Measures invariant under group actions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
A measure μ : measure α is said to be invariant under an action of a group G if scalar
multiplication by c : G is a measure preserving map for all c. In this file we define a
typeclass for measures invariant under action of an (additive or multiplicative) group and prove
some basic properties of such measures.
- measure_preimage_vadd : ∀ (c : M) ⦃s : set α⦄, measurable_set s → ⇑μ ((λ (x : α), c +ᵥ x) ⁻¹' s) = ⇑μ s
A measure μ : measure α is invariant under an additive action of M on α if for any
measurable set s : set α and c : M, the measure of its preimage under λ x, c +ᵥ x is equal to
the measure of s.
Instances of this typeclass
- measure_theory.vadd_invariant_measure.zero
- measure_theory.vadd_invariant_measure.add
- measure_theory.vadd_invariant_measure.vadd
- measure_theory.vadd_invariant_measure.vadd_nnreal
- measure_theory.is_mul_left_invariant.vadd_invariant_measure
- measure_theory.is_mul_right_invariant.to_vadd_invariant_measure_op
- measure_theory.subgroup.vadd_invariant_measure
- measure_preimage_smul : ∀ (c : M) ⦃s : set α⦄, measurable_set s → ⇑μ ((λ (x : α), c • x) ⁻¹' s) = ⇑μ s
A measure μ : measure α is invariant under a multiplicative action of M on α if for any
measurable set s : set α and c : M, the measure of its preimage under λ x, c • x is equal to
the measure of s.
Instances of this typeclass
- measure_theory.smul_invariant_measure.zero
- measure_theory.smul_invariant_measure.add
- measure_theory.smul_invariant_measure.smul
- measure_theory.smul_invariant_measure.smul_nnreal
- measure_theory.is_mul_left_invariant.smul_invariant_measure
- measure_theory.is_mul_right_invariant.to_smul_invariant_measure_op
- measure_theory.subgroup.smul_invariant_measure
Equivalent definitions of a measure invariant under a multiplicative action of a group.
-
0:
smul_invariant_measure G α μ; -
1: for every
c : Gand a measurable sets, the measure of the preimage ofsunder scalar multiplication bycis equal to the measure ofs; -
2: for every
c : Gand a measurable sets, the measure of the imagec • sofsunder scalar multiplication bycis equal to the measure ofs; -
3, 4: properties 2, 3 for any set, including non-measurable ones;
-
5: for any
c : G, scalar multiplication bycmapsμtoμ; -
6: for any
c : G, scalar multiplication bycis a measure preserving map.
Equivalent definitions of a measure invariant under an additive action of a group.
-
0:
vadd_invariant_measure G α μ; -
1: for every
c : Gand a measurable sets, the measure of the preimage ofsunder vector addition(+ᵥ) cis equal to the measure ofs; -
2: for every
c : Gand a measurable sets, the measure of the imagec +ᵥ sofsunder vector addition(+ᵥ) cis equal to the measure ofs; -
3, 4: properties 2, 3 for any set, including non-measurable ones;
-
5: for any
c : G, vector addition ofcmapsμtoμ; -
6: for any
c : G, vector addition ofcis a measure preserving map.
If measure μ is invariant under an additive group action and is nonzero on a compact set K,
then it is positive on any nonempty open set. In case of a regular measure, one can assume μ ≠ 0
instead of μ K ≠ 0, see measure_theory.measure_is_open_pos_of_vadd_invariant_of_ne_zero.
If measure μ is invariant under a group action and is nonzero on a compact set K, then it is
positive on any nonempty open set. In case of a regular measure, one can assume μ ≠ 0 instead of
μ K ≠ 0, see measure_theory.measure_is_open_pos_of_smul_invariant_of_ne_zero.