Skip to content

Commit

Permalink
chore(analysis/special_functions/exp_log): add some missing dot notat…
Browse files Browse the repository at this point in the history
…ion lemmas (#9405)
  • Loading branch information
urkud committed Sep 27, 2021
1 parent 9175158 commit f181d81
Showing 1 changed file with 27 additions and 0 deletions.
27 changes: 27 additions & 0 deletions src/analysis/special_functions/exp_log.lean
Original file line number Diff line number Diff line change
Expand Up @@ -164,6 +164,33 @@ complex.times_cont_diff_exp.times_cont_diff_at.comp_times_cont_diff_within_at x

end

section

variable {α : Type*}

open complex

lemma filter.tendsto.cexp {l : filter α} {f : α → ℂ} {z : ℂ} (hf : tendsto f l (𝓝 z)) :
tendsto (λ x, exp (f x)) l (𝓝 (exp z)) :=
(continuous_exp.tendsto _).comp hf

variables [topological_space α] {f : α → ℂ} {s : set α} {x : α}

lemma continuous_within_at.cexp (h : continuous_within_at f s x) :
continuous_within_at (λ y, exp (f y)) s x :=
h.cexp

lemma continuous_at.cexp (h : continuous_at f x) : continuous_at (λ y, exp (f y)) x :=
h.cexp

lemma continuous_on.cexp (h : continuous_on f s) : continuous_on (λ y, exp (f y)) s :=
λ x hx, (h x hx).cexp

lemma continuous.cexp (h : continuous f) : continuous (λ y, exp (f y)) :=
continuous_iff_continuous_at.2 $ λ x, h.continuous_at.cexp

end

namespace real

variables {x y z : ℝ}
Expand Down

0 comments on commit f181d81

Please sign in to comment.