Extension Hahn-Banach theorem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove the analytic Hahn-Banach theorem. For any continuous linear function on a subspace, we can extend it to a function on the entire space without changing its norm.
We prove
real.exists_extension_norm_eq
: Hahn-Banach theorem for continuous linear functions on normed spaces overℝ
.exists_extension_norm_eq
: Hahn-Banach theorem for continuous linear functions on normed spaces overℝ
orℂ
.
In order to state and prove the corollaries uniformly, we prove the statements for a field 𝕜
satisfying is_R_or_C 𝕜
.
In this setting, exists_dual_vector
states that, for any nonzero x
, there exists a continuous
linear form g
of norm 1
with g x = ‖x‖
(where the norm has to be interpreted as an element
of 𝕜
).
Hahn-Banach theorem for continuous linear functions over 𝕜
satisyfing is_R_or_C 𝕜
.
Corollary of Hahn-Banach. Given a nonzero element x
of a normed space, there exists an
element of the dual space, of norm 1
, whose value on x
is ‖x‖
.
Variant of Hahn-Banach, eliminating the hypothesis that x
be nonzero, and choosing
the dual element arbitrarily when x = 0
.
Variant of Hahn-Banach, eliminating the hypothesis that x
be nonzero, but only ensuring that
the dual element has norm at most 1
(this can not be improved for the trivial
vector space).