src/HOL/TLA/Memory/MemoryImplementation.thy
changeset 27117 97e9dae57284
parent 27100 889613625e2b
child 27208 5fe899199f85
--- a/src/HOL/TLA/Memory/MemoryImplementation.thy	Tue Jun 10 16:43:07 2008 +0200
+++ b/src/HOL/TLA/Memory/MemoryImplementation.thy	Tue Jun 10 16:43:14 2008 +0200
@@ -763,12 +763,11 @@
 *)
 ML {*
 fun split_idle_tac ss simps i =
-    EVERY [TRY (rtac @{thm actionI} i),
-           DatatypePackage.case_tac "(s,t) |= unchanged (e p, c p, r p, m p, rmhist!p)" i,
-           rewrite_goals_tac @{thms action_rews},
-           forward_tac [temp_use @{thm Step1_4_7}] i,
-           asm_full_simp_tac (ss addsimps simps) i
-          ]
+  TRY (rtac @{thm actionI} i) THEN
+  case_split_tac "(s,t) |= unchanged (e p, c p, r p, m p, rmhist!p)" i THEN
+  rewrite_goals_tac @{thms action_rews} THEN
+  forward_tac [temp_use @{thm Step1_4_7}] i THEN
+  asm_full_simp_tac (ss addsimps simps) i
 *}
 (* ----------------------------------------------------------------------
    Combine steps 1.2 and 1.4 to prove that the implementation satisfies