mathlib3 documentation

analysis.mean_inequalities

Mean value inequalities #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

In this file we prove several inequalities for finite sums, including AM-GM inequality, Young's inequality, Hölder inequality, and Minkowski inequality. Versions for integrals of some of these inequalities are available in measure_theory.mean_inequalities.

Main theorems #

AM-GM inequality: #

The inequality says that the geometric mean of a tuple of non-negative numbers is less than or equal to their arithmetic mean. We prove the weighted version of this inequality: if $w$ and $z$ are two non-negative vectors and $\sum_{i\in s} w_i=1$, then $$ \prod_{i\in s} z_i^{w_i} ≤ \sum_{i\in s} w_iz_i. $$ The classical version is a special case of this inequality for $w_i=\frac{1}{n}$.

We prove a few versions of this inequality. Each of the following lemmas comes in two versions: a version for real-valued non-negative functions is in the real namespace, and a version for nnreal-valued functions is in the nnreal namespace.

Young's inequality #

Young's inequality says that for non-negative numbers a, b, p, q such that $\frac{1}{p}+\frac{1}{q}=1$ we have $$ ab ≤ \frac{a^p}{p} + \frac{b^q}{q}. $$

This inequality is a special case of the AM-GM inequality. It is then used to prove Hölder's inequality (see below).

Hölder's inequality #

The inequality says that for two conjugate exponents p and q (i.e., for two positive numbers such that $\frac{1}{p}+\frac{1}{q}=1$) and any two non-negative vectors their inner product is less than or equal to the product of the $L_p$ norm of the first vector and the $L_q$ norm of the second vector: $$ \sum_{i\in s} a_ib_i ≤ \sqrt[p]{\sum_{i\in s} a_i^p}\sqrt[q]{\sum_{i\in s} b_i^q}. $$

We give versions of this result in , ℝ≥0 and ℝ≥0∞.

There are at least two short proofs of this inequality. In our proof we prenormalize both vectors, then apply Young's inequality to each $a_ib_i$. Another possible proof would be to deduce this inequality from the generalized mean inequality for well-chosen vectors and weights.

Minkowski's inequality #

The inequality says that for p ≥ 1 the function $$ \|a\|_p=\sqrt[p]{\sum_{i\in s} a_i^p} $$ satisfies the triangle inequality $\|a+b\|_p\le \|a\|_p+\|b\|_p$.

We give versions of this result in real, ℝ≥0 and ℝ≥0∞.

We deduce this inequality from Hölder's inequality. Namely, Hölder inequality implies that $\|a\|_p$ is the maximum of the inner product $\sum_{i\in s}a_ib_i$ over b such that $\|b\|_q\le 1$. Now Minkowski's inequality follows from the fact that the maximum value of the sum of two functions is less than or equal to the sum of the maximum values of the summands.

TODO #

AM-GM inequality #

theorem real.geom_mean_le_arith_mean_weighted {ι : Type u} (s : finset ι) (w z : ι ) (hw : (i : ι), i s 0 w i) (hw' : s.sum (λ (i : ι), w i) = 1) (hz : (i : ι), i s 0 z i) :
s.prod (λ (i : ι), z i ^ w i) s.sum (λ (i : ι), w i * z i)

AM-GM inequality: the geometric mean is less than or equal to the arithmetic mean, weighted version for real-valued nonnegative functions.

theorem real.geom_mean_weighted_of_constant {ι : Type u} (s : finset ι) (w z : ι ) (x : ) (hw : (i : ι), i s 0 w i) (hw' : s.sum (λ (i : ι), w i) = 1) (hz : (i : ι), i s 0 z i) (hx : (i : ι), i s w i 0 z i = x) :
s.prod (λ (i : ι), z i ^ w i) = x
theorem real.arith_mean_weighted_of_constant {ι : Type u} (s : finset ι) (w z : ι ) (x : ) (hw' : s.sum (λ (i : ι), w i) = 1) (hx : (i : ι), i s w i 0 z i = x) :
s.sum (λ (i : ι), w i * z i) = x
theorem real.geom_mean_eq_arith_mean_weighted_of_constant {ι : Type u} (s : finset ι) (w z : ι ) (x : ) (hw : (i : ι), i s 0 w i) (hw' : s.sum (λ (i : ι), w i) = 1) (hz : (i : ι), i s 0 z i) (hx : (i : ι), i s w i 0 z i = x) :
s.prod (λ (i : ι), z i ^ w i) = s.sum (λ (i : ι), w i * z i)
theorem nnreal.geom_mean_le_arith_mean_weighted {ι : Type u} (s : finset ι) (w z : ι nnreal) (hw' : s.sum (λ (i : ι), w i) = 1) :
s.prod (λ (i : ι), z i ^ (w i)) s.sum (λ (i : ι), w i * z i)

The geometric mean is less than or equal to the arithmetic mean, weighted version for nnreal-valued functions.

theorem nnreal.geom_mean_le_arith_mean2_weighted (w₁ w₂ p₁ p₂ : nnreal) :
w₁ + w₂ = 1 p₁ ^ w₁ * p₂ ^ w₂ w₁ * p₁ + w₂ * p₂

The geometric mean is less than or equal to the arithmetic mean, weighted version for two nnreal numbers.

theorem nnreal.geom_mean_le_arith_mean3_weighted (w₁ w₂ w₃ p₁ p₂ p₃ : nnreal) :
w₁ + w₂ + w₃ = 1 p₁ ^ w₁ * p₂ ^ w₂ * p₃ ^ w₃ w₁ * p₁ + w₂ * p₂ + w₃ * p₃
theorem nnreal.geom_mean_le_arith_mean4_weighted (w₁ w₂ w₃ w₄ p₁ p₂ p₃ p₄ : nnreal) :
w₁ + w₂ + w₃ + w₄ = 1 p₁ ^ w₁ * p₂ ^ w₂ * p₃ ^ w₃ * p₄ ^ w₄ w₁ * p₁ + w₂ * p₂ + w₃ * p₃ + w₄ * p₄
theorem real.geom_mean_le_arith_mean2_weighted {w₁ w₂ p₁ p₂ : } (hw₁ : 0 w₁) (hw₂ : 0 w₂) (hp₁ : 0 p₁) (hp₂ : 0 p₂) (hw : w₁ + w₂ = 1) :
p₁ ^ w₁ * p₂ ^ w₂ w₁ * p₁ + w₂ * p₂
theorem real.geom_mean_le_arith_mean3_weighted {w₁ w₂ w₃ p₁ p₂ p₃ : } (hw₁ : 0 w₁) (hw₂ : 0 w₂) (hw₃ : 0 w₃) (hp₁ : 0 p₁) (hp₂ : 0 p₂) (hp₃ : 0 p₃) (hw : w₁ + w₂ + w₃ = 1) :
p₁ ^ w₁ * p₂ ^ w₂ * p₃ ^ w₃ w₁ * p₁ + w₂ * p₂ + w₃ * p₃
theorem real.geom_mean_le_arith_mean4_weighted {w₁ w₂ w₃ w₄ p₁ p₂ p₃ p₄ : } (hw₁ : 0 w₁) (hw₂ : 0 w₂) (hw₃ : 0 w₃) (hw₄ : 0 w₄) (hp₁ : 0 p₁) (hp₂ : 0 p₂) (hp₃ : 0 p₃) (hp₄ : 0 p₄) (hw : w₁ + w₂ + w₃ + w₄ = 1) :
p₁ ^ w₁ * p₂ ^ w₂ * p₃ ^ w₃ * p₄ ^ w₄ w₁ * p₁ + w₂ * p₂ + w₃ * p₃ + w₄ * p₄

Young's inequality #

theorem real.young_inequality_of_nonneg {a b p q : } (ha : 0 a) (hb : 0 b) (hpq : p.is_conjugate_exponent q) :
a * b a ^ p / p + b ^ q / q

Young's inequality, a version for nonnegative real numbers.

theorem real.young_inequality (a b : ) {p q : } (hpq : p.is_conjugate_exponent q) :
a * b |a| ^ p / p + |b| ^ q / q

Young's inequality, a version for arbitrary real numbers.

theorem nnreal.young_inequality (a b : nnreal) {p q : nnreal} (hp : 1 < p) (hpq : 1 / p + 1 / q = 1) :
a * b a ^ p / p + b ^ q / q

Young's inequality, ℝ≥0 version. We use {p q : ℝ≥0} in order to avoid constructing witnesses of 0 ≤ p and 0 ≤ q for the denominators.

theorem nnreal.young_inequality_real (a b : nnreal) {p q : } (hpq : p.is_conjugate_exponent q) :
a * b a ^ p / p.to_nnreal + b ^ q / q.to_nnreal

Young's inequality, ℝ≥0 version with real conjugate exponents.

theorem ennreal.young_inequality (a b : ennreal) {p q : } (hpq : p.is_conjugate_exponent q) :

Young's inequality, ℝ≥0∞ version with real conjugate exponents.

Hölder's and Minkowski's inequalities #

theorem nnreal.inner_le_Lp_mul_Lq {ι : Type u} (s : finset ι) (f g : ι nnreal) {p q : } (hpq : p.is_conjugate_exponent q) :
s.sum (λ (i : ι), f i * g i) s.sum (λ (i : ι), f i ^ p) ^ (1 / p) * s.sum (λ (i : ι), g i ^ q) ^ (1 / q)

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. Version for sums over finite sets, with ℝ≥0-valued functions.

theorem nnreal.inner_le_Lp_mul_Lq_tsum {ι : Type u} {f g : ι nnreal} {p q : } (hpq : p.is_conjugate_exponent q) (hf : summable (λ (i : ι), f i ^ p)) (hg : summable (λ (i : ι), g i ^ q)) :
summable (λ (i : ι), f i * g i) ∑' (i : ι), f i * g i (∑' (i : ι), f i ^ p) ^ (1 / p) * (∑' (i : ι), g i ^ q) ^ (1 / q)

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. A version for nnreal-valued functions. For an alternative version, convenient if the infinite sums are already expressed as p-th powers, see inner_le_Lp_mul_Lq_has_sum.

theorem nnreal.summable_mul_of_Lp_Lq {ι : Type u} {f g : ι nnreal} {p q : } (hpq : p.is_conjugate_exponent q) (hf : summable (λ (i : ι), f i ^ p)) (hg : summable (λ (i : ι), g i ^ q)) :
summable (λ (i : ι), f i * g i)
theorem nnreal.inner_le_Lp_mul_Lq_tsum' {ι : Type u} {f g : ι nnreal} {p q : } (hpq : p.is_conjugate_exponent q) (hf : summable (λ (i : ι), f i ^ p)) (hg : summable (λ (i : ι), g i ^ q)) :
∑' (i : ι), f i * g i (∑' (i : ι), f i ^ p) ^ (1 / p) * (∑' (i : ι), g i ^ q) ^ (1 / q)
theorem nnreal.inner_le_Lp_mul_Lq_has_sum {ι : Type u} {f g : ι nnreal} {A B : nnreal} {p q : } (hpq : p.is_conjugate_exponent q) (hf : has_sum (λ (i : ι), f i ^ p) (A ^ p)) (hg : has_sum (λ (i : ι), g i ^ q) (B ^ q)) :
(C : nnreal), C A * B has_sum (λ (i : ι), f i * g i) C

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. A version for nnreal-valued functions. For an alternative version, convenient if the infinite sums are not already expressed as p-th powers, see inner_le_Lp_mul_Lq_tsum.

theorem nnreal.rpow_sum_le_const_mul_sum_rpow {ι : Type u} (s : finset ι) (f : ι nnreal) {p : } (hp : 1 p) :
s.sum (λ (i : ι), f i) ^ p (s.card) ^ (p - 1) * s.sum (λ (i : ι), f i ^ p)

For 1 ≤ p, the p-th power of the sum of f i is bounded above by a constant times the sum of the p-th powers of f i. Version for sums over finite sets, with ℝ≥0-valued functions.

theorem nnreal.is_greatest_Lp {ι : Type u} (s : finset ι) (f : ι nnreal) {p q : } (hpq : p.is_conjugate_exponent q) :
is_greatest ((λ (g : ι nnreal), s.sum (λ (i : ι), f i * g i)) '' {g : ι nnreal | s.sum (λ (i : ι), g i ^ q) 1}) (s.sum (λ (i : ι), f i ^ p) ^ (1 / p))

The L_p seminorm of a vector f is the greatest value of the inner product ∑ i in s, f i * g i over functions g of L_q seminorm less than or equal to one.

theorem nnreal.Lp_add_le {ι : Type u} (s : finset ι) (f g : ι nnreal) {p : } (hp : 1 p) :
s.sum (λ (i : ι), (f i + g i) ^ p) ^ (1 / p) s.sum (λ (i : ι), f i ^ p) ^ (1 / p) + s.sum (λ (i : ι), g i ^ p) ^ (1 / p)

Minkowski inequality: the L_p seminorm of the sum of two vectors is less than or equal to the sum of the L_p-seminorms of the summands. A version for nnreal-valued functions.

theorem nnreal.Lp_add_le_tsum {ι : Type u} {f g : ι nnreal} {p : } (hp : 1 p) (hf : summable (λ (i : ι), f i ^ p)) (hg : summable (λ (i : ι), g i ^ p)) :
summable (λ (i : ι), (f i + g i) ^ p) (∑' (i : ι), (f i + g i) ^ p) ^ (1 / p) (∑' (i : ι), f i ^ p) ^ (1 / p) + (∑' (i : ι), g i ^ p) ^ (1 / p)

Minkowski inequality: the L_p seminorm of the infinite sum of two vectors is less than or equal to the infinite sum of the L_p-seminorms of the summands, if these infinite sums both exist. A version for nnreal-valued functions. For an alternative version, convenient if the infinite sums are already expressed as p-th powers, see Lp_add_le_has_sum_of_nonneg.

theorem nnreal.summable_Lp_add {ι : Type u} {f g : ι nnreal} {p : } (hp : 1 p) (hf : summable (λ (i : ι), f i ^ p)) (hg : summable (λ (i : ι), g i ^ p)) :
summable (λ (i : ι), (f i + g i) ^ p)
theorem nnreal.Lp_add_le_tsum' {ι : Type u} {f g : ι nnreal} {p : } (hp : 1 p) (hf : summable (λ (i : ι), f i ^ p)) (hg : summable (λ (i : ι), g i ^ p)) :
(∑' (i : ι), (f i + g i) ^ p) ^ (1 / p) (∑' (i : ι), f i ^ p) ^ (1 / p) + (∑' (i : ι), g i ^ p) ^ (1 / p)
theorem nnreal.Lp_add_le_has_sum {ι : Type u} {f g : ι nnreal} {A B : nnreal} {p : } (hp : 1 p) (hf : has_sum (λ (i : ι), f i ^ p) (A ^ p)) (hg : has_sum (λ (i : ι), g i ^ p) (B ^ p)) :
(C : nnreal), C A + B has_sum (λ (i : ι), (f i + g i) ^ p) (C ^ p)

Minkowski inequality: the L_p seminorm of the infinite sum of two vectors is less than or equal to the infinite sum of the L_p-seminorms of the summands, if these infinite sums both exist. A version for nnreal-valued functions. For an alternative version, convenient if the infinite sums are not already expressed as p-th powers, see Lp_add_le_tsum_of_nonneg.

theorem real.inner_le_Lp_mul_Lq {ι : Type u} (s : finset ι) (f g : ι ) {p q : } (hpq : p.is_conjugate_exponent q) :
s.sum (λ (i : ι), f i * g i) s.sum (λ (i : ι), |f i| ^ p) ^ (1 / p) * s.sum (λ (i : ι), |g i| ^ q) ^ (1 / q)

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. Version for sums over finite sets, with real-valued functions.

theorem real.rpow_sum_le_const_mul_sum_rpow {ι : Type u} (s : finset ι) (f : ι ) {p : } (hp : 1 p) :
s.sum (λ (i : ι), |f i|) ^ p (s.card) ^ (p - 1) * s.sum (λ (i : ι), |f i| ^ p)

For 1 ≤ p, the p-th power of the sum of f i is bounded above by a constant times the sum of the p-th powers of f i. Version for sums over finite sets, with -valued functions.

theorem real.Lp_add_le {ι : Type u} (s : finset ι) (f g : ι ) {p : } (hp : 1 p) :
s.sum (λ (i : ι), |f i + g i| ^ p) ^ (1 / p) s.sum (λ (i : ι), |f i| ^ p) ^ (1 / p) + s.sum (λ (i : ι), |g i| ^ p) ^ (1 / p)

Minkowski inequality: the L_p seminorm of the sum of two vectors is less than or equal to the sum of the L_p-seminorms of the summands. A version for real-valued functions.

theorem real.inner_le_Lp_mul_Lq_of_nonneg {ι : Type u} (s : finset ι) {f g : ι } {p q : } (hpq : p.is_conjugate_exponent q) (hf : (i : ι), i s 0 f i) (hg : (i : ι), i s 0 g i) :
s.sum (λ (i : ι), f i * g i) s.sum (λ (i : ι), f i ^ p) ^ (1 / p) * s.sum (λ (i : ι), g i ^ q) ^ (1 / q)

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. Version for sums over finite sets, with real-valued nonnegative functions.

theorem real.inner_le_Lp_mul_Lq_tsum_of_nonneg {ι : Type u} {f g : ι } {p q : } (hpq : p.is_conjugate_exponent q) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : summable (λ (i : ι), f i ^ p)) (hg_sum : summable (λ (i : ι), g i ^ q)) :
summable (λ (i : ι), f i * g i) ∑' (i : ι), f i * g i (∑' (i : ι), f i ^ p) ^ (1 / p) * (∑' (i : ι), g i ^ q) ^ (1 / q)

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. A version for -valued functions. For an alternative version, convenient if the infinite sums are already expressed as p-th powers, see inner_le_Lp_mul_Lq_has_sum_of_nonneg.

theorem real.summable_mul_of_Lp_Lq_of_nonneg {ι : Type u} {f g : ι } {p q : } (hpq : p.is_conjugate_exponent q) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : summable (λ (i : ι), f i ^ p)) (hg_sum : summable (λ (i : ι), g i ^ q)) :
summable (λ (i : ι), f i * g i)
theorem real.inner_le_Lp_mul_Lq_tsum_of_nonneg' {ι : Type u} {f g : ι } {p q : } (hpq : p.is_conjugate_exponent q) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : summable (λ (i : ι), f i ^ p)) (hg_sum : summable (λ (i : ι), g i ^ q)) :
∑' (i : ι), f i * g i (∑' (i : ι), f i ^ p) ^ (1 / p) * (∑' (i : ι), g i ^ q) ^ (1 / q)
theorem real.inner_le_Lp_mul_Lq_has_sum_of_nonneg {ι : Type u} {f g : ι } {p q : } (hpq : p.is_conjugate_exponent q) {A B : } (hA : 0 A) (hB : 0 B) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : has_sum (λ (i : ι), f i ^ p) (A ^ p)) (hg_sum : has_sum (λ (i : ι), g i ^ q) (B ^ q)) :
(C : ), 0 C C A * B has_sum (λ (i : ι), f i * g i) C

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. A version for nnreal-valued functions. For an alternative version, convenient if the infinite sums are not already expressed as p-th powers, see inner_le_Lp_mul_Lq_tsum_of_nonneg.

theorem real.rpow_sum_le_const_mul_sum_rpow_of_nonneg {ι : Type u} (s : finset ι) {f : ι } {p : } (hp : 1 p) (hf : (i : ι), i s 0 f i) :
s.sum (λ (i : ι), f i) ^ p (s.card) ^ (p - 1) * s.sum (λ (i : ι), f i ^ p)

For 1 ≤ p, the p-th power of the sum of f i is bounded above by a constant times the sum of the p-th powers of f i. Version for sums over finite sets, with nonnegative -valued functions.

theorem real.Lp_add_le_of_nonneg {ι : Type u} (s : finset ι) {f g : ι } {p : } (hp : 1 p) (hf : (i : ι), i s 0 f i) (hg : (i : ι), i s 0 g i) :
s.sum (λ (i : ι), (f i + g i) ^ p) ^ (1 / p) s.sum (λ (i : ι), f i ^ p) ^ (1 / p) + s.sum (λ (i : ι), g i ^ p) ^ (1 / p)

Minkowski inequality: the L_p seminorm of the sum of two vectors is less than or equal to the sum of the L_p-seminorms of the summands. A version for -valued nonnegative functions.

theorem real.Lp_add_le_tsum_of_nonneg {ι : Type u} {f g : ι } {p : } (hp : 1 p) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : summable (λ (i : ι), f i ^ p)) (hg_sum : summable (λ (i : ι), g i ^ p)) :
summable (λ (i : ι), (f i + g i) ^ p) (∑' (i : ι), (f i + g i) ^ p) ^ (1 / p) (∑' (i : ι), f i ^ p) ^ (1 / p) + (∑' (i : ι), g i ^ p) ^ (1 / p)

Minkowski inequality: the L_p seminorm of the infinite sum of two vectors is less than or equal to the infinite sum of the L_p-seminorms of the summands, if these infinite sums both exist. A version for -valued functions. For an alternative version, convenient if the infinite sums are already expressed as p-th powers, see Lp_add_le_has_sum_of_nonneg.

theorem real.summable_Lp_add_of_nonneg {ι : Type u} {f g : ι } {p : } (hp : 1 p) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : summable (λ (i : ι), f i ^ p)) (hg_sum : summable (λ (i : ι), g i ^ p)) :
summable (λ (i : ι), (f i + g i) ^ p)
theorem real.Lp_add_le_tsum_of_nonneg' {ι : Type u} {f g : ι } {p : } (hp : 1 p) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) (hf_sum : summable (λ (i : ι), f i ^ p)) (hg_sum : summable (λ (i : ι), g i ^ p)) :
(∑' (i : ι), (f i + g i) ^ p) ^ (1 / p) (∑' (i : ι), f i ^ p) ^ (1 / p) + (∑' (i : ι), g i ^ p) ^ (1 / p)
theorem real.Lp_add_le_has_sum_of_nonneg {ι : Type u} {f g : ι } {p : } (hp : 1 p) (hf : (i : ι), 0 f i) (hg : (i : ι), 0 g i) {A B : } (hA : 0 A) (hB : 0 B) (hfA : has_sum (λ (i : ι), f i ^ p) (A ^ p)) (hgB : has_sum (λ (i : ι), g i ^ p) (B ^ p)) :
(C : ), 0 C C A + B has_sum (λ (i : ι), (f i + g i) ^ p) (C ^ p)

Minkowski inequality: the L_p seminorm of the infinite sum of two vectors is less than or equal to the infinite sum of the L_p-seminorms of the summands, if these infinite sums both exist. A version for -valued functions. For an alternative version, convenient if the infinite sums are not already expressed as p-th powers, see Lp_add_le_tsum_of_nonneg.

theorem ennreal.inner_le_Lp_mul_Lq {ι : Type u} (s : finset ι) (f g : ι ennreal) {p q : } (hpq : p.is_conjugate_exponent q) :
s.sum (λ (i : ι), f i * g i) s.sum (λ (i : ι), f i ^ p) ^ (1 / p) * s.sum (λ (i : ι), g i ^ q) ^ (1 / q)

Hölder inequality: the scalar product of two functions is bounded by the product of their L^p and L^q norms when p and q are conjugate exponents. Version for sums over finite sets, with ℝ≥0∞-valued functions.

theorem ennreal.rpow_sum_le_const_mul_sum_rpow {ι : Type u} (s : finset ι) (f : ι ennreal) {p : } (hp : 1 p) :
s.sum (λ (i : ι), f i) ^ p (s.card) ^ (p - 1) * s.sum (λ (i : ι), f i ^ p)

For 1 ≤ p, the p-th power of the sum of f i is bounded above by a constant times the sum of the p-th powers of f i. Version for sums over finite sets, with ℝ≥0∞-valued functions.

theorem ennreal.Lp_add_le {ι : Type u} (s : finset ι) (f g : ι ennreal) {p : } (hp : 1 p) :
s.sum (λ (i : ι), (f i + g i) ^ p) ^ (1 / p) s.sum (λ (i : ι), f i ^ p) ^ (1 / p) + s.sum (λ (i : ι), g i ^ p) ^ (1 / p)

Minkowski inequality: the L_p seminorm of the sum of two vectors is less than or equal to the sum of the L_p-seminorms of the summands. A version for ℝ≥0∞ valued nonnegative functions.