File tree Expand file tree Collapse file tree 3 files changed +19
-10
lines changed Expand file tree Collapse file tree 3 files changed +19
-10
lines changed Original file line number Diff line number Diff line change 26
26
module Algebra.Module.Bundles where
27
27
28
28
open import Algebra.Bundles
29
- open import Algebra.Core
29
+ using (Semiring; Ring; CommutativeSemiring; CommutativeRing;
30
+ CommutativeMonoid; AbelianGroup)
31
+ open import Algebra.Core using (Op₁; Op₂)
30
32
open import Algebra.Definitions using (Involutive)
31
33
import Algebra.Module.Bundles.Raw as Raw
32
- open import Algebra.Module.Core
34
+ open import Algebra.Module.Core using (Opₗ; Opᵣ)
33
35
open import Algebra.Module.Structures
36
+ using (IsLeftSemimodule; IsRightSemimodule; IsBisemimodule;
37
+ IsSemimodule; IsLeftModule; IsRightModule; IsModule; IsBimodule)
34
38
open import Algebra.Module.Definitions
35
- open import Algebra.Properties.Group
36
- open import Function.Base
37
- open import Level
39
+ open import Function.Base using (flip)
40
+ open import Level using (Level; _⊔_; suc)
38
41
open import Relation.Binary.Core using (Rel)
39
42
open import Relation.Nullary using (¬_)
40
43
import Relation.Binary.Reasoning.Setoid as ≈-Reasoning
Original file line number Diff line number Diff line change @@ -13,11 +13,14 @@ open import Relation.Binary.Structures using (IsEquivalence)
13
13
module Algebra.Module.Structures where
14
14
15
15
open import Algebra.Bundles
16
- open import Algebra.Core
17
- open import Algebra.Module.Core
16
+ using (Semiring; Ring; CommutativeSemiring; CommutativeRing)
17
+ open import Algebra.Core using (Op₁; Op₂)
18
+ open import Algebra.Module.Core using (Opₗ; Opᵣ)
18
19
import Algebra.Definitions as Defs
19
20
open import Algebra.Module.Definitions
20
- open import Algebra.Structures
21
+ using (module LeftDefs ; module RightDefs ; module BiDefs ;
22
+ module SimultaneousBiDefs )
23
+ open import Algebra.Structures using (IsCommutativeMonoid; IsAbelianGroup)
21
24
open import Data.Product.Base using (_,_; proj₁; proj₂)
22
25
open import Level using (Level; _⊔_)
23
26
Original file line number Diff line number Diff line change @@ -14,10 +14,13 @@ open import Relation.Binary.Structures using (IsEquivalence)
14
14
module Algebra.Module.Structures.Biased where
15
15
16
16
open import Algebra.Bundles
17
- open import Algebra.Core
18
- open import Algebra.Module.Core
17
+ using (Semiring; Ring; CommutativeSemiring; CommutativeRing)
18
+ open import Algebra.Core using (Op₁; Op₂)
19
+ open import Algebra.Module.Core using (Opₗ; Opᵣ)
19
20
open import Algebra.Module.Consequences
20
21
open import Algebra.Module.Structures
22
+ using (IsLeftSemimodule; IsRightSemimodule; IsBisemimodule;
23
+ IsSemimodule; IsLeftModule; IsRightModule; IsModule)
21
24
open import Function.Base using (flip)
22
25
open import Level using (Level; _⊔_)
23
26
You can’t perform that action at this time.
0 commit comments