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:
strict_convex_on_exp
: The exponential function is strictly convex.even.convex_on_pow
: For an evenn : ℕ
,λ x, x ^ n
is convex.convex_on_pow
: Forn : ℕ
,λ x, x ^ n
is convex on $[0, +∞)$.convex_on_zpow
: Form : ℤ
,λ x, x ^ m
is convex on $[0, +∞)$.strict_concave_on_log_Ioi
,strict_concave_on_log_Iio
:real.log
is strictly concave on $(0, +∞)$ and $(-∞, 0)$ respectively.convex_on_rpow
,strict_convex_on_rpow
: Forp : ℝ
,λ x, x ^ p
is convex on $[0, +∞)$ when1 ≤ p
and strictly convex when1 < p
.
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.