src/HOL/Orderings.thy
changeset 61955 e96292f32c3c
parent 61824 dcbe9f756ae0
child 62521 6383440f41a8
--- a/src/HOL/Orderings.thy	Mon Dec 28 19:23:15 2015 +0100
+++ b/src/HOL/Orderings.thy	Mon Dec 28 21:47:32 2015 +0100
@@ -93,25 +93,25 @@
 begin
 
 notation
-  less_eq  ("op <=") and
-  less_eq  ("(_/ <= _)" [51, 51] 50) and
+  less_eq  ("op \<le>") and
+  less_eq  ("(_/ \<le> _)"  [51, 51] 50) and
   less  ("op <") and
   less  ("(_/ < _)"  [51, 51] 50)
 
-notation (xsymbols)
-  less_eq  ("op \<le>") and
-  less_eq  ("(_/ \<le> _)"  [51, 51] 50)
+abbreviation (input)
+  greater_eq  (infix "\<ge>" 50)
+  where "x \<ge> y \<equiv> y \<le> x"
 
 abbreviation (input)
-  greater_eq  (infix ">=" 50) where
-  "x >= y \<equiv> y <= x"
+  greater  (infix ">" 50)
+  where "x > y \<equiv> y < x"
+
+notation (ASCII)
+  less_eq  ("op <=") and
+  less_eq  ("(_/ <= _)" [51, 51] 50)
 
 notation (input)
-  greater_eq  (infix "\<ge>" 50)
-
-abbreviation (input)
-  greater  (infix ">" 50) where
-  "x > y \<equiv> y < x"
+  greater_eq  (infix ">=" 50)
 
 end
 
@@ -652,7 +652,7 @@
 
 subsection \<open>Bounded quantifiers\<close>
 
-syntax
+syntax (ASCII)
   "_All_less" :: "[idt, 'a, bool] => bool"    ("(3ALL _<_./ _)"  [0, 0, 10] 10)
   "_Ex_less" :: "[idt, 'a, bool] => bool"    ("(3EX _<_./ _)"  [0, 0, 10] 10)
   "_All_less_eq" :: "[idt, 'a, bool] => bool"    ("(3ALL _<=_./ _)" [0, 0, 10] 10)
@@ -663,7 +663,7 @@
   "_All_greater_eq" :: "[idt, 'a, bool] => bool"    ("(3ALL _>=_./ _)" [0, 0, 10] 10)
   "_Ex_greater_eq" :: "[idt, 'a, bool] => bool"    ("(3EX _>=_./ _)" [0, 0, 10] 10)
 
-syntax (xsymbols)
+syntax
   "_All_less" :: "[idt, 'a, bool] => bool"    ("(3\<forall>_<_./ _)"  [0, 0, 10] 10)
   "_Ex_less" :: "[idt, 'a, bool] => bool"    ("(3\<exists>_<_./ _)"  [0, 0, 10] 10)
   "_All_less_eq" :: "[idt, 'a, bool] => bool"    ("(3\<forall>_\<le>_./ _)" [0, 0, 10] 10)