Documentation

Mathlib.Data.Complex.Exponential

Exponential Function #

This file contains the definitions of the real and complex exponential function.

theorem Complex.isCauSeq_abs_exp (z : ) :
IsCauSeq _root_.abs fun (n : ) => mFinset.range n, abs (z ^ m / m.factorial)
theorem Complex.isCauSeq_exp (z : ) :
IsCauSeq abs fun (n : ) => mFinset.range n, z ^ m / m.factorial
def Complex.exp' (z : ) :

The Cauchy sequence consisting of partial sums of the Taylor series of the complex exponential function

Equations
Instances For
    def Complex.exp (z : ) :

    The complex exponential function, defined via its Taylor series

    Equations
    Instances For

      scoped notation for the complex exponential function

      Equations
      Instances For
        def Real.exp (x : ) :

        The real exponential function, defined as the real part of the complex exponential

        Equations
        Instances For

          scoped notation for the real exponential function

          Equations
          Instances For
            @[simp]
            theorem Complex.exp_zero :
            exp 0 = 1
            theorem Complex.exp_add (x y : ) :
            exp (x + y) = exp x * exp y

            the exponential function as a monoid hom from Multiplicative to

            Equations
            Instances For
              theorem Complex.exp_sum {α : Type u_1} (s : Finset α) (f : α) :
              exp (∑ xs, f x) = xs, exp (f x)
              theorem Complex.exp_nsmul (x : ) (n : ) :
              exp (n x) = exp x ^ n
              theorem Complex.exp_nat_mul (x : ) (n : ) :
              exp (n * x) = exp x ^ n
              @[simp]
              theorem Complex.exp_ne_zero (x : ) :
              exp x 0
              theorem Complex.exp_neg (x : ) :
              exp (-x) = (exp x)⁻¹
              theorem Complex.exp_sub (x y : ) :
              exp (x - y) = exp x / exp y
              theorem Complex.exp_int_mul (z : ) (n : ) :
              exp (n * z) = exp z ^ n
              @[simp]
              @[simp]
              theorem Complex.ofReal_exp_ofReal_re (x : ) :
              (exp x).re = exp x
              @[simp]
              theorem Complex.ofReal_exp (x : ) :
              (Real.exp x) = exp x
              @[simp]
              theorem Complex.exp_ofReal_im (x : ) :
              (exp x).im = 0
              @[simp]
              theorem Real.exp_zero :
              exp 0 = 1
              theorem Real.exp_add (x y : ) :
              exp (x + y) = exp x * exp y

              the exponential function as a monoid hom from Multiplicative to

              Equations
              Instances For
                theorem Real.exp_sum {α : Type u_1} (s : Finset α) (f : α) :
                exp (∑ xs, f x) = xs, exp (f x)
                theorem Real.exp_nsmul (x : ) (n : ) :
                exp (n x) = exp x ^ n
                theorem Real.exp_nat_mul (x : ) (n : ) :
                exp (n * x) = exp x ^ n
                @[simp]
                theorem Real.exp_ne_zero (x : ) :
                exp x 0
                theorem Real.exp_neg (x : ) :
                exp (-x) = (exp x)⁻¹
                theorem Real.exp_sub (x y : ) :
                exp (x - y) = exp x / exp y
                theorem Real.sum_le_exp_of_nonneg {x : } (hx : 0 x) (n : ) :
                iFinset.range n, x ^ i / i.factorial exp x
                theorem Real.pow_div_factorial_le_exp (x : ) (hx : 0 x) (n : ) :
                x ^ n / n.factorial exp x
                theorem Real.quadratic_le_exp_of_nonneg {x : } (hx : 0 x) :
                1 + x + x ^ 2 / 2 exp x
                theorem Real.one_le_exp {x : } (hx : 0 x) :
                1 exp x
                theorem Real.exp_pos (x : ) :
                0 < exp x
                theorem Real.exp_nonneg (x : ) :
                0 exp x
                @[simp]
                theorem Real.abs_exp (x : ) :
                |exp x| = exp x
                theorem Real.exp_abs_le (x : ) :
                exp |x| exp x + exp (-x)
                theorem Real.exp_lt_exp_of_lt {x y : } (h : x < y) :
                exp x < exp y
                theorem Real.exp_le_exp_of_le {x y : } (h : x y) :
                exp x exp y
                @[simp]
                theorem Real.exp_lt_exp {x y : } :
                exp x < exp y x < y
                @[simp]
                theorem Real.exp_le_exp {x y : } :
                exp x exp y x y
                @[simp]
                theorem Real.exp_eq_exp {x y : } :
                exp x = exp y x = y
                @[simp]
                theorem Real.exp_eq_one_iff (x : ) :
                exp x = 1 x = 0
                @[simp]
                theorem Real.one_lt_exp_iff {x : } :
                1 < exp x 0 < x
                @[simp]
                theorem Real.exp_lt_one_iff {x : } :
                exp x < 1 x < 0
                @[simp]
                theorem Real.exp_le_one_iff {x : } :
                exp x 1 x 0
                @[simp]
                theorem Real.one_le_exp_iff {x : } :
                1 exp x 0 x
                theorem Complex.sum_div_factorial_le {α : Type u_1} [LinearOrderedField α] (n j : ) (hn : 0 < n) :
                mFinset.filter (fun (m : ) => n m) (Finset.range j), 1 / m.factorial n.succ / (n.factorial * n)
                theorem Complex.exp_bound {x : } (hx : abs x 1) {n : } (hn : 0 < n) :
                abs (exp x - mFinset.range n, x ^ m / m.factorial) abs x ^ n * (n.succ * (n.factorial * n)⁻¹)
                theorem Complex.exp_bound' {x : } {n : } (hx : abs x / n.succ 1 / 2) :
                abs (exp x - mFinset.range n, x ^ m / m.factorial) abs x ^ n / n.factorial * 2
                theorem Complex.abs_exp_sub_one_le {x : } (hx : abs x 1) :
                abs (exp x - 1) 2 * abs x
                theorem Complex.abs_exp_sub_one_sub_id_le {x : } (hx : abs x 1) :
                abs (exp x - 1 - x) abs x ^ 2
                theorem Complex.abs_exp_sub_sum_le_exp_abs_sub_sum (x : ) (n : ) :
                abs (exp x - mFinset.range n, x ^ m / m.factorial) Real.exp (abs x) - mFinset.range n, abs x ^ m / m.factorial
                theorem Complex.abs_exp_sub_sum_le_abs_mul_exp (x : ) (n : ) :
                abs (exp x - mFinset.range n, x ^ m / m.factorial) abs x ^ n * Real.exp (abs x)
                theorem Real.exp_bound {x : } (hx : |x| 1) {n : } (hn : 0 < n) :
                |exp x - mFinset.range n, x ^ m / m.factorial| |x| ^ n * (n.succ / (n.factorial * n))
                theorem Real.exp_bound' {x : } (h1 : 0 x) (h2 : x 1) {n : } (hn : 0 < n) :
                exp x mFinset.range n, x ^ m / m.factorial + x ^ n * (n + 1) / (n.factorial * n)
                theorem Real.abs_exp_sub_one_le {x : } (hx : |x| 1) :
                |exp x - 1| 2 * |x|
                theorem Real.abs_exp_sub_one_sub_id_le {x : } (hx : |x| 1) :
                |exp x - 1 - x| x ^ 2
                noncomputable def Real.expNear (n : ) (x r : ) :

                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.

                Equations
                Instances For
                  @[simp]
                  theorem Real.expNear_zero (x r : ) :
                  expNear 0 x r = r
                  @[simp]
                  theorem Real.expNear_succ (n : ) (x r : ) :
                  expNear (n + 1) x r = expNear n x (1 + x / (n + 1) * r)
                  theorem Real.expNear_sub (n : ) (x r₁ r₂ : ) :
                  expNear n x r₁ - expNear n x r₂ = x ^ n / n.factorial * (r₁ - r₂)
                  theorem Real.exp_approx_end (n m : ) (x : ) (e₁ : n + 1 = m) (h : |x| 1) :
                  |exp x - expNear m x 0| |x| ^ m / m.factorial * ((m + 1) / m)
                  theorem Real.exp_approx_succ {n : } {x a₁ b₁ : } (m : ) (e₁ : n + 1 = m) (a₂ b₂ : ) (e : |1 + x / m * a₂ - a₁| b₁ - |x| / m * b₂) (h : |exp x - expNear m x a₂| |x| ^ m / m.factorial * b₂) :
                  |exp x - expNear n x a₁| |x| ^ n / n.factorial * b₁
                  theorem Real.exp_approx_end' {n : } {x a b : } (m : ) (e₁ : n + 1 = m) (rm : ) (er : m = rm) (h : |x| 1) (e : |1 - a| b - |x| / rm * ((rm + 1) / rm)) :
                  |exp x - expNear n x a| |x| ^ n / n.factorial * b
                  theorem Real.exp_1_approx_succ_eq {n : } {a₁ b₁ : } {m : } (en : n + 1 = m) {rm : } (er : m = rm) (h : |exp 1 - expNear m 1 ((a₁ - 1) * rm)| |1| ^ m / m.factorial * (b₁ * rm)) :
                  |exp 1 - expNear n 1 a₁| |1| ^ n / n.factorial * b₁
                  theorem Real.exp_approx_start (x a b : ) (h : |exp x - expNear 0 x a| |x| ^ 0 / (Nat.factorial 0) * b) :
                  |exp x - a| b
                  theorem Real.exp_bound_div_one_sub_of_interval' {x : } (h1 : 0 < x) (h2 : x < 1) :
                  exp x < 1 / (1 - x)
                  theorem Real.exp_bound_div_one_sub_of_interval {x : } (h1 : 0 x) (h2 : x < 1) :
                  exp x 1 / (1 - x)
                  theorem Real.add_one_lt_exp {x : } (hx : x 0) :
                  x + 1 < exp x
                  theorem Real.add_one_le_exp (x : ) :
                  x + 1 exp x
                  theorem Real.one_sub_lt_exp_neg {x : } (hx : x 0) :
                  1 - x < exp (-x)
                  theorem Real.one_sub_le_exp_neg (x : ) :
                  1 - x exp (-x)
                  theorem Real.one_sub_div_pow_le_exp_neg {n : } {t : } (ht' : t n) :
                  (1 - t / n) ^ n exp (-t)
                  theorem Real.le_inv_mul_exp (x : ) {c : } (hc : 0 < c) :
                  x c⁻¹ * exp (c * x)

                  Extension for the positivity tactic: Real.exp is always positive.

                  Instances For
                    @[simp]
                    theorem Complex.abs_exp_ofReal (x : ) :
                    abs (exp x) = Real.exp x