(******************************************************************************* Project: Refining Authenticated Key Agreement with Strong Adversaries Module: Messages.thy (Isabelle/HOL 2016-1) ID: $Id: Messages.thy 133008 2017-01-17 13:53:14Z csprenge $ Author: Joseph Lallemand, INRIA Nancy <joseph.lallemand@loria.fr> Christoph Sprenger, ETH Zurich <sprenger@inf.ethz.ch> Message datatype and quotient construction based on Diffie-Hellman equational theory. Copyright (c) 2015-2016 Joseph Lallemand and Christoph Sprenger Licence: LGPL *******************************************************************************) section ‹Message definitions› theory Messages imports Main begin (****************************************************************************************) subsection ‹Messages› (****************************************************************************************) text ‹Agents› datatype agent = Agent nat text ‹Nonces› typedecl fid_t datatype fresh_t = mk_fresh "fid_t" "nat" (infixr ‹$› 65) fun fid :: "fresh_t ⇒ fid_t" where "fid (f $ n) = f" fun num :: "fresh_t ⇒ nat" where "num (f $ n) = n" datatype nonce_t = nonce_fresh "fresh_t" | nonce_atk "nat" text ‹Keys›