2015-07-18 |
wenzelm |
2015-07-18 |
prefer tactics with explicit context;
|
file | diff | annotate |
2015-02-10 |
wenzelm |
2015-02-10 |
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
occasionally clarified use of context;
|
file | diff | annotate |
2014-11-10 |
wenzelm |
2014-11-10 |
proper context for assume_tac (atac remains as fall-back without context);
|
file | diff | annotate |
2014-11-02 |
wenzelm |
2014-11-02 |
modernized header uniformly as section;
|
file | diff | annotate |
2014-09-11 |
blanchet |
2014-09-11 |
updated news
|
file | diff | annotate |
2014-09-11 |
blanchet |
2014-09-11 |
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
|
file | diff | annotate |
2013-09-06 |
noschinl |
2013-09-06 |
use case_of_simps
|
file | diff | annotate |
2012-02-14 |
wenzelm |
2012-02-14 |
prefer high-level elim_format;
|
file | diff | annotate |
2011-11-20 |
wenzelm |
2011-11-20 |
eliminated obsolete "standard";
|
file | diff | annotate |
2011-02-02 |
paulson |
2011-02-02 |
Introduction of metis calls and other cosmetic modifications.
|
file | diff | annotate |
2010-08-31 |
bulwahn |
2010-08-31 |
renewing specifications in HOL-Auth
|
file | diff | annotate |
2010-07-22 |
wenzelm |
2010-07-22 |
updated some headers;
|
file | diff | annotate |
2009-10-17 |
wenzelm |
2009-10-17 |
eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;
|
file | diff | annotate |
2009-08-14 |
paulson |
2009-08-14 |
sledgehammer used to streamline protocol proofs
|
file | diff | annotate |
2009-03-16 |
wenzelm |
2009-03-16 |
simplified method setup;
|
file | diff | annotate |
2009-03-13 |
wenzelm |
2009-03-13 |
unified type Proof.method and pervasive METHOD combinators;
|
file | diff | annotate |
2008-06-16 |
wenzelm |
2008-06-16 |
eliminated OldGoals.inst;
|
file | diff | annotate |
2008-06-11 |
wenzelm |
2008-06-11 |
OldGoals.inst;
|
file | diff | annotate |
2007-08-01 |
wenzelm |
2007-08-01 |
tuned ML bindings (for multithreading);
|
file | diff | annotate |
2006-11-29 |
wenzelm |
2006-11-29 |
simplified method setup;
|
file | diff | annotate |
2006-11-17 |
wenzelm |
2006-11-17 |
more robust syntax for definition/abbreviation/notation;
|
file | diff | annotate |
2006-09-28 |
wenzelm |
2006-09-28 |
replaced syntax/translations by abbreviation;
|
file | diff | annotate |
2006-01-04 |
paulson |
2006-01-04 |
a few more named lemmas
|
file | diff | annotate |
2005-10-26 |
paulson |
2005-10-26 |
tidied away duplicate thm
|
file | diff | annotate |
2005-06-17 |
haftmann |
2005-06-17 |
migrated theory headers to new format
|
file | diff | annotate |
2003-09-23 |
paulson |
2003-09-23 |
Removal of the Key_supply axiom (affects many possbility proofs) and minor
changes
|
file | diff | annotate |
2003-07-24 |
paulson |
2003-07-24 |
Tidying and replacement of some axioms by specifications
|
file | diff | annotate |
2003-05-05 |
paulson |
2003-05-05 |
improved presentation of HOL/Auth theories
|
file | diff | annotate |
2003-04-29 |
paulson |
2003-04-29 |
tweaks
|
file | diff | annotate |
2003-04-26 |
paulson |
2003-04-26 |
converting more HOL-Auth to new-style theories
|
file | diff | annotate |
2003-04-25 |
paulson |
2003-04-25 |
Changes required by the certified email protocol
Public-key model now provides separate signature/encryption keys and also
long-term symmetric keys.
|
file | diff | annotate |
2001-08-06 |
paulson |
2001-08-06 |
three new theorems
|
file | diff | annotate |
2001-05-19 |
paulson |
2001-05-19 |
spelling check
|
file | diff | annotate |
2001-03-05 |
paulson |
2001-03-05 |
a few basic X-symbols
|
file | diff | annotate |
2001-03-02 |
paulson |
2001-03-02 |
conversion of Message.thy to Isar format
|
file | diff | annotate |
2001-02-13 |
paulson |
2001-02-13 |
partial conversion to Isar script style
simplified unicity proofs
|
file | diff | annotate |
1999-03-18 |
paulson |
1999-03-18 |
exchanged the order of Gets and Notes in datatype event
|
file | diff | annotate |
1999-03-09 |
paulson |
1999-03-09 |
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.
|
file | diff | annotate |
1998-07-24 |
berghofe |
1998-07-24 |
Adapted to new datatype package.
|
file | diff | annotate |
1997-09-18 |
paulson |
1997-09-18 |
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
|
file | diff | annotate |
1997-09-17 |
paulson |
1997-09-17 |
Spy can see Notes of the compromised agents
|
file | diff | annotate |
1997-07-14 |
paulson |
1997-07-14 |
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.
|
file | diff | annotate |
1997-07-11 |
paulson |
1997-07-11 |
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".
|
file | diff | annotate |
1996-09-26 |
paulson |
1996-09-26 |
Introduction of "lost" argument
Changed Enemy -> Spy
Ran expandshort
|
file | diff | annotate |
1996-09-03 |
paulson |
1996-09-03 |
Renaming and simplification
|
file | diff | annotate |
1996-08-21 |
paulson |
1996-08-21 |
Addition of message NS5
|
file | diff | annotate |
1996-08-20 |
paulson |
1996-08-20 |
Working version of NS, messages 1-4!
|
file | diff | annotate |
1996-08-20 |
paulson |
1996-08-20 |
Working version of NS, messages 1-3, WITH INTERLEAVING
|
file | diff | annotate |
1996-08-19 |
paulson |
1996-08-19 |
Renaming of functions, and tidying
|
file | diff | annotate |
1996-07-29 |
paulson |
1996-07-29 |
Works up to main theorem, then XXX...X
|
file | diff | annotate |
1996-07-26 |
paulson |
1996-07-26 |
Auth proofs work up to the XXX...
|
file | diff | annotate |
1996-07-11 |
paulson |
1996-07-11 |
Added Msg 3; works up to Says_Server_imp_Key_newK
|
file | diff | annotate |
1996-06-28 |
paulson |
1996-06-28 |
Proving safety properties of authentication protocols
|
file | diff | annotate |