Skip to content

Commit

Permalink
feat(SpecialFunctions/Log): add tendsto_log_nhdsWithin_zero_right (#…
Browse files Browse the repository at this point in the history
…8554)

I use this lemma several times in an external project.
Also, this lemma doesn't rely on our non-canonical extension of `Real.log` to negative numbers.
  • Loading branch information
urkud committed Nov 27, 2023
1 parent 1412ef2 commit b70e89f
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Mathlib/Analysis/SpecialFunctions/Log/Basic.lean
Expand Up @@ -347,6 +347,9 @@ theorem tendsto_log_nhdsWithin_zero : Tendsto log (𝓝[≠] 0) atBot := by
simpa [← tendsto_comp_exp_atBot] using tendsto_id
#align real.tendsto_log_nhds_within_zero Real.tendsto_log_nhdsWithin_zero

lemma tendsto_log_nhdsWithin_zero_right : Tendsto log (𝓝[>] 0) atBot :=
tendsto_log_nhdsWithin_zero.mono_left <| nhdsWithin_mono _ fun _ h ↦ ne_of_gt h

theorem continuousOn_log : ContinuousOn log {0}ᶜ := by
simp (config := { unfoldPartialApp := true }) only [continuousOn_iff_continuous_restrict,
restrict]
Expand Down

0 comments on commit b70e89f

Please sign in to comment.