Selected Solutions to Graph Theory, 3 rd Edition

Size: px
Start display at page:

Download "Selected Solutions to Graph Theory, 3 rd Edition"

Transcription

1 Selected Solutions to Graph Theory, 3 rd Edition Reinhard Diestel of Institute Technology Indian :: Jana Guwahati Research Scholar Mathematics Rakesh :: Rakesh Jana Department of Mathematics May 1, 2016

2 Acknowledgement These solutions are the result of taking CS-520(Advanced Graph Theory) course in the Jan-July semester of 2016 at Indian Institute of Technology Guwahati. This is not a complete set of solutions in that book. It may happen that solution of some problem may be wrong. I have not verified these problem from some expart. It is my kind request you that do not belive the answer blindly. If you found any mistake please inform me. I know these article must contain some typographical errors, in that case please inform me. If you have any better solution in any of these problem please let me know. I will upload that solution in this content with your name. If you want to discuss any of these solution with me please ping me in my given address or meet me in research scholar office (RS-E1-010) Department of Mathematics,. You can find List of Solved Exercises at the end. Please jana.rakesh. math@gmail.com or j.rakesh@iitg.ernet.in for any corrections and suggestions. Copyright c , Rakesh Jana

3 Contents 1 The Basics 3 2 Matching, Covering and Packing 10 3 Connectivity 14 4 Planar Graphs 18 5 Colouring 19 9 Ramsey Theory for Graphs Some Arbitary Problem 22 1 The Basics Matching Connectivity Planar graph Colouring Solved Exercise Reference 27

4 1 The Basics See some extra problem on basic in the end( problem problem ). Exercise 1.1. What is the number of edges in K n? Proof. Notice that first vertex adjacent to other n 1 vertices. Now compute how many vertices are adjacent to second vertex except first vertex, obviously answer is n 2. Similarly compute how many vertices are adjacent to third vertex except first and second vertices, answer is n 3, and so on. Thus total number of edge is K n is (n 1) + (n 2) = n(n 1). 2 Exercise 1.2. Determine the average degree, number of edges, diameter, girth, and circumference of the hypercube graph Q d. Proof. Since V is the set of all 0 1 sequences of length d. Thus total number of vertices is 2 d, since in each place we can assign two number 0, 1. Since two such sequence form an edge if and only if they differ in exactly one position. Thus each vertices has degree d. Now we know that 2 E = v V d(v) E = d 2d 2 Thus average degree of Q d = 2 E V = d. = d 2 d 1. Notice that the distance between any two vertices depends on the number of different bits, so diameter is d, i.e. diam G = d. Girth(Q 1 ) =, because there are no cycles on hypercube graph Q 1. Girth(Q d ) = 4, where d 2, this is because Q d = K 2 Q d 1. Circumference of Q d is 2 d. Exercise 1.3. Let G be a graph containing a cycle C, and assume that G contains a path of length at least k between two vertices of C. Show that G contains a cycle of length at least k. Is this best possible? 3

5 Proof. Let the path P start at x and end at y where x, y are lie on C. Suppose that P leaves C for the i th time at vertex x i, and arrives at C for the i th time at vertex y i (it is possible for x i+1 = y i ). Then the x i, y i -portion of P together with the x i, y i -portion of C forms a cycle of length at least 1 + l i, where l i = dist P (x i, y i ). Let among x i s and y i s there are t many distict vertices. Without loss of any generality Now if t k then we can take a path along C connecting these distinct vertices and then traverse C then we will get a cycle of length atleast k + 1. Let t < k. Let us consider subpath of path P, P i = x i P y i and P i = y i P x i+1. Then there are atmost t many internally disjoint subpath of P. Let P k be the subpath of P with maximum length, say l(p k ) = m. Then k l(p ) tm km Thus m > k. Hence we have a subpath of the path P of lenght atleast k whose end points are in C and also distinct. Hence We get a cycle of length atleast k. Notice in the solution that we can improve the size of cycle from k to k + 1. Exercise 1.4. We know that from proposition that every graph containing a cycle satisfying g(g) 2 diam G + 1. Is the bound is best possible? Proof. Yes. It is the best possible bound because equality occur when G = K 3. Exercise 1.5. Show that rad G diam G 2 rad G. Proof. We know that diam G = max x,y v(g) d G (x, y). rad G = min x V (G) min x V (G) = diam G. max d G(x, y) y V (G) max diam G y V (G) To show diam G 2 rad G. Let a, b, v V (G) such that d G (a, b) = diam G and rad G = max y V (G) d G (v, y). diam G = d G (a, b) d G (a, v) + d G (v, b) rad G + rad G = 2 rad G. 4

6 Exercise 1.6. Prove the weakening of Theorem obtained by replacing average with minimum degree. Deduce that G n 0 (d/2, g) for every graph G as given in the theorem. Proof. Case 1: Consider g = 2r + 1, r N. This proof is similar to proof of proposition Let v V (G) be any vertex in G. Let us consider D i = {u V (G) : d G (u, v) = i}, for i N {0}. It is clear that D i D j =, i j and V (G) = i 0 D i. Since v can not contained in any cycle of length lesser then 2r + 1. Thus for any u, w D i, 0 i r 1, N(u) D i+1 is disjoint from N(w) D i+1, otherwise we can construct a cycle of length atmost r r 1 = 2r < 2r +1, a contradiction. Hence each vertex in D i, 0 i r 1 is connected to exactly one vertex in D i 1 and atleast δ 1 vertices in D i+1. Hence D 0 = 1, D 1 δ and D i δ(δ 1) i 1, for 2 i r. Thus V (G) r 1 i=0 r 1 D i = 1 + δ (δ 1) i 1. Case-2: Consider g = 2r, r N. In this case proof is same as previous one instead of a vertex we have to start with two adjacent vertices. Let uv E(G). Similar way consider for i N {0}, i=0 D u i = {y : ˆd(u, y) = i} D v i = {y : ˆd(v, y) = i} where ˆd(x, y) := d G uv (x, y). Similar way as case-1, for any x {u, v}, Di x Dj x = for i j and for any a, b Di x, N(a) Di+1 x is disjoint from N(b) Di+1 x for 1 i < r 1. Also each vertex in Di x (0 i < r 1) is connected to exactly one vertex in Di 1 x and atleast δ 1 vertices in Di+1. x Now D0 x = 1, D1 x δ 1 and Di x (δ 1) i, for 1 i r 1. Let us define for x {u, v}, T x = Di x. 0 i r 1 Notice that T x = r 1 i=0 (δ 1)i for any x {u, v}. Claim. T u T v =. To prove this claim first notice that D u i D v j =, for all 0 i, j r 1. If not let x D u i D v j for some 0 i, j r 1. Then there exist a cycle in G of length atmost r 1 + r = 2r 1 < 2r, a contradiction. Hence T u T v =. Hence V (G) T u + T v = 2 r 1 i=0 (δ 1)i. 5

7 Lemma 1.1. Let P be a path in a connected graph G. If there is u V (G) \ V (P ), then there exist v V (G) \ V (P ) adjacent to P. Proof. Let u V (G)\V (P ) and w V (P ). Since G is connected there exist a u w path in G, say Q. Now consider last common vertex p V (P ) V (Q) (traversing from w to u) then there exist a vertex in v V (Q) \ V (P ) such that vp E(G). Exercise 1.7. Show that every connected graph G contains a path of length at least min{2δg, G 1}. Proof. Let us consider P = x 0 x 1 x k be a longest path in G. We have to show k min{2δg, G 1}. If possible let k < min{2δg, G 1}. Now G is connected E(G) G 1. Since k < G 1 there exist u V (G) \ V (P ) and by lemma 1.1 there exist y V (G) \ V (P ) such that yx i E(G), for some 0 i k. Now if x 0 x k E(G) we can get a path P = yx i P x k x 0 P x i which is longer then P, a contradiction. Thus x 0 x k / E(G). Now N(x 0 ) V (P ) and N(x k ) V (P ), since P is the longest path. Let us consider S = {x j x j+1 N(x 0 ), 0 j k 2}. Clearly S δ(g). Since k < 2δ(G) gives V (P ) \ (S {x k }) δ(g). By pigeonhole principle there exist x j S such that x j x k E(G). Hence we get a cycle C = x 0 P x j x k P x j+1 x 0. Now consider the path P = yx i C x i which is longer then P, a contradiction. Hence k min{2δg, G 1}. Exercise 1.8. Find a good lower bound for the order of a connected graph in terms of its diameter and minimum degree. Proof. The following claim gives the lower bound for the order of connected graph. Claim. Let G be any connected graph with diam G = k and δ(g) = d then G kd/3. Let d G (x, y) = k, for some x, y V (G) and distance achieve by the path P = x 0 x 1 x k, where x 0 = x, x k = y. Let u be a vertex not on P that is adjacent to some vertex on P. Let i be the smallest integer such that x i is adjacent to v. Notice that if v is adjacent to x j for j > i + 2 then we can get a path x 0 P x i vx j P x k and which is shorter then P, a contradiction to d G (x, y) = k. Hence each v V (G) \ V (P ) can adjacent to at most 3 vertices on P. Exercise Show that every 2-connected graph conatains a cycle. 6

8 Proof. Let G be a 2-connected graph. Then δ(g) 2, since if d(v) = 1 or 0, for some v V (G) then that vertex will be either a cut vertex or isolated, in both case it contradict that G is 2-connected. Hence by proposition-1.3.1, it has a cycle of length atleast δ(g) + 1. Exercise Determine κ(g) and λ(g) for G = P m, C n, K n, K m,n, and Q d ; d, m, n 3. Proof. Recall. κ(g) denote for connectivity(vertex) of a graph G and λ(g) denote edge-connectivity of graph G. Also by proposition-1.4.2, κ(g) λ(g) δ(g). Given graphs are all connected. κ(p m ) = 1, for m 2 it is clear, for m > 2 if you remove an interior vertex of P m, it becomes a disconnect graph. λ(p m ) = 1, as if you delete any edge, the graph becomes disconnected. κ(c n ) = 2, because if you remove any vertex you will get P n 1, hence if you delete any two vertex from C n then it becomes a disconnect graph. λ(c n ) = 2, as if you delete any edge, the graph becomes P n and if you delete one more edge it become disconnected. Similarly, κ(k n ) = n 1 λ(k n ) = n 1 κ(k m,n ) = min{m, n} λ(k m,n ) = min{m, n} κ(q d ) = d λ(q d ) = d. Exercise Is there any function f : N N such that, for all k N, every graph of minimum degree atleast f(k) is k connected? Proof. No. Suppose f(1) = t N. Then there exist graphs G and H with both have minimum degree t but one of them is connected and other is not. For instance take G = K t+1 and take H be two disjoint component of K t+1. Exercise Show that every tree T has atleast (T ) leaves. Proof. Exercise Show that a tree without a vertex of degree 2 has more leaves than other vertices. Can you find a very short proof that does not use induction? 7

9 Proof. Let T be a tree with no vertex of degree 2. Let V i = {v V (G) : d G (v) = i}. Notice that V 2 =. Now average degree of a tree is 2 E 2( V 1) = < 2. Now V V Hence we get, V 1 + V 1 i=3 2 > This complete the answer. v V d G(v) V = V V 1 i=3 V i V = V + 2 V 1 i=3 V i V V 1 V i = V > 2 i=3 V 1 i=1 i V i V = V 1 + V 1 i=3 i V i V = V 1 i=3 V i V V i = V 1 > V 1 Exercise Let G be a connected graph, and let r G be a vertex. Starting from r, move along the edges of G, going whenever possible to a vertex not visited so far. If there is no such vertex, go back along the edge by which the current vertex was first reached (unless the current vertex is r; then stop).(this procedure has earned those trees the name of depth-first search trees.) Show that the edges traversed in depth-first search form a normal spanning tree in G with root r. Proof. First notice that in dfs we always get a tree, since we always add a vertex to the current subgraph if it is not end point of any edge of current subgraph, so cannot create a cycle. To show it is spanning. Suppose it not spanning tree of G then there is a vertex v which is not in the tree but adjacent to a vertex u in the tree. But then when we left u for the last time we would have visited v instead of returning to r. So we get a contradiction that depth-first search completed. Hence we get a spanning tree, say T. To show T is normal. Last part remaining Exercise Show that a graph is bipartite if and only if every induced cycle has even length. Proof. Recall. An induced cycle in G is a cycle in G forming an induced subgraph without any chords. i=3 V i. 8

10 If a graph is bipartite then it does not have any odd cycle by proposition-1.6.1, hence does not have any induced cycle of odd length. To prove reverse part. Let us assume G is not bipartite. Since G is not bipartite so it has an odd cycle. Let C be a smallest odd cycle in G. Then C can not be induced cycle, since all induced cycle are even lengths. Then there exist x, y V (C) but xy / E(C). Thus we get two cycle C 1 = xcyx, C 2 = ycxy (traverse clockwise direction), among them one is odd and other is even. Hence we get a shorter odd cycle, a contradiction. This proves the result. Exercise Find a function f : N N such that, for all k N, every graph of average degree at least f ( k) has a bipartite subgraph of minimum degree at least k. Proof. Define a map f : N N by f(k) = 4k, k N. The idea behind to consider this function is following: Every graph with an average degree of 4k have a subgraph H with minimum degree 2k, and we will lose another factor of 2 in moving H to its bipartite subgraph. Let H be the bipartite subgraph of H with the maximal number of edges. My claim is that H have minimum degree atleast k. If not, let v H such that d H (v) < k. This means v lost more then half of its neighbours in the process to form H to H. This means v is on the same partition with its looses neighbours. But in that case if we consider v in the other partition we can able to connect those previously looses vertices to v and form a new bipartite subgraph of H with more edges then H have, a contradiction. Hence it proves of my claim. Exercise Prove or Disprove that every connected graph contains a walk that traverses each of its edges exactly once in each direction. Proof. Let W = v 0 v 1 v k be a longest walk in G that traverses every edge exactly once in each direction. If possible let there exist a vertex v not visited by W. Without loss of any generality let us assume v N(v i ) for some 0 i k. Now consider a walk v 0 W v i vv i W v k which is longer then W and also traverses each of its edges exactly once in each direction, a contradiction. So each vertex in G visited by W. Again suppose that W doesn t contain all the edges, since W visits every vertex in G so G has an edge e = v i v j (i < j) not traversed by W. Consider a new walk v 0 W v i v j v i W v k which is longer then W and also traverses each of its edges exactly once in each direction, a contradiction. So each edge in G visited by W. Hence every connected graph contains a walk that traverses each of its edges exactly once in each direction. 9

11 2 Matching, Covering and Packing See some extra problem on Matching, Covering and Packing in the end( problem problem ). Exercise 2.2. Describe an algorithm that finds, as efficiently as possible, a matching of maximum cardinality in any bipartite graph. Proof. We already know that A matching M is maximum in a graph G if and only if there are no augmenting paths with respect to M. Let A and B be the bipartition of G, and let M be the matching in G, initially M =. Following algorithm known as Hungarian Method. Algorithm 1 Maximum-Matching (G, A, B, M) 1: if M saturates every vertex in A then 2: stop; 3: Let u be an an M-unsaturated vertex in A. 4: Set S = {u}, T =. 5: if N(S) = T then N(S) < S, since T = S 1 then by Hall s theorem there is no matching that saturates every vertex in A then 6: stop; 7: Let v N(S) \ T. 8: if v is M-saturated, let vw M then 9: Set S = S {w}, T = T {v}; (Observe that T = S 1 is maintained). 10: goto step-5. 11: Otherwise we get an M-augmenting u v path. 12: M = M P = (M \ P ) (P \ M); (symmetric difference of the two sets of edges) 13: Maximum-Matching (G, A, B, M) Exercise 2.3. Show that if there exist injective function A B and B A between two infinite set A and B then there exist a bijection between A B. Proof. The above problem is known as Cantor-Schrouder-Bernstein theorem. Although the statement seemingly obvious statement is surprisingly difficult to prove. The the strategy of the proof is following: Let f : A B and g : B A be two injective map. First, we apply f(a) = B 1 B. Next, g(b 1 ) = A 2 A. Iterating this, we keep bouncing back and forth between 10

12 smaller and smaller subsets of A and B until the process stabilizes and we end up with some sets Ā A and B B for which f(ā) = B and g( B) = Ā. This implies that Ā B. The next task is to show that A \ Ā B \ B. Finally, we conclude that A B. You can get complete proof of this result in the book Introductory Real Analysis by A. N. Kolmogorov and S. V. Fomin, 1st edition, Dover Publications. Exercise 2.4. Find an infinite counterexample to the statement of the marriage theorem. Proof. Let A = Z + {a} and B = Z +, here a is an alphabet. Let us consider a graph G with vertex set V (G) = A B, (consider A and B are different set). Let xy E(G), x A and y B if and only if x = y or x = a. Then for any S A, N(S) S. But a matching saturating A must saturate Z + A, and since these vertices have degree 1 and they already matched with every vertex in B, it cannot saturate a. Hence there is no matching saturating A. Exercise 2.5. Let k be an integer. Show that any two partitions of a finite set into k-sets admit a common choice of representatives. Proof. Let k N. Let X be a set of n elements with k n and m = n, and let k A 1,, A m and B 1,, B m are partitions of V into k-sets. Let us define a bipartite graph G with the vertex set V (G) = A B where A = {A 1,, A m } and B = {B 1,, B m }, viewing each set A i as a vertex. Let A i B j E(G) if and only if A i B j. We want to apply Hall theorem. Let S A and we have to estimate N(S). Let S contain t many element of A. Then number of element of X contain in S is tk. Now number of element of B covering these tk element is atleast t, since each element B j contains k elements. It follows that N(S) S. Hence Hall condition holds. Now by Halls theorem, we have a matching saturaing A, that is, we have a perfect matching. Therefore, any two partitions of a finite set into k-sets admit a common choice of representatives. Exercise 2.6. Let A be a finite set with subsets A 1,, A n, and let d 1,, d n N. Show that there are disjoint subsets D k A k, with D k = d k for all k n, if and only if A i d i i I i I for all I {1,, n}. Proof. Suppose i I A i i I d i holds for all I {1,, n}. Let us denote the elements of A i as follows, A i = {a i1, a i2,, a iti }, for 1 i n. Clearly for each 11

13 i, d i t i. Let us construct a bipartite graph G with bipartition {X, A}, where X = n i=1 {a ij : 1 j d i } and join a ij X to a A if and only if a A i. Notice that in G for any S X, N(S) S. Thus by Hall s theorem G contains a matching saturaing X. That matching gives us disjoint subsets D k A k, with D k = d k for all k n. If there exist disjoint subsets D k A k, with D k = d k for all k n then this is equivalent to that there exist a matching in the bipartite graph G (which is constructed earlier). saturating X. Hence, by the Hall s theorem, for any S X, N(S) S. Now for any I {1,, n} consider S = i I D i gives, i I A i i I d i. Exercise 2.8. Find a bipartite graph and a set of preferences such that no matching of maximum size is stable and no stable matching has maximal size. Proof. Try C 6. Exercise 2.9. Find a non-bipartite graph and a set of preferences that has no stable matching. Proof. Try K 3. Exercise Show that all stable matchings of a given bipartite graph cover the same vertices. (In particular, they have same size.) Proof. Suppose M 1 and M 2 are two stable matchings of G that don t cover the same vertices. Then there exist some vertex x which is matched under M 1 but unmatched under M 2. Let xy M 1. Notice that y must be matched in M 2, otherwise there exist a edge xy whose both end points are unmatched under M 2, a contradiction that M 2 is a stable matching. Since y is matched in M 2 thus there exist z V (G) such that yz M 2. Thus we have xyz path with edges alternately in M 1 and M 2. Continue this way we get a path P = v 0 v 1 v n for some n 2 where v 0 = x, v 1 = y, v 2 = z. Notice that v n 2 < vn 1 v n in M 2, but v n < vn 1 v n 2 in M 1, a contradiction. Thus M 1 and M 2 cover same vertices. Exercise Show that a graph G contains k independent edges if and only if q(g S) S + G 2k for all sets S V (G). Exercise Find a cubic graph without a 1-factor. Proof. From Theorem we know that A graph G has a 1-factor if and only if g(g S) S for all S V (G). Consider the following graph G, 12

14 Figure 1: Cubic graph G Figure 2: Graph G S Let us consider S V (G) to be red colored vertices. Thus q(g S) = 6 > S = 4. Hence G can not have 1 factor. Exercise Derive the merriage theorem from Tutte s theorem. Proof. 13

15 3 Connectivity See some extra problem on connectivity in the end( problem problem ). Exercise 3.4. Let X and X be minimal separating vertex sets in G such that X meets at least two components of G X. Show that X meets all the components of G X, and that X meets all the components of G X. Proof. Suppose that X meets G X in only one component, say C. Then X X C. So the components of G X are components which come from C X and a component which contains the rest of G. So, X meets only one component of G X. This is a contradiction. Hence, X meets at least two components of G X. Then, it follows from symmetry that X meets every component of G X. Exercise 3.7. Show, without using Menger s theorem, that any two vertices of a 2-connected graph lie on a common cycle (that is there exist two internally vertex disjoint path between those two vertices). Proof. This problem is known as Whitney s theorem which is solved in You can find this theorem in many books such as Graph theory with application by Bondy & Murty. But third solution in this note which given by Kewen Zhao is simplier then any other solutions. First Solution 1 : I have to show between any two vertices in a biconnected graph there exist two internally vertex disjoint path. I will show it by inductively by using induction on their distance. Let us assume x, y be any two vertex set in G and d = dist G (x, y). If d = 1, that is xy E(G). since G is biconnected thus there exist another x y path in G, otherwise xy is a bridge in G, a contradiction. Let us assume the statement is hold for any vertex of degree less than d 2. Let S be the shortest path between x and y. Let v V (S) with lesser distance to y in S.Then dist G (x, v) = d 1 < d. Thus by induction hypothesis there exist two internally vertex disjoint x v path in G, say P 1, P 2. Now if y is a vertex of any one of these path, say P 1 then xp 1 y and P 2 y gives us two different paths, as in xp 1 y path v will not come as v is the end vertex and y comes before v. Let us assume y / V (P 1 ) V (P 2 ). Since G {v} is connected there exist a x y path in G {v}, say Q. Now consider the last vertex w V (Q)(according to the distance from x in Q) such that w V (P 1 ) V (P 2 ). Since w v thus either w V (P 1 ) or w V (P 2 ). Without loss of any generality assume w V (P 1 ). Now consider a new path P 3 := xp 1 wqy. Notice that V (P 3 ) V (P 2 ) = {x}. Thus consider another path P 4 := xp 2 vy. Hence P 3, P 4 are two internal vertex disjoint x y path. 1 Based on Theorem-3.2(pp ), Bondy & Murty Book. 14

16 Second solution: 2 Suppose that there are two vertices u, v such that they are not on a cycle. Then we want to show that there is a cut vertex separating u and v. To argue about the paths from u to v, we want to first order the vertices. One way to do this is to do a depth first search of G from u, label all the vertices in a pre-order traversal, and for each vertex w let a(w) be the smallest ancestor that can be reached from w through one of its descendants; note that there can only be back edges in this traversal, since G is undirected. We want to characterize when are two vertices u and v on a cycle in such a DFS. It is clear that if a(v) = u then they are on a cycle, however, this is not necessary. The only other possibility is the following: consider the path between v and a(v); if there is a vertex w on this path such that a(w) = u then u and v are also on a cycle. Thus two vertices are on a cycle iff in the path P from v to a(v) there is a vertex w such that a(w) = u. In our setting, however, u and v are not on a cycle. The cut vertex separating u and v is the ancestor a(w), where w P, closest to u. Third solution: 3 Let G be 2-connected graph and assume there exist two vertices u and v without two internally-disjoint u v paths. Let P and Q be two u v paths with the common vertex set S as small as possible. Let w S \ {u, v} and P 1 := up w, P 2 = wp v and Q 1 := uqw, Q 2 := wqv. Since G is 2-connected, let R denote a shortest path from some vertex x (V (P 1 ) V (Q 1 )) \ {w} to some vertex y (V (P 2 ) V (Q 2 )) \ {w} without passing through w. We may assume, without loss of generality, that x is in P 1 and y in Q 2. Let T denote the u v path composed of up 1 xryq 2 v. Clearly the common vertices of T and the u v path composed of Q 1 P 2 are all in S \ {w}. This contradicts the choice of both P and Q as having the smallest number of vertices common. Exercise 3.9. Let G be a 2-connected graph but not a triangle, and let e be an edge of G. Show that either G e or G/e is again 2-connected. Deduce a constructive characterization of a 2-connected graphs analogous to Theorem Proof. Exercise Let G be a 3-connected graph, and let xy be an edge of G. Show that G/xy is 3-connected if and only if G {x, y} is 2-connected. Proof. Given that G is 3-connected with an edge xy E(G). Let G/xy is 3 connected. To show G {x, y} is 2 connected. Suppose if possible G {x, y} is not 2 connected. Then there exist a vertex z in G {xy} which separate G {x, y}. Then {z, v xy } becomes a separating set of G/xy, a contradiction. Hence G {x, y} is 2-connected A simple proof of Whitney s theorem on connectivity in a graph by Kewen Zhao. 15

17 Conversely, suppose G {x, y} is 2 connected. To show G/xy is 3 connected. If possible let G/xy is not 3-connected. Then there exist a separating set {u, v} in G/xy which separate G/xy. Now if u, v v xy then {u, v} becomes a separating set of G, a contradiction. Suppose u = v xy. Then v separates G {x, y}, a contradiction. Hence G/xy is 3 connected. Exercise Show that every cubic 3-edge-connected graph is 3-connected. Proof. Lemma 3.1. Let G be a k 2 connected graph. Let S be the set of k vertices and u V \ S. Then there exist k many u S path contianing u as only common vertex. Proof of lemma: Let us consider a graph G such that V (G ) = V (G) {x} and E(G ) = E(G) {xy y S}. Then G is k-connected graph. By Menger s theorem there exist k (internal) vertex disjoint u x path in G. These path must passes through vertices of S. Since S = k, every path contain exactly one element from S. Consider corresponding path in G gives required k paths. Exercise Let k 2. Show that every k-connected graph of order at least 2k contains a cycle of length at least 2k. Proof. Let C be the longest cycle in G. If v V (C), for all v V (G) then we are done. Let there exist v V (G) \ V (C). Then by lemma-3.1 there exist k vertex disjoint (only common vertex is v) v C paths. Now if C < 2k then by pigeonhole principle there exist two paths whose end points are adjacent on C. We can construct a longer cycle by detouring along these paths, a contradiction. Exercise Let k 2. Show that in a k-connected graph any k vertices lie on a common cycle. Proof. I will prove this statement using induction on k. The base case of induction is k = 2. It is directly follows from Menger s theorem although I have given a alternating proof of this result in problem-3.7. For induction hypothesis let us assume for any k 1 connected graph the statment holds. Now let G be a k-connected graph and S = {v 1,, v k } are k many vertices in G. Now since G is k-connected, then G v 1 is k 1 connected. By induction hypothesis we get vertices v 2,, v k are lie on a common cycle in G v 1, say C. Now conside two vertex set {v 1 } and V (C). Case-1: Let l(c) = k 1. Consider v V \V (C) and C {v}. Then by lemma-3.1 there k 1 many internal vertex disjoint v 1 C path in G haveing v 1 is their only common vertex. Hence we can construct a new path containing all those k vertices. 16

18 Case-2: Let l(c) k. Then there k many internal vertex disjoint v 1 C path in G, say P i, 1 i k such that if x i be the end points of P i then V (P i ) C = {x i } and x i x j, for each i j. Such type of path exist by lemma-3.1. Without loss of generality assume that x i are present in C in anticlockwise order. Then these many paths devide C into k segment. Let C i = x i Cx i+1 for 1 i k (consider k + 1 = 1) are the segment of C. Since S {v 1 } = k 1 then by pigeonhole principle atleast one segment does not contain any vertices of S {v 1 }, say C i. Then we can get a new cycle C = v 1 P i+1 x i+1 Cx i P i v 1. Here x i+1 Cx i taken anticlockwise direction. Hence C contain all k vertices of S. Exercise

19 4 Planar Graphs See some extra problem apart from Diestel books on planar graphs in the end( problem problem ). Exercise 4.5. Show that every planar graph is unioin of three forests. Exercise For every k N, construct a triangle free k-chromatic graph. Proof. The following construction is known as Tutte s construction of triangle-free k-chromatic graph. G H to be the graph obtained by joining every vertex in G with every vertex in H. For k 5 it is easy to construct. Now let k > 5. Clearly χ(g H) = χ(g)+χ(h). (Exercise ). Notice that χ(c 5 C 5 ) = 6. Consider G 6 = C 5 C 5 and for k > 6, consider G k = G k 1 G k 1. Claim. G k is triangle free. Proof. We will prove it by induction on k. Notice that G 2 = K 2, triangle free. Let G k 1 triangle free. Claim. χ(g k ) = k. 18

20 5 Colouring See some extra problem on colouring in the end( problem problem ). Exercise 4.5. Show that every graph G has a vertex ordering for which the greedy algorithm uses only χ(g) colours. Proof. Since G is χ(g) colourable there exist a colouring of G which takes χ(g) colours. According to this colouring partition the vertex set V (G) into χ(g) parts. Let these parts are V 1,, V χ(g). Notice that all vertices belongs to same partition are independent. Now apply Greddy algorithm as follows: first colour all vertices of V 1 by colour 1, after colour all vertices of V 2 by colour 1 or 2. This is because each such vertex may not have any neighbours among vertices from V 1. In general, color all vertices of V i with the colour from {1, 2,, i} because some vertices of V i may not adjacent to any already-colored vertices. Hence Greddy algorithm will use atmost χ(g) colour. Since G can not be colour by lower then χ(g) colour. Hence Greddy algorithm will use exactly χ(g) colour. Exercise 4.6. For evry n > 1, find a bipartite graph on 2n vertices, ordered in such a way that the greddy algorithm uses n rather than 2 colours. Proof. Consider complete K n,n graph with bipartition A, B. Let A = {a 1,, a n } and B = {b 1,, b n }. Suppose M = {a i b i : 1 i n} be the perfect matching of K n,n. Let us consider a new bipartite graph G = K n,n \ M (removing only edges). Now apply Greddy algorithm in G with the vertex order {a 1, b 1,, a n, b n }. Then a 1 and b 1 will be assigned color 1, since they are not adjacent to any already-colored vertices. Since a 2 and b 2 are each adjacent to a vertex already assigned color 1 they will be assigned color 2. Agian a 3 and b 3, each adjacent to vertices of colors 1 and 2, must be assigned color 3 and so on. Since a n and b n each adjacent to vertices of every color from 1 to n 1 it must be assigned color n. Exercise 4.9. Find a lower bound for the colouring number in terms of average degree. Proof. Recall proposition-1.2.2: Every graph G with atleast one degree has a subgraph H with δ(h ) > ɛ(h ) ɛ(g) = d(g). 2 It is clear that, Hence d(g) χ(g). χ(g) = max H G δ(h) + 1 δ(h ) + 1 = d(g)

21 Exercise A k-chromatic graph is called critically k-chromatic, or just critical, if χ(g v) < k for every v V (G). Show that every k-chromatic graph has a critical k-chromatic induced subgraph, and that any such subgraph has minimum degree atleast k 1 Proof. For first part use induction. If the graph G itself is critically k-chromatic, then we are done, otherwise there exists a vertex v in G such that χ(g v) = k. Then apply induction hypothesis to the graph G v to find a critically k-chromatic subgraph of G. Let G be itself a critically k-chromatic graph. It is enough to show that, if there exist a vertex v G such that deg(v) < χ(g) 1 then χ(g) = χ(g v). Let there exist a vertex v G such that deg(v) = χ(g) 2. Since χ(g v) < k thus we can color G v using k 1 color. Since v is adjacent to k 2 edges so its neighbours will get atmost k 2 colors so we can color v with remaining one color. Thus G is k 1 colourable, a contradiction. Exercise Determine the critical 3-chromatic graphs. Proof. We will prove that a graph is critical 3-chromatic graph if and only if it is an odd cycle. Since we know that every odd cycle is 3-chromatic and if we delete any one vertex of this cycle, we will get a path which is 2-colourable. Hence every odd cycle is critical 3-chromatic. Let G be a critical 3-chromatic graph. Then G can not be a bipartite graph. Thus G had an odd cycle,say C. Claim is G = C. If not then there exist a vertex v G C. Now notice that G v contain an odd cycle C so its chromatic number is 3, but since G is crticial 3-chromatic graph, χ(g v) < 3, a contradiction. Hence G = C. 20

22 9 Ramsey Theory for Graphs Exercise 9.6. Use Ramsey s theorem to show that for any k, l N there is an n N such that every sequence of n distinct integers contains an increasing subsequence of length k + 1 or a decreasing subsequence of length l + 1. Find an example showing that n > kl. Then prove the theorem of Erdos and Szekeres that n = kl + 1 will do. Proof. Exercise 9.7. Sketch a proof of the following theorem of Erdos and Szekeres: for every k N there is an n N such that among any n points in the plane, no three of them collinear, there are k points spanning a convex k-gon, i.e. such that none of them lies in the convex hull of the others. Proof. Exercise 9.8. Prove the following result of Schur: for every k N there is an n N such that, for every partition of {1,, n} into k sets, at least one of the subsets contains numbers x, y, z such that x + y = z. Proof. 21

23 10 Some Arbitary Problem 1 The Basics Exercise Prove that the number of simple even graphs (degree of all vertices is even) with n vertices is 2 (n 1 2 ) Proof. There is a bijection between simple graphs with n 1 vertices and even simple graphs on n vertices. Given a simple graph G with V (G) = {v 1,, v n } we can construct a even simple graph of n vertices. We know that no of vertices of odd degree is even. Construct a new graph G with V (G ) = V (G) {v n } and E(G ) = E(G) {v i v n : v i V (G), deg G (v i ) is odd}. Then G is a even simple graph. Conversely given a even simple graph G we will get back G by G v n. Since in a simple graph of n 1 vertices can have atmost ( n 1 2 graph of n vertices is 2 (n 1 2 ). Exercise Matching ) edges thus no of even simple Exercise Prove that a nonempty bipartite graph has a matching such that all vertices of maximal degree are saturated. Exercise Show that the following obvious algorithm need not pro- duce a stable matching in a bipartite graph. Starting with any matching. If the current matching is not maximal, add an edge. If it is maximal but not stable, insert an edge that creates instability, deleting any current matching edges at its ends. Proof. Consider a bipartite graph G with bipartition {A, B} where A = {1, 2, 3, 4} and B = {a, b}. Consider preferences: 1 a 2 b 3 4 Let us consider the following matching: a : 3 > 2 > 1 > 4 b : 2 > 3 > 4 > 1 1 : b > a 2 : a > b 3 : b > a 4 : a > b 22

24 1 a 2 b a 2 b a 2 b a 2 b 3 4 Notice that a prefers 2 over 1, and 2 prefers a, so this is not a stable matching. Delete the two edges consider 2a as new matching edge with another independent edge. Notice that a prefers 3 over 2, and 3 is unmatched, so this is not a stable matching. Again doing same operation. Notice that b prefers 3 over 4, and 3 also prefer b, so this is not a stable matching. Again doing same operation. Notice that b prefers 2 over 3, and 2 is unmatched, so this is not a stable matching. Again doing same operation. Hence we get looped back to where we started. 1 a b Thus given algorithm need not produce a stable matching. 23

25 Exercise A matching M in a graph is of maximal cardinality if and only if the graph has no augmenting path with respect to M. Exercise Prove that every tree has atmost one perfect martching. Exercise Connectivity Exercise Exercise Let G be a biconnected graph with δ(g) 3. Prove that there exist a vertex v V (G) such that G v is also biconnected. Exercise Planar graph Exercise Prove that every planar graph has a vertex of degree atmost 5. Exercise Prove that there does not exist any 6-connected planar graph. Exercise Prove that every planar 5-connected graph has atleast 12 vertices. Exercise For which r there exist a planar r-regular graph. Exercise Show that the petersen graph is not planar. 5 Colouring Exercise Find chromatic number of graphs a) K n ; b) K n,m ; c) P n ; d) C n ; e) Petersen graph. Exercise Prove that if every block of a graph is k-colorable then the graph is k-colorable. Exercise Let G, H be any two graph. Show that χg H) = χ(g) + χ(h). Exercise Prove that difference (G) χ(g) maybe arbitarily large. Exercise Prove that the number of edges of a graph G is atleast χ(g)(χ(g) 1)/2. 24

26 Proof. Let 0 < i, j < χ(g) and i j. Then there exist an edge whose end vertices color with i and j, otherwise we can color G with lesser number of color then χ(g). Hence total no of edge is atleast ( ) χ(g) 2 = χ(g)(χ(g) 1). 2 Exercise Find all counterexample to this statement: every connected graph G contains a vertex such that deg v χ(g) Exercise

27 T 4 T 2 T 1 T 3 T 5 c a d a b d b 1 c Figure 3: Labeling of edges and identification of vertices in P. a b x 0 x 1 d c Figure 4: Sketch of A = π(bd P ). 26

28 11 Solved Exercise Reference List of Solved Exercises 1 The Basics 3 Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Matching, Covering and Packing 10 Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Connectivity 14 Exercise Exercise Exercise Exercise Exercise Exercise Exercise Exercise Planar Graphs 18 Exercise Exercise Colouring 19 Exercise Exercise Exercise Exercise Exercise Ramsey Theory for Graphs 21 Exercise Exercise Exercise Some Arbitary Problem 22 1 The Basics Matching Connectivity Planar graph Colouring Solved Exercise Reference 27 27

HW Graph Theory SOLUTIONS (hbovik)

HW Graph Theory SOLUTIONS (hbovik) Diestel 1.3: Let G be a graph containing a cycle C, and assume that G contains a path P of length at least k between two vertices of C. Show that G contains a cycle of length at least k. If C has length

More information

Part II. Graph Theory. Year

Part II. Graph Theory. Year Part II Year 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2017 53 Paper 3, Section II 15H Define the Ramsey numbers R(s, t) for integers s, t 2. Show that R(s, t) exists for all s,

More information

Exercise set 2 Solutions

Exercise set 2 Solutions Exercise set 2 Solutions Let H and H be the two components of T e and let F E(T ) consist of the edges of T with one endpoint in V (H), the other in V (H ) Since T is connected, F Furthermore, since T

More information

Assignment 1 Introduction to Graph Theory CO342

Assignment 1 Introduction to Graph Theory CO342 Assignment 1 Introduction to Graph Theory CO342 This assignment will be marked out of a total of thirty points, and is due on Thursday 18th May at 10am in class. Throughout the assignment, the graphs are

More information

Module 7. Independent sets, coverings. and matchings. Contents

Module 7. Independent sets, coverings. and matchings. Contents Module 7 Independent sets, coverings Contents and matchings 7.1 Introduction.......................... 152 7.2 Independent sets and coverings: basic equations..... 152 7.3 Matchings in bipartite graphs................

More information

List of Theorems. Mat 416, Introduction to Graph Theory. Theorem 1 The numbers R(p, q) exist and for p, q 2,

List of Theorems. Mat 416, Introduction to Graph Theory. Theorem 1 The numbers R(p, q) exist and for p, q 2, List of Theorems Mat 416, Introduction to Graph Theory 1. Ramsey s Theorem for graphs 8.3.11. Theorem 1 The numbers R(p, q) exist and for p, q 2, R(p, q) R(p 1, q) + R(p, q 1). If both summands on the

More information

4. (a) Draw the Petersen graph. (b) Use Kuratowski s teorem to prove that the Petersen graph is non-planar.

4. (a) Draw the Petersen graph. (b) Use Kuratowski s teorem to prove that the Petersen graph is non-planar. UPPSALA UNIVERSITET Matematiska institutionen Anders Johansson Graph Theory Frist, KandMa, IT 010 10 1 Problem sheet 4 Exam questions Solve a subset of, say, four questions to the problem session on friday.

More information

MATH 363 Final Wednesday, April 28. Final exam. You may use lemmas and theorems that were proven in class and on assignments unless stated otherwise.

MATH 363 Final Wednesday, April 28. Final exam. You may use lemmas and theorems that were proven in class and on assignments unless stated otherwise. Final exam This is a closed book exam. No calculators are allowed. Unless stated otherwise, justify all your steps. You may use lemmas and theorems that were proven in class and on assignments unless stated

More information

K 4 C 5. Figure 4.5: Some well known family of graphs

K 4 C 5. Figure 4.5: Some well known family of graphs 08 CHAPTER. TOPICS IN CLASSICAL GRAPH THEORY K, K K K, K K, K K, K C C C C 6 6 P P P P P. Graph Operations Figure.: Some well known family of graphs A graph Y = (V,E ) is said to be a subgraph of a graph

More information

Matching Algorithms. Proof. If a bipartite graph has a perfect matching, then it is easy to see that the right hand side is a necessary condition.

Matching Algorithms. Proof. If a bipartite graph has a perfect matching, then it is easy to see that the right hand side is a necessary condition. 18.433 Combinatorial Optimization Matching Algorithms September 9,14,16 Lecturer: Santosh Vempala Given a graph G = (V, E), a matching M is a set of edges with the property that no two of the edges have

More information

Graph Connectivity G G G

Graph Connectivity G G G Graph Connectivity 1 Introduction We have seen that trees are minimally connected graphs, i.e., deleting any edge of the tree gives us a disconnected graph. What makes trees so susceptible to edge deletions?

More information

MATH 350 GRAPH THEORY & COMBINATORICS. Contents

MATH 350 GRAPH THEORY & COMBINATORICS. Contents MATH 350 GRAPH THEORY & COMBINATORICS PROF. SERGEY NORIN, FALL 2013 Contents 1. Basic definitions 1 2. Connectivity 2 3. Trees 3 4. Spanning Trees 3 5. Shortest paths 4 6. Eulerian & Hamiltonian cycles

More information

Assignment 4 Solutions of graph problems

Assignment 4 Solutions of graph problems Assignment 4 Solutions of graph problems 1. Let us assume that G is not a cycle. Consider the maximal path in the graph. Let the end points of the path be denoted as v 1, v k respectively. If either of

More information

Matching Theory. Figure 1: Is this graph bipartite?

Matching Theory. Figure 1: Is this graph bipartite? Matching Theory 1 Introduction A matching M of a graph is a subset of E such that no two edges in M share a vertex; edges which have this property are called independent edges. A matching M is said to

More information

Adjacent: Two distinct vertices u, v are adjacent if there is an edge with ends u, v. In this case we let uv denote such an edge.

Adjacent: Two distinct vertices u, v are adjacent if there is an edge with ends u, v. In this case we let uv denote such an edge. 1 Graph Basics What is a graph? Graph: a graph G consists of a set of vertices, denoted V (G), a set of edges, denoted E(G), and a relation called incidence so that each edge is incident with either one

More information

Definition For vertices u, v V (G), the distance from u to v, denoted d(u, v), in G is the length of a shortest u, v-path. 1

Definition For vertices u, v V (G), the distance from u to v, denoted d(u, v), in G is the length of a shortest u, v-path. 1 Graph fundamentals Bipartite graph characterization Lemma. If a graph contains an odd closed walk, then it contains an odd cycle. Proof strategy: Consider a shortest closed odd walk W. If W is not a cycle,

More information

Problem Set 3. MATH 776, Fall 2009, Mohr. November 30, 2009

Problem Set 3. MATH 776, Fall 2009, Mohr. November 30, 2009 Problem Set 3 MATH 776, Fall 009, Mohr November 30, 009 1 Problem Proposition 1.1. Adding a new edge to a maximal planar graph of order at least 6 always produces both a T K 5 and a T K 3,3 subgraph. Proof.

More information

PACKING DIGRAPHS WITH DIRECTED CLOSED TRAILS

PACKING DIGRAPHS WITH DIRECTED CLOSED TRAILS PACKING DIGRAPHS WITH DIRECTED CLOSED TRAILS PAUL BALISTER Abstract It has been shown [Balister, 2001] that if n is odd and m 1,, m t are integers with m i 3 and t i=1 m i = E(K n) then K n can be decomposed

More information

Key Graph Theory Theorems

Key Graph Theory Theorems Key Graph Theory Theorems Rajesh Kumar MATH 239 Intro to Combinatorics August 19, 2008 3.3 Binary Trees 3.3.1 Problem (p.82) Determine the number, t n, of binary trees with n edges. The number of binary

More information

Math 170- Graph Theory Notes

Math 170- Graph Theory Notes 1 Math 170- Graph Theory Notes Michael Levet December 3, 2018 Notation: Let n be a positive integer. Denote [n] to be the set {1, 2,..., n}. So for example, [3] = {1, 2, 3}. To quote Bud Brown, Graph theory

More information

Characterizing Graphs (3) Characterizing Graphs (1) Characterizing Graphs (2) Characterizing Graphs (4)

Characterizing Graphs (3) Characterizing Graphs (1) Characterizing Graphs (2) Characterizing Graphs (4) S-72.2420/T-79.5203 Basic Concepts 1 S-72.2420/T-79.5203 Basic Concepts 3 Characterizing Graphs (1) Characterizing Graphs (3) Characterizing a class G by a condition P means proving the equivalence G G

More information

9 Connectivity. Contents. 9.1 Vertex Connectivity

9 Connectivity. Contents. 9.1 Vertex Connectivity 9 Connectivity Contents 9.1 Vertex Connectivity.............................. 205 Connectivity and Local Connectivity............... 206 Vertex Cuts and Menger s Theorem................. 207 9.2 The Fan

More information

Lecture 6: Graph Properties

Lecture 6: Graph Properties Lecture 6: Graph Properties Rajat Mittal IIT Kanpur In this section, we will look at some of the combinatorial properties of graphs. Initially we will discuss independent sets. The bulk of the content

More information

Chapter 3: Paths and Cycles

Chapter 3: Paths and Cycles Chapter 3: Paths and Cycles 5 Connectivity 1. Definitions: Walk: finite sequence of edges in which any two consecutive edges are adjacent or identical. (Initial vertex, Final vertex, length) Trail: walk

More information

Math 776 Homework. Austin Mohr. June 15, Theorem 1.1. The following assertions are equivalent for a graph T : (i) T is a tree;

Math 776 Homework. Austin Mohr. June 15, Theorem 1.1. The following assertions are equivalent for a graph T : (i) T is a tree; Math 776 Homework Austin Mohr June 15, 2012 1 Problem 1 Theorem 1.1. The following assertions are equivalent for a graph T : (i) T is a tree; (ii) Any two vertices of T are linked by a unique path in T

More information

Number Theory and Graph Theory

Number Theory and Graph Theory 1 Number Theory and Graph Theory Chapter 6 Basic concepts and definitions of graph theory By A. Satyanarayana Reddy Department of Mathematics Shiv Nadar University Uttar Pradesh, India E-mail: satya8118@gmail.com

More information

Vertex coloring, chromatic number

Vertex coloring, chromatic number Vertex coloring, chromatic number A k-coloring of a graph G is a labeling f : V (G) S, where S = k. The labels are called colors; the vertices of one color form a color class. A k-coloring is proper if

More information

Graph Theory S 1 I 2 I 1 S 2 I 1 I 2

Graph Theory S 1 I 2 I 1 S 2 I 1 I 2 Graph Theory S I I S S I I S Graphs Definition A graph G is a pair consisting of a vertex set V (G), and an edge set E(G) ( ) V (G). x and y are the endpoints of edge e = {x, y}. They are called adjacent

More information

Two Characterizations of Hypercubes

Two Characterizations of Hypercubes Two Characterizations of Hypercubes Juhani Nieminen, Matti Peltola and Pasi Ruotsalainen Department of Mathematics, University of Oulu University of Oulu, Faculty of Technology, Mathematics Division, P.O.

More information

{ 1} Definitions. 10. Extremal graph theory. Problem definition Paths and cycles Complete subgraphs

{ 1} Definitions. 10. Extremal graph theory. Problem definition Paths and cycles Complete subgraphs Problem definition Paths and cycles Complete subgraphs 10. Extremal graph theory 10.1. Definitions Let us examine the following forbidden subgraph problems: At most how many edges are in a graph of order

More information

Theorem 3.1 (Berge) A matching M in G is maximum if and only if there is no M- augmenting path.

Theorem 3.1 (Berge) A matching M in G is maximum if and only if there is no M- augmenting path. 3 Matchings Hall s Theorem Matching: A matching in G is a subset M E(G) so that no edge in M is a loop, and no two edges in M are incident with a common vertex. A matching M is maximal if there is no matching

More information

On vertex-coloring edge-weighting of graphs

On vertex-coloring edge-weighting of graphs Front. Math. China DOI 10.1007/s11464-009-0014-8 On vertex-coloring edge-weighting of graphs Hongliang LU 1, Xu YANG 1, Qinglin YU 1,2 1 Center for Combinatorics, Key Laboratory of Pure Mathematics and

More information

Lecture Notes on Graph Theory

Lecture Notes on Graph Theory Lecture Notes on Graph Theory Vadim Lozin 1 Introductory concepts A graph G = (V, E) consists of two finite sets V and E. The elements of V are called the vertices and the elements of E the edges of G.

More information

Combinatorics Summary Sheet for Exam 1 Material 2019

Combinatorics Summary Sheet for Exam 1 Material 2019 Combinatorics Summary Sheet for Exam 1 Material 2019 1 Graphs Graph An ordered three-tuple (V, E, F ) where V is a set representing the vertices, E is a set representing the edges, and F is a function

More information

Basic Combinatorics. Math 40210, Section 01 Fall Homework 4 Solutions

Basic Combinatorics. Math 40210, Section 01 Fall Homework 4 Solutions Basic Combinatorics Math 40210, Section 01 Fall 2012 Homework 4 Solutions 1.4.2 2: One possible implementation: Start with abcgfjiea From edge cd build, using previously unmarked edges: cdhlponminjkghc

More information

Module 11. Directed Graphs. Contents

Module 11. Directed Graphs. Contents Module 11 Directed Graphs Contents 11.1 Basic concepts......................... 256 Underlying graph of a digraph................ 257 Out-degrees and in-degrees.................. 258 Isomorphism..........................

More information

Bipartite Roots of Graphs

Bipartite Roots of Graphs Bipartite Roots of Graphs Lap Chi Lau Department of Computer Science University of Toronto Graph H is a root of graph G if there exists a positive integer k such that x and y are adjacent in G if and only

More information

Fundamental Properties of Graphs

Fundamental Properties of Graphs Chapter three In many real-life situations we need to know how robust a graph that represents a certain network is, how edges or vertices can be removed without completely destroying the overall connectivity,

More information

Vertex coloring, chromatic number

Vertex coloring, chromatic number Vertex coloring, chromatic number A k-coloring of a graph G is a labeling f : V (G) S, where S = k. The labels are called colors; the vertices of one color form a color class. A k-coloring is proper if

More information

by conservation of flow, hence the cancelation. Similarly, we have

by conservation of flow, hence the cancelation. Similarly, we have Chapter 13: Network Flows and Applications Network: directed graph with source S and target T. Non-negative edge weights represent capacities. Assume no edges into S or out of T. (If necessary, we can

More information

On the Relationships between Zero Forcing Numbers and Certain Graph Coverings

On the Relationships between Zero Forcing Numbers and Certain Graph Coverings On the Relationships between Zero Forcing Numbers and Certain Graph Coverings Fatemeh Alinaghipour Taklimi, Shaun Fallat 1,, Karen Meagher 2 Department of Mathematics and Statistics, University of Regina,

More information

Triple Connected Domination Number of a Graph

Triple Connected Domination Number of a Graph International J.Math. Combin. Vol.3(2012), 93-104 Triple Connected Domination Number of a Graph G.Mahadevan, Selvam Avadayappan, J.Paulraj Joseph and T.Subramanian Department of Mathematics Anna University:

More information

Characterizations of graph classes by forbidden configurations

Characterizations of graph classes by forbidden configurations Characterizations of graph classes by forbidden configurations Zdeněk Dvořák September 14, 2015 We consider graph classes that can be described by excluding some fixed configurations. Let us give some

More information

A graph is finite if its vertex set and edge set are finite. We call a graph with just one vertex trivial and all other graphs nontrivial.

A graph is finite if its vertex set and edge set are finite. We call a graph with just one vertex trivial and all other graphs nontrivial. 2301-670 Graph theory 1.1 What is a graph? 1 st semester 2550 1 1.1. What is a graph? 1.1.2. Definition. A graph G is a triple (V(G), E(G), ψ G ) consisting of V(G) of vertices, a set E(G), disjoint from

More information

Problem Set 2 Solutions

Problem Set 2 Solutions Problem Set 2 Solutions Graph Theory 2016 EPFL Frank de Zeeuw & Claudiu Valculescu 1. Prove that the following statements about a graph G are equivalent. - G is a tree; - G is minimally connected (it is

More information

1 Matchings in Graphs

1 Matchings in Graphs Matchings in Graphs J J 2 J 3 J 4 J 5 J J J 6 8 7 C C 2 C 3 C 4 C 5 C C 7 C 8 6 J J 2 J 3 J 4 J 5 J J J 6 8 7 C C 2 C 3 C 4 C 5 C C 7 C 8 6 Definition Two edges are called independent if they are not adjacent

More information

5.1 Min-Max Theorem for General Matching

5.1 Min-Max Theorem for General Matching CSC5160: Combinatorial Optimization and Approximation Algorithms Topic: General Matching Date: 4/01/008 Lecturer: Lap Chi Lau Scribe: Jennifer X.M. WU In this lecture, we discuss matchings in general graph.

More information

DO NOT RE-DISTRIBUTE THIS SOLUTION FILE

DO NOT RE-DISTRIBUTE THIS SOLUTION FILE Professor Kindred Math 104, Graph Theory Homework 2 Solutions February 7, 2013 Introduction to Graph Theory, West Section 1.2: 26, 38, 42 Section 1.3: 14, 18 Section 2.1: 26, 29, 30 DO NOT RE-DISTRIBUTE

More information

Math 776 Graph Theory Lecture Note 1 Basic concepts

Math 776 Graph Theory Lecture Note 1 Basic concepts Math 776 Graph Theory Lecture Note 1 Basic concepts Lectured by Lincoln Lu Transcribed by Lincoln Lu Graph theory was founded by the great Swiss mathematician Leonhard Euler (1707-178) after he solved

More information

Sources for this lecture. 3. Matching in bipartite and general graphs. Symmetric difference

Sources for this lecture. 3. Matching in bipartite and general graphs. Symmetric difference S-72.2420 / T-79.5203 Matching in bipartite and general graphs 1 3. Matching in bipartite and general graphs Let G be a graph. A matching M in G is a set of nonloop edges with no shared endpoints. Let

More information

Subdivisions of Graphs: A Generalization of Paths and Cycles

Subdivisions of Graphs: A Generalization of Paths and Cycles Subdivisions of Graphs: A Generalization of Paths and Cycles Ch. Sobhan Babu and Ajit A. Diwan Department of Computer Science and Engineering, Indian Institute of Technology Bombay, Powai, Mumbai 400076,

More information

Chapter 2 Graphs. 2.1 Definition of Graphs

Chapter 2 Graphs. 2.1 Definition of Graphs Chapter 2 Graphs Abstract Graphs are discrete structures that consist of vertices and edges connecting some of these vertices. Graphs have many applications in Mathematics, Computer Science, Engineering,

More information

HW Graph Theory SOLUTIONS (hbovik) - Q

HW Graph Theory SOLUTIONS (hbovik) - Q 1, Diestel 9.3: An arithmetic progression is an increasing sequence of numbers of the form a, a+d, a+ d, a + 3d.... Van der Waerden s theorem says that no matter how we partition the natural numbers into

More information

Lecture 3: Recap. Administrivia. Graph theory: Historical Motivation. COMP9020 Lecture 4 Session 2, 2017 Graphs and Trees

Lecture 3: Recap. Administrivia. Graph theory: Historical Motivation. COMP9020 Lecture 4 Session 2, 2017 Graphs and Trees Administrivia Lecture 3: Recap Assignment 1 due 23:59 tomorrow. Quiz 4 up tonight, due 15:00 Thursday 31 August. Equivalence relations: (S), (R), (T) Total orders: (AS), (R), (T), (L) Partial orders: (AS),

More information

Advanced Combinatorial Optimization September 17, Lecture 3. Sketch some results regarding ear-decompositions and factor-critical graphs.

Advanced Combinatorial Optimization September 17, Lecture 3. Sketch some results regarding ear-decompositions and factor-critical graphs. 18.438 Advanced Combinatorial Optimization September 17, 2009 Lecturer: Michel X. Goemans Lecture 3 Scribe: Aleksander Madry ( Based on notes by Robert Kleinberg and Dan Stratila.) In this lecture, we

More information

Characterizations of Trees

Characterizations of Trees Characterizations of Trees Lemma Every tree with at least two vertices has at least two leaves. Proof. 1. A connected graph with at least two vertices has an edge. 2. In an acyclic graph, an end point

More information

Matchings in Graphs. Definition 1 Let G = (V, E) be a graph. M E is called as a matching of G if v V we have {e M : v is incident on e E} 1.

Matchings in Graphs. Definition 1 Let G = (V, E) be a graph. M E is called as a matching of G if v V we have {e M : v is incident on e E} 1. Lecturer: Scribe: Meena Mahajan Rajesh Chitnis Matchings in Graphs Meeting: 1 6th Jan 010 Most of the material in this lecture is taken from the book Fast Parallel Algorithms for Graph Matching Problems

More information

Ma/CS 6b Class 4: Matchings in General Graphs

Ma/CS 6b Class 4: Matchings in General Graphs Ma/CS 6b Class 4: Matchings in General Graphs By Adam Sheffer Reminder: Hall's Marriage Theorem Theorem. Let G = V 1 V 2, E be a bipartite graph. There exists a matching of size V 1 in G if and only if

More information

8 Colouring Planar Graphs

8 Colouring Planar Graphs 8 Colouring Planar Graphs The Four Colour Theorem Lemma 8.1 If G is a simple planar graph, then (i) 12 v V (G)(6 deg(v)) with equality for triangulations. (ii) G has a vertex of degree 5. Proof: For (i),

More information

5 Matchings in Bipartite Graphs and Their Applications

5 Matchings in Bipartite Graphs and Their Applications 5 Matchings in Bipartite Graphs and Their Applications 5.1 Matchings Definition 5.1 A matching M in a graph G is a set of edges of G, none of which is a loop, such that no two edges in M have a common

More information

CMSC Honors Discrete Mathematics

CMSC Honors Discrete Mathematics CMSC 27130 Honors Discrete Mathematics Lectures by Alexander Razborov Notes by Justin Lubin The University of Chicago, Autumn 2017 1 Contents I Number Theory 4 1 The Euclidean Algorithm 4 2 Mathematical

More information

Weak Dynamic Coloring of Planar Graphs

Weak Dynamic Coloring of Planar Graphs Weak Dynamic Coloring of Planar Graphs Caroline Accurso 1,5, Vitaliy Chernyshov 2,5, Leaha Hand 3,5, Sogol Jahanbekam 2,4,5, and Paul Wenger 2 Abstract The k-weak-dynamic number of a graph G is the smallest

More information

1 Matchings with Tutte s Theorem

1 Matchings with Tutte s Theorem 1 Matchings with Tutte s Theorem Last week we saw a fairly strong necessary criterion for a graph to have a perfect matching. Today we see that this condition is in fact sufficient. Theorem 1 (Tutte, 47).

More information

Bounds on distances for spanning trees of graphs. Mr Mthobisi Luca Ntuli

Bounds on distances for spanning trees of graphs. Mr Mthobisi Luca Ntuli Bounds on distances for spanning trees of graphs Mr Mthobisi Luca Ntuli March 8, 2018 To Mphemba Legacy iii Acknowledgments I would like to thank my supervisors, Dr MJ Morgan and Prof S Mukwembi. It

More information

Graph theory. Po-Shen Loh. June We begin by collecting some basic facts which can be proved via bare-hands techniques.

Graph theory. Po-Shen Loh. June We begin by collecting some basic facts which can be proved via bare-hands techniques. Graph theory Po-Shen Loh June 013 1 Basic results We begin by collecting some basic facts which can be proved via bare-hands techniques. 1. The sum of all of the degrees is equal to twice the number of

More information

AMS /672: Graph Theory Homework Problems - Week V. Problems to be handed in on Wednesday, March 2: 6, 8, 9, 11, 12.

AMS /672: Graph Theory Homework Problems - Week V. Problems to be handed in on Wednesday, March 2: 6, 8, 9, 11, 12. AMS 550.47/67: Graph Theory Homework Problems - Week V Problems to be handed in on Wednesday, March : 6, 8, 9,,.. Assignment Problem. Suppose we have a set {J, J,..., J r } of r jobs to be filled by a

More information

Chromatic Transversal Domatic Number of Graphs

Chromatic Transversal Domatic Number of Graphs International Mathematical Forum, 5, 010, no. 13, 639-648 Chromatic Transversal Domatic Number of Graphs L. Benedict Michael Raj 1, S. K. Ayyaswamy and I. Sahul Hamid 3 1 Department of Mathematics, St.

More information

Some Upper Bounds for Signed Star Domination Number of Graphs. S. Akbari, A. Norouzi-Fard, A. Rezaei, R. Rotabi, S. Sabour.

Some Upper Bounds for Signed Star Domination Number of Graphs. S. Akbari, A. Norouzi-Fard, A. Rezaei, R. Rotabi, S. Sabour. Some Upper Bounds for Signed Star Domination Number of Graphs S. Akbari, A. Norouzi-Fard, A. Rezaei, R. Rotabi, S. Sabour Abstract Let G be a graph with the vertex set V (G) and edge set E(G). A function

More information

6. Lecture notes on matroid intersection

6. Lecture notes on matroid intersection Massachusetts Institute of Technology 18.453: Combinatorial Optimization Michel X. Goemans May 2, 2017 6. Lecture notes on matroid intersection One nice feature about matroids is that a simple greedy algorithm

More information

Discrete Mathematics I So Practice Sheet Solutions 1

Discrete Mathematics I So Practice Sheet Solutions 1 Discrete Mathematics I So 2016 Tibor Szabó Shagnik Das Practice Sheet Solutions 1 Provided below are possible solutions to the questions from the practice sheet issued towards the end of the course. Exercise

More information

Graph Theory Day Four

Graph Theory Day Four Graph Theory Day Four February 8, 018 1 Connected Recall from last class, we discussed methods for proving a graph was connected. Our two methods were 1) Based on the definition, given any u, v V(G), there

More information

Topics in Combinatorial Optimization February 5, Lecture 2

Topics in Combinatorial Optimization February 5, Lecture 2 8.997 Topics in Combinatorial Optimization February 5, 2004 Lecture 2 Lecturer: Michel X. Goemans Scribe: Robert Kleinberg In this lecture, we will: Present Edmonds algorithm for computing a maximum matching

More information

Discrete mathematics II. - Graphs

Discrete mathematics II. - Graphs Emil Vatai April 25, 2018 Basic definitions Definition of an undirected graph Definition (Undirected graph) An undirected graph or (just) a graph is a triplet G = (ϕ, E, V ), where V is the set of vertices,

More information

5 Graphs

5 Graphs 5 Graphs jacques@ucsd.edu Some of the putnam problems are to do with graphs. They do not assume more than a basic familiarity with the definitions and terminology of graph theory. 5.1 Basic definitions

More information

2. Lecture notes on non-bipartite matching

2. Lecture notes on non-bipartite matching Massachusetts Institute of Technology 18.433: Combinatorial Optimization Michel X. Goemans February 15th, 013. Lecture notes on non-bipartite matching Given a graph G = (V, E), we are interested in finding

More information

Elements of Graph Theory

Elements of Graph Theory Elements of Graph Theory Quick review of Chapters 9.1 9.5, 9.7 (studied in Mt1348/2008) = all basic concepts must be known New topics we will mostly skip shortest paths (Chapter 9.6), as that was covered

More information

Pebble Sets in Convex Polygons

Pebble Sets in Convex Polygons 2 1 Pebble Sets in Convex Polygons Kevin Iga, Randall Maddox June 15, 2005 Abstract Lukács and András posed the problem of showing the existence of a set of n 2 points in the interior of a convex n-gon

More information

Small Survey on Perfect Graphs

Small Survey on Perfect Graphs Small Survey on Perfect Graphs Michele Alberti ENS Lyon December 8, 2010 Abstract This is a small survey on the exciting world of Perfect Graphs. We will see when a graph is perfect and which are families

More information

Chapter 6 GRAPH COLORING

Chapter 6 GRAPH COLORING Chapter 6 GRAPH COLORING A k-coloring of (the vertex set of) a graph G is a function c : V (G) {1, 2,..., k} such that c (u) 6= c (v) whenever u is adjacent to v. Ifak-coloring of G exists, then G is called

More information

Graph Theory. Connectivity, Coloring, Matching. Arjun Suresh 1. 1 GATE Overflow

Graph Theory. Connectivity, Coloring, Matching. Arjun Suresh 1. 1 GATE Overflow Graph Theory Connectivity, Coloring, Matching Arjun Suresh 1 1 GATE Overflow GO Classroom, August 2018 Thanks to Subarna/Sukanya Das for wonderful figures Arjun, Suresh (GO) Graph Theory GATE 2019 1 /

More information

Modules. 6 Hamilton Graphs (4-8 lectures) Introduction Necessary conditions and sufficient conditions Exercises...

Modules. 6 Hamilton Graphs (4-8 lectures) Introduction Necessary conditions and sufficient conditions Exercises... Modules 6 Hamilton Graphs (4-8 lectures) 135 6.1 Introduction................................ 136 6.2 Necessary conditions and sufficient conditions............. 137 Exercises..................................

More information

Abstract. A graph G is perfect if for every induced subgraph H of G, the chromatic number of H is equal to the size of the largest clique of H.

Abstract. A graph G is perfect if for every induced subgraph H of G, the chromatic number of H is equal to the size of the largest clique of H. Abstract We discuss a class of graphs called perfect graphs. After defining them and getting intuition with a few simple examples (and one less simple example), we present a proof of the Weak Perfect Graph

More information

ECS 20 Lecture 17b = Discussion D8 Fall Nov 2013 Phil Rogaway

ECS 20 Lecture 17b = Discussion D8 Fall Nov 2013 Phil Rogaway 1 ECS 20 Lecture 17b = Discussion D8 Fall 2013 25 Nov 2013 Phil Rogaway Today: Using discussion section to finish up graph theory. Much of these notes the same as those prepared for last lecture and the

More information

Applied Mathematical Sciences, Vol. 5, 2011, no. 49, Július Czap

Applied Mathematical Sciences, Vol. 5, 2011, no. 49, Július Czap Applied Mathematical Sciences, Vol. 5, 011, no. 49, 437-44 M i -Edge Colorings of Graphs Július Czap Department of Applied Mathematics and Business Informatics Faculty of Economics, Technical University

More information

γ(ɛ) (a, b) (a, d) (d, a) (a, b) (c, d) (d, d) (e, e) (e, a) (e, e) (a) Draw a picture of G.

γ(ɛ) (a, b) (a, d) (d, a) (a, b) (c, d) (d, d) (e, e) (e, a) (e, e) (a) Draw a picture of G. MAD 3105 Spring 2006 Solutions for Review for Test 2 1. Define a graph G with V (G) = {a, b, c, d, e}, E(G) = {r, s, t, u, v, w, x, y, z} and γ, the function defining the edges, is given by the table ɛ

More information

How many colors are needed to color a map?

How many colors are needed to color a map? How many colors are needed to color a map? Is 4 always enough? Two relevant concepts How many colors do we need to color a map so neighboring countries get different colors? Simplifying assumption (not

More information

The Restrained Edge Geodetic Number of a Graph

The Restrained Edge Geodetic Number of a Graph International Journal of Computational and Applied Mathematics. ISSN 0973-1768 Volume 11, Number 1 (2016), pp. 9 19 Research India Publications http://www.ripublication.com/ijcam.htm The Restrained Edge

More information

Graph Theory: Matchings and Factors

Graph Theory: Matchings and Factors Graph Theory: Matchings and Factors Pallab Dasgupta, Professor, Dept. of Computer Sc. and Engineering, IIT Kharagpur pallab@cse.iitkgp.ernet.in Matchings A matching of size k in a graph G is a set of k

More information

CLAW-FREE 3-CONNECTED P 11 -FREE GRAPHS ARE HAMILTONIAN

CLAW-FREE 3-CONNECTED P 11 -FREE GRAPHS ARE HAMILTONIAN CLAW-FREE 3-CONNECTED P 11 -FREE GRAPHS ARE HAMILTONIAN TOMASZ LUCZAK AND FLORIAN PFENDER Abstract. We show that every 3-connected claw-free graph which contains no induced copy of P 11 is hamiltonian.

More information

16 1. The Basics. x = t 1 >...>t k <...<t n = y

16 1. The Basics. x = t 1 >...>t k <...<t n = y 16 1. The Basics [8.2.3] [8.6.8] Lemma 1.5.5. Let T be a normal tree in G. (i) Any two vertices x, y T are separated in G by the set x y. (ii) If S V (T )=V(G) and S is down-closed, then the components

More information

Week 9-10: Connectivity

Week 9-10: Connectivity Week 9-0: Connectiity October 3, 206 Vertex Connectiity Let G = (V, E) be a graph. Gien two ertices x, y V. Two (x, y)-path are said to be internally disjoint if they hae no internal ertices in common.

More information

Solution for Homework set 3

Solution for Homework set 3 TTIC 300 and CMSC 37000 Algorithms Winter 07 Solution for Homework set 3 Question (0 points) We are given a directed graph G = (V, E), with two special vertices s and t, and non-negative integral capacities

More information

Restricted edge connectivity and restricted connectivity of graphs

Restricted edge connectivity and restricted connectivity of graphs Restricted edge connectivity and restricted connectivity of graphs Litao Guo School of Applied Mathematics Xiamen University of Technology Xiamen Fujian 361024 P.R.China ltguo2012@126.com Xiaofeng Guo

More information

Matching and Covering

Matching and Covering Matching and Covering Matchings A matching of size k in a graph G is a set of k pairwise disjoint edges The vertices belonging to the edges of a matching are saturated by the matching; the others are unsaturated

More information

Topics in Combinatorics. Dorottya Sziráki Gergő Nemes

Topics in Combinatorics. Dorottya Sziráki Gergő Nemes Topics in Combinatorics Dorottya Sziráki Gergő Nemes ii Preface These notes are based on the lectures of the course titled Topics in Combinatorics, which were given by Ervin Győri in the winter trimester

More information

DO NOT RE-DISTRIBUTE THIS SOLUTION FILE

DO NOT RE-DISTRIBUTE THIS SOLUTION FILE Professor Kindred Math 104, Graph Theory Homework 3 Solutions February 14, 2013 Introduction to Graph Theory, West Section 2.1: 37, 62 Section 2.2: 6, 7, 15 Section 2.3: 7, 10, 14 DO NOT RE-DISTRIBUTE

More information

Mathematical and Algorithmic Foundations Linear Programming and Matchings

Mathematical and Algorithmic Foundations Linear Programming and Matchings Adavnced Algorithms Lectures Mathematical and Algorithmic Foundations Linear Programming and Matchings Paul G. Spirakis Department of Computer Science University of Patras and Liverpool Paul G. Spirakis

More information

MATH 682 Notes Combinatorics and Graph Theory II. One interesting class of graphs rather akin to trees and acyclic graphs is the bipartite graph:

MATH 682 Notes Combinatorics and Graph Theory II. One interesting class of graphs rather akin to trees and acyclic graphs is the bipartite graph: 1 Bipartite graphs One interesting class of graphs rather akin to trees and acyclic graphs is the bipartite graph: Definition 1. A graph G is bipartite if the vertex-set of G can be partitioned into two

More information

Some Elementary Lower Bounds on the Matching Number of Bipartite Graphs

Some Elementary Lower Bounds on the Matching Number of Bipartite Graphs Some Elementary Lower Bounds on the Matching Number of Bipartite Graphs Ermelinda DeLaViña and Iride Gramajo Department of Computer and Mathematical Sciences University of Houston-Downtown Houston, Texas

More information

Planar graphs. Chapter 8

Planar graphs. Chapter 8 Chapter 8 Planar graphs Definition 8.1. A graph is called planar if it can be drawn in the plane so that edges intersect only at vertices to which they are incident. Example 8.2. Different representations

More information