Skip to content

Commit

Permalink
line edits
Browse files Browse the repository at this point in the history
  • Loading branch information
emilyriehl committed Jan 29, 2025
1 parent 41bcf03 commit 4296cdc
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 8 deletions.
Original file line number Diff line number Diff line change
Expand Up @@ -115,8 +115,6 @@ theorem twoSimplex_δ2 (X₀ X₁ X₂ : WalkingIso) :
unfold twoSimplex oneSimplex
sorry



theorem twoSimplex_ext {X₀ X₁ X₂ Y₀ Y₁ Y₂ : WalkingIso}
(e₀ : X₀ = Y₀) (e₁ : X₁ = Y₁) (e₂ : X₂ = Y₂) : twoSimplex X₀ X₁ X₂ = twoSimplex Y₀ Y₁ Y₂ :=
congrArg (yonedaEquiv coherentIso _).symm (ComposableArrows.ext₂ e₀ e₁ e₂ rfl rfl)
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -69,8 +69,8 @@ noncomputable def map01Coprod34 : (Δ[1] ⨿ Δ[1] ⟶ Sq : Type u) :=
coprod.desc (delta01 ≫ (pushout.inl delta12 delta01)) (delta01 ≫ (pushout.inr delta12 delta01))
noncomputable def map01Coprod34' : (Δ[1] ⨿ Δ[1] ⟶ Sq' : Type u) :=
coprod.desc
((stdSimplex.δ 1) ≫ (pushout.inl delta12' delta01'))
((stdSimplex.δ 1) ≫ (pushout.inr delta12' delta01'))
((stdSimplex.δ 1) ≫ (pushout.inl (stdSimplex.δ 0) (stdSimplex.δ 2)))
((stdSimplex.δ 1) ≫ (pushout.inr (stdSimplex.δ 0) (stdSimplex.δ 2)))

/--
The pushout of the diagram
Expand Down Expand Up @@ -105,12 +105,10 @@ noncomputable def map2dModel'toCoherentIso : Model2dCoherentIso' ⟶ coherentIso
· exact coprod.desc (coherentIso.pt WalkingIso.zero) (coherentIso.pt WalkingIso.one)
· unfold map0Coprod0' map01Coprod34'
apply coprod.hom_ext
· unfold delta01' delta12'
simp only [coprod.desc_comp, Category.assoc, colimit.ι_desc, PushoutCocone.mk_pt,
· simp only [coprod.desc_comp, Category.assoc, colimit.ι_desc, PushoutCocone.mk_pt,
PushoutCocone.mk_ι_app, BinaryCofan.ι_app_left, BinaryCofan.mk_inl, coprod.map_desc]
rw [coherentIso.twoSimplex_δ1 _ _ _, ← coherentIso.oneSimplex_const]
· unfold delta01' delta12'
simp only [coprod.desc_comp, Category.assoc, colimit.ι_desc,
· simp only [coprod.desc_comp, Category.assoc, colimit.ι_desc,
PushoutCocone.mk_pt, PushoutCocone.mk_ι_app,
BinaryCofan.mk_pt, BinaryCofan.ι_app_right, BinaryCofan.mk_inr, coprod.map_desc]
rw [coherentIso.twoSimplex_δ1 _ _ _, ← coherentIso.oneSimplex_const]
Expand Down

0 comments on commit 4296cdc

Please sign in to comment.