src/FOLP/FOLP.thy
changeset 60754 02924903a6fd
parent 59498 50b60f501b05
child 60770 240563fbf41d
--- a/src/FOLP/FOLP.thy	Sat Jul 18 20:53:05 2015 +0200
+++ b/src/FOLP/FOLP.thy	Sat Jul 18 20:54:56 2015 +0200
@@ -56,7 +56,7 @@
     and r2: "!!y. y:Q ==> g(y):R"
   shows "?p : R"
   apply (rule excluded_middle [THEN disjE])
-   apply (tactic {* DEPTH_SOLVE (atac 1 ORELSE
+   apply (tactic {* DEPTH_SOLVE (assume_tac @{context} 1 ORELSE
        resolve_tac @{context} [@{thm r1}, @{thm r2}, @{thm major} RS @{thm mp}] 1) *})
   done
 
@@ -80,8 +80,9 @@
   apply (insert major)
   apply (unfold iff_def)
   apply (rule conjE)
-  apply (tactic {* DEPTH_SOLVE_1 (etac @{thm impCE} 1 ORELSE
-      eresolve_tac @{context} [@{thm notE}, @{thm impE}] 1 THEN atac 1 ORELSE atac 1 ORELSE
+  apply (tactic {* DEPTH_SOLVE_1 (eresolve_tac @{context} @{thms impCE} 1 ORELSE
+      eresolve_tac @{context} [@{thm notE}, @{thm impE}] 1 THEN assume_tac @{context} 1 ORELSE
+      assume_tac @{context} 1 ORELSE
       resolve_tac @{context} [@{thm r1}, @{thm r2}] 1) *})+
   done
 
@@ -107,7 +108,7 @@
   val mp = @{thm mp}
   val not_elim = @{thm notE}
   val swap = @{thm swap}
-  val hyp_subst_tacs = [hyp_subst_tac]
+  fun hyp_subst_tacs ctxt = [hyp_subst_tac ctxt]
 );
 open Cla;