Skip to content

Commit 4fa1e39

Browse files
committed
Jiggle comment
1 parent 193992b commit 4fa1e39

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

src/Algebra/Ideal.agda

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -17,9 +17,12 @@ import Algebra.Module.Construct.TensorUnit as TU
1717
open import Algebra.NormalSubgroup (+-group)
1818
open import Level
1919

20+
------------------------------------------------------------------------
21+
-- Definition
22+
23+
-- a (two sided) ideal is exactly a subbimodule of R considered as a bimodule over itself
2024
record Ideal c′ ℓ′ : Set (c ⊔ ℓ ⊔ suc (c′ ⊔ ℓ′)) where
2125
field
22-
-- a (two sided) ideal is exactly a subbimodule of R considered as a bimodule over itself
2326
subbimodule : Subbimodule (TU.bimodule {R = R}) c′ ℓ′
2427

2528
open Subbimodule subbimodule public

0 commit comments

Comments
 (0)