Zulip Chat Archive
Stream: Is there code for X?
Topic: Adding big-O
Gareth Ma (May 05 2024 at 16:28):
Is there code for the following?
example {f g h : ℤ → ℝ} (hf : f =O[atTop] h) (hg : g =O[atTop] h) : (f + g) =O[atTop] h := by
sorry
Yaël Dillies (May 05 2024 at 16:29):
Gareth Ma (May 05 2024 at 16:30):
wtf I swear when I tried hf.add
5 minutes ago it didn't work
Gareth Ma (May 05 2024 at 16:30):
Thanks sorry
Jireh Loreaux (May 05 2024 at 21:34):
@Gareth Ma You can also do the following, which fails to find anything because the terms are kind of eta-expanded (not exactly).
@loogle ⊢ (?f + ?g) =O[?l] ?h
Jireh Loreaux (May 05 2024 at 21:34):
@loogle ⊢ (?f + ?g) =O[?l] ?h
loogle (May 05 2024 at 21:35):
:shrug: nothing found
Jireh Loreaux (May 05 2024 at 21:35):
3rd hit:
@loogle HAdd.hAdd, ⊢ ?f =O[?l] ?h
loogle (May 05 2024 at 21:35):
:search: Asymptotics.IsLittleO.right_isBigO_add, Asymptotics.IsLittleO.right_isBigO_add', and 11 more
Jireh Loreaux (May 05 2024 at 21:36):
1st hit:
@loogle ⊢ (fun x ↦ ?f x + ?g x) =O[?l] ?h
loogle (May 05 2024 at 21:36):
:search: Asymptotics.IsBigO.add, Asymptotics.IsBigO.add_isLittleO, and 2 more
Last updated: May 02 2025 at 03:31 UTC