src/CTT/CTT.thy
changeset 59498 50b60f501b05
parent 59164 ff40c53d1af9
child 59755 f8d164ab0dc1
--- a/src/CTT/CTT.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/CTT/CTT.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -453,13 +453,13 @@
 
 fun safestep_tac ctxt thms i =
     form_tac ctxt ORELSE
-    resolve_tac thms i  ORELSE
-    biresolve_tac safe0_brls i  ORELSE  mp_tac ctxt i  ORELSE
-    DETERM (biresolve_tac safep_brls i)
+    resolve_tac ctxt thms i  ORELSE
+    biresolve_tac ctxt safe0_brls i  ORELSE  mp_tac ctxt i  ORELSE
+    DETERM (biresolve_tac ctxt safep_brls i)
 
 fun safe_tac ctxt thms i = DEPTH_SOLVE_1 (safestep_tac ctxt thms i)
 
-fun step_tac ctxt thms = safestep_tac ctxt thms  ORELSE'  biresolve_tac unsafe_brls
+fun step_tac ctxt thms = safestep_tac ctxt thms  ORELSE'  biresolve_tac ctxt unsafe_brls
 
 (*Fails unless it solves the goal!*)
 fun pc_tac ctxt thms = DEPTH_SOLVE_1 o (step_tac ctxt thms)