(************************************************************************) (* v * The Coq Proof Assistant / The Coq Development Team *) (* Logic.eq==>iff) Zlt. Proof. repeat red; intros; subst; auto. Qed. Definition le_lteq := Zle_lt_or_eq_iff. Definition compare_spec := Zcompare_spec. End Z_as_OT. (** Note that [Z_as_OT] can also be seen as a [UsualOrderedType] and a [OrderedType] (and also as a [DecidableType]). *) (** * An [order] tactic for integers *) Module ZOrder := OTF_to_OrderTac Z_as_OT. Ltac z_order := ZOrder.order. (** Note that [z_order] is domain-agnostic: it will not prove [1<=2] or [x<=x+x], but rather things like [x<=y -> y<=x -> x=y]. *)