Zulip Chat Archive
Stream: mathlib4
Topic: linarith does not know trichotomy?
Siddharth Bhat (Oct 24 2023 at 02:44):
Consider the MWE:
import Mathlib.Tactic
theorem linarith_failure (x y : nat) (h1 : ¬ (x = y)) (h2 : ¬ (x < y)) : x > y :=
by
try linarith
sorry
shouldn't linarith
be able to prove this?
Mario Carneiro (Oct 24 2023 at 03:08):
note re: MWEs: don't suppress errors which are the point of the test. Just use linarith
, not try linarith; sorry
Mario Carneiro (Oct 24 2023 at 03:15):
import Mathlib.Tactic
theorem linarith_failure (x y : Nat) (h1 : ¬ (x = y)) (h2 : ¬ (x < y)) : x > y := by
linarith (config := {splitNe := true})
Last updated: Dec 20 2023 at 11:08 UTC