Skip to content

Commit

Permalink
feat(algebra/group_with_zero): add zero_mul_eq_const and mul_zero_eq_…
Browse files Browse the repository at this point in the history
…const (#11021)

These are to match the corresponding lemmas about unapplied application of multiplication by 1. Like those lemmas, these are not marked simp.
  • Loading branch information
eric-wieser committed Dec 27, 2021
1 parent a360354 commit 463be88
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/algebra/group_with_zero/basic.lean
Expand Up @@ -90,6 +90,12 @@ lemma mul_eq_zero_of_ne_zero_imp_eq_zero {a b : M₀} (h : a ≠ 0 → b = 0) :
a * b = 0 :=
if ha : a = 0 then by rw [ha, zero_mul] else by rw [h ha, mul_zero]

/-- To match `one_mul_eq_id`. -/
lemma zero_mul_eq_const : ((*) (0 : M₀)) = function.const _ 0 := funext zero_mul

/-- To match `mul_one_eq_id`. -/
lemma mul_zero_eq_const : (* (0 : M₀)) = function.const _ 0 := funext mul_zero

end mul_zero_class

/-- Pushforward a `no_zero_divisors` instance along an injective function. -/
Expand Down

0 comments on commit 463be88

Please sign in to comment.