src/HOL/Integ/NatBin.thy
changeset 15129 fbf90acc5bf4
parent 15013 34264f5e4691
child 15131 c69542757a4d
--- a/src/HOL/Integ/NatBin.thy	Sat Aug 14 16:27:56 2004 +0200
+++ b/src/HOL/Integ/NatBin.thy	Mon Aug 16 12:29:09 2004 +0200
@@ -839,8 +839,8 @@
   "uminus" :: "int => int"      ("`~")
   "op +" :: "int => int => int" ("(_ `+/ _)")
   "op *" :: "int => int => int" ("(_ `*/ _)")
-  "op div" :: "int => int => int" ("(_ `div/ _)")
-  "op mod" :: "int => int => int" ("(_ `mod/ _)")
+  "op div" :: "int => int => int" ("(_ div/ _)")
+  "op mod" :: "int => int => int" ("(_ mod/ _)")
   "op <" :: "int => int => bool" ("(_ </ _)")
   "op <=" :: "int => int => bool" ("(_ <=/ _)")
   "neg"                         ("(_ < 0)")