File tree Expand file tree Collapse file tree 1 file changed +4
-2
lines changed Expand file tree Collapse file tree 1 file changed +4
-2
lines changed Original file line number Diff line number Diff line change @@ -222,10 +222,12 @@ variable [CommMagma G] {a : G}
222222@[to_additive]
223223theorem mul_comm : ∀ a b : G, a * b = b * a := CommMagma.mul_comm
224224
225- @[simp] lemma isLeftRegular_iff_isRegular : IsLeftRegular a ↔ IsRegular a := by
225+ @[to_additive (attr := simp)]
226+ lemma isLeftRegular_iff_isRegular : IsLeftRegular a ↔ IsRegular a := by
226227 simp [isRegular_iff, IsLeftRegular, IsRightRegular, mul_comm]
227228
228- @[simp] lemma isRightRegular_iff_isRegular : IsRightRegular a ↔ IsRegular a := by
229+ @[to_additive (attr := simp)]
230+ lemma isRightRegular_iff_isRegular : IsRightRegular a ↔ IsRegular a := by
229231 simp [isRegular_iff, IsLeftRegular, IsRightRegular, mul_comm]
230232
231233/-- Any `CommMagma G` that satisfies `IsRightCancelMul G` also satisfies `IsLeftCancelMul G`. -/
You can’t perform that action at this time.
0 commit comments