playground/coq/misc/lia-stuff.v

17 lines
331 B
Coq

Require Import ssreflect Lia.
Locate "_ <= _".
Search not lt le.
Goal forall (a b: nat),
~(a < b) -> b <= a.
Proof.
lia.
Show Proof. (* Quite big and incomprehensible.
Price to be paid for automation *)
Restart.
move => a b H.
by rewrite -PeanoNat.Nat.nlt_ge.
Show Proof. (* Simpler. More readable *)
Qed.