Zulip Chat Archive
Stream: mathlib4
Topic: Two simple calculus lemmas
Michael Stoll (Nov 18 2024 at 16:49):
I need the following two results, but find it hard to produce elegant proofs:
import Mathlib
open Topology Filter
lemma foo {f : ℝ → ℝ} {x : ℝ} (hf : ContinuousAt f x) :
∃ C : ℝ, ∀ᶠ (y : ℝ) in (𝓝 x), C ≤ f y := by
sorry
lemma bar {a : ℝ} (ha : a > 0) (b : ℝ) :
Tendsto (fun x : ℝ ↦ a / (x - b)) (𝓝[>] b) atTop := by
sorry
Any pointers?
Alex Kontorovich (Nov 18 2024 at 17:22):
For the first one, won't something like use f x - 1
and then eventually_lt_of_tendsto_lt work?
Matt Diamond (Nov 18 2024 at 17:33):
lemma foo {f : ℝ → ℝ} {x : ℝ} (hf : ContinuousAt f x) :
∃ C : ℝ, ∀ᶠ (y : ℝ) in (𝓝 x), C ≤ f y :=
⟨f x - 1, eventually_ge_of_tendsto_gt (by simp) hf.tendsto⟩
Alex Kontorovich (Nov 18 2024 at 17:38):
lemma foo {f : ℝ → ℝ} {x : ℝ} (hf : ContinuousAt f x) :
∃ C : ℝ, ∀ᶠ (y : ℝ) in (𝓝 x), C ≤ f y := by
exact ⟨f x - 1, eventually_ge_of_tendsto_gt (by linarith) hf⟩
Alex Kontorovich (Nov 18 2024 at 17:42):
Second one should use tendsto_inv_zero_atTop
. (inv
is better than ...)
Michael Stoll (Nov 18 2024 at 18:40):
Thanks! This helps.
Michael Stoll (Nov 18 2024 at 18:41):
And is there a better way of showing Tendsto (fun x ↦ x - 1) (𝓝[>] 1) (𝓝[>] 0)
than going via epsilons and deltas? apply?
is decidedly unhelpful in this part of the library...
Jireh Loreaux (Nov 18 2024 at 19:07):
You'll want to use docs#ContinuousWithinAt.tendsto_nhdsWithin_image
Jireh Loreaux (Nov 18 2024 at 19:08):
Note that 𝓝[>] 1
is just notation for nhdsWithin 1 (Set.Ioi 1)
Last updated: May 02 2025 at 03:31 UTC