KG1 W2021 Lecture 08
KG1 W2021 Lecture 08
Lecture #8
Menger’s theorems and the Ear lemma
Irena Penev
In what follows, all graphs are finite, simple (i.e. have no loops and no
parallel edges), and non-null.
1 Menger’s theorems
Menger’s theorem (vertex version). Let G be a graph, and let A, B ⊆
V (G).1 Then the minimum number of vertices separating A from B in G is
equal to the maximum number of pairwise disjoint A-B paths in G.2
a4 = b1 A = {a1 , a2 , a3 , a4 }
a1 b2 B = {b1 , b2 , b3 }
a2 b3
a3
set of vertices
separating
A from B
Proof. We assume inductively that the theorem holds for graphs that have
fewer than |E(G)| edges. More precisely, we assume that for all graphs
G′ such that |E(G′ )| < |E(G)|, and all sets A′ , B ′ ⊆ V (G′ ), the minimum
number of vertices separating A′ from B ′ in G′ is equal to the maximum
number of pairwise disjoint A′ -B ′ paths in G′ . We must prove that this holds
for G as well. From now on, we let k be the minimum number of vertices
separating A from B in G.
1
A and B need not be disjoint.
2
“Pairwise disjoint” here means that no two paths have a vertex in common (and
consequently, no two paths have an edge in common).
1
First, we claim that there can be no more than k pairwise disjoint paths
from A to B in G. Indeed, let X ⊆ V (G) be a k-vertex set separating A
from B in G, and let P be any collection of pairwise disjoint paths from A
to B. By definition, every path in P contains at least one vertex of X, and
since paths in P are pairwise disjoint, no two paths in P contain the same
vertex of X. So, |P| ≤ |X| = k, as we had claimed.
It remains to show that there are at least k pairwise disjoint paths from
A to B. Clearly, for any set X ⊆ V (G) separating A from B in G, we have
that A ∩ B ⊆ X; consequently, |A ∩ B| ≤ k. Now, if E(G) = ∅, then A ∩ B
separates A from B in G, and so |A ∩ B| = k; in this case, the vertices of
A ∩ B form k pairwise disjoint one-vertex paths from A to B, and we are
done. From now on, we assume that G has at least one edge, say xy. Let
Gxy := G/xy, i.e. let Gxy be the graph obtained from G by contracting the
edge xy, and let vxy be the vertex obtained by contracting xy.3
x y vxy
G G/xy
2
X = {x1 , . . . , xk }.
We now consider the graph G \ xy, i.e. the graph obtained from G by
deleting the edge xy.10 Since x, y ∈ X, we know that any set of vertices
separating A from X in G \ xy also separates A from B in G;11 consequently,
any such set has at least k vertices, and so by the induction hypothesis,
there are k pairwise disjoint paths from A to X in G, call them P1 , . . . , Pk .
Similarly, there are k pairwise disjoint paths from B to X in G, call them
Q1 , . . . , Qk . We may assume that for all i ∈ {1, . . . , k}, xi is an endpoint
both of Pi and of Qi . So, P1 − x1 − Q1 , . . . , Pk − xk − Qk are pairwise disjoint
walks from A to B. But in fact, each of these walks is a path, for otherwise,
it would contain a path from A to B that contains no vertex of X.12 So,
there are at least k pairwise disjoint paths from A to B in G.
3
number of vertices of V (G) \ {s, t} separating S from T in G \ {s, t}.13
Similarly, the maximum number of pairwise internally disjoint s-t paths
in G is equal to the maximum number of pairwise disjoint S-T paths in
G. By Menger’s theorem (vertex version), the minimum number of vertices
separating S from T in G \ {s, t} is equal to the maximum number of pairwise
disjoint S-T paths in G \ {s, t}. So, the minimum number of vertices of
V (G) \ {s, t} separating s from t in G is equal to the maximum number of
pairwise internally disjoint s-t paths in G. This completes the argument.
Our next goal is to prove the edge version of Menger’s theorem. The
line graph of a graph G, denoted by L(G), is the graph whose vertex set is
E(G), and in which e, f ∈ L(V (G)) = E(G) are adjacent if and only if e and
f share an endpoint in G.
f1
f1
e1 e4 e1 e4
e5 e5
e2 e3 e2 e3
f2
f2
G L(G)
4
in G, we know that there is a path v1 , . . . , vr in G, with v1 = s and vr = t,
that does not use any edge of X. But now v1 v2 , v2 v3 , . . . , vr−1 vr is a path
from S to T in L(G) that does not use any vertex (in L(G)) in X. So, X
does not separate S from T in L(G).
s t
Proof. Suppose first that (i) holds, and fix ℓ pairwise edge-disjoint s-t paths
in G, say P1 , . . . , Pℓ . For all i ∈ {1, . . . , ℓ}, set Pi = v1i , . . . , vri i . Now, for all
i ∈ {1, . . . , ℓ}, set PiL = v1i v2i , v2i v3i , . . . , vri i −1 vri i (with v1i = s and vri i = t).
Clearly, P1L , . . . , PℓL are pairwise disjoint S-T paths in L(G).
Suppose now that (ii) holds, and fix ℓ pairwise disjoint S-T paths in
G, say QL L L i i
1 , . . . , Qℓ . For all i ∈ {1, . . . , ℓ}, set Qi = e1 , . . . , eri . Now, for
i
all i ∈ {1, . . . , ℓ} and j ∈ {1, . . . , ri }, let vj be a common vertex of the
edges eij and eij+1 in G, and set Qi = s, v1i , . . . , vri i −1 , t. Then Q1 , . . . , Qℓ are
pairwise edge-disjoint s-t walks in G, and we deduce that there are ℓ pairwise
edge-disjoint s-t paths in G.
s t
5
Proof. Let S be the set of all edges in G incident with s, and let T be the set
of all edges in G incident with t. By Proposition 1.2, the minimum number
of edges separating s from t in G is equal to the minimum number of vertices
separating S from T in L(G). By Proposition 1.3, the maximum number
of pairwise edge-disjoint s-t paths in G is equal to the maximum number
of pairwise disjoint S-T paths in G. By Menger’s theorem (vertex version),
the minimum number of vertices separating S from T in L(G) is equal to
the maximum number of pairwise disjoint S-T paths in G. We now deduce
that the minimum number of edges separating s from t in G is equal to the
maximum number of pairwise edge-disjoint s-t paths in G. This completes
the argument.
6
such that |X| ≤ k − 1 and G \ X is disconnected. Then G \ X has at least
two components, and we choose vertices s and t from distinct components of
G \ X. Now X ⊆ V (G) \ {s, t} separates s from t, and so by Corollary 1.1,
there can be at most |X| ≤ k − 1 internally disjoint paths between s and t
in G. But this contradicts the fact that there are k internally disjoint paths
between any two distinct vertices of G.
We now prove (b). Suppose that G is ℓ-edge-connected. Fix distinct
vertices s, t ∈ V (G). Since G is ℓ-edge-connected, s cannot be separated from
t with fewer than ℓ edges of G, and so by Menger’s theorem (edge version),
there are at least ℓ pairwise edge-disjoint paths between s and t in G.
Suppose now that G is not ℓ-edge connected. Then there exists a set
F ⊆ E(G) such that |F | ≤ ℓ − 1 and G \ F is disconnected. Since G \ F is
disconnected, it has at least two components; let s and t be vertices from
distinct components of G \ F . Now F separates s from t, and in particular, s
can be separated from t by at most |F | ≤ ℓ − 1 edges of G. So, by Menger’s
theorem (edge version), there are at most ℓ − 1 pairwise edge-disjoint paths
between s and t in G.
cut-vertex
7
In this section, we give a full structural description of 2-connected graphs.
A path addition (sometimes called open ear addition) to a graph H is the
addition to H of a path between two distinct vertices of H in such a way
that no internal vertex and no edge of the path belongs to H. In the picture
below, we show how the cube graph can be constructed by starting with a
cycle of length four and then repeatedly adding open ears (the path/open
ear added at each step is in red).
Proof. We first prove the “if” (i.e. “⇐=”) part of the lemma. Clearly, cycles
are 2-connected (indeed, every cycle has at least three vertices, is connected,
and has no cut-vertices).20 Further, if a graph G can be obtained from a
2-connected graph H by adding a path, then G has at least three vertices
(because H does), and it is easy to see that G is connected and has no
cut-vertices;21 so, G is 2-connected. It now follows by an easy induction
(e.g. on the number of paths added) that any graph obtained from a cycle
by repeated path addition is 2-connected. This proves the “if” part of the
lemma.
It remains to prove the “only if” (i.e. “=⇒”) part of the lemma. Fix a
2-connected graph G. By Lemma 2.1, G contains a cycle.22 Now, let H be
a maximal subgraph of G that either is a cycle or can be obtained from a
cycle by repeated path addition.23 We must show that H = G.
First, we claim that H is an induced subgraph of G.24 If not, then there
exist distinct vertices u, v ∈ V (H) that are adjacent in G, but not in H; but
then the graph obtained from H by adding the one-edge path u, v contradicts
the maximality of H. So, H is indeed an induced subgraph of G.
20
Alternatively, this follows from Lemma 2.1.
21
Check this!
22
Indeed, G has at least three vertices (because it is 2-connected), and by Lemma 2.1,
any two of them lie on a common cycle. So, G contains a cycle.
23
This means that no subgraph H ∗ of G that either is a cycle or can be obtained from a
cycle by repeated path addition contains H as a proper subgraph.
24
A graph H is an induced subgraph of a graph G if V (H) ⊆ V (G), and for all distinct
u, v ∈ V (H), we have that uv ∈ E(H) if and only if uv ∈ E(G).
8
u
v
H G
This proves that V (H) = V (G). Since we already know that H is an induced
subgraph of G, it follows that H = G. This proves the “only if” part of the
lemma.
25
Otherwise, we fix a minimal index i ∈ {1, . . . , t − 1} such that pi ∈ V (H), and we
consider the path v, p1 , . . . , pi instead of v, p1 , . . . , pt .