wenzelm [Tue, 20 Oct 2009 21:37:06 +0200] rev 33032
fixed SML/NJ toplevel pp;
tuned;
wenzelm [Tue, 20 Oct 2009 21:26:45 +0200] rev 33031
backpatching of structure Proof and ProofContext -- avoid odd aliases;
renamed transfer_proof to raw_transfer;
indicate firm naming conventions for theory, Proof.context, Context.generic;
wenzelm [Tue, 20 Oct 2009 21:22:37 +0200] rev 33030
tuned;
wenzelm [Tue, 20 Oct 2009 20:54:31 +0200] rev 33029
uniform use of Integer.min/max;
wenzelm [Tue, 20 Oct 2009 20:03:23 +0200] rev 33028
modernized session SET_Protocol;
wenzelm [Tue, 20 Oct 2009 19:52:04 +0200] rev 33027
modernized session Metis_Examples;
wenzelm [Tue, 20 Oct 2009 19:37:09 +0200] rev 33026
modernized session Isar_Examples;
wenzelm [Tue, 20 Oct 2009 19:36:52 +0200] rev 33025
tuned header;
wenzelm [Tue, 20 Oct 2009 19:29:24 +0200] rev 33024
more accurate dependencies for HOL-SMT, which is a session with image;
misc cleanup;
wenzelm [Tue, 20 Oct 2009 19:28:01 +0200] rev 33023
removed unused map_force;
paulson [Tue, 20 Oct 2009 15:02:48 +0100] rev 33022
Removal of the unused atpset concept, the atp attribute and some related code.
boehmes [Tue, 20 Oct 2009 15:03:17 +0200] rev 33021
additional schematic rules for Z3's rewrite rule
nipkow [Tue, 20 Oct 2009 14:44:19 +0200] rev 33020
merged
nipkow [Tue, 20 Oct 2009 14:44:02 +0200] rev 33019
added Hilbert_Choice section
boehmes [Tue, 20 Oct 2009 14:22:54 +0200] rev 33018
merged
boehmes [Tue, 20 Oct 2009 14:22:02 +0200] rev 33017
eliminated extraneous wrapping of public records,
replaced simp_tac by best_tac (simplifier failed),
less strict condition for rewrite (can also handle equations with single literal on left-hand side)
boehmes [Tue, 20 Oct 2009 12:06:17 +0200] rev 33016
proper exceptions instead of unhandled partiality
nipkow [Tue, 20 Oct 2009 13:37:56 +0200] rev 33015
footnote: inv via inv_onto
nipkow [Tue, 20 Oct 2009 13:20:42 +0200] rev 33014
added inv_def for compatibility as a lemma
wenzelm [Tue, 20 Oct 2009 11:36:19 +0200] rev 33013
slightly less context-sensitive settings;
wenzelm [Tue, 20 Oct 2009 11:08:50 +0200] rev 33012
merged
boehmes [Tue, 20 Oct 2009 10:29:47 +0200] rev 33011
corrected paths to certificates,
added note how to re-generate the certificates
boehmes [Tue, 20 Oct 2009 10:11:30 +0200] rev 33010
added proof reconstructon for Z3,
added certificates for simpler re-checking of proofs (no need to invoke external solvers),
added examples and certificates for all examples,
removed Unsynchronized.ref (in smt_normalize.ML)
wenzelm [Tue, 20 Oct 2009 10:46:42 +0200] rev 33009
merged
haftmann [Tue, 20 Oct 2009 08:10:47 +0200] rev 33008
merged
haftmann [Tue, 20 Oct 2009 08:10:31 +0200] rev 33007
more accurate checkpoints
haftmann [Mon, 19 Oct 2009 16:34:12 +0200] rev 33006
dropped lazy code equations
haftmann [Mon, 19 Oct 2009 16:32:03 +0200] rev 33005
CONTRIBUTORS
wenzelm [Mon, 19 Oct 2009 23:02:56 +0200] rev 33004
always qualify NJ's old List.foldl/foldr in Isabelle/ML;
wenzelm [Mon, 19 Oct 2009 23:02:23 +0200] rev 33003
eliminated duplicate fold1 -- beware of argument order!