Additive Haar measure constructed from a basis #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Given a basis of a finite-dimensional real vector space, we define the corresponding Lebesgue
measure, which gives measure 1
to the parallelepiped spanned by the basis.
Main definitions #
parallelepiped v
is the parallelepiped spanned by a finite family of vectors.basis.parallelepiped
is the parallelepiped associated to a basis, seen as a compact set with nonempty interior.basis.add_haar
is the Lebesgue measure associated to a basis, giving measure1
to the corresponding parallelepiped.
In particular, we declare a measure_space
instance on any finite-dimensional inner product space,
by using the Lebesgue measure associated to some orthonormal basis (which is in fact independent
of the basis).
The closed parallelepiped spanned by a finite family of vectors.
Equations
- parallelepiped v = (λ (t : ι → ℝ), finset.univ.sum (λ (i : ι), t i • v i)) '' set.Icc 0 1
Reindexing a family of vectors does not change their parallelepiped.
A parallelepiped
is the convex hull of its vertices
The axis aligned parallelepiped over ι → ℝ
is a cuboid.
The parallelepiped spanned by a basis, as a compact set with nonempty interior.
Equations
- b.parallelepiped = {to_compacts := {carrier := parallelepiped ⇑b, is_compact' := _}, interior_nonempty' := _}
The Lebesgue measure associated to a basis, giving measure 1
to the parallelepiped spanned
by the basis.
Equations
Instances for basis.add_haar
A finite dimensional inner product space has a canonical measure, the Lebesgue measure giving
volume 1
to the parallelepiped spanned by any orthonormal basis. We define the measure using
some arbitrary choice of orthonormal basis. The fact that it works with any orthonormal basis
is proved in orthonormal_basis.volume_parallelepiped
.
Equations
- measure_space_of_inner_product_space = {to_measurable_space := _inst_6, volume := (std_orthonormal_basis ℝ E).to_basis.add_haar}
Miscellaneous instances for euclidean_space
#
In combination with measure_space_of_inner_product_space
, these put a measure_space
structure
on euclidean_space
.
pi_Lp.equiv
as a measurable_equiv
.
Equations
- euclidean_space.measurable_equiv ι = {to_equiv := pi_Lp.equiv 2 (λ (i : ι), ℝ), measurable_to_fun := _, measurable_inv_fun := _}