Skip to content

Commit b707d83

Browse files
committed
fix: tidy up
1 parent c05773b commit b707d83

File tree

1 file changed

+1
-2
lines changed

1 file changed

+1
-2
lines changed

src/Algebra/Construct/Sub/Ring/Ideal.agda

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -12,15 +12,14 @@ module Algebra.Construct.Sub.Ring.Ideal {c ℓ} (R : Ring c ℓ) where
1212

1313
open import Algebra.Module.Construct.Sub.Bimodule using (Subbimodule)
1414
open import Algebra.Module.Construct.TensorUnit using (bimodule)
15-
open import Level
15+
open import Level using (suc; _⊔_)
1616

1717
------------------------------------------------------------------------
1818
-- Definition
1919
-- a (two sided) ideal is exactly a subbimodule of R considered as a bimodule over itself
2020

2121
record Ideal c′ ℓ′ : Set (c ⊔ ℓ ⊔ suc (c′ ⊔ ℓ′)) where
2222
field
23-
2423
subbimodule : Subbimodule {R = R} bimodule c′ ℓ′
2524

2625
open Subbimodule subbimodule public

0 commit comments

Comments
 (0)