Zulip Chat Archive
Stream: general
Topic: reflection inside rw
Kenny Lau (May 16 2020 at 07:35):
let's say I have this:
theorem test : 1 = 0 :=
by rw [by (tactic.get_goals >>= tactic.trace)]
it seems like tactic.get_goals >>= tactic.trace
cannot see the state outside (i.e. 1 = 0
)
Kenny Lau (May 16 2020 at 07:35):
is there a way to access the outer scope from within rw
?
Keeley Hoek (May 16 2020 at 19:34):
No
Last updated: Dec 20 2023 at 11:08 UTC