make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
(* Author: Lawrence C Paulson, Cambridge University Computer Laboratory
Copyright 1996 University of Cambridge
*)
header {* Blanqui's "guard" concept: protocol-independent secrecy *}
theory Auth_Guard_Public
imports
"P1"
"P2"
"Guard_NS_Public"
"Proto"
begin
end