Zulip Chat Archive

Stream: mathlib4

Topic: measurability regression


Gareth Ma (Oct 29 2023 at 19:01):

Mathlib 3:

import measure_theory.function.floor

example : measurable (λ (y : ), int.fract y * y ⁻¹) :=
begin
  measurability
end

Mathlib 4:

import Mathlib.MeasureTheory.Function.Floor

example : Measurable (fun (y : )  Int.fract y * y ⁻¹) := by
  measurability

fails with error

 4:3-4:16: error:
tactic 'aesop' failed, failed to prove the goal after exhaustive search.
 Measurable fun y => Int.fract y * y⁻¹

Gareth Ma (Oct 29 2023 at 19:01):

Am I missing some imports or something?

Gareth Ma (Oct 29 2023 at 19:08):

Solution is Measurable.mul measurable_fract measurable_inv

Junyan Xu (Oct 30 2023 at 19:09):

Possibly related: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Regression.20in.20continuity


Last updated: Dec 20 2023 at 11:08 UTC