diff -r cd7f9ea58338 -r c26eeb000470 src/ZF/Constructible/WF_absolute.thy --- a/src/ZF/Constructible/WF_absolute.thy Tue Jul 16 16:28:49 2002 +0200 +++ b/src/ZF/Constructible/WF_absolute.thy Tue Jul 16 16:29:36 2002 +0200 @@ -611,19 +611,6 @@ apply (simp add: wfrec_relativize, blast) done -lemma (in M_wfrank) wfrec_closed_lemma [rule_format]: - "[|wf(r); M(r); - strong_replacement(M, \x y. y = \x, wfrec(r, x, H)\); - \x[M]. \g[M]. function(g) --> M(H(x,g)) |] - ==> M(a) --> M(wfrec(r,a,H))" -apply (rule_tac a=a in wf_induct, assumption+) -apply (subst wfrec, assumption, clarify) -apply (drule_tac x1=x and x="\x\r -`` {x}. wfrec(r, x, H)" - in rspec [THEN rspec]) -apply (simp_all add: function_lam) -apply (blast intro: dest: pair_components_in_M ) -done - text{*Full version not assuming transitivity, but maybe not very useful.*} theorem (in M_wfrank) wfrec_closed: "[|wf(r); M(r); M(a);