Zulip Chat Archive
Stream: Is there code for X?
Topic: dominated integrability
Alex Kontorovich (May 14 2024 at 16:44):
I can't seem to find this in the library: If g is integrable on , say, and atTop, then f is integrable:
import Mathlib.MeasureTheory.Integral.IntegrableOn
import Mathlib.Order.Filter.AtTopBot
import Mathlib.MeasureTheory.Measure.Haar.OfBasis
open MeasureTheory Set Filter
example (f g : ℝ → ℝ) (g_integrableOn : IntegrableOn g (Ioi (0 : ℝ)))
(f_le_g_atTop : f =O[atTop] g) : IntegrableOn f (Ioi (0 : ℝ)) := by
sorry
Any hints would be much appreciated; thanks!
Mitchell Lee (May 14 2024 at 16:49):
I don't think this is true because you need a hypothesis about the behavior of f on atBot as well.
Mitchell Lee (May 14 2024 at 16:50):
Also, that f is locally integrable.
Alex Kontorovich (May 14 2024 at 16:51):
Sure, not atBot I think (since I'm only integrating down to 0), but local integrability might be needed. Is there some theorem like this one, with sufficient hypotheses?... Thanks!
Mitchell Lee (May 14 2024 at 16:52):
What about this?
Mitchell Lee (May 14 2024 at 16:52):
Mitchell Lee (May 14 2024 at 16:53):
Or this one: docs#MeasureTheory.LocallyIntegrable.integrable_of_isBigO_cocompact
Alex Kontorovich (May 14 2024 at 16:55):
Great, thanks! This should do what I needed: docs#MeasureTheory.LocallyIntegrableOn.integrableOn_of_isBigO_atTop
Last updated: May 02 2025 at 03:31 UTC