be a path in L G ; we can associated to P the following alternating sequence of vertices and edges in G:

Size: px
Start display at page:

Download "be a path in L G ; we can associated to P the following alternating sequence of vertices and edges in G:"

Transcription

1 1. The line graph of a graph. Let G = (V, E) be a graph with E. The line graph of G is the graph L G such that V (L G ) = E and E(L G ) = {ef : e, f E : e and f are adjacent}. Examples 1.1. (1) If G is a path of length n, then L G is a path of length n 1. (2) If G is a cycle of length n, then L G = G. (3) If G is a star with n vertices i.e. G 3 and G has a vertex u such that E = {vu, v V {u}}, then L G = K n 1. The converses also hold, see Exercise 1.6. For an edge uv V we write (uv) V (L G ) for the corresponding vertex of the line graph. But we abuse notation using the same symbol for edges, or subsets of edges, in G and vertices, or subsets of vertices, in L G. Lemma 1.2. Let G be a graph with E(G). Then (1) E(L G ) = ( ) d(v) ; 2 v V (2) for any F E(G) we have L G F = L G F ; (3) for any v V (G) we have L G v = L G E(v). Proof. For any v V (G), every pair of edges in E(v) corresponds to an edge in L G, and all the edges of L G are obtained in this way. Hence the first formula follows. The remaining two identitities follow trivially from the definition. Let P = e 0... e m L G be a path in L G ; we can associated to P the following alternating sequence of vertices and edges in G: w 0, e 0, w 1, e 1,... w m, e m, w m+1, where w i V (G) are such that e 0 = w 0 w 1, e m = w m w m+1 and w i is the vertex adjacent to e i 1 and e i for i = 1,..., m. By definition w 0 w 1 and w m w m+1, while we may have w i = w j for the remaining cases; see Example 1.4. From the above sequence we extract the following sequence of (not necessarily distinct) vertices in G (1.1) ω(p ) := (w 0, w 1,..., w m, w m+1 ). We shall use this notation in the next basic Lemma. Lemma - Definition 1.3. Let G be a graph and L G its line graph. (1) Let Q = v 0... v n G be a path. L Q is a path in L G. (2) Let P L G be a path such that ω(p ) consists of distinct vertices. Then there exists a path Q P G such that P = L QP. We have and V (Q P ) = ω(p ) length(q P ) = length(p ) + 1 1

2 2 (3) Fix e, f E(G) and let P L G be an ef-path of minimal length. Then P satisfies the assumption of (2). (4) Let P L G be an ef-path. Then there exists an ef-path P L G such that ω(p ) ω(p ) and such that P satisfies the assumption of (2). Proof. (1). Let Q = v 0... v n be a path in G, we already noticed that L Q is a path. Now v i v i+1 E and hence (v i v i+1 ) is a vertex of L G ; as the v i are all distinct, the (v i v i+1 ) are all distinct. Now, the edges v i v i+1 and v i 1 v i are adjacent for all i 1, hence (v i 1 v i )(v i v i+1 ) is an edge of L G. Therefore L Q L G. (2). Keeping the above notation, assume w 0,..., w m+1 are all distinct. By definition, G has the edge w i w i+1 = e i for all i m, hence Q = w 0 w 1... w m+1 is a path in G. Finally, L Q = P since, as we just noticed, the vertex (w i w i+1 ) equals the vertex e i in L G. We set Q = Q P and we are done. (3). We need to prove that if P = e 0... e m has minimal length between e = e 0 and f = e m, then the elements in ω(p ) are all distinct. By contradiction, let h be minimum such that there exists k > h with w h = w k. If h > 0 then e h 1 is adjacent to e k, hence (1.2) P 1 = e 0... e h 1 e k... e m is a path from e to f shorter than P, which is not possible. If h = 0 then k 2, hence the following (1.3) P 2 = e 0 e k... e m is too short a path from e to f, a contradiction. (4). Let P = e 0... e m be a path from e = e 0 to f = e m and ω(p ) = (w 0, w 1,..., w m+1 ) the associated sequence of vertices. If ω(p ) has no multiple vertices (i.e. if w i w j for all i j) then, by (2), we can take P = P and we are done. We shall prove (4) by induction on the number of multiple vertices in ω(p ), i.e. the number M P = {i = 0,..., m + 1 : j i : w i = w j }. The induction base, M P = 0, has already been treated. Let h be minimum such that there exists k > h with w h = w k. Then, arguing exactly as in the proof of (3), we construct a shorter path from e to f. More precisely, if h > 0, then the path is P 1, given in (1.2), and ω(p 1 ) = (w 0, w 1,..., w h, w k+1,... w m+1 ) ω(p ) with h < k; thus the multiple vertex w k is not in ω(p 1 ), hence M P1 M P 1. The iduction hypotesis gives an ef-path P 1 satisfying (2) and such that ω(p 1 ) ω(p 1 ) ω(p ). So we are done. In the case where the path is P 2, given in (1.3), we have ω(p 2 ) = (w 1, w 0, w k+1,... w m+1 ) ω(p ) with k 2, so the same argument as before applies. The next example illustrates parts of the Lemma and of its proof.

3 3 Example 1.4. In the picture below we have a star graph, G, and its line graph, where we highlighted the path P described in the sequel. In G we set e i = v i v 0 for all i = 1,..., 5. Next, consider the following path in L G joining e 1 and e 5 P = e 1 e 3 e 4 e 2 e 5 L G hence ω(p ) = (v 1, v 0, v 0, v 0, v 0, v 5 ). The proof yields ω(p ) = (v 1, v 0, v 5 ) and P = e 1 e 5. Finally, Q P = v 1 v 0 v 5 G and, of course, L v1 v 0 v 5 = (v 1 v 0 )(v 0 v 5 ) = e 1 e 5. v 1 v 2 G = v 5 v 0 e 1 e 2 v 3 L G = e 5 e 3 v 4 e 4 Figure 1 Lemma 1.5. Let G = (V, E) be a graph and L G its line graph. G is connected if and only if L G is connected and δ(g) 1. Proof. Suppose G connected, let e = uw and f = xy be two edges of G; we need to find a path in L G between e and f. Let Q = uv 1... v n x be a ux-path in G of minimal length. Consider the path L Q L G. If L Q contains e and f we are done. If L Q does not contain e, then, by the minimality of Q, the vertex w is not in Q. Hence el Q is a path in L G containing e. If this path does not contain f, arguing as above we have the path el Q f contains e and f. So we are done. Conversely, assume L G connected and G free from isolated vertices. Fix x, y V (G); we need to find a path joining x and y. Pick two edges, e x and e y, adjacent to each of them (if e x = e y then we are done). Let P = e 0... e n be a path of minimal length in L G such that e x = e 0 and e y = e n. By Lemma 1.3 there exists a path Q P G such that L QP = P ; by part (2) of the Lemma the vertices of the path Q P are those in ω(p ), which contains x and y; so Q P contains x and y, and we are done. Exercise 1.6. Let G be such that δ(g) > 0. Prove the following. (1) If L G is a path of length n, then G is a path of length n + 1. (2) If L G is a cycle, then G = L G. (3) If L G = K n, then G is a star with n edges.

4 4 Exercise 1.7. Let G = (V, E) and e, f E such that e = xy and f = uv. Set M = min{d(x, u), d(x, v), d(y, u), d(y, v)}. Show that d LG (e, f) = M Connectivity via paths The definition of a connected graph is based on the notion of path. Indeed let G = (V, E) be a graph. Then, by definition, G is 1-connected if and only if for every x, y V there exists an xy-path P G. Next, already know that G is 2-connected if and only if for every x, y V there exist two independent xy-paths P 1, P 2 G (recall that to say that P 1 and P 2 are independent is to say that i.e. P 1 P 2 = {x, y}). We shall prove in Theorem 2.7 that the analog holds for every k. For now we prove the following result, which is the easy implication of Theorem 2.7. Proposition 2.1. Let G be a graph containing k independent xy-paths for every pair of vertices x, y. Then G is k-connected. Proof. To prove that G is k-connected pick a pair of vertices x, y any a set S V {x, y} separating x from y; we need to show that S k. Now, let P 1,..., P k be k independent xy-paths in G; then S each of them must intersect S, so let s i S V (P i ); since the P i are independent, we have s i s j for all i j; hence S k. The proof of the converse is non-trivial, and it is based on an important auxiliary result, interesting in its own right. To begin with, we introduce the following notation: for any graph G = (V, E) and any A, B V (not necessarily disjoint) we set (2.1) κ G (A, B) = min{ S : S V (G) : S separates A from B} and (2.2) π G (A, B) = maximum number of disjoint AB-paths in G. Example 2.2. Assume G connected. If A = {x} and B = {y} with x y we can separate x from y with {x}; moreover it is clear that two xy-paths will never be disjoint, hence κ G (x, y) = π G (x, y) = 1. Example 2.3. Suppose B = V. Then an AB-path P must be of type P = v with v A (for otherwise P would intersect B in two points, which is not possible). Hence π G (A, V ) = A ; now a set S intersecting every AB-path must contain A, therefore κ G (A, V ) = A Lemma 2.4. Let G = (V, E) be k-connected and let x, y V be distinct and not adjacent. Then k G (N(x), N(y)) k.

5 Proof. Set A = N(x) and B = N(y); to every xy-path we can associate an AB-path as follows {xy paths} {AB paths} xv 1... v n y v 1... v n which is well defined, as xy E. We denote by P be the image of the above map; observe that P is the set of AB-paths not containing x or y, and it is not empty, as G is connected. Let now S V be a set separating A and B. Then S intersects every path in P, hence S {x, y} intersects every path in P, hence S {x, y} intersects every xy-path, hence S {x, y} separates x and y. As G is k-connected, S {x, y} k and hence, a fortiori, S k. Therefore k G (A, B) k as wanted. Now, since every S V separating A and B must contain a vertex from every AB-path is clear that π G (A, B) κ G (A, B). It is quite remarkable that, just as in the previous example, equality holds in general, as the following theorem states. Theorem 2.5. Fix a graph G = (V, E) and two subsets A, B of V. Then the minimum number of vertices separating A and B equals the maximum number of disjoint AB-paths. In symbols π G (A, B) = κ G (A, B). Proof. By what we observed above, it suffices to show that G has at least κ G (A, B) disjoint AB-paths. We shall do that by proving the following claim. Let P be a set of disjoint AB-paths with P < κ G (A, B); then there exists a set P of disjoint AB-paths such that P = P + 1 and such that the set of endpoints in B of the paths in P contains the set of endpoints of the paths in P. We shall prove the claim by descending induction on B ; observe that the claim is stronger than the theorem, but the additional requirement on the endpoints is needed for the proof to work. The basis of the induction is the case B = V, which has been treated in Example 2.3 above. We set k = κ G (A, B). Let P be a set of AB-paths as above; to simplify the terminology, by an endpoint of P we shall mean an endpoint of a path in P. Let S be the set of endpoints of P lying in B; since S < k, by hypothesis S cannot separate A and B. Hence there exists an AB path, R, not contained in P. If R is disjoint from the paths in P we are done. If not, let v be the last vertex of R lying in a path, P, in P. Now consider the following set B V B = B V (vr) V (vp ) and the following set of disjoint AB -paths P = P {P } {P v} (P is gotten from P by replacing P with its truncation at v). By construction B B, hence k G (A, B ) k G (A, B), and hence P < k G (A, B ); therefore we can apply the induction hypothesis to B and P. 5

6 6 This gives a set, P, of P + 1 disjoint AB -paths whose endpoints in B contain the endpoints of the paths in P. In particular, P contains a path, P, from A to v and a path, Q, from A to a point y B other than the endpoints of P. Hence P {P, Q } is made of disjoint AB-paths; we will conclude the proof by showing how to replace P and Q with AB-paths so as to get a set P satisfying the claim. There are two possibilities, y vp or y vp. If y vp we replace P with P = P + vp and if y B, we replace Q with Q = Q + yr; if y B we leave Q = Q. If y vp we replace P with P = P + yr and we replace Q with Q = Q + yp. Finally, the set P := P {P, Q } {P, Q } is a set of P + 1 disjoint AB-paths, as we wanted. Corollary 2.6. Let G = (V, E) be k-connected; fix A V with A k and v V A. Then G contains k independent xa-paths with different endpoints in A. Proof. Set B = N(x); we claim k G (A, B) k. Indeed, let U V be such that U k 1; pick a A U and b B U; as G is k-connected G U is connected, hence it contains an ab-path. This shows that U does not separate A and B. By Theorem 2.5, G contains k disjoint BA-paths, P 1,..., P k. Now x P i, since x A; therefore xp 1,..., xp k are independent xa-paths with different endpoints in A. The previous Theorem 2.5 is a key ingredient in the proof of the following. Theorem 2.7 (Menger). A graph G is k-connected if and only if for every pair of vertices x, y it contains k independent xy-paths. Proof. We proved one implication in Proposition 2.1. We shall now show that for any x, y V distinct, G contains k independent xy-paths. We first assume x and y not adjacent. By Lemma 2.4 and Theorem 2.5 there exist k disjoint N(x)N(y)-paths in G, written P 1,..., P k. Set P i = v 0 v 1... v n ; we claim that P i does not contain x or y. Indeed if, say, x = v h then we have h 0 (for x N(x)) and h n (for x N(y)); hence v h 1 and v h+1 are in P N(x), which is not possible as P meets N(x) only in v 0. The claim is proved. As P i does not contain x or y the following P i := xv 0 v 1... v n y is an xypath for i = 1,..., k. It is clear that P 1,..., P k are independent xy-paths, so we are done. Now suppose x and y adjacent. By contradiction, assume G has at most k 1 independent xy-paths; hence G e has at most k 2 independent xypaths. Recall now that G e is (k 1)-connected, since G is k-connected. But then, by the previous part of the proof, G e has k 1 independent xy-paths, as x and y are not adjacent in G e. This is a contradiction. Exercise 2.8. Set k 3; show that in a k-connected graphs any k vertices lie in a common cycle. (The case k = 2 is already known.)

7 Exercise 2.9. Let G be a k-connected graph with at least 2k-vertices. Then G contains a cycle of length at least 2k. 3. Edge-connectivity Definition 3.1. Let k 0. The graph G = (V, E) is k-edge-connected if V > 1 and for any F E with F k 1 the graph G F is connected. Remark 3.2. (1) If G is k-connected, G is k-edge-connnected. (2) If G is k-edge-connnected, then δ(g) k. (3) G is 1-edge-connected if and only if it is 1-connected if and only if it is connected and not K 1. (4) G is 2-connected if and only if it is connected and has no bridges. Recall that for a graph G its line graph, introduced in Section 1, is denoted by L G. Proposition 3.3. A graph G is k-edge-connected if and only if L G is k- connected and δ(g) k. Proof. The first statement follows directly from the definition of line graph. For the second, we can assume k 2 by Lemma 1.5. Assume G is k-edge-connected, then δ(g) k and hence V (L G ) = E(G) > k (here we use k 2, exercise). Let F V (L G ) be such that the graph L G F is disconnected, hence, by (2), L G F is disconnected. Now Lemma 1.5 yields that G F is disconnected, hence F k; this proves that L G is k-connected. Conversely, assume L G is k-connected and δ(g) k; hence V (G) > k. For any F E(G) such that F k 1 we have δ(g F ) 1; therefore, by Lemma 1.5 and (2), if G F is disconnected so is L G F ; now this is not possible because L G is k-connected. This proves that G is k-edgeconnected. The assumption on δ(g) in the second part of the Proposition is really needed: in Example 1.4 we have a graph G with δ(g) = 1, hence not 2- edge-connected, whereas L G is 2-connected (in fact 4-connected!). The following is a consequence of the previous result. Theorem 3.4 (Menger). A graph G is k-edge-connected if and only if every pair of vertices is joined by k edge disjoint paths. Proof. Of course, we can assume k 2. One implication is easy. If G contains k edge-disjoint paths between any two vertices, any set of edges F E such that G F is disconnected must contain at least an edge for each of those paths, hence F k, and hence G is k-edge-connected. Conversely, suppose G is k-edge connected; then, by the previous proposition, its line graph, L G, is k-connected. Consider the sets of edges adjacent to them, E(x) and E(y), and the denote the corresponding sets of vertices in the line graph by A = E(x) V (L G ) and B = E(y) V (L G ). As L G is k-connected, the minimum number of vertices separating A and B is at least k; hence, by Theorem 2.5, there exist k disjoint AB-paths, P 1,..., P k, in L G. Now we apply Lemma 1.3; we replace each P i by the path P i defined 7

8 8 in (4) of that Lemma; then P i is again an AB-path, and since P i and P j are disjoint, one easily checks that P i and P j are disjoint. Moreover, again by the Lemma, for every i = 1,..., k there is a path Q i G such that L Qi = P i. By construction the paths Q 1,..., Q k are edge-disjoint; moreover, as P i is an AB-path, Q i is an xy-path. The proof is complete. Exercise 3.5. Let G be a graph. Show that G is k-edge connected if and only if G > 1 and for every x, y V, any set F E separating x and y satisfies F k. Exercise 3.6. Let G be k-edge-connected with k 1; show that G e is (k 1)-edge-connected for any e E. Give an example of a k-edge-connected graph such that G x is not (k 1)-edge-connected for some x V.

HW Graph Theory SOLUTIONS (hbovik) - Q

HW Graph Theory SOLUTIONS (hbovik) - Q 1, Diestel 3.5: Deduce the k = 2 case of Menger s theorem (3.3.1) from Proposition 3.1.1. Let G be 2-connected, and let A and B be 2-sets. We handle some special cases (thus later in the induction if these

More information

Observation 4.1 G has a proper separation of order 0 if and only if G is disconnected.

Observation 4.1 G has a proper separation of order 0 if and only if G is disconnected. 4 Connectivity 2-connectivity Separation: A separation of G of order k is a pair of subgraphs (H, K) with H K = G and E(H K) = and V (H) V (K) = k. Such a separation is proper if V (H) \ V (K) and V (K)

More information

Observation 4.1 G has a proper separation of order 0 if and only if G is disconnected.

Observation 4.1 G has a proper separation of order 0 if and only if G is disconnected. 4 Connectivity 2-connectivity Separation: A separation of G of order k is a pair of subgraphs (H 1, H 2 ) so that H 1 H 2 = G E(H 1 ) E(H 2 ) = V (H 1 ) V (H 2 ) = k Such a separation is proper if V (H

More information

Ring Sums, Bridges and Fundamental Sets

Ring Sums, Bridges and Fundamental Sets 1 Ring Sums Definition 1 Given two graphs G 1 = (V 1, E 1 ) and G 2 = (V 2, E 2 ) we define the ring sum G 1 G 2 = (V 1 V 2, (E 1 E 2 ) (E 1 E 2 )) with isolated points dropped. So an edge is in G 1 G

More information

Partial cubes: structures, characterizations, and constructions

Partial cubes: structures, characterizations, and constructions Partial cubes: structures, characterizations, and constructions Sergei Ovchinnikov San Francisco State University, Mathematics Department, 1600 Holloway Ave., San Francisco, CA 94132 Abstract Partial cubes

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

Disjoint Hamiltonian Cycles in Bipartite Graphs

Disjoint Hamiltonian Cycles in Bipartite Graphs Disjoint Hamiltonian Cycles in Bipartite Graphs Michael Ferrara 1, Ronald Gould 1, Gerard Tansey 1 Thor Whalen Abstract Let G = (X, Y ) be a bipartite graph and define σ (G) = min{d(x) + d(y) : xy / E(G),

More information

Thus, X is connected by Problem 4. Case 3: X = (a, b]. This case is analogous to Case 2. Case 4: X = (a, b). Choose ε < b a

Thus, X is connected by Problem 4. Case 3: X = (a, b]. This case is analogous to Case 2. Case 4: X = (a, b). Choose ε < b a Solutions to Homework #6 1. Complete the proof of the backwards direction of Theorem 12.2 from class (which asserts the any interval in R is connected). Solution: Let X R be a closed interval. Case 1:

More information

Topological properties

Topological properties CHAPTER 4 Topological properties 1. Connectedness Definitions and examples Basic properties Connected components Connected versus path connected, again 2. Compactness Definition and first examples Topological

More information

Economics 204 Fall 2012 Problem Set 3 Suggested Solutions

Economics 204 Fall 2012 Problem Set 3 Suggested Solutions Economics 204 Fall 2012 Problem Set 3 Suggested Solutions 1. Give an example of each of the following (and prove that your example indeed works): (a) A complete metric space that is bounded but not compact.

More information

Strongly chordal and chordal bipartite graphs are sandwich monotone

Strongly chordal and chordal bipartite graphs are sandwich monotone Strongly chordal and chordal bipartite graphs are sandwich monotone Pinar Heggernes Federico Mancini Charis Papadopoulos R. Sritharan Abstract A graph class is sandwich monotone if, for every pair of its

More information

Discrete Mathematics

Discrete Mathematics Discrete Mathematics 309 (009) 3811 380 Contents lists available at ScienceDirect Discrete Mathematics journal homepage: www.elsevier.com/locate/disc Disjoint hamiltonian cycles in bipartite graphs Michael

More information

Cographs; chordal graphs and tree decompositions

Cographs; chordal graphs and tree decompositions Cographs; chordal graphs and tree decompositions Zdeněk Dvořák September 14, 2015 Let us now proceed with some more interesting graph classes closed on induced subgraphs. 1 Cographs The class of cographs

More information

Degree Sequence and Supereulerian Graphs

Degree Sequence and Supereulerian Graphs Degree Sequence and Supereulerian Graphs Suohai Fan, Hong-Jian Lai, Yehong Shao, Taoye Zhang and Ju Zhou January 29, 2007 Abstract A sequence d = (d 1, d 2,, d n ) is graphic if there is a simple graph

More information

Decompositions of graphs into cycles with chords

Decompositions of graphs into cycles with chords Decompositions of graphs into cycles with chords Paul Balister Hao Li Richard Schelp May 22, 2017 In memory of Dick Schelp, who passed away shortly after the submission of this paper Abstract We show that

More information

Path decompositions and Gallai s conjecture

Path decompositions and Gallai s conjecture Journal of Combinatorial Theory, Series B 93 (005) 117 15 www.elsevier.com/locate/jctb Path decompositions and Gallai s conjecture Genghua Fan Department of Mathematics, Fuzhou University, Fuzhou, Fujian

More information

5 Flows and cuts in digraphs

5 Flows and cuts in digraphs 5 Flows and cuts in digraphs Recall that a digraph or network is a pair G = (V, E) where V is a set and E is a multiset of ordered pairs of elements of V, which we refer to as arcs. Note that two vertices

More information

Hamilton cycles and closed trails in iterated line graphs

Hamilton cycles and closed trails in iterated line graphs Hamilton cycles and closed trails in iterated line graphs Paul A. Catlin, Department of Mathematics Wayne State University, Detroit MI 48202 USA Iqbalunnisa, Ramanujan Institute University of Madras, Madras

More information

Distance between two k-sets and Path-Systems Extendibility

Distance between two k-sets and Path-Systems Extendibility Distance between two k-sets and Path-Systems Extendibility December 2, 2003 Ronald J. Gould (Emory University), Thor C. Whalen (Metron, Inc.) Abstract Given a simple graph G on n vertices, let σ 2 (G)

More information

Graphs with large maximum degree containing no odd cycles of a given length

Graphs with large maximum degree containing no odd cycles of a given length Graphs with large maximum degree containing no odd cycles of a given length Paul Balister Béla Bollobás Oliver Riordan Richard H. Schelp October 7, 2002 Abstract Let us write f(n, ; C 2k+1 ) for the maximal

More information

arxiv: v2 [math.co] 7 Jan 2016

arxiv: v2 [math.co] 7 Jan 2016 Global Cycle Properties in Locally Isometric Graphs arxiv:1506.03310v2 [math.co] 7 Jan 2016 Adam Borchert, Skylar Nicol, Ortrud R. Oellermann Department of Mathematics and Statistics University of Winnipeg,

More information

CLIQUES IN THE UNION OF GRAPHS

CLIQUES IN THE UNION OF GRAPHS CLIQUES IN THE UNION OF GRAPHS RON AHARONI, ELI BERGER, MARIA CHUDNOVSKY, AND JUBA ZIANI Abstract. Let B and R be two simple graphs with vertex set V, and let G(B, R) be the simple graph with vertex set

More information

The edge-density for K 2,t minors

The edge-density for K 2,t minors The edge-density for K,t minors Maria Chudnovsky 1 Columbia University, New York, NY 1007 Bruce Reed McGill University, Montreal, QC Paul Seymour Princeton University, Princeton, NJ 08544 December 5 007;

More information

CHAPTER 7. Connectedness

CHAPTER 7. Connectedness CHAPTER 7 Connectedness 7.1. Connected topological spaces Definition 7.1. A topological space (X, T X ) is said to be connected if there is no continuous surjection f : X {0, 1} where the two point set

More information

Independent Transversals in r-partite Graphs

Independent Transversals in r-partite Graphs Independent Transversals in r-partite Graphs Raphael Yuster Department of Mathematics Raymond and Beverly Sackler Faculty of Exact Sciences Tel Aviv University, Tel Aviv, Israel Abstract Let G(r, n) denote

More information

A short course on matching theory, ECNU Shanghai, July 2011.

A short course on matching theory, ECNU Shanghai, July 2011. A short course on matching theory, ECNU Shanghai, July 2011. Sergey Norin LECTURE 3 Tight cuts, bricks and braces. 3.1. Outline of Lecture Ear decomposition of bipartite graphs. Tight cut decomposition.

More information

Eulerian Subgraphs and Hamilton-Connected Line Graphs

Eulerian Subgraphs and Hamilton-Connected Line Graphs Eulerian Subgraphs and Hamilton-Connected Line Graphs Hong-Jian Lai Department of Mathematics West Virginia University Morgantown, WV 2606, USA Dengxin Li Department of Mathematics Chongqing Technology

More information

Math 541 Fall 2008 Connectivity Transition from Math 453/503 to Math 541 Ross E. Staffeldt-August 2008

Math 541 Fall 2008 Connectivity Transition from Math 453/503 to Math 541 Ross E. Staffeldt-August 2008 Math 541 Fall 2008 Connectivity Transition from Math 453/503 to Math 541 Ross E. Staffeldt-August 2008 Closed sets We have been operating at a fundamental level at which a topological space is a set together

More information

HAMILTONICITY AND FORBIDDEN SUBGRAPHS IN 4-CONNECTED GRAPHS

HAMILTONICITY AND FORBIDDEN SUBGRAPHS IN 4-CONNECTED GRAPHS HAMILTONICITY AND FORBIDDEN SUBGRAPHS IN 4-CONNECTED GRAPHS FLORIAN PFENDER Abstract. Let T be the line graph of the unique tree F on 8 vertices with degree sequence (3, 3, 3,,,,, ), i.e. T is a chain

More information

Upper Bounds of Dynamic Chromatic Number

Upper Bounds of Dynamic Chromatic Number Upper Bounds of Dynamic Chromatic Number Hong-Jian Lai, Bruce Montgomery and Hoifung Poon Department of Mathematics West Virginia University, Morgantown, WV 26506-6310 June 22, 2000 Abstract A proper vertex

More information

Advanced Topics in Discrete Math: Graph Theory Fall 2010

Advanced Topics in Discrete Math: Graph Theory Fall 2010 21-801 Advanced Topics in Discrete Math: Graph Theory Fall 2010 Prof. Andrzej Dudek notes by Brendan Sullivan October 18, 2010 Contents 0 Introduction 1 1 Matchings 1 1.1 Matchings in Bipartite Graphs...................................

More information

Maximising the number of induced cycles in a graph

Maximising the number of induced cycles in a graph Maximising the number of induced cycles in a graph Natasha Morrison Alex Scott April 12, 2017 Abstract We determine the maximum number of induced cycles that can be contained in a graph on n n 0 vertices,

More information

Branchwidth of graphic matroids.

Branchwidth of graphic matroids. Branchwidth of graphic matroids. Frédéric Mazoit and Stéphan Thomassé Abstract Answering a question of Geelen, Gerards, Robertson and Whittle [2], we prove that the branchwidth of a bridgeless graph is

More information

K 4 -free graphs with no odd holes

K 4 -free graphs with no odd holes K 4 -free graphs with no odd holes Maria Chudnovsky 1 Columbia University, New York NY 10027 Neil Robertson 2 Ohio State University, Columbus, Ohio 43210 Paul Seymour 3 Princeton University, Princeton

More information

4 CONNECTED PROJECTIVE-PLANAR GRAPHS ARE HAMILTONIAN. Robin Thomas* Xingxing Yu**

4 CONNECTED PROJECTIVE-PLANAR GRAPHS ARE HAMILTONIAN. Robin Thomas* Xingxing Yu** 4 CONNECTED PROJECTIVE-PLANAR GRAPHS ARE HAMILTONIAN Robin Thomas* Xingxing Yu** School of Mathematics Georgia Institute of Technology Atlanta, Georgia 30332, USA May 1991, revised 23 October 1993. Published

More information

Some hard families of parameterised counting problems

Some hard families of parameterised counting problems Some hard families of parameterised counting problems Mark Jerrum and Kitty Meeks School of Mathematical Sciences, Queen Mary University of London {m.jerrum,k.meeks}@qmul.ac.uk September 2014 Abstract

More information

Eulerian Subgraphs in Graphs with Short Cycles

Eulerian Subgraphs in Graphs with Short Cycles Eulerian Subgraphs in Graphs with Short Cycles Paul A. Catlin Hong-Jian Lai Abstract P. Paulraja recently showed that if every edge of a graph G lies in a cycle of length at most 5 and if G has no induced

More information

AALBORG UNIVERSITY. Total domination in partitioned graphs. Allan Frendrup, Preben Dahl Vestergaard and Anders Yeo

AALBORG UNIVERSITY. Total domination in partitioned graphs. Allan Frendrup, Preben Dahl Vestergaard and Anders Yeo AALBORG UNIVERSITY Total domination in partitioned graphs by Allan Frendrup, Preben Dahl Vestergaard and Anders Yeo R-2007-08 February 2007 Department of Mathematical Sciences Aalborg University Fredrik

More information

Citation for pulished version (APA): Henning, M. A., & Yeo, A. (2016). Transversals in 4-uniform hypergraphs. Journal of Combinatorics, 23(3).

Citation for pulished version (APA): Henning, M. A., & Yeo, A. (2016). Transversals in 4-uniform hypergraphs. Journal of Combinatorics, 23(3). Syddansk Universitet Transversals in 4-uniform hypergraphs Henning, Michael A; Yeo, Anders Published in: Journal of Combinatorics Publication date: 2016 Document version Forlagets udgivne version Document

More information

Graph Theory. Thomas Bloom. February 6, 2015

Graph Theory. Thomas Bloom. February 6, 2015 Graph Theory Thomas Bloom February 6, 2015 1 Lecture 1 Introduction A graph (for the purposes of these lectures) is a finite set of vertices, some of which are connected by a single edge. Most importantly,

More information

arxiv: v1 [cs.dm] 12 Jun 2016

arxiv: v1 [cs.dm] 12 Jun 2016 A Simple Extension of Dirac s Theorem on Hamiltonicity Yasemin Büyükçolak a,, Didem Gözüpek b, Sibel Özkana, Mordechai Shalom c,d,1 a Department of Mathematics, Gebze Technical University, Kocaeli, Turkey

More information

ON THE NUMBER OF COMPONENTS OF A GRAPH

ON THE NUMBER OF COMPONENTS OF A GRAPH Volume 5, Number 1, Pages 34 58 ISSN 1715-0868 ON THE NUMBER OF COMPONENTS OF A GRAPH HAMZA SI KADDOUR AND ELIAS TAHHAN BITTAR Abstract. Let G := (V, E be a simple graph; for I V we denote by l(i the number

More information

A Randomized Rounding Approach to the Traveling Salesman Problem

A Randomized Rounding Approach to the Traveling Salesman Problem A Randomized Rounding Approach to the Traveling Salesman Problem Shayan Oveis Gharan Amin Saberi. Mohit Singh. Abstract For some positive constant ɛ 0, we give a ( 3 2 ɛ 0)-approximation algorithm for

More information

Connectivity of addable graph classes

Connectivity of addable graph classes Connectivity of addable graph classes Paul Balister Béla Bollobás Stefanie Gerke July 6, 008 A non-empty class A of labelled graphs is weakly addable if for each graph G A and any two distinct components

More information

arxiv: v1 [math.co] 22 Jan 2018

arxiv: v1 [math.co] 22 Jan 2018 arxiv:1801.07025v1 [math.co] 22 Jan 2018 Spanning trees without adjacent vertices of degree 2 Kasper Szabo Lyngsie, Martin Merker Abstract Albertson, Berman, Hutchinson, and Thomassen showed in 1990 that

More information

Domination and Total Domination Contraction Numbers of Graphs

Domination and Total Domination Contraction Numbers of Graphs Domination and Total Domination Contraction Numbers of Graphs Jia Huang Jun-Ming Xu Department of Mathematics University of Science and Technology of China Hefei, Anhui, 230026, China Abstract In this

More information

On the Graph Bisection Cut Polytope

On the Graph Bisection Cut Polytope On the Graph Bisection Cut Polytope Michael Armbruster, Christoph Helmberg Chemnitz University of Technology Contact: helmberg@mathematik.tu-chemnitz.de Marzena Fügenschuh, Alexander Martin Darmstadt University

More information

2. Introduction to commutative rings (continued)

2. Introduction to commutative rings (continued) 2. Introduction to commutative rings (continued) 2.1. New examples of commutative rings. Recall that in the first lecture we defined the notions of commutative rings and field and gave some examples of

More information

2. Metric Spaces. 2.1 Definitions etc.

2. Metric Spaces. 2.1 Definitions etc. 2. Metric Spaces 2.1 Definitions etc. The procedure in Section for regarding R as a topological space may be generalized to many other sets in which there is some kind of distance (formally, sets with

More information

Rainbow matchings and rainbow connectedness

Rainbow matchings and rainbow connectedness Rainbow matchings and rainbow connectedness Alexey Pokrovskiy arxiv:1504.05373v1 [math.co] 21 Apr 2015 Methods for Discrete Structures, Freie Universität, Berlin, Germany. Email: alja123@gmail.com Keywords:

More information

CYCLE STRUCTURES IN GRAPHS. Angela K. Harris. A thesis submitted to the. University of Colorado Denver. in partial fulfillment

CYCLE STRUCTURES IN GRAPHS. Angela K. Harris. A thesis submitted to the. University of Colorado Denver. in partial fulfillment CYCLE STRUCTURES IN GRAPHS by Angela K. Harris Master of Science, University of South Alabama, 003 A thesis submitted to the University of Colorado Denver in partial fulfillment of the requirements for

More information

ALL GRAPHS WITH PAIRED-DOMINATION NUMBER TWO LESS THAN THEIR ORDER. Włodzimierz Ulatowski

ALL GRAPHS WITH PAIRED-DOMINATION NUMBER TWO LESS THAN THEIR ORDER. Włodzimierz Ulatowski Opuscula Math. 33, no. 4 (2013), 763 783 http://dx.doi.org/10.7494/opmath.2013.33.4.763 Opuscula Mathematica ALL GRAPHS WITH PAIRED-DOMINATION NUMBER TWO LESS THAN THEIR ORDER Włodzimierz Ulatowski Communicated

More information

Bichain graphs: geometric model and universal graphs

Bichain graphs: geometric model and universal graphs Bichain graphs: geometric model and universal graphs Robert Brignall a,1, Vadim V. Lozin b,, Juraj Stacho b, a Department of Mathematics and Statistics, The Open University, Milton Keynes MK7 6AA, United

More information

9. Birational Maps and Blowing Up

9. Birational Maps and Blowing Up 72 Andreas Gathmann 9. Birational Maps and Blowing Up In the course of this class we have already seen many examples of varieties that are almost the same in the sense that they contain isomorphic dense

More information

Every line graph of a 4-edge-connected graph is Z 3 -connected

Every line graph of a 4-edge-connected graph is Z 3 -connected European Journal of Combinatorics 0 (2009) 595 601 Contents lists available at ScienceDirect European Journal of Combinatorics journal homepage: www.elsevier.com/locate/ejc Every line graph of a 4-edge-connected

More information

arxiv: v1 [math.co] 13 May 2016

arxiv: v1 [math.co] 13 May 2016 GENERALISED RAMSEY NUMBERS FOR TWO SETS OF CYCLES MIKAEL HANSSON arxiv:1605.04301v1 [math.co] 13 May 2016 Abstract. We determine several generalised Ramsey numbers for two sets Γ 1 and Γ 2 of cycles, in

More information

MATROID PACKING AND COVERING WITH CIRCUITS THROUGH AN ELEMENT

MATROID PACKING AND COVERING WITH CIRCUITS THROUGH AN ELEMENT MATROID PACKING AND COVERING WITH CIRCUITS THROUGH AN ELEMENT MANOEL LEMOS AND JAMES OXLEY Abstract. In 1981, Seymour proved a conjecture of Welsh that, in a connected matroid M, the sum of the maximum

More information

Tight Bounds on Vertex Connectivity Under Vertex Sampling

Tight Bounds on Vertex Connectivity Under Vertex Sampling Tight Bounds on Vertex Connectivity Under Vertex Sampling Keren Censor-Hillel Mohsen Ghaffari George Giakkoupis Bernhard Haeupler Fabian Kuhn Abstract A fundamental result by Karger [10] states that for

More information

Every 3-connected, essentially 11-connected line graph is hamiltonian

Every 3-connected, essentially 11-connected line graph is hamiltonian Every 3-connected, essentially 11-connected line graph is hamiltonian Hong-Jian Lai, Yehong Shao, Hehui Wu, Ju Zhou October 2, 25 Abstract Thomassen conjectured that every 4-connected line graph is hamiltonian.

More information

5 Set Operations, Functions, and Counting

5 Set Operations, Functions, and Counting 5 Set Operations, Functions, and Counting Let N denote the positive integers, N 0 := N {0} be the non-negative integers and Z = N 0 ( N) the positive and negative integers including 0, Q the rational numbers,

More information

Saturation numbers for Ramsey-minimal graphs

Saturation numbers for Ramsey-minimal graphs Saturation numbers for Ramsey-minimal graphs Martin Rolek and Zi-Xia Song Department of Mathematics University of Central Florida Orlando, FL 3816 August 17, 017 Abstract Given graphs H 1,..., H t, a graph

More information

arxiv: v2 [math.co] 25 Jul 2016

arxiv: v2 [math.co] 25 Jul 2016 Partitioning a graph into a cycle and a sparse graph Alexey Pokrovskiy arxiv:1607.03348v [math.co] 5 Jul 016 ETH Zürich, Zürich, Switzerland Keywords: Partitioning graphs, Ramsey theory, cycles. July 6,

More information

Connectivity of addable graph classes

Connectivity of addable graph classes Connectivity of addable graph classes Paul Balister Béla Bollobás Stefanie Gerke January 8, 007 A non-empty class A of labelled graphs that is closed under isomorphism is weakly addable if for each graph

More information

ON THE CORE OF A GRAPHf

ON THE CORE OF A GRAPHf ON THE CORE OF A GRAPHf By FRANK HARARY and MICHAEL D. PLUMMER [Received 8 October 1965] 1. Introduction Let G be a graph. A set of points M is said to cover all the lines of G if every line of G has at

More information

Technical Results on Regular Preferences and Demand

Technical Results on Regular Preferences and Demand Division of the Humanities and Social Sciences Technical Results on Regular Preferences and Demand KC Border Revised Fall 2011; Winter 2017 Preferences For the purposes of this note, a preference relation

More information

Graph Theory Notes. January 15, H. A. Kierstead

Graph Theory Notes. January 15, H. A. Kierstead Graph Theory Notes January 15, 2019 H. A. Kierstead CHAPTER 1 Introduction This is an on going project. There will be changes to the material not yet covered, especially just before each lecture. There

More information

Mid Term-1 : Practice problems

Mid Term-1 : Practice problems Mid Term-1 : Practice problems These problems are meant only to provide practice; they do not necessarily reflect the difficulty level of the problems in the exam. The actual exam problems are likely to

More information

Compatible Circuit Decompositions of 4-Regular Graphs

Compatible Circuit Decompositions of 4-Regular Graphs Compatible Circuit Decompositions of 4-Regular Graphs Herbert Fleischner, François Genest and Bill Jackson Abstract A transition system T of an Eulerian graph G is a family of partitions of the edges incident

More information

ON THE NUMBERS OF CUT-VERTICES AND END-BLOCKS IN 4-REGULAR GRAPHS

ON THE NUMBERS OF CUT-VERTICES AND END-BLOCKS IN 4-REGULAR GRAPHS Discussiones Mathematicae Graph Theory 34 (2014) 127 136 doi:10.7151/dmgt.1724 ON THE NUMBERS OF CUT-VERTICES AND END-BLOCKS IN 4-REGULAR GRAPHS Dingguo Wang 2,3 and Erfang Shan 1,2 1 School of Management,

More information

Advanced Combinatorial Optimization September 22, Lecture 4

Advanced Combinatorial Optimization September 22, Lecture 4 8.48 Advanced Combinatorial Optimization September 22, 2009 Lecturer: Michel X. Goemans Lecture 4 Scribe: Yufei Zhao In this lecture, we discuss some results on edge coloring and also introduce the notion

More information

Introduction to Graph Theory

Introduction to Graph Theory Introduction to Graph Theory George Voutsadakis 1 1 Mathematics and Computer Science Lake Superior State University LSSU Math 351 George Voutsadakis (LSSU) Introduction to Graph Theory August 2018 1 /

More information

DR.RUPNATHJI( DR.RUPAK NATH )

DR.RUPNATHJI( DR.RUPAK NATH ) Contents 1 Sets 1 2 The Real Numbers 9 3 Sequences 29 4 Series 59 5 Functions 81 6 Power Series 105 7 The elementary functions 111 Chapter 1 Sets It is very convenient to introduce some notation and terminology

More information

Trees. A tree is a graph which is. (a) Connected and. (b) has no cycles (acyclic).

Trees. A tree is a graph which is. (a) Connected and. (b) has no cycles (acyclic). Trees A tree is a graph which is (a) Connected and (b) has no cycles (acyclic). 1 Lemma 1 Let the components of G be C 1, C 2,..., C r, Suppose e = (u, v) / E, u C i, v C j. (a) i = j ω(g + e) = ω(g).

More information

Maximal and Maximum Independent Sets In Graphs With At Most r Cycles

Maximal and Maximum Independent Sets In Graphs With At Most r Cycles Maximal and Maximum Independent Sets In Graphs With At Most r Cycles Bruce E. Sagan Department of Mathematics Michigan State University East Lansing, MI sagan@math.msu.edu Vincent R. Vatter Department

More information

Hamilton Cycles in Digraphs of Unitary Matrices

Hamilton Cycles in Digraphs of Unitary Matrices Hamilton Cycles in Digraphs of Unitary Matrices G. Gutin A. Rafiey S. Severini A. Yeo Abstract A set S V is called an q + -set (q -set, respectively) if S has at least two vertices and, for every u S,

More information

Long cycles have the edge-erdős-pósa property

Long cycles have the edge-erdős-pósa property Long cycles have the edge-erdős-pósa property Henning Bruhn, Matthias Heinlein and Felix Joos Abstract We prove that the set of long cycles has the edge-erdős-pósa property: for every fixed integer l 3

More information

FRACTIONAL CLIQUE DECOMPOSITIONS OF DENSE PARTITE GRAPHS

FRACTIONAL CLIQUE DECOMPOSITIONS OF DENSE PARTITE GRAPHS FRACTIONAL CLIQUE DECOMPOSITIONS OF DENSE PARTITE GRAPHS RICHARD MONTGOMERY Abstract. We give a minimum degree condition sufficent to ensure the existence of a fractional K r-decomposition in a balanced

More information

Double domination edge removal critical graphs

Double domination edge removal critical graphs AUSTRALASIAN JOURNAL OF COMBINATORICS Volume 48 (2010), Pages 285 299 Double domination edge removal critical graphs Soufiane Khelifi Laboratoire LMP2M, Bloc des laboratoires Université demédéa Quartier

More information

Stability in the Erdős Gallai Theorems on cycles and paths

Stability in the Erdős Gallai Theorems on cycles and paths Journal of Combinatorial Theory, Series B 11 (016) 197 8 Contents lists available at ScienceDirect Journal of Combinatorial Theory, Series B www.elsevier.com/locate/jctb Stability in the Erdős Gallai Theorems

More information

Def. A topological space X is disconnected if it admits a non-trivial splitting: (We ll abbreviate disjoint union of two subsets A and B meaning A B =

Def. A topological space X is disconnected if it admits a non-trivial splitting: (We ll abbreviate disjoint union of two subsets A and B meaning A B = CONNECTEDNESS-Notes Def. A topological space X is disconnected if it admits a non-trivial splitting: X = A B, A B =, A, B open in X, and non-empty. (We ll abbreviate disjoint union of two subsets A and

More information

Induced Saturation of Graphs

Induced Saturation of Graphs Induced Saturation of Graphs Maria Axenovich a and Mónika Csikós a a Institute of Algebra and Geometry, Karlsruhe Institute of Technology, Englerstraße 2, 76128 Karlsruhe, Germany Abstract A graph G is

More information

3 COUNTABILITY AND CONNECTEDNESS AXIOMS

3 COUNTABILITY AND CONNECTEDNESS AXIOMS 3 COUNTABILITY AND CONNECTEDNESS AXIOMS Definition 3.1 Let X be a topological space. A subset D of X is dense in X iff D = X. X is separable iff it contains a countable dense subset. X satisfies the first

More information

Spaces of continuous functions

Spaces of continuous functions Chapter 2 Spaces of continuous functions 2.8 Baire s Category Theorem Recall that a subset A of a metric space (X, d) is dense if for all x X there is a sequence from A converging to x. An equivalent definition

More information

Math 5707: Graph Theory, Spring 2017 Midterm 3

Math 5707: Graph Theory, Spring 2017 Midterm 3 University of Minnesota Math 5707: Graph Theory, Spring 2017 Midterm 3 Nicholas Rancourt (edited by Darij Grinberg) December 25, 2017 1 Exercise 1 1.1 Problem Let G be a connected multigraph. Let x, y,

More information

If g is also continuous and strictly increasing on J, we may apply the strictly increasing inverse function g 1 to this inequality to get

If g is also continuous and strictly increasing on J, we may apply the strictly increasing inverse function g 1 to this inequality to get 18:2 1/24/2 TOPIC. Inequalities; measures of spread. This lecture explores the implications of Jensen s inequality for g-means in general, and for harmonic, geometric, arithmetic, and related means in

More information

Averaging 2-Rainbow Domination and Roman Domination

Averaging 2-Rainbow Domination and Roman Domination Averaging 2-Rainbow Domination and Roman Domination José D. Alvarado 1, Simone Dantas 1, and Dieter Rautenbach 2 arxiv:1507.0899v1 [math.co] 17 Jul 2015 1 Instituto de Matemática e Estatística, Universidade

More information

On improving matchings in trees, via bounded-length augmentations 1

On improving matchings in trees, via bounded-length augmentations 1 On improving matchings in trees, via bounded-length augmentations 1 Julien Bensmail a, Valentin Garnero a, Nicolas Nisse a a Université Côte d Azur, CNRS, Inria, I3S, France Abstract Due to a classical

More information

Some Nordhaus-Gaddum-type Results

Some Nordhaus-Gaddum-type Results Some Nordhaus-Gaddum-type Results Wayne Goddard Department of Mathematics Massachusetts Institute of Technology Cambridge, USA Michael A. Henning Department of Mathematics University of Natal Pietermaritzburg,

More information

INVERSE LIMITS AND PROFINITE GROUPS

INVERSE LIMITS AND PROFINITE GROUPS INVERSE LIMITS AND PROFINITE GROUPS BRIAN OSSERMAN We discuss the inverse limit construction, and consider the special case of inverse limits of finite groups, which should best be considered as topological

More information

Homework 1 Real Analysis

Homework 1 Real Analysis Homework 1 Real Analysis Joshua Ruiter March 23, 2018 Note on notation: When I use the symbol, it does not imply that the subset is proper. In writing A X, I mean only that a A = a X, leaving open the

More information

arxiv: v1 [math.co] 28 Oct 2016

arxiv: v1 [math.co] 28 Oct 2016 More on foxes arxiv:1610.09093v1 [math.co] 8 Oct 016 Matthias Kriesell Abstract Jens M. Schmidt An edge in a k-connected graph G is called k-contractible if the graph G/e obtained from G by contracting

More information

The super line graph L 2

The super line graph L 2 Discrete Mathematics 206 (1999) 51 61 www.elsevier.com/locate/disc The super line graph L 2 Jay S. Bagga a;, Lowell W. Beineke b, Badri N. Varma c a Department of Computer Science, College of Science and

More information

Locating-Total Dominating Sets in Twin-Free Graphs: a Conjecture

Locating-Total Dominating Sets in Twin-Free Graphs: a Conjecture Locating-Total Dominating Sets in Twin-Free Graphs: a Conjecture Florent Foucaud Michael A. Henning Department of Pure and Applied Mathematics University of Johannesburg Auckland Park, 2006, South Africa

More information

Minimal Paths and Cycles in Set Systems

Minimal Paths and Cycles in Set Systems Minimal Paths and Cycles in Set Systems Dhruv Mubayi Jacques Verstraëte July 9, 006 Abstract A minimal k-cycle is a family of sets A 0,..., A k 1 for which A i A j if and only if i = j or i and j are consecutive

More information

1 Some loose ends from last time

1 Some loose ends from last time Cornell University, Fall 2010 CS 6820: Algorithms Lecture notes: Kruskal s and Borůvka s MST algorithms September 20, 2010 1 Some loose ends from last time 1.1 A lemma concerning greedy algorithms and

More information

10. Noether Normalization and Hilbert s Nullstellensatz

10. Noether Normalization and Hilbert s Nullstellensatz 10. Noether Normalization and Hilbert s Nullstellensatz 91 10. Noether Normalization and Hilbert s Nullstellensatz In the last chapter we have gained much understanding for integral and finite ring extensions.

More information

Combined degree and connectivity conditions for H-linked graphs

Combined degree and connectivity conditions for H-linked graphs Combined degree and connectivity conditions for H-linked graphs FLORIAN PFENDER Universität Rostock Institut für Mathematik D-18055 Rostock, Germany Florian.Pfender@uni-rostock.de Abstract For a given

More information

Spanning Paths in Infinite Planar Graphs

Spanning Paths in Infinite Planar Graphs Spanning Paths in Infinite Planar Graphs Nathaniel Dean AT&T, ROOM 2C-415 600 MOUNTAIN AVENUE MURRAY HILL, NEW JERSEY 07974-0636, USA Robin Thomas* Xingxing Yu SCHOOL OF MATHEMATICS GEORGIA INSTITUTE OF

More information

SEMI-STRONG SPLIT DOMINATION IN GRAPHS. Communicated by Mehdi Alaeiyan. 1. Introduction

SEMI-STRONG SPLIT DOMINATION IN GRAPHS. Communicated by Mehdi Alaeiyan. 1. Introduction Transactions on Combinatorics ISSN (print): 2251-8657, ISSN (on-line): 2251-8665 Vol. 3 No. 2 (2014), pp. 51-63. c 2014 University of Isfahan www.combinatorics.ir www.ui.ac.ir SEMI-STRONG SPLIT DOMINATION

More information

Every 3-connected, essentially 11-connected line graph is Hamiltonian

Every 3-connected, essentially 11-connected line graph is Hamiltonian Journal of Combinatorial Theory, Series B 96 (26) 571 576 www.elsevier.com/locate/jctb Every 3-connected, essentially 11-connected line graph is Hamiltonian Hong-Jian Lai a, Yehong Shao b, Hehui Wu a,

More information