src/ZF/ex/Primrec.thy
changeset 1155 928a16e02f9f
parent 753 ec86863e87c8
child 1401 0c439768f45c
--- a/src/ZF/ex/Primrec.thy	Thu Jun 22 12:58:39 1995 +0200
+++ b/src/ZF/ex/Primrec.thy	Thu Jun 22 17:13:05 1995 +0200
@@ -39,12 +39,12 @@
   COMP_def  "COMP(g,fs) == lam l:list(nat). g ` map(%f. f`l, fs)"
 
   (*Note that g is applied first to PREC(f,g)`y and then to y!*)
-  PREC_def  "PREC(f,g) == \
-\            lam l:list(nat). list_case(0, \
-\                      %x xs. rec(x, f`xs, %y r. g ` Cons(r, Cons(y, xs))), l)"
+  PREC_def  "PREC(f,g) == 
+            lam l:list(nat). list_case(0, 
+                      %x xs. rec(x, f`xs, %y r. g ` Cons(r, Cons(y, xs))), l)"
   
-  ACK_def   "ACK(i) == rec(i, SC, \
-\                      %z r. PREC (CONST (r`[1]), COMP(r,[PROJ(0)])))"
+  ACK_def   "ACK(i) == rec(i, SC, 
+                      %z r. PREC (CONST (r`[1]), COMP(r,[PROJ(0)])))"
 
 
 inductive
@@ -57,8 +57,8 @@
     PREC     "[| f: primrec; g: primrec |] ==> PREC(f,g): primrec"
   monos      "[list_mono]"
   con_defs   "[SC_def,CONST_def,PROJ_def,COMP_def,PREC_def]"
-  type_intrs "nat_typechecks @ list.intrs @   		        \
-\	      [lam_type, list_case_type, drop_type, map_type,   \
-\	      apply_type, rec_type]"
+  type_intrs "nat_typechecks @ list.intrs @   		        
+	      [lam_type, list_case_type, drop_type, map_type,   
+	      apply_type, rec_type]"
 
 end