src/ZF/ex/Term.thy
changeset 1155 928a16e02f9f
parent 753 ec86863e87c8
child 1401 0c439768f45c
--- a/src/ZF/ex/Term.thy	Thu Jun 22 12:58:39 1995 +0200
+++ b/src/ZF/ex/Term.thy	Thu Jun 22 17:13:05 1995 +0200
@@ -28,8 +28,8 @@
 
 defs
   term_rec_def
-   "term_rec(t,d) == \
-\   Vrec(t, %t g. term_case(%x zs. d(x, zs, map(%z.g`z, zs)), t))"
+   "term_rec(t,d) == 
+   Vrec(t, %t g. term_case(%x zs. d(x, zs, map(%z.g`z, zs)), t))"
 
   term_map_def	"term_map(f,t) == term_rec(t, %x zs rs. Apply(f(x), rs))"