Documentation

Mathlib.Analysis.SpecialFunctions.Sigmoid

Sigmoid function #

In this file we define the sigmoid function x : ℝ ↦ (1 + exp (-x))⁻¹ and prove some of its analytic properties.

We then show that the sigmoid function can be seen as an order embedding from to I = [0, 1] and that this embedding is both a topological embedding and a measurable embedding. We also prove that the composition of this embedding with the measurable embedding from a standard Borel space α to is a measurable embedding from α to I.

Main definitions and results #

Sigmoid as a function from to #

Sigmoid as a function from to I #

Sigmoid as an OrderEmbedding from to I #

Tags #

sigmoid, embedding, measurable embedding, topological embedding

noncomputable def Real.sigmoid (x : ) :

The sigmoid function from to .

Equations
Instances For
    theorem Real.sigmoid_def (x : ) :
    x.sigmoid = (1 + exp (-x))⁻¹
    theorem Real.sigmoid_pos (x : ) :
    theorem Real.sigmoid_le {a b : } :
    a ba.sigmoid b.sigmoid
    theorem Real.sigmoid_lt {a b : } :
    a < ba.sigmoid < b.sigmoid
    @[simp]
    theorem Real.sigmoid_inj {a b : } :
    theorem Real.sigmoid_neg (x : ) :
    theorem Real.deriv_sigmoid :
    deriv sigmoid = fun (x : ) => x.sigmoid * (1 - x.sigmoid)
    theorem AnalyticAt.sigmoid {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {x : E} (fa : AnalyticAt f x) :
    theorem AnalyticAt.sigmoid' {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {x : E} (fa : AnalyticAt f x) :
    AnalyticAt (fun (z : E) => (f z).sigmoid) x
    theorem AnalyticOn.sigmoid {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {s : Set E} (fs : AnalyticOn f s) :
    theorem AnalyticWithinAt.sigmoid {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {f : E} {s : Set E} {x : E} (fa : AnalyticWithinAt f s x) :
    noncomputable def unitInterval.sigmoid :

    The sigmoid function from to I.

    Equations
    Instances For
      theorem unitInterval.sigmoid_lt {a b : } :
      a < bsigmoid a < sigmoid b
      @[simp]
      theorem unitInterval.sigmoid_inj {a b : } :