Documentation

Convex.Function.Lsmooth

Lsmooth #

Main results #

This file mainly concentrates on the properties of the L smooth function.

The main theorem is given as:

theorem lipschitz_continuous_upper_bound {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {f' : EE →L[] } {l : NNReal} (h₁ : ∀ (x₁ : E), HasFDerivAt f (f' x₁) x₁) (h₂ : LipschitzWith l f') (x : E) (y : E) :
f y f x + (f' x) (y - x) + l / 2 * y - x ^ 2
theorem lipschitz_continuos_upper_bound' {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {l : NNReal} (h₁ : ∀ (x₁ : E), HasGradientAt f (f' x₁) x₁) (h₂ : LipschitzWith l f') (x : E) (y : E) :
f y f x + f' x, y - x⟫_ + l / 2 * y - x ^ 2
theorem lipschitz_minima_lower_bound {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {xm : E} {l : NNReal} (h₁ : ∀ (x : E), HasGradientAt f (f' x) x) (h₂ : LipschitzWith l f') (min : IsMinOn f Set.univ xm) (hl : l > 0) (x : E) :
1 / (2 * l) * f' x ^ 2 f x - f xm
theorem lipschitz_to_lnorm_sub_convex {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {s : Set E} {l : NNReal} (hs : Convex s) (h₁ : xs, HasGradientAt f (f' x) x) (h₂ : LipschitzOnWith l f' s) (hl : l > 0) :
ConvexOn s fun (x : E) => l / 2 * x ^ 2 - f x
theorem convex_to_lower {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {l : } (h₁ : ∀ (x : E), HasGradientAt f (f' x) x) (h₂ : ConvexOn Set.univ fun (x : E) => l / 2 * x ^ 2 - f x) (lp : l > 0) (hfun : ConvexOn Set.univ f) (x : E) (y : E) :
f' x - f' y, x - y⟫_ 1 / l * f' x - f' y ^ 2
theorem lipschitz_to_lower {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {l : NNReal} (h₁ : ∀ (x : E), HasGradientAt f (f' x) x) (h₂ : LipschitzWith l f') (hfun : ConvexOn Set.univ f) (hl : l > 0) (x : E) (y : E) :
f' x - f' y, x - y⟫_ 1 / l * f' x - f' y ^ 2
theorem lower_to_lipschitz {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] {f' : EE} {l : NNReal} (h₂ : ∀ (x y : E), f' x - f' y, x - y⟫_ 1 / l * f' x - f' y ^ 2) (hl : l > 0) :
theorem lower_iff_lipschitz {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {l : NNReal} (h₁ : ∀ (x : E), HasGradientAt f (f' x) x) (hfun : ConvexOn Set.univ f) (hl : l > 0) :
LipschitzWith l f' ∀ (x y : E), f' x - f' y, x - y⟫_ 1 / l * f' x - f' y ^ 2
theorem lipshictz_iff_lnorm_sub_convex {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {l : NNReal} (h₁ : ∀ (x : E), HasGradientAt f (f' x) x) (hfun : ConvexOn Set.univ f) (hl : l > 0) :
LipschitzWith l f' ConvexOn Set.univ fun (x : E) => l / 2 * x ^ 2 - f x
theorem lower_iff_lnorm_sub_convex {E : Type u_1} [NormedAddCommGroup E] [InnerProductSpace E] [CompleteSpace E] {f : E} {f' : EE} {l : NNReal} (h₁ : ∀ (x : E), HasGradientAt f (f' x) x) (hfun : ConvexOn Set.univ f) (hl : l > 0) :
(ConvexOn Set.univ fun (x : E) => l / 2 * x ^ 2 - f x) ∀ (x y : E), f' x - f' y, x - y⟫_ 1 / l * f' x - f' y ^ 2