src/Doc/Tutorial/Protocol/Message.thy
changeset 82630 2bb4a8d0111d
parent 81261 0c9075bdff38
equal deleted inserted replaced
82629:9c4daf15261c 82630:2bb4a8d0111d
   848    (SELECT_GOAL
   848    (SELECT_GOAL
   849      (EVERY 
   849      (EVERY 
   850       [  (*push in occurrences of X...*)
   850       [  (*push in occurrences of X...*)
   851        (REPEAT o CHANGED)
   851        (REPEAT o CHANGED)
   852          (Rule_Insts.res_inst_tac ctxt [((("x", 1), Position.none), "X")] []
   852          (Rule_Insts.res_inst_tac ctxt [((("x", 1), Position.none), "X")] []
   853            (insert_commute RS ssubst) 1),
   853            (@{thm insert_commute} RS ssubst) 1),
   854        (*...allowing further simplifications*)
   854        (*...allowing further simplifications*)
   855        simp_tac ctxt 1,
   855        simp_tac ctxt 1,
   856        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   856        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   857        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   857        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   858 \<close>
   858 \<close>