batteries icon indicating copy to clipboard operation
batteries copied to clipboard

Bug: `simp?` does not take reverse directions into account

Open sgouezel opened this issue 1 year ago • 1 comments

MWE:

import Std
def foo : Nat → Nat := sorry
theorem foo_eq_iff (z : Nat) : z = 17 ↔ foo z = 3 := sorry
theorem fail (z : Nat) (h : z = 17) : foo z = 3 := by
  simp? [← foo_eq_iff]
  exact h

The simp? works fine, but the suggestion is to use simp only [foo_eq_iff].

sgouezel avatar Sep 15 '23 13:09 sgouezel

Caused by core: leanprover/lean4#2131

JLimperg avatar Sep 18 '23 10:09 JLimperg