Zulip Chat Archive
Stream: new members
Topic: Proving the derivative of a polynomial evaluates to zero
oishi (Dec 28 2024 at 11:59):
How should I prove this example? Specifically, I want to prove that the derivative evaluates to 0 when x=1. (I'm not sure if my formulation of this expression is correct.) I would like to complete this proof using a polynomial.
import Mathlib
example (h: m < n): Polynomial.eval 1 ((⇑Polynomial.derivative)^[m] ((Polynomial.C (1:ℝ) - Polynomial.X) ^ n)) = 0 := by sorry
Ruben Van de Velde (Dec 28 2024 at 12:05):
Are you perhaps missing an assumption on m and n?
oishi (Dec 28 2024 at 12:06):
oh, yes, m < n.
Ruben Van de Velde (Dec 28 2024 at 12:10):
My first step was found by rw?
:
rw [@Polynomial.iterate_derivative_eq_factorial_smul_sum]
oishi (Dec 28 2024 at 12:30):
I find something like this.
theorem Polynomial.aeval_iterate_derivative_of_lt
{R : Type u_1} [CommSemiring R] {A : Type u_3} [CommRing A] [Algebra R A]
(p : Polynomial R) (q : ℕ) (r : A) {p' : Polynomial A}
(hp : Polynomial.map (algebraMap R A) p = (Polynomial.X - Polynomial.C r) ^ q * p')
{k : ℕ} (hk : k < q) :
(Polynomial.aeval r) ((⇑Polynomial.derivative)^[k] p) = 0
Last updated: May 02 2025 at 03:31 UTC