Skip to content

Commit 523f8fb

Browse files
wuprkbuzzard
authored andcommitted
feat(Algebra/Group/TypeTags): Add toMul_eq_one and toAdd_eq_zero (#14097)
1 parent a326c8c commit 523f8fb

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

Mathlib/Algebra/Group/TypeTags.lean

+10
Original file line numberDiff line numberDiff line change
@@ -249,6 +249,11 @@ theorem ofMul_eq_zero {A : Type*} [One A] {x : A} : Additive.ofMul x = 0 ↔ x =
249249
theorem toMul_zero [One α] : toMul (0 : Additive α) = 1 := rfl
250250
#align to_mul_zero toMul_zero
251251

252+
@[simp]
253+
lemma toMul_eq_one {α : Type*} [One α] {x : Additive α} :
254+
Additive.toMul x = 1 ↔ x = 0 :=
255+
Iff.rfl
256+
252257
instance [Zero α] : One (Multiplicative α) :=
253258
⟨Multiplicative.ofAdd 0
254259

@@ -267,6 +272,11 @@ theorem toAdd_one [Zero α] : toAdd (1 : Multiplicative α) = 0 :=
267272
rfl
268273
#align to_add_one toAdd_one
269274

275+
@[simp]
276+
lemma toAdd_eq_zero {α : Type*} [Zero α] {x : Multiplicative α} :
277+
Multiplicative.toAdd x = 0 ↔ x = 1 :=
278+
Iff.rfl
279+
270280
instance Additive.addZeroClass [MulOneClass α] : AddZeroClass (Additive α) where
271281
zero := 0
272282
add := (· + ·)

0 commit comments

Comments
 (0)