try to avoid races again (cf. 8c37cb84065f and fd3a36e48b09);
(* Author: Lawrence C Paulson, Cambridge University Computer Laboratory
Copyright 1996 University of Cambridge
*)
header {* Blanqui's "guard" concept: protocol-independent secrecy *}
theory Auth_Guard_Shared
imports
"Guard_OtwayRees"
"Guard_Yahalom"
begin
end