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
Trying to use simp? in conv mode gives an error "unexpected identifier; expected command".
Context
simp and simp only are valid tactics in conv mode. So it would be natural if simp? would also work (and allow to replace simp calls by simp only calls for efficiency).
Prerequisites
Please put an X between the brackets as you perform the following steps:
https://github.com/leanprover/lean4/issues
Avoid dependencies to Mathlib or Batteries.
https://live.lean-lang.org/#project=lean-nightly
(You can also use the settings there to switch to “Lean nightly”)
Description
Trying to use
simp?
inconv
mode gives an error "unexpected identifier; expected command".Context
simp
andsimp only
are valid tactics inconv
mode. So it would be natural ifsimp?
would also work (and allow to replacesimp
calls bysimp only
calls for efficiency).See the discussion on Zulip.
Steps to Reproduce
MWE:
Expected behavior:
simp?
should work inconv
mode in the same way as it does normally.Actual behavior:
simp?
inconv
mode results in an error.Versions
Lean 4.15.0-nightly-2024-11-21
Target: x86_64-unknown-linux-gnu
Impact
Add 👍 to issues you consider important. If others are impacted by this issue, please ask them to add 👍 to it.
The text was updated successfully, but these errors were encountered: