mathlib documentation

analysis.complex.removable_singularity

Removable singularity theorem #

In this file we prove Riemann's removable singularity theorem: if f : ℂ → E is complex differentiable in a punctured neighborhood of a point c and is bounded in a punctured neighborhood of c (or, more generally, $f(z) - f(c)=o((z-c)^{-1})$), then it has a limit at c and the function function.update f c (lim (𝓝[≠] c) f) is complex differentiable in a neighborhood of c.

Removable singularity theorem, weak version. If f : ℂ → E is differentiable in a punctured neighborhood of a point and is continuous at this point, then it is analytic at this point.

theorem complex.differentiable_on_update_lim_of_is_o {E : Type u} [normed_group E] [normed_space E] [measurable_space E] [borel_space E] [topological_space.second_countable_topology E] [complete_space E] {f : → E} {s : set } {c : } (hc : s 𝓝 c) (hd : differentiable_on f (s \ {c})) (ho : asymptotics.is_o (λ (z : ), f z - f c) (λ (z : ), (z - c)⁻¹) (𝓝[{c}] c)) :

Removable singularity theorem: if s is a neighborhood of c : ℂ, a function f : ℂ → E is complex differentiable on s \ {c}, and $f(z) - f(c)=o((z-c)^{-1})$, then f redefined to be equal to lim (𝓝[≠] c) f at c is complex differentiable on s.

theorem complex.differentiable_on_update_lim_insert_of_is_o {E : Type u} [normed_group E] [normed_space E] [measurable_space E] [borel_space E] [topological_space.second_countable_topology E] [complete_space E] {f : → E} {s : set } {c : } (hc : s 𝓝[{c}] c) (hd : differentiable_on f s) (ho : asymptotics.is_o (λ (z : ), f z - f c) (λ (z : ), (z - c)⁻¹) (𝓝[{c}] c)) :

Removable singularity theorem: if s is a punctured neighborhood of c : ℂ, a function f : ℂ → E is complex differentiable on s, and $f(z) - f(c)=o((z-c)^{-1})$, then f redefined to be equal to lim (𝓝[≠] c) f at c is complex differentiable on {c} ∪ s.

Removable singularity theorem: if s is a neighborhood of c : ℂ, a function f : ℂ → E is complex differentiable and is bounded on s \ {c}, then f redefined to be equal to lim (𝓝[≠] c) f at c is complex differentiable on s.

theorem complex.tendsto_lim_of_differentiable_on_punctured_nhds_of_is_o {E : Type u} [normed_group E] [normed_space E] [measurable_space E] [borel_space E] [topological_space.second_countable_topology E] [complete_space E] {f : → E} {c : } (hd : ∀ᶠ (z : ) in 𝓝[{c}] c, differentiable_at f z) (ho : asymptotics.is_o (λ (z : ), f z - f c) (λ (z : ), (z - c)⁻¹) (𝓝[{c}] c)) :
filter.tendsto f (𝓝[{c}] c) (𝓝 (lim (𝓝[{c}] c) f))

Removable singularity theorem: if a function f : ℂ → E is complex differentiable on a punctured neighborhood of c and $f(z) - f(c)=o((z-c)^{-1})$, then f has a limit at c.

Removable singularity theorem: if a function f : ℂ → E is complex differentiable and bounded on a punctured neighborhood of c, then f has a limit at c.