(******************************************************************************* Project: Development of Security Protocols by Refinement Module: Refinement/Runs.thy (Isabelle/HOL 2016-1) ID: $Id: Runs.thy 132773 2016-12-09 15:30:22Z csprenge $ Author: Christoph Sprenger, ETH Zurich <sprenger@inf.ethz.ch> Protocol runs: local state of executing protocol roles Copyright (c) 2010-2016 Christoph Sprenger Licence: LGPL *******************************************************************************) section ‹Protocol runs› theory Runs imports Atoms begin (******************************************************************************) subsection ‹Runs› (******************************************************************************) text ‹Define some typical roles.›