src/Doc/Tutorial/Protocol/Message.thy
changeset 82630 2bb4a8d0111d
parent 81261 0c9075bdff38
--- a/src/Doc/Tutorial/Protocol/Message.thy	Fri May 16 20:44:51 2025 +0200
+++ b/src/Doc/Tutorial/Protocol/Message.thy	Sun May 18 14:33:01 2025 +0000
@@ -850,7 +850,7 @@
       [  (*push in occurrences of X...*)
        (REPEAT o CHANGED)
          (Rule_Insts.res_inst_tac ctxt [((("x", 1), Position.none), "X")] []
-           (insert_commute RS ssubst) 1),
+           (@{thm insert_commute} RS ssubst) 1),
        (*...allowing further simplifications*)
        simp_tac ctxt 1,
        REPEAT (FIRSTGOAL (resolve_tac ctxt [allI,impI,notI,conjI,iffI])),