mathlib3 documentation

analysis.complex.abs_max

Maximum modulus principle #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

In this file we prove several versions of the maximum modulus principle. There are several statements that can be called "the maximum modulus principle" for maps between normed complex spaces. They differ by assumptions on the domain (any space, a nontrivial space, a finite dimensional space), assumptions on the codomain (any space, a strictly convex space), and by conclusion (either equality of norms or of the values of the function).

Main results #

Theorems for any codomain #

Consider a function f : E → F that is complex differentiable on a set s, is continuous on its closure, and ‖f x‖ has a maximum on s at c. We prove the following theorems.

Theorems for a strictly convex codomain #

If the codomain F is a strictly convex space, then in the lemmas from the previous section we can prove f w = f c instead of ‖f w‖ = ‖f c‖, see complex.eq_on_of_is_preconnected_of_is_max_on_norm, complex.eq_on_closure_of_is_preconnected_of_is_max_on_norm, complex.eq_of_is_max_on_of_ball_subset, complex.eq_on_closed_ball_of_is_max_on_norm, and complex.eventually_eq_of_is_local_max_norm.

Values on the frontier #

Finally, we prove some corollaries that relate the (norm of the) values of a function on a set to its values on the frontier of the set. All these lemmas assume that E is a nontrivial space. In this section f g : E → F are functions that are complex differentiable on a bounded set s and are continuous on its closure. We prove the following theorems.

Tags #

maximum modulus principle, complex analysis

Auxiliary lemmas #

We split the proof into a series of lemmas. First we prove the principle for a function f : ℂ → F with an additional assumption that F is a complete space, then drop unneeded assumptions one by one.

The lemmas with names *_auxₙ are considered to be private and should not be used outside of this file.

Now we drop the assumption complete_space F by embedding F into its completion.

Then we replace the assumption is_max_on (norm ∘ f) (closed_ball z r) z with a seemingly weaker assumption is_max_on (norm ∘ f) (ball z r) z.

theorem complex.norm_max_aux₃ {F : Type v} [normed_add_comm_group F] [normed_space F] {f : F} {z w : } {r : } (hr : has_dist.dist w z = r) (hd : diff_cont_on_cl f (metric.ball z r)) (hz : is_max_on (has_norm.norm f) (metric.ball z r) z) :

Maximum modulus principle for any codomain #

If we do not assume that the codomain is a strictly convex space, then we can only claim that the norm ‖f x‖ is locally constant.

Finally, we generalize the theorem from a disk in to a closed ball in any normed space.

Maximum modulus principle on a closed ball: if f : E → F is continuous on a closed ball, is complex differentiable on the corresponding open ball, and the norm ‖f w‖ takes its maximum value on the open ball at its center, then the norm ‖f w‖ is constant on the closed ball.

theorem complex.norm_eq_norm_of_is_max_on_of_ball_subset {E : Type u} [normed_add_comm_group E] [normed_space E] {F : Type v} [normed_add_comm_group F] [normed_space F] {f : E F} {s : set E} {z w : E} (hd : diff_cont_on_cl f s) (hz : is_max_on (has_norm.norm f) s z) (hsub : metric.ball z (has_dist.dist w z) s) :

Maximum modulus principle: if f : E → F is complex differentiable on a set s, the norm of f takes it maximum on s at z, and w is a point such that the closed ball with center z and radius dist w z is included in s, then ‖f w‖ = ‖f z‖.

Maximum modulus principle: if f : E → F is complex differentiable in a neighborhood of c and the norm ‖f z‖ has a local maximum at c, then ‖f z‖ is locally constant in a neighborhood of c.

Maximum modulus principle on a connected set. Let U be a (pre)connected open set in a complex normed space. Let f : E → F be a function that is complex differentiable on U. Suppose that ‖f x‖ takes its maximum value on U at c ∈ U. Then ‖f x‖ = ‖f c‖ for all x ∈ U.

Maximum modulus principle on a connected set. Let U be a (pre)connected open set in a complex normed space. Let f : E → F be a function that is complex differentiable on U and is continuous on its closure. Suppose that ‖f x‖ takes its maximum value on U at c ∈ U. Then ‖f x‖ = ‖f c‖ for all x ∈ closure U.

The case of a strictly convex codomain #

If the codomain F is a strictly convex space, then we can claim equalities like f w = f z instead of ‖f w‖ = ‖f z‖.

Instead of repeating the proof starting with lemmas about integrals, we apply a corresponding lemma above twice: for f and for λ x, f x + f c. Then we have ‖f w‖ = ‖f z‖ and ‖f w + f z‖ = ‖f z + f z‖, thus ‖f w + f z‖ = ‖f w‖ + ‖f z‖. This is only possible if f w = f z, see eq_of_norm_eq_of_norm_add_eq.

Maximum modulus principle on a connected set. Let U be a (pre)connected open set in a complex normed space. Let f : E → F be a function that is complex differentiable on U. Suppose that ‖f x‖ takes its maximum value on U at c ∈ U. Then f x = f c for all x ∈ U.

TODO: change assumption from is_max_on to is_local_max.

Maximum modulus principle on a connected set. Let U be a (pre)connected open set in a complex normed space. Let f : E → F be a function that is complex differentiable on U and is continuous on its closure. Suppose that ‖f x‖ takes its maximum value on U at c ∈ U. Then f x = f c for all x ∈ closure U.

theorem complex.eq_of_is_max_on_of_ball_subset {E : Type u} [normed_add_comm_group E] [normed_space E] {F : Type v} [normed_add_comm_group F] [normed_space F] [strict_convex_space F] {f : E F} {s : set E} {z w : E} (hd : diff_cont_on_cl f s) (hz : is_max_on (has_norm.norm f) s z) (hsub : metric.ball z (has_dist.dist w z) s) :
f w = f z

Maximum modulus principle. Let f : E → F be a function between complex normed spaces. Suppose that the codomain F is a strictly convex space, f is complex differentiable on a set s, f is continuous on the closure of s, the norm of f takes it maximum on s at z, and w is a point such that the closed ball with center z and radius dist w z is included in s, then f w = f z.

Maximum modulus principle on a closed ball. Suppose that a function f : E → F from a normed complex space to a strictly convex normed complex space has the following properties:

  • it is continuous on a closed ball metric.closed_ball z r,
  • it is complex differentiable on the corresponding open ball;
  • the norm ‖f w‖ takes its maximum value on the open ball at its center.

Then f is a constant on the closed ball.

Maximum modulus principle: if f : E → F is complex differentiable in a neighborhood of c and the norm ‖f z‖ has a local maximum at c, then f is locally constant in a neighborhood of c.

theorem complex.eventually_eq_or_eq_zero_of_is_local_min_norm {E : Type u} [normed_add_comm_group E] [normed_space E] {f : E } {c : E} (hf : ∀ᶠ (z : E) in nhds c, differentiable_at f z) (hc : is_local_min (has_norm.norm f) c) :
(∀ᶠ (z : E) in nhds c, f z = f c) f c = 0

Maximum on a set vs maximum on its frontier #

In this section we prove corollaries of the maximum modulus principle that relate the values of a function on a set to its values on the frontier of this set.

Maximum modulus principle: if f : E → F is complex differentiable on a nonempty bounded set U and is continuous on its closure, then there exists a point z ∈ frontier U such that λ z, ‖f z‖ takes it maximum value on closure U at z.

theorem complex.norm_le_of_forall_mem_frontier_norm_le {E : Type u} [normed_add_comm_group E] [normed_space E] {F : Type v} [normed_add_comm_group F] [normed_space F] [nontrivial E] {f : E F} {U : set E} (hU : metric.bounded U) (hd : diff_cont_on_cl f U) {C : } (hC : (z : E), z frontier U f z C) {z : E} (hz : z closure U) :
f z C

Maximum modulus principle: if f : E → F is complex differentiable on a bounded set U and ‖f z‖ ≤ C for any z ∈ frontier U, then the same is true for any z ∈ closure U.

If two complex differentiable functions f g : E → F are equal on the boundary of a bounded set U, then they are equal on closure U.

theorem complex.eq_on_of_eq_on_frontier {E : Type u} [normed_add_comm_group E] [normed_space E] {F : Type v} [normed_add_comm_group F] [normed_space F] [nontrivial E] {f g : E F} {U : set E} (hU : metric.bounded U) (hf : diff_cont_on_cl f U) (hg : diff_cont_on_cl g U) (hfg : set.eq_on f g (frontier U)) :
set.eq_on f g U

If two complex differentiable functions f g : E → F are equal on the boundary of a bounded set U, then they are equal on U.