Documentation

Mathlib.Analysis.Complex.LocallyUniformLimit

Locally uniform limits of holomorphic functions #

This file gathers some results about locally uniform limits of holomorphic functions on an open subset of the complex plane.

Main results #

noncomputable def Complex.cderiv {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] (r : ) (f : E) (z : ) :
E

A circle integral which coincides with deriv f z whenever one can apply the Cauchy formula for the derivative. It is useful in the proof that locally uniform limits of holomorphic functions are holomorphic, because it depends continuously on f for the uniform topology.

Equations
Instances For
    theorem Complex.cderiv_eq_deriv {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {z : } {r : } {f : E} (hU : IsOpen U) (hf : DifferentiableOn f U) (hr : 0 < r) (hzr : Metric.closedBall z r U) :
    theorem Complex.norm_cderiv_le {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {z : } {M : } {r : } {f : E} (hr : 0 < r) (hf : wMetric.sphere z r, f w M) :
    theorem Complex.cderiv_sub {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {z : } {r : } {f : E} {g : E} (hr : 0 < r) (hf : ContinuousOn f (Metric.sphere z r)) (hg : ContinuousOn g (Metric.sphere z r)) :
    theorem Complex.norm_cderiv_lt {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {z : } {M : } {r : } {f : E} (hr : 0 < r) (hfM : wMetric.sphere z r, f w < M) (hf : ContinuousOn f (Metric.sphere z r)) :
    theorem Complex.norm_cderiv_sub_lt {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {z : } {M : } {r : } {f : E} {g : E} (hr : 0 < r) (hfg : wMetric.sphere z r, f w - g w < M) (hf : ContinuousOn f (Metric.sphere z r)) (hg : ContinuousOn g (Metric.sphere z r)) :
    theorem TendstoUniformlyOn.cderiv {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] {K : Set } {δ : } {φ : Filter ι} {F : ιE} {f : E} (hF : TendstoUniformlyOn F f φ (Metric.cthickening δ K)) (hδ : 0 < δ) (hFn : ∀ᶠ (n : ι) in φ, ContinuousOn (F n) (Metric.cthickening δ K)) :
    theorem Complex.tendstoUniformlyOn_deriv_of_cthickening_subset {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {K : Set } {φ : Filter ι} {F : ιE} {f : E} (hf : TendstoLocallyUniformlyOn F f φ U) (hF : ∀ᶠ (n : ι) in φ, DifferentiableOn (F n) U) {δ : } (hδ : 0 < δ) (hK : IsCompact K) (hU : IsOpen U) (hKU : Metric.cthickening δ K U) :
    TendstoUniformlyOn (deriv F) (Complex.cderiv δ f) φ K
    theorem Complex.exists_cthickening_tendstoUniformlyOn {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {K : Set } {φ : Filter ι} {F : ιE} {f : E} (hf : TendstoLocallyUniformlyOn F f φ U) (hF : ∀ᶠ (n : ι) in φ, DifferentiableOn (F n) U) (hK : IsCompact K) (hU : IsOpen U) (hKU : K U) :
    δ > 0, Metric.cthickening δ K U TendstoUniformlyOn (deriv F) (Complex.cderiv δ f) φ K
    theorem TendstoLocallyUniformlyOn.differentiableOn {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {φ : Filter ι} {F : ιE} {f : E} [φ.NeBot] (hf : TendstoLocallyUniformlyOn F f φ U) (hF : ∀ᶠ (n : ι) in φ, DifferentiableOn (F n) U) (hU : IsOpen U) :

    A locally uniform limit of holomorphic functions on an open domain of the complex plane is holomorphic (the derivatives converge locally uniformly to that of the limit, which is proved as TendstoLocallyUniformlyOn.deriv).

    theorem TendstoLocallyUniformlyOn.deriv {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {φ : Filter ι} {F : ιE} {f : E} (hf : TendstoLocallyUniformlyOn F f φ U) (hF : ∀ᶠ (n : ι) in φ, DifferentiableOn (F n) U) (hU : IsOpen U) :
    theorem Complex.differentiableOn_tsum_of_summable_norm {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {F : ιE} {u : ι} (hu : Summable u) (hf : ∀ (i : ι), DifferentiableOn (F i) U) (hU : IsOpen U) (hF_le : ∀ (i : ι), wU, F i w u i) :
    DifferentiableOn (fun (w : ) => ∑' (i : ι), F i w) U

    If the terms in the sum ∑' (i : ι), F i are uniformly bounded on U by a summable function, and each term in the sum is differentiable on U, then so is the sum.

    theorem Complex.hasSum_deriv_of_summable_norm {E : Type u_1} {ι : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {U : Set } {z : } {F : ιE} {u : ι} (hu : Summable u) (hf : ∀ (i : ι), DifferentiableOn (F i) U) (hU : IsOpen U) (hF_le : ∀ (i : ι), wU, F i w u i) (hz : z U) :
    HasSum (fun (i : ι) => deriv (F i) z) (deriv (fun (w : ) => ∑' (i : ι), F i w) z)

    If the terms in the sum ∑' (i : ι), F i are uniformly bounded on U by a summable function, then the sum of deriv F i at a point in U is the derivative of the sum.