Documentation

Convex.Analysis.Lemmas

Lemmas #

Main results #

This file contains the following parts of basic properties of continuous and differentiable lemmas

theorem ContinuousAt_Convergence {E : Type u_1} [NormedAddCommGroup E] {f : E} {x : E} (h : ContinuousAt f x) (ε : ) :
ε > 0δ > 0, ∀ (x' : E), x - x' δf x' - f x ε
theorem Convergence_ContinuousAt {E : Type u_1} [NormedAddCommGroup E] {f : E} {x : E} (h : ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x ε) :
theorem ContinuousAt_iff_Convergence {E : Type u_1} [NormedAddCommGroup E] {f : E} {x : E} :
ContinuousAt f x ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x ε
theorem continuous {E : Type u_1} [NormedAddCommGroup E] {f : E} {x : E} (h : ContinuousAt f x) (ε : ) :
ε > 0δ > 0, ∀ (y : E), y - x < δf y - f x < ε
theorem deriv_function_comp_segment {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {f' : EE →L[] } (x : E) (y : E) (h₁ : ∀ (x₁ : E), HasFDerivAt f (f' x₁) x₁) (t₀ : ) :
HasDerivAt (fun (t : ) => f (x + t (y - x))) ((fun (t : ) => (f' (x + t (y - x))) (y - x)) t₀) t₀
theorem HasFDeriv_Convergence {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {f' : EE →L[] } {x : E} (h : HasFDerivAt f (f' x) x) (ε : ) :
ε > 0δ > 0, ∀ (x' : E), x - x' δf x' - f x - (f' x) (x' - x) ε * x - x'
theorem Convergence_HasFDeriv {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {f' : EE →L[] } {x : E} (h : ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x - (f' x) (x' - x) ε * x - x') :
HasFDerivAt f (f' x) x
theorem HasFDeriv_iff_Convergence_Point {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {x : E} {f'x : E →L[] } :
HasFDerivAt f f'x x ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x - f'x (x' - x) ε * x - x'
theorem HasFDeriv_iff_Convergence {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {f' : EE →L[] } {x : E} :
HasFDerivAt f (f' x) x ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x - (f' x) (x' - x) ε * x - x'
theorem HasGradient_Convergence {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {x : E} {f : E} {f' : EE} (h : HasGradientAt f (f' x) x) (ε : ) :
ε > 0δ > 0, ∀ (x' : E), x - x' δf x' - f x - f' x, x' - x⟫_ ε * x - x'
theorem Convergence_HasGradient {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {x : E} {f : E} {f' : EE} (h : ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x - f' x, x' - x⟫_ ε * x - x') :
HasGradientAt f (f' x) x
theorem HasGradient_iff_Convergence_Point {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {x : E} {f : E} {f'x : E} :
HasGradientAt f f'x x ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x - f'x, x' - x⟫_ ε * x - x'
theorem HasGradient_iff_Convergence {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {x : E} {f : E} {f' : EE} :
HasGradientAt f (f' x) x ε > 0, δ > 0, ∀ (x' : E), x - x' δf x' - f x - f' x, x' - x⟫_ ε * x - x'
theorem gradient_norm_sq_eq_two_self {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] (x : E) :
HasGradientAt (fun (x : E) => x ^ 2) (2 x) x
theorem gradient_of_inner_const {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] (x : E) (a : E) :
HasGradientAt (fun (x : E) => a, x⟫_) a x
theorem gradient_of_const_mul_norm {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] (l : ) (z : E) :
HasGradientAt (fun (x : E) => l / 2 * x ^ 2) (l z) z
theorem gradient_of_sq {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {x : E} (u : E) :
HasGradientAt (fun (u : E) => u - x ^ 2 / 2) (u - x) u
theorem sub_normsquare_gradient {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {s : Set E} (hf : xs, HasGradientAt f (f' x) x) (m : ) (x : E) :
x sHasGradientAt (fun (x : E) => f x - m / 2 * x ^ 2) (f' x - m x) x
theorem gradient_continuous_of_contdiff {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {x : E} {ε : } (f : E) (he : ε > 0) (hf : ContDiffOn 1 f (Metric.ball x ε)) :
ContinuousAt (fun (x : E) => gradient f x) x
theorem expansion {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} (hf : ∀ (x : E), HasGradientAt f (f' x) x) (x : E) (p : E) :
t > 0, t < 1 f (x + p) = f x + f' (x + t p), p⟫_
theorem general_expansion {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} (x : E) (p : E) (hf : yMetric.closedBall x p, HasGradientAt f (f' y) y) :
t > 0, t < 1 f (x + p) = f x + f' (x + t p), p⟫_
theorem lagrange {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {s : Set E} (hs : Convex s) (hf : xs, HasGradientAt f (f' x) x) (x : E) :
x sys, cSet.Ioo 0 1, f' (x + c (y - x)), y - x⟫_ = f y - f x