File tree 1 file changed +4
-5
lines changed
src/Algebra/Module/Construct
1 file changed +4
-5
lines changed Original file line number Diff line number Diff line change @@ -64,16 +64,15 @@ module Nagata (ring : Ring r ℓr) (bimodule : Bimodule ring ring m ℓm) where
64
64
renaming (Carrierᴹ to M)
65
65
66
66
open AbelianGroup M.+ᴹ-abelianGroup
67
- renaming (setoid to setoidᴹ; sym to symᴹ)
68
67
hiding (_≈_)
69
68
70
- +ᴹ-middleFour = Consequences.comm∧assoc⇒middleFour setoidᴹ +ᴹ-cong +ᴹ-comm +ᴹ-assoc
69
+ +ᴹ-middleFour = Consequences.comm∧assoc⇒middleFour ≈ᴹ-setoid +ᴹ-cong +ᴹ-comm +ᴹ-assoc
71
70
72
- open ≈-Reasoning setoidᴹ
71
+ open ≈-Reasoning ≈ᴹ-setoid
73
72
74
73
open module N = Bimodule (DirectProduct.bimodule TensorUnit.bimodule bimodule)
75
74
using ()
76
- renaming (Carrierᴹ to N
75
+ renaming ( Carrierᴹ to N
77
76
; _≈ᴹ_ to _≈_
78
77
; _+ᴹ_ to _+_
79
78
; 0ᴹ to 0#
@@ -138,7 +137,7 @@ module Nagata (ring : Ring r ℓr) (bimodule : Bimodule ring ring m ℓm) where
138
137
r₁ *ₗ (r₂ *ₗ m₃) +ᴹ (r₁ *ₗ (m₂ *ᵣ r₃) +ᴹ (m₁ *ᵣ r₂) *ᵣ r₃)
139
138
≈⟨ +ᴹ-assoc (r₁ *ₗ (r₂ *ₗ m₃)) (r₁ *ₗ (m₂ *ᵣ r₃)) ((m₁ *ᵣ r₂) *ᵣ r₃) ⟨
140
139
(r₁ *ₗ (r₂ *ₗ m₃) +ᴹ r₁ *ₗ (m₂ *ᵣ r₃)) +ᴹ (m₁ *ᵣ r₂) *ᵣ r₃
141
- ≈⟨ +ᴹ-cong (symᴹ (*ₗ-distribˡ r₁ (r₂ *ₗ m₃) (m₂ *ᵣ r₃))) (*ᵣ-assoc m₁ r₂ r₃) ⟩
140
+ ≈⟨ +ᴹ-cong (≈ᴹ-sym (*ₗ-distribˡ r₁ (r₂ *ₗ m₃) (m₂ *ᵣ r₃))) (*ᵣ-assoc m₁ r₂ r₃) ⟩
142
141
r₁ *ₗ (r₂ *ₗ m₃ +ᴹ m₂ *ᵣ r₃) +ᴹ m₁ *ᵣ (r₂ R.* r₃) ∎)
143
142
144
143
distribˡ : _*_ DistributesOverˡ _+_
You can’t perform that action at this time.
0 commit comments