Skip to content

Commit e14c050

Browse files
committed
[ fix ] Module exports
1 parent c2cff82 commit e14c050

File tree

1 file changed

+9
-19
lines changed

1 file changed

+9
-19
lines changed

src/Algebra/Module/Bundles.agda

+9-19
Original file line numberDiff line numberDiff line change
@@ -295,27 +295,17 @@ record Module {r ℓr} (commutativeRing : CommutativeRing r ℓr) m ℓm
295295

296296
open IsModule isModule public
297297

298-
{- TODO: #898
299-
semimodule : Semimodule commutativeSemiring m ℓm
300-
semimodule = record { isSemimodule = isSemimodule }
301-
302-
open Semimodule semimodule public
303-
using ( leftSemimodule; isLeftSemimodule; rightSemimodule
304-
; isRightSemimodule; _*ᵣ_; *ₗ-comm; *ᵣ-comm; *ᵣ-cong
305-
; *ᵣ-zeroʳ; *ᵣ-distribˡ; *ᵣ-identityʳ; *ᵣ-assoc; *ᵣ-zeroˡ
306-
; *ᵣ-distribʳ)
307-
-}
308-
309-
leftModule : LeftModule ring m ℓm
310-
leftModule = record { isLeftModule = isLeftModule }
298+
bimodule : Bimodule ring ring m ℓm
299+
bimodule = record { isBimodule = isBimodule }
311300

312-
open LeftModule leftModule public
313-
using ( leftSemimodule
301+
open Bimodule bimodule public
302+
using ( leftModule; rightModule; leftSemimodule; rightSemimodule
314303
; +ᴹ-abelianGroup; +ᴹ-group; +ᴹ-commutativeMonoid; +ᴹ-monoid
315304
; +ᴹ-semigroup; +ᴹ-magma ; +ᴹ-rawMonoid; +ᴹ-rawMagma)
316305

317-
rightModule : RightModule ring m ℓm
318-
rightModule = record { isRightModule = isRightModule }
306+
{- TODO: #898
307+
semimodule : Semimodule commutativeSemiring m ℓm
308+
semimodule = record { isSemimodule = isSemimodule }
319309
320-
open RightModule rightModule public
321-
using (rightSemimodule)
310+
open Semimodule semimodule public using (*ₗ-comm; *ᵣ-comm)
311+
-}

0 commit comments

Comments
 (0)