(******************************************************************************* Project: Development of Security Protocols by Refinement Module: Refinement/Keys.thy (Isabelle/HOL 2016-1) ID: $Id: Keys.thy 132773 2016-12-09 15:30:22Z csprenge $ Author: Christoph Sprenger, ETH Zurich <sprenger@inf.ethz.ch> Symmetric (shared) and asymmetric (public/private) keys. (based on Larry Paulson's theory Public.thy) Copyright (c) 2012-2016 Christoph Sprenger Licence: LGPL *******************************************************************************) section ‹Symmetric and Assymetric Keys› theory Keys imports Agents begin text ‹Divide keys into session and long-term keys. Define different kinds of long-term keys in second step.›