src/HOL/Orderings.thy
changeset 20588 c847c56edf0c
parent 19984 29bb4659f80a
child 20714 6a122dba034c
--- a/src/HOL/Orderings.thy	Tue Sep 19 15:21:41 2006 +0200
+++ b/src/HOL/Orderings.thy	Tue Sep 19 15:21:42 2006 +0200
@@ -8,18 +8,16 @@
 header {* Type classes for $\le$ *}
 
 theory Orderings
-imports Lattice_Locales
+imports OperationalEquality Lattice_Locales
 uses ("antisym_setup.ML")
 begin
 
 subsection {* Order signatures and orders *}
 
-axclass
-  ord < type
-
-consts
-  less  :: "['a::ord, 'a] => bool"
-  less_eq  :: "['a::ord, 'a] => bool"
+class ord = eq +
+  constrains eq :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
+  fixes less_eq :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
+  fixes less    :: "'a \<Rightarrow> 'a \<Rightarrow> bool"
 
 const_syntax
   less  ("op <")