Zulip Chat Archive

Stream: Is there code for X?

Topic: Tendsto on divison of linear functions


EdwardW (Sep 24 2024 at 15:17):

Hi :)

Was trying something of the sort:

theorem linear_div_tendsto {𝕂 : Type u_1} [RCLike 𝕂] (a b c d : 𝕂) (hc : c β‰  0) :

Β  Β  Tendsto (fun (x:ℝ) ↦ β€–(a * x + b) / (c * x + d)β€–) atTop (nhds β€–a/cβ€–) := by sorry

This can be solved by dividing through by xx, but that requires x≠0x \neq 0 and is messy algebra. I couldn't find anything particularly helpful in Mathlib. Polynomial.div_tendsto_leadingCoeff_div_of_degree_eq is the closest I can find, but that required an ordered field, which is not necessary here.

Thanks!

Kevin Buzzard (Sep 25 2024 at 07:17):

If I were doing this from first principles on paper I'd subtract and add a/c from ax+b/cx+d to get a/c+(bc-ad)/c(cx+d) and then just prove that the latter tends to zero.

EdwardW (Sep 25 2024 at 08:36):

Yes exactly, I guess I'll do it the hard way, I might investigate the tendsto API as that could do with some additional infrastructure

Bhavik Mehta (Sep 25 2024 at 09:46):

I'd do the proof by dividing through by x, using the fact that (ax+b)/(cx+d) =αΆ [atTop] (a+b/x)/(c+d/x), and then the denominator is eventually nonzero too. Once you state everything in terms of eventually atTop, you can filter upwards and get x != 0 as a hypothesis, then field_simp + ring should make the algebra really easy

EdwardW (Sep 25 2024 at 11:04):

Seems like more effort than Kevin's way, but yes that seems like the way I was going to do it originally

Kevin Buzzard (Sep 25 2024 at 11:27):

It looks to me like about the same amount of effort. The trick is to move away from (ax+b)/(cx+d) (which there won't be any lemmas about, I guess) to functions like b/x or constant functions, which hopefully there will be lemmas about (and then apply results about sum of limits is limit of sums etc)

EdwardW (Sep 25 2024 at 11:44):

For sure, saying that it would definitely be useful to have division of two polynomials, or higher degree polynomials/arbitrary polynomials become really messy

Kevin Buzzard (Sep 25 2024 at 12:38):

Can you formalise the statement about division of two polynomials which you think we should have?

EdwardW (Sep 26 2024 at 12:37):

Probably

theorem Polynomial.RCLike.div_tendsto_leadingCoeff_div_of_degree_eq {π•œ : Type u_1} [RCLike π•œ]
    (P Q : π•œ[X]) (hdeg : P.degree = Q.degree) : Tendsto
    (fun x : β„• ↦ eval ↑x P / eval ↑x Q) atTop (𝓝 (P.leadingCoeff / Q.leadingCoeff)) := by sorry

?

Perhaps I am mistaken, but this doesn't seem trivial, in fact I was working on it just now and it seems like tendsto support for RCLike is somewhat lacking, perhaps this is because this is covered by another typeclass?

Jireh Loreaux (Sep 26 2024 at 14:06):

I think it's not the statement you want. There's no reason to restrict to sequences.

import Mathlib

open Bornology Filter Topology Polynomial

theorem Polynomial.tendsto_div_cobounded_of_degree_eq
    {π•œ : Type*} [NontriviallyNormedField π•œ] (P Q : π•œ[X]) (hdeg : P.degree = Q.degree) :
    Tendsto (fun x : π•œ ↦ eval x P / eval x Q) (cobounded π•œ) (𝓝 (P.leadingCoeff / Q.leadingCoeff)) := by
  sorry

Jireh Loreaux (Sep 26 2024 at 14:14):

Actually, maybe you only need NormedField because of Filter.tendsto_invβ‚€_cobounded

EdwardW (Sep 26 2024 at 14:15):

You are correct, I wasn't sure how to generalise my idea, I suppose then that mine is obtained by composition on an algebraMap. Would it be helpful if I proved this statement?

EdwardW (Sep 26 2024 at 14:18):

/ attempted to :face_with_peeking_eye:

Bhavik Mehta (Nov 12 2024 at 10:21):

I just came across docs#div_tendsto_leadingCoeff_div_of_degree_eq which looks really similar to this, although it's for x atTop rather than cobounded. Maybe it helps here, or for others coming across this thread in the future

Anatole Dedecker (Nov 12 2024 at 12:15):

Yes, in an ideal world everything would follow docs#Polynomial.isEquivalent_atTop_lead. I remember at the time I added this the most annoying part in using it was computing concrete things about concrete polynomials, do we have tactics to do that now?

EdwardW (Nov 12 2024 at 12:34):

Hmm probably not, it would be nice to be corrected. I suppose ring tactics etc would help though


Last updated: May 02 2025 at 03:31 UTC