The iterated derivative of an analytic function #
If a function is analytic, written as f (x + y) = ∑ pₙ (y, ..., y)
then its n
-th iterated
derivative at x
is given by (v₁, ..., vₙ) ↦ ∑ pₙ (v_{σ (1)}, ..., v_{σ (n)})
where the sum
is over all permutations of {1, ..., n}
. In particular, it is symmetric.
This generalizes the result of HasFPowerSeriesOnBall.factorial_smul
giving
D^n f (v, ..., v) = n! * pₙ (v, ..., v)
.
Main result #
HasFPowerSeriesOnBall.iteratedFDeriv_eq_sum
shows thatiteratedFDeriv 𝕜 n f x v = ∑ σ : Perm (Fin n), p n (fun i ↦ v (σ i))
, whenf
hasp
as power series within the sets
on the ballB (x, r)
.ContDiffAt.iteratedFDeriv_comp_perm
proves the symmetry of the iterated derivative of an analytic function, in the formiteratedFDeriv 𝕜 n f x (v ∘ σ) = iteratedFDeriv 𝕜 n f x v
for any permutationσ
ofFin n
.
Versions within sets are also given.
Implementation #
To prove the formula for the iterated derivative, we decompose an analytic function as
the sum of fun y ↦ pₙ (y, ..., y)
and the rest. For the former, its iterated derivative follows
from the formula for iterated derivatives of multilinear maps
(see ContinuousMultilinearMap.iteratedFDeriv_comp_diagonal
). For the latter, we show by
induction on n
that if the n
-th term in a power series is zero, then the n
-th iterated
derivative vanishes (see HasFPowerSeriesWithinOnBall.iteratedFDerivWithin_eq_zero
).
All these results are proved assuming additionally that the function is analytic on the relevant set (which does not follow from the fact that the function has a power series, if the target space is not complete). This makes it possible to avoid all completeness assumptions in the final statements. When needed, we give versions of some statements assuming completeness and dropping analyticity, for ease of use.
Formal multilinear series associated to the iterated derivative, defined by iterating
p ↦ p.derivSeries
and currying suitably. It is defined so that, if a function has p
as a power
series, then its iterated derivative of order k
has p.iteratedFDerivSeries k
as a power
series.
Equations
- One or more equations did not get rendered due to their size.
- p.iteratedFDerivSeries 0 = (↑(continuousMultilinearCurryFin0 𝕜 E F).symm.toContinuousLinearEquiv).compFormalMultilinearSeries p
Instances For
If a function has a power series on a ball, then so do its iterated derivatives.
If the n
-th term in a power series is zero, then the n
-th derivative of the corresponding
function vanishes.
If a function has a power series in a ball, then its n
-th iterated derivative is given by
(v₁, ..., vₙ) ↦ ∑ pₙ (v_{σ (1)}, ..., v_{σ (n)})
where the sum is over all
permutations of {1, ..., n}
.
If a function has a power series in a ball, then its n
-th iterated derivative is given by
(v₁, ..., vₙ) ↦ ∑ pₙ (v_{σ (1)}, ..., v_{σ (n)})
where the sum is over all
permutations of {1, ..., n}
.
If a function has a power series in a ball, then its n
-th iterated derivative is given by
(v₁, ..., vₙ) ↦ ∑ pₙ (v_{σ (1)}, ..., v_{σ (n)})
where the sum is over all
permutations of {1, ..., n}
.
If a function has a power series in a ball, then its n
-th iterated derivative is given by
(v₁, ..., vₙ) ↦ ∑ pₙ (v_{σ (1)}, ..., v_{σ (n)})
where the sum is over all
permutations of {1, ..., n}
.
The n
-th iterated derivative of an analytic function on a set is symmetric.
The n
-th iterated derivative of an analytic function on a set is symmetric.
The n
-th iterated derivative of an analytic function is symmetric.
The n
-th iterated derivative of an analytic function is symmetric.