src/ZF/Resid/Redex.thy
changeset 3840 e0baea4d485a
parent 2874 b1e7e2179597
child 6046 2c8a8be36c94
--- a/src/ZF/Resid/Redex.thy	Fri Oct 10 18:17:17 1997 +0200
+++ b/src/ZF/Resid/Redex.thy	Fri Oct 10 18:23:31 1997 +0200
@@ -22,7 +22,7 @@
 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))"
+   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