Skip to content

Commit

Permalink
feat(Combinatorics/SimpleGraph/Matching): add `IsPerfectMatching.toSu…
Browse files Browse the repository at this point in the history
…bgraph_spanningCoe_iff` (#19094)

Just a small lemma about perfect matchings and `spanningCoe`.
In preparation for Tutte's theorem.
  • Loading branch information
Pim Otte committed Nov 18, 2024
1 parent 62c5318 commit 277fb94
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions Mathlib/Combinatorics/SimpleGraph/Matching.lean
Original file line number Diff line number Diff line change
Expand Up @@ -204,6 +204,11 @@ lemma IsPerfectMatching.induce_connectedComponent_isMatching (h : M.IsPerfectMat
(c : ConnectedComponent G) : (M.induce c.supp).IsMatching := by
simpa [h.2.verts_eq_univ] using h.1.induce_connectedComponent c

@[simp]
lemma IsPerfectMatching.toSubgraph_spanningCoe_iff (h : M.spanningCoe ≤ G') :
(G'.toSubgraph M.spanningCoe h).IsPerfectMatching ↔ M.IsPerfectMatching := by
simp only [isPerfectMatching_iff, toSubgraph_adj, spanningCoe_adj]

end Subgraph

namespace ConnectedComponent
Expand Down

0 comments on commit 277fb94

Please sign in to comment.