src/ZF/ZF.thy
changeset 6068 2d8f3e1f1151
parent 3940 1d5bee4d047f
child 6340 7d5cbd5819a0
--- a/src/ZF/ZF.thy	Wed Jan 06 15:00:12 1999 +0100
+++ b/src/ZF/ZF.thy	Thu Jan 07 10:56:05 1999 +0100
@@ -40,8 +40,16 @@
   (* Descriptions *)
 
   The         :: (i => o) => i      (binder "THE " 10)
-  if          :: [o, i, i] => i
+  If          :: [o, i, i] => i     ("(if (_)/ then (_)/ else (_))" [10] 10)
+
+syntax
+  old_if      :: [o, i, i] => i   ("if '(_,_,_')")
 
+translations
+  "if(P,a,b)" => "If(P,a,b)"
+
+
+consts
   (* Finite Sets *)
 
   Upair, cons :: [i, i] => i