src/HOL/Wellfounded_Relations.thy
changeset 19769 c40ce2de2020
parent 19623 12e6cc4382ae
child 22261 9e185f78e7d4
--- a/src/HOL/Wellfounded_Relations.thy	Sun Jun 04 10:52:47 2006 +0200
+++ b/src/HOL/Wellfounded_Relations.thy	Mon Jun 05 14:22:58 2006 +0200
@@ -70,11 +70,13 @@
 apply blast
 done
 
+lemma in_inv_image[simp]: "((x,y) : inv_image r f) = ((f x, f y) : r)"
+  by (auto simp:inv_image_def)
 
 subsubsection{*Finally, All Measures are Wellfounded.*}
 
 lemma in_measure[simp]: "((x,y) : measure f) = (f x < f y)"
-by (auto simp:measure_def inv_image_def)
+  by (simp add:measure_def)
 
 lemma wf_measure [iff]: "wf (measure f)"
 apply (unfold measure_def)
@@ -118,6 +120,10 @@
 apply (drule spec, erule mp, blast) 
 done
 
+lemma in_lex_prod[simp]: 
+  "(((a,b),(a',b')): r <*lex*> s) = ((a,a'): r \<or> (a = a' \<and> (b, b') : s))"
+  by (auto simp:lex_prod_def)
+
 text{*Transitivity of WF combinators.*}
 lemma trans_lex_prod [intro!]: 
     "[| trans R1; trans R2 |] ==> trans (R1 <*lex*> R2)"