eliminated Plain_HOLCF.thy (see also 8e92772bc0e8): it was modeled after HOL/Plain.thy which was discontinued later;
(* Author: Lawrence C Paulson, Cambridge University Computer Laboratory
Copyright 1996 University of Cambridge
*)
section \<open>Conventional protocols: rely on conventional Message, Event and Public -- Shared-key protocols\<close>
theory Auth_Shared
imports
"NS_Shared"
"Kerberos_BAN"
"Kerberos_BAN_Gets"
"KerberosIV"
"KerberosIV_Gets"
"KerberosV"
"OtwayRees"
"OtwayRees_AN"
"OtwayRees_Bad"
"OtwayReesBella"
"WooLam"
"Recur"
"Yahalom"
"Yahalom2"
"Yahalom_Bad"
"ZhouGollmann"
begin
end