src/ZF/Resid/Redex.thy
changeset 1155 928a16e02f9f
parent 1048 5ba0314f8214
child 1401 0c439768f45c
--- a/src/ZF/Resid/Redex.thy	Thu Jun 22 12:58:39 1995 +0200
+++ b/src/ZF/Resid/Redex.thy	Thu Jun 22 17:13:05 1995 +0200
@@ -21,8 +21,8 @@
  
 defs
   redex_rec_def
-   "redex_rec(p,b,c,d) == \
-\   Vrec(p, %p g.redexes_case(b, %x.c(x,g`x),   \
-\                             %n x y.d(n, x, y, g`x, g`y), p))"
+   "redex_rec(p,b,c,d) == 
+   Vrec(p, %p g.redexes_case(b, %x.c(x,g`x),   
+                             %n x y.d(n, x, y, g`x, g`y), p))"
 end