Finite measures #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the type of finite measures on a given measurable space. When the underlying
space has a topology and the measurable space structure (sigma algebra) is finer than the Borel
sigma algebra, then the type of finite measures is equipped with the topology of weak convergence
of measures. The topology of weak convergence is the coarsest topology w.r.t. which
for every bounded continuous ℝ≥0
-valued function f
, the integration of f
against the
measure is continuous.
Main definitions #
The main definitions are
- the type
measure_theory.finite_measure Ω
with the topology of weak convergence; measure_theory.finite_measure.to_weak_dual_bcnn : finite_measure Ω → (weak_dual ℝ≥0 (Ω →ᵇ ℝ≥0))
allowing to interpret a finite measure as a continuous linear functional on the space of bounded continuous nonnegative functions onΩ
. This is used for the definition of the topology of weak convergence.
Main results #
- Finite measures
μ
onΩ
give rise to continuous linear functionals on the space of bounded continuous nonnegative functions onΩ
via integration:measure_theory.finite_measure.to_weak_dual_bcnn : finite_measure Ω → (weak_dual ℝ≥0 (Ω →ᵇ ℝ≥0))
measure_theory.finite_measure.tendsto_iff_forall_integral_tendsto
: Convergence of finite measures is characterized by the convergence of integrals of all bounded continuous functions. This shows that the chosen definition of topology coincides with the common textbook definition of weak convergence of measures. A similar characterization by the convergence of integrals (in themeasure_theory.lintegral
sense) of all bounded continuous nonnegative functions ismeasure_theory.finite_measure.tendsto_iff_forall_lintegral_tendsto
.
Implementation notes #
The topology of weak convergence of finite Borel measures is defined using a mapping from
measure_theory.finite_measure Ω
to weak_dual ℝ≥0 (Ω →ᵇ ℝ≥0)
, inheriting the topology from the
latter.
The implementation of measure_theory.finite_measure Ω
and is directly as a subtype of
measure_theory.measure Ω
, and the coercion to a function is the composition ennreal.to_nnreal
and the coercion to function of measure_theory.measure Ω
. Another alternative would have been to
use a bijection with measure_theory.vector_measure Ω ℝ≥0
as an intermediate step. Some
considerations:
- Potential advantages of using the
nnreal
-valued vector measure alternative:- The coercion to function would avoid need to compose with
ennreal.to_nnreal
, thennreal
-valued API could be more directly available.
- The coercion to function would avoid need to compose with
- Potential drawbacks of the vector measure alternative:
- The coercion to function would lose monotonicity, as non-measurable sets would be defined to have measure 0.
- No integration theory directly. E.g., the topology definition requires
measure_theory.lintegral
w.r.t. a coercion tomeasure_theory.measure Ω
in any case.
References #
Tags #
weak convergence of measures, finite measure
Finite measures #
In this section we define the Type
of finite_measure Ω
, when Ω
is a measurable space. Finite
measures on Ω
are a module over ℝ≥0
.
If Ω
is moreover a topological space and the sigma algebra on Ω
is finer than the Borel sigma
algebra (i.e. [opens_measurable_space Ω]
), then finite_measure Ω
is equipped with the topology
of weak convergence of measures. This is implemented by defining a pairing of finite measures μ
on Ω
with continuous bounded nonnegative functions f : Ω →ᵇ ℝ≥0
via integration, and using the
associated weak topology (essentially the weak-star topology on the dual of Ω →ᵇ ℝ≥0
).
Finite measures are defined as the subtype of measures that have the property of being finite measures (i.e., their total mass is finite).
Equations
Instances for measure_theory.finite_measure
- measure_theory.finite_measure.measure_theory.measure.has_coe
- measure_theory.finite_measure.has_coe_to_fun
- measure_theory.finite_measure.has_zero
- measure_theory.finite_measure.inhabited
- measure_theory.finite_measure.has_add
- measure_theory.finite_measure.has_smul
- measure_theory.finite_measure.add_comm_monoid
- measure_theory.finite_measure.module
- measure_theory.finite_measure.topological_space
A finite measure can be interpreted as a measure.
Equations
- measure_theory.finite_measure.has_coe_to_fun = {coe := λ (μ : measure_theory.finite_measure Ω) (s : set Ω), (⇑μ s).to_nnreal}
The (total) mass of a finite measure μ
is μ univ
, i.e., the cast to nnreal
of
(μ : measure Ω) univ
.
Equations
- measure_theory.finite_measure.has_zero = {zero := ⟨0, _⟩}
Equations
Equations
- measure_theory.finite_measure.has_add = {add := λ (μ ν : measure_theory.finite_measure Ω), ⟨↑μ + ↑ν, _⟩}
Equations
- measure_theory.finite_measure.has_smul = {smul := λ (c : R) (μ : measure_theory.finite_measure Ω), ⟨c • ↑μ, _⟩}
Equations
- measure_theory.finite_measure.add_comm_monoid = function.injective.add_comm_monoid coe measure_theory.finite_measure.coe_injective measure_theory.finite_measure.coe_zero measure_theory.finite_measure.coe_add measure_theory.finite_measure.add_comm_monoid._proof_3
Coercion is an add_monoid_hom
.
Equations
- measure_theory.finite_measure.coe_add_monoid_hom = {to_fun := coe coe_to_lift, map_zero' := _, map_add' := _}
Equations
- measure_theory.finite_measure.module = function.injective.module nnreal measure_theory.finite_measure.coe_add_monoid_hom measure_theory.finite_measure.coe_injective measure_theory.finite_measure.module._proof_4
Restrict a finite measure μ to a set A.
The pairing of a finite (Borel) measure μ
with a nonnegative bounded continuous
function is obtained by (Lebesgue) integrating the (test) function against the measure.
This is finite_measure.test_against_nn
.
Finite measures yield elements of the weak_dual
of bounded continuous nonnegative
functions via measure_theory.finite_measure.test_against_nn
, i.e., integration.
Equations
- μ.to_weak_dual_bcnn = {to_linear_map := {to_fun := λ (f : bounded_continuous_function Ω nnreal), μ.test_against_nn f, map_add' := _, map_smul' := _}, cont := _}
The topology of weak convergence on measure_theory.finite_measure Ω
is inherited (induced)
from the weak-* topology on weak_dual ℝ≥0 (Ω →ᵇ ℝ≥0)
via the function
measure_theory.finite_measure.to_weak_dual_bcnn
.
The total mass of a finite measure depends continuously on the measure.
Convergence of finite measures implies the convergence of their total masses.
If the total masses of finite measures tend to zero, then the measures tend to
zero. This formulation concerns the associated functionals on bounded continuous
nonnegative test functions. See finite_measure.tendsto_zero_of_tendsto_zero_mass
for
a formulation stating the weak convergence of measures.
If the total masses of finite measures tend to zero, then the measures tend to zero.
A characterization of weak convergence in terms of integrals of bounded continuous nonnegative functions.
Bounded convergence results for finite measures #
This section is about bounded convergence theorems for finite measures.
A bounded convergence theorem for a finite measure: If bounded continuous non-negative functions are uniformly bounded by a constant and tend to a limit, then their integrals against the finite measure tend to the integral of the limit. This formulation assumes:
- the functions tend to a limit along a countably generated filter;
- the limit is in the almost everywhere sense;
- boundedness holds almost everywhere;
- integration is
measure_theory.lintegral
, i.e., the functions and their integrals areℝ≥0∞
-valued.
A bounded convergence theorem for a finite measure:
If a sequence of bounded continuous non-negative functions are uniformly bounded by a constant
and tend pointwise to a limit, then their integrals (measure_theory.lintegral
) against the finite
measure tend to the integral of the limit.
A related result with more general assumptions is
measure_theory.finite_measure.tendsto_lintegral_nn_filter_of_le_const
.
A bounded convergence theorem for a finite measure: If bounded continuous non-negative functions are uniformly bounded by a constant and tend to a limit, then their integrals against the finite measure tend to the integral of the limit. This formulation assumes:
- the functions tend to a limit along a countably generated filter;
- the limit is in the almost everywhere sense;
- boundedness holds almost everywhere;
- integration is the pairing against non-negative continuous test functions
(
measure_theory.finite_measure.test_against_nn
).
A related result using measure_theory.lintegral
for integration is
measure_theory.finite_measure.tendsto_lintegral_nn_filter_of_le_const
.
A bounded convergence theorem for a finite measure:
If a sequence of bounded continuous non-negative functions are uniformly bounded by a constant and
tend pointwise to a limit, then their integrals (measure_theory.finite_measure.test_against_nn
)
against the finite measure tend to the integral of the limit.
Related results:
measure_theory.finite_measure.tendsto_test_against_nn_filter_of_le_const
: more general assumptionsmeasure_theory.finite_measure.tendsto_lintegral_nn_of_le_const
: usingmeasure_theory.lintegral
for integration.
Weak convergence of finite measures with bounded continuous real-valued functions #
In this section we characterize the weak convergence of finite measures by the usual (defining) condition that the integrals of all bounded continuous real-valued functions converge.
A characterization of weak convergence in terms of integrals of bounded continuous real-valued functions.