leanprover-community / mathlib4

The math library of Lean 4

Home Page:https://leanprover-community.github.io/mathlib4_docs

Geek Repo:Geek Repo

Github PK Tool:Github PK Tool

Support `Fact` for the `slim_check` tactic

grhkm21 opened this issue · comments

Currently, this fails:

import Mathlib.Tactic.SlimCheck

example {a : ℕ} [Fact a.Prime] : a + 1 = 1 + a := by
  slim_check

While replacing the [Fact a.Prime] instance with (ha : a.Prime) makes it work (with a warning of "Gave up 3 times"). It would be nice for slim_check to support Fact too!