File tree Expand file tree Collapse file tree 4 files changed +7
-6
lines changed Expand file tree Collapse file tree 4 files changed +7
-6
lines changed Original file line number Diff line number Diff line change 8
8
9
9
module Algebra.Bundles.Raw where
10
10
11
- open import Algebra.Core
11
+ open import Algebra.Core using (Op₁; Op₂)
12
12
open import Relation.Binary.Core using (Rel)
13
13
open import Relation.Binary.Bundles.Raw using (RawSetoid)
14
14
open import Level using (suc; _⊔_)
Original file line number Diff line number Diff line change 10
10
module Algebra.Consequences.Base
11
11
{a} {A : Set a} where
12
12
13
- open import Algebra.Core
13
+ open import Algebra.Core using (Op₁; Op₂)
14
14
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)
17
18
open import Relation.Binary.Definitions using (Reflexive)
18
19
19
20
module _ {ℓ} {_•_ : Op₂ A} (_≈_ : Rel A ℓ) where
Original file line number Diff line number Diff line change @@ -19,8 +19,8 @@ open import Relation.Binary.PropositionalEquality.Core
19
19
open import Relation.Binary.PropositionalEquality.Properties
20
20
using (setoid)
21
21
open import Relation.Unary using (Pred)
22
+ open import Algebra.Core using (Op₁; Op₂)
22
23
23
- open import Algebra.Core
24
24
open import Algebra.Definitions {A = A} _≡_
25
25
import Algebra.Consequences.Setoid (setoid A) as Base
26
26
Original file line number Diff line number Diff line change 7
7
8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
- open import Relation.Binary.Core using (Rel)
11
10
open import Relation.Binary.Bundles using (Setoid)
12
11
open import Relation.Binary.Definitions
13
12
using (Substitutive; Symmetric; Total)
@@ -22,6 +21,7 @@ open import Data.Product.Base using (_,_)
22
21
open import Function.Base using (_$_; id; _∘_)
23
22
open import Function.Definitions
24
23
import Relation.Binary.Consequences as Bin
24
+ open import Relation.Binary.Core using (Rel)
25
25
open import Relation.Binary.Reasoning.Setoid S
26
26
open import Relation.Unary using (Pred)
27
27
You can’t perform that action at this time.
0 commit comments