Zulip Chat Archive

Stream: general

Topic: lt_of_le_of_ne{,'}


Johan Commelin (Feb 12 2019 at 12:19):

Is there any reason for this?

#print lt_of_le_of_ne
-- theorem lt_of_le_of_ne : ∀ {α : Type u} [_inst_1 : partial_order α] {a b : α},
-- a ≤ b → a ≠ b → a < b := _
#print lt_of_le_of_ne'
-- theorem lt_of_le_of_ne' : ∀ {α : Type u} [_inst_1 : partial_order α] {a b : α},
-- a ≤ b → a ≠ b → a < b := _

Mario Carneiro (Feb 12 2019 at 12:19):

the proof is different, probably

Kevin Buzzard (Feb 12 2019 at 12:19):

IIRC one uses an axiom

Kevin Buzzard (Feb 12 2019 at 12:20):

and Kenny wasn't happy

Kevin Buzzard (Feb 12 2019 at 12:20):

Not all proofs are equal after all!

Mario Carneiro (Feb 12 2019 at 12:21):

aha

#print axioms lt_of_le_of_ne
-- classical.choice
-- quot.sound
-- propext
#print axioms lt_of_le_of_ne'
-- no axioms

Johan Commelin (Feb 12 2019 at 12:23):

Aaahrg... I see.

Johan Commelin (Feb 12 2019 at 12:23):

Ok, I'll be nice, and use the ' version.

Mario Carneiro (Feb 12 2019 at 12:24):

if you don't care, probably don't bother

Johan Commelin (Feb 12 2019 at 12:24):

It would be nice if there was a comment explaining this reason in the source (@Kenny Lau, you are missing chances to spread the word)

Mario Carneiro (Feb 12 2019 at 12:24):

one day the tick will go away and that's one less thing to fix in your proof

Kevin Buzzard (Feb 12 2019 at 12:25):

an axiomall the axioms

Kenny Lau (Feb 12 2019 at 13:13):

what is the format of the title of this thread? It doesn't look like regex

Johan Commelin (Feb 12 2019 at 13:15):

It's a bashism

Johan Commelin (Feb 12 2019 at 13:16):

mv file.{txt,tex} will do mv file.txt file.tex


Last updated: Dec 20 2023 at 11:08 UTC