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.
getVert_map
Walk.map
1 parent 20a0747 commit c15bb2eCopy full SHA for c15bb2e
Mathlib/Combinatorics/SimpleGraph/Walks/Maps.lean
@@ -100,6 +100,10 @@ theorem edges_map : (p.map f).edges = p.edges.map (Sym2.map f) := by
100
@[simp]
101
theorem edgeSet_map : (p.map f).edgeSet = Sym2.map f '' p.edgeSet := by ext; simp
102
103
+@[simp]
104
+theorem getVert_map (n : ℕ) : (p.map f).getVert n = f (p.getVert n) := by
105
+ induction p generalizing n <;> cases n <;> simp [*]
106
+
107
theorem map_injective_of_injective {f : G →g G'} (hinj : Function.Injective f) (u v : V) :
108
Function.Injective (Walk.map f : G.Walk u v → G'.Walk (f u) (f v)) := by
109
intro p p' h
0 commit comments