Finite dimensional topological vector spaces over complete fields #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Let π
be a complete nontrivially normed field, and E
a topological vector space (TVS) over
π
(i.e we have [add_comm_group E] [module π E] [topological_space E] [topological_add_group E]
and [has_continuous_smul π E]
).
If E
is finite dimensional and Hausdorff, then all linear maps from E
to any other TVS are
continuous.
When E
is a normed space, this gets us the equivalence of norms in finite dimension.
Main results : #
linear_map.continuous_iff_is_closed_ker
: a linear form is continuous if and only if its kernel is closed.linear_map.continuous_of_finite_dimensional
: a linear map on a finite-dimensional Hausdorff space over a complete field is continuous.
TODO #
Generalize more of analysis/normed_space/finite_dimension
to general TVSs.
Implementation detail #
The main result from which everything follows is the fact that, if ΞΎ : ΞΉ β E
is a finite basis,
then ΞΎ.equiv_fun : E ββ (ΞΉ β π)
is continuous. However, for technical reasons, it is easier to
prove this when ΞΉ
and E
live ine the same universe. So we start by doing that as a private
lemma, then we deduce linear_map.continuous_of_finite_dimensional
from it, and then the general
result follows as continuous_equiv_fun_basis
.
The space of continuous linear maps between finite-dimensional spaces is finite-dimensional.
If π
is a nontrivially normed field, any T2 topology on π
which makes it a topological
vector space over itself (with the norm topology) is equal to the norm topology.
Any linear form on a topological vector space over a nontrivially normed field is continuous if its kernel is closed.
Any linear form on a topological vector space over a nontrivially normed field is continuous if and only if its kernel is closed.
Over a nontrivially normed field, any linear form which is nonzero on a nonempty open set is automatically continuous.
Any linear map on a finite dimensional space over a complete field is continuous.
Equations
In finite dimensions over a non-discrete complete normed field, the canonical identification
(in terms of a basis) with π^n
(endowed with the product topology) is continuous.
This is the key fact wich makes all linear maps from a T2 finite dimensional TVS over such a field
continuous (see linear_map.continuous_of_finite_dimensional
), which in turn implies that all
norms are equivalent in finite dimensions.
The continuous linear map induced by a linear map on a finite dimensional space
A surjective linear map f
with finite dimensional codomain is an open map.
Equations
The continuous linear equivalence induced by a linear equivalence on a finite dimensional space.
Equations
- e.to_continuous_linear_equiv = {to_linear_equiv := {to_fun := e.to_fun, map_add' := _, map_smul' := _, inv_fun := e.inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Equations
Two finite-dimensional topological vector spaces over a complete normed field are continuously linearly equivalent if they have the same (finite) dimension.
Two finite-dimensional topological vector spaces over a complete normed field are continuously linearly equivalent if and only if they have the same (finite) dimension.
A continuous linear equivalence between two finite-dimensional topological vector spaces over a complete normed field of the same (finite) dimension.
Equations
Construct a continuous linear map given the value at a finite basis.
The continuous linear equivalence between a vector space over π
with a finite basis and
functions from its basis indexing type to π
.
Equations
- v.equiv_funL = {to_linear_equiv := {to_fun := v.equiv_fun.to_fun, map_add' := _, map_smul' := _, inv_fun := v.equiv_fun.inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Builds a continuous linear equivalence from a continuous linear map on a finite-dimensional vector space whose determinant is nonzero.