Skip to content

Commit

Permalink
Make variables names _∙∙_∙∙_ consistent with those in doubleComp-face…
Browse files Browse the repository at this point in the history
…s and remove an unnecessary space
  • Loading branch information
ShreckYe committed Aug 4, 2023
1 parent b56db83 commit 0d90ad3
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Cubical/Foundations/Prelude.agda
Original file line number Diff line number Diff line change
Expand Up @@ -110,12 +110,12 @@ congP₂ f p q i = f i (p i) (q i)
`doubleCompPath-filler p q r` gives the whole square
-}

doubleComp-faces : {x y z w : A } (p : x ≡ y) (r : z ≡ w)
doubleComp-faces : {x y z w : A} (p : x ≡ y) (r : z ≡ w)
(i : I) (j : I) Partial (i ∨ ~ i) A
doubleComp-faces p r i j (i = i0) = p (~ j)
doubleComp-faces p r i j (i = i1) = r j

_∙∙_∙∙_ : wx xy yz wz
_∙∙_∙∙_ : xy yz zw xw
(p ∙∙ q ∙∙ r) i =
hcomp (doubleComp-faces p r i) (q i)

Expand Down

0 comments on commit 0d90ad3

Please sign in to comment.