Skip to content

Commit fe42b2c

Browse files
committed
Add new law to constructed modules
1 parent c456702 commit fe42b2c

File tree

2 files changed

+4
-0
lines changed

2 files changed

+4
-0
lines changed

src/Algebra/Module/Construct/DirectProduct.agda

+2
Original file line numberDiff line numberDiff line change
@@ -97,6 +97,7 @@ semimodule M N = record
9797
{ isSemimodule = record
9898
{ isBisemimodule = Bisemimodule.isBisemimodule
9999
(bisemimodule M.bisemimodule N.bisemimodule)
100+
; *ₗ-*ᵣ-comm = λ x m M.*ₗ-*ᵣ-comm x (proj₁ m) , N.*ₗ-*ᵣ-comm x (proj₂ m)
100101
}
101102
} where module M = Semimodule M; module N = Semimodule N
102103

@@ -155,5 +156,6 @@ bimodule M N = record
155156
⟨module⟩ M N = record
156157
{ isModule = record
157158
{ isBimodule = Bimodule.isBimodule (bimodule M.bimodule N.bimodule)
159+
; *ₗ-*ᵣ-comm = λ x m M.*ₗ-*ᵣ-comm x (proj₁ m) , N.*ₗ-*ᵣ-comm x (proj₂ m)
158160
}
159161
} where module M = Module M; module N = Module N

src/Algebra/Module/Construct/TensorUnit.agda

+2
Original file line numberDiff line numberDiff line change
@@ -77,6 +77,7 @@ semimodule : {R : CommutativeSemiring c ℓ} → Semimodule R c ℓ
7777
semimodule {R = commutativeSemiring} = record
7878
{ isSemimodule = record
7979
{ isBisemimodule = Bisemimodule.isBisemimodule bisemimodule
80+
; *ₗ-*ᵣ-comm = λ x m *-comm x m
8081
}
8182
} where open CommutativeSemiring commutativeSemiring
8283

@@ -113,5 +114,6 @@ bimodule {R = ring} = record
113114
⟨module⟩ {R = commutativeRing} = record
114115
{ isModule = record
115116
{ isBimodule = Bimodule.isBimodule bimodule
117+
; *ₗ-*ᵣ-comm = λ x m *-comm x m
116118
}
117119
} where open CommutativeRing commutativeRing

0 commit comments

Comments
 (0)