diff -r 6061ae1f90f2 -r 9bc16273c2d4 doc-src/TutorialI/Protocol/Message.thy --- a/doc-src/TutorialI/Protocol/Message.thy Fri Jun 17 11:35:35 2005 +0200 +++ b/doc-src/TutorialI/Protocol/Message.thy Fri Jun 17 16:12:49 2005 +0200 @@ -7,8 +7,8 @@ Inductive relations "parts", "analz" and "synth" *) -theory Message = Main -files ("Message_lemmas.ML"): +theory Message imports Main +uses ("Message_lemmas.ML") begin (*Needed occasionally with spy_analz_tac, e.g. in analz_insert_Key_newK*) lemma [simp] : "A Un (B Un A) = B Un A"