Skip to content

Commit

Permalink
Merge branch 'eric-wieser/MonoidAlgebra.smul_single' into eric-wieser…
Browse files Browse the repository at this point in the history
…/MonoidAlgebra.isLocalHom
  • Loading branch information
eric-wieser committed Jan 22, 2025
2 parents 9a072a9 + f37f1ed commit c3e8710
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Polynomial/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -430,7 +430,7 @@ theorem monomial_pow (n : ℕ) (r : R) (k : ℕ) : monomial n r ^ k = monomial (

theorem smul_monomial {S} [SMulZeroClass S R] (a : S) (n : ℕ) (b : R) :
a • monomial n b = monomial n (a • b) :=
toFinsupp_injective <| by simp; rw [smul_single]
toFinsupp_injective <| AddMonoidAlgebra.smul_single _ _ _

theorem monomial_injective (n : ℕ) : Function.Injective (monomial n : R → R[X]) :=
(toFinsuppIso R).symm.injective.comp (single_injective n)
Expand Down

0 comments on commit c3e8710

Please sign in to comment.