src/ZF/AC/DC.thy
changeset 27678 85ea2be46c71
parent 24893 b8ef7afe3a6b
child 32960 69916a850301
--- a/src/ZF/AC/DC.thy	Mon Jul 21 16:30:49 2008 +0200
+++ b/src/ZF/AC/DC.thy	Fri Jul 25 07:35:53 2008 +0200
@@ -5,7 +5,9 @@
 The proofs concerning the Axiom of Dependent Choice
 *)
 
-theory DC imports AC_Equiv Hartog Cardinal_aux begin
+theory DC
+imports AC_Equiv Hartog Cardinal_aux
+begin
 
 lemma RepFun_lepoll: "Ord(a) ==> {P(b). b \<in> a} \<lesssim> a"
 apply (unfold lepoll_def)
@@ -95,7 +97,7 @@
 	   transrec(b, %c r. THE x. first(x, {x \<in> X. <r``c, x> \<in> R}, Q))"
 
 
-locale (open) DC0_imp =
+locale DC0_imp =
   fixes XX and RR and X and R
 
   assumes all_ex: "\<forall>Y \<in> Pow(X). Y \<prec> nat --> (\<exists>x \<in> X. <Y, x> \<in> R)"
@@ -237,16 +239,16 @@
 apply (elim allE)
 apply (erule impE)
    (*these three results comprise Lemma 1*)
-apply (blast intro!: DC0_imp.lemma1_1 DC0_imp.lemma1_2 DC0_imp.lemma1_3)
+apply (blast intro!: DC0_imp.lemma1_1 [OF DC0_imp.intro] DC0_imp.lemma1_2 [OF DC0_imp.intro] DC0_imp.lemma1_3 [OF DC0_imp.intro])
 apply (erule bexE)
 apply (rule_tac x = "\<lambda>n \<in> nat. f`succ (n) `n" in rev_bexI)
- apply (rule lam_type, blast dest!: DC0_imp.lemma2 intro: fun_weaken_type)
+ apply (rule lam_type, blast dest!: DC0_imp.lemma2 [OF DC0_imp.intro] intro: fun_weaken_type)
 apply (rule oallI)
-apply (frule DC0_imp.lemma2, assumption)
+apply (frule DC0_imp.lemma2 [OF DC0_imp.intro], assumption)
   apply (blast intro: fun_weaken_type)
  apply (erule ltD) 
 (** LEVEL 11: last subgoal **)
-apply (subst DC0_imp.lemma3, assumption+) 
+apply (subst DC0_imp.lemma3 [OF DC0_imp.intro], assumption+) 
   apply (fast elim!: fun_weaken_type)
  apply (erule ltD) 
 apply (force simp add: lt_def) 
@@ -293,7 +295,7 @@
 done
 
 
-locale (open) imp_DC0 =
+locale imp_DC0 =
   fixes XX and RR and x and R and f and allRR
   defines XX_def: "XX == (\<Union>n \<in> nat.
 		      {f \<in> succ(n)->domain(R). \<forall>k \<in> n. <f`k, f`succ(k)> \<in> R})"