File tree Expand file tree Collapse file tree 3 files changed +7
-36
lines changed
src/Relation/Binary/Domain Expand file tree Collapse file tree 3 files changed +7
-36
lines changed Original file line number Diff line number Diff line change 6
6
7
7
module Relation.Binary.Domain.Bundles where
8
8
9
+ open import Level using (Level; _⊔_; suc)
9
10
open import Relation.Binary.Bundles using (Poset)
10
- open import Relation.Binary.Core using (Rel)
11
- open import Level using (Level; _⊔_; suc; Lift; lift; lower)
12
- open import Function using (_∘_; id)
13
- open import Data.Product using (∃-syntax; _×_; _,_; proj₁; proj₂)
14
- open import Relation.Unary using (Pred)
15
- open import Relation.Binary.PropositionalEquality using (_≡_; subst; cong)
16
- open import Relation.Binary.Reasoning.PartialOrder
17
- open import Relation.Binary.Structures
18
- open import Data.Bool using (Bool; true; false; if_then_else_)
19
- open import Relation.Binary.Morphism.Structures
20
- open import Relation.Binary.Morphism.Structures using (IsOrderHomomorphism)
21
- open import Data.Nat.Properties using (≤-trans)
22
-
23
11
open import Relation.Binary.Domain.Structures
24
12
open import Relation.Binary.Domain.Definitions
25
13
@@ -45,7 +33,6 @@ module _ {c ℓ₁ ℓ₂ : Level} (P : Poset c ℓ₁ ℓ₂) where
45
33
open IsDCPO DcpoStr public
46
34
47
35
module _ {c ℓ₁ ℓ₂ : Level} {P : Poset c ℓ₁ ℓ₂} {Q : Poset c ℓ₁ ℓ₂} where
48
-
49
36
private
50
37
module P = Poset P
51
38
module Q = Poset Q
Original file line number Diff line number Diff line change 6
6
7
7
module Relation.Binary.Domain.Definitions where
8
8
9
+ open import Data.Product using (∃-syntax; _×_; _,_)
10
+ open import Level using (Level; _⊔_)
9
11
open import Relation.Binary.Bundles using (Poset)
10
- open import Relation.Binary.Core using (Rel)
11
- open import Level using (Level; _⊔_; suc; Lift; lift; lower)
12
- open import Function using (_∘_; id)
13
- open import Data.Product using (∃-syntax; _×_; _,_; proj₁; proj₂)
14
- open import Relation.Unary using (Pred)
15
- open import Relation.Binary.PropositionalEquality using (_≡_; subst; cong)
16
- open import Relation.Binary.Reasoning.PartialOrder
17
- open import Relation.Binary.Morphism.Structures
18
12
open import Relation.Binary.Morphism.Structures using (IsOrderHomomorphism)
19
- open import Data.Nat.Properties using (≤-trans)
20
13
21
14
private variable
22
15
c o ℓ e o' ℓ' e' ℓ₂ : Level
@@ -29,7 +22,6 @@ module _ where
29
22
30
23
module _ {c ℓ₁ ℓ₂ : Level} (P : Poset c ℓ₁ ℓ₂) where
31
24
open Poset P
32
-
33
25
IsSemidirectedFamily : ∀ {Ix : Set c} → (s : Ix → Carrier) → Set _
34
26
IsSemidirectedFamily s = ∀ i j → ∃[ k ] (s i ≤ s k × s j ≤ s k)
35
27
Original file line number Diff line number Diff line change 6
6
7
7
module Relation.Binary.Domain.Structures where
8
8
9
- open import Relation.Binary.Bundles using (Poset)
10
- open import Relation.Binary.Core using (Rel)
11
- open import Level using (Level; _⊔_; suc; Lift; lift; lower)
12
- open import Function using (_∘_; id)
13
- open import Data.Product using (∃-syntax; _×_; _,_; proj₁; proj₂)
14
- open import Relation.Unary using (Pred)
15
- open import Relation.Binary.PropositionalEquality using (_≡_; subst; cong)
16
- open import Relation.Binary.Reasoning.PartialOrder
17
- open import Relation.Binary.Structures
18
- open import Data.Bool using (Bool; true; false; if_then_else_)
19
- open import Relation.Binary.Morphism.Structures
20
- open import Relation.Binary.Morphism.Structures using (IsOrderHomomorphism)
9
+ open import Data.Product using (_×_; _,_)
21
10
open import Data.Nat.Properties using (≤-trans)
11
+ open import Function using (_∘_)
12
+ open import Level using (Level; _⊔_; suc)
13
+ open import Relation.Binary.Bundles using (Poset)
22
14
open import Relation.Binary.Domain.Definitions
23
15
24
16
private variable
You can’t perform that action at this time.
0 commit comments