diff -r 304a47739407 -r 04ce6bb14d85 src/HOL/Wellfounded.thy --- a/src/HOL/Wellfounded.thy Thu Sep 24 19:14:18 2009 +0200 +++ b/src/HOL/Wellfounded.thy Fri Sep 25 09:50:31 2009 +0200 @@ -267,8 +267,8 @@ lemma wfP_SUP: "\i. wfP (r i) \ \i j. r i \ r j \ inf (DomainP (r i)) (RangeP (r j)) = bot \ wfP (SUPR UNIV r)" - by (rule wf_UN [where I=UNIV and r="\i. {(x, y). r i x y}", to_pred SUP_UN_eq2 pred_equals_eq]) - (simp_all add: bot_fun_eq bot_bool_eq) + by (rule wf_UN [where I=UNIV and r="\i. {(x, y). r i x y}", to_pred SUP_UN_eq2]) + (simp_all add: Collect_def) lemma wf_Union: "[| ALL r:R. wf r;