src/HOL/Ord.thy
changeset 8882 9df44a4f1bf7
parent 7357 d0e16da40ea2
child 10227 692e29b9d2b2
--- a/src/HOL/Ord.thy	Thu May 18 11:40:57 2000 +0200
+++ b/src/HOL/Ord.thy	Thu May 18 11:43:57 2000 +0200
@@ -12,26 +12,26 @@
 axclass
   ord < term
 
-global
-
 syntax
   "op <"        :: ['a::ord, 'a] => bool             ("op <")
   "op <="       :: ['a::ord, 'a] => bool             ("op <=")
 
+global
+
 consts
   "op <"        :: ['a::ord, 'a] => bool             ("(_/ < _)"  [50, 51] 50)
   "op <="       :: ['a::ord, 'a] => bool             ("(_/ <= _)" [50, 51] 50)
-  mono          :: ['a::ord => 'b::ord] => bool       (*monotonicity*)
-  min, max      :: ['a::ord, 'a] => 'a
 
-  Least         :: ('a::ord=>bool) => 'a             (binder "LEAST " 10)
+local
 
 syntax (symbols)
   "op <="       :: ['a::ord, 'a] => bool             ("op \\<le>")
   "op <="       :: ['a::ord, 'a] => bool             ("(_/ \\<le> _)"  [50, 51] 50)
 
-
-local
+consts
+  mono          :: ['a::ord => 'b::ord] => bool      (*monotonicity*)
+  min, max      :: ['a::ord, 'a] => 'a
+  Least         :: ('a::ord=>bool) => 'a             (binder "LEAST " 10)
 
 defs
   mono_def      "mono(f) == (!A B. A <= B --> f(A) <= f(B))"