mathlib documentation

data.​complex.​exponential

data.​complex.​exponential

Exponential, trigonometric and hyperbolic trigonometric functions

This file contains the definitions of the real and complex exponential, sine, cosine, tangent, hyperbolic sine, hypebolic cosine, and hyperbolic tangent functions.

theorem forall_ge_le_of_forall_le_succ {α : Type u_1} [preorder α] (f : → α) {m : } (h : ∀ (n : ), n mf n.succ f n) {l : } (k : ) :
k mk lf l f k

theorem is_cau_of_decreasing_bounded {α : Type u_1} [discrete_linear_ordered_field α] [archimedean α] (f : → α) {a : α} {m : } :
(∀ (n : ), n mabs (f n) a)(∀ (n : ), n mf n.succ f n)is_cau_seq abs f

theorem is_cau_of_mono_bounded {α : Type u_1} [discrete_linear_ordered_field α] [archimedean α] (f : → α) {a : α} {m : } :
(∀ (n : ), n mabs (f n) a)(∀ (n : ), n mf n f n.succ)is_cau_seq abs f

theorem is_cau_series_of_abv_le_cau {α : Type u_1} {β : Type u_2} [ring β] [discrete_linear_ordered_field α] {abv : β → α} [is_absolute_value abv] {f : → β} {g : → α} (n : ) :
(∀ (m : ), n mabv (f m) g m)is_cau_seq abs (λ (n : ), (finset.range n).sum (λ (i : ), g i))is_cau_seq abv (λ (n : ), (finset.range n).sum (λ (i : ), f i))

theorem is_cau_series_of_abv_cau {α : Type u_1} {β : Type u_2} [ring β] [discrete_linear_ordered_field α] {abv : β → α} [is_absolute_value abv] {f : → β} :
is_cau_seq abs (λ (m : ), (finset.range m).sum (λ (n : ), abv (f n)))is_cau_seq abv (λ (m : ), (finset.range m).sum (λ (n : ), f n))

theorem is_cau_geo_series {α : Type u_1} [discrete_linear_ordered_field α] [archimedean α] {β : Type u_2} [field β] {abv : β → α} [is_absolute_value abv] (x : β) :
abv x < 1is_cau_seq abv (λ (n : ), (finset.range n).sum (λ (m : ), x ^ m))

theorem is_cau_geo_series_const {α : Type u_1} [discrete_linear_ordered_field α] [archimedean α] (a : α) {x : α} :
abs x < 1is_cau_seq abs (λ (m : ), (finset.range m).sum (λ (n : ), a * x ^ n))

theorem series_ratio_test {α : Type u_1} {β : Type u_2} [ring β] [discrete_linear_ordered_field α] [archimedean α] {abv : β → α} [is_absolute_value abv] {f : → β} (n : ) (r : α) :
0 rr < 1(∀ (m : ), n mabv (f m.succ) r * abv (f m))is_cau_seq abv (λ (m : ), (finset.range m).sum (λ (n : ), f n))

theorem sum_range_diag_flip {α : Type u_1} [add_comm_monoid α] (n : ) (f : → α) :
(finset.range n).sum (λ (m : ), (finset.range (m + 1)).sum (λ (k : ), f k (m - k))) = (finset.range n).sum (λ (m : ), (finset.range (n - m)).sum (λ (k : ), f m k))

theorem sum_range_sub_sum_range {α : Type u_1} [add_comm_group α] {f : → α} {n m : } :
n m(finset.range m).sum (λ (k : ), f k) - (finset.range n).sum (λ (k : ), f k) = (finset.filter (λ (k : ), n k) (finset.range m)).sum (λ (k : ), f k)

theorem abv_sum_le_sum_abv {α : Type u_1} {β : Type u_2} [ring β] [discrete_linear_ordered_field α] {abv : β → α} [is_absolute_value abv] {γ : Type u_3} (f : γ → β) (s : finset γ) :
abv (s.sum (λ (k : γ), f k)) s.sum (λ (k : γ), abv (f k))

theorem cauchy_product {α : Type u_1} {β : Type u_2} [ring β] [discrete_linear_ordered_field α] {abv : β → α} [is_absolute_value abv] {a b : → β} (ha : is_cau_seq abs (λ (m : ), (finset.range m).sum (λ (n : ), abv (a n)))) (hb : is_cau_seq abv (λ (m : ), (finset.range m).sum (λ (n : ), b n))) (ε : α) :
0 < ε(∃ (i : ), ∀ (j : ), j iabv ((finset.range j).sum (λ (k : ), a k) * (finset.range j).sum (λ (k : ), b k) - (finset.range j).sum (λ (n : ), (finset.range (n + 1)).sum (λ (m : ), a m * b (n - m)))) < ε)

theorem complex.​is_cau_abs_exp (z : ) :
is_cau_seq abs (λ (n : ), (finset.range n).sum (λ (m : ), complex.abs (z ^ m / (m.fact))))

theorem complex.​is_cau_exp (z : ) :
is_cau_seq complex.abs (λ (n : ), (finset.range n).sum (λ (m : ), z ^ m / (m.fact)))

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

Equations
def complex.​exp  :

The complex exponential function, defined via its Taylor series

Equations
def complex.​sin  :

The complex sine function, defined via exp

Equations
def complex.​cos  :

The complex cosine function, defined via exp

Equations
def complex.​tan  :

The complex tangent function, defined as sin z / cos z

Equations
def complex.​sinh  :

The complex hyperbolic sine function, defined via exp

Equations
def complex.​cosh  :

The complex hyperbolic cosine function, defined via exp

Equations
def complex.​tanh  :

The complex hyperbolic tangent function, defined as sinh z / cosh z

Equations
def real.​exp  :

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

Equations
def real.​sin  :

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

Equations
def real.​cos  :

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

Equations
def real.​tan  :

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

Equations
def real.​sinh  :

The real hypebolic sine function, defined as the real part of the complex hyperbolic sine

Equations
def real.​cosh  :

The real hypebolic cosine function, defined as the real part of the complex hyperbolic cosine

Equations
def real.​tanh  :

The real hypebolic tangent function, defined as the real part of the complex hyperbolic tangent

Equations
@[simp]

theorem complex.​exp_sum {α : Type u_1} (s : finset α) (f : α → ) :
complex.exp (s.sum (λ (x : α), f x)) = s.prod (λ (x : α), complex.exp (f x))

theorem complex.​exp_nat_mul (x : ) (n : ) :

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

@[simp]

theorem complex.​cos_two_mul (x : ) :
complex.cos (2 * x) = 2 * complex.cos x ^ 2 - 1

theorem complex.​cos_square (x : ) :
complex.cos x ^ 2 = 1 / 2 + complex.cos (2 * x) / 2

@[simp]
theorem real.​exp_zero  :

theorem real.​exp_add (x y : ) :

theorem real.​exp_sum {α : Type u_1} (s : finset α) (f : α → ) :
real.exp (s.sum (λ (x : α), f x)) = s.prod (λ (x : α), real.exp (f x))

theorem real.​exp_nat_mul (x : ) (n : ) :

theorem real.​exp_ne_zero (x : ) :

theorem real.​exp_neg (x : ) :

theorem real.​exp_sub (x y : ) :

@[simp]
theorem real.​sin_zero  :

@[simp]
theorem real.​sin_neg (x : ) :

theorem real.​sin_add (x y : ) :

@[simp]
theorem real.​cos_zero  :

@[simp]
theorem real.​cos_neg (x : ) :

theorem real.​cos_add (x y : ) :

theorem real.​sin_sub (x y : ) :

theorem real.​cos_sub (x y : ) :

@[simp]
theorem real.​tan_zero  :

@[simp]
theorem real.​tan_neg (x : ) :

theorem real.​sin_sq_add_cos_sq (x : ) :
real.sin x ^ 2 + real.cos x ^ 2 = 1

theorem real.​sin_sq_le_one (x : ) :
real.sin x ^ 2 1

theorem real.​cos_sq_le_one (x : ) :
real.cos x ^ 2 1

theorem real.​abs_sin_le_one (x : ) :

theorem real.​abs_cos_le_one (x : ) :

theorem real.​sin_le_one (x : ) :

theorem real.​cos_le_one (x : ) :

theorem real.​neg_one_le_sin (x : ) :

theorem real.​neg_one_le_cos (x : ) :

theorem real.​cos_two_mul (x : ) :
real.cos (2 * x) = 2 * real.cos x ^ 2 - 1

theorem real.​sin_two_mul (x : ) :

theorem real.​cos_square (x : ) :
real.cos x ^ 2 = 1 / 2 + real.cos (2 * x) / 2

theorem real.​sin_square (x : ) :
real.sin x ^ 2 = 1 - real.cos x ^ 2

theorem real.​sinh_eq (x : ) :

The definition of sinh in terms of exp.

@[simp]
theorem real.​sinh_zero  :

@[simp]
theorem real.​sinh_neg (x : ) :

theorem real.​cosh_eq (x : ) :

The definition of cosh in terms of exp.

@[simp]
theorem real.​cosh_zero  :

@[simp]
theorem real.​cosh_neg (x : ) :

@[simp]
theorem real.​tanh_zero  :

@[simp]
theorem real.​tanh_neg (x : ) :

theorem real.​add_one_le_exp_of_nonneg {x : } :
0 xx + 1 real.exp x

theorem real.​one_le_exp {x : } :
0 x1 real.exp x

theorem real.​exp_pos (x : ) :

@[simp]
theorem real.​abs_exp (x : ) :

theorem real.​exp_monotone {x y : } :
x yreal.exp x real.exp y

theorem real.​exp_lt_exp {x y : } :

theorem real.​exp_le_exp {x y : } :

@[simp]
theorem real.​exp_eq_one_iff (x : ) :
real.exp x = 1 x = 0

theorem real.​one_lt_exp_iff {x : } :
1 < real.exp x 0 < x

theorem real.​exp_lt_one_iff {x : } :
real.exp x < 1 x < 0

theorem real.​cosh_pos (x : ) :

real.cosh is always positive

theorem complex.​sum_div_fact_le {α : Type u_1} [discrete_linear_ordered_field α] (n j : ) :
0 < n(finset.filter (λ (k : ), n k) (finset.range j)).sum (λ (m : ), 1 / (m.fact)) (n.succ) * ((n.fact) * n)⁻¹

theorem complex.​exp_bound {x : } (hx : complex.abs x 1) {n : } :
0 < ncomplex.abs (complex.exp x - (finset.range n).sum (λ (m : ), x ^ m / (m.fact))) complex.abs x ^ n * ((n.succ) * ((n.fact) * n)⁻¹)

theorem real.​cos_bound {x : } :
abs x 1abs (real.cos x - (1 - x ^ 2 / 2)) abs x ^ 4 * (5 / 96)

theorem real.​sin_bound {x : } :
abs x 1abs (real.sin x - (x - x ^ 3 / 6)) abs x ^ 4 * (5 / 96)

theorem real.​cos_pos_of_le_one {x : } :
abs x 10 < real.cos x

theorem real.​sin_pos_of_pos_of_le_one {x : } :
0 < xx 10 < real.sin x

theorem real.​sin_pos_of_pos_of_le_two {x : } :
0 < xx 20 < real.sin x

theorem real.​cos_one_le  :
real.cos 1 2 / 3