Documentation

Mathlib.Analysis.Calculus.SmoothSeries

Smoothness of series #

We show that series of functions are differentiable, or smooth, when each individual function in the series is and additionally suitable uniform summable bounds are satisfied.

More specifically,

We also give versions of these statements which are localized to a set.

Differentiability #

theorem summable_of_summable_hasFDerivAt_of_isPreconnected {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {f' : ฮฑ โ†’ E โ†’ E โ†’L[๐•œ] F} {s : Set E} {xโ‚€ : E} {x : E} (hu : Summable u) (hs : IsOpen s) (h's : IsPreconnected s) (hf : โˆ€ (n : ฮฑ), โˆ€ x โˆˆ s, HasFDerivAt (f n) (f' n x) x) (hf' : โˆ€ (n : ฮฑ), โˆ€ x โˆˆ s, โ€–f' n xโ€– โ‰ค u n) (hxโ‚€ : xโ‚€ โˆˆ s) (hf0 : Summable fun (x : ฮฑ) => f x xโ‚€) (hx : x โˆˆ s) :
Summable fun (n : ฮฑ) => f n x

Consider a series of functions โˆ‘' n, f n x on a preconnected open set. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series converges everywhere on the set.

theorem summable_of_summable_hasDerivAt_of_isPreconnected {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {g' : ฮฑ โ†’ ๐•œ โ†’ F} {t : Set ๐•œ} {yโ‚€ : ๐•œ} {y : ๐•œ} (hu : Summable u) (ht : IsOpen t) (h't : IsPreconnected t) (hg : โˆ€ (n : ฮฑ), โˆ€ y โˆˆ t, HasDerivAt (g n) (g' n y) y) (hg' : โˆ€ (n : ฮฑ), โˆ€ y โˆˆ t, โ€–g' n yโ€– โ‰ค u n) (hyโ‚€ : yโ‚€ โˆˆ t) (hg0 : Summable fun (x : ฮฑ) => g x yโ‚€) (hy : y โˆˆ t) :
Summable fun (n : ฮฑ) => g n y

Consider a series of functions โˆ‘' n, f n x on a preconnected open set. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series converges everywhere on the set.

theorem hasFDerivAt_tsum_of_isPreconnected {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {f' : ฮฑ โ†’ E โ†’ E โ†’L[๐•œ] F} {s : Set E} {xโ‚€ : E} {x : E} (hu : Summable u) (hs : IsOpen s) (h's : IsPreconnected s) (hf : โˆ€ (n : ฮฑ), โˆ€ x โˆˆ s, HasFDerivAt (f n) (f' n x) x) (hf' : โˆ€ (n : ฮฑ), โˆ€ x โˆˆ s, โ€–f' n xโ€– โ‰ค u n) (hxโ‚€ : xโ‚€ โˆˆ s) (hf0 : Summable fun (n : ฮฑ) => f n xโ‚€) (hx : x โˆˆ s) :
HasFDerivAt (fun (y : E) => โˆ‘' (n : ฮฑ), f n y) (โˆ‘' (n : ฮฑ), f' n x) x

Consider a series of functions โˆ‘' n, f n x on a preconnected open set. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series is differentiable on the set and its derivative is the sum of the derivatives.

theorem hasDerivAt_tsum_of_isPreconnected {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {g' : ฮฑ โ†’ ๐•œ โ†’ F} {t : Set ๐•œ} {yโ‚€ : ๐•œ} {y : ๐•œ} (hu : Summable u) (ht : IsOpen t) (h't : IsPreconnected t) (hg : โˆ€ (n : ฮฑ), โˆ€ y โˆˆ t, HasDerivAt (g n) (g' n y) y) (hg' : โˆ€ (n : ฮฑ), โˆ€ y โˆˆ t, โ€–g' n yโ€– โ‰ค u n) (hyโ‚€ : yโ‚€ โˆˆ t) (hg0 : Summable fun (n : ฮฑ) => g n yโ‚€) (hy : y โˆˆ t) :
HasDerivAt (fun (z : ๐•œ) => โˆ‘' (n : ฮฑ), g n z) (โˆ‘' (n : ฮฑ), g' n y) y

Consider a series of functions โˆ‘' n, f n x on a preconnected open set. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series is differentiable on the set and its derivative is the sum of the derivatives.

theorem summable_of_summable_hasFDerivAt {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {f' : ฮฑ โ†’ E โ†’ E โ†’L[๐•œ] F} {xโ‚€ : E} (hu : Summable u) (hf : โˆ€ (n : ฮฑ) (x : E), HasFDerivAt (f n) (f' n x) x) (hf' : โˆ€ (n : ฮฑ) (x : E), โ€–f' n xโ€– โ‰ค u n) (hf0 : Summable fun (n : ฮฑ) => f n xโ‚€) (x : E) :
Summable fun (n : ฮฑ) => f n x

Consider a series of functions โˆ‘' n, f n x. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series converges everywhere.

theorem summable_of_summable_hasDerivAt {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {g' : ฮฑ โ†’ ๐•œ โ†’ F} {yโ‚€ : ๐•œ} (hu : Summable u) (hg : โˆ€ (n : ฮฑ) (y : ๐•œ), HasDerivAt (g n) (g' n y) y) (hg' : โˆ€ (n : ฮฑ) (y : ๐•œ), โ€–g' n yโ€– โ‰ค u n) (hg0 : Summable fun (n : ฮฑ) => g n yโ‚€) (y : ๐•œ) :
Summable fun (n : ฮฑ) => g n y

Consider a series of functions โˆ‘' n, f n x. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series converges everywhere.

theorem hasFDerivAt_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {f' : ฮฑ โ†’ E โ†’ E โ†’L[๐•œ] F} {xโ‚€ : E} (hu : Summable u) (hf : โˆ€ (n : ฮฑ) (x : E), HasFDerivAt (f n) (f' n x) x) (hf' : โˆ€ (n : ฮฑ) (x : E), โ€–f' n xโ€– โ‰ค u n) (hf0 : Summable fun (n : ฮฑ) => f n xโ‚€) (x : E) :
HasFDerivAt (fun (y : E) => โˆ‘' (n : ฮฑ), f n y) (โˆ‘' (n : ฮฑ), f' n x) x

Consider a series of functions โˆ‘' n, f n x. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series is differentiable and its derivative is the sum of the derivatives.

theorem hasDerivAt_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {g' : ฮฑ โ†’ ๐•œ โ†’ F} {yโ‚€ : ๐•œ} (hu : Summable u) (hg : โˆ€ (n : ฮฑ) (y : ๐•œ), HasDerivAt (g n) (g' n y) y) (hg' : โˆ€ (n : ฮฑ) (y : ๐•œ), โ€–g' n yโ€– โ‰ค u n) (hg0 : Summable fun (n : ฮฑ) => g n yโ‚€) (y : ๐•œ) :
HasDerivAt (fun (z : ๐•œ) => โˆ‘' (n : ฮฑ), g n z) (โˆ‘' (n : ฮฑ), g' n y) y

Consider a series of functions โˆ‘' n, f n x. If the series converges at a point, and all functions in the series are differentiable with a summable bound on the derivatives, then the series is differentiable and its derivative is the sum of the derivatives.

theorem differentiable_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {f' : ฮฑ โ†’ E โ†’ E โ†’L[๐•œ] F} (hu : Summable u) (hf : โˆ€ (n : ฮฑ) (x : E), HasFDerivAt (f n) (f' n x) x) (hf' : โˆ€ (n : ฮฑ) (x : E), โ€–f' n xโ€– โ‰ค u n) :
Differentiable ๐•œ fun (y : E) => โˆ‘' (n : ฮฑ), f n y

Consider a series of functions โˆ‘' n, f n x. If all functions in the series are differentiable with a summable bound on the derivatives, then the series is differentiable. Note that our assumptions do not ensure the pointwise convergence, but if there is no pointwise convergence then the series is zero everywhere so the result still holds.

theorem differentiable_tsum' {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {g' : ฮฑ โ†’ ๐•œ โ†’ F} (hu : Summable u) (hg : โˆ€ (n : ฮฑ) (y : ๐•œ), HasDerivAt (g n) (g' n y) y) (hg' : โˆ€ (n : ฮฑ) (y : ๐•œ), โ€–g' n yโ€– โ‰ค u n) :
Differentiable ๐•œ fun (z : ๐•œ) => โˆ‘' (n : ฮฑ), g n z

Consider a series of functions โˆ‘' n, f n x. If all functions in the series are differentiable with a summable bound on the derivatives, then the series is differentiable. Note that our assumptions do not ensure the pointwise convergence, but if there is no pointwise convergence then the series is zero everywhere so the result still holds.

theorem fderiv_tsum_apply {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {xโ‚€ : E} (hu : Summable u) (hf : โˆ€ (n : ฮฑ), Differentiable ๐•œ (f n)) (hf' : โˆ€ (n : ฮฑ) (x : E), โ€–fderiv ๐•œ (f n) xโ€– โ‰ค u n) (hf0 : Summable fun (n : ฮฑ) => f n xโ‚€) (x : E) :
fderiv ๐•œ (fun (y : E) => โˆ‘' (n : ฮฑ), f n y) x = โˆ‘' (n : ฮฑ), fderiv ๐•œ (f n) x
theorem deriv_tsum_apply {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {yโ‚€ : ๐•œ} (hu : Summable u) (hg : โˆ€ (n : ฮฑ), Differentiable ๐•œ (g n)) (hg' : โˆ€ (n : ฮฑ) (y : ๐•œ), โ€–deriv (g n) yโ€– โ‰ค u n) (hg0 : Summable fun (n : ฮฑ) => g n yโ‚€) (y : ๐•œ) :
deriv (fun (z : ๐•œ) => โˆ‘' (n : ฮฑ), g n z) y = โˆ‘' (n : ฮฑ), deriv (g n) y
theorem fderiv_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {xโ‚€ : E} (hu : Summable u) (hf : โˆ€ (n : ฮฑ), Differentiable ๐•œ (f n)) (hf' : โˆ€ (n : ฮฑ) (x : E), โ€–fderiv ๐•œ (f n) xโ€– โ‰ค u n) (hf0 : Summable fun (n : ฮฑ) => f n xโ‚€) :
(fderiv ๐•œ fun (y : E) => โˆ‘' (n : ฮฑ), f n y) = fun (x : E) => โˆ‘' (n : ฮฑ), fderiv ๐•œ (f n) x
theorem deriv_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup F] [CompleteSpace F] {u : ฮฑ โ†’ โ„} [NormedSpace ๐•œ F] {g : ฮฑ โ†’ ๐•œ โ†’ F} {yโ‚€ : ๐•œ} (hu : Summable u) (hg : โˆ€ (n : ฮฑ), Differentiable ๐•œ (g n)) (hg' : โˆ€ (n : ฮฑ) (y : ๐•œ), โ€–deriv (g n) yโ€– โ‰ค u n) (hg0 : Summable fun (n : ฮฑ) => g n yโ‚€) :
(deriv fun (y : ๐•œ) => โˆ‘' (n : ฮฑ), g n y) = fun (y : ๐•œ) => โˆ‘' (n : ฮฑ), deriv (g n) y

Higher smoothness #

theorem iteratedFDeriv_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {v : โ„• โ†’ ฮฑ โ†’ โ„} {N : โ„•โˆž} (hf : โˆ€ (i : ฮฑ), ContDiff ๐•œ N (f i)) (hv : โˆ€ (k : โ„•), โ†‘k โ‰ค N โ†’ Summable (v k)) (h'f : โˆ€ (k : โ„•) (i : ฮฑ) (x : E), โ†‘k โ‰ค N โ†’ โ€–iteratedFDeriv ๐•œ k (f i) xโ€– โ‰ค v k i) {k : โ„•} (hk : โ†‘k โ‰ค N) :
(iteratedFDeriv ๐•œ k fun (y : E) => โˆ‘' (n : ฮฑ), f n y) = fun (x : E) => โˆ‘' (n : ฮฑ), iteratedFDeriv ๐•œ k (f n) x

Consider a series of smooth functions, with summable uniform bounds on the successive derivatives. Then the iterated derivative of the sum is the sum of the iterated derivative.

theorem iteratedFDeriv_tsum_apply {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {v : โ„• โ†’ ฮฑ โ†’ โ„} {N : โ„•โˆž} (hf : โˆ€ (i : ฮฑ), ContDiff ๐•œ N (f i)) (hv : โˆ€ (k : โ„•), โ†‘k โ‰ค N โ†’ Summable (v k)) (h'f : โˆ€ (k : โ„•) (i : ฮฑ) (x : E), โ†‘k โ‰ค N โ†’ โ€–iteratedFDeriv ๐•œ k (f i) xโ€– โ‰ค v k i) {k : โ„•} (hk : โ†‘k โ‰ค N) (x : E) :
iteratedFDeriv ๐•œ k (fun (y : E) => โˆ‘' (n : ฮฑ), f n y) x = โˆ‘' (n : ฮฑ), iteratedFDeriv ๐•œ k (f n) x

Consider a series of smooth functions, with summable uniform bounds on the successive derivatives. Then the iterated derivative of the sum is the sum of the iterated derivative.

theorem contDiff_tsum {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {v : โ„• โ†’ ฮฑ โ†’ โ„} {N : โ„•โˆž} (hf : โˆ€ (i : ฮฑ), ContDiff ๐•œ N (f i)) (hv : โˆ€ (k : โ„•), โ†‘k โ‰ค N โ†’ Summable (v k)) (h'f : โˆ€ (k : โ„•) (i : ฮฑ) (x : E), โ†‘k โ‰ค N โ†’ โ€–iteratedFDeriv ๐•œ k (f i) xโ€– โ‰ค v k i) :
ContDiff ๐•œ N fun (x : E) => โˆ‘' (i : ฮฑ), f i x

Consider a series of functions โˆ‘' i, f i x. Assume that each individual function f i is of class C^N, and moreover there is a uniform summable upper bound on the k-th derivative for each k โ‰ค N. Then the series is also C^N.

theorem contDiff_tsum_of_eventually {ฮฑ : Type u_1} {๐•œ : Type u_3} {E : Type u_4} {F : Type u_5} [RCLike ๐•œ] [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [CompleteSpace F] [NormedSpace ๐•œ F] {f : ฮฑ โ†’ E โ†’ F} {v : โ„• โ†’ ฮฑ โ†’ โ„} {N : โ„•โˆž} (hf : โˆ€ (i : ฮฑ), ContDiff ๐•œ N (f i)) (hv : โˆ€ (k : โ„•), โ†‘k โ‰ค N โ†’ Summable (v k)) (h'f : โˆ€ (k : โ„•), โ†‘k โ‰ค N โ†’ โˆ€แถ  (i : ฮฑ) in Filter.cofinite, โˆ€ (x : E), โ€–iteratedFDeriv ๐•œ k (f i) xโ€– โ‰ค v k i) :
ContDiff ๐•œ N fun (x : E) => โˆ‘' (i : ฮฑ), f i x

Consider a series of functions โˆ‘' i, f i x. Assume that each individual function f i is of class C^N, and moreover there is a uniform summable upper bound on the k-th derivative for each k โ‰ค N (except maybe for finitely many is). Then the series is also C^N.