The First-Derivative Test #
We prove the first-derivative test from calculus, in the strong form given on Wikipedia.
The test is proved over the real numbers ℝ
using monotoneOn_of_deriv_nonneg
from [Mathlib.Analysis.Calculus.MeanValue].
The Second-Derivative Test #
We prove the Second-Derivative Test using the First-Derivative Test. Source: Wikipedia.
Main results #
isLocalMax_of_deriv_Ioo
: Supposef
is a real-valued function of a real variable defined on some interval containing the pointa
. Further suppose thatf
is continuous ata
and differentiable on some open interval containinga
, except possibly ata
itself.If there exists a positive number
r > 0
such that for everyx
in(a − r, a)
we havef′(x) ≥ 0
, and for everyx
in(a, a + r)
we havef′(x) ≤ 0
, thenf
has a local maximum ata
.isLocalMin_of_deriv_Ioo
: The dual offirst_derivative_max
, for minima.isLocalMax_of_deriv
: 1st derivative test for maxima using filters.isLocalMin_of_deriv
: 1st derivative test for minima using filters.isLocalMin_of_deriv_deriv_pos
: The second-derivative test, minimum version.
Tags #
derivative test, calculus
The First-Derivative Test from calculus, maxima version.
Suppose a < b < c
, f : ℝ → ℝ
is continuous at b
,
the derivative f'
is nonnegative on (a,b)
, and
the derivative f'
is nonpositive on (b,c)
. Then f
has a local maximum at a
.
The First-Derivative Test from calculus, minima version.
The First-Derivative Test from calculus, maxima version, expressed in terms of left and right filters.
The First-Derivative Test from calculus, minima version, expressed in terms of left and right filters.
The First Derivative test, maximum version.
The First Derivative test, minimum version.
The First Derivative test with a hypothesis on the sign of the derivative, maximum version.
The First Derivative test with a hypothesis on the sign of the derivative, minimum version.
The Second-Derivative Test from calculus, minimum version.
Applies to functions like x^2 + 1[x ≥ 0]
as well as twice differentiable
functions.
The Second-Derivative Test from calculus, maximum version.