Circle integral transform #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the circle integral transform of a function f with complex domain. This is
defined as $(2πi)^{-1}\frac{f(x)}{x-w}$ where x moves along a circle. We then prove some basic
facts about these functions.
These results are useful for proving that the uniform limit of a sequence of holomorphic functions is holomorphic.
Given a function f : ℂ → E, circle_transform R z w f is the functions mapping θ to
(2 * ↑π * I)⁻¹ • deriv (circle_map z R) θ • ((circle_map z R θ) - w)⁻¹ • f (circle_map z R θ).
If f is differentiable and w is in the interior of the ball, then the integral from 0 to
2 * π of this gives the value f(w).
Equations
- complex.circle_transform R z w f θ = (2 * ↑real.pi * complex.I)⁻¹ • deriv (circle_map z R) θ • (circle_map z R θ - w)⁻¹ • f (circle_map z R θ)
The derivative of circle_transform w.r.t w.
Equations
- complex.circle_transform_deriv R z w f θ = (2 * ↑real.pi * complex.I)⁻¹ • deriv (circle_map z R) θ • ((circle_map z R θ - w) ^ 2)⁻¹ • f (circle_map z R θ)
A useful bound for circle integrals (with complex codomain)
Equations
- complex.circle_transform_bounding_function R z w = complex.circle_transform_deriv R z w.fst (λ (x : ℂ), 1) w.snd
The derivative of a circle_transform is locally bounded.