(******************************************************************************* Project: Development of Security Protocols by Refinement Module: Refinement/Atoms.thy (Isabelle/HOL 2016-1) ID: $Id: Atoms.thy 132773 2016-12-09 15:30:22Z csprenge $ Author: Christoph Sprenger, ETH Zurich <sprenger@inf.ethz.ch> Atomic messages for L1-L2 protocols Copyright (c) 2009-2016 Christoph Sprenger Licence: LGPL *******************************************************************************) section ‹Atomic messages› theory Atoms imports Keys begin (******************************************************************************) subsection ‹Atoms datatype› (******************************************************************************)