History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Auth/Shared.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;


# 34a0be19 12-Feb-2014 blanchet <none@none>

adapted theories to 'xxx_case' to 'case_xxx'
* * *
'char_case' -> 'case_char' and same for 'rec'
* * *
compile
* * *
renamed 'xxx_case' to 'case_xxx'


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

use case_of_simps


# 0928b2db 18-Apr-2013 wenzelm <none@none>

simplifier uses proper Proof.context instead of historic type simpset;


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

Introduction of metis calls and other cosmetic modifications.


# 077493ab 08-Sep-2010 haftmann <none@none>

modernized primrec


# 4ca87fa3 08-Sep-2010 paulson <none@none>

tidied using inductive_simps


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

updated some headers;


# 0ddc87cf 21-Sep-2009 haftmann <none@none>

common base for protocols with symmetric keys

--HG--
rename : src/HOL/Auth/ROOT.ML => src/HOL/Auth/All_Symmetric.thy


# a4b600c4 23-Jul-2009 wenzelm <none@none>

renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;


# 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;


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

tuned ML bindings (for multithreading);


# 95ee7518 21-Jul-2007 wenzelm <none@none>

tactics: avoid dynamic reference to accidental theory context (via ML_Context.the_context etc.);


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

simplified method setup;


# 48fb0751 07-Jul-2006 wenzelm <none@none>

tactic/method simpset: maintain proper context;


# 963ca45e 23-Jan-2006 paulson <none@none>

replacement of bool by a datatype (making problems first-order). More lemma names


# 2f8b86a7 04-Oct-2005 paulson <none@none>

theorems need names


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

migrated theory headers to new format


# 0d9b3ba0 11-Jul-2004 wenzelm <none@none>

local_cla/simpset_of;


# ba486add 21-Jun-2004 wenzelm <none@none>

avoid \...\;


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

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


# 91c79bda 04-Sep-2003 paulson <none@none>

new, separate specifications


# 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


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

converting more HOL-Auth to new-style theories


# 4584fe6a 08-Apr-2003 paulson <none@none>

tidying


# 05b61f85 17-Aug-2002 paulson <none@none>

tidying of Isar scripts


# 29210ae9 07-Dec-2001 paulson <none@none>

Slightly generalized the agents' knowledge theorems


# a887046d 27-Apr-2001 paulson <none@none>

better treatment of methods: uses Method.ctxt_args to refer to current
simpset and claset. Needed to fix problems with Recur.thy


# 68aabf0f 29-Mar-2001 paulson <none@none>

misc tidying; changing the predicate isSymKey to the set symKeys


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

partial conversion to Isar script style
simplified unicity proofs


# 609bc635 09-Jan-2001 nipkow <none@none>

`` -> ` and ``` -> ``


# 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


# 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".


# 819edde7 01-Jul-1997 paulson <none@none>

Deleted the obsolete operators newK, newN and nPair


# 606b411f 05-Jun-1997 nipkow <none@none>

Modified a few defs and proofs because of the changes to theory Finite.thy.


# 5b1e40e3 16-Jan-1997 paulson <none@none>

Now with Andy Gordon's treatment of freshness to replace newN/K


# 2176d339 19-Dec-1996 paulson <none@none>

Extensive tidying and simplification, largely stemming from
changing newN and newK to take an integer argument


# 0ab925a1 13-Dec-1996 paulson <none@none>

Temporary additions (random) for the nested Otway-Rees protocol
They will need to be rationalized


# e9d73437 05-Dec-1996 paulson <none@none>

Updating of comments


# b917424c 28-Nov-1996 paulson <none@none>

Weaking of injectivity assumptions for newK and newN:
they are no longer assumed injective over all traces, merely over the
length of a trace


# 2ba1b43e 09-Oct-1996 paulson <none@none>

New version of axiom sees1_Says:
Previously it only allowed the SENDER to see the content of messages...
Now instead the RECIPIENT sees the messages. This change had no effect
on subsequent proofs because protocol rules refer specifically to the
relevant messages sent to an agent.


# fb338176 07-Oct-1996 paulson <none@none>

Simple tidying


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

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


# 3aaf8238 23-Sep-1996 paulson <none@none>

Removal of the Notes constructor


# 85fed2c2 09-Sep-1996 paulson <none@none>

"bad" set simplifies statements of many theorems


# fefa3205 09-Sep-1996 paulson <none@none>

Stronger proofs; work for Otway-Rees


# 04cbbed4 03-Sep-1996 paulson <none@none>

Renaming and simplification


# 7a1b609b 21-Aug-1996 paulson <none@none>

Separation of theory Event into two parts:
Shared for general shared-key material
NS_Shared for the Needham-Schroeder shared-key protocol