Zulip Chat Archive
Stream: lean4
Topic: goal at the end of `simp at`
Horațiu Cheval (Aug 03 2022 at 15:22):
It seems that ⊢
can only be placed last in the list of a simp at
tactic call.
example (h h' : True) : True ∧ False := by
simp at h ⊢ h'
-- unknown tactic
but simp at h h' ⊢
works. Is this by design?
Mario Carneiro (Aug 03 2022 at 16:28):
It's a pretty meaningless piece of syntax flexibility
Last updated: Dec 20 2023 at 11:08 UTC