File tree Expand file tree Collapse file tree 2 files changed +3
-3
lines changed Expand file tree Collapse file tree 2 files changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -23,7 +23,7 @@ private variable
23
23
Ix A B : Set o
24
24
P : Poset c ℓ e
25
25
26
- module _ where
26
+ module _ where
27
27
IsMonotone : (P : Poset o ℓ e) → (Q : Poset o' ℓ' e') → (f : Poset.Carrier P → Poset.Carrier Q) → Set (o ⊔ ℓ ⊔ e ⊔ ℓ' ⊔ e')
28
28
IsMonotone P Q f = IsOrderHomomorphism (Poset._≈_ P) (Poset._≈_ Q) (Poset._≤_ P) (Poset._≤_ Q) f
29
29
@@ -32,4 +32,4 @@ module _ {c ℓ₁ ℓ₂ : Level} (P : Poset c ℓ₁ ℓ₂) where
32
32
33
33
IsSemidirectedFamily : ∀ {Ix : Set c} → (s : Ix → Carrier) → Set _
34
34
IsSemidirectedFamily s = ∀ i j → ∃[ k ] (s i ≤ s k × s j ≤ s k)
35
-
35
+
Original file line number Diff line number Diff line change @@ -174,4 +174,4 @@ module _ {c ℓ₁ ℓ₂} {P : Poset c ℓ₁ ℓ₂} {D E : DCPO P c ℓ₁
174
174
(IsOrderHomomorphism.cong mono (uniqueLub {D = D} (D.⋁ _ dir) lub (D.⋁-isLub _ dir) x))
175
175
(pres-⋁ _ dir)
176
176
; PreserveEquality = IsOrderHomomorphism.cong mono }
177
-
177
+
You can’t perform that action at this time.
0 commit comments