Product measures #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define and prove properties about finite products of measures (and at some point, countable products of measures).
Main definition #
measure_theory.measure.pi
: The product of finitely many σ-finite measures. Givenμ : Π i : ι, measure (α i)
for[fintype ι]
it has typemeasure (Π i : ι, α i)
.
To apply Fubini along some subset of the variables, use
measure_theory.measure_preserving_pi_equiv_pi_subtype_prod
to reduce to the situation of a product
of two measures: this lemma states that the bijection
measurable_equiv.pi_equiv_pi_subtype_prod α p
between (Π i : ι, α i)
and
(Π i : {i // p i}, α i) × (Π i : {i // ¬ p i}, α i)
maps a product measure to a direct product of
product measures, to which one can apply the usual Fubini for direct product of measures.
Implementation Notes #
We define measure_theory.outer_measure.pi
, the product of finitely many outer measures, as the
maximal outer measure n
with the property that n (pi univ s) ≤ ∏ i, m i (s i)
,
where pi univ s
is the product of the sets {s i | i : ι}
.
We then show that this induces a product of measures, called measure_theory.measure.pi
.
For a collection of σ-finite measures μ
and a collection of measurable sets s
we show that
measure.pi μ (pi univ s) = ∏ i, m i (s i)
. To do this, we follow the following steps:
- We know that there is some ordering on
ι
, given by an element of[countable ι]
. - Using this, we have an equivalence
measurable_equiv.pi_measurable_equiv_tprod
betweenΠ ι, α i
and an iterated product ofα i
, calledlist.tprod α l
for some listl
. - On this iterated product we can easily define a product measure
measure_theory.measure.tprod
by iteratingmeasure_theory.measure.prod
- Using the previous two steps we construct
measure_theory.measure.pi'
onΠ ι, α i
for countableι
. - We know that
measure_theory.measure.pi'
sends products of sets to products of measures, and sincemeasure_theory.measure.pi
is the maximal such measure (or at least, it comes from an outer measure which is the maximal such outer measure), we get the same rule formeasure_theory.measure.pi
.
Tags #
finitary product measure
We start with some measurability properties
Boxes form a π-system.
The product of generated σ-algebras is the one generated by boxes, if both generating sets are countably spanning.
If C
and D
generate the σ-algebras on α
resp. β
, then rectangles formed by C
and D
generate the σ-algebra on α × β
.
The product σ-algebra is generated from boxes, i.e. s ×ˢ t
for sets s : set α
and
t : set β
.
An upper bound for the measure in a finite product space. It is defined to by taking the image of the set under all projections, and taking the product of the measures of these images. For measurable boxes it is equal to the correct measure.
Equations
- measure_theory.pi_premeasure m s = finset.univ.prod (λ (i : ι), ⇑(m i) (function.eval i '' s))
outer_measure.pi m
is the finite product of the outer measures {m i | i : ι}
.
It is defined to be the maximal outer measure n
with the property that
n (pi univ s) ≤ ∏ i, m i (s i)
, where pi univ s
is the product of the sets
{s i | i : ι}
.
A product of measures in tprod α l
.
Equations
- measure_theory.measure.tprod l μ = list.rec (measure_theory.measure.dirac punit.star) (λ (i : δ) (l : list δ) (ih : measure_theory.measure (list.tprod π l)), (μ i).prod ih) l
Instances for measure_theory.measure.tprod
The product measure on an encodable finite type, defined by mapping measure.tprod
along the
equivalence measurable_equiv.pi_measurable_equiv_tprod
.
The definition measure_theory.measure.pi
should be used instead of this one.
measure.pi μ
is the finite product of the measures {μ i | i : ι}
.
It is defined to be measure corresponding to measure_theory.outer_measure.pi
.
Equations
- measure_theory.measure.pi μ = (measure_theory.outer_measure.pi (λ (i : ι), (μ i).to_outer_measure)).to_measure _
Instances for measure_theory.measure.pi
- measure_theory.measure.pi.sigma_finite
- measure_theory.measure.pi.measure_theory.has_no_atoms
- measure_theory.measure.pi.measure_theory.is_locally_finite_measure
- measure_theory.measure.pi.is_mul_left_invariant
- measure_theory.measure.pi.is_add_left_invariant
- measure_theory.measure.pi.is_mul_right_invariant
- measure_theory.measure.pi.is_add_right_invariant
- measure_theory.measure.pi.is_inv_invariant
- measure_theory.measure.pi.is_neg_invariant
- measure_theory.measure.pi.is_open_pos_measure
- measure_theory.measure.pi.is_finite_measure_on_compacts
- measure_theory.measure.pi.is_haar_measure
- measure_theory.measure.pi.is_add_haar_measure
measure.pi μ
has finite spanning sets in rectangles of finite spanning sets.
A measure on a finite product space equals the product measure if they are equal on rectangles with as sides sets that generate the corresponding σ-algebras.
A measure on a finite product space equals the product measure if they are equal on rectangles.
If one of the measures μ i
has no atoms, them measure.pi µ
has no atoms. The instance below assumes that all μ i
have no atoms.
Equations
We intentionally restrict this only to the nondependent function space, since
type-class inference cannot find an instance for ι → ℝ
when this is stated for dependent function
spaces.
We intentionally restrict this only to the nondependent function space, since type-class
inference cannot find an instance for ι → ℝ
when this is stated for dependent function spaces.
We intentionally restrict this only to the nondependent function space, since type-class
inference cannot find an instance for ι → ℝ
when this is stated for dependent function spaces.
We intentionally restrict this only to the nondependent function space, since
type-class inference cannot find an instance for ι → ℝ
when this is stated for dependent function
spaces.
Measure preserving equivalences #
In this section we prove that some measurable equivalences (e.g., between fin 1 → α
and α
or
between fin 2 → α
and α × α
) preserve measure or volume. These lemmas can be used to prove that
measures of corresponding sets (images or preimages) have equal measures and functions f ∘ e
and
f
have equal integrals, see lemmas in the measure_theory.measure_preserving
prefix.