src/HOL/UNITY/Project.thy
changeset 46471 2289a3869c88
parent 45477 11d9c2768729
child 46912 e0cd5c4df8e6
--- a/src/HOL/UNITY/Project.thy	Tue Feb 14 20:57:05 2012 +0100
+++ b/src/HOL/UNITY/Project.thy	Tue Feb 14 21:19:39 2012 +0100
@@ -544,7 +544,7 @@
      "[| F\<squnion>project h UNIV G \<in> A ensures B;   
          G \<in> stable (extend_set h A - extend_set h B) |]  
       ==> extend h F\<squnion>G \<in> (extend_set h A) ensures (extend_set h B)"
-apply (rule project_ensures_D_lemma [of _ UNIV, THEN revcut_rl], auto)
+apply (rule project_ensures_D_lemma [of _ UNIV, elim_format], auto)
 done
 
 lemma (in Extend) project_Ensures_D: 
@@ -553,7 +553,7 @@
                      extend_set h B) |]  
       ==> extend h F\<squnion>G \<in> (extend_set h A) Ensures (extend_set h B)"
 apply (unfold Ensures_def)
-apply (rule project_ensures_D_lemma [THEN revcut_rl])
+apply (rule project_ensures_D_lemma [elim_format])
 apply (auto simp add: project_set_reachable_extend_eq [symmetric])
 done