Finite dimensional normed spaces over complete fields #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Over a complete nontrivially normed field, in finite dimension, all norms are equivalent and all linear maps are continuous. Moreover, a finite-dimensional subspace is always complete and closed.
Main results: #
finite_dimensional.complete
: a finite-dimensional space over a complete field is complete. This is not registered as an instance, as the field would be an unknown metavariable in typeclass resolution.submodule.closed_of_finite_dimensional
: a finite-dimensional subspace over a complete field is closedfinite_dimensional.proper
: a finite-dimensional space over a proper field is proper. This is not registered as an instance, as the field would be an unknown metavariable in typeclass resolution. It is however registered as an instance for𝕜 = ℝ
and𝕜 = ℂ
. As properness implies completeness, there is no need to also registerfinite_dimensional.complete
onℝ
orℂ
.finite_dimensional_of_is_compact_closed_ball
: Riesz' theorem: if the closed unit ball is compact, then the space is finite-dimensional.
Implementation notes #
The fact that all norms are equivalent is not written explicitly, as it would mean having two norms
on a single space, which is not the way type classes work. However, if one has a
finite-dimensional vector space E
with a norm, and a copy E'
of this type with another norm,
then the identities from E
to E'
and from E'
to E
are continuous thanks to
linear_map.continuous_of_finite_dimensional
. This gives the desired norm equivalence.
A linear isometry between finite dimensional spaces of equal dimension can be upgraded to a linear isometry equivalence.
Equations
- li.to_linear_isometry_equiv h = {to_linear_equiv := li.to_linear_map.linear_equiv_of_injective _ h, norm_map' := _}
An affine isometry between finite dimensional spaces of equal dimension can be upgraded to an affine isometry equivalence.
Equations
- li.to_affine_isometry_equiv h = affine_isometry_equiv.mk' ⇑li (li.linear_isometry.to_linear_isometry_equiv h) (arbitrary P₁) _
Reinterpret an affine equivalence as a homeomorphism.
Equations
- f.to_homeomorph_of_finite_dimensional = {to_equiv := f.to_equiv, continuous_to_fun := _, continuous_inv_fun := _}
Any K
-Lipschitz map from a subset s
of a metric space α
to a finite-dimensional real
vector space E'
can be extended to a Lipschitz map on the whole space α
, with a slightly worse
constant C * K
where C
only depends on E'
. We record a working value for this constant C
as lipschitz_extension_constant E'
.
Equations
- lipschitz_extension_constant E' = let A : E' ≃L[ℝ] ↥(basis.of_vector_space_index ℝ E') → ℝ := (basis.of_vector_space ℝ E').equiv_fun.to_continuous_linear_equiv in linear_order.max (‖A.symm.to_continuous_linear_map‖₊ * ‖A.to_continuous_linear_map‖₊) 1
Any K
-Lipschitz map from a subset s
of a metric space α
to a finite-dimensional real
vector space E'
can be extended to a Lipschitz map on the whole space α
, with a slightly worse
constant lipschitz_extension_constant E' * K
.
A weaker version of basis.op_nnnorm_le
that abstracts away the value of C
.
A weaker version of basis.op_norm_le
that abstracts away the value of C
.
A finite-dimensional subspace is complete.
A finite-dimensional subspace is closed.
In an infinite dimensional space, given a finite number of points, one may find a point
with norm at most R
which is at distance at least 1
of all these points.
In an infinite-dimensional normed space, there exists a sequence of points which are all
bounded by R
and at distance at least 1
. For a version not assuming c
and R
, see
exists_seq_norm_le_one_le_norm_sub
.
Riesz's theorem: if a closed ball with center zero of positive radius is compact in a vector space, then the space is finite-dimensional.
Riesz's theorem: if a closed ball of positive radius is compact in a vector space, then the space is finite-dimensional.
If a function has compact support, then either the function is trivial or the space if finite-dimensional.
If a function has compact multiplicative support, then either the function is trivial or the space if finite-dimensional.
An injective linear map with finite-dimensional domain is a closed embedding.
Continuous linear equivalence between continuous linear functions 𝕜ⁿ → E
and Eⁿ
.
The spaces 𝕜ⁿ
and Eⁿ
are represented as ι → 𝕜
and ι → E
, respectively,
where ι
is a finite type.
Equations
- continuous_linear_equiv.pi_ring ι = {to_linear_equiv := {to_fun := (linear_map.to_continuous_linear_map.symm.trans (linear_equiv.pi_ring 𝕜 E ι 𝕜)).to_fun, map_add' := _, map_smul' := _, inv_fun := (linear_map.to_continuous_linear_map.symm.trans (linear_equiv.pi_ring 𝕜 E ι 𝕜)).inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
A family of continuous linear maps is continuous on s
if all its applications are.
Any finite-dimensional vector space over a proper field is proper.
We do not register this as an instance to avoid an instance loop when trying to prove the
properness of 𝕜
, and the search for 𝕜
as an unknown metavariable. Declare the instance
explicitly when needed.
If E
is a finite dimensional normed real vector space, x : E
, and s
is a neighborhood of
x
that is not equal to the whole space, then there exists a point y ∈ frontier s
at distance
metric.inf_dist x sᶜ
from x
. See also
is_compact.exists_mem_frontier_inf_dist_compl_eq_dist
.
If K
is a compact set in a nontrivial real normed space and x ∈ K
, then there exists a point
y
of the boundary of K
at distance metric.inf_dist x Kᶜ
from x
. See also
exists_mem_frontier_inf_dist_compl_eq_dist
.
In a finite dimensional vector space over ℝ
, the series ∑ x, ‖f x‖
is unconditionally
summable if and only if the series ∑ x, f x
is unconditionally summable. One implication holds in
any complete normed space, while the other holds only in finite dimensional spaces.