Zulip Chat Archive
Stream: mathlib4
Topic: timeout synthesizing MeasurableDiv2 R
llllvvuu (Apr 02 2024 at 06:21):
I was reminded of this again today: https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/MeasurableDiv.20for.20Complex.20and.20Real.20types/near/419670355
I wrote it off at the time, but I wonder if the UX can/should be improved here? (if intended behavior, no problem, otherwise I'd be interested to learn how to fix this!)
In PNT+ I've put the following:
-- TODO: why do we need to bump this?
instance : MeasurableDiv₂ ℝ := by
haveI (G : Type) [DivInvMonoid G] [MeasurableSpace G] [MeasurableInv G] [MeasurableMul₂ G] :
MeasurableDiv₂ G := inferInstance
exact this ℝ
Mario Carneiro (Apr 02 2024 at 06:27):
#mwe?
llllvvuu (Apr 02 2024 at 06:30):
The one from the linked message still works:
import Mathlib
instance : MeasurableDiv₂ ℂ := inferInstance
instance : MeasurableDiv₂ ℝ := inferInstance
failed to synthesize
MeasurableDiv₂ ℂ
(deterministic) timeout at 'typeclass', maximum number of heartbeats (20000) has been reached
I'm not well-versed in reading synthInstance traces but it looks like a maybe a wide search or a search that's getting stuck on non-true goals like DiscreteMeasurableSpace
?
Last updated: May 02 2025 at 03:31 UTC