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


# 6688eecc 17-Feb-2016 haftmann <none@none>

prefer abbreviations for compound operators INFIMUM and SUPREMUM


# ce5e1da3 28-Dec-2015 wenzelm <none@none>

more symbols;


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

isabelle update_cartouches -c -t;


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


# 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


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


# 7b63d2a6 11-Jul-2007 berghofe <none@none>

Adapted to new inductive definition package.


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


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

migrated theory headers to new format


# 5442a36e 26-Sep-2003 paulson <none@none>

Conversion of all main protocols from "Shared" to "Public".
Removal of Key_supply_ax: modifications to possibility theorems.
Improved presentation.


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

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


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

improved presentation of HOL/Auth theories


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

tweaks


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


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

tidying of Isar scripts


# 4962745e 03-Oct-2001 wenzelm <none@none>

tuned parentheses in relational expressions;


# 58383ae7 03-May-2001 paulson <none@none>

minor tweaks


# 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


# 153d8df2 23-Apr-2001 paulson <none@none>

(rough) conversion of Auth/Recur to Isar format


# 22bc9d8c 27-Feb-2001 paulson <none@none>

Some X-symbols for <notin>, <noteq>, <forall>, <exists>
Streamlining of Yahalom proofs
Removal of redundant proofs


# 9aca3040 08-Sep-1998 paulson <none@none>

Got rid of not_Says_to_self and most uses of ~= in definitions and theorems


# d06dcde6 21-Aug-1998 paulson <none@none>

Tidying


# dbcff1b4 10-Jan-1998 paulson <none@none>

Simplified proofs by omitting PA = {|XA, ...|} from RA2


# 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


# 5f61de48 04-Sep-1997 paulson <none@none>

Renamed "evs" to "evs1", "evs2", etc. in protocol inductive definition


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


# c2cffc3b 27-Jun-1997 paulson <none@none>

Corrected indentations and margins after the renaming of "set_of_list"


# 8628ff0b 26-Jun-1997 nipkow <none@none>

set_of_list -> set


# 6e20702e 23-Jan-1997 paulson <none@none>

Re-ordering of certificates so that session keys appear in decreasing order


# 842553e0 21-Jan-1997 paulson <none@none>

Improved layout and updated comments


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

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


# 79d4553e 07-Jan-1997 paulson <none@none>

Simplification of some proofs, especially by eliminating
the equality in RA2


# d2fcef87 07-Jan-1997 paulson <none@none>

Now uses HPair


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

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


# f9feace9 18-Dec-1996 paulson <none@none>

Recursive Authentication Protocol