(******************************************************************************* Title: HOL/Auth/Message Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1996 University of Cambridge Datatypes of agents and messages; Inductive relations "parts", "analz" and "synth" ******************************************************************************** Module: Refinement/Message.thy (Isabelle/HOL 2016-1) ID: $Id: Message.thy 133856 2017-03-20 18:05:54Z csprenge $ Edited: Christoph Sprenger <sprenger@inf.ethz.ch>, ETH Zurich Integrated and adapted for security protocol refinement *******************************************************************************) section ‹Theory of Agents and Messages for Security Protocols› theory Message imports Keys begin (*Needed occasionally with spy_analz_tac, e.g. in analz_insert_Key_newK*) lemma Un_idem_collapse [simp]: "A ∪ (B ∪ A) = B ∪ A" by blast