haftmann [Wed, 21 Oct 2009 08:14:38 +0200] rev 33038
dropped redundant gen_ prefix
haftmann [Tue, 20 Oct 2009 16:13:01 +0200] rev 33037
replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
kleing [Wed, 21 Oct 2009 16:41:22 +1100] rev 33036
find_theorems: better handling of abbreviations (by Timothy Bourke)
wenzelm [Wed, 21 Oct 2009 00:36:12 +0200] rev 33035
standardized basic operations on type option;
wenzelm [Tue, 20 Oct 2009 23:25:04 +0200] rev 33034
eliminated THENL -- use THEN RANGE;
eliminated TRY' -- use TRY with op o;
observe naming convention ctxt: Proof.context;
tuned whitespace;
wenzelm [Tue, 20 Oct 2009 22:46:24 +0200] rev 33033
tuned;
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!
wenzelm [Mon, 19 Oct 2009 21:54:57 +0200] rev 33002
uniform use of Integer.add/mult/sum/prod;
berghofe [Mon, 19 Oct 2009 16:47:21 +0200] rev 33001
Removed dead code in function mk_deftab.
berghofe [Mon, 19 Oct 2009 16:45:52 +0200] rev 33000
Removed unneeded reference to inv_def.
berghofe [Mon, 19 Oct 2009 16:45:00 +0200] rev 32999
Replaced inv by the_inv_onto.
berghofe [Mon, 19 Oct 2009 16:43:45 +0200] rev 32998
Renamed inv to the_inv and turned it into an abbreviation (based on the_inv_onto).
wenzelm [Sun, 18 Oct 2009 22:19:05 +0200] rev 32997
fixed proof (cf. d1d4d7a08a66);
wenzelm [Sun, 18 Oct 2009 22:16:37 +0200] rev 32996
removed disjunctive group cancellation -- provers run independently;
sledgehammer: kill earlier session, and removed obsolete max_atps;
tuned;
wenzelm [Sun, 18 Oct 2009 21:13:29 +0200] rev 32995
tuned;
wenzelm [Sun, 18 Oct 2009 20:53:40 +0200] rev 32994
removed some unreferenced material;
tuned;
nipkow [Sun, 18 Oct 2009 18:08:04 +0200] rev 32993
merged
nipkow [Sun, 18 Oct 2009 18:07:44 +0200] rev 32992
certificates for sos
nipkow [Sun, 18 Oct 2009 16:25:59 +0200] rev 32991
merged
nipkow [Sun, 18 Oct 2009 16:25:04 +0200] rev 32990
added sums of squares for standard deviation
nipkow [Sun, 18 Oct 2009 12:07:56 +0200] rev 32989
merged
nipkow [Sun, 18 Oct 2009 12:07:25 +0200] rev 32988
Inv -> inv_onto, inv abbr. inv_onto UNIV.
wenzelm [Sun, 18 Oct 2009 00:10:20 +0200] rev 32987
disable indent-tabs-mode in Proof General / Emacs;
wenzelm [Sat, 17 Oct 2009 23:48:09 +0200] rev 32986
merged
wenzelm [Sat, 17 Oct 2009 23:47:27 +0200] rev 32985
made SML/NJ happy;
ballarin [Sat, 17 Oct 2009 23:07:53 +0200] rev 32984
Merged.
ballarin [Sat, 17 Oct 2009 22:58:18 +0200] rev 32983
Finished revisions of locales tutorial.
ballarin [Thu, 15 Oct 2009 22:22:08 +0200] rev 32982
Changed part of the examples to int.
ballarin [Thu, 15 Oct 2009 22:07:18 +0200] rev 32981
Save current state of locales tutorial.
ballarin [Thu, 15 Oct 2009 22:06:43 +0200] rev 32980
Observe order of declaration when printing registrations.
wenzelm [Sat, 17 Oct 2009 22:35:28 +0200] rev 32979
disable sunbroy2 for now;
wenzelm [Sat, 17 Oct 2009 22:34:19 +0200] rev 32978
tuned/moved divide_and_conquer';
wenzelm [Sat, 17 Oct 2009 21:14:08 +0200] rev 32977
tuned;
wenzelm [Sat, 17 Oct 2009 20:37:38 +0200] rev 32976
removed separate record_quick_and_dirty_sensitive;
wenzelm [Sat, 17 Oct 2009 20:15:59 +0200] rev 32975
simplified tactics;
use proper SUBGOAL/CSUBGOAL;
wenzelm [Sat, 17 Oct 2009 19:04:35 +0200] rev 32974
eliminated old List.foldr and OldTerm operations;
misc tuning;
wenzelm [Sat, 17 Oct 2009 18:14:47 +0200] rev 32973
removed unused names;
wenzelm [Sat, 17 Oct 2009 18:01:24 +0200] rev 32972
misc tuning and simplification;
wenzelm [Sat, 17 Oct 2009 17:18:59 +0200] rev 32971
less pervasive names;
wenzelm [Sat, 17 Oct 2009 16:58:03 +0200] rev 32970
operations of structure Skip_Proof (formerly SkipProof) no longer require quick_and_dirty mode;
wenzelm [Sat, 17 Oct 2009 16:40:41 +0200] rev 32969
Method.cheating: check quick_and_dirty here;
wenzelm [Sat, 17 Oct 2009 16:34:39 +0200] rev 32968
tuned;
wenzelm [Sat, 17 Oct 2009 16:33:14 +0200] rev 32967
Unsynchronized.set etc.;
wenzelm [Sat, 17 Oct 2009 15:57:51 +0200] rev 32966
indicate CRITICAL nature of various setmp combinators;
wenzelm [Sat, 17 Oct 2009 15:55:57 +0200] rev 32965
ISABELLE_TOOL;
wenzelm [Sat, 17 Oct 2009 15:42:36 +0200] rev 32964
tuned signature;
observe coding conventions of this file;
wenzelm [Sat, 17 Oct 2009 14:51:30 +0200] rev 32963
merged
nipkow [Sat, 17 Oct 2009 13:46:55 +0200] rev 32962
merged
nipkow [Sat, 17 Oct 2009 13:46:39 +0200] rev 32961
added the_inv_onto
wenzelm [Sat, 17 Oct 2009 14:43:18 +0200] rev 32960
eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;
wenzelm [Sat, 17 Oct 2009 01:05:59 +0200] rev 32959
removed obsolete old goal command;
wenzelm [Sat, 17 Oct 2009 00:53:18 +0200] rev 32958
legacy Drule.standard is no longer pervasive;
wenzelm [Sat, 17 Oct 2009 00:52:37 +0200] rev 32957
explicitly qualify Drule.standard;
wenzelm [Fri, 16 Oct 2009 10:55:07 +0200] rev 32956
tuned white space;
wenzelm [Fri, 16 Oct 2009 10:45:10 +0200] rev 32955
local channels for tracing/debugging;
wenzelm [Fri, 16 Oct 2009 00:26:19 +0200] rev 32954
made SML/NJ happy;
wenzelm [Thu, 15 Oct 2009 23:51:22 +0200] rev 32953
sunbroy2: back to single-threaded mode for now -- deadlock in Poly/ML 5.3-SVN-900;
wenzelm [Thu, 15 Oct 2009 23:28:10 +0200] rev 32952
replaced String.concat by implode;
replaced String.concatWith by space_implode;
replaced (Seq.flat o Seq.map) by Seq.maps;
replaced List.mapPartial by map_filter;
replaced List.concat by flat;
replaced (flat o map) by maps, which produces less garbage;
wenzelm [Thu, 15 Oct 2009 23:10:35 +0200] rev 32951
space_implode;
wenzelm [Thu, 15 Oct 2009 21:28:39 +0200] rev 32950
normalized aliases of Output operations;
wenzelm [Thu, 15 Oct 2009 21:08:03 +0200] rev 32949
eliminated slightly odd get/set operations in favour of Unsynchronized.ref;
eliminated aliases of Output operations;
print_cert: use warning for increased chance that the user actually sees the output;
misc tuning and simplification;
wenzelm [Thu, 15 Oct 2009 17:49:30 +0200] rev 32948
natural argument order for prover;
renamed atp_problem to problem;
standard naming convention for the_system;
wenzelm [Thu, 15 Oct 2009 17:06:19 +0200] rev 32947
ATP_Manager.get_prover: canonical argument order;
eliminated various aliases of existing operations, notably Output channels;
tuned messages;
misc tuning and clarification;
wenzelm [Thu, 15 Oct 2009 17:04:45 +0200] rev 32946
tuned proof (via atp_minimized);
wenzelm [Thu, 15 Oct 2009 16:15:22 +0200] rev 32945
sort_strings (cf. Pure/library.ML);
wenzelm [Thu, 15 Oct 2009 15:53:33 +0200] rev 32944
clarified File.platform_path vs. File.shell_path;
tuned;
wenzelm [Thu, 15 Oct 2009 15:45:50 +0200] rev 32943
exported File.shell_quote;
wenzelm [Thu, 15 Oct 2009 12:23:24 +0200] rev 32942
misc tuning and recovery of Isabelle coding style;
wenzelm [Thu, 15 Oct 2009 11:49:27 +0200] rev 32941
eliminated extraneous wrapping of public records;
tuned;
wenzelm [Thu, 15 Oct 2009 11:23:03 +0200] rev 32940
tuned signature;
tuned;
wenzelm [Thu, 15 Oct 2009 11:12:09 +0200] rev 32939
renamed functor HeapFun to Heap;
wenzelm [Thu, 15 Oct 2009 10:59:10 +0200] rev 32938
misc tuning and clarification;
wenzelm [Thu, 15 Oct 2009 00:55:29 +0200] rev 32937
structure ATP_Manager: eliminated slightly odd get/set operations in favour of Unsynchronized.ref;
uniform interpretation of ATP_Manager.atps via ATP_Manager.get_atps;
wenzelm [Wed, 14 Oct 2009 23:44:37 +0200] rev 32936
modernized structure names;
wenzelm [Wed, 14 Oct 2009 23:13:38 +0200] rev 32935
show direct GC time (which is included in CPU time);
wenzelm [Wed, 14 Oct 2009 22:57:44 +0200] rev 32934
eliminated obsolete C/flip combinator;
nipkow [Wed, 14 Oct 2009 21:14:53 +0200] rev 32933
added List.nth
wenzelm [Wed, 14 Oct 2009 16:45:26 +0200] rev 32932
tuned make parameters for sunbroy2;
wenzelm [Wed, 14 Oct 2009 16:39:35 +0200] rev 32931
accomodate old version of "tail", e.g. on sunbroy2;
wenzelm [Wed, 14 Oct 2009 16:08:51 +0200] rev 32930
settings for parallel experimental Poly/ML 5.3;
haftmann [Wed, 14 Oct 2009 13:56:56 +0200] rev 32929
sharpened name
haftmann [Wed, 14 Oct 2009 12:20:01 +0200] rev 32928
more explicit notion of canonized code equations
haftmann [Wed, 14 Oct 2009 12:19:17 +0200] rev 32927
more explicit notion of canonized code equations
haftmann [Wed, 14 Oct 2009 12:04:16 +0200] rev 32926
tuned whitespace
haftmann [Wed, 14 Oct 2009 12:03:16 +0200] rev 32925
tuned whitespace
haftmann [Wed, 14 Oct 2009 11:56:44 +0200] rev 32924
dropped Code_Printer prefix where feasible; fixed whitespace issues; more coherent terminology
haftmann [Tue, 13 Oct 2009 14:57:53 +0200] rev 32923
merged
haftmann [Tue, 13 Oct 2009 14:08:01 +0200] rev 32922
deactivated Datatype.distinct_simproc
haftmann [Tue, 13 Oct 2009 14:08:00 +0200] rev 32921
dropped Datatype.distinct_simproc; tuned
hoelzl [Tue, 13 Oct 2009 13:40:26 +0200] rev 32920
order conjunctions to be printed without parentheses
hoelzl [Tue, 13 Oct 2009 12:02:55 +0200] rev 32919
approximation now fails earlier when using interval splitting; value [approximate] now supports bounded variables; renamed Var -> Atom for better readability
haftmann [Tue, 13 Oct 2009 09:13:24 +0200] rev 32918
merged
haftmann [Mon, 12 Oct 2009 16:16:44 +0200] rev 32917
added add_tyconames; tuned
haftmann [Tue, 13 Oct 2009 08:36:53 +0200] rev 32916
merged
haftmann [Tue, 13 Oct 2009 08:36:39 +0200] rev 32915
more appropriate abstraction over distinctness rules
haftmann [Mon, 12 Oct 2009 15:48:12 +0200] rev 32914
merged
haftmann [Mon, 12 Oct 2009 15:46:38 +0200] rev 32913
intro_base_names combinator
haftmann [Mon, 12 Oct 2009 15:26:50 +0200] rev 32912
merged
haftmann [Mon, 12 Oct 2009 15:26:40 +0200] rev 32911
dropped dist_ss