diff -r 4c2514625873 -r 2eef5e71edd6 doc-src/TutorialI/Protocol/Event.thy --- a/doc-src/TutorialI/Protocol/Event.thy Mon Mar 16 17:51:07 2009 +0100 +++ b/doc-src/TutorialI/Protocol/Event.thy Mon Mar 16 17:51:24 2009 +0100 @@ -287,7 +287,7 @@ intro: analz_subset_parts [THEN subsetD] parts_mono [THEN [2] rev_subsetD]) method_setup analz_mono_contra = {* - Method.no_args (SIMPLE_METHOD (REPEAT_FIRST analz_mono_contra_tac)) *} + Scan.succeed (K (SIMPLE_METHOD (REPEAT_FIRST analz_mono_contra_tac))) *} "for proving theorems of the form X \ analz (knows Spy evs) --> P" subsubsection{*Useful for case analysis on whether a hash is a spoof or not*} @@ -344,7 +344,7 @@ *} method_setup synth_analz_mono_contra = {* - Method.no_args (SIMPLE_METHOD (REPEAT_FIRST synth_analz_mono_contra_tac)) *} + Scan.succeed (K (SIMPLE_METHOD (REPEAT_FIRST synth_analz_mono_contra_tac))) *} "for proving theorems of the form X \ synth (analz (knows Spy evs)) --> P" (*>*)