Measures on Groups #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We develop some properties of measures on (topological) groups
- We define properties on measures: measures that are left or right invariant w.r.t. multiplication.
- We define the measure
μ.inv : A ↦ μ(A⁻¹)
and show that it is right invariant iffμ
is left invariant. - We define a class
is_haar_measure μ
, requiring that the measureμ
is left-invariant, finite on compact sets, and positive on open sets.
We also give analogues of all these notions in the additive world.
- map_add_left_eq_self : ∀ (g : G), measure_theory.measure.map (has_add.add g) μ = μ
A measure μ
on a measurable additive group is left invariant
if the measure of left translations of a set are equal to the measure of the set itself.
Instances of this typeclass
- measure_theory.measure.is_add_haar_measure.to_is_add_left_invariant
- measure_theory.is_add_left_invariant_smul
- measure_theory.is_add_left_invariant_smul_nnreal
- measure_theory.measure.prod.measure.is_add_left_invariant
- measure_theory.measure.neg.is_add_left_invariant
- measure_theory.measure.pi.is_add_left_invariant
- measure_theory.pi.is_add_left_invariant_volume
- measure_theory.measure.is_add_left_invariant_add_haar_measure
- measure_theory.measure.alternating_map.measure.is_add_left_invariant
- measure_theory.measure.hausdorff_measure.measure.is_add_left_invariant
- map_mul_left_eq_self : ∀ (g : G), measure_theory.measure.map (has_mul.mul g) μ = μ
A measure μ
on a measurable group is left invariant
if the measure of left translations of a set are equal to the measure of the set itself.
Instances of this typeclass
- measure_theory.measure.is_haar_measure.to_is_mul_left_invariant
- measure_theory.is_mul_left_invariant_smul
- measure_theory.is_mul_left_invariant_smul_nnreal
- measure_theory.measure.prod.measure.is_mul_left_invariant
- measure_theory.measure.inv.is_mul_left_invariant
- measure_theory.measure.pi.is_mul_left_invariant
- measure_theory.pi.is_mul_left_invariant_volume
- measure_theory.measure.is_mul_left_invariant_haar_measure
- measure_theory.measure.hausdorff_measure.measure.is_mul_left_invariant
- map_add_right_eq_self : ∀ (g : G), measure_theory.measure.map (λ (_x : G), _x + g) μ = μ
A measure μ
on a measurable additive group is right invariant
if the measure of right translations of a set are equal to the measure of the set itself.
Instances of this typeclass
- is_add_left_invariant.is_add_right_invariant
- measure_theory.is_add_right_invariant_smul
- measure_theory.is_add_right_invariant_smul_nnreal
- measure_theory.measure.prod.measure.is_add_right_invariant
- measure_theory.measure.neg.is_add_right_invariant
- measure_theory.measure.pi.is_add_right_invariant
- measure_theory.measure.hausdorff_measure.measure.is_add_right_invariant
- map_mul_right_eq_self : ∀ (g : G), measure_theory.measure.map (λ (_x : G), _x * g) μ = μ
A measure μ
on a measurable group is right invariant
if the measure of right translations of a set are equal to the measure of the set itself.
Instances of this typeclass
- measure_theory.is_mul_left_invariant.is_mul_right_invariant
- measure_theory.is_mul_right_invariant_smul
- measure_theory.is_mul_right_invariant_smul_nnreal
- measure_theory.measure.prod.measure.is_mul_right_invariant
- measure_theory.measure.inv.is_mul_right_invariant
- measure_theory.measure.pi.is_mul_right_invariant
- measure_theory.measure.hausdorff_measure.measure.is_mul_right_invariant
An alternative way to prove that μ
is left invariant under addition.
An alternative way to prove that μ
is left invariant under multiplication.
An alternative way to prove that μ
is right invariant under multiplication.
An alternative way to prove that μ
is right invariant under addition.
We shorten this from measure_preimage_add_left
, since left invariant is the
preferred option for measures in this formalization.
We shorten this from measure_preimage_mul_left
, since left invariant is the preferred option
for measures in this formalization.
The measure A ↦ μ (A⁻¹)
, where A⁻¹
is the pointwise inverse of A
.
Equations
The measure A ↦ μ (- A)
, where - A
is the pointwise negation of A
.
Equations
A measure is invariant under negation if - μ = μ
. Equivalently, this means that for all
measurable A
we have μ (- A) = μ A
, where - A
is the pointwise negation of A
.
A measure is invariant under inversion if μ⁻¹ = μ
. Equivalently, this means that for all
measurable A
we have μ (A⁻¹) = μ A
, where A⁻¹
is the pointwise inverse of A
.
If a left-invariant measure gives positive mass to a compact set, then it gives positive mass to any open set.
If a left-invariant measure gives positive mass to a compact set, then it gives positive mass to any open set.
A nonzero left-invariant regular measure gives positive mass to any open set.
A nonzero left-invariant regular measure gives positive mass to any open set.
If a left-invariant measure gives finite mass to a nonempty open set, then it gives finite mass to any compact set.
If a left-invariant measure gives finite mass to a nonempty open set, then it gives finite mass to any compact set.
If a left-invariant measure gives finite mass to a set with nonempty interior, then it gives finite mass to any compact set.
If a left-invariant measure gives finite mass to a set with nonempty interior, then it gives finite mass to any compact set.
In a noncompact locally compact group, a left-invariant measure which is positive on open sets has infinite mass.
In a noncompact locally compact additive group, a left-invariant measure which is positive on open sets has infinite mass.
In an abelian additive
group every left invariant measure is also right-invariant. We don't declare the converse as an
instance, since that would loop type-class inference, and we use is_add_left_invariant
as the
default hypothesis in abelian groups.
In an abelian group every left invariant measure is also right-invariant.
We don't declare the converse as an instance, since that would loop type-class inference, and
we use is_mul_left_invariant
as the default hypothesis in abelian groups.
- to_is_finite_measure_on_compacts : measure_theory.is_finite_measure_on_compacts μ
- to_is_add_left_invariant : μ.is_add_left_invariant
- to_is_open_pos_measure : μ.is_open_pos_measure
A measure on an additive group is an additive Haar measure if it is left-invariant, and gives finite mass to compact sets and positive mass to open sets.
Instances of this typeclass
- measure_theory.measure.prod.is_add_haar_measure
- measure_theory.measure.pi.is_add_haar_measure
- measure_theory.measure.is_add_haar_measure_add_haar_measure
- is_add_haar_measure_basis_add_haar
- measure_theory.is_add_haar_measure_volume_pi
- measure_theory.measure.map_continuous_linear_equiv.is_add_haar_measure
- measure_theory.measure.map_linear_equiv.is_add_haar_measure
- add_circle.measure_theory.measure_space.volume.measure_theory.measure.is_add_haar_measure
- add_circle.haar_add_circle.is_add_haar_measure
- to_is_finite_measure_on_compacts : measure_theory.is_finite_measure_on_compacts μ
- to_is_mul_left_invariant : μ.is_mul_left_invariant
- to_is_open_pos_measure : μ.is_open_pos_measure
A measure on a group is a Haar measure if it is left-invariant, and gives finite mass to compact sets and positive mass to open sets.
Record that a Haar measure on a locally compact space is locally finite. This is needed as the fact that a measure which is finite on compacts is locally finite is not registered as an instance, to avoid an instance loop.
Record that an additive Haar measure on a locally compact space is locally finite. This is needed as the fact that a measure which is finite on compacts is locally finite is not registered as an instance, to avoid an instance loop.
If a left-invariant measure gives positive mass to some compact set with nonempty interior, then it is a Haar measure.
If a left-invariant measure gives positive mass to some compact set with nonempty interior, then it is an additive Haar measure.
The image of a Haar measure under a continuous surjective proper group homomorphism is again
a Haar measure. See also mul_equiv.is_haar_measure_map
.
The image of an additive Haar measure under a continuous surjective proper additive
group homomorphism is again an additive Haar measure. See also
add_equiv.is_add_haar_measure_map
.
A convenience wrapper for measure_theory.measure.is_haar_measure_map
.
A convenience wrapper for measure_theory.measure.is_add_haar_measure_map
.
A Haar measure on a σ-compact space is σ-finite.
A Haar measure on a σ-compact space is σ-finite.
If the neutral element of a group is not isolated, then a Haar measure on this group has no atoms.
The additive version of this instance applies in particular to show that an additive Haar measure on a nontrivial finite-dimensional real vector space has no atom.
If the zero element of an additive group is not isolated, then an additive Haar measure on this group has no atoms.
This applies in particular to show that an additive Haar measure on a nontrivial finite-dimensional real vector space has no atom.