Inner product space derived from a norm #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines an inner_product_space
instance from a norm that respects the
parallellogram identity. The parallelogram identity is a way to express the inner product of x
and
y
in terms of the norms of x
, y
, x + y
, x - y
.
Main results #
inner_product_space.of_norm
: a normed space whose norm respects the parallellogram identity, can be seen as an inner product space.
Implementation notes #
We define inner_
$$\langle x, y \rangle := \frac{1}{4} (‖x + y‖^2 - ‖x - y‖^2 + i ‖ix + y‖ ^ 2 - i ‖ix - y‖^2)$$
and use the parallelogram identity
$$‖x + y‖^2 + ‖x - y‖^2 = 2 (‖x‖^2 + ‖y‖^2)$$
to prove it is an inner product, i.e., that it is conjugate-symmetric (inner_.conj_symm
) and
linear in the first argument. add_left
is proved by judicious application of the parallelogram
identity followed by tedious arithmetic. smul_left
is proved step by step, first noting that
$\langle λ x, y \rangle = λ \langle x, y \rangle$ for $λ ∈ ℕ$, $λ = -1$, hence $λ ∈ ℤ$ and $λ ∈ ℚ$
by arithmetic. Then by continuity and the fact that ℚ is dense in ℝ, the same is true for ℝ.
The case of ℂ then follows by applying the result for ℝ and more arithmetic.
TODO #
Move upstream to analysis.inner_product_space.basic
.
References #
- Jordan, P. and von Neumann, J., On inner products in linear, metric spaces
- https://math.stackexchange.com/questions/21792/norms-induced-by-inner-products-and-the-parallelogram-law
- https://math.dartmouth.edu/archive/m113w10/public_html/jordan-vneumann-thm.pdf
Tags #
inner product space, Hilbert space, norm
- parallelogram_identity : ∀ (x y : E), ‖x + y‖ * ‖x + y‖ + ‖x - y‖ * ‖x - y‖ = 2 * (‖x‖ * ‖x‖ + ‖y‖ * ‖y‖)
Predicate for the parallelogram identity to hold in a normed group. This is a scalar-less
version of inner_product_space
. If you have an inner_product_spaceable
assumption, you can
locally upgrade that to inner_product_space 𝕜 E
using casesI nonempty_inner_product_space 𝕜 E
.
Instances of this typeclass
Fréchet–von Neumann–Jordan Theorem. A normed space E
whose norm satisfies the
parallelogram identity can be given a compatible inner product.
Equations
- inner_product_space.of_norm 𝕜 h = {to_normed_space := _inst_3, to_has_inner := {inner := inner_ 𝕜 _inst_3}, norm_sq_eq_inner := _, conj_symm := _, add_left := _, smul_left := _}
Fréchet–von Neumann–Jordan Theorem. A normed space E
whose norm satisfies the
parallelogram identity can be given a compatible inner product. Do
casesI nonempty_inner_product_space 𝕜 E
to locally upgrade inner_product_spaceable E
to
inner_product_space 𝕜 E
.