File tree 2 files changed +4
-0
lines changed
src/Algebra/Module/Construct
2 files changed +4
-0
lines changed Original file line number Diff line number Diff line change @@ -97,6 +97,7 @@ semimodule M N = record
97
97
{ isSemimodule = record
98
98
{ isBisemimodule = Bisemimodule.isBisemimodule
99
99
(bisemimodule M.bisemimodule N.bisemimodule)
100
+ ; *ₗ-*ᵣ-comm = λ x m → M.*ₗ-*ᵣ-comm x (proj₁ m) , N.*ₗ-*ᵣ-comm x (proj₂ m)
100
101
}
101
102
} where module M = Semimodule M; module N = Semimodule N
102
103
@@ -155,5 +156,6 @@ bimodule M N = record
155
156
⟨module⟩ M N = record
156
157
{ isModule = record
157
158
{ isBimodule = Bimodule.isBimodule (bimodule M.bimodule N.bimodule)
159
+ ; *ₗ-*ᵣ-comm = λ x m → M.*ₗ-*ᵣ-comm x (proj₁ m) , N.*ₗ-*ᵣ-comm x (proj₂ m)
158
160
}
159
161
} where module M = Module M; module N = Module N
Original file line number Diff line number Diff line change @@ -77,6 +77,7 @@ semimodule : {R : CommutativeSemiring c ℓ} → Semimodule R c ℓ
77
77
semimodule {R = commutativeSemiring} = record
78
78
{ isSemimodule = record
79
79
{ isBisemimodule = Bisemimodule.isBisemimodule bisemimodule
80
+ ; *ₗ-*ᵣ-comm = λ x m → *-comm x m
80
81
}
81
82
} where open CommutativeSemiring commutativeSemiring
82
83
@@ -113,5 +114,6 @@ bimodule {R = ring} = record
113
114
⟨module⟩ {R = commutativeRing} = record
114
115
{ isModule = record
115
116
{ isBimodule = Bimodule.isBimodule bimodule
117
+ ; *ₗ-*ᵣ-comm = λ x m → *-comm x m
116
118
}
117
119
} where open CommutativeRing commutativeRing
You can’t perform that action at this time.
0 commit comments