diff -r 443c19953137 -r 62ab1968c1f4 doc-src/TutorialI/Protocol/Message.thy --- a/doc-src/TutorialI/Protocol/Message.thy Wed Jun 11 15:40:20 2008 +0200 +++ b/doc-src/TutorialI/Protocol/Message.thy Wed Jun 11 15:40:44 2008 +0200 @@ -862,7 +862,8 @@ (EVERY [ (*push in occurrences of X...*) (REPEAT o CHANGED) - (res_inst_tac [("x1","X")] (insert_commute RS ssubst) 1), + (RuleInsts.res_inst_tac (Simplifier.the_context ss) + [(("x", 1), "X")] (insert_commute RS ssubst) 1), (*...allowing further simplifications*) simp_tac ss 1, REPEAT (FIRSTGOAL (resolve_tac [allI,impI,notI,conjI,iffI])),