Skip to content

Commit 982fcae

Browse files
authored
import cleaning Module 1 (#2607)
1 parent 183c6b0 commit 982fcae

File tree

6 files changed

+12
-10
lines changed

6 files changed

+12
-10
lines changed

src/Algebra/Module/Definitions/Bi.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ module Algebra.Module.Definitions.Bi
1515
{a a′ b ℓb} (A : Set a) (A′ : Set a′) {B : Set b} (_≈_ : Rel B ℓb)
1616
where
1717

18-
open import Algebra.Module.Core
18+
open import Algebra.Module.Core using (Opₗ; Opᵣ)
1919

2020
Associative : Opₗ A B Opᵣ A′ B Set _
2121
Associative _∙ₗ_ _∙ᵣ_ = x m y ((x ∙ₗ m) ∙ᵣ y) ≈ (x ∙ₗ (m ∙ᵣ y))

src/Algebra/Module/Definitions/Bi/Simultaneous.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -6,13 +6,13 @@
66

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

9-
open import Relation.Binary
9+
open import Relation.Binary using (Rel)
1010

1111
module Algebra.Module.Definitions.Bi.Simultaneous
1212
{a b ℓb} (A : Set a) {B : Set b} (_≈_ : Rel B ℓb)
1313
where
1414

15-
open import Algebra.Module.Core
15+
open import Algebra.Module.Core using (Opₗ; Opᵣ)
1616

1717
Coincident : Opₗ A B Opᵣ A B Set _
1818
Coincident _∙ₗ_ _∙ᵣ_ = x m (x ∙ₗ m) ≈ (m ∙ᵣ x)

src/Algebra/Module/Definitions/Left.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -19,8 +19,8 @@ module Algebra.Module.Definitions.Left
1919
------------------------------------------------------------------------
2020
-- Binary operations
2121

22-
open import Algebra.Core
23-
open import Algebra.Module.Core
22+
open import Algebra.Core using (Op₂)
23+
open import Algebra.Module.Core using (Opₗ)
2424

2525
------------------------------------------------------------------------
2626
-- Properties of operations

src/Algebra/Module/Definitions/Right.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -19,8 +19,8 @@ module Algebra.Module.Definitions.Right
1919
------------------------------------------------------------------------
2020
-- Binary operations
2121

22-
open import Algebra.Core
23-
open import Algebra.Module.Core
22+
open import Algebra.Core using (Op₂)
23+
open import Algebra.Module.Core using (Opᵣ)
2424

2525
------------------------------------------------------------------------
2626
-- Properties of operations

src/Algebra/Module/Morphism/Construct/Composition.agda

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -9,10 +9,12 @@
99
module Algebra.Module.Morphism.Construct.Composition where
1010

1111
open import Algebra.Module.Bundles.Raw
12+
using (RawLeftSemimodule; RawLeftModule; RawRightSemimodule; RawRightModule;
13+
RawBisemimodule; RawBimodule; RawSemimodule; RawModule)
1214
open import Algebra.Module.Morphism.Structures
13-
open import Algebra.Morphism.Construct.Composition
15+
open import Algebra.Morphism.Construct.Composition using (isMonoidHomomorphism; isGroupHomomorphism)
1416
open import Function.Base using (_∘_)
15-
import Function.Construct.Composition as Func
17+
import Function.Construct.Composition as Func using (surjective)
1618
open import Level using (Level)
1719
open import Relation.Binary.Definitions using (Transitive)
1820

src/Algebra/Module/Morphism/Construct/Identity.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -19,7 +19,7 @@ open import Algebra.Module.Morphism.Structures
1919
; module SemimoduleMorphisms
2020
; module ModuleMorphisms
2121
)
22-
open import Algebra.Morphism.Construct.Identity
22+
open import Algebra.Morphism.Construct.Identity using ( isMonoidHomomorphism; isGroupHomomorphism)
2323
open import Data.Product.Base using (_,_)
2424
open import Function.Base using (id)
2525
import Function.Construct.Identity as Id

0 commit comments

Comments
 (0)