added same_fstI
authoroheimb
Tue, 20 Feb 2001 18:47:30 +0100
changeset 11167 2c90a6167b0b
parent 11166 eca861fd1eb5
child 11168 b964accc9307
added same_fstI
src/HOL/Wellfounded_Relations.ML
--- a/src/HOL/Wellfounded_Relations.ML	Tue Feb 20 18:47:29 2001 +0100
+++ b/src/HOL/Wellfounded_Relations.ML	Tue Feb 20 18:47:30 2001 +0100
@@ -205,6 +205,10 @@
  * Wellfoundedness of same_fst
  *---------------------------------------------------------------------------*)
 
+Goalw[same_fst_def] "[| P x; (y',y) : R x |] ==> ((x,y'),(x,y)) : same_fst P R";
+by (Asm_simp_tac 1);
+qed "same_fstI";
+
 val prems = goalw thy [same_fst_def]
   "(!!x. P x ==> wf(R x)) ==> wf(same_fst P R)";
 by(full_simp_tac (simpset() delcongs [imp_cong] addsimps [wf_def]) 1);