Weak convergence of (finite) measures #
This file will define the topology of weak convergence of finite measures and probability measures
on topological spaces. 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.
TODOs:
- Define the topologies (the current version only defines the types) via
weak_dual ℝ≥0 (α →ᵇ ℝ≥0)
. - Prove that an equivalent definition of the topologies is obtained requiring continuity of
integration of bounded continuous
ℝ
-valued functions instead. - Include the portmanteau theorem on characterizations of weak convergence of (Borel) probability measures.
Main definitions #
The main definitions are the
- types
finite_measure α
andprobability_measure α
; to_weak_dual_bounded_continuous_nnreal : 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 will be used for the definition of the topology of weak convergence.
TODO:
- Define the topologies on the above types.
Main results #
- Finite measures
μ
onα
give rise to continuous linear functionals on the space of bounded continuous nonnegative functions onα
via integration:to_weak_dual_of_bounded_continuous_nnreal : finite_measure α → (weak_dual ℝ≥0 (α →ᵇ ℝ≥0))
.
TODO:
- Portmanteau theorem.
Notations #
No new notation is introduced.
Implementation notes #
The topology of weak convergence of finite Borel measures will be defined using a mapping from
finite_measure α
to weak_dual ℝ≥0 (α →ᵇ ℝ≥0)
, inheriting the topology from the latter.
The current implementation of finite_measure α
and probability_measure α
is directly as
subtypes of measure α
, and the coercion to a function is the composition ennreal.to_nnreal
and the coercion to function of measure α
. Another alternative would be to use a bijection
with vector_measure α ℝ≥0
as an intermediate step. The choice of implementation should not have
drastic downstream effects, so it can be changed later if appropriate.
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. 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
lintegral
w.r.t. a coercion tomeasure α
in any case.
References #
Tags #
weak convergence of measures, finite measure, probability measure
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
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_scalar = {smul := λ (c : ℝ≥0) (μ : measure_theory.finite_measure α), ⟨c • ↑μ, _⟩}
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' := _}
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 finite_measure.test_against_nn
, i.e., integration.
Equations
- μ.to_weak_dual_bounded_continuous_nnreal = {to_linear_map := {to_fun := λ (f : α →ᵇ ℝ≥0), μ.test_against_nn f, map_add' := _, map_smul' := _}, cont := _}
Probability measures are defined as the subtype of measures that have the property of being probability measures (i.e., their total mass is one).
Equations
A probability measure can be interpreted as a measure.
Equations
- measure_theory.probability_measure.has_coe_to_fun = {coe := λ (μ : measure_theory.probability_measure α) (s : set α), (⇑μ s).to_nnreal}
A probability measure can be interpreted as a finite measure.
Equations
- μ.to_finite_measure = ⟨↑μ, _⟩
The pairing of a (Borel) probability measure μ
with a nonnegative bounded continuous
function is obtained by (Lebesgue) integrating the (test) function against the measure. This
is probability_measure.test_against_nn
.
Equations
- μ.test_against_nn f = (measure_theory.lintegral ↑μ (coe ∘ ⇑f)).to_nnreal
Probability measures yield elements of the weak_dual
of bounded continuous nonnegative
functions via probability_measure.test_against_nn
, i.e., integration.
Equations
- μ.to_weak_dual_bounded_continuous_nnreal = {to_linear_map := {to_fun := λ (f : α →ᵇ ℝ≥0), μ.test_against_nn f, map_add' := _, map_smul' := _}, cont := _}