Deficiency (graph theory)

Deficiency is a concept in graph theory that is used to refine various theorems related to perfect matching in graphs, such as Hall's marriage theorem. Is was first studied by Øystein Ore.[1][2]:17 A related property is surplus.

Definition of deficiency


Let G = (V, E) be a graph, and let U be an independent set of vertices - a subset of V in which no two vertices are connected by an edge. Denote by NG(U) the set of neighbors of U - a subset of V that contains all vertices that are connected by an edge to one or more vertices of U. The deficiency of the set U is defined by:

defG(U) := |U| - |NG(U)|

Suppose G is a bipartite graph, with bipartition V = X u Y. The deficiency of G with respect to one of its parts (say X), is the maximum deficiency of a subset of X:

def(G;X) := max [U subset of X] defG(U)

Sometimes this quantity is called the critical difference of G.[3]

Note that defG of the empty subset is 0, so def(G;X) ≥ 0.

Deficiency and matching

If def(G;X) = 0, it means that for all subsets U of X, |NG(U)| ≥ |U|. Hence, by Hall's marriage theorem, G admits a perfect matching.

In contrast, if def(G;X) > 0, it means that for some subsets U of X, |NG(U)| < |U|. Hence, by the same theorem, G does not admit a perfect matching. Moreover, using the notion of deficiency, it is possible to state a quantitative version of Hall's theorem:

Every bipartite graph G = (X+Y, E) admits a matching in which at most def(G;X) vertices of X are unmatched.

Proof. Let d = def(G;X). This means that, for every subset U of X, |NG(U)| ≥ |U|-d. Add d dummy vertices to Y, and connect every dummy vertex to all vertices of X. After the addition, for every subset U of X, |NG(U)| ≥ |U|. By Hall's marriage theorem, the new graph admits a matching in which all vertices of X are matched. Now, restore the origial graph by removing the d dummy vertices; this leaves at most d vertices of X unmatched. Other ways to state this theorem are:[2]:17

where ν(G) the is size of a maximum matching in G (also called the matching number of G).

Properties of the deficiency function

In a bipartite graph G = (X+Y, E), the deficiency function is a supermodular set function: for every two subsets X1, X2 of X:[2]:Lem.1.3.2

A tight subset is a subset of X whose deficiency equals the deficiency of the entire graph (i.e., equals the maximum). The intersection and union of tight sets are tight; this follows from properties of upper-bounded supermodular set functions.[2]:Lem.1.3.3

In a non-bipartite graph, the deficiency function is, in general, not supermodular.

Strong Hall property

A graph G has the Hall property if Hall's marriage theorem holds for that graph, namely, if G has either a perfect matching or a vertex set with a positive deficiency. A graph has the strong Hall property if def(G) = |V| - 2 ν(G). Obviously, the strong Hall property implies the Hall property. Bipartite graphs have both of these properties, however there are classes of non-bipartite graphs that have these properties.

In particular, a graph has the strong Hall property if-and-only-if it is stable - its maximum matching size equals its maximum fractional matching size.[3]

Surplus

The surplus of a subset U of V is defined by:

surG(U) := |NG(U)| - |U| = - defG(U)

The surplus of a graph G w.r.t. a subset X is defined by the minimum surplus of non-empty subsets of X:[2]:19

sur(G;X) := min [U a non-empty subset of X] surG(U)

Note the restriction to non-empty subsets: without it, the surplus of all graphs would always be 0. Note also that:

def(G;X) = max[0, - sur(G; X)]

In a bipartite graph G = (X+Y, E), the surplus function is a submodular set function: for every two subsets X1, X2 of X:

A surplus-tight subset is a subset of X whose surplus equals the surplus of the entire graph (i.e., equals the minimum). The intersection and union of tight sets with non-empty intersection are tight; this follows from properties of lower-bounded submodular set functions.[2]:Lem.1.3.5

For a bipartite graph G with def(G;X) = 0, the number sur(G;X) is the largest integer s satisfying the following property for every vertex x in X: if we add s new vertices to X and connect them to the vertices in NG(x), the resulting graph has a non-negative surplus.[2]:Thm.1.3.6

If G is a bipartite graph with a positive surplus, such that deleting any edge from G decreases sur(G;X), then every vertex in X has degree sur(G;X)+1.[4]

A bipartite graph has a positive surplus (w.r.t. X) if-and-only-if it contains a forest F such that every vertex in X has degree 2 in F.[2]:Thm.1.3.8

Graphs with a positive surplus play an important role in the theory of graph structures; see the Gallai–Edmonds decomposition.

In a non-bipartite graph, the surplus function is, in general, not submodular.

References

  1. Ore, Oystein (1955-12-01). "Graphs and matching theorems". Duke Mathematical Journal. 22 (4): 625–639. doi:10.1215/S0012-7094-55-02268-7. ISSN 0012-7094.
  2. Lovász, László; Plummer, M. D. (1986), Matching Theory, Annals of Discrete Mathematics, 29, North-Holland, ISBN 0-444-87916-1, MR 0859549
  3. Beckenbach, Isabel; Borndörfer, Ralf (2018-10-01). "Hall's and Kőnig's theorem in graphs and hypergraphs". Discrete Mathematics. 341 (10): 2753–2761. doi:10.1016/j.disc.2018.06.013. ISSN 0012-365X.
  4. Lovász, L. (1970-09-01). "A generalization of Kónig's theorem". Acta Mathematica Academiae Scientiarum Hungaricae. 21 (3): 443–446. doi:10.1007/BF01894789. ISSN 1588-2632. S2CID 121333106.
This article is issued from Wikipedia. The text is licensed under Creative Commons - Attribution - Sharealike. Additional terms may apply for the media files.