src/HOL/Lfp.ML
changeset 3842 b55686a7b22c
parent 1873 b07ee188f061
child 5098 48e70d9fe05f
--- a/src/HOL/Lfp.ML	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOL/Lfp.ML	Fri Oct 10 19:02:28 1997 +0200
@@ -41,7 +41,7 @@
 
 val [lfp,mono,indhyp] = goal Lfp.thy
     "[| a: lfp(f);  mono(f);                            \
-\       !!x. [| x: f(lfp(f) Int {x.P(x)}) |] ==> P(x)   \
+\       !!x. [| x: f(lfp(f) Int {x. P(x)}) |] ==> P(x)   \
 \    |] ==> P(a)";
 by (res_inst_tac [("a","a")] (Int_lower2 RS subsetD RS CollectD) 1);
 by (rtac (lfp RSN (2, lfp_lowerbound RS subsetD)) 1);
@@ -66,7 +66,7 @@
 
 val rew::prems = goal Lfp.thy
     "[| A == lfp(f);  mono(f);   a:A;                   \
-\       !!x. [| x: f(A Int {x.P(x)}) |] ==> P(x)        \
+\       !!x. [| x: f(A Int {x. P(x)}) |] ==> P(x)        \
 \    |] ==> P(a)";
 by (EVERY1 [rtac induct,        (*backtracking to force correct induction*)
             REPEAT1 o (ares_tac (map (rewrite_rule [rew]) prems))]);