Zulip Chat Archive
Stream: general
Topic: simp documentation
Simon Hudon (Mar 15 2018 at 00:19):
@Kevin Buzzard I'm having a look at your recent PR. In "When it is unadvisable to use simp", why not use show
instead of suffices
?
Kevin Buzzard (Mar 15 2018 at 00:20):
I think that's kind of backwards
Kevin Buzzard (Mar 15 2018 at 00:20):
let's say you're a long way from a goal
Kevin Buzzard (Mar 15 2018 at 00:20):
and simp makes tiny progress
Kevin Buzzard (Mar 15 2018 at 00:21):
no wait
Kevin Buzzard (Mar 15 2018 at 00:21):
simp changes your goal slightly
Kevin Buzzard (Mar 15 2018 at 00:21):
it makes it into X
Kevin Buzzard (Mar 15 2018 at 00:21):
then suffices X, simpa [this]
does the same thing
Kevin Buzzard (Mar 15 2018 at 00:21):
but show won't work
Kevin Buzzard (Mar 15 2018 at 00:21):
becuase X isn't defeq to the original goal
Kevin Buzzard (Mar 15 2018 at 00:23):
The idiom (is that the right word?) is that if simp changes your goal to X, then why not make a new goal and instantly close it with simp.
Simon Hudon (Mar 15 2018 at 00:24):
Good point. Then you can only choose show
in the special case where the new goal is defeq
to the old one.
Simon Hudon (Mar 15 2018 at 00:25):
It might be worth having a shortcut for suffices : (simplified thing), by simpa [this]
Kevin Buzzard (Mar 15 2018 at 00:30):
yeah, it's simp
;-)
Kevin Buzzard (Mar 15 2018 at 00:31):
simp to (simplified thing)
?
Mario Carneiro (Mar 15 2018 at 00:31):
simpa
was intended for basically exactly that use case. It's not exactly wasting that many keywords as it is
Kevin Buzzard (Mar 15 2018 at 00:31):
yeah but golf
Mario Carneiro (Mar 15 2018 at 00:32):
for golf, simpa [bla] using bla
is even more effective
Kevin Buzzard (Mar 15 2018 at 00:32):
simp {answer := simplified thing}
Mario Carneiro (Mar 15 2018 at 00:33):
also, you can just write suffices : (simplified thing), {simpa}
Last updated: Dec 20 2023 at 11:08 UTC