src/HOL/Hilbert_Choice.thy
changeset 54295 45a5523d4a63
parent 52143 36ffe23b25f8
child 54578 9387251b6a46
--- a/src/HOL/Hilbert_Choice.thy	Sun Nov 10 10:02:34 2013 +0100
+++ b/src/HOL/Hilbert_Choice.thy	Sun Nov 10 15:05:06 2013 +0100
@@ -741,7 +741,7 @@
 | "bacc r (Suc n) = (bacc r n \<union> {x. \<forall>y. (y, x) \<in> r \<longrightarrow> y \<in> bacc r n})"
 
 lemma bacc_subseteq_acc:
-  "bacc r n \<subseteq> acc r"
+  "bacc r n \<subseteq> Wellfounded.acc r"
   by (induct n) (auto intro: acc.intros)
 
 lemma bacc_mono:
@@ -761,10 +761,10 @@
 
 lemma acc_subseteq_bacc:
   assumes "finite r"
-  shows "acc r \<subseteq> (\<Union>n. bacc r n)"
+  shows "Wellfounded.acc r \<subseteq> (\<Union>n. bacc r n)"
 proof
   fix x
-  assume "x : acc r"
+  assume "x : Wellfounded.acc r"
   then have "\<exists> n. x : bacc r n"
   proof (induct x arbitrary: rule: acc.induct)
     case (accI x)
@@ -788,7 +788,7 @@
 lemma acc_bacc_eq:
   fixes A :: "('a :: finite \<times> 'a) set"
   assumes "finite A"
-  shows "acc A = bacc A (card (UNIV :: 'a set))"
+  shows "Wellfounded.acc A = bacc A (card (UNIV :: 'a set))"
   using assms by (metis acc_subseteq_bacc bacc_subseteq_acc bacc_upper_bound order_eq_iff)