Zulip Chat Archive

Stream: general

Topic: bug with refine + rw


Kenny Lau (Dec 18 2018 at 08:46):

example (H : (0 = 0  0 = 1)  true) : true :=
begin
  refine H (λ h, _), rw h --fails
/-
rewrite tactic failed, lemma is not an equality nor a iff
state:
H : (0 = 0 → 0 = 1) → true,
h : 0 = 0
⊢ 0 = 1
-/
end


example (H : (0 = 0  0 = 1)  true) : true :=
begin
  refine H _, intro h, rw h --works
end

Kenny Lau (Dec 18 2018 at 08:48):

and also workaround:

example (H : (0 = 0  0 = 1)  true) : true :=
begin
  refine H (λ h, _),
  change _ at h, rw h --works
end

Last updated: Dec 20 2023 at 11:08 UTC