src/ZF/WF.thy
changeset 1401 0c439768f45c
parent 1155 928a16e02f9f
child 1478 2b8c2a7547ab
--- a/src/ZF/WF.thy	Fri Dec 08 19:48:15 1995 +0100
+++ b/src/ZF/WF.thy	Sat Dec 09 13:36:11 1995 +0100
@@ -8,13 +8,13 @@
 
 WF = Trancl + "mono" + "equalities" +
 consts
-  wf           :: "i=>o"
-  wf_on        :: "[i,i]=>o"			("wf[_]'(_')")
+  wf           :: i=>o
+  wf_on        :: [i,i]=>o			("wf[_]'(_')")
 
-  wftrec,wfrec :: "[i, i, [i,i]=>i] =>i"
-  wfrec_on     :: "[i, i, i, [i,i]=>i] =>i"	("wfrec[_]'(_,_,_')")
-  is_recfun    :: "[i, i, [i,i]=>i, i] =>o"
-  the_recfun   :: "[i, i, [i,i]=>i] =>i"
+  wftrec,wfrec :: [i, i, [i,i]=>i] =>i
+  wfrec_on     :: [i, i, i, [i,i]=>i] =>i	("wfrec[_]'(_,_,_')")
+  is_recfun    :: [i, i, [i,i]=>i, i] =>o
+  the_recfun   :: [i, i, [i,i]=>i] =>i
 
 defs
   (*r is a well-founded relation*)