We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
support_injective
1 parent f0b4174 commit 4f51227Copy full SHA for 4f51227
Mathlib/Combinatorics/SimpleGraph/Walk.lean
@@ -1136,6 +1136,9 @@ lemma ext_support {u v} {p q : G.Walk u v} (h : p.support = q.support) :
1136
have : (p.copy h rfl).support = q.support := by simpa
1137
simp [← ih this]
1138
1139
+lemma support_injective {u v : V} : (support (G := G) (u := u) (v := v)).Injective :=
1140
+ fun _ _ ↦ ext_support
1141
+
1142
lemma ext_getVert_le_length {u v} {p q : G.Walk u v} (hl : p.length = q.length)
1143
(h : ∀ k ≤ p.length, p.getVert k = q.getVert k) :
1144
p = q := by
0 commit comments