L²
inner product space structure on finite products of inner product spaces #
The L²
norm on a finite product of inner product spaces is compatible with an inner product
$$
\langle x, y\rangle = \sum \langle x_i, y_i \rangle.
$$
This is recorded in this file as an inner product space instance on pi_Lp 2
.
Main definitions #
-
euclidean_space 𝕜 n
: defined to bepi_Lp 2 (n → 𝕜)
for anyfintype n
, i.e., the space from functions ton
to𝕜
with theL²
norm. We register several instances on it (notably that it is a finite-dimensional inner product space). -
basis.isometry_euclidean_of_orthonormal
: provides the isometry to Euclidean space from a given finite-dimensional inner product space, induced by a basis of the space. -
linear_isometry_equiv.of_inner_product_space
: provides an arbitrary isometry to Euclidean space from a given finite-dimensional inner product space, induced by choosing an arbitrary basis. -
complex.isometry_euclidean
: standard isometry fromℂ
toeuclidean_space ℝ (fin 2)
Equations
- pi_Lp.inner_product_space f = {to_normed_group := pi_Lp.normed_group 2 f (λ (i : ι), inner_product_space.to_normed_group 𝕜), to_normed_space := pi_Lp.normed_space 2 f 𝕜 (λ (i : ι), inner_product_space.to_normed_space), to_has_inner := {inner := λ (x y : pi_Lp 2 f), ∑ (i : ι), inner (x i) (y i)}, norm_sq_eq_inner := _, conj_sym := _, add_left := _, smul_left := _}
The standard real/complex Euclidean space, functions on a finite type. For an n
-dimensional
space use euclidean_space 𝕜 (fin n)
.
Equations
- euclidean_space 𝕜 n = pi_Lp 2 (λ (i : n), 𝕜)
Equations
- euclidean_space.inner_product_space = pi_Lp.inner_product_space (λ (i : ι), 𝕜)
A finite, mutually orthogonal family of subspaces of E
, which span E
, induce an isometry
from E
to pi_Lp 2
of the subspaces equipped with the L2
inner product.
Equations
- hV.isometry_L2_of_orthogonal_family hV' = let e₁ : (⨁ (i : ι), (λ (i : ι), ↥(V i)) i) ≃ₗ[𝕜] Π (i : ι), (λ (i : ι), ↥(V i)) i := direct_sum.linear_equiv_fun_on_fintype 𝕜 ι (λ (i : ι), ↥(V i)), e₂ : (⨁ (i : ι), ↥(V i)) ≃ₗ[𝕜] E := linear_equiv.of_bijective (direct_sum.submodule_coe V) _ _ in (e₂.symm.trans e₁).isometry_of_inner _
An orthonormal basis on a fintype ι
for an inner product space induces an isometry with
euclidean_space 𝕜 ι
.
Equations
If f : E ≃ₗᵢ[𝕜] E'
is a linear isometry of inner product spaces then an orthonormal basis v
of E
determines a linear isometry e : E' ≃ₗᵢ[𝕜] euclidean_space 𝕜 ι
. This result states that
e
may be obtained either by transporting v
to E'
or by composing with the linear isometry
E ≃ₗᵢ[𝕜] euclidean_space 𝕜 ι
provided by v
.
ℂ
is isometric to ℝ²
with the Euclidean inner product.
Equations
- complex.isometry_euclidean = complex.basis_one_I.isometry_euclidean_of_orthonormal complex.isometry_euclidean._proof_1
Given a natural number n
equal to the finrank
of a finite-dimensional inner product space,
there exists an isometry from the space to euclidean_space 𝕜 (fin n)
.
Given a natural number n
one less than the finrank
of a finite-dimensional inner product
space, there exists an isometry from the orthogonal complement of a nonzero singleton to
euclidean_space 𝕜 (fin n)
.