src/FOLP/ex/If.thy
changeset 19796 d86e7b1fc472
parent 17480 fd19f77dcf60
child 25991 31b38a39e589
--- a/src/FOLP/ex/If.thy	Tue Jun 06 19:24:05 2006 +0200
+++ b/src/FOLP/ex/If.thy	Tue Jun 06 20:42:25 2006 +0200
@@ -5,7 +5,7 @@
 begin
 
 constdefs
-  if :: "[o,o,o]=>o"
+  "if" :: "[o,o,o]=>o"
   "if(P,Q,R) == P&Q | ~P&R"
 
 ML {* use_legacy_bindings (the_context ()) *}