Open
Description
Lean4's smart unfolding relies on the markers markSmartUnfoldigMatch
and markSmartUnfoldigMatchAlt
. Since they are not present in mathbin definitions, definitional equality checks sometimes loop:
import Mathbin.Data.Int.Basic
example (n : ℕ) (x y : ℤ) : npowRec n x = npowRec n y := rfl
-- maximum recursion depth has been reached (use `set_option maxRecDepth <num>` to increase limit)
Metadata
Metadata
Assignees
Labels
No labels