src/HOL/Nat.thy
author slotosch
Fri, 04 Apr 1997 16:04:28 +0200
changeset 2909 22a8a97b66be
parent 2608 450c9b682a92
child 3370 5c5fdce3a4e4
permissions -rw-r--r--
Added Example Quot CVS ----------------------------------------------------------------------

(*  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