prefer generic elimination rules for even/odd over specialized unfold rules for nat
(*  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