src/HOL/Main.thy
changeset 55065 6d0af3c10864
parent 55062 6d3fad6f01c9
child 55066 4e5ddf3162ac
--- a/src/HOL/Main.thy	Mon Jan 20 18:24:56 2014 +0100
+++ b/src/HOL/Main.thy	Mon Jan 20 18:24:56 2014 +0100
@@ -18,10 +18,10 @@
   sup (infixl "\<squnion>" 65) and
   Inf ("\<Sqinter>_" [900] 900) and
   Sup ("\<Squnion>_" [900] 900) and
-  ordLeq2 ("<=o") and
-  ordLeq3 ("\<le>o") and
-  ordLess2 ("<o") and
-  ordIso2 ("=o") and
+  ordLeq2 (infix "<=o" 50) and
+  ordLeq3 (infix "\<le>o" 50) and
+  ordLess2 (infix "<o" 50) and
+  ordIso2 (infix "=o" 50) and
   csum (infixr "+c" 65) and
   cprod (infixr "*c" 80) and
   cexp (infixr "^c" 90)