Properties of inner product spaces #
This file proves many basic properties of inner product spaces (real or complex).
Main results #
inner_mul_inner_self_le
: the Cauchy-Schwartz inequality (one of many variants).norm_inner_eq_norm_iff
: the equality criteion in the Cauchy-Schwartz inequality (also in many variants).inner_eq_sum_norm_sq_div_four
: the polarization identity.- We show that the inner product is continuous,
continuous_inner
, and bundle it as the continuous sesquilinear mapinnerSL
(see alsoinnerββ
for the non-continuous version).
Tags #
inner product space, Hilbert space, norm
See inner_smul_left
for the common special when π = π
.
Special case of inner_smul_left_eq_star_smul
when the acting ring has a trivial star
(eg β
, β€
, ββ₯0
, β
, β
).
See inner_smul_right
for the common special when π = π
.
See inner_smul_left_eq_star_smul
for the case of a general algebra action.
See inner_smul_right_eq_smul
for the case of a general algebra action.
The inner product as a sesquilinear form.
Note that in the case π = β
this is a bilinear form.
Equations
- sesqFormOfInner = LinearMap.mkβ'ββ (RingHom.id π) (starRingEnd π) (fun (x y : E) => inner y x) β― β― β― β―
Instances For
The real inner product as a bilinear form.
Note that unlike sesqFormOfInner
, this does not reverse the order of the arguments.
Equations
Instances For
An inner product with a sum on the left, Finsupp
version.
An inner product with a sum on the right, Finsupp
version.
CauchyβSchwarz inequality for real inner products.
A family of vectors is linearly independent if they are nonzero and orthogonal.
CauchyβSchwarz inequality with norm
CauchyβSchwarz inequality with norm
Polarization identity: The real part of the inner product, in terms of the norm.
Polarization identity: The real part of the inner product, in terms of the norm.
Polarization identity: The real part of the inner product, in terms of the norm.
Polarization identity: The imaginary part of the inner product, in terms of the norm.
Polarization identity: The inner product, in terms of the norm.
Polarization identity: The real inner product, in terms of the norm.
Polarization identity: The real inner product, in terms of the norm.
Pythagorean theorem, vector inner product form.
Pythagorean theorem, subtracting vectors, if-and-only-if vector inner product form.
Pythagorean theorem, subtracting vectors, if-and-if vector inner product form using square roots.
The real inner product of two vectors, divided by the product of their norms, has absolute value at most 1.
When an inner product space E
over π
is considered as a real normed space, its inner
product satisfies IsBoundedBilinearMap
.
In order to state these results, we need a NormedSpace β E
instance. We will later establish
such an instance by restriction-of-scalars, InnerProductSpace.rclikeToReal π E
, but this
instance may be not definitionally equal to some other βnaturalβ instance. So, we assume
[NormedSpace β E]
.
The inner product of two weighted sums, where the weights in each sum add to 0, in terms of the norms of pairwise differences.
Formula for the distance between the images of two nonzero points under an inversion with center
zero. See also EuclideanGeometry.dist_inversion_inversion
for inversions around a general
point.
The inner product of a nonzero vector with a nonzero multiple of itself, divided by the product of their norms, has absolute value
The inner product of a nonzero vector with a nonzero multiple of itself, divided by the product of their norms, has absolute value
The inner product of a nonzero vector with a positive multiple of itself, divided by the product of their norms, has value 1.
The inner product of a nonzero vector with a negative multiple of itself, divided by the product of their norms, has value -1.
If the inner product of two vectors is equal to the product of their norms, then the two vectors
are multiples of each other. One form of the equality case for Cauchy-Schwarz.
Compare inner_eq_norm_mul_iff
, which takes the stronger hypothesis βͺx, yβ« = βxβ * βyβ
.
The inner product of two vectors, divided by the product of their norms, has absolute value 1 if and only if they are nonzero and one is a multiple of the other. One form of equality case for Cauchy-Schwarz.
The inner product of two vectors, divided by the product of their norms, has absolute value 1 if and only if they are nonzero and one is a multiple of the other. One form of equality case for Cauchy-Schwarz.
If the inner product of two vectors is equal to the product of their norms (i.e.,
βͺx, yβ« = βxβ * βyβ
), then the two vectors are nonnegative real multiples of each other. One form
of the equality case for Cauchy-Schwarz.
Compare norm_inner_eq_norm_iff
, which takes the weaker hypothesis abs βͺx, yβ« = βxβ * βyβ
.
If the inner product of two vectors is equal to the product of their norms (i.e.,
βͺx, yβ« = βxβ * βyβ
), then the two vectors are nonnegative real multiples of each other. One form
of the equality case for Cauchy-Schwarz.
Compare norm_inner_eq_norm_iff
, which takes the weaker hypothesis abs βͺx, yβ« = βxβ * βyβ
.
The inner product of two vectors, divided by the product of their norms, has value 1 if and only if they are nonzero and one is a positive multiple of the other.
The inner product of two vectors, divided by the product of their norms, has value -1 if and only if they are nonzero and one is a negative multiple of the other.
If the inner product of two unit vectors is 1
, then the two vectors are equal. One form of
the equality case for Cauchy-Schwarz.
If the inner product of two unit vectors is strictly less than 1
, then the two vectors are
distinct. One form of the equality case for Cauchy-Schwarz.
The sphere of radius r = βyβ
is tangent to the plane βͺx, yβ« = βyβ ^ 2
at x = y
.
A field π
satisfying RCLike
is itself a π
-inner product space.
Equations
- RCLike.innerProductSpace = InnerProductSpace.mk β― β― β― β―
A general inner product implies a real inner product. This is not registered as an instance
since π
does not appear in the return type Inner β E
.
Equations
- Inner.rclikeToReal π E = { inner := fun (x y : E) => RCLike.re (inner x y) }
Instances For
A general inner product space structure implies a real inner product structure.
This is not registered as an instance since
π
does not appear in the return typeInnerProductSpace β E
,- It is likely to create instance diamonds, as it builds upon the diamond-prone
NormedSpace.restrictScalars
.
However, it can be used in a proof to obtain a real inner product space structure from a given
π
-inner product space structure.
Equations
- InnerProductSpace.rclikeToReal π E = InnerProductSpace.mk β― β― β― β―
Instances For
A complex inner product implies a real inner product. This cannot be an instance since it
creates a diamond with PiLp.innerProductSpace
because re (sum i, inner (x i) (y i))
and
sum i, re (inner (x i) (y i))
are not defeq.
Instances For
An RCLike
field is a real inner product space.
Equations
- RCLike.toInnerProductSpaceReal = InnerProductSpace.mk β― β― β― β―