Zulip Chat Archive

Stream: Is there code for X?

Topic: IntervalIntegrable tactics?


Alex Kontorovich (Mar 28 2024 at 21:57):

Are there integrability tactics that make proving something like this less mind-numbingly tedious? Thanks!

import Mathlib

lemma integrability_aux {a b : } (a_lt_b : a < b) :
    IntervalIntegrable (fun (x : )  (x : ) + 1 / 2 - x) MeasureTheory.volume a b := sorry

Floris van Doorn (Mar 28 2024 at 22:00):

docs#Continuous.intervalIntegrable + the tactic fun_prop?

Floris van Doorn (Mar 28 2024 at 22:00):

Oh, oops, I misread floor as abs.

Floris van Doorn (Mar 28 2024 at 22:03):

Do we have Measurable + Bounded range = Interval integrable? fun_prop can deal with Measurable (maybe with some lemmas about floor tagged), and bounded range is hopefully not too hard.

Vincent Beffara (Mar 28 2024 at 22:29):

You can cook it with docs#IntervalIntegrable.mono_fun' and docs#intervalIntegrable_const


Last updated: May 02 2025 at 03:31 UTC