Skip to content

Commit 80f01cd

Browse files
authored
[imports] Algebra.Bundles .. Algebra.Consequences.* (#2596)
* Algebra Bundles Consequences * Algebra Bundles Consequences * space * lines * cleaning import
1 parent 0305d6b commit 80f01cd

File tree

4 files changed

+7
-6
lines changed

4 files changed

+7
-6
lines changed

src/Algebra/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.Bundles.Raw where
1010

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

src/Algebra/Consequences/Base.agda

Lines changed: 4 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -10,10 +10,11 @@
1010
module Algebra.Consequences.Base
1111
{a} {A : Set a} where
1212

13-
open import Algebra.Core
13+
open import Algebra.Core using (Op₁; Op₂)
1414
open import Algebra.Definitions
15-
open import Data.Sum.Base
16-
open import Relation.Binary.Core
15+
using (Selective; Idempotent; SelfInverse; Involutive)
16+
open import Data.Sum.Base using (_⊎_; reduce)
17+
open import Relation.Binary.Core using (Rel)
1718
open import Relation.Binary.Definitions using (Reflexive)
1819

1920
module _ {ℓ} {_•_ : Op₂ A} (_≈_ : Rel A ℓ) where

src/Algebra/Consequences/Propositional.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -19,8 +19,8 @@ open import Relation.Binary.PropositionalEquality.Core
1919
open import Relation.Binary.PropositionalEquality.Properties
2020
using (setoid)
2121
open import Relation.Unary using (Pred)
22+
open import Algebra.Core using (Op₁; Op₂)
2223

23-
open import Algebra.Core
2424
open import Algebra.Definitions {A = A} _≡_
2525
import Algebra.Consequences.Setoid (setoid A) as Base
2626

src/Algebra/Consequences/Setoid.agda

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

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

10-
open import Relation.Binary.Core using (Rel)
1110
open import Relation.Binary.Bundles using (Setoid)
1211
open import Relation.Binary.Definitions
1312
using (Substitutive; Symmetric; Total)
@@ -22,6 +21,7 @@ open import Data.Product.Base using (_,_)
2221
open import Function.Base using (_$_; id; _∘_)
2322
open import Function.Definitions
2423
import Relation.Binary.Consequences as Bin
24+
open import Relation.Binary.Core using (Rel)
2525
open import Relation.Binary.Reasoning.Setoid S
2626
open import Relation.Unary using (Pred)
2727

0 commit comments

Comments
 (0)