src/ZF/Constructible/WF_absolute.thy
changeset 13269 3ba9be497c33
parent 13268 240509babf00
child 13293 09276ee04361
--- a/src/ZF/Constructible/WF_absolute.thy	Mon Jul 01 18:16:18 2002 +0200
+++ b/src/ZF/Constructible/WF_absolute.thy	Tue Jul 02 13:28:08 2002 +0200
@@ -1,20 +1,5 @@
 theory WF_absolute = WFrec:
 
-(*????move to Wellorderings.thy*)
-lemma (in M_axioms) wellfounded_on_field_imp_wellfounded:
-     "wellfounded_on(M, field(r), r) ==> wellfounded(M,r)"
-by (simp add: wellfounded_def wellfounded_on_iff_wellfounded, fast)
-
-lemma (in M_axioms) wellfounded_iff_wellfounded_on_field:
-     "M(r) ==> wellfounded(M,r) <-> wellfounded_on(M, field(r), r)"
-by (blast intro: wellfounded_imp_wellfounded_on
-                 wellfounded_on_field_imp_wellfounded)
-
-lemma (in M_axioms) wellfounded_on_subset_A:
-     "[| wellfounded_on(M,A,r);  B<=A |] ==> wellfounded_on(M,B,r)"
-by (simp add: wellfounded_on_def, blast)
-
-
 subsection{*Every well-founded relation is a subset of some inverse image of
       an ordinal*}