src/HOL/TLA/Memory/MemoryImplementation.thy
changeset 59498 50b60f501b05
parent 58963 26bf09b95dda
child 59802 684cfaa12e47
--- a/src/HOL/TLA/Memory/MemoryImplementation.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/TLA/Memory/MemoryImplementation.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -800,7 +800,7 @@
    (TRY (rtac @{thm actionI} 1) THEN
     Induct_Tacs.case_tac ctxt "(s,t) |= unchanged (e p, c p, r p, m p, rmhist!p)" 1 THEN
     rewrite_goals_tac ctxt @{thms action_rews} THEN
-    forward_tac [temp_use ctxt @{thm Step1_4_7}] 1 THEN
+    forward_tac ctxt [temp_use ctxt @{thm Step1_4_7}] 1 THEN
     asm_full_simp_tac ctxt 1);
 *}