Documentation

Convex.Function.StronglyConvex

the properties of strongly convex function and gradient descent method for strongly convex function

theorem Strongly_Convex_Bound {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] {s : Set E} {f : E} (m : ) (strongly_convex : StrongConvexOn s m f) ⦃x : E :
x s∀ ⦃y : E⦄, y s∀ ⦃a : ⦄, 0 < a∀ ⦃b : ⦄, 0 < ba + b = 1f (a x + b y) a * f x + b * f y - m / 2 * a * b * x - y ^ 2
theorem stronglyConvexOn_def {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] {s : Set E} {f : E} {m : } (hs : Convex s) (hfun : ∀ ⦃x : E⦄, x s∀ ⦃y : E⦄, y s∀ ⦃a : ⦄, 0 a∀ ⦃b : ⦄, 0 ba + b = 1f (a x + b y) a * f x + b * f y - m / 2 * a * b * x - y ^ 2) :
theorem Strongly_Convex_Unique_Minima {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] {s : Set E} {f : E} {m : } {xm : E} {xm' : E} {mp : m > 0} (hsc : StrongConvexOn s m f) (min : IsMinOn f s xm) (min' : IsMinOn f s xm') (hxm : xm s) (hxm' : xm' s) :
xm = xm'
theorem Strong_Convex_lower {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {s : Set E} {f : E} {m : } {f' : EE} (hsc : StrongConvexOn s m f) (hf : xs, HasGradientAt f (f' x) x) (x : E) :
x sys, f' x - f' y, x - y⟫_ m * x - y ^ 2
theorem Lower_Strong_Convex {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {s : Set E} {f : E} {m : } {f' : EE} (hf : xs, HasGradientAt f (f' x) x) (hs : Convex s) (h : xs, ys, f' x - f' y, x - y⟫_ m * x - y ^ 2) :
theorem Strong_Convex_iff_lower {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {s : Set E} {f : E} {m : } {f' : EE} (hf : xs, HasGradientAt f (f' x) x) (hs : Convex s) :
StrongConvexOn s m f xs, ys, f' x - f' y, x - y⟫_ m * x - y ^ 2
theorem Strong_Convex_second_lower {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {s : Set E} {f : E} {m : } {f' : EE} (hsc : StrongConvexOn s m f) (hf : xs, HasGradientAt f (f' x) x) (x : E) :
x sys, f y f x + f' x, y - x⟫_ + m / 2 * y - x ^ 2