Fundamental domain of a group action #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
A set s
is said to be a fundamental domain of an action of a group G
on a measurable space α
with respect to a measure μ
if
-
s
is a measurable set; -
the sets
g • s
over allg : G
cover almost all points of the whole space; -
the sets
g • s
, are pairwise a.e. disjoint, i.e.,μ (g₁ • s ∩ g₂ • s) = 0
wheneverg₁ ≠ g₂
; we require this forg₂ = 1
in the definition, then deduce it for any twog₁ ≠ g₂
.
In this file we prove that in case of a countable group G
and a measure preserving action, any two
fundamental domains have the same measure, and for a G
-invariant function, its integrals over any
two fundamental domains are equal to each other.
We also generate additive versions of all theorems in this file using the to_additive
attribute.
Main declarations #
measure_theory.is_fundamental_domain
: Predicate for a set to be a fundamental domain of the action of a groupmeasure_theory.fundamental_frontier
: Fundamental frontier of a set under the action of a group. Elements ofs
that belong to some other translate ofs
.measure_theory.fundamental_interior
: Fundamental interior of a set under the action of a group. Elements ofs
that do not belong to any other translate ofs
.
- null_measurable_set : measure_theory.null_measurable_set s μ
- ae_covers : ∀ᵐ (x : α) ∂μ, ∃ (g : G), g +ᵥ x ∈ s
- ae_disjoint : pairwise (measure_theory.ae_disjoint μ on λ (g : G), g +ᵥ s)
A measurable set s
is a fundamental domain for an additive action of an additive group G
on a measurable space α
with respect to a measure α
if the sets g +ᵥ s
, g : G
, are pairwise
a.e. disjoint and cover the whole space.
- null_measurable_set : measure_theory.null_measurable_set s μ
- ae_covers : ∀ᵐ (x : α) ∂μ, ∃ (g : G), g • x ∈ s
- ae_disjoint : pairwise (measure_theory.ae_disjoint μ on λ (g : G), g • s)
A measurable set s
is a fundamental domain for an action of a group G
on a measurable
space α
with respect to a measure α
if the sets g • s
, g : G
, are pairwise a.e. disjoint and
cover the whole space.
If for each x : α
, exactly one of g • x
, g : G
, belongs to a measurable set s
, then s
is a fundamental domain for the action of G
on α
.
If for each x : α
, exactly one of g +ᵥ x
, g : G
, belongs to a measurable set
s
, then s
is a fundamental domain for the additive action of G
on α
.
For s
to be a fundamental domain, it's enough to check ae_disjoint (g • s) s
for g ≠ 1
.
For s
to be a fundamental domain, it's enough to check ae_disjoint (g +ᵥ s) s
for
g ≠ 0
.
If a measurable space has a finite measure μ
and a countable additive group G
acts
quasi-measure-preservingly, then to show that a set s
is a fundamental domain, it is sufficient
to check that its translates g +ᵥ s
are (almost) disjoint and that the sum ∑' g, μ (g +ᵥ s)
is
sufficiently large.
If a measurable space has a finite measure μ
and a countable group G
acts
quasi-measure-preservingly, then to show that a set s
is a fundamental domain, it is sufficient
to check that its translates g • s
are (almost) disjoint and that the sum ∑' g, μ (g • s)
is
sufficiently large.
Given a measure space with an action of a finite group G
, the measure of any G
-invariant set
is determined by the measure of its intersection with a fundamental domain for the action of G
.
Given a measure space with an action of a
finite additive group G
, the measure of any G
-invariant set is determined by the measure of its
intersection with a fundamental domain for the action of G
.
If s
and t
are two fundamental domains of the same action, then their measures are equal.
If s
and t
are two fundamental domains of the same action, then their measures
are equal.
If the additive action of a countable group G
admits an invariant measure μ
with
a fundamental domain s
, then every null-measurable set t
such that the sets g +ᵥ t ∩ s
are
pairwise a.e.-disjoint has measure at most μ s
.
If the action of a countable group G
admits an invariant measure μ
with a fundamental domain
s
, then every null-measurable set t
such that the sets g • t ∩ s
are pairwise a.e.-disjoint
has measure at most μ s
.
If the action of a countable group G
admits an invariant measure μ
with a fundamental domain
s
, then every null-measurable set t
of measure strictly greater than μ s
contains two
points x y
such that g • x = y
for some g ≠ 1
.
If the additive action of a countable group G
admits an invariant measure μ
with
a fundamental domain s
, then every null-measurable set t
of measure strictly greater than μ s
contains two points x y
such that g +ᵥ x = y
for some g ≠ 0
.
If f
is invariant under the action of a countable group G
, and μ
is a G
-invariant
measure with a fundamental domain s
, then the ess_sup
of f
restricted to s
is the same as
that of f
on all of its domain.
If f
is invariant under the action of a countable additive group G
, and μ
is a
G
-invariant measure with a fundamental domain s
, then the ess_sup
of f
restricted to s
is
the same as that of f
on all of its domain.
Interior/frontier of a fundamental domain #
The boundary of a fundamental domain, those points of the domain that also lie in a nontrivial translate.
The boundary of a fundamental domain, those points of the domain that also lie in a nontrivial translate.
The interior of a fundamental domain, those points of the domain not lying in any translate.
The interior of a fundamental domain, those points of the domain not lying in any translate.