src/HOL/SET_Protocol/Message_SET.thy
changeset 59755 f8d164ab0dc1
parent 59498 50b60f501b05
child 59763 56d2c357e6b5
equal deleted inserted replaced
59754:696d87036f04 59755:f8d164ab0dc1
   869   DETERM
   869   DETERM
   870    (SELECT_GOAL
   870    (SELECT_GOAL
   871      (EVERY
   871      (EVERY
   872       [  (*push in occurrences of X...*)
   872       [  (*push in occurrences of X...*)
   873        (REPEAT o CHANGED)
   873        (REPEAT o CHANGED)
   874            (res_inst_tac ctxt [(("x", 1), "X")] (insert_commute RS ssubst) 1),
   874            (res_inst_tac ctxt [((("x", 1), Position.none), "X")] (insert_commute RS ssubst) 1),
   875        (*...allowing further simplifications*)
   875        (*...allowing further simplifications*)
   876        simp_tac ctxt 1,
   876        simp_tac ctxt 1,
   877        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   877        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),
   878        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   878        DEPTH_SOLVE (atomic_spy_analz_tac ctxt 1)]) i);
   879 *}
   879 *}