Set integral
In this file we prove some properties of ∫ x in s, f x ∂μ. Recall that this notation
is defined as ∫ x, f x ∂(μ.restrict s). In integral_indicator we prove that for a measurable
function f and a measurable set s this definition coincides with another natural definition:
∫ x, indicator s f x ∂μ = ∫ x in s, f x ∂μ, where indicator s f x is equal to f x for x ∈ s
and is zero otherwise.
Since ∫ x in s, f x ∂μ is a notation, one can rewrite or apply any theorem about ∫ x, f x ∂μ
directly. In this file we prove some theorems about dependence of ∫ x in s, f x ∂μ on s, e.g.
integral_union, integral_empty, integral_univ.
We also define integrable_on f s μ := integrable f (μ.restrict s) and prove theorems like
integrable_on_union : integrable_on f (s ∪ t) μ ↔ integrable_on f s μ ∧ integrable_on f t μ.
Next we define a predicate integrable_at_filter (f : α → E) (l : filter α) (μ : measure α)
saying that f is integrable at some set s ∈ l and prove that a measurable function is integrable
at l with respect to μ provided that f is bounded above at l ⊓ μ.ae and μ is finite
at l.
Finally, we prove a version of the
Fundamental theorem of calculus
for set integral, see filter.tendsto.integral_sub_linear_is_o_ae and its corollaries.
Namely, consider a measurably generated filter l, a measure μ finite at this filter, and
a function f that has a finite limit c at l ⊓ μ.ae. Then ∫ x in s, f x ∂μ = μ s • c + o(μ s)
as s tends to l.lift' powerset, i.e. for any ε>0 there exists t ∈ l such that
∥∫ x in s, f x ∂μ - μ s • c∥ ≤ ε * μ s whenever s ⊆ t. We also formulate a version of this
theorem for a locally finite measure μ and a function f continuous at a point a.
Notation
∫ a in s, f a is measure_theory.integral (s.indicator f)
TODO
The file ends with over a hundred lines of commented out code. This is the old contents of this file
using the indicator approach to the definition of ∫ x in s, f x ∂μ. This code should be
migrated to the new definition.
A function is integrable_on a set s if it is a measurable function and if the integral of
its pointwise norm over s is less than infinity.
Equations
We say that a function f is integrable at filter l if it is integrable on some
set s ∈ l. Equivalently, it is eventually integrable on s in l.lift' powerset.
Equations
- measure_theory.integrable_at_filter f l μ = ∃ (s : set α) (H : s ∈ l), measure_theory.integrable_on f s μ
If μ is a measure finite at filter l and f is a function such that its norm is bounded
above at l, then f is integrable at l.
To prove something for an arbitrary measurable + integrable function in a second countable Borel normed group, it suffices to show that
- the property holds for (multiples of) characteristic functions;
- is closed under addition;
- the set of functions in the
L¹space for which the property holds is closed. - the property is closed under the almost-everywhere equal relation.
It is possible to make the hypotheses in the induction steps a bit stronger, and such conditions
can be added once we need them (for example in h_sum it is only necessary to consider the sum of
a simple function with a multiple of a characteristic function and that the intersection
of their images is a subset of {0}).
For a measurable function f and a measurable set s, the integral of indicator s f
over the whole space is equal to ∫ x in s, f x ∂μ defined as ∫ x, f x ∂(μ.restrict s).
Fundamental theorem of calculus for set integrals: if μ is a measure that is finite
at a filter l and f is a measurable function that has a finite limit b at l ⊓ μ.ae,
then ∫ x in s, f x ∂μ = μ s • b + o(μ s) as s tends to l.lift' powerset. Since μ s is
an ennreal number, we use (μ s).to_real in the actual statement.
If a function is integrable at 𝓝[s] x for each point x of a compact set s, then it is
integrable on s.
A function f continuous on a compact set s is integrable on this set with respect to any
locally finite measure.
A continuous function f is integrable on any compact set with respect to any locally finite
measure.
Fundamental theorem of calculus for set integrals, nhds version: if μ is a locally finite
measure that and f is a measurable function that is continuous at a point a,
then ∫ x in s, f x ∂μ = μ s • f a + o(μ s) as s tends to (𝓝 a).lift' powerset.
Since μ s is an ennreal number, we use (μ s).to_real in the actual statement.
### Continuous linear maps composed with integration
The goal of this section is to prove that integration commutes with continuous linear maps.
The first step is to prove that, given a function φ : α → E which is measurable and integrable,
and a continuous linear map L : E →L[ℝ] F, the function λ a, L(φ a) is also measurable
and integrable. Note we cannot write this as L ∘ φ since the type of L is not an actual
function type.
The next step is translate this to l1, replacing the function φ by a term with type
α →₁[μ] E (an equivalence class of integrable functions).
The corresponding "composition" is L.comp_l1 φ : α →₁[μ] F. This is then upgraded to
a linear map L.comp_l1ₗ : (α →₁[μ] E) →ₗ[ℝ] (α →₁[μ] F) and a continuous linear map
L.comp_l1L : (α →₁[μ] E) →L[ℝ] (α →₁[μ] F).
Then we can prove the commutation result using continuity of all relevant operations and the result on simple functions.
Composing φ : α →₁[μ] E with L : E →L[ℝ] F.
Equations
- L.comp_l1 φ = measure_theory.l1.of_fun (λ (a : α), ⇑L (⇑φ a)) _
Composing φ : α →₁[μ] E with L : E →L[ℝ] F, seen as a ℝ-linear map on α →₁[μ] E.
Composing φ : α →₁[μ] E with L : E →L[ℝ] F, seen as a continuous ℝ-linear map on
α →₁[μ] E.