We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 29d6a82 commit b6ef030Copy full SHA for b6ef030
src/Algebra/Ideal.agda
@@ -17,9 +17,12 @@ import Algebra.Module.Construct.TensorUnit as TU
17
open import Algebra.NormalSubgroup (+-group)
18
open import Level
19
20
+------------------------------------------------------------------------
21
+-- Definition
22
+
23
+-- a (two sided) ideal is exactly a subbimodule of R considered as a bimodule over itself
24
record Ideal c′ ℓ′ : Set (c ⊔ ℓ ⊔ suc (c′ ⊔ ℓ′)) where
25
field
- -- a (two sided) ideal is exactly a subbimodule of R considered as a bimodule over itself
26
subbimodule : Subbimodule (TU.bimodule {R = R}) c′ ℓ′
27
28
open Subbimodule subbimodule public
0 commit comments