src/HOL/Nat.thy
author nipkow
Wed, 12 Feb 1997 18:53:59 +0100
changeset 2608 450c9b682a92
parent 2541 70aa00ed3025
child 3370 5c5fdce3a4e4
permissions -rw-r--r--
New class "order" and accompanying changes. In particular reflexivity of <= is now one rewrite rule.

(*  Title:      HOL/Nat.thy
    ID:         $Id$
    Author:     Tobias Nipkow
    Copyright   1997 TU Muenchen

Nat is a partial order
*)

Nat = NatDef +

instance nat :: order (le_refl,le_trans,le_anti_sym,nat_less_le)

end