Skip to content

Commit

Permalink
feat(AlgebraicTopology/SimplicialSet): Add auxiliary ext lemma for pa…
Browse files Browse the repository at this point in the history
…ths (#19349)

We implement the generalization of the path extensionality lemmas suggested by @joelriou in #19057. Two paths of the same nonzero length can be identified by constructing an identification between each of their arrows.

Co-Authored-By: [Joël Riou](https://github.com/joelriou)
  • Loading branch information
gio256 committed Nov 22, 2024
1 parent 178af37 commit 3d401e0
Showing 1 changed file with 12 additions and 0 deletions.
12 changes: 12 additions & 0 deletions Mathlib/AlgebraicTopology/SimplicialSet/Path.lean
Original file line number Diff line number Diff line change
Expand Up @@ -73,4 +73,16 @@ lemma spine_map_subinterval {n : ℕ} (j l : ℕ) (hjl : j + l ≤ n) (Δ : X _[
· simp only [spine_arrow, Path.interval, ← FunctorToTypes.map_comp_apply, ← op_comp,
mkOfSucc_subinterval_eq]

/-- Two paths of the same nonzero length are equal if all of their arrows are equal. -/
@[ext]
lemma Path.ext' {n : ℕ} {f g : Path X (n + 1)}
(h : ∀ i : Fin (n + 1), f.arrow i = g.arrow i) :
f = g := by
ext j
· rcases Fin.eq_castSucc_or_eq_last j with ⟨k, hk⟩ | hl
· rw [hk, ← f.arrow_src k, ← g.arrow_src k, h]
· simp only [hl, ← Fin.succ_last]
rw [← f.arrow_tgt (Fin.last n), ← g.arrow_tgt (Fin.last n), h]
· exact h j

end SSet

0 comments on commit 3d401e0

Please sign in to comment.