Skip to content

Commit 4925719

Browse files
authored
end construct import cleaning (#2600)
* end construct import * cleaning import
1 parent 021b69c commit 4925719

File tree

6 files changed

+8
-10
lines changed

6 files changed

+8
-10
lines changed

src/Algebra/Construct/Initial.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ open import Algebra.Bundles.Raw
2121
open import Algebra.Core using (Op₂)
2222
open import Algebra.Definitions using (Congruent₂)
2323
open import Algebra.Structures using (IsMagma; IsSemigroup; IsBand)
24-
open import Data.Empty.Polymorphic
24+
open import Data.Empty.Polymorphic using (⊥)
2525
open import Relation.Binary.Core using (Rel)
2626
open import Relation.Binary.Structures using (IsEquivalence)
2727
open import Relation.Binary.Definitions

src/Algebra/Construct/LiftedChoice.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ open import Algebra
1010

1111
module Algebra.Construct.LiftedChoice where
1212

13-
open import Algebra.Consequences.Base
13+
open import Algebra.Consequences.Base using (sel⇒idem)
1414
open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂; [_,_]; [_,_]′)
1515
open import Data.Product.Base using (_×_; _,_)
1616
open import Function.Base using (const; _$_)

src/Algebra/Construct/Pointwise.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,7 @@ open import Algebra.Core using (Op₁; Op₂)
1717
open import Algebra.Structures
1818
open import Data.Product.Base using (_,_)
1919
open import Function.Base using (id; _∘′_; const)
20-
open import Level
20+
open import Level using (Level; _⊔_)
2121
open import Relation.Binary.Core using (Rel)
2222
open import Relation.Binary.Bundles using (Setoid)
2323
open import Relation.Binary.Structures using (IsEquivalence)

src/Algebra/Construct/Subst/Equality.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@
1010
{-# OPTIONS --cubical-compatible --safe #-}
1111

1212
open import Data.Product.Base as Product
13-
open import Relation.Binary.Core
13+
open import Relation.Binary.Core using (Rel; _⇔_)
1414

1515
module Algebra.Construct.Subst.Equality
1616
{a ℓ₁ ℓ₂} {A : Set a} {≈₁ : Rel A ℓ₁} {≈₂ : Rel A ℓ₂}
@@ -20,7 +20,7 @@ module Algebra.Construct.Subst.Equality
2020
open import Algebra.Definitions
2121
open import Algebra.Structures
2222
import Data.Sum.Base as Sum
23-
open import Function.Base
23+
open import Function.Base using (id; _∘_)
2424
open import Relation.Binary.Construct.Subst.Equality equiv
2525

2626
------------------------------------------------------------------------

src/Algebra/Construct/Terminal.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ open import Level using (Level)
1515
module Algebra.Construct.Terminal {c ℓ : Level} where
1616

1717
open import Algebra.Bundles
18-
open import Data.Unit.Polymorphic
18+
open import Data.Unit.Polymorphic using (⊤)
1919
open import Relation.Binary.Core using (Rel)
2020

2121
------------------------------------------------------------------------

src/Algebra/Construct/Zero.agda

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -19,10 +19,8 @@ open import Level using (Level)
1919

2020
module Algebra.Construct.Zero {c ℓ : Level} where
2121

22-
open import Algebra.Bundles.Raw
23-
using (RawMagma)
24-
open import Algebra.Bundles
25-
using (Magma; Semigroup; Band)
22+
open import Algebra.Bundles.Raw using (RawMagma)
23+
open import Algebra.Bundles using (Magma; Semigroup; Band)
2624

2725
------------------------------------------------------------------------
2826
-- Re-export those algebras which are both initial and terminal

0 commit comments

Comments
 (0)