Zulip Chat Archive
Stream: new members
Topic: a > a is false
Debendro Mookerjee (Mar 15 2020 at 01:12):
Is there any way to show that a > a is false in lean?
Bryan Gin-ge Chen (Mar 15 2020 at 01:21):
Here's one way:
import tactic example (a : ℕ) : ¬ a < a := by library_search -- Try this: exact irrefl a example (a : ℕ) : ¬ a < a := irrefl a
Daniel Keys (Mar 15 2020 at 01:23):
Here's another:
lemma L1 (a : ℕ) : ¬ a > a := begin push_neg, apply le_iff_lt_or_eq.2, right, refl, end
Debendro Mookerjee (Mar 15 2020 at 01:26):
Thanks appreciate it!
Last updated: Dec 20 2023 at 11:08 UTC