Complex and real exponential #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove continuity of complex.exp and real.exp. We also prove a few facts about
limits of real.exp at infinity.
Tags #
exp
The real exponential function tends to +∞ at +∞.
The real exponential function tends to 0 at -∞ or, equivalently, exp(-x) tends to 0
at +∞
The real exponential function tends to 1 at 0.
The function exp(x)/x^n tends to +∞ at +∞, for any natural number n
The function x^n * exp(-x) tends to 0 at +∞, for any natural number n.
The function (b * exp x + c) / (x ^ n) tends to +∞ at +∞, for any natural number
n and any real numbers b and c such that b is positive.
The function (x ^ n) / (b * exp x + c) tends to 0 at +∞, for any natural number
n and any real numbers b and c such that b is nonzero.
real.exp as an order isomorphism between ℝ and (0, +∞).
Equations
- real.exp_order_iso = strict_mono.order_iso_of_surjective (set.cod_restrict rexp (set.Ioi 0) real.exp_pos) real.exp_order_iso._proof_1 real.exp_order_iso._proof_2
complex.abs (complex.exp z) → ∞ as complex.re z → ∞. TODO: use bornology.cobounded.
complex.exp z → 0 as complex.re z → -∞.