Zulip Chat Archive
Stream: Is there code for X?
Topic: not some implies none
Marcus Rossel (Jul 15 2021 at 08:17):
Is there a lemma for solving: ?
example {α : Type*} (a : option α) (h : ∀ b, ¬(a = some b)) : a = none := sorry
Or is this only true when α
is inhabited?
Eric Wieser (Jul 15 2021 at 08:23):
Does library_search
help?
Eric Wieser (Jul 15 2021 at 08:24):
cases a
should make quick progress
Eric Rodriguez (Jul 15 2021 at 08:26):
by tidy
solves it
Kevin Buzzard (Jul 15 2021 at 08:30):
I should think the first thing you should do with such a proof is replace it by by tidy?
and see what it actually did, and then remove all the stuff that it did which it didn't need to do
Scott Morrison (Jul 17 2021 at 01:20):
Maybe someone should work on tidy
again: presumably one could generate better output for tidy?
by detecting some common useless steps.
Last updated: Dec 20 2023 at 11:08 UTC