Commit 2024-02-01 09:38 f8b99c79

View on Github β†’

feat(Analysis.Calculus.FDeriv.Analytic + Analysis.Complex.TaylorSeries): Taylor series of holomorphic functions (#10087) See here on Zulip. This adds some general lemmas due to Junyan Xu, culminating in

theorem HasFPowerSeriesOnBall.hasSum_iteratedFDeriv {π•œ : Type*} [NontriviallyNormedField π•œ] {E : Type*}
    [ NormedAddCommGroup E] [NormedSpace π•œ E] {F : Type*} [NormedAddCommGroup F]
    [NormedSpace π•œ F] {p : FormalMultilinearSeries π•œ E F} {f : E β†’ F} {x : E} {r : ℝβ‰₯0∞}
    (h : HasFPowerSeriesOnBall f p x r) [CompleteSpace F] [CharZero π•œ] {y : E} (hy : y ∈ EMetric.ball 0 r) :+1:
    HasSum (fun n ↦ (n ! : π•œ)⁻¹‒ (iteratedFDeriv π•œ n f x) fun x ↦ y) (f (x + y))

and uses this to show that the Taylor series of a function that is complex differentiable on an open ball in β„‚ converges there to the function; similarly for functions that are holomorphic on all of β„‚:

lemma Complex.hasSum_taylorSeries_on_ball {E : Type*} [NormedAddCommGroup E] [NormedSpace β„‚ E]
    [CompleteSpace E] ⦃f : β„‚ β†’ E⦄ ⦃c : ℂ⦄ ⦃r : NNReal⦄ (hf : DifferentiableOn β„‚ f (Metric.ball c ↑r)) ⦃z : ℂ⦄
    (hz : z ∈ Metric.ball c ↑r) :
    HasSum (fun n ↦ (n ! : β„‚)⁻¹ β€’ (z - c) ^ n β€’ iteratedDeriv n f c) (f z)
lemma Complex.taylorSeries_eq_on_ball {E : Type*} [NormedAddCommGroup E] [NormedSpace β„‚ E]
    [CompleteSpace E] ⦃f : β„‚ β†’ E⦄ ⦃c : ℂ⦄ ⦃r : NNReal⦄ (hf : DifferentiableOn β„‚ f (Metric.ball c ↑r)) ⦃z : ℂ⦄
    (hz : z ∈ Metric.ball c ↑r) : 
    βˆ‘' (n : β„•), (n ! : β„‚)⁻¹ β€’ (z - c) ^ n β€’ iteratedDeriv n f c = f z
lemma Complex.taylorSeries_eq_on_ball' ⦃c : ℂ⦄ ⦃r : NNReal⦄ ⦃z : ℂ⦄ (hz : z ∈ Metric.ball c ↑r) {f : β„‚ β†’ β„‚}
    (hf : DifferentiableOn β„‚ f (Metric.ball c ↑r)) : 
    βˆ‘' (n : β„•), (n ! : β„‚)⁻¹ * iteratedDeriv n f c * (z - c) ^ n = f z

and similar lemmas for EMetric.balls and entire functions.

Estimated changes