Documentation

Mathlib.Analysis.Calculus.LocalExtr.LineDeriv

Local extremum and line derivatives #

If f has a local extremum at a point, then the derivative at this point is zero. In this file we prove several versions of this fact for line derivatives.

theorem IsExtrFilter.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {a : E} {b : E} {f' : } {l : Filter E} (h : IsExtrFilter f l a) (hd : HasLineDerivAt f f' a b) (h' : Filter.Tendsto (fun (t : ) => a + t b) (nhds 0) l) :
f' = 0
theorem IsExtrFilter.lineDeriv_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {a : E} {b : E} {l : Filter E} (h : IsExtrFilter f l a) (h' : Filter.Tendsto (fun (t : ) => a + t b) (nhds 0) l) :
lineDeriv f a b = 0
theorem IsExtrOn.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} {f' : } (h : IsExtrOn f s a) (hd : HasLineDerivAt f f' a b) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
f' = 0
theorem IsExtrOn.lineDeriv_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} (h : IsExtrOn f s a) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
lineDeriv f a b = 0
theorem IsMinOn.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} {f' : } (h : IsMinOn f s a) (hd : HasLineDerivAt f f' a b) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
f' = 0
theorem IsMinOn.lineDeriv_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} (h : IsMinOn f s a) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
lineDeriv f a b = 0
theorem IsMaxOn.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} {f' : } (h : IsMaxOn f s a) (hd : HasLineDerivAt f f' a b) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
f' = 0
theorem IsMaxOn.lineDeriv_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} (h : IsMaxOn f s a) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
lineDeriv f a b = 0
theorem IsExtrOn.hasLineDerivWithinAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} {f' : } (h : IsExtrOn f s a) (hd : HasLineDerivWithinAt f f' s a b) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
f' = 0
theorem IsExtrOn.lineDerivWithin_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} (h : IsExtrOn f s a) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
theorem IsMinOn.hasLineDerivWithinAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} {f' : } (h : IsMinOn f s a) (hd : HasLineDerivWithinAt f f' s a b) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
f' = 0
theorem IsMinOn.lineDerivWithin_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} (h : IsMinOn f s a) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
theorem IsMaxOn.hasLineDerivWithinAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} {f' : } (h : IsMaxOn f s a) (hd : HasLineDerivWithinAt f f' s a b) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
f' = 0
theorem IsMaxOn.lineDerivWithin_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] {f : E} {s : Set E} {a : E} {b : E} (h : IsMaxOn f s a) (h' : ∀ᶠ (t : ) in nhds 0, a + t b s) :
theorem IsLocalExtr.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [ContinuousAdd E] [ContinuousSMul E] {f : E} {a : E} {b : E} {f' : } (h : IsLocalExtr f a) (hd : HasLineDerivAt f f' a b) :
f' = 0
theorem IsLocalMin.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [ContinuousAdd E] [ContinuousSMul E] {f : E} {a : E} {b : E} {f' : } (h : IsLocalMin f a) (hd : HasLineDerivAt f f' a b) :
f' = 0
theorem IsLocalMin.lineDeriv_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [ContinuousAdd E] [ContinuousSMul E] {f : E} {a : E} (h : IsLocalMin f a) :
theorem IsLocalMax.hasLineDerivAt_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [ContinuousAdd E] [ContinuousSMul E] {f : E} {a : E} {b : E} {f' : } (h : IsLocalMax f a) (hd : HasLineDerivAt f f' a b) :
f' = 0
theorem IsLocalMax.lineDeriv_eq_zero {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [ContinuousAdd E] [ContinuousSMul E] {f : E} {a : E} (h : IsLocalMax f a) :