Zulip Chat Archive

Stream: mathlib4

Topic: IsLittleO as Tendsto


Yury G. Kudryashov (Nov 13 2023 at 05:02):

In a project I'm working on, I need the following filter:

def myFilter : Filter  :=  (c : ) (_ : 0 < c), 𝓟 {z | |z.im|  c * z.re ^ 2}

lemma tendsto_myFilter {α} {f : α  } {l} :
    Tendsto f l myFilter  (fun x  (f x).im) =o[l] (fun x  (f x).re ^ 2) := sorry

Yury G. Kudryashov (Nov 13 2023 at 05:05):

I think about addint a more general version to Mathlib. E.g.,

def Filter.littleO (f : α  E) (g : α  F) : Filter α :=  (c : ) (_ : 0 < c), 𝓟 {x | f x  c * g x}

Yury G. Kudryashov (Nov 13 2023 at 05:05):

Is there a better approach?


Last updated: Dec 20 2023 at 11:08 UTC