Chebyshev polynomials over the reals: some extremal properties #
Chebyshev polynomials have largest leading coefficient, following proof in https://math.stackexchange.com/a/978145/1277
Main statements #
- leadingCoeff_le_of_forall_abs_le_one: If
Pis a real polynomial of degree at mostnand|P (x)| ≤ 1for allx ∈ [-1, 1]then the leading coefficient ofPis at most2 ^ (n - 1) - leadingCoeff_eq_iff_of_forall_abs_le_one: When
n ≥ 2, equality holds iffP = T_n
Implementation #
By monotonicity of 2 ^ (n - 1), we can assume that P has degree exactly n.
Using Lagrange interpolation, we can give a formula for the leading coefficient of P
as a linear combination of the values of P on the Chebyshev nodes (sumNodes_eq_coeff).
The Chebyshev polynomial T_n has value ±1 on the nodes, with the same signs as the
coefficients of the linear combination (negOnePow_mul_leadingCoeffC_pos).
Since |P (x)| ≤ 1 on the nodes, this implies that the leading coefficient of P is bounded
by that of T_n, which is known to equal 2 ^ (n - 1).
Moreover, equality holds iff P and T_n agree on the nodes, which implies that they coincide.
For a polynomial P and coefficient function c, sumNodes n c P is a linear combination
of P evaluated at the n'th order Chebyshev nodes, with coefficients taken from c.
Equations
- Polynomial.Chebyshev.sumNodes n c P = ∑ i ∈ Finset.Iic n, Polynomial.eval (Polynomial.Chebyshev.node n i) P * c i