leanprover / lean4

Lean 4 programming language and theorem prover
https://lean-lang.org
Apache License 2.0
3.82k stars 325 forks source link

`rw?` regression from `v4.7.0` #4062

Open Seasawher opened 2 weeks ago

Seasawher commented 2 weeks ago

Description

in Lean v4.7.0 and mathlib 4.7.0, this code success: (see https://github.com/Seasawher/v470playground/blob/main/V470playground/Basic.lean)

import Mathlib.Tactic

variable (n m : Nat)

example (h : n + m = 0) : n = 0 ↔ m = 0 := by
  /-
  Try this: rw [propext (eq_zero_iff_eq_zero_of_add_eq_zero h)]
  -- "no goals"
  -/
  rw?
  done

But in v4.8.0-rc1, we get "unsolved goals" error.

Additional Information

I am unable to find an example without mathlib dependencies. rw? is not in Lean v4.7.0.

Impact

Add :+1: to issues you consider important. If others are impacted by this issue, please ask them to add :+1: to it.

semorrison commented 2 weeks ago

Oh, sorry, this is a known regression, that rw? no longer works on Iff goals. No immediate plans to work on this.

semorrison commented 2 weeks ago

(But I'd review a PR.)