Zulip Chat Archive
Stream: new members
Topic: What is `simp only []`
Vaibhav Karve (Jul 01 2020 at 22:34):
What is the list of reductions used by simp only []
? I could not figure it out from the mathlib API documentation at
https://leanprover-community.github.io/mathlib_docs/tactics.html#simp
Mario Carneiro (Jul 01 2020 at 22:36):
Nothing with a name, but it will perform beta reduction and constructor injectivity
Last updated: May 02 2025 at 03:31 UTC