Skip to content

Commit e18c588

Browse files
committed
Rearrange imports
1 parent 1edd49c commit e18c588

File tree

1 file changed

+5
-6
lines changed

1 file changed

+5
-6
lines changed

src/Algebra/Construct/Quotient/Ring.agda

Lines changed: 5 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -11,21 +11,20 @@ open import Algebra.Ideal using (Ideal)
1111

1212
module Algebra.Construct.Quotient.Ring {c ℓ} (R : Ring c ℓ) {c′ ℓ′} (I : Ideal R c′ ℓ′) where
1313

14+
open import Algebra.Morphism.Structures using (IsRingHomomorphism)
15+
open import Algebra.Properties.Ring R
16+
open import Algebra.Structures
17+
open import Level
18+
1419
open Ring R
1520
private module I = Ideal I
1621
open I using (ι; normalSubgroup)
1722

1823
open import Algebra.Construct.Quotient.Group +-group normalSubgroup public
1924
using (_≋_; _by_; ≋-refl; ≋-sym; ≋-trans; ≋-isEquivalence; ≈⇒≋; quotientIsGroup; quotientGroup; π; π-surjective)
2025
renaming (≋-∙-cong to ≋-+-cong; ≋-⁻¹-cong to ≋‿-‿cong)
21-
2226
open import Algebra.Definitions _≋_
23-
open import Algebra.Morphism.Structures using (IsRingHomomorphism)
2427
open import Algebra.Properties.Semiring semiring
25-
open import Algebra.Properties.Ring R
26-
open import Algebra.Structures
27-
open import Function.Definitions using (Surjective)
28-
open import Level
2928
open import Relation.Binary.Reasoning.Setoid setoid
3029

3130
≋-*-cong : Congruent₂ _*_

0 commit comments

Comments
 (0)