Primitives of Holomorphic Functions #
In this file, we give conditions under which holomorphic functions have primitives. The main goal
is to prove that holomorphic functions on simply connected domains have primitives. As a first step,
we prove that holomorphic functions on disks have primitives. The approach is based on Morera's
theorem, that a continuous function (on a disk) whose integral round a rectangle vanishes on all
rectangles contained in the disk has a primitive. (Coupled with the fact that holomorphic functions
satisfy this property.) To prove Morera's theorem, we first define the Complex.wedgeIntegral
,
which is the integral of a function over a "wedge" (a horizontal segment followed by a vertical
segment in the disk), and compute its derivative.
Main results #
Complex.IsConservativeOn.isExactOn_ball
: Morera's Theorem: On a disk, a continuous function whose integrals on rectangles vanish, has primitives.DifferentiableOn.isExactOn_ball
: On a disk, a holomorphic function has primitives.
TODO: Extend to holomorphic functions on simply connected domains.
The (z, w)
-wedge-integral of f
, is the integral of f
over two sides of the rectangle
determined by z
and w
.
Equations
Instances For
A function f
IsConservativeOn
in U
if, for any rectangle contained in U
the integral of f
over the rectangle is zero.
Equations
- Complex.IsConservativeOn f U = ∀ (z w : ℂ), z.Rectangle w ⊆ U → z.wedgeIntegral w f = -w.wedgeIntegral z f
Instances For
A function f
IsExactOn
in U
if it is the complex derivative of a function on U
.
In complex variable theory, this is also referred to as "having a primitive".
Equations
- Complex.IsExactOn f U = ∃ (g : ℂ → E), ∀ z ∈ U, HasDerivAt g (f z) z
Instances For
If a function f
IsConservativeOn
on a disk of center c
, then for points z
in this disk,
the wedge integral from c
to z
is additive under a detour through a nearby point w
.
The wedgeIntegral
has derivative at z
equal to f z
.
Morera's theorem for a disk On a disk, a continuous function whose integrals on rectangles vanish, has primitives.
Morera's theorem for a disk On a disk, a holomorphic function has primitives.