You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
This is a regression from mathlib's exact? which got removed on the v4.7.0 version bump.
In certain situations, Lean autogenerates constants with names like proof_1 or proof_2. These are not intended to be visible to the end user, but exact? can sometimes suggest them, shadowing more-canonical lemmas.
import Mathlib.Data.PNat.Basic
example (f : Nat → Nat) (a : Nat) (hae : f a = 0)
(h : 0 < Nat.zero) : False := by
exact?
-- Try this: exact PNat.caseStrongInductionOn.proof_1 h
If I comment out the mathlib import, then exact? gives me something more reasonable:
Try this: exact Nat.not_succ_le_zero 0 h
The text was updated successfully, but these errors were encountered:
This is a regression from mathlib's
exact?
which got removed on the v4.7.0 version bump.In certain situations, Lean autogenerates constants with names like
proof_1
orproof_2
. These are not intended to be visible to the end user, butexact?
can sometimes suggest them, shadowing more-canonical lemmas.If I comment out the mathlib import, then exact? gives me something more reasonable:
The text was updated successfully, but these errors were encountered: