Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-1000
-240
+240
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
Moved Option into core HOL which caused a few local changes.
1996-09-24, by nipkow
Proofs made more robust to work in presence of le_refl
1996-09-23, by paulson
Now uses init_html
1996-09-23, by paulson
Simplification of proof of unique_session_keys
1996-09-23, by paulson
Correction of protocol; addition of Reveal message; proofs of
1996-09-23, by paulson
Proof of Says_imp_old_keys is now more robust
1996-09-23, by paulson
Removal of the Notes constructor
1996-09-23, by paulson
New laws for messages
1996-09-23, by paulson
Simplification of definition of synth
1996-09-23, by paulson
Addition of le_refl to default simpset/claset
1996-09-23, by paulson
Removal of reference Nipkow-LICS-93
1996-09-23, by paulson
Proof of mult_le_mono is now more robust
1996-09-23, by paulson
New infix syntax: breaks line BEFORE operator
1996-09-23, by paulson
Optimized version of SELECT_GOAL, up to 10% faster
1996-09-23, by paulson
New operations on cterms. Now same names as in Logic
1996-09-23, by paulson
Addition of gensym
1996-09-23, by paulson
Bad version of Otway-Rees and the new attack on it
1996-09-23, by paulson
Reformatting; proved B_gets_secure_key
1996-09-13, by paulson
Abstraction of enemy_analz_tac over its argument
1996-09-13, by paulson
Reformatting
1996-09-13, by paulson
Reordering of premises for cut theorems, and new law MPair_synth_analz
1996-09-13, by paulson
No longer assumes Alice is not the Enemy in NS3.
1996-09-13, by paulson
Uses the improved enemy_analz_tac of Shared.ML, with simpler proofs
1996-09-13, by paulson
Addition of Yahalom protocol
1996-09-13, by paulson
Removal of obsolete thm Fake_parts_insert
1996-09-13, by paulson
Addition of enemy_analz_tac and safe_solver
1996-09-13, by paulson
added flat_eq,
1996-09-12, by oheimb
renamed adm_disj_lemma11 to adm_lemma11
1996-09-12, by oheimb
added comment on is_flat
1996-09-12, by oheimb
added stric
1996-09-12, by oheimb
undo last revision
1996-09-12, by oheimb
bin/isa2latex: copy the binary to bin/isa2latex instead of linking it there
1996-09-12, by oheimb
new \subsubsection{Configuring conversion tables and keyboard bindings}
1996-09-12, by oheimb
Tidied many proofs, using AddIffs to let equivalences take
1996-09-12, by paulson
Installed AddIffs, and some code from HOL.ML
1996-09-12, by paulson
Simplification and tidying of definitions
1996-09-12, by paulson
Now hologic.ML is loaded in HOL.ML
1996-09-12, by paulson
New file cladata.ML
1996-09-12, by paulson
Split off classical reasoning code to cladata.ML
1996-09-12, by paulson
Change to best_tac required to prevent looping
1996-09-12, by paulson
Moved RSLIST here from ../Relation.ML
1996-09-11, by paulson
Removal of univ_cs
1996-09-11, by paulson
Reformatting
1996-09-11, by paulson
renamed cterm_lift_inst_rule to term_lift_inst_rule and made it take
1996-09-11, by nipkow
Removed refs to clasets like rel_cs etc. Used implicit claset.
1996-09-11, by nipkow
Converted proofs to use default clasets.
1996-09-10, by nipkow
Added Auth to the test target
1996-09-10, by paulson
Now runs all Auth proofs
1996-09-10, by paulson
Now uses DB-ROOT.ML, which is separate from ROOT.ML
1996-09-10, by paulson
Dedicated root file for making the Auth database
1996-09-10, by paulson
Beefed-up auto-tactic: now repeatedly simplifies if needed
1996-09-10, by paulson
"bad" set simplifies statements of many theorems
1996-09-09, by paulson
added cterm_lift_inst_rule
1996-09-09, by nipkow
Stronger proofs; work for Otway-Rees
1996-09-09, by paulson
Stronger proofs; work for Otway-Rees
1996-09-09, by paulson
These simpsets must not use miniscoping
1996-09-09, by paulson
Corrected associativity: must be to right, as the type dictatess
1996-09-09, by paulson
Removal of (EX x. P) <-> P and (ALL x. P) <-> P
1996-09-09, by paulson
Improved error handling: if there are syntax or type-checking
1996-09-06, by paulson
Modified proof to work with miniscoping
1996-09-06, by paulson
Now uses thin_tac
1996-09-05, by paulson
Now uses thin_tac
1996-09-05, by paulson
Renaming of _rews to _simps
1996-09-05, by paulson
Added thin_tac to signature; previous change was useless
1996-09-05, by paulson
Some renaming. Note that this miniscoping is more
1996-09-05, by paulson
Introduction of miniscoping for FOL
1996-09-05, by paulson
Pretty-printing change to emphasize the scope of assumptions
1996-09-05, by paulson
Declared thin_tac
1996-09-05, by paulson
Miniscoping rules are deleted, as these brittle proofs
1996-09-05, by paulson
Simplified some proofs for compatibility with miniscoping
1996-09-05, by paulson
Added miniscoping to the simplifier: quantifiers are now pushed in
1996-09-05, by paulson
Fixed pretty-printing of {|...|}
1996-09-03, by paulson
New theorems for Fake case
1996-09-03, by paulson
A further tidying
1996-09-03, by paulson
ROOT file for Auth directory
1996-09-03, by paulson
Renaming and simplification
1996-09-03, by paulson
Renaming and simplification
1996-09-03, by paulson
Initial working proof of Otway-Rees protocol
1996-09-03, by paulson
Swaped two conditions in the completeness statement.
1996-08-23, by nipkow
Generalized my_lemma1: (c3,s3) |--> cs3
1996-08-23, by nipkow
Now deepen_tac can take advantage of wrappers --
1996-08-22, by paulson
Proved mem_if
1996-08-22, by paulson
Proved set_of_list_subset_Cons
1996-08-22, by paulson
For building the security theory as a separate database
1996-08-22, by paulson
Separation of theory Event into two parts:
1996-08-21, by paulson
Addition of message NS5
1996-08-21, by paulson
Tidying: removing redundant args in classical reasoner calls
1996-08-21, by paulson
Added le_eq_less_Suc; fixed some comments;
1996-08-21, by paulson
Working version of NS, messages 1-4!
1996-08-20, by paulson
Working version of NS, messages 1-3, WITH INTERLEAVING
1996-08-20, by paulson
Added ref to allow suppression of error msgs
1996-08-20, by paulson
New classical reasoner: warns of, and ignores, redundant rules.
1996-08-20, by paulson
Addition of function set_of_list
1996-08-20, by paulson
Some tidying. This brittle proof depends upon
1996-08-20, by paulson
Corrected for new classical reasoner: redundant rules
1996-08-20, by paulson
updated html-link
1996-08-19, by nipkow
Installation of auto_tac; re-organization
1996-08-19, by paulson
Tidied up the proofs
1996-08-19, by paulson
Added impOfSubs
1996-08-19, by paulson
Now less_zeroE is a Safe Elim rule
1996-08-19, by paulson
Improved comment
1996-08-19, by paulson
Added proof of Un_insert_right
1996-08-19, by paulson
Changed precedences to remove ambiguities in r^+ notation
1996-08-19, by paulson
Improved the proof of Problem 38
1996-08-19, by paulson
Added a lot of basic laws, from HOL/simpdata
1996-08-19, by paulson
Renaming of functions, and tidying
1996-08-19, by paulson
Now starts with set_current_thy
1996-08-19, by paulson
Tidied some proofs
1996-08-19, by paulson
Tidied some proofs, maybe using less_SucE
1996-08-19, by paulson
Removal of less_SucE as default SE rule
1996-08-19, by paulson
Renamed setOfList to set_of_list
1996-08-19, by paulson
Minor improvements of the scripts
1996-08-16, by oheimb
Improved (?) wording of error message
1996-08-12, by paulson
Added a new section on Definitions
1996-08-12, by paulson
Rewording: parameters->arguments!
1996-08-12, by paulson
Initial revision of thy_data.ML
1996-08-08, by berghofe
Added function for storing default claset in theory.
1996-08-08, by berghofe
Removed unnecessary Addsimps.
1996-08-08, by berghofe
Simplified primrec definitions.
1996-08-08, by berghofe
Classical tactics now use default claset.
1996-08-02, by berghofe
Simplified primrec definitions.
1996-08-02, by berghofe
Replaced prove_case_cong by Konrad Slinds optimized version.
1996-08-02, by berghofe
Simplified primrec - definitions.
1996-07-30, by berghofe
Now also Deepen_tac and Best_tac are used.
1996-07-30, by berghofe
Classical tactics now use default claset.
1996-07-30, by berghofe
Works up to main theorem, then XXX...X
1996-07-29, by paulson
Added two new distributive laws
1996-07-29, by paulson
Addition of rev_notE
1996-07-26, by paulson
Inserted spaces in error messages to improve readability
1996-07-26, by paulson
Addition of contra_subsetD and rev_contra_subsetD
1996-07-26, by paulson
Removal of cfast_tac
1996-07-26, by paulson
Removed clash with "range" constant
1996-07-26, by paulson
Redefining "range" as a macro -- new proof needed
1996-07-26, by paulson
Auth proofs work up to the XXX...
1996-07-26, by paulson
Proved insert_image
1996-07-26, by paulson
Redefining "range" as a macro
1996-07-26, by paulson
Proved bex_False
1996-07-26, by paulson
unnecessary files removed
1996-07-23, by oheimb
Corrected typo regarding the type of set_oracle
1996-07-23, by paulson
Added insert_commute
1996-07-22, by paulson
Updated BibTeX identifiers
1996-07-22, by paulson
Acknowledged Martin Simons
1996-07-22, by paulson
Corrected typo involving derivations
1996-07-22, by paulson
Classical tactics now use default claset.
1996-07-19, by berghofe
Corrected o_assoc lemma
1996-07-17, by pusch
removed superfluous Park-induct rule
1996-07-17, by pusch
renamed adm_impl to adm_imp
1996-07-17, by oheimb
Edited in response to referees comments; new references
1996-07-17, by paulson
correction of recent typo
1996-07-17, by oheimb
Added section about current claset.
1996-07-16, by berghofe
Put in minimal simpset to avoid excessive simplification,
Isabelle94-6
1996-07-16, by paulson
corrected comment
1996-07-16, by paulson
Acknowledged Stefan Berghofer for finding errors
1996-07-16, by paulson
Fixed typo regarding lifting over P|P
1996-07-16, by paulson
Increased revision number
1996-07-16, by paulson
Tidied up; added "syntax" decl
1996-07-16, by paulson
New dummy .thy files to document dependencies
1996-07-15, by paulson
Uses minimal simpset (min_ss) and full_simp_tac
1996-07-15, by paulson
Documented simplification tactics which make use of the implicit simpset.
1996-07-15, by nipkow
updated syntax of primrec definitions
1996-07-15, by berghofe
*** empty log message ***
1996-07-12, by oheimb
bug fix: Glam_ast_tr
1996-07-12, by oheimb
added configuration for STEM
1996-07-12, by oheimb
minor bug fix
1996-07-12, by oheimb
updated syntax of primrec definitions
1996-07-12, by berghofe
replaced setsolver ... by addsolver
1996-07-12, by oheimb
Added Msg 3; works up to Says_Server_imp_Key_newK
1996-07-11, by paulson
Corrected indentation
1996-07-11, by paulson
Oracles can now be strings instead of identifiers
1996-07-11, by paulson
Added insert_mono
1996-07-11, by paulson
Added ML reference
1996-07-11, by paulson
Modified to reject certain inputs -- illustrates error handling
1996-07-11, by paulson
Documentation of oracles and their syntax
1996-07-11, by paulson
Simplified syntax of primrec definitions.
1996-07-05, by berghofe
Removed a use of eq_cs
1996-06-28, by paulson
Removed the unused eq_cs, and added some distributive laws
1996-06-28, by paulson
Removed the unused rel_eq_cs
1996-06-28, by paulson
Added contra_subsetD and rev_contra_subsetD
1996-06-28, by paulson
Added rev_notE by analogy with rev_mp
1996-06-28, by paulson
Proving safety properties of authentication protocols
1996-06-28, by paulson
Updated reference to Slinds paper on TFL
1996-06-28, by paulson
Now set_cs is just taken from !claset
1996-06-28, by paulson
Added type-checking to rule "combination". This corrects a fault
1996-06-28, by paulson
Restored warning comment
1996-06-28, by paulson
re-added when_funs to library.ML
1996-06-27, by oheimb
patches for Holcfb.thy removed
1996-06-27, by oheimb
removed old version of LEAST operator
1996-06-27, by oheimb
repaired 8bit pragma
1996-06-26, by oheimb
adapted path to 8bit package
1996-06-26, by oheimb
function names in when_rews now meta-quantified
1996-06-26, by oheimb
when_funs removed
1996-06-26, by oheimb
*** empty log message ***
1996-06-25, by oheimb
Initial revision
1996-06-25, by oheimb
Changed argument order of nat_rec.
1996-06-25, by berghofe
Changed argument order of nat_rec.
1996-06-25, by berghofe
Replaced occurrence of fast_tac by Fast_tac .
1996-06-21, by berghofe
Replaced occurrence of set_cs by claset_of "Fun" .
1996-06-21, by berghofe
Added function Addss.
1996-06-21, by berghofe
Classical tactics now use default claset.
1996-06-21, by berghofe
minor fix of index_vnames: name "O" is occupied (used in HOL/Relation.thy)
1996-06-21, by oheimb
Restored Addsimps [Suc_le_lessD], as it cannot be added
1996-06-20, by paulson
Corrected comment
1996-06-20, by paulson
New rewrites for vacuous quantification
1996-06-18, by paulson
Addition of setOfList
1996-06-18, by paulson
Addition of Safe_step_tac
1996-06-18, by paulson
Translation infixes <->, etc., no longer available at top-level
1996-06-18, by paulson
Addition of setOfList
1996-06-18, by paulson
Removal of list_all
1996-06-18, by paulson
Translation infixes <->, etc., no longer available at top-level
1996-06-18, by paulson
Inserted comment about problem 43
1996-06-17, by paulson
Removed quantification over lists
1996-06-17, by paulson
Now exports Delrules
1996-06-17, by paulson
Converted to use constdefs instead of defs
1996-06-17, by paulson
Explicitly included add_mult_distrib & add_mult_distrib2
1996-06-14, by paulson
New example of greatest common divisor
1996-06-14, by paulson
Added Primes to list of theories in target ex
1996-06-14, by paulson
Now del_simp catches the right exception!
1996-06-14, by paulson
Added delete function for brls
1996-06-14, by paulson
Now implements delrules
1996-06-14, by paulson
Added new Primes theory
1996-06-14, by paulson
Explicitly included add_mult_distrib & add_mult_distrib2
1996-06-14, by paulson
Updated list of theories for target ex
1996-06-14, by paulson
Tidied spacing
1996-06-14, by paulson
New lemmas for gcd example
1996-06-14, by paulson
Obsolete relics concerned with recursion
1996-06-14, by paulson
New example of GCDs and divides relation
1996-06-13, by paulson
The "divides" relation, the greatest common divisor and Euclid's algorithm
1996-06-13, by paulson
Addition of converse_iff, domain_converse, range_converse as rewrites
1996-06-07, by paulson
Quotes now optional around inductive set
1996-06-06, by paulson
Quotes now optional around inductive set
1996-06-06, by paulson
Quotes now optional around inductive set
1996-06-06, by paulson
Tidied some proofs
1996-06-04, by paulson
best_tac, deepen_tac and safe_tac now also use default claset.
1996-06-03, by berghofe
Shortened some proofs
1996-06-03, by paulson
Added a new theorem, UN_Int_subset
1996-06-03, by paulson
Used 2 instead of Suc(Suc 0)
1996-06-03, by paulson
Shortened a proof
1996-06-03, by paulson
adapted use of monofun_cfun_arg
1996-05-31, by oheimb
adapted proof of flat_codom
1996-05-31, by oheimb
introduced forgotten bind_thm calls
1996-05-31, by oheimb
less
more
|
(0)
-1000
-240
+240
+1000
+3000
+10000
+30000
tip