Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2020-04-30 07:10 b14a26ee

View on Github →

refactor(analysis/complex/exponential): split into three files in special_functions/ (#2565) The file analysis/complex/exponential.lean was growing out of control (2500 lines) and was dealing with complex and real exponentials, trigonometric functions, and power functions. I split it into three files corresponding to these three topics, and put them instead in analysis/special_functions/, as it was not specifically complex. This is purely a refactor, so absolutely no new material nor changed proof. Related Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.232565.20exponential.20split

Estimated changes

added theorem complex.continuous_exp
added theorem complex.deriv_exp
added theorem complex.iter_deriv_exp
added theorem deriv_cexp
added theorem deriv_exp
added theorem deriv_log'
added theorem deriv_within_cexp
added theorem deriv_within_exp
added theorem deriv_within_log'
added theorem differentiable.cexp
added theorem differentiable.exp
added theorem differentiable.log
added theorem differentiable_at.cexp
added theorem differentiable_at.exp
added theorem differentiable_at.log
added theorem differentiable_on.cexp
added theorem differentiable_on.exp
added theorem differentiable_on.log
added theorem has_deriv_at.cexp
added theorem has_deriv_at.exp
added theorem has_deriv_at.log
added theorem real.continuous_at_log
added theorem real.continuous_exp
added theorem real.continuous_log'
added theorem real.continuous_log
added theorem real.deriv_exp
added theorem real.exp_log
added theorem real.exp_log_eq_abs
added theorem real.has_deriv_at_exp
added theorem real.has_deriv_at_log
added theorem real.iter_deriv_exp
added theorem real.log_abs
added theorem real.log_exp
added theorem real.log_le_log
added theorem real.log_lt_log
added theorem real.log_lt_log_iff
added theorem real.log_mul
added theorem real.log_neg
added theorem real.log_neg_eq_log
added theorem real.log_neg_iff
added theorem real.log_nonneg
added theorem real.log_nonpos
added theorem real.log_one
added theorem real.log_pos
added theorem real.log_pos_iff
added theorem real.log_zero
added theorem complex.abs_cpow_real
added theorem complex.cpow_add
added theorem complex.cpow_def
added theorem complex.cpow_eq_pow
added theorem complex.cpow_int_cast
added theorem complex.cpow_mul
added theorem complex.cpow_nat_cast
added theorem complex.cpow_neg
added theorem complex.cpow_one
added theorem complex.cpow_zero
added theorem complex.of_real_cpow
added theorem complex.one_cpow
added theorem complex.zero_cpow
added theorem filter.tendsto.nnrpow
added theorem nnreal.coe_rpow
added theorem nnreal.mul_rpow
added theorem nnreal.one_le_rpow
added theorem nnreal.one_lt_rpow
added theorem nnreal.one_rpow
added theorem nnreal.rpow_add
added theorem nnreal.rpow_eq_pow
added theorem nnreal.rpow_le_one
added theorem nnreal.rpow_le_rpow
added theorem nnreal.rpow_lt_one
added theorem nnreal.rpow_lt_rpow
added theorem nnreal.rpow_mul
added theorem nnreal.rpow_nat_cast
added theorem nnreal.rpow_neg
added theorem nnreal.rpow_one
added theorem nnreal.rpow_zero
added theorem nnreal.zero_rpow
added theorem real.continuous_rpow
added theorem real.continuous_sqrt
added theorem real.mul_rpow
added theorem real.one_le_rpow
added theorem real.one_lt_rpow
added theorem real.one_rpow
added theorem real.rpow_add
added theorem real.rpow_def
added theorem real.rpow_def_of_neg
added theorem real.rpow_def_of_pos
added theorem real.rpow_eq_pow
added theorem real.rpow_int_cast
added theorem real.rpow_le_one
added theorem real.rpow_le_rpow
added theorem real.rpow_lt_one
added theorem real.rpow_lt_rpow
added theorem real.rpow_mul
added theorem real.rpow_nat_cast
added theorem real.rpow_neg
added theorem real.rpow_one
added theorem real.rpow_pos_of_pos
added theorem real.rpow_zero
added theorem real.sqrt_eq_rpow
added theorem real.zero_rpow
deleted theorem complex.abs_cpow_inv_nat
deleted theorem complex.abs_cpow_real
deleted theorem complex.continuous_exp
deleted theorem complex.cpow_add
deleted theorem complex.cpow_def
deleted theorem complex.cpow_eq_pow
deleted theorem complex.cpow_eq_zero_iff
deleted theorem complex.cpow_int_cast
deleted theorem complex.cpow_mul
deleted theorem complex.cpow_nat_cast
deleted theorem complex.cpow_nat_inv_pow
deleted theorem complex.cpow_neg
deleted theorem complex.cpow_one
deleted theorem complex.cpow_zero
deleted theorem complex.deriv_exp
deleted theorem complex.has_deriv_at_exp
deleted theorem complex.iter_deriv_exp
deleted theorem complex.of_real_cpow
deleted theorem complex.one_cpow
deleted theorem complex.zero_cpow
deleted theorem deriv_cexp
deleted theorem deriv_exp
deleted theorem deriv_log'
deleted theorem deriv_within_cexp
deleted theorem deriv_within_exp
deleted theorem deriv_within_log'
deleted theorem differentiable.cexp
deleted theorem differentiable.exp
deleted theorem differentiable.log
deleted theorem differentiable_at.cexp
deleted theorem differentiable_at.exp
deleted theorem differentiable_at.log
deleted theorem differentiable_on.cexp
deleted theorem differentiable_on.exp
deleted theorem differentiable_on.log
deleted theorem filter.tendsto.nnrpow
deleted theorem has_deriv_at.cexp
deleted theorem has_deriv_at.exp
deleted theorem has_deriv_at.log
deleted theorem has_deriv_at.rexp
deleted theorem has_deriv_within_at.cexp
deleted theorem has_deriv_within_at.exp
deleted theorem has_deriv_within_at.log
deleted theorem has_deriv_within_at.rexp
deleted theorem nnreal.coe_rpow
deleted theorem nnreal.continuous_at_rpow
deleted theorem nnreal.mul_rpow
deleted theorem nnreal.one_le_rpow
deleted theorem nnreal.one_lt_rpow
deleted theorem nnreal.one_rpow
deleted theorem nnreal.rpow_add
deleted theorem nnreal.rpow_eq_pow
deleted theorem nnreal.rpow_eq_zero_iff
deleted theorem nnreal.rpow_le_one
deleted theorem nnreal.rpow_le_rpow
deleted theorem nnreal.rpow_lt_one
deleted theorem nnreal.rpow_lt_rpow
deleted theorem nnreal.rpow_mul
deleted theorem nnreal.rpow_nat_cast
deleted theorem nnreal.rpow_neg
deleted theorem nnreal.rpow_one
deleted theorem nnreal.rpow_zero
deleted theorem nnreal.zero_rpow
deleted theorem real.abs_rpow_le_abs_rpow
deleted theorem real.continuous_at_log
deleted theorem real.continuous_at_rpow
deleted theorem real.continuous_exp
deleted theorem real.continuous_log'
deleted theorem real.continuous_log
deleted theorem real.continuous_rpow
deleted theorem real.continuous_rpow_aux1
deleted theorem real.continuous_rpow_aux2
deleted theorem real.continuous_rpow_aux3
deleted theorem real.continuous_sqrt
deleted theorem real.deriv_exp
deleted theorem real.differentiable_exp
deleted theorem real.exists_exp_eq_of_pos
deleted theorem real.exp_log
deleted theorem real.exp_log_eq_abs
deleted theorem real.has_deriv_at_exp
deleted theorem real.has_deriv_at_log
deleted theorem real.iter_deriv_exp
deleted theorem real.log_abs
deleted theorem real.log_exp
deleted theorem real.log_le_log
deleted theorem real.log_lt_log
deleted theorem real.log_lt_log_iff
deleted theorem real.log_mul
deleted theorem real.log_neg
deleted theorem real.log_neg_eq_log
deleted theorem real.log_neg_iff
deleted theorem real.log_nonneg
deleted theorem real.log_nonpos
deleted theorem real.log_one
deleted theorem real.log_pos
deleted theorem real.log_pos_iff
deleted theorem real.log_zero
deleted theorem real.mul_rpow
deleted theorem real.one_le_rpow
deleted theorem real.one_lt_rpow
deleted theorem real.one_rpow
deleted theorem real.pow_nat_rpow_nat_inv
deleted theorem real.rpow_add
deleted theorem real.rpow_def
deleted theorem real.rpow_def_of_neg
deleted theorem real.rpow_def_of_nonneg
deleted theorem real.rpow_def_of_nonpos
deleted theorem real.rpow_def_of_pos
deleted theorem real.rpow_eq_pow
deleted theorem real.rpow_int_cast
deleted theorem real.rpow_le_one
deleted theorem real.rpow_le_rpow
deleted theorem real.rpow_lt_one
deleted theorem real.rpow_lt_rpow
deleted theorem real.rpow_mul
deleted theorem real.rpow_nat_cast
deleted theorem real.rpow_nat_inv_pow_nat
deleted theorem real.rpow_neg
deleted theorem real.rpow_one
deleted theorem real.rpow_pos_of_pos
deleted theorem real.rpow_zero
deleted theorem real.sqrt_eq_rpow
deleted theorem real.tendsto_exp_at_top
deleted theorem real.tendsto_log_one_zero
deleted theorem real.zero_rpow