Skip to content

Commit c15bb2e

Browse files
committed
feat(Combinatorics/SimpleGraph): add simp lemma getVert_map for Walk.map (#32102)
1 parent 20a0747 commit c15bb2e

File tree

1 file changed

+4
-0
lines changed
  • Mathlib/Combinatorics/SimpleGraph/Walks

1 file changed

+4
-0
lines changed

Mathlib/Combinatorics/SimpleGraph/Walks/Maps.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -100,6 +100,10 @@ theorem edges_map : (p.map f).edges = p.edges.map (Sym2.map f) := by
100100
@[simp]
101101
theorem edgeSet_map : (p.map f).edgeSet = Sym2.map f '' p.edgeSet := by ext; simp
102102

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+
103107
theorem map_injective_of_injective {f : G →g G'} (hinj : Function.Injective f) (u v : V) :
104108
Function.Injective (Walk.map f : G.Walk u v → G'.Walk (f u) (f v)) := by
105109
intro p p' h

0 commit comments

Comments
 (0)