src/HOL/Real/Real.thy
author wenzelm
Wed, 14 Apr 1999 14:44:04 +0200
changeset 6426 9a2ace82b68e
parent 5588 a3ab526bb891
child 7077 60b098bb8b8a
permissions -rw-r--r--
intrs: names and atts;

(*  Title:      Real/Real.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

Type "real" is a linear order
*)

Real = RealDef +

instance real :: order (real_le_refl,real_le_trans,real_le_anti_sym,real_less_le)
instance real :: linorder (real_le_linear)

end