src/HOL/Real/Real.thy
author paulson
Thu, 10 Jun 1999 10:39:38 +0200
changeset 6811 4700ca722bbd
parent 5588 a3ab526bb891
child 7077 60b098bb8b8a
permissions -rw-r--r--
Always_LeadsTo_pre. Always_LeadsTo_post: new equivalences suggested by Misra

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