Conditional expectation in L1 #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains two more steps of the construction of the conditional expectation, which is
completed in measure_theory.function.conditional_expectation.basic
. See that file for a
description of the full process.
The contitional expectation of an L²
function is defined in
measure_theory.function.conditional_expectation.condexp_L2
. In this file, we perform two steps.
- Show that the conditional expectation of the indicator of a measurable set with finite measure
is integrable and define a map
set α → (E →L[ℝ] (α →₁[μ] E))
which to a set associates a linear map. That linear map sendsx ∈ E
to the conditional expectation of the indicator of the set with valuex
. - Extend that map to
condexp_L1_clm : (α →₁[μ] E) →L[ℝ] (α →₁[μ] E)
. This is done using the same construction as the Bochner integral (see the filemeasure_theory/integral/set_to_L1
).
Main definitions #
condexp_L1
: Conditional expectation of a function as a linear map fromL1
to itself.
Conditional expectation of an indicator as a continuous linear map. #
The goal of this section is to build
condexp_ind (hm : m ≤ m0) (μ : measure α) (s : set s) : G →L[ℝ] α →₁[μ] G
, which
takes x : G
to the conditional expectation of the indicator of the set s
with value x
,
seen as an element of α →₁[μ] G
.
Conditional expectation of the indicator of a measurable set with finite measure, as a function in L1.
Equations
- measure_theory.condexp_ind_L1_fin hm hs hμs x = measure_theory.integrable.to_L1 ⇑(measure_theory.condexp_ind_smul hm hs hμs x) _
Conditional expectation of the indicator of a set, as a function in L1. Its value for sets which are not both measurable and of finite measure is not used: we set it to 0.
Equations
- measure_theory.condexp_ind_L1 hm μ s x = dite (measurable_set s ∧ ⇑μ s ≠ ⊤) (λ (hs : measurable_set s ∧ ⇑μ s ≠ ⊤), measure_theory.condexp_ind_L1_fin hm _ _ x) (λ (hs : ¬(measurable_set s ∧ ⇑μ s ≠ ⊤)), 0)
Conditional expectation of the indicator of a set, as a linear map from G
to L1.
Equations
- measure_theory.condexp_ind hm μ s = {to_linear_map := {to_fun := measure_theory.condexp_ind_L1 hm μ s _inst_13, map_add' := _, map_smul' := _}, cont := _}
Conditional expectation of a function as a linear map from α →₁[μ] F'
to itself.
Equations
Auxiliary lemma used in the proof of set_integral_condexp_L1_clm
.
The integral of the conditional expectation condexp_L1_clm
over an m
-measurable set is equal
to the integral of f
on that set. See also set_integral_condexp
, the similar statement for
condexp
.
Conditional expectation of a function, in L1. Its value is 0 if the function is not
integrable. The function-valued condexp
should be used instead in most cases.
Equations
- measure_theory.condexp_L1 hm μ f = measure_theory.set_to_fun μ (measure_theory.condexp_ind hm μ) _ f
The integral of the conditional expectation condexp_L1
over an m
-measurable set is equal to
the integral of f
on that set. See also set_integral_condexp
, the similar statement for
condexp
.