Mean value inequalities for integrals #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove several inequalities on integrals, notably the Hölder inequality and
the Minkowski inequality. The versions for finite sums are in analysis.mean_inequalities
.
Main results #
Hölder's inequality for the Lebesgue integral of ℝ≥0∞
and ℝ≥0
functions: we prove
∫ (f * g) ∂μ ≤ (∫ f^p ∂μ) ^ (1/p) * (∫ g^q ∂μ) ^ (1/q)
for p
, q
conjugate real exponents
and α→(e)nnreal
functions in two cases,
ennreal.lintegral_mul_le_Lp_mul_Lq
: ℝ≥0∞ functions,nnreal.lintegral_mul_le_Lp_mul_Lq
: ℝ≥0 functions.
Minkowski's inequality for the Lebesgue integral of measurable functions with ℝ≥0∞
values:
we prove (∫ (f + g)^p ∂μ) ^ (1/p) ≤ (∫ f^p ∂μ) ^ (1/p) + (∫ g^p ∂μ) ^ (1/p)
for 1 ≤ p
.
Hölder's inequality for the Lebesgue integral of ℝ≥0∞ and nnreal functions #
We prove ∫ (f * g) ∂μ ≤ (∫ f^p ∂μ) ^ (1/p) * (∫ g^q ∂μ) ^ (1/q)
for p
, q
conjugate real exponents and α→(e)nnreal
functions in several cases, the first two being useful
only to prove the more general results:
ennreal.lintegral_mul_le_one_of_lintegral_rpow_eq_one
: ℝ≥0∞ functions for which the integrals on the right are equal to 1,ennreal.lintegral_mul_le_Lp_mul_Lq_of_ne_zero_of_ne_top
: ℝ≥0∞ functions for which the integrals on the right are neither ⊤ nor 0,ennreal.lintegral_mul_le_Lp_mul_Lq
: ℝ≥0∞ functions,nnreal.lintegral_mul_le_Lp_mul_Lq
: nnreal functions.
Function multiplied by the inverse of its p-seminorm (∫⁻ f^p ∂μ) ^ 1/p
Hölder's inequality in case of finite non-zero integrals
Hölder's inequality for functions α → ℝ≥0∞
. The integral of the product of two functions
is bounded by the product of their ℒp
and ℒq
seminorms when p
and q
are conjugate
exponents.
Minkowski's inequality for functions α → ℝ≥0∞
: the ℒp
seminorm of the sum of two
functions is bounded by the sum of their ℒp
seminorms.
Variant of Minkowski's inequality for functions α → ℝ≥0∞
in ℒp
with p ≤ 1
: the ℒp
seminorm of the sum of two functions is bounded by a constant multiple of the sum
of their ℒp
seminorms.
Hölder's inequality for functions α → ℝ≥0
. The integral of the product of two functions
is bounded by the product of their ℒp
and ℒq
seminorms when p
and q
are conjugate
exponents.