Skip to content

Commit

Permalink
feat: StrictSegal.spineToSimplex_map lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
gio256 committed Jan 18, 2025
1 parent 7a07689 commit 06edc34
Showing 1 changed file with 21 additions and 1 deletion.
22 changes: 21 additions & 1 deletion Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -123,7 +123,20 @@ theorem spineToSimplex_edge (f : Path X m) (j l : ℕ) (hjl : j + l ≤ m) :

end spineToSimplex

/- TODO: spineToSimplex_map -/
open Opposite in
/-- For any `σ : X ⟶ Y` between `n + 1`-truncated `StrictSegal` simplicial sets,
`spineToSimplex` commutes with `Path.map`. -/
lemma spineToSimplex_map {X Y : SSet.Truncated.{u} (n + 1)}
(sx : StrictSegal X) (sy : StrictSegal Y)
(m : ℕ) (h : m ≤ n := by leq) (f : Path X (m + 1)) (σ : X ⟶ Y) :
sy.spineToSimplex (m + 1) (by leq) (f.map σ) =
σ.app (op [m + 1]ₙ₊₁) (sx.spineToSimplex (m + 1) (by leq) f) := by
apply sy.spineInjective (m + 1)
ext k
dsimp only [spineEquiv, Equiv.coe_fn_mk, spine_arrow]
rw [← types_comp_apply (σ.app _) (Y.map _), ← σ.naturality]
simp only [spineToSimplex_arrow, types_comp_apply]
rfl

section spine_δ

Expand Down Expand Up @@ -276,6 +289,13 @@ theorem spineToSimplex_edge :

end interval

/-- For any `σ : X ⟶ Y` between `StrictSegal` simplicial sets, `spineToSimplex`
commutes with `Path.map`. -/
lemma spineToSimplex_map {X Y : SSet.{u}} (sx : StrictSegal X)
(sy : StrictSegal Y) {n : ℕ} (f : Path X (n + 1)) (σ : X ⟶ Y) :
sy.spineToSimplex (f.map σ) = σ.app _ (sx.spineToSimplex f) :=
sx (n + 1) |>.spineToSimplex_map (sy _) n (by leq) f ((truncation _).map σ)

variable (f : Path X (n + 1))
variable {i : Fin (n + 1)} {j : Fin (n + 2)}

Expand Down

0 comments on commit 06edc34

Please sign in to comment.