(************************************************************************) (* * The Coq Proof Assistant / The Coq Development Team *) (* v * INRIA, CNRS and contributors - Copyright 1999-2018 *) (* y<=x -> x=y]. *) Local Open Scope N_scope. Section TestOrder. Let test : forall x y, x<=y -> y<=x -> x=y. Proof. N.order. Qed. End TestOrder.