--- a/src/HOL/Integ/IntDef.thy Thu Mar 16 20:19:25 2006 +0100
+++ b/src/HOL/Integ/IntDef.thy Fri Mar 17 09:34:23 2006 +0100
@@ -891,8 +891,8 @@
"HOL.uminus" :: "int => int" ("~")
"HOL.plus" :: "int => int => int" ("(_ +/ _)")
"HOL.times" :: "int => int => int" ("(_ */ _)")
- "op <" :: "int => int => bool" ("(_ </ _)")
- "op <=" :: "int => int => bool" ("(_ <=/ _)")
+ "Orderings.less" :: "int => int => bool" ("(_ </ _)")
+ "Orderings.less_eq" :: "int => int => bool" ("(_ <=/ _)")
"neg" ("(_ < 0)")
code_syntax_tyco int