File tree Expand file tree Collapse file tree 6 files changed +8
-10
lines changed Expand file tree Collapse file tree 6 files changed +8
-10
lines changed Original file line number Diff line number Diff line change @@ -21,7 +21,7 @@ open import Algebra.Bundles.Raw
21
21
open import Algebra.Core using (Op₂)
22
22
open import Algebra.Definitions using (Congruent₂)
23
23
open import Algebra.Structures using (IsMagma; IsSemigroup; IsBand)
24
- open import Data.Empty.Polymorphic
24
+ open import Data.Empty.Polymorphic using (⊥)
25
25
open import Relation.Binary.Core using (Rel)
26
26
open import Relation.Binary.Structures using (IsEquivalence)
27
27
open import Relation.Binary.Definitions
Original file line number Diff line number Diff line change @@ -10,7 +10,7 @@ open import Algebra
10
10
11
11
module Algebra.Construct.LiftedChoice where
12
12
13
- open import Algebra.Consequences.Base
13
+ open import Algebra.Consequences.Base using (sel⇒idem)
14
14
open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂; [_,_]; [_,_]′)
15
15
open import Data.Product.Base using (_×_; _,_)
16
16
open import Function.Base using (const; _$_)
Original file line number Diff line number Diff line change @@ -17,7 +17,7 @@ open import Algebra.Core using (Op₁; Op₂)
17
17
open import Algebra.Structures
18
18
open import Data.Product.Base using (_,_)
19
19
open import Function.Base using (id; _∘′_; const)
20
- open import Level
20
+ open import Level using (Level; _⊔_)
21
21
open import Relation.Binary.Core using (Rel)
22
22
open import Relation.Binary.Bundles using (Setoid)
23
23
open import Relation.Binary.Structures using (IsEquivalence)
Original file line number Diff line number Diff line change 10
10
{-# OPTIONS --cubical-compatible --safe #-}
11
11
12
12
open import Data.Product.Base as Product
13
- open import Relation.Binary.Core
13
+ open import Relation.Binary.Core using (Rel; _⇔_)
14
14
15
15
module Algebra.Construct.Subst.Equality
16
16
{a ℓ₁ ℓ₂} {A : Set a} {≈₁ : Rel A ℓ₁} {≈₂ : Rel A ℓ₂}
@@ -20,7 +20,7 @@ module Algebra.Construct.Subst.Equality
20
20
open import Algebra.Definitions
21
21
open import Algebra.Structures
22
22
import Data.Sum.Base as Sum
23
- open import Function.Base
23
+ open import Function.Base using (id; _∘_)
24
24
open import Relation.Binary.Construct.Subst.Equality equiv
25
25
26
26
------------------------------------------------------------------------
Original file line number Diff line number Diff line change @@ -15,7 +15,7 @@ open import Level using (Level)
15
15
module Algebra.Construct.Terminal {c ℓ : Level} where
16
16
17
17
open import Algebra.Bundles
18
- open import Data.Unit.Polymorphic
18
+ open import Data.Unit.Polymorphic using (⊤)
19
19
open import Relation.Binary.Core using (Rel)
20
20
21
21
------------------------------------------------------------------------
Original file line number Diff line number Diff line change @@ -19,10 +19,8 @@ open import Level using (Level)
19
19
20
20
module Algebra.Construct.Zero {c ℓ : Level} where
21
21
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)
26
24
27
25
------------------------------------------------------------------------
28
26
-- Re-export those algebras which are both initial and terminal
You can’t perform that action at this time.
0 commit comments