src/Doc/Tutorial/Protocol/Message.thy
changeset 59755 f8d164ab0dc1
parent 59498 50b60f501b05
child 59763 56d2c357e6b5
equal deleted inserted replaced
59754:696d87036f04 59755:f8d164ab0dc1
   854   DETERM
   854   DETERM
   855    (SELECT_GOAL
   855    (SELECT_GOAL
   856      (EVERY 
   856      (EVERY 
   857       [  (*push in occurrences of X...*)
   857       [  (*push in occurrences of X...*)
   858        (REPEAT o CHANGED)
   858        (REPEAT o CHANGED)
   859            (res_inst_tac ctxt [(("x", 1), "X")] (insert_commute RS ssubst) 1),
   859            (res_inst_tac ctxt [((("x", 1), Position.none), "X")] (insert_commute RS ssubst) 1),
   860        (*...allowing further simplifications*)
   860        (*...allowing further simplifications*)
   861        simp_tac ctxt 1,
   861        simp_tac ctxt 1,
   862        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   862        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   863        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   863        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   864 *}
   864 *}