--- a/doc-src/TutorialI/Protocol/Message.thy Wed Aug 22 23:23:48 2012 +0200
+++ b/doc-src/TutorialI/Protocol/Message.thy Wed Aug 22 23:45:49 2012 +0200
@@ -8,8 +8,9 @@
header{*Theory of Agents and Messages for Security Protocols*}
-theory Message imports Main uses "../../antiquote_setup.ML" begin
-setup {* Antiquote_Setup.setup *}
+theory Message imports Main begin
+ML_file "../../antiquote_setup.ML"
+setup Antiquote_Setup.setup
(*Needed occasionally with spy_analz_tac, e.g. in analz_insert_Key_newK*)
lemma [simp] : "A \<union> (B \<union> A) = B \<union> A"