Skip to content

Commit

Permalink
Fix whitespace
Browse files Browse the repository at this point in the history
  • Loading branch information
LuuBluum committed Sep 7, 2024
1 parent 96d8ccc commit f60761c
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Cubical/Relation/Binary/Order/Poset/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -356,7 +356,7 @@ IsPosetEquivRespectsJoin : {P : Poset ℓ₀ ℓ₀'} {S : Poset ℓ₁ ℓ₁'}
(equivFun (e .fst) a)
(equivFun (e .fst) b)
(equivFun (e .fst) a∨b)

IsPosetEquivRespectsJoin {P = P} {S = S} (e , posEq) a b a∨b
= propBiimpl→Equiv (isPropIsJoin proP a b a∨b)
(isPropIsJoin proS (equivFun e a) (equivFun e b) (equivFun e a∨b))
Expand Down
6 changes: 3 additions & 3 deletions Cubical/Relation/Binary/Order/Toset/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -143,8 +143,8 @@ module _

private
pos = isToset→isPoset tos
pre = isPoset→isProset pos

pre = isPoset→isProset pos

prop = IsToset.is-prop-valued tos

Expand All @@ -159,7 +159,7 @@ module _
module _
{P : Embedding A ℓ''}
where

private
toA = fst (snd P)

Expand Down

0 comments on commit f60761c

Please sign in to comment.