src/HOL/HOL.thy
changeset 19039 8eae46249628
parent 18887 6ad81e3fa478
child 19121 d7fd5415a781
--- a/src/HOL/HOL.thy	Tue Feb 14 17:07:11 2006 +0100
+++ b/src/HOL/HOL.thy	Tue Feb 14 17:07:48 2006 +0100
@@ -1397,9 +1397,9 @@
   "op -->" "HOL.op_implies"
   "op &" "HOL.op_and"
   "op |" "HOL.op_or"
-  "op +" "IntDef.op_add"
-  "op -" "IntDef.op_minus"
-  "op *" "IntDef.op_times"
+  "op +" "HOL.op_add"
+  "op -" "HOL.op_minus"
+  "op *" "HOL.op_times"
   Not "HOL.not"
   uminus "HOL.uminus"
   arbitrary "HOL.arbitrary"
@@ -1419,9 +1419,9 @@
     ml (infixl 0 "orelse")
     haskell (infixl 2 "||")
   If
-    ml ("if __/ then __/ else __")
-    haskell ("if __/ then __/ else __")
-  "op =" (* an intermediate solution *)
+    ml (target_atom "(if __/ then __/ else __)")
+    haskell (target_atom "(if __/ then __/ else __)")
+  "op =" (* an intermediate solution for polymorphic equality *)
     ml (infixl 6 "=")
     haskell (infixl 4 "==")
   arbitrary