Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit ee74e7f

Browse files
committed
feat(analysis/special_functions/exp_log): tendsto real.log at_top at_top (#3826)
1 parent 863bf79 commit ee74e7f

File tree

1 file changed

+11
-0
lines changed

1 file changed

+11
-0
lines changed

src/analysis/special_functions/exp_log.lean

Lines changed: 11 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -460,6 +460,17 @@ lemma tendsto_pow_mul_exp_neg_at_top_nhds_0 (n : ℕ) : tendsto (λx, x^n * exp
460460
(tendsto_inv_at_top_zero.comp (tendsto_exp_div_pow_at_top n)).congr $ λx,
461461
by rw [function.comp_app, inv_eq_one_div, div_div_eq_mul_div, one_mul, div_eq_mul_inv, exp_neg]
462462

463+
/-- The real logarithm function tends to `+∞` at `+∞`. -/
464+
lemma tendsto_log_at_top : tendsto log at_top at_top :=
465+
begin
466+
rw tendsto_at_top_at_top,
467+
intro b,
468+
use exp b,
469+
intros a hab,
470+
rw [← exp_le_exp, exp_log_eq_abs (ne_of_gt $ lt_of_lt_of_le (exp_pos b) hab)],
471+
exact le_trans hab (le_abs_self a)
472+
end
473+
463474
open_locale big_operators
464475

465476
/-- A crude lemma estimating the difference between `log (1-x)` and its Taylor series at `0`,

0 commit comments

Comments
 (0)