src/HOL/TLA/Memory/MemoryImplementation.thy
changeset 27100 889613625e2b
parent 26342 0f65fa163304
child 27117 97e9dae57284
equal deleted inserted replaced
27099:2a91d9575935 27100:889613625e2b
   762    steps of the implementation, and try to solve the idling case by simplification
   762    steps of the implementation, and try to solve the idling case by simplification
   763 *)
   763 *)
   764 ML {*
   764 ML {*
   765 fun split_idle_tac ss simps i =
   765 fun split_idle_tac ss simps i =
   766     EVERY [TRY (rtac @{thm actionI} i),
   766     EVERY [TRY (rtac @{thm actionI} i),
   767            case_tac "(s,t) |= unchanged (e p, c p, r p, m p, rmhist!p)" i,
   767            DatatypePackage.case_tac "(s,t) |= unchanged (e p, c p, r p, m p, rmhist!p)" i,
   768            rewrite_goals_tac @{thms action_rews},
   768            rewrite_goals_tac @{thms action_rews},
   769            forward_tac [temp_use @{thm Step1_4_7}] i,
   769            forward_tac [temp_use @{thm Step1_4_7}] i,
   770            asm_full_simp_tac (ss addsimps simps) i
   770            asm_full_simp_tac (ss addsimps simps) i
   771           ]
   771           ]
   772 *}
   772 *}