File tree Expand file tree Collapse file tree 4 files changed +16
-16
lines changed
src/Algebra/Lattice/Construct Expand file tree Collapse file tree 4 files changed +16
-16
lines changed Original file line number Diff line number Diff line change 13
13
14
14
{-# OPTIONS --cubical-compatible --safe #-}
15
15
16
- open import Algebra
17
- open import Algebra.Lattice
16
+ module Algebra.Lattice.Construct.DirectProduct where
17
+
18
+ open import Algebra using (Band)
19
+ open import Algebra.Lattice using (Semilattice)
18
20
import Algebra.Construct.DirectProduct as DirectProduct
19
21
open import Data.Product.Base using (_,_; _<*>_)
20
- open import Data.Product.Relation.Binary.Pointwise.NonDependent
21
22
open import Level using (Level; _⊔_)
22
23
23
- module Algebra.Lattice.Construct.DirectProduct where
24
-
25
24
private
26
25
variable
27
26
a b ℓ₁ ℓ₂ : Level
Original file line number Diff line number Diff line change 6
6
7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
+ module Algebra.Lattice.Construct.LiftedChoice where
10
+
9
11
open import Algebra
10
- open import Algebra.Lattice
11
- open import Algebra.Construct.LiftedChoice
12
+ using (Op₂; IsSelectiveMagma; Associative; Commutative)
13
+ open import Algebra.Lattice.Structures using (IsSemilattice)
14
+ open import Algebra.Construct.LiftedChoice using (Lift; isBand; comm)
12
15
open import Relation.Binary.Core using (Rel; _Preserves_⟶_)
13
16
open import Relation.Binary.Structures using (IsEquivalence)
14
17
open import Level using (Level)
15
18
16
- module Algebra.Lattice.Construct.LiftedChoice where
17
-
18
19
private
19
20
variable
20
21
a b p ℓ : Level
Original file line number Diff line number Diff line change 9
9
10
10
{-# OPTIONS --cubical-compatible --safe #-}
11
11
12
- open import Algebra.Core using (Op₂)
13
- open import Algebra.Definitions
14
- open import Algebra.Lattice.Structures
15
12
open import Data.Product.Base using (_,_)
16
- open import Function.Base
17
- open import Relation.Binary.Core
13
+ open import Relation.Binary.Core using (Rel ; _⇔_)
18
14
19
15
module Algebra.Lattice.Construct.Subst.Equality
20
16
{a ℓ₁ ℓ₂} {A : Set a} {≈₁ : Rel A ℓ₁} {≈₂ : Rel A ℓ₂}
21
17
(equiv@(to , from) : ≈₁ ⇔ ≈₂)
22
18
where
23
19
20
+ open import Algebra.Core using (Op₂)
21
+ open import Algebra.Lattice.Structures
22
+ using (IsSemilattice ;IsLattice ;IsDistributiveLattice ;IsBooleanAlgebra )
23
+ open import Function.Base using (id)
24
24
open import Algebra.Construct.Subst.Equality equiv
25
25
open import Relation.Binary.Construct.Subst.Equality equiv
26
26
Original file line number Diff line number Diff line change @@ -17,8 +17,8 @@ open import Level using (Level)
17
17
18
18
module Algebra.Lattice.Construct.Zero {c ℓ : Level} where
19
19
20
- open import Algebra.Lattice.Bundles
21
- open import Data.Unit.Polymorphic
20
+ open import Algebra.Lattice.Bundles using (Semilattice)
21
+ open import Data.Unit.Polymorphic using (⊤)
22
22
23
23
------------------------------------------------------------------------
24
24
-- Bundles
You can’t perform that action at this time.
0 commit comments