src/HOL/Wellfounded.thy
changeset 32244 a99723d77ae0
parent 32235 8f9b8d14fc9f
child 32263 8bc0fd4a23a0
--- a/src/HOL/Wellfounded.thy	Tue Jul 28 08:48:48 2009 +0200
+++ b/src/HOL/Wellfounded.thy	Tue Jul 28 08:48:56 2009 +0200
@@ -886,30 +886,6 @@
   qed
 qed
 
-text {*Wellfoundedness of @{text same_fst}*}
-
-definition
- same_fst :: "('a => bool) => ('a => ('b * 'b)set) => (('a*'b)*('a*'b))set"
-where
-    "same_fst P R == {((x',y'),(x,y)) . x'=x & P x & (y',y) : R x}"
-   --{*For @{text rec_def} declarations where the first n parameters
-       stay unchanged in the recursive call. *}
-
-lemma same_fstI [intro!]:
-     "[| P x; (y',y) : R x |] ==> ((x,y'),(x,y)) : same_fst P R"
-by (simp add: same_fst_def)
-
-lemma wf_same_fst:
-  assumes prem: "(!!x. P x ==> wf(R x))"
-  shows "wf(same_fst P R)"
-apply (simp cong del: imp_cong add: wf_def same_fst_def)
-apply (intro strip)
-apply (rename_tac a b)
-apply (case_tac "wf (R a)")
- apply (erule_tac a = b in wf_induct, blast)
-apply (blast intro: prem)
-done
-
 
 subsection{*Weakly decreasing sequences (w.r.t. some well-founded order) 
    stabilize.*}