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 88
99module Algebra.Lattice.Bundles.Raw where
1010
11- open import Algebra.Core
11+ open import Algebra.Core using (Op₂)
1212open import Algebra.Bundles.Raw using (RawMagma)
1313open import Level using (suc; _⊔_)
1414open import Relation.Binary.Core using (Rel)
Original file line number Diff line number Diff line change 88{-# OPTIONS --cubical-compatible --safe #-}
99
1010open import Algebra.Construct.NaturalChoice.Base
11- import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp
11+ using (MaxOperator; MaxOp⇒ MinOp)
1212open import Relation.Binary.Bundles using (TotalPreorder)
1313
1414module Algebra.Lattice.Construct.NaturalChoice.MaxOp
1515 {a ℓ₁ ℓ₂} {O : TotalPreorder a ℓ₁ ℓ₂} (maxOp : MaxOperator O)
1616 where
1717
18+ import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp
19+
1820private
1921 module Min = MinOp (MaxOp⇒MinOp maxOp)
2022
Original file line number Diff line number Diff line change 66
77{-# OPTIONS --cubical-compatible --safe #-}
88
9- open import Algebra.Lattice.Bundles
10- open import Algebra.Construct.NaturalChoice.Base
9+ open import Algebra.Construct.NaturalChoice.Base using (MinOperator; MaxOperator)
1110open import Relation.Binary.Bundles using (TotalPreorder)
1211
1312module Algebra.Lattice.Construct.NaturalChoice.MinMaxOp
@@ -22,6 +21,7 @@ open MaxOperator maxOp
2221
2322open import Algebra.Lattice.Structures _≈_
2423open import Algebra.Construct.NaturalChoice.MinMaxOp minOp maxOp
24+ open import Algebra.Lattice.Bundles using (Lattice; DistributiveLattice)
2525open import Relation.Binary.Reasoning.Preorder preorder
2626
2727------------------------------------------------------------------------
Original file line number Diff line number Diff line change 77
88{-# OPTIONS --cubical-compatible --safe #-}
99
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)
1311open import Relation.Binary.Bundles using (TotalPreorder)
1412
1513module Algebra.Lattice.Construct.NaturalChoice.MinOp
@@ -18,8 +16,9 @@ module Algebra.Lattice.Construct.NaturalChoice.MinOp
1816open TotalPreorder O
1917open MinOperator minOp
2018
21- open import Algebra.Lattice.Structures _≈_
2219open import Algebra.Construct.NaturalChoice.MinOp minOp
20+ open import Algebra.Lattice.Bundles using (Semilattice)
21+ open import Algebra.Lattice.Structures _≈_
2322
2423------------------------------------------------------------------------
2524-- Structures
You can’t perform that action at this time.
0 commit comments