src/HOL/Real/RealOrd.thy
author paulson
Wed, 07 Jun 2000 12:14:18 +0200
changeset 9043 ca761fe227d8
parent 9013 9dd0274f76af
child 14265 95b42e69436c
permissions -rw-r--r--
First round of changes, towards installation of simprocs * replacing 0r by (0::real0 * better rewriting, especially pulling out signs in (-x)*y = - (x*y), etc.

(*  Title:	 Real/RealOrd.thy
    ID: 	 $Id$
    Author:      Jacques D. Fleuriot and Lawrence C. Paulson
    Copyright:   1998  University of Cambridge
    Description: Type "real" is a linear order and also 
                 satisfies plus_ac0: + is an AC-operator with zero
*)

RealOrd = RealDef +

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

instance real :: plus_ac0 (real_add_commute,real_add_assoc,real_add_zero_left)

end