src/HOL/Real/RealOrd.thy
author paulson
Tue, 21 Sep 1999 10:39:33 +0200
changeset 7545 1578f1fd62cf
parent 7334 a90fc1e5fb19
child 7588 26384af93359
permissions -rw-r--r--
fixed SOUNDNESS BUG concerning the map from terms like ?f x y to SVC variables

(*  Title:	Real/RealOrd.thy
    ID: 	$Id$
    Author:     Lawrence C. Paulson
                Jacques D. Fleuriot
    Copyright:   1998  University of Cambridge
    Description: Type "real" is a linear order
*)

RealOrd = RealDef +

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

end