Zulip Chat Archive

Stream: general

Topic: Find what simprocs were used


Heather Macbeth (Aug 28 2024 at 01:26):

On the following example, I believe a simproc is being used:

set_option trace.Debug.Meta.Tactic.simp true
example : (-1:Int) + 1 = 0 := by simp [-eq_self]

The trace shows

[Debug.Meta.Tactic.simp] simproc result -1 + 1 => 0

Is there an option I can set to see which simproc this is?

Heather Macbeth (Aug 28 2024 at 01:29):

:woman_facepalming: I guess simp? [-eq_self] is doing it already:

Try this: simp only [Int.reduceNeg, Int.reduceAdd, Int.reduceEq]

Last updated: May 02 2025 at 03:31 UTC