Documentation

Mathlib.MeasureTheory.Function.ConditionalExpectation.CondexpL1

Conditional expectation in L1 #

This file contains two more steps of the construction of the conditional expectation, which is completed in MeasureTheory.Function.ConditionalExpectation.Basic. See that file for a description of the full process.

The conditional expectation of an function is defined in MeasureTheory.Function.ConditionalExpectation.CondexpL2. In this file, we perform two steps.

Main definitions #

Conditional expectation of an indicator as a continuous linear map. #

The goal of this section is to build condexpInd (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.

def MeasureTheory.condexpIndL1Fin {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] (hm : m m0) [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x : G) :
(Lp G 1 μ)

Conditional expectation of the indicator of a measurable set with finite measure, as a function in L1.

Equations
Instances For
    theorem MeasureTheory.condexpIndL1Fin_ae_eq_condexpIndSMul {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] (hm : m m0) [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x : G) :
    (condexpIndL1Fin hm hs hμs x) =ᶠ[ae μ] (condexpIndSMul hm hs hμs x)
    theorem MeasureTheory.condexpIndL1Fin_add {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x y : G) :
    condexpIndL1Fin hm hs hμs (x + y) = condexpIndL1Fin hm hs hμs x + condexpIndL1Fin hm hs hμs y
    theorem MeasureTheory.condexpIndL1Fin_smul {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (c : ) (x : G) :
    condexpIndL1Fin hm hs hμs (c x) = c condexpIndL1Fin hm hs hμs x
    theorem MeasureTheory.condexpIndL1Fin_smul' {α : Type u_1} {F : Type u_2} {𝕜 : Type u_6} [RCLike 𝕜] [NormedAddCommGroup F] [NormedSpace 𝕜 F] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} {hm : m m0} [SigmaFinite (μ.trim hm)] [NormedSpace F] [SMulCommClass 𝕜 F] (hs : MeasurableSet s) (hμs : μ s ) (c : 𝕜) (x : F) :
    condexpIndL1Fin hm hs hμs (c x) = c condexpIndL1Fin hm hs hμs x
    theorem MeasureTheory.norm_condexpIndL1Fin_le {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x : G) :
    condexpIndL1Fin hm hs hμs x (μ s).toReal * x
    theorem MeasureTheory.condexpIndL1Fin_disjoint_union {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s t : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (ht : MeasurableSet t) (hμs : μ s ) (hμt : μ t ) (hst : Disjoint s t) (x : G) :
    condexpIndL1Fin hm x = condexpIndL1Fin hm hs hμs x + condexpIndL1Fin hm ht hμt x
    def MeasureTheory.condexpIndL1 {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] [NormedSpace G] {m m0 : MeasurableSpace α} (hm : m m0) (μ : Measure α) (s : Set α) [SigmaFinite (μ.trim hm)] (x : G) :
    (Lp G 1 μ)

    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
    Instances For
      theorem MeasureTheory.condexpIndL1_of_measurableSet_of_measure_ne_top {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x : G) :
      condexpIndL1 hm μ s x = condexpIndL1Fin hm hs hμs x
      theorem MeasureTheory.condexpIndL1_of_measure_eq_top {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hμs : μ s = ) (x : G) :
      condexpIndL1 hm μ s x = 0
      theorem MeasureTheory.condexpIndL1_of_not_measurableSet {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : ¬MeasurableSet s) (x : G) :
      condexpIndL1 hm μ s x = 0
      theorem MeasureTheory.condexpIndL1_add {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (x y : G) :
      condexpIndL1 hm μ s (x + y) = condexpIndL1 hm μ s x + condexpIndL1 hm μ s y
      theorem MeasureTheory.condexpIndL1_smul {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (c : ) (x : G) :
      condexpIndL1 hm μ s (c x) = c condexpIndL1 hm μ s x
      theorem MeasureTheory.condexpIndL1_smul' {α : Type u_1} {F : Type u_2} {𝕜 : Type u_6} [RCLike 𝕜] [NormedAddCommGroup F] [NormedSpace 𝕜 F] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} {hm : m m0} [SigmaFinite (μ.trim hm)] [NormedSpace F] [SMulCommClass 𝕜 F] (c : 𝕜) (x : F) :
      condexpIndL1 hm μ s (c x) = c condexpIndL1 hm μ s x
      theorem MeasureTheory.norm_condexpIndL1_le {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (x : G) :
      condexpIndL1 hm μ s x (μ s).toReal * x
      theorem MeasureTheory.continuous_condexpIndL1 {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] :
      Continuous fun (x : G) => condexpIndL1 hm μ s x
      theorem MeasureTheory.condexpIndL1_disjoint_union {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s t : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (ht : MeasurableSet t) (hμs : μ s ) (hμt : μ t ) (hst : Disjoint s t) (x : G) :
      condexpIndL1 hm μ (s t) x = condexpIndL1 hm μ s x + condexpIndL1 hm μ t x
      def MeasureTheory.condexpInd {α : Type u_1} (G : Type u_4) [NormedAddCommGroup G] [NormedSpace G] {m m0 : MeasurableSpace α} (hm : m m0) (μ : Measure α) [SigmaFinite (μ.trim hm)] (s : Set α) :
      G →L[] (Lp G 1 μ)

      Conditional expectation of the indicator of a set, as a linear map from G to L1.

      Equations
      Instances For
        theorem MeasureTheory.condexpInd_ae_eq_condexpIndSMul {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] (hm : m m0) [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x : G) :
        ((condexpInd G hm μ s) x) =ᶠ[ae μ] (condexpIndSMul hm hs hμs x)
        theorem MeasureTheory.aestronglyMeasurable'_condexpInd {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (x : G) :
        AEStronglyMeasurable' m (↑((condexpInd G hm μ s) x)) μ
        @[simp]
        theorem MeasureTheory.condexpInd_empty {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] :
        condexpInd G hm μ = 0
        theorem MeasureTheory.condexpInd_smul' {α : Type u_1} {F : Type u_2} {𝕜 : Type u_6} [RCLike 𝕜] [NormedAddCommGroup F] [NormedSpace 𝕜 F] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} {hm : m m0} [SigmaFinite (μ.trim hm)] [NormedSpace F] [SMulCommClass 𝕜 F] (c : 𝕜) (x : F) :
        (condexpInd F hm μ s) (c x) = c (condexpInd F hm μ s) x
        theorem MeasureTheory.norm_condexpInd_apply_le {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (x : G) :
        (condexpInd G hm μ s) x (μ s).toReal * x
        theorem MeasureTheory.norm_condexpInd_le {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] :
        condexpInd G hm μ s (μ s).toReal
        theorem MeasureTheory.condexpInd_disjoint_union_apply {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s t : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (ht : MeasurableSet t) (hμs : μ s ) (hμt : μ t ) (hst : Disjoint s t) (x : G) :
        (condexpInd G hm μ (s t)) x = (condexpInd G hm μ s) x + (condexpInd G hm μ t) x
        theorem MeasureTheory.condexpInd_disjoint_union {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s t : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (ht : MeasurableSet t) (hμs : μ s ) (hμt : μ t ) (hst : Disjoint s t) :
        condexpInd G hm μ (s t) = condexpInd G hm μ s + condexpInd G hm μ t
        theorem MeasureTheory.dominatedFinMeasAdditive_condexpInd {α : Type u_1} (G : Type u_4) [NormedAddCommGroup G] {m m0 : MeasurableSpace α} [NormedSpace G] (hm : m m0) (μ : Measure α) [SigmaFinite (μ.trim hm)] :
        theorem MeasureTheory.setIntegral_condexpInd {α : Type u_1} {G' : Type u_5} [NormedAddCommGroup G'] [NormedSpace G'] [CompleteSpace G'] {m m0 : MeasurableSpace α} {μ : Measure α} {s t : Set α} {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (ht : MeasurableSet t) (hμs : μ s ) (hμt : μ t ) (x : G') :
        (a : α) in s, ((condexpInd G' hm μ t) x) a μ = (μ (t s)).toReal x
        @[deprecated MeasureTheory.setIntegral_condexpInd (since := "2024-04-17")]
        theorem MeasureTheory.set_integral_condexpInd {α : Type u_1} {G' : Type u_5} [NormedAddCommGroup G'] [NormedSpace G'] [CompleteSpace G'] {m m0 : MeasurableSpace α} {μ : Measure α} {s t : Set α} {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (ht : MeasurableSet t) (hμs : μ s ) (hμt : μ t ) (x : G') :
        (a : α) in s, ((condexpInd G' hm μ t) x) a μ = (μ (t s)).toReal x

        Alias of MeasureTheory.setIntegral_condexpInd.

        theorem MeasureTheory.condexpInd_of_measurable {α : Type u_1} {G : Type u_4} [NormedAddCommGroup G] {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} [NormedSpace G] {hm : m m0} [SigmaFinite (μ.trim hm)] (hs : MeasurableSet s) (hμs : μ s ) (c : G) :
        (condexpInd G hm μ s) c = indicatorConstLp 1 hμs c
        theorem MeasureTheory.condexpInd_nonneg {α : Type u_1} {m m0 : MeasurableSpace α} {μ : Measure α} {s : Set α} {hm : m m0} [SigmaFinite (μ.trim hm)] {E : Type u_7} [NormedLatticeAddCommGroup E] [NormedSpace E] [OrderedSMul E] (hs : MeasurableSet s) (hμs : μ s ) (x : E) (hx : 0 x) :
        0 (condexpInd E hm μ s) x
        def MeasureTheory.condexpL1CLM {α : Type u_1} (F' : Type u_3) [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} (hm : m m0) (μ : Measure α) [SigmaFinite (μ.trim hm)] :
        (Lp F' 1 μ) →L[] (Lp F' 1 μ)

        Conditional expectation of a function as a linear map from α →₁[μ] F' to itself.

        Equations
        Instances For
          theorem MeasureTheory.condexpL1CLM_smul {α : Type u_1} {F' : Type u_3} {𝕜 : Type u_6} [RCLike 𝕜] [NormedAddCommGroup F'] [NormedSpace 𝕜 F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (c : 𝕜) (f : (Lp F' 1 μ)) :
          (condexpL1CLM F' hm μ) (c f) = c (condexpL1CLM F' hm μ) f
          theorem MeasureTheory.condexpL1CLM_indicatorConstLp {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {s : Set α} (hs : MeasurableSet s) (hμs : μ s ) (x : F') :
          (condexpL1CLM F' hm μ) (indicatorConstLp 1 hs hμs x) = (condexpInd F' hm μ s) x
          theorem MeasureTheory.condexpL1CLM_indicatorConst {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {s : Set α} (hs : MeasurableSet s) (hμs : μ s ) (x : F') :
          (condexpL1CLM F' hm μ) (Lp.simpleFunc.indicatorConst 1 hs hμs x) = (condexpInd F' hm μ s) x
          theorem MeasureTheory.setIntegral_condexpL1CLM_of_measure_ne_top {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {s : Set α} (f : (Lp F' 1 μ)) (hs : MeasurableSet s) (hμs : μ s ) :
          (x : α) in s, ((condexpL1CLM F' hm μ) f) x μ = (x : α) in s, f x μ

          Auxiliary lemma used in the proof of setIntegral_condexpL1CLM.

          @[deprecated MeasureTheory.setIntegral_condexpL1CLM_of_measure_ne_top (since := "2024-04-17")]
          theorem MeasureTheory.set_integral_condexpL1CLM_of_measure_ne_top {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {s : Set α} (f : (Lp F' 1 μ)) (hs : MeasurableSet s) (hμs : μ s ) :
          (x : α) in s, ((condexpL1CLM F' hm μ) f) x μ = (x : α) in s, f x μ

          Alias of MeasureTheory.setIntegral_condexpL1CLM_of_measure_ne_top.


          Auxiliary lemma used in the proof of setIntegral_condexpL1CLM.

          theorem MeasureTheory.setIntegral_condexpL1CLM {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {s : Set α} (f : (Lp F' 1 μ)) (hs : MeasurableSet s) :
          (x : α) in s, ((condexpL1CLM F' hm μ) f) x μ = (x : α) in s, f x μ

          The integral of the conditional expectation condexpL1CLM over an m-measurable set is equal to the integral of f on that set. See also setIntegral_condexp, the similar statement for condexp.

          @[deprecated MeasureTheory.setIntegral_condexpL1CLM (since := "2024-04-17")]
          theorem MeasureTheory.set_integral_condexpL1CLM {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {s : Set α} (f : (Lp F' 1 μ)) (hs : MeasurableSet s) :
          (x : α) in s, ((condexpL1CLM F' hm μ) f) x μ = (x : α) in s, f x μ

          Alias of MeasureTheory.setIntegral_condexpL1CLM.


          The integral of the conditional expectation condexpL1CLM over an m-measurable set is equal to the integral of f on that set. See also setIntegral_condexp, the similar statement for condexp.

          theorem MeasureTheory.aestronglyMeasurable'_condexpL1CLM {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (f : (Lp F' 1 μ)) :
          AEStronglyMeasurable' m (↑((condexpL1CLM F' hm μ) f)) μ
          theorem MeasureTheory.condexpL1CLM_lpMeas {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (f : (lpMeas F' m 1 μ)) :
          (condexpL1CLM F' hm μ) f = f
          theorem MeasureTheory.condexpL1CLM_of_aestronglyMeasurable' {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (f : (Lp F' 1 μ)) (hfm : AEStronglyMeasurable' m (↑f) μ) :
          (condexpL1CLM F' hm μ) f = f
          def MeasureTheory.condexpL1 {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} (hm : m m0) (μ : Measure α) [SigmaFinite (μ.trim hm)] (f : αF') :
          (Lp F' 1 μ)

          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
          Instances For
            theorem MeasureTheory.condexpL1_undef {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f : αF'} (hf : ¬Integrable f μ) :
            condexpL1 hm μ f = 0
            theorem MeasureTheory.condexpL1_eq {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f : αF'} (hf : Integrable f μ) :
            condexpL1 hm μ f = (condexpL1CLM F' hm μ) (Integrable.toL1 f hf)
            @[simp]
            theorem MeasureTheory.condexpL1_zero {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] :
            condexpL1 hm μ 0 = 0
            @[simp]
            theorem MeasureTheory.condexpL1_measure_zero {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {f : αF'} (hm : m m0) :
            condexpL1 hm 0 f = 0
            theorem MeasureTheory.aestronglyMeasurable'_condexpL1 {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f : αF'} :
            AEStronglyMeasurable' m (↑(condexpL1 hm μ f)) μ
            theorem MeasureTheory.condexpL1_congr_ae {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {f g : αF'} (hm : m m0) [SigmaFinite (μ.trim hm)] (h : f =ᶠ[ae μ] g) :
            condexpL1 hm μ f = condexpL1 hm μ g
            theorem MeasureTheory.integrable_condexpL1 {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (f : αF') :
            Integrable (↑(condexpL1 hm μ f)) μ
            theorem MeasureTheory.setIntegral_condexpL1 {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f : αF'} {s : Set α} (hf : Integrable f μ) (hs : MeasurableSet s) :
            (x : α) in s, (condexpL1 hm μ f) x μ = (x : α) in s, f x μ

            The integral of the conditional expectation condexpL1 over an m-measurable set is equal to the integral of f on that set. See also setIntegral_condexp, the similar statement for condexp.

            @[deprecated MeasureTheory.setIntegral_condexpL1 (since := "2024-04-17")]
            theorem MeasureTheory.set_integral_condexpL1 {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f : αF'} {s : Set α} (hf : Integrable f μ) (hs : MeasurableSet s) :
            (x : α) in s, (condexpL1 hm μ f) x μ = (x : α) in s, f x μ

            Alias of MeasureTheory.setIntegral_condexpL1.


            The integral of the conditional expectation condexpL1 over an m-measurable set is equal to the integral of f on that set. See also setIntegral_condexp, the similar statement for condexp.

            theorem MeasureTheory.condexpL1_add {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f g : αF'} (hf : Integrable f μ) (hg : Integrable g μ) :
            condexpL1 hm μ (f + g) = condexpL1 hm μ f + condexpL1 hm μ g
            theorem MeasureTheory.condexpL1_neg {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (f : αF') :
            condexpL1 hm μ (-f) = -condexpL1 hm μ f
            theorem MeasureTheory.condexpL1_smul {α : Type u_1} {F' : Type u_3} {𝕜 : Type u_6} [RCLike 𝕜] [NormedAddCommGroup F'] [NormedSpace 𝕜 F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] (c : 𝕜) (f : αF') :
            condexpL1 hm μ (c f) = c condexpL1 hm μ f
            theorem MeasureTheory.condexpL1_sub {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f g : αF'} (hf : Integrable f μ) (hg : Integrable g μ) :
            condexpL1 hm μ (f - g) = condexpL1 hm μ f - condexpL1 hm μ g
            theorem MeasureTheory.condexpL1_of_aestronglyMeasurable' {α : Type u_1} {F' : Type u_3} [NormedAddCommGroup F'] [NormedSpace F'] [CompleteSpace F'] {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {f : αF'} (hfm : AEStronglyMeasurable' m f μ) (hfi : Integrable f μ) :
            (condexpL1 hm μ f) =ᶠ[ae μ] f
            theorem MeasureTheory.condexpL1_mono {α : Type u_1} {m m0 : MeasurableSpace α} {μ : Measure α} {hm : m m0} [SigmaFinite (μ.trim hm)] {E : Type u_7} [NormedLatticeAddCommGroup E] [CompleteSpace E] [NormedSpace E] [OrderedSMul E] {f g : αE} (hf : Integrable f μ) (hg : Integrable g μ) (hfg : f ≤ᶠ[ae μ] g) :
            (condexpL1 hm μ f) ≤ᶠ[ae μ] (condexpL1 hm μ g)