src/HOL/Orderings.thy
changeset 19277 f7602e74d948
parent 19039 8eae46249628
child 19527 9b5c38e8e780
--- a/src/HOL/Orderings.thy	Thu Mar 16 20:19:25 2006 +0100
+++ b/src/HOL/Orderings.thy	Fri Mar 17 09:34:23 2006 +0100
@@ -18,24 +18,20 @@
   ord < type
 
 syntax
-  "op <"        :: "['a::ord, 'a] => bool"             ("op <")
-  "op <="       :: "['a::ord, 'a] => bool"             ("op <=")
-
-global
+  "less"        :: "['a::ord, 'a] => bool"             ("op <")
+  "less_eq"     :: "['a::ord, 'a] => bool"             ("op <=")
 
 consts
-  "op <"        :: "['a::ord, 'a] => bool"             ("(_/ < _)"  [50, 51] 50)
-  "op <="       :: "['a::ord, 'a] => bool"             ("(_/ <= _)" [50, 51] 50)
-
-local
+  "less"        :: "['a::ord, 'a] => bool"             ("(_/ < _)"  [50, 51] 50)
+  "less_eq"     :: "['a::ord, 'a] => bool"             ("(_/ <= _)" [50, 51] 50)
 
 syntax (xsymbols)
-  "op <="       :: "['a::ord, 'a] => bool"             ("op \<le>")
-  "op <="       :: "['a::ord, 'a] => bool"             ("(_/ \<le> _)"  [50, 51] 50)
+  "less_eq"     :: "['a::ord, 'a] => bool"             ("op \<le>")
+  "less_eq"     :: "['a::ord, 'a] => bool"             ("(_/ \<le> _)"  [50, 51] 50)
 
 syntax (HTML output)
-  "op <="       :: "['a::ord, 'a] => bool"             ("op \<le>")
-  "op <="       :: "['a::ord, 'a] => bool"             ("(_/ \<le> _)"  [50, 51] 50)
+  "less_eq"     :: "['a::ord, 'a] => bool"             ("op \<le>")
+  "less_eq"     :: "['a::ord, 'a] => bool"             ("(_/ \<le> _)"  [50, 51] 50)
 
 text{* Syntactic sugar: *}
 
@@ -310,11 +306,11 @@
 	    if of_sort t1
 	    then SOME (t1, "=", t2)
 	    else NONE
-	| dec (Const ("op <=",  _) $ t1 $ t2) =
+	| dec (Const ("Orderings.less_eq",  _) $ t1 $ t2) =
 	    if of_sort t1
 	    then SOME (t1, "<=", t2)
 	    else NONE
-	| dec (Const ("op <",  _) $ t1 $ t2) =
+	| dec (Const ("Orderings.less",  _) $ t1 $ t2) =
 	    if of_sort t1
 	    then SOME (t1, "<", t2)
 	    else NONE
@@ -548,35 +544,35 @@
     if v=v' andalso not (v mem (map fst (Term.add_frees n [])))
     then Syntax.const q $ Syntax.mark_bound v' $ n $ P else raise Match;
   fun all_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op -->",_) $ (Const ("op <",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
+               Const("op -->",_) $ (Const ("Orderings.less",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
     mk v v' "_lessAll" n P
 
   | all_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op -->",_) $ (Const ("op <=",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
+               Const("op -->",_) $ (Const ("Orderings.less_eq",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
     mk v v' "_leAll" n P
 
   | all_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op -->",_) $ (Const ("op <",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
+               Const("op -->",_) $ (Const ("Orderings.less",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
     mk v v' "_gtAll" n P
 
   | all_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op -->",_) $ (Const ("op <=",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
+               Const("op -->",_) $ (Const ("Orderings.less_eq",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
     mk v v' "_geAll" n P;
 
   fun ex_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op &",_) $ (Const ("op <",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
+               Const("op &",_) $ (Const ("Orderings.less",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
     mk v v' "_lessEx" n P
 
   | ex_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op &",_) $ (Const ("op <=",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
+               Const("op &",_) $ (Const ("Orderings.less_eq",_) $ (Const ("_bound",_) $ Free (v',_)) $ n ) $ P] =
     mk v v' "_leEx" n P
 
   | ex_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op &",_) $ (Const ("op <",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
+               Const("op &",_) $ (Const ("Orderings.less",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
     mk v v' "_gtEx" n P
 
   | ex_tr' [Const ("_bound",_) $ Free (v,_),
-               Const("op &",_) $ (Const ("op <=",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
+               Const("op &",_) $ (Const ("Orderings.less_eq",_) $ n $ (Const ("_bound",_) $ Free (v',_))) $ P] =
     mk v v' "_geEx" n P
 in
 [("ALL ", all_tr'), ("EX ", ex_tr')]
@@ -703,10 +699,4 @@
   leave out the "(xtrans)" above.
 *)
 
-subsection {* Code generator setup *}
-
-code_alias
-  "op <=" "Orderings.op_le"
-  "op <" "Orderings.op_lt"
-
 end