History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Auth/Event.thy
Revision Date Author Comments
# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# f5796e6d 14-Feb-2018 wenzelm <none@none>

more symbols;


# 5385dbfa 16-Jan-2018 wenzelm <none@none>

standardized towards new-style formal comments: isabelle update_comments;


# 2df4ddef 10-Aug-2016 nipkow <none@none>

"split add" -> "split"


# feca4ab8 10-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 7f7de75b 18-Jul-2015 wenzelm <none@none>

prefer tactics with explicit context;


# b8d56fe6 10-Feb-2015 wenzelm <none@none>

proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
occasionally clarified use of context;


# 4eae0352 10-Nov-2014 wenzelm <none@none>

proper context for assume_tac (atac remains as fall-back without context);


# 794edf80 02-Nov-2014 wenzelm <none@none>

modernized header uniformly as section;


# 5fc26177 11-Sep-2014 blanchet <none@none>

updated news


# 6a7662be 11-Sep-2014 blanchet <none@none>

renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'


# f0361b5e 06-Sep-2013 noschinl <none@none>

use case_of_simps


# 324e98e6 14-Feb-2012 wenzelm <none@none>

prefer high-level elim_format;


# f4961062 20-Nov-2011 wenzelm <none@none>

eliminated obsolete "standard";


# 898b7628 02-Feb-2011 paulson <none@none>

Introduction of metis calls and other cosmetic modifications.


# 4625a9a3 31-Aug-2010 bulwahn <none@none>

renewing specifications in HOL-Auth


# deac04eb 22-Jul-2010 wenzelm <none@none>

updated some headers;


# 079cde2d 17-Oct-2009 wenzelm <none@none>

eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;


# 2d43315f 14-Aug-2009 paulson <none@none>

sledgehammer used to streamline protocol proofs


# b1258973 16-Mar-2009 wenzelm <none@none>

simplified method setup;


# 77d6b267 13-Mar-2009 wenzelm <none@none>

unified type Proof.method and pervasive METHOD combinators;


# a5551838 16-Jun-2008 wenzelm <none@none>

eliminated OldGoals.inst;


# 6284a6de 11-Jun-2008 wenzelm <none@none>

OldGoals.inst;


# df5ccfe2 01-Aug-2007 wenzelm <none@none>

tuned ML bindings (for multithreading);


# f7800759 29-Nov-2006 wenzelm <none@none>

simplified method setup;


# cd65d9bc 16-Nov-2006 wenzelm <none@none>

more robust syntax for definition/abbreviation/notation;


# 8d37dcbe 28-Sep-2006 wenzelm <none@none>

replaced syntax/translations by abbreviation;


# 7ca981cd 04-Jan-2006 paulson <none@none>

a few more named lemmas


# 928211c1 26-Oct-2005 paulson <none@none>

tidied away duplicate thm


# a7060872 17-Jun-2005 haftmann <none@none>

migrated theory headers to new format


# d66531ec 23-Sep-2003 paulson <none@none>

Removal of the Key_supply axiom (affects many possbility proofs) and minor
changes


# f6663d03 24-Jul-2003 paulson <none@none>

Tidying and replacement of some axioms by specifications


# 7a4d9400 05-May-2003 paulson <none@none>

improved presentation of HOL/Auth theories


# a03be07c 28-Apr-2003 paulson <none@none>

tweaks


# 63be96be 25-Apr-2003 paulson <none@none>

converting more HOL-Auth to new-style theories


# c5f9f5e4 25-Apr-2003 paulson <none@none>

Changes required by the certified email protocol

Public-key model now provides separate signature/encryption keys and also
long-term symmetric keys.


# 152beace 06-Aug-2001 paulson <none@none>

three new theorems


# 9c6192fe 18-May-2001 paulson <none@none>

spelling check


# 0c13cd01 04-Mar-2001 paulson <none@none>

a few basic X-symbols


# 158d88c6 02-Mar-2001 paulson <none@none>

conversion of Message.thy to Isar format


# 7da6eee0 13-Feb-2001 paulson <none@none>

partial conversion to Isar script style
simplified unicity proofs


# f61219de 18-Mar-1999 paulson <none@none>

exchanged the order of Gets and Notes in datatype event


# 5ed22e3e 09-Mar-1999 paulson <none@none>

Added Bella's "Gets" model for Otway_Rees. Also affects some other theories.
Changing "spies" to "knows Spy", etc. Retaining the constant "spies" as a
translation.


# df41c559 24-Jul-1998 berghofe <none@none>

Adapted to new datatype package.


# 99c390e7 18-Sep-1997 paulson <none@none>

Global change: lost->bad and sees Spy->spies
First change just gives a more sensible name.
Second change eliminates the agent parameter of "sees" to simplify
definitions and theorems


# edfd4df1 17-Sep-1997 paulson <none@none>

Spy can see Notes of the compromised agents


# 5276b175 13-Jul-1997 paulson <none@none>

Changing "lost" from a parameter of protocol definitions to a constant.

Advantages: no "lost" argument everywhere; fewer Vars in subgoals;
less need for specially instantiated rules
Disadvantage: can no longer prove "Agent_not_see_encrypted_key", but this
theorem was never used, and its original proof was also broken
the introduction of the "Notes" constructor.


# 4055b9c9 11-Jul-1997 paulson <none@none>

Moving common declarations and proofs from theories "Shared"
and "Public" to "Event". NB the original "Event" theory was later renamed "Shared".

Addition of the Notes constructor to datatype "event".


# ac9b0212 22-Nov-1996 paulson <none@none>

Have been obsolete for months; contents are now in Shared and NS_Shared


# e2feb658 25-Sep-1996 paulson <none@none>

Introduction of "lost" argument
Changed Enemy -> Spy
Ran expandshort


# b91abd12 03-Sep-1996 paulson <none@none>

Renaming and simplification


# 02107313 21-Aug-1996 paulson <none@none>

Addition of message NS5


# 1b438cf6 20-Aug-1996 paulson <none@none>

Working version of NS, messages 1-4!


# 6f044346 20-Aug-1996 paulson <none@none>

Working version of NS, messages 1-3, WITH INTERLEAVING


# 49ed9cfd 19-Aug-1996 paulson <none@none>

Renaming of functions, and tidying


# b6572432 29-Jul-1996 paulson <none@none>

Works up to main theorem, then XXX...X


# a3a15df5 25-Jul-1996 paulson <none@none>

Auth proofs work up to the XXX...


# 328a4f3a 11-Jul-1996 paulson <none@none>

Added Msg 3; works up to Says_Server_imp_Key_newK


# 782f2f44 28-Jun-1996 paulson <none@none>

Proving safety properties of authentication protocols