Zulip Chat Archive

Stream: Is there code for X?

Topic: Limit of composition


Gareth Ma (Mar 12 2024 at 23:01):

Is there something like this?

example (f g :   ) (h : f =O[atTop] g) (F :   ) (hF : Monotone F) :
    (F  f) =O[atTop] (F  g) := by
  sorry

The idea is simply that if f(x)Cg(x)f(x) \leq Cg(x) then F(f(x))F(Cg(x))F(f(x)) \leq F(Cg(x)) from monotonenes. Add the absolute values yourself...

Gareth Ma (Mar 12 2024 at 23:01):

Also is Moogle down or are there no results?

Screenshot-2024-03-12-at-23.01.38.png

Kevin Buzzard (Mar 12 2024 at 23:03):

Jesse told me earlier today that it was server migration.

Gareth Ma (Mar 12 2024 at 23:13):

Oh I might need some positivity conditions, but yes

Anatole Dedecker (Mar 12 2024 at 23:16):

I’m getting tired but I don’t think this is true ? Sticking to natural numbers for simplicity, take f(n)=n+1f(n)=n +1, g(n)=ng(n) = n, F(n)=n!F(n)=n!. Then for sure f=O(g)f=O(g) but F(f(n))F(g(n))=n+1\frac{F(f(n))}{F(g(n))} = n+1 so we don’t have Ff=O(Fg)F\circ f=O(F\circ g)

Anatole Dedecker (Mar 12 2024 at 23:17):

(deleted)

Gareth Ma (Mar 12 2024 at 23:17):

You probably mean to flip it around? But I think you’re correct

Anatole Dedecker (Mar 12 2024 at 23:18):

Ah yes flipping it seems to work (fixed)

Gareth Ma (Mar 12 2024 at 23:18):

No I think n!∉O((n+1)!)n! \not \in O((n + 1)!).

Gareth Ma (Mar 12 2024 at 23:18):

Yeah

Gareth Ma (Mar 12 2024 at 23:19):

My original goal was to prove that log(1+o(1))=O(1)\log(1 + o(1)) = O(1), and my plan was first prove 1+xexp(x)1 + x \leq \exp(x) i.e. 1+x=O(exp(x))1 + x = O(\exp(x)), then take log for log(1+x)=O(x)\log(1 + x) = O(x)

Gareth Ma (Mar 12 2024 at 23:20):

Actually wait, I can just take log of the inequality directly to get log(1+x)log(exp(x))\log(1 + x) \leq \log(\exp(x))... :man_facepalming: okay I'm getting tired too

Gareth Ma (Mar 12 2024 at 23:20):

Thanks for the help

Anatole Dedecker (Mar 12 2024 at 23:20):

Aaaaaah no I deleted the wrong message

Gareth Ma (Mar 12 2024 at 23:20):

Haha you can recover in the EDITED history

Anatole Dedecker (Mar 12 2024 at 23:23):

Yes but not restore the LaTeX...

Gareth Ma (Mar 12 2024 at 23:23):

:(

Gareth Ma (Mar 12 2024 at 23:24):

I can read it from the history :D

Jesse Michael Han (Mar 13 2024 at 04:17):

Gareth Ma said:

Also is Moogle down or are there no results?

Screenshot-2024-03-12-at-23.01.38.png

Moogle is back online! happy moogling

Notification Bot (Mar 26 2024 at 11:06):

A message was moved from this topic to #general > Moogle down by Jireh Loreaux.


Last updated: May 02 2025 at 03:31 UTC