shifted Legendre Polynomials #
In this file, we define the shifted Legendre polynomials shiftedLegendre n
for n : ℕ
as a
polynomial in ℤ[X]
. We prove some basic properties of the Legendre polynomials.
factorial_mul_shiftedLegendre_eq
: The analogue of Rodrigues' formula for the shifted Legendre polynomials;shiftedLegendre_eval_symm
: The values of the shifted Legendre polynomial atx
and1 - x
differ by a factor(-1)ⁿ
.
Reference #
Tags #
shifted Legendre polynomials, derivative
shiftedLegendre n
is an integer polynomial for each n : ℕ
, defined by:
Pₙ(x) = ∑ k ∈ Finset.range (n + 1), (-1)ᵏ * choose n k * choose (n + k) n * xᵏ
These polynomials appear in combinatorics and the theory of orthogonal polynomials.
Equations
- Polynomial.shiftedLegendre n = ∑ k ∈ Finset.range (n + 1), Polynomial.C ((-1) ^ k * ↑(n.choose k) * ↑((n + k).choose n)) * Polynomial.X ^ k
Instances For
The shifted Legendre polynomial multiplied by a factorial equals the higher-order derivative of
the combinatorial function X ^ n * (1 - X) ^ n
. This is the analogue of Rodrigues' formula for
the shifted Legendre polynomials.
The degree of shiftedLegendre n
is n
.
The values of the Legendre polynomial at x
and 1 - x
differ by a factor (-1)ⁿ
.