leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

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: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll