Skip to content

Commit b99cfe8

Browse files
authored
cleaning import Lattice 1 (#2602)
* Cleaning import Lattice 1 * Cleaning import Lattice 1 * Cleaning import Lattice 1 * import cleaning
1 parent 3faa8c4 commit b99cfe8

File tree

4 files changed

+9
-8
lines changed

4 files changed

+9
-8
lines changed

src/Algebra/Lattice/Bundles/Raw.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,7 @@
88

99
module Algebra.Lattice.Bundles.Raw where
1010

11-
open import Algebra.Core
11+
open import Algebra.Core using (Op₂)
1212
open import Algebra.Bundles.Raw using (RawMagma)
1313
open import Level using (suc; _⊔_)
1414
open import Relation.Binary.Core using (Rel)

src/Algebra/Lattice/Construct/NaturalChoice/MaxOp.agda

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,13 +8,15 @@
88
{-# OPTIONS --cubical-compatible --safe #-}
99

1010
open import Algebra.Construct.NaturalChoice.Base
11-
import Algebra.Lattice.Construct.NaturalChoice.MinOp as MinOp
11+
using (MaxOperator; MaxOp⇒MinOp)
1212
open import Relation.Binary.Bundles using (TotalPreorder)
1313

1414
module 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+
1820
private
1921
module Min = MinOp (MaxOp⇒MinOp maxOp)
2022

src/Algebra/Lattice/Construct/NaturalChoice/MinMaxOp.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -6,8 +6,7 @@
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)
1110
open import Relation.Binary.Bundles using (TotalPreorder)
1211

1312
module Algebra.Lattice.Construct.NaturalChoice.MinMaxOp
@@ -22,6 +21,7 @@ open MaxOperator maxOp
2221

2322
open import Algebra.Lattice.Structures _≈_
2423
open import Algebra.Construct.NaturalChoice.MinMaxOp minOp maxOp
24+
open import Algebra.Lattice.Bundles using (Lattice; DistributiveLattice)
2525
open import Relation.Binary.Reasoning.Preorder preorder
2626

2727
------------------------------------------------------------------------

src/Algebra/Lattice/Construct/NaturalChoice/MinOp.agda

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -7,9 +7,7 @@
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)
1311
open import Relation.Binary.Bundles using (TotalPreorder)
1412

1513
module Algebra.Lattice.Construct.NaturalChoice.MinOp
@@ -18,8 +16,9 @@ module Algebra.Lattice.Construct.NaturalChoice.MinOp
1816
open TotalPreorder O
1917
open MinOperator minOp
2018

21-
open import Algebra.Lattice.Structures _≈_
2219
open import Algebra.Construct.NaturalChoice.MinOp minOp
20+
open import Algebra.Lattice.Bundles using (Semilattice)
21+
open import Algebra.Lattice.Structures _≈_
2322

2423
------------------------------------------------------------------------
2524
-- Structures

0 commit comments

Comments
 (0)