Documentation

Mathlib.Analysis.Convex.Integral

Jensen's inequality for integrals #

In this file we prove several forms of Jensen's inequality for integrals.

TODO #

Tags #

convex, integral, center mass, average value, Jensen's inequality

Non-strict Jensen's inequality #

theorem Convex.integral_mem {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} [MeasureTheory.IsProbabilityMeasure μ] (hs : Convex s) (hsc : IsClosed s) (hf : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) :
∫ (x : α), f xμ s

If μ is a probability measure on α, s is a convex closed set in E, and f is an integrable function sending μ-a.e. points to s, then the expected value of f belongs to s: ∫ x, f x ∂μ ∈ s. See also Convex.sum_mem for a finite sum version of this lemma.

theorem Convex.average_mem {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} [MeasureTheory.IsFiniteMeasure μ] [NeZero μ] (hs : Convex s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) :
⨍ (x : α), f xμ s

If μ is a non-zero finite measure on α, s is a convex closed set in E, and f is an integrable function sending μ-a.e. points to s, then the average value of f belongs to s: ⨍ x, f x ∂μ ∈ s. See also Convex.centerMass_mem for a finite sum version of this lemma.

theorem Convex.set_average_mem {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} (hs : Convex s) (hsc : IsClosed s) (h0 : μ t 0) (ht : μ t ) (hfs : ∀ᵐ (x : α) ∂μ.restrict t, f x s) (hfi : MeasureTheory.IntegrableOn f t μ) :
⨍ (x : α) in t, f xμ s

If μ is a non-zero finite measure on α, s is a convex closed set in E, and f is an integrable function sending μ-a.e. points to s, then the average value of f belongs to s: ⨍ x, f x ∂μ ∈ s. See also Convex.centerMass_mem for a finite sum version of this lemma.

theorem Convex.set_average_mem_closure {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} (hs : Convex s) (h0 : μ t 0) (ht : μ t ) (hfs : ∀ᵐ (x : α) ∂μ.restrict t, f x s) (hfi : MeasureTheory.IntegrableOn f t μ) :
⨍ (x : α) in t, f xμ closure s

If μ is a non-zero finite measure on α, s is a convex set in E, and f is an integrable function sending μ-a.e. points to s, then the average value of f belongs to closure s: ⨍ x, f x ∂μ ∈ s. See also Convex.centerMass_mem for a finite sum version of this lemma.

theorem ConvexOn.average_mem_epigraph {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsFiniteMeasure μ] [NeZero μ] (hg : ConvexOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
(⨍ (x : α), f xμ, ⨍ (x : α), g (f x)μ) {p : E × | p.1 s g p.1 p.2}
theorem ConcaveOn.average_mem_hypograph {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsFiniteMeasure μ] [NeZero μ] (hg : ConcaveOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
(⨍ (x : α), f xμ, ⨍ (x : α), g (f x)μ) {p : E × | p.1 s p.2 g p.1}
theorem ConvexOn.map_average_le {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsFiniteMeasure μ] [NeZero μ] (hg : ConvexOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
g (⨍ (x : α), f xμ) ⨍ (x : α), g (f x)μ

Jensen's inequality: if a function g : E → ℝ is convex and continuous on a convex closed set s, μ is a finite non-zero measure on α, and f : α → E is a function sending μ-a.e. points to s, then the value of g at the average value of f is less than or equal to the average value of g ∘ f provided that both f and g ∘ f are integrable. See also ConvexOn.map_centerMass_le for a finite sum version of this lemma.

theorem ConcaveOn.le_map_average {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsFiniteMeasure μ] [NeZero μ] (hg : ConcaveOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
⨍ (x : α), g (f x)μ g (⨍ (x : α), f xμ)

Jensen's inequality: if a function g : E → ℝ is concave and continuous on a convex closed set s, μ is a finite non-zero measure on α, and f : α → E is a function sending μ-a.e. points to s, then the average value of g ∘ f is less than or equal to the value of g at the average value of f provided that both f and g ∘ f are integrable. See also ConcaveOn.le_map_centerMass for a finite sum version of this lemma.

theorem ConvexOn.set_average_mem_epigraph {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} {g : E} (hg : ConvexOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (h0 : μ t 0) (ht : μ t ) (hfs : ∀ᵐ (x : α) ∂μ.restrict t, f x s) (hfi : MeasureTheory.IntegrableOn f t μ) (hgi : MeasureTheory.IntegrableOn (g f) t μ) :
(⨍ (x : α) in t, f xμ, ⨍ (x : α) in t, g (f x)μ) {p : E × | p.1 s g p.1 p.2}

Jensen's inequality: if a function g : E → ℝ is convex and continuous on a convex closed set s, μ is a finite non-zero measure on α, and f : α → E is a function sending μ-a.e. points of a set t to s, then the value of g at the average value of f over t is less than or equal to the average value of g ∘ f over t provided that both f and g ∘ f are integrable.

theorem ConcaveOn.set_average_mem_hypograph {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} {g : E} (hg : ConcaveOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (h0 : μ t 0) (ht : μ t ) (hfs : ∀ᵐ (x : α) ∂μ.restrict t, f x s) (hfi : MeasureTheory.IntegrableOn f t μ) (hgi : MeasureTheory.IntegrableOn (g f) t μ) :
(⨍ (x : α) in t, f xμ, ⨍ (x : α) in t, g (f x)μ) {p : E × | p.1 s p.2 g p.1}

Jensen's inequality: if a function g : E → ℝ is concave and continuous on a convex closed set s, μ is a finite non-zero measure on α, and f : α → E is a function sending μ-a.e. points of a set t to s, then the average value of g ∘ f over t is less than or equal to the value of g at the average value of f over t provided that both f and g ∘ f are integrable.

theorem ConvexOn.map_set_average_le {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} {g : E} (hg : ConvexOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (h0 : μ t 0) (ht : μ t ) (hfs : ∀ᵐ (x : α) ∂μ.restrict t, f x s) (hfi : MeasureTheory.IntegrableOn f t μ) (hgi : MeasureTheory.IntegrableOn (g f) t μ) :
g (⨍ (x : α) in t, f xμ) ⨍ (x : α) in t, g (f x)μ

Jensen's inequality: if a function g : E → ℝ is convex and continuous on a convex closed set s, μ is a finite non-zero measure on α, and f : α → E is a function sending μ-a.e. points of a set t to s, then the value of g at the average value of f over t is less than or equal to the average value of g ∘ f over t provided that both f and g ∘ f are integrable.

theorem ConcaveOn.le_map_set_average {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} {g : E} (hg : ConcaveOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (h0 : μ t 0) (ht : μ t ) (hfs : ∀ᵐ (x : α) ∂μ.restrict t, f x s) (hfi : MeasureTheory.IntegrableOn f t μ) (hgi : MeasureTheory.IntegrableOn (g f) t μ) :
⨍ (x : α) in t, g (f x)μ g (⨍ (x : α) in t, f xμ)

Jensen's inequality: if a function g : E → ℝ is concave and continuous on a convex closed set s, μ is a finite non-zero measure on α, and f : α → E is a function sending μ-a.e. points of a set t to s, then the average value of g ∘ f over t is less than or equal to the value of g at the average value of f over t provided that both f and g ∘ f are integrable.

theorem ConvexOn.map_integral_le {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsProbabilityMeasure μ] (hg : ConvexOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
g (∫ (x : α), f xμ) ∫ (x : α), g (f x)μ

Jensen's inequality: if a function g : E → ℝ is convex and continuous on a convex closed set s, μ is a probability measure on α, and f : α → E is a function sending μ-a.e. points to s, then the value of g at the expected value of f is less than or equal to the expected value of g ∘ f provided that both f and g ∘ f are integrable. See also ConvexOn.map_centerMass_le for a finite sum version of this lemma.

theorem ConcaveOn.le_map_integral {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsProbabilityMeasure μ] (hg : ConcaveOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
∫ (x : α), g (f x)μ g (∫ (x : α), f xμ)

Jensen's inequality: if a function g : E → ℝ is concave and continuous on a convex closed set s, μ is a probability measure on α, and f : α → E is a function sending μ-a.e. points to s, then the expected value of g ∘ f is less than or equal to the value of g at the expected value of f provided that both f and g ∘ f are integrable.

Strict Jensen's inequality #

theorem ae_eq_const_or_exists_average_ne_compl {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {f : αE} [MeasureTheory.IsFiniteMeasure μ] (hfi : MeasureTheory.Integrable f μ) :
μ.ae.EventuallyEq f (Function.const α (⨍ (x : α), f xμ)) ∃ (t : Set α), MeasurableSet t μ t 0 μ t 0 ⨍ (x : α) in t, f xμ ⨍ (x : α) in t, f xμ

If f : α → E is an integrable function, then either it is a.e. equal to the constant ⨍ x, f x ∂μ or there exists a measurable set such that μ t ≠ 0, μ tᶜ ≠ 0, and the average values of f over t and tᶜ are different.

theorem Convex.average_mem_interior_of_set {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {t : Set α} {f : αE} [MeasureTheory.IsFiniteMeasure μ] (hs : Convex s) (h0 : μ t 0) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (ht : ⨍ (x : α) in t, f xμ interior s) :
⨍ (x : α), f xμ interior s

If an integrable function f : α → E takes values in a convex set s and for some set t of positive measure, the average value of f over t belongs to the interior of s, then the average of f over the whole space belongs to the interior of s.

theorem StrictConvex.ae_eq_const_or_average_mem_interior {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} [MeasureTheory.IsFiniteMeasure μ] (hs : StrictConvex s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) :
μ.ae.EventuallyEq f (Function.const α (⨍ (x : α), f xμ)) ⨍ (x : α), f xμ interior s

If an integrable function f : α → E takes values in a strictly convex closed set s, then either it is a.e. equal to its average value, or its average value belongs to the interior of s.

theorem StrictConvexOn.ae_eq_const_or_map_average_lt {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsFiniteMeasure μ] (hg : StrictConvexOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
μ.ae.EventuallyEq f (Function.const α (⨍ (x : α), f xμ)) g (⨍ (x : α), f xμ) < ⨍ (x : α), g (f x)μ

Jensen's inequality, strict version: if an integrable function f : α → E takes values in a convex closed set s, and g : E → ℝ is continuous and strictly convex on s, then either f is a.e. equal to its average value, or g (⨍ x, f x ∂μ) < ⨍ x, g (f x) ∂μ.

theorem StrictConcaveOn.ae_eq_const_or_lt_map_average {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {s : Set E} {f : αE} {g : E} [MeasureTheory.IsFiniteMeasure μ] (hg : StrictConcaveOn s g) (hgc : ContinuousOn g s) (hsc : IsClosed s) (hfs : ∀ᵐ (x : α) ∂μ, f x s) (hfi : MeasureTheory.Integrable f μ) (hgi : MeasureTheory.Integrable (g f) μ) :
μ.ae.EventuallyEq f (Function.const α (⨍ (x : α), f xμ)) ⨍ (x : α), g (f x)μ < g (⨍ (x : α), f xμ)

Jensen's inequality, strict version: if an integrable function f : α → E takes values in a convex closed set s, and g : E → ℝ is continuous and strictly concave on s, then either f is a.e. equal to its average value, or ⨍ x, g (f x) ∂μ < g (⨍ x, f x ∂μ).

theorem ae_eq_const_or_norm_average_lt_of_norm_le_const {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {f : αE} {C : } [StrictConvexSpace E] (h_le : ∀ᵐ (x : α) ∂μ, f x C) :
μ.ae.EventuallyEq f (Function.const α (⨍ (x : α), f xμ)) ⨍ (x : α), f xμ < C

If E is a strictly convex normed space and f : α → E is a function such that ‖f x‖ ≤ C a.e., then either this function is a.e. equal to its average value, or the norm of its average value is strictly less than C.

theorem ae_eq_const_or_norm_integral_lt_of_norm_le_const {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {f : αE} {C : } [StrictConvexSpace E] [MeasureTheory.IsFiniteMeasure μ] (h_le : ∀ᵐ (x : α) ∂μ, f x C) :
μ.ae.EventuallyEq f (Function.const α (⨍ (x : α), f xμ)) ∫ (x : α), f xμ < (μ Set.univ).toReal * C

If E is a strictly convex normed space and f : α → E is a function such that ‖f x‖ ≤ C a.e., then either this function is a.e. equal to its average value, or the norm of its integral is strictly less than (μ univ).toReal * C.

theorem ae_eq_const_or_norm_setIntegral_lt_of_norm_le_const {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {t : Set α} {f : αE} {C : } [StrictConvexSpace E] (ht : μ t ) (h_le : ∀ᵐ (x : α) ∂μ.restrict t, f x C) :
(μ.restrict t).ae.EventuallyEq f (Function.const α (⨍ (x : α) in t, f xμ)) ∫ (x : α) in t, f xμ < (μ t).toReal * C

If E is a strictly convex normed space and f : α → E is a function such that ‖f x‖ ≤ C a.e. on a set t of finite measure, then either this function is a.e. equal to its average value on t, or the norm of its integral over t is strictly less than (μ t).toReal * C.

@[deprecated ae_eq_const_or_norm_setIntegral_lt_of_norm_le_const]
theorem ae_eq_const_or_norm_set_integral_lt_of_norm_le_const {α : Type u_1} {E : Type u_2} {m0 : MeasurableSpace α} [NormedAddCommGroup E] [NormedSpace E] [CompleteSpace E] {μ : MeasureTheory.Measure α} {t : Set α} {f : αE} {C : } [StrictConvexSpace E] (ht : μ t ) (h_le : ∀ᵐ (x : α) ∂μ.restrict t, f x C) :
(μ.restrict t).ae.EventuallyEq f (Function.const α (⨍ (x : α) in t, f xμ)) ∫ (x : α) in t, f xμ < (μ t).toReal * C

Alias of ae_eq_const_or_norm_setIntegral_lt_of_norm_le_const.


If E is a strictly convex normed space and f : α → E is a function such that ‖f x‖ ≤ C a.e. on a set t of finite measure, then either this function is a.e. equal to its average value on t, or the norm of its integral over t is strictly less than (μ t).toReal * C.