src/ZF/Constructible/WF_absolute.thy
changeset 13647 7f6f0ffc45c3
parent 13634 99a593b49b04
child 16417 9bc16273c2d4
--- a/src/ZF/Constructible/WF_absolute.thy	Mon Oct 14 10:44:32 2002 +0200
+++ b/src/ZF/Constructible/WF_absolute.thy	Mon Oct 14 11:32:00 2002 +0200
@@ -3,7 +3,7 @@
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
 *)
 
-header {*Absoluteness for Well-Founded Relations and Well-Founded Recursion*}
+header {*Absoluteness of Well-Founded Recursion*}
 
 theory WF_absolute = WFrec:
 
@@ -175,13 +175,8 @@
   apply (simp_all add: trancl_type [THEN field_rel_subset])
 done
 
-text{*Relativized to M: Every well-founded relation is a subset of some
-inverse image of an ordinal.  Key step is the construction (in M) of a
-rank function.*}
 
-
-
-text{*absoluteness for wfrec-defined functions.*}
+text{*Absoluteness for wfrec-defined functions.*}
 
 (*first use is_recfun, then M_is_recfun*)