Measures on Groups #
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
- measure_theory.measure.is_add_haar_measure.to_is_add_left_invariant
- measure_theory.has_scalar.smul.measure.is_add_left_invariant
- measure_theory.measure.neg.measure.is_add_left_invariant
- measure_theory.measure.pi.is_add_left_invariant
- measure_theory.pi.is_add_left_invariant_volume
- real.is_add_left_invariant_real_volume
- real.is_add_left_invariant_real_volume_pi
- measure_theory.measure.is_add_left_invariant_add_haar_measure
- measure_theory.is_add_left_invariant_real_volume_pi
- 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
- measure_theory.measure.is_haar_measure.to_is_mul_left_invariant
- measure_theory.has_scalar.smul.measure.is_mul_left_invariant
- measure_theory.measure.inv.measure.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
- 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.
- 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.
An alternative way to prove that μ
is left invariant under multiplication.
An alternative way to prove that μ
is left invariant under multiplication.
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
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.
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.
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 default hypotheses 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.
- 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.
If a left-invariant measure gives positive mass to some compact set with nonempty interior, then it is a Haar measure
The image of a Haar measure under a group homomorphism which is also a homeomorphism is again a Haar measure.
A Haar measure on a sigma-compact space is sigma-finite.
If the neutral element of a group is not isolated, then a Haar measure on this group has no atom.
This applies in particular to show that an additive Haar measure on a nontrivial finite-dimensional real vector space has no atom.