mathlib3 documentation

analysis.convex.specific_functions.basic

Collection of convex functions #

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

In this file we prove that the following functions are convex or strictly convex:

The proofs in this file are deliberately elementary, not by appealing to the sign of the second derivative. This is in order to keep this file early in the import hierarchy, since it is on the path to Hölder's and Minkowski's inequalities and after that to Lp spaces and most of measure theory.

TODO #

For p : ℝ, prove that λ x, x ^ p is concave when 0 ≤ p ≤ 1 and strictly concave when 0 < p < 1.

exp is strictly convex on the whole real line.

We give an elementary proof rather than using the second derivative test, since this lemma is needed early in the analysis library.

exp is convex on the whole real line.

theorem convex_on_pow (n : ) :
convex_on (set.Ici 0) (λ (x : ), x ^ n)

x^n, n : ℕ is convex on [0, +∞) for all n.

We give an elementary proof rather than using the second derivative test, since this lemma is needed early in the analysis library.

theorem even.convex_on_pow {n : } (hn : even n) :
convex_on set.univ (λ (x : ), x ^ n)

x^n, n : ℕ is convex on the whole real line whenever n is even.

We give an elementary proof rather than using the second derivative test, since this lemma is needed early in the analysis library.

theorem convex_on_zpow (m : ) :
convex_on (set.Ioi 0) (λ (x : ), x ^ m)

x^m, m : ℤ is convex on (0, +∞) for all m.

We give an elementary proof rather than using the second derivative test, since this lemma is needed early in the analysis library.

theorem one_add_mul_self_lt_rpow_one_add {s : } (hs : -1 s) (hs' : s 0) {p : } (hp : 1 < p) :
1 + p * s < (1 + s) ^ p

Bernoulli's inequality for real exponents, strict version: for 1 < p and -1 ≤ s, with s ≠ 0, we have 1 + p * s < (1 + s) ^ p.

theorem one_add_mul_self_le_rpow_one_add {s : } (hs : -1 s) {p : } (hp : 1 p) :
1 + p * s (1 + s) ^ p

Bernoulli's inequality for real exponents, non-strict version: for 1 ≤ p and -1 ≤ s we have 1 + p * s ≤ (1 + s) ^ p.

theorem strict_convex_on_rpow {p : } (hp : 1 < p) :
strict_convex_on (set.Ici 0) (λ (x : ), x ^ p)
theorem convex_on_rpow {p : } (hp : 1 p) :
convex_on (set.Ici 0) (λ (x : ), x ^ p)