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
axiomα : Typeaxiomβ : Typeaxiomp : α → Propaxiomq : α → Propaxiomr : α → Propaxiomrp : {x : α} → r x ↔ p x
axiomrq : {x : α} → r x ↔ q x
axiomf : (x : α) → p x → β
axiomg : (x : α) → q x → β
axiomy : β
axiomfx : (x : α) → (hx : r x) → f x (rp.mp hx) = g x (rq.mp hx)
example (x : α) (hx : r x) : g x (rq.mp hx) = y := byhave test : y = f x (rp.mp hx) := bysorryhave test₂ : 0 = 0 := by rfl
rw [fx _] at test
exact test.symm
The following code would fail at
exact test.symm
:If remove
test₂
, it would works. I posted this phenomenon to the Zulip channel at https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/A.20subtle.20detail.20about.20Lean.20.60rw.60.20tactic. I also posted some analysis of Lean source code on the thread, and Eric Wieser suggested me to file a bug.The text was updated successfully, but these errors were encountered: