Skip to content

Commit

Permalink
Fix whitespace
Browse files Browse the repository at this point in the history
  • Loading branch information
Trebor-Huang committed Sep 19, 2024
1 parent a181af8 commit 54a2b1f
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 3 deletions.
4 changes: 2 additions & 2 deletions Cubical/HITs/Wedge/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -618,7 +618,7 @@ module _ (X∙ @ (X , x₀) : Pointed ℓ) (Y∙ @ (Y , y₀) : Pointed ℓ') wh
{-
The proof proceeds by applying the pasting lemma twice:
1 ----> Y
↓ ↓
↓ ↓
X --> X ⋁ Y --> X
↓ mid ↓ bot ↓
1 ----> Y ----> 1
Expand Down Expand Up @@ -646,6 +646,6 @@ module _ (X∙ @ (X , x₀) : Pointed ℓ) (Y∙ @ (Y , y₀) : Pointed ℓ') wh
where
open PushoutPasteDown (rotatePushoutSquare (_ , midPushout))
fX (terminal X) (terminal Y) refl

Pushout⋁≃Unit : Pushout fX fY ≃ Unit
Pushout⋁≃Unit = _ , botPushout
1 change: 0 additions & 1 deletion Cubical/Homotopy/Loopspace.agda
Original file line number Diff line number Diff line change
Expand Up @@ -538,4 +538,3 @@ module _ {ℓ} {B C : Type ℓ} (b₀ : B) (π : B → C) where
-- splitting and splitting∙ agrees
splitting-typ : cong typ splitting∙ ≡ splitting
splitting-typ = congFunct typ presplit twisted∙

0 comments on commit 54a2b1f

Please sign in to comment.