src/HOL/Wellfounded.thy
changeset 32263 8bc0fd4a23a0
parent 32244 a99723d77ae0
child 32461 eee4fa79398f
--- a/src/HOL/Wellfounded.thy	Tue Jul 28 08:49:03 2009 +0200
+++ b/src/HOL/Wellfounded.thy	Tue Jul 28 13:37:08 2009 +0200
@@ -283,8 +283,10 @@
 apply (blast elim!: allE)  
 done
 
-lemmas wfP_SUP = wf_UN [where I=UNIV and r="\<lambda>i. {(x, y). r i x y}",
-  to_pred SUP_UN_eq2 bot_empty_eq pred_equals_eq, simplified, standard]
+lemma wfP_SUP:
+  "\<forall>i. wfP (r i) \<Longrightarrow> \<forall>i j. r i \<noteq> r j \<longrightarrow> inf (DomainP (r i)) (RangeP (r j)) = bot \<Longrightarrow> wfP (SUPR UNIV r)"
+  by (rule wf_UN [where I=UNIV and r="\<lambda>i. {(x, y). r i x y}", to_pred SUP_UN_eq2 pred_equals_eq])
+    (simp_all add: bot_fun_eq bot_bool_eq)
 
 lemma wf_Union: 
  "[| ALL r:R. wf r;