src/HOL/Main.thy
changeset 16587 b34c8aa657a5
parent 15965 f422f8283491
child 16635 bf7de5723c60
--- a/src/HOL/Main.thy	Tue Jun 28 15:26:45 2005 +0200
+++ b/src/HOL/Main.thy	Tue Jun 28 15:27:45 2005 +0200
@@ -26,7 +26,7 @@
   "Not"     ("not")
   "op |"    ("(_ orelse/ _)")
   "op &"    ("(_ andalso/ _)")
-  "If"      ("(if _/ then _/ else _)")
+  "HOL.If"      ("(if _/ then _/ else _)")
 
   "wfrec"   ("wf'_rec?")