Contents #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we work with contents. A content λ
is a function from a certain class of subsets
(such as the compact subsets) to ℝ≥0
that is
- additive: If
K₁
andK₂
are disjoint sets in the domain ofλ
, thenλ(K₁ ∪ K₂) = λ(K₁) + λ(K₂)
; - subadditive: If
K₁
andK₂
are in the domain ofλ
, thenλ(K₁ ∪ K₂) ≤ λ(K₁) + λ(K₂)
; - monotone: If
K₁ ⊆ K₂
are in the domain ofλ
, thenλ(K₁) ≤ λ(K₂)
.
We show that:
- Given a content
λ
on compact sets, let us define a functionλ*
on open sets, by lettingλ* U
be the supremum ofλ K
forK
included inU
. This is a countably subadditive map that vanishes at∅
. In Halmos (1950) this is called the inner contentλ*
ofλ
, and formalized asinner_content
. - Given an inner content, we define an outer measure
μ*
, by lettingμ* E
be the infimum ofλ* U
over the open setsU
containingE
. This is indeed an outer measure. It is formalized asouter_measure
. - Restricting this outer measure to Borel sets gives a regular measure
μ
.
We define bundled contents as content
.
In this file we only work on contents on compact sets, and inner contents on open sets, and both
contents and inner contents map into the extended nonnegative reals. However, in other applications
other choices can be made, and it is not a priori clear what the best interface should be.
Main definitions #
For μ : content G
, we define
μ.inner_content
: the inner content associated toμ
.μ.outer_measure
: the outer measure associated toμ
.μ.measure
: the Borel measure associated toμ
.
We prove that, on a locally compact space, the measure μ.measure
is regular.
References #
- Paul Halmos (1950), Measure Theory, §53
- https://en.wikipedia.org/wiki/Content_(measure_theory)
- to_fun : topological_space.compacts G → nnreal
- mono' : ∀ (K₁ K₂ : topological_space.compacts G), ↑K₁ ⊆ ↑K₂ → self.to_fun K₁ ≤ self.to_fun K₂
- sup_disjoint' : ∀ (K₁ K₂ : topological_space.compacts G), disjoint ↑K₁ ↑K₂ → self.to_fun (K₁ ⊔ K₂) = self.to_fun K₁ + self.to_fun K₂
- sup_le' : ∀ (K₁ K₂ : topological_space.compacts G), self.to_fun (K₁ ⊔ K₂) ≤ self.to_fun K₁ + self.to_fun K₂
A content is an additive function on compact sets taking values in ℝ≥0
. It is a device
from which one can define a measure.
Instances for measure_theory.content
- measure_theory.content.has_sizeof_inst
- measure_theory.content.inhabited
- measure_theory.content.has_coe_to_fun
Equations
- measure_theory.content.inhabited = {default := {to_fun := λ (K : topological_space.compacts G), 0, mono' := _, sup_disjoint' := _, sup_le' := _}}
Although the to_fun
field of a content takes values in ℝ≥0
, we register a coercion to
functions taking values in ℝ≥0∞
as most constructions below rely on taking suprs and infs, which
is more convenient in a complete lattice, and aim at constructing a measure.
Equations
- measure_theory.content.has_coe_to_fun = {coe := λ (μ : measure_theory.content G) (s : topological_space.compacts G), ↑(μ.to_fun s)}
Constructing the inner content of a content. From a content defined on the compact sets, we obtain a function defined on all open sets, by taking the supremum of the content of all compact subsets.
Equations
- μ.inner_content U = ⨆ (K : topological_space.compacts G) (h : ↑K ⊆ ↑U), ⇑μ K
This is "unbundled", because that it required for the API of induced_outer_measure
.
The inner content of a supremum of opens is at most the sum of the individual inner contents.
The inner content of a union of sets is at most the sum of the individual inner contents.
This is the "unbundled" version of inner_content_Sup_nat
.
It required for the API of induced_outer_measure
.
Extending a content on compact sets to an outer measure on all sets.
Equations
- μ.outer_measure = measure_theory.induced_outer_measure (λ (U : set G) (hU : is_open U), μ.inner_content {carrier := U, is_open' := hU}) is_open_empty _
For the outer measure coming from a content, all Borel sets are measurable.
The measure induced by the outer measure coming from a content, on the Borel sigma-algebra.
Equations
- μ.measure = μ.outer_measure.to_measure _
Instances for measure_theory.content.measure
In a locally compact space, any measure constructed from a content is regular.
A content μ
is called regular if for every compact set K
,
μ(K) = inf {μ(K') : K ⊂ int K' ⊂ K'
. See Paul Halmos (1950), Measure Theory, §54
Equations
- μ.content_regular = ∀ ⦃K : topological_space.compacts G⦄, ⇑μ K = ⨅ (K' : topological_space.compacts G) (hK : ↑K ⊆ interior ↑K'), ⇑μ K'
If μ
is a regular content, then the measure induced by μ
will agree with μ
on compact sets.