src/Doc/Tutorial/Protocol/Message.thy
changeset 59780 23b67731f4f0
parent 59763 56d2c357e6b5
child 61992 6d02bb8b5fe1
equal deleted inserted replaced
59778:fe5b796d6b2a 59780:23b67731f4f0
   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          (Rule_Insts.res_inst_tac ctxt [((("x", 1), Position.none), "X")] (insert_commute RS ssubst) 1),
   859          (Rule_Insts.res_inst_tac ctxt [((("x", 1), Position.none), "X")] []
       
   860            (insert_commute RS ssubst) 1),
   860        (*...allowing further simplifications*)
   861        (*...allowing further simplifications*)
   861        simp_tac ctxt 1,
   862        simp_tac ctxt 1,
   862        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   863        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   863        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   864        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   864 *}
   865 *}