Skip to content

Commit 5ac10dd

Browse files
authored
[imports] Algebra.Lattice.Construct.* (#2603)
* Cleaning import Lattice 2 * t * fix
1 parent 80f01cd commit 5ac10dd

File tree

4 files changed

+16
-16
lines changed

4 files changed

+16
-16
lines changed

src/Algebra/Lattice/Construct/DirectProduct.agda

Lines changed: 4 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -13,15 +13,14 @@
1313

1414
{-# OPTIONS --cubical-compatible --safe #-}
1515

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)
1820
import Algebra.Construct.DirectProduct as DirectProduct
1921
open import Data.Product.Base using (_,_; _<*>_)
20-
open import Data.Product.Relation.Binary.Pointwise.NonDependent
2122
open import Level using (Level; _⊔_)
2223

23-
module Algebra.Lattice.Construct.DirectProduct where
24-
2524
private
2625
variable
2726
a b ℓ₁ ℓ₂ : Level

src/Algebra/Lattice/Construct/LiftedChoice.agda

Lines changed: 5 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -6,15 +6,16 @@
66

77
{-# OPTIONS --cubical-compatible --safe #-}
88

9+
module Algebra.Lattice.Construct.LiftedChoice where
10+
911
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)
1215
open import Relation.Binary.Core using (Rel; _Preserves_⟶_)
1316
open import Relation.Binary.Structures using (IsEquivalence)
1417
open import Level using (Level)
1518

16-
module Algebra.Lattice.Construct.LiftedChoice where
17-
1819
private
1920
variable
2021
a b p ℓ : Level

src/Algebra/Lattice/Construct/Subst/Equality.agda

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -9,18 +9,18 @@
99

1010
{-# OPTIONS --cubical-compatible --safe #-}
1111

12-
open import Algebra.Core using (Op₂)
13-
open import Algebra.Definitions
14-
open import Algebra.Lattice.Structures
1512
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 ; _⇔_)
1814

1915
module Algebra.Lattice.Construct.Subst.Equality
2016
{a ℓ₁ ℓ₂} {A : Set a} {≈₁ : Rel A ℓ₁} {≈₂ : Rel A ℓ₂}
2117
(equiv@(to , from) : ≈₁ ⇔ ≈₂)
2218
where
2319

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)
2424
open import Algebra.Construct.Subst.Equality equiv
2525
open import Relation.Binary.Construct.Subst.Equality equiv
2626

src/Algebra/Lattice/Construct/Zero.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -17,8 +17,8 @@ open import Level using (Level)
1717

1818
module Algebra.Lattice.Construct.Zero {c ℓ : Level} where
1919

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 (⊤)
2222

2323
------------------------------------------------------------------------
2424
-- Bundles

0 commit comments

Comments
 (0)