Skip to content

Commit 1edd49c

Browse files
committed
Paramaterize Subbimodule rather than TU.bimodule
1 parent b6ef030 commit 1edd49c

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Algebra/Ideal.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -23,7 +23,7 @@ open import Level
2323
-- a (two sided) ideal is exactly a subbimodule of R considered as a bimodule over itself
2424
record Ideal c′ ℓ′ : Set (c ⊔ ℓ ⊔ suc (c′ ⊔ ℓ′)) where
2525
field
26-
subbimodule : Subbimodule (TU.bimodule {R = R}) c′ ℓ′
26+
subbimodule : Subbimodule {R = R} TU.bimodule c′ ℓ′
2727

2828
open Subbimodule subbimodule public
2929

0 commit comments

Comments
 (0)