Skip to content

Commit b5d3e50

Browse files
committed
fix-whitespace
1 parent b4edd11 commit b5d3e50

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/Relation/Binary/Domain/Definitions.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -23,7 +23,7 @@ private variable
2323
Ix A B : Set o
2424
P : Poset c ℓ e
2525

26-
module _ where
26+
module _ where
2727
IsMonotone : (P : Poset o ℓ e) (Q : Poset o' ℓ' e') (f : Poset.Carrier P Poset.Carrier Q) Set (o ⊔ ℓ ⊔ e ⊔ ℓ' ⊔ e')
2828
IsMonotone P Q f = IsOrderHomomorphism (Poset._≈_ P) (Poset._≈_ Q) (Poset._≤_ P) (Poset._≤_ Q) f
2929

@@ -32,4 +32,4 @@ module _ {c ℓ₁ ℓ₂ : Level} (P : Poset c ℓ₁ ℓ₂) where
3232

3333
IsSemidirectedFamily : {Ix : Set c} (s : Ix Carrier) Set _
3434
IsSemidirectedFamily s = i j ∃[ k ] (s i ≤ s k × s j ≤ s k)
35-
35+

src/Relation/Binary/Properties/Domain.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -174,4 +174,4 @@ module _ {c ℓ₁ ℓ₂} {P : Poset c ℓ₁ ℓ₂} {D E : DCPO P c ℓ₁
174174
(IsOrderHomomorphism.cong mono (uniqueLub {D = D} (D.⋁ _ dir) lub (D.⋁-isLub _ dir) x))
175175
(pres-⋁ _ dir)
176176
; PreserveEquality = IsOrderHomomorphism.cong mono }
177-
177+

0 commit comments

Comments
 (0)