src/HOL/Integ/IntDef.thy
changeset 21552 da4e5237dda2
parent 21454 a1937c51ed88
child 21820 2f2b6a965ccc
--- a/src/HOL/Integ/IntDef.thy	Mon Nov 27 13:42:47 2006 +0100
+++ b/src/HOL/Integ/IntDef.thy	Mon Nov 27 13:42:48 2006 +0100
@@ -921,7 +921,7 @@
   (SML "!((_ : IntInf.int) = _)")
   (Haskell infixl 4 "==")
 
-code_const "op <= \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
+code_const "op \<le> \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
   (SML "IntInf.<= (_, _)")
   (Haskell infix 4 "<=")