mathlib documentation

analysis.​special_functions.​exp_log

analysis.​special_functions.​exp_log

Complex and real exponential, real logarithm

Main statements

This file establishes the basic analytical properties of the complex and real exponential functions (continuity, differentiability, computation of the derivative).

It also contains the definition of the real logarithm function (as the inverse of the exponential on (0, +∞), extended to by setting log (-x) = log x) and its basic properties (continuity, differentiability, formula for the derivative).

The complex logarithm is not defined in this file as it relies on trigonometric functions. See instead trigonometric.lean.

Tags

exp, log

The complex exponential is everywhere differentiable, with the derivative exp x.

theorem has_deriv_at.​cexp {f : } {f' x : } :
has_deriv_at f f' xhas_deriv_at (λ (x : ), complex.exp (f x)) (complex.exp (f x) * f') x

theorem has_deriv_within_at.​cexp {f : } {f' x : } {s : set } :
has_deriv_within_at f f' s xhas_deriv_within_at (λ (x : ), complex.exp (f x)) (complex.exp (f x) * f') s x

@[simp]
theorem differentiable_at.​cexp {f : } {x : } :

theorem differentiable_on.​cexp {f : } {s : set } :

@[simp]
theorem differentiable.​cexp {f : } :

theorem deriv_within_cexp {f : } {x : } {s : set } :

@[simp]
theorem deriv_cexp {f : } {x : } :
differentiable_at f xderiv (λ (x : ), complex.exp (f x)) x = complex.exp (f x) * deriv f x

Register lemmas for the derivatives of the composition of real.exp, real.cos, real.sin, real.cosh and real.sinh with a differentiable function, for standalone use and use with simp.

real.exp

theorem has_deriv_at.​exp {f : } {f' x : } :
has_deriv_at f f' xhas_deriv_at (λ (x : ), real.exp (f x)) (real.exp (f x) * f') x

theorem has_deriv_within_at.​exp {f : } {f' x : } {s : set } :
has_deriv_within_at f f' s xhas_deriv_within_at (λ (x : ), real.exp (f x)) (real.exp (f x) * f') s x

theorem differentiable_within_at.​exp {f : } {x : } {s : set } :

@[simp]
theorem differentiable_at.​exp {f : } {x : } :

theorem differentiable_on.​exp {f : } {s : set } :

@[simp]
theorem differentiable.​exp {f : } :

theorem deriv_within_exp {f : } {x : } {s : set } :

@[simp]
theorem deriv_exp {f : } {x : } :
differentiable_at f xderiv (λ (x : ), real.exp (f x)) x = real.exp (f x) * deriv f x

theorem real.​exists_exp_eq_of_pos {x : } :
0 < x(∃ (y : ), real.exp y = x)

def real.​log  :

The real logarithm function, equal to the inverse of the exponential for x > 0, to log |x| for x < 0, and to 0 for 0. We use this unconventional extension to (-∞, 0] as it gives the formula log (x * y) = log x + log y for all nonzero x and y, and the derivative of log is 1/x away from 0.

Equations
theorem real.​exp_log_eq_abs {x : } :
x 0real.exp (real.log x) = abs x

theorem real.​exp_log {x : } :
0 < xreal.exp (real.log x) = x

theorem real.​exp_log_of_neg {x : } :
x < 0real.exp (real.log x) = -x

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

@[simp]
theorem real.​log_zero  :

@[simp]
theorem real.​log_one  :

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

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

theorem real.​log_mul {x y : } :
x 0y 0real.log (x * y) = real.log x + real.log y

@[simp]

theorem real.​log_le_log {x y : } :
0 < x0 < y(real.log x real.log y x y)

theorem real.​log_lt_log {x y : } :
0 < xx < yreal.log x < real.log y

theorem real.​log_lt_log_iff {x y : } :
0 < x0 < y(real.log x < real.log y x < y)

theorem real.​log_pos_iff {x : } :
0 < x(0 < real.log x 1 < x)

theorem real.​log_pos {x : } :
1 < x0 < real.log x

theorem real.​log_neg_iff {x : } :
0 < x(real.log x < 0 x < 1)

theorem real.​log_neg {x : } :
0 < xx < 1real.log x < 0

theorem real.​log_nonneg {x : } :
1 x0 real.log x

theorem real.​log_nonpos {x : } :
0 xx 1real.log x 0

theorem real.​continuous_log'  :
continuous (λ (x : {x // 0 < x}), real.log x.val)

theorem real.​continuous_log {α : Type u_1} [topological_space α] {f : α → } :
(∀ (a : α), 0 < f a)continuous fcontinuous (λ (a : α), real.log (f a))

Three forms of the continuity of real.log are provided. For the other two forms, see real.continuous_log' and real.continuous_at_log

theorem has_deriv_within_at.​log {f : } {x f' : } {s : set } :
has_deriv_within_at f f' s xf x 0has_deriv_within_at (λ (y : ), real.log (f y)) (f' / f x) s x

theorem has_deriv_at.​log {f : } {x f' : } :
has_deriv_at f f' xf x 0has_deriv_at (λ (y : ), real.log (f y)) (f' / f x) x

theorem differentiable_within_at.​log {f : } {x : } {s : set } :
differentiable_within_at f s xf x 0differentiable_within_at (λ (x : ), real.log (f x)) s x

@[simp]
theorem differentiable_at.​log {f : } {x : } :
differentiable_at f xf x 0differentiable_at (λ (x : ), real.log (f x)) x

theorem differentiable_on.​log {f : } {s : set } :
differentiable_on f s(∀ (x : ), x sf x 0)differentiable_on (λ (x : ), real.log (f x)) s

@[simp]
theorem differentiable.​log {f : } :
differentiable f(∀ (x : ), f x 0)differentiable (λ (x : ), real.log (f x))

theorem deriv_within_log' {f : } {x : } {s : set } :
differentiable_within_at f s xf x 0unique_diff_within_at s xderiv_within (λ (x : ), real.log (f x)) s x = deriv_within f s x / f x

@[simp]
theorem deriv_log' {f : } {x : } :
differentiable_at f xf x 0deriv (λ (x : ), real.log (f x)) x = deriv f x / f x

The real exponential function tends to +∞ at +∞.

The real exponential function tends to 0 at -infinity or, equivalently, exp(-x) tends to 0 at +infinity

The function exp(x)/x^n tends to +infinity at +infinity, for any natural number n

The function x^n * exp(-x) tends to 0 at +∞, for any natural number n.

The real logarithm function tends to +∞ at +∞.

theorem real.​abs_log_sub_add_sum_range_le {x : } (h : abs x < 1) (n : ) :
abs ((finset.range n).sum (λ (i : ), x ^ (i + 1) / (i + 1)) + real.log (1 - x)) abs x ^ (n + 1) / (1 - abs x)

A crude lemma estimating the difference between log (1-x) and its Taylor series at 0, where the main point of the bound is that it tends to 0. The goal is to deduce the series expansion of the logarithm, in has_sum_pow_div_log_of_abs_lt_1.

theorem real.​has_sum_pow_div_log_of_abs_lt_1 {x : } :
abs x < 1has_sum (λ (n : ), x ^ (n + 1) / (n + 1)) (-real.log (1 - x))

Power series expansion of the logarithm around 1.