mathlib documentation

measure_theory.group.measure

Measures on Groups #

We develop some properties of measures on (topological) groups

We also give analogues of all these notions in the additive world.

@[class]

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
@[class]

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
theorem measure_theory.map_add_right_eq_self {G : Type u_1} [measurable_space G] [has_add G] (μ : measure_theory.measure G) [μ.is_add_right_invariant] (g : G) :
(measure_theory.measure.map (λ (_x : G), _x + g)) μ = μ
theorem measure_theory.map_mul_right_eq_self {G : Type u_1} [measurable_space G] [has_mul G] (μ : measure_theory.measure G) [μ.is_mul_right_invariant] (g : G) :
(measure_theory.measure.map (λ (_x : G), _x * g)) μ = μ
theorem measure_theory.forall_measure_preimage_add_iff {G : Type u_1} [measurable_space G] [has_add G] [has_measurable_add G] (μ : measure_theory.measure G) :
(∀ (g : G) (A : set G), measurable_set Aμ ((λ (h : G), g + h) ⁻¹' A) = μ A) μ.is_add_left_invariant
theorem measure_theory.forall_measure_preimage_mul_iff {G : Type u_1} [measurable_space G] [has_mul G] [has_measurable_mul G] (μ : measure_theory.measure G) :
(∀ (g : G) (A : set G), measurable_set Aμ ((λ (h : G), g * h) ⁻¹' A) = μ A) μ.is_mul_left_invariant

An alternative way to prove that μ is left invariant under multiplication.

theorem measure_theory.forall_measure_preimage_mul_right_iff {G : Type u_1} [measurable_space G] [has_mul G] [has_measurable_mul G] (μ : measure_theory.measure G) :
(∀ (g : G) (A : set G), measurable_set Aμ ((λ (h : G), h * g) ⁻¹' A) = μ A) μ.is_mul_right_invariant

An alternative way to prove that μ is left invariant under multiplication.

theorem measure_theory.forall_measure_preimage_add_right_iff {G : Type u_1} [measurable_space G] [has_add G] [has_measurable_add G] (μ : measure_theory.measure G) :
(∀ (g : G) (A : set G), measurable_set Aμ ((λ (h : G), h + g) ⁻¹' A) = μ A) μ.is_add_right_invariant
@[simp]
theorem measure_theory.measure_preimage_add {G : Type u_1} [measurable_space G] [add_group G] [has_measurable_add G] (μ : measure_theory.measure G) [μ.is_add_left_invariant] (g : G) (A : set G) :
μ ((λ (h : G), g + h) ⁻¹' A) = μ A
@[simp]
theorem measure_theory.measure_preimage_mul {G : Type u_1} [measurable_space G] [group G] [has_measurable_mul G] (μ : measure_theory.measure G) [μ.is_mul_left_invariant] (g : G) (A : set G) :
μ ((λ (h : G), g * h) ⁻¹' A) = μ A

We shorten this from measure_preimage_mul_left, since left invariant is the preferred option for measures in this formalization.

@[simp]
theorem measure_theory.measure_preimage_add_right {G : Type u_1} [measurable_space G] [add_group G] [has_measurable_add G] (μ : measure_theory.measure G) [μ.is_add_right_invariant] (g : G) (A : set G) :
μ ((λ (h : G), h + g) ⁻¹' A) = μ A
@[simp]
theorem measure_theory.measure_preimage_mul_right {G : Type u_1} [measurable_space G] [group G] [has_measurable_mul G] (μ : measure_theory.measure G) [μ.is_mul_right_invariant] (g : G) (A : set G) :
μ ((λ (h : G), h * g) ⁻¹' A) = μ A
@[protected]

The measure A ↦ μ (A⁻¹), where A⁻¹ is the pointwise inverse of A.

Equations
@[protected]

The measure A ↦ μ (- A), where - A is the pointwise negation of A.

Equations
theorem measure_theory.measure.neg_apply {G : Type u_1} [measurable_space G] [add_group G] [has_measurable_neg G] (μ : measure_theory.measure G) (s : set G) :
(μ.neg) s = μ (-s)
@[protected, simp]
@[protected, simp]

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.

@[protected, instance]

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.

@[class]

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
@[class]

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.

Instances

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.

@[protected, instance]

A Haar measure on a sigma-compact space is sigma-finite.

@[protected, instance]

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.