doc-src/ZF/If.thy
changeset 35416 d8d7d1b785af
parent 19792 e8e3da6d3ff7
child 42637 381fdcab0f36
--- a/doc-src/ZF/If.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/doc-src/ZF/If.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -8,8 +8,7 @@
 
 theory If imports FOL begin
 
-constdefs
-  "if" :: "[o,o,o]=>o"
+definition "if" :: "[o,o,o]=>o" where
   "if(P,Q,R) == P&Q | ~P&R"
 
 lemma ifI: