Commit 523f8fb 1 parent a326c8c commit 523f8fb Copy full SHA for 523f8fb
File tree 1 file changed +10
-0
lines changed
1 file changed +10
-0
lines changed Original file line number Diff line number Diff line change @@ -249,6 +249,11 @@ theorem ofMul_eq_zero {A : Type*} [One A] {x : A} : Additive.ofMul x = 0 ↔ x =
249
249
theorem toMul_zero [One α] : toMul (0 : Additive α) = 1 := rfl
250
250
#align to_mul_zero toMul_zero
251
251
252
+ @[simp]
253
+ lemma toMul_eq_one {α : Type *} [One α] {x : Additive α} :
254
+ Additive.toMul x = 1 ↔ x = 0 :=
255
+ Iff.rfl
256
+
252
257
instance [Zero α] : One (Multiplicative α) :=
253
258
⟨Multiplicative.ofAdd 0 ⟩
254
259
@@ -267,6 +272,11 @@ theorem toAdd_one [Zero α] : toAdd (1 : Multiplicative α) = 0 :=
267
272
rfl
268
273
#align to_add_one toAdd_one
269
274
275
+ @[simp]
276
+ lemma toAdd_eq_zero {α : Type *} [Zero α] {x : Multiplicative α} :
277
+ Multiplicative.toAdd x = 0 ↔ x = 1 :=
278
+ Iff.rfl
279
+
270
280
instance Additive.addZeroClass [MulOneClass α] : AddZeroClass (Additive α) where
271
281
zero := 0
272
282
add := (· + ·)
You can’t perform that action at this time.
0 commit comments