src/ZF/ex/PropLog.thy
changeset 3840 e0baea4d485a
parent 1478 2b8c2a7547ab
child 6046 2c8a8be36c94
--- a/src/ZF/ex/PropLog.thy	Fri Oct 10 18:17:17 1997 +0200
+++ b/src/ZF/ex/PropLog.thy	Fri Oct 10 18:23:31 1997 +0200
@@ -48,7 +48,7 @@
 
   prop_rec_def
    "prop_rec(p,b,c,h) == 
-   Vrec(p, %p g.prop_case(b, c, %x y. h(x, y, g`x, g`y), p))"
+   Vrec(p, %p g. prop_case(b, c, %x y. h(x, y, g`x, g`y), p))"
 
   (** Semantics of propositional logic **)
   is_true_def