Zulip Chat Archive
Stream: Is there code for X?
Topic: L'Hôpital's rule for infinity/infinity
Aaron Hill (Feb 02 2025 at 18:15):
I found https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Calculus/LHopital.html but it only seems to handle the 0/0 case, not the infinity/infinity case. Do we have any theorems for that case?
Kevin Buzzard (Feb 02 2025 at 18:42):
Can you state the theorem that you're looking for (ideally in lean but even in maths would be a start)
Aaron Hill (Feb 03 2025 at 01:25):
What I'd like is that if f(x) -> infinity
and g(x) -> infinity
as x -> infinity
, then f(x)/g(x) -> f'(x)/g'(x)
(assuming both are differentiable). Specifically, an atTop
(instead of nhds 0
) version of https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Calculus/LHopital.html#HasDerivAt.lhopital_zero_atTop:
import Mathlib
import Mathlib.Topology.Defs.Filter
open Filter
open Topology
theorem lhopital_atTop_atTop {a b : ℝ} {l : Filter ℝ} {f f' g g' : ℝ → ℝ} (hff' : ∀ᶠ x in atTop, HasDerivAt f (f' x) x)
(hgg' : ∀ᶠ x in atTop, HasDerivAt g (g' x) x) (hg' : ∀ᶠ x in atTop, g' x ≠ 0)
(hftop : Tendsto f atTop atTop) (hgtop : Tendsto g atTop atTop)
(hdiv : Tendsto (fun x => f' x / g' x) atTop l) : Tendsto (fun x => f x / g x) atTop l := by
sorry
Last updated: May 02 2025 at 03:31 UTC