Zulip Chat Archive

Stream: mathlib4

Topic: exact? regression?


Kevin Buzzard (Mar 05 2024 at 09:51):

I just upgraded my mathlib and now I have this:

import Mathlib

example (a b c : ) (hc : c  0) (h : a * c = b * c) : a = b := by
  exact?
  /-
  function expected
    @ι' (φ j)
  -/

Was that a thing before?

Sébastien Gouëzel (Mar 05 2024 at 09:53):

It's a known issue, soon to be fixed, see https://leanprover.zulipchat.com/#narrow/stream/113486-announce/topic/v4.2E7.2E0-rc1/near/424799730. It should work with fewer imports.

Kevin Buzzard (Mar 05 2024 at 09:54):

Oh yeah I just realised this myself. Thanks!

Kim Morrison (Mar 06 2024 at 10:45):

This is fixed now on master.

Kevin Buzzard (Mar 06 2024 at 16:59):

Indeed, now exact? fails for an older reason :-) (it doesn't find mul_right_cancel₀ hc h because exact? doesn't seem to work on equalities in general)


Last updated: May 02 2025 at 03:31 UTC