File tree Expand file tree Collapse file tree 4 files changed +9
-8
lines changed Expand file tree Collapse file tree 4 files changed +9
-8
lines changed Original file line number Diff line number Diff line change 8
8
9
9
module Algebra.Lattice.Bundles.Raw where
10
10
11
- open import Algebra.Core
11
+ open import Algebra.Core using (Op₂)
12
12
open import Algebra.Bundles.Raw using (RawMagma)
13
13
open import Level using (suc; _⊔_)
14
14
open import Relation.Binary.Core using (Rel)
Original file line number Diff line number Diff line change 8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
10
open import Algebra.Construct.NaturalChoice.Base
11
- import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp
11
+ using (MaxOperator; MaxOp⇒ MinOp)
12
12
open import Relation.Binary.Bundles using (TotalPreorder)
13
13
14
14
module Algebra.Lattice.Construct.NaturalChoice.MaxOp
15
15
{a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂} (maxOp : MaxOperator O)
16
16
where
17
17
18
+ import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp
19
+
18
20
private
19
21
module Min = MinOp (MaxOp⇒MinOp maxOp)
20
22
Original file line number Diff line number Diff line change 6
6
7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
- open import Algebra.Lattice.Bundles
10
- open import Algebra.Construct.NaturalChoice.Base
9
+ open import Algebra.Construct.NaturalChoice.Base using (MinOperator; MaxOperator)
11
10
open import Relation.Binary.Bundles using (TotalPreorder)
12
11
13
12
module Algebra.Lattice.Construct.NaturalChoice.MinMaxOp
@@ -22,6 +21,7 @@ open MaxOperator maxOp
22
21
23
22
open import Algebra.Lattice.Structures _≈_
24
23
open import Algebra.Construct.NaturalChoice.MinMaxOp minOp maxOp
24
+ open import Algebra.Lattice.Bundles using (Lattice; DistributiveLattice)
25
25
open import Relation.Binary.Reasoning.Preorder preorder
26
26
27
27
------------------------------------------------------------------------
Original file line number Diff line number Diff line change 7
7
8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
- open import Algebra.Bundles
11
- open import Algebra.Lattice.Bundles
12
- open import Algebra.Construct.NaturalChoice.Base
10
+ open import Algebra.Construct.NaturalChoice.Base using (MinOperator)
13
11
open import Relation.Binary.Bundles using (TotalPreorder)
14
12
15
13
module Algebra.Lattice.Construct.NaturalChoice.MinOp
@@ -18,8 +16,9 @@ module Algebra.Lattice.Construct.NaturalChoice.MinOp
18
16
open TotalPreorder O
19
17
open MinOperator minOp
20
18
21
- open import Algebra.Lattice.Structures _≈_
22
19
open import Algebra.Construct.NaturalChoice.MinOp minOp
20
+ open import Algebra.Lattice.Bundles using (Semilattice)
21
+ open import Algebra.Lattice.Structures _≈_
23
22
24
23
------------------------------------------------------------------------
25
24
-- Structures
You can’t perform that action at this time.
0 commit comments