Skip to content

Commit

Permalink
chore(finsupp/basic): weaken hypotheses (#18874)
Browse files Browse the repository at this point in the history
these are already in mathlib4, I just missed them in mathlib3.
  • Loading branch information
ericrbg committed Apr 26, 2023
1 parent 9b2b58d commit 57911c5
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/data/finsupp/basic.lean
Expand Up @@ -1259,16 +1259,16 @@ Throughout this section, some `monoid` and `semiring` arguments are specified wi
`[]`. See note [implicit instance arguments].
-/

@[simp] lemma coe_smul [add_monoid M] [smul_zero_class R M]
@[simp] lemma coe_smul [has_zero M] [smul_zero_class R M]
(b : R) (v : α →₀ M) : ⇑(b • v) = b • v := rfl
lemma smul_apply [add_monoid M] [smul_zero_class R M]
lemma smul_apply [has_zero M] [smul_zero_class R M]
(b : R) (v : α →₀ M) (a : α) : (b • v) a = b • (v a) := rfl

lemma _root_.is_smul_regular.finsupp [add_monoid M] [smul_zero_class R M] {k : R}
lemma _root_.is_smul_regular.finsupp [has_zero M] [smul_zero_class R M] {k : R}
(hk : is_smul_regular M k) : is_smul_regular (α →₀ M) k :=
λ _ _ h, ext $ λ i, hk (congr_fun h i)

instance [nonempty α] [add_monoid M] [smul_zero_class R M] [has_faithful_smul R M] :
instance [nonempty α] [has_zero M] [smul_zero_class R M] [has_faithful_smul R M] :
has_faithful_smul R (α →₀ M) :=
{ eq_of_smul_eq_smul := λ r₁ r₂ h, let ⟨a⟩ := ‹nonempty α› in eq_of_smul_eq_smul $ λ m : M,
by simpa using congr_fun (h (single a m)) a }
Expand Down

0 comments on commit 57911c5

Please sign in to comment.