Skip to content

Commit

Permalink
tweak
Browse files Browse the repository at this point in the history
  • Loading branch information
Trebor-Huang committed Sep 19, 2024
1 parent a4b23dd commit 98bbb7a
Showing 1 changed file with 2 additions and 3 deletions.
5 changes: 2 additions & 3 deletions Cubical/HITs/Join/SuspWedgeEquiv.agda
Original file line number Diff line number Diff line change
Expand Up @@ -121,6 +121,5 @@ module _ {ℓ ℓ'} (X∙ @ (X , x₀) : Pointed ℓ) (Y∙ @ (Y , y₀) : Point
H3 = λ _ refl
} ∙ sym (Susp≡PushoutSusp* {ℓ-max ℓ ℓ'})

join≡Susp : Susp (X∙ ⋀ Y∙) ≡ join X Y
join≡Susp = sym A□○≡Σ ∙ 3x3-lemma smash-span ∙ A○□≡join

Susp≡join : Susp (X∙ ⋀ Y∙) ≡ join X Y
Susp≡join = sym A□○≡Σ ∙ 3x3-lemma smash-span ∙ A○□≡join

0 comments on commit 98bbb7a

Please sign in to comment.