Exponential Function #
This file contains the definitions of the real and complex exponential function.
The Cauchy sequence consisting of partial sums of the Taylor series of the complex exponential function
Equations
- Complex.exp' z = ⟨fun (n : ℕ) => ∑ m ∈ Finset.range n, z ^ m / ↑m.factorial, ⋯⟩
Instances For
The complex exponential function, defined via its Taylor series
Equations
- Complex.exp z = (Complex.exp' z).lim
Instances For
scoped notation for the complex exponential function
Equations
- Complex.termCexp = Lean.ParserDescr.node `Complex.termCexp 1024 (Lean.ParserDescr.symbol "cexp")
Instances For
scoped notation for the real exponential function
Equations
- Real.termRexp = Lean.ParserDescr.node `Real.termRexp 1024 (Lean.ParserDescr.symbol "rexp")
Instances For
the exponential function as a monoid hom from Multiplicative ℂ
to ℂ
Equations
- Complex.expMonoidHom = { toFun := fun (z : Multiplicative ℂ) => Complex.exp (Multiplicative.toAdd z), map_one' := Complex.expMonoidHom.proof_1, map_mul' := Complex.expMonoidHom.proof_2 }
Instances For
the exponential function as a monoid hom from Multiplicative ℝ
to ℝ
Equations
- Real.expMonoidHom = { toFun := fun (x : Multiplicative ℝ) => Real.exp (Multiplicative.toAdd x), map_one' := Real.expMonoidHom.proof_1, map_mul' := Real.expMonoidHom.proof_2 }
Instances For
A finite initial segment of the exponential series, followed by an arbitrary tail.
For fixed n
this is just a linear map wrt r
, and each map is a simple linear function
of the previous (see expNear_succ
), with expNear n x r ⟶ exp x
as n ⟶ ∞
,
for any r
.
Instances For
Extension for the positivity
tactic: Real.exp
is always positive.