Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+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.
automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
2011-02-09, by blanchet
renamed field
2011-02-09, by blanchet
added "Z3 as an ATP" support to Sledgehammer locally
2011-02-09, by blanchet
remove Z3 wrapper script, which is no longer necessary now that the SMT module generates SMT-LIB compliant files
2011-02-09, by blanchet
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
2011-02-09, by blanchet
tuned scope of Multithreading.interrupted vs. Multithreading.with_attributes;
2011-02-09, by wenzelm
merged
2011-02-09, by bulwahn
changing auto-quickcheck to be considered a non-interactive invocation of quickcheck
2011-02-08, by bulwahn
discontinued obsolete lib/scripts/polyml-platform;
2011-02-08, by wenzelm
clarified comment -- ancienct PG 3.7.x is still in use;
2011-02-08, by wenzelm
discontinued obsolete alias HOL.thy for @{theory HOL} in ML;
2011-02-08, by wenzelm
prefer polyml-5.2.1 over odd polyml-5.3.0-old;
2011-02-08, by wenzelm
some shuffling of isatest settings, to ensure coverage of polyml-5.2.1, polyml-5.3.0, polyml-5.4.0, polyml-5.4.1 (SVN), smlnj/110.72;
2011-02-08, by wenzelm
reverted slightly odd eb5900951702: isatest-doc should work again due to 4b08499b3db1 (polyml-5.3.0 supports proper TimeLimit, as required for HOL-Nitpick-Examples);
2011-02-08, by wenzelm
merged
2011-02-08, by wenzelm
available_provers ~> supported_provers (for clarity)
2011-02-08, by blanchet
sort E weights
2011-02-08, by blanchet
added support for bleeding-edge E weighting function "SymOffsetsWeight"
2011-02-08, by blanchet
transformed lie into truth
2011-02-08, by blanchet
enable SMT weights and triggers, since they lead to slight improvements according to the Judgment Day suite
2011-02-08, by blanchet
improving sum type and option type term constructions for correct presentation in Smallcheck
2011-02-08, by bulwahn
Explicitly build HOLCF and ZF images. They are not part of the release any more.
2011-02-08, by kleing
added termination lemmas
2011-02-08, by nipkow
improving term construction of product types in Smallcheck which enables correct presentation of counterexamples
2011-02-07, by bulwahn
discontinued support for Poly/ML 5.2, which was the last version without proper multithreading and TimeLimit implementation;
2011-02-08, by wenzelm
tuned headers;
2011-02-08, by wenzelm
updated to polyml-5.3.0, which is presently known as the most robust version;
2011-02-08, by wenzelm
explicit Multithreading.interrupted to ensure that interrupts stay within the boundaries of managed evaluation blocks;
2011-02-08, by wenzelm
always test/clear Multithreading.interrupted, indepently of thread attributes;
2011-02-08, by wenzelm
added Multithreading.interrupted (cf. java.lang.Thread.interrupted);
2011-02-08, by wenzelm
more robust TimeLimit: make double sure that watchdog has terminated and interrupts received during uninterruptible state are propagated (NB: Thread.testInterrupt requires InterruptSynch in Poly/ML 5.4.0 or earlier);
2011-02-07, by wenzelm
more tracing information via Par_List.map_name;
2011-02-05, by wenzelm
clarified bootstrapping of structure TimeLimit;
2011-02-05, by wenzelm
more scalable collections of tasks, notably for totality of known group members;
2011-02-04, by wenzelm
tuned signature;
2011-02-04, by wenzelm
merged
2011-02-04, by wenzelm
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
2011-02-04, by hoelzl
add auto support for AE_mp
2011-02-04, by hoelzl
add borel_fubini_integrable; remove unused bijectivity rules for measureable functions
2011-02-04, by hoelzl
parallelization of nested Isar proofs is subject to Goal.parallel_proofs_threshold;
2011-02-04, by wenzelm
Task_Queue.update_timing: more precise treatment of interruptibility;
2011-02-04, by wenzelm
Lazy.force_result: more standard treatment of interruptibility, potentially addressing races of exceptions vs. interrupts;
2011-02-04, by wenzelm
thm_proof: visible fulfill_body only, without joining nested thms -- retain proof irrelevance, which is important for parallel performance;
2011-02-03, by wenzelm
tuned comments;
2011-02-03, by wenzelm
clarified Proofterm.proofs_enabled;
2011-02-03, by wenzelm
explicit is better than implicit;
2011-02-03, by wenzelm
tuned odd conditional expression;
2011-02-02, by wenzelm
eliminated slightly odd abstract type Task_Queue.deps;
2011-02-02, by wenzelm
merged
2011-02-02, by wenzelm
Introduction of metis calls and other cosmetic modifications.
2011-02-02, by paulson
merged
2011-02-02, by boehmes
avoid ML structure aliases (especially single-letter abbreviations)
2011-02-02, by boehmes
making the bash script swipl_version closer to Isabelle's conventional bash scripts
2011-02-02, by bulwahn
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
2011-02-02, by hoelzl
merged
2011-02-02, by bulwahn
scala serializer adds parentheses around function literals
2011-02-02, by bulwahn
made SML/NJ happy
2011-02-02, by krauss
term style 'isub': ad-hoc subscripting of variables that end with digits (x1, x23, ...)
2011-02-01, by krauss
refined Task_Queue.dequeue_deps (more incremental);
2011-02-02, by wenzelm
maintain Task_Queue.group within Task_Queue.task;
2011-02-02, by wenzelm
tuned comment;
2011-02-02, by wenzelm
Future.join_results: discontinued post-hoc recording of dynamic dependencies;
2011-02-02, by wenzelm
more informative task timing: some dependency tracking;
2011-02-01, by wenzelm
refined task timing: joining vs. waiting;
2011-02-01, by wenzelm
simplified trace;
2011-02-01, by wenzelm
more specific Goal.fork_name;
2011-01-31, by wenzelm
name "passive" tasks (practically lazy values);
2011-01-31, by wenzelm
tuned trivial cases;
2011-01-31, by wenzelm
tuned signature;
2011-01-31, by wenzelm
support named tasks, for improved tracing;
2011-01-31, by wenzelm
more direct Future.bulk, which potentially reduces overhead for Par_List;
2011-01-31, by wenzelm
tuned isatest settings;
2011-01-31, by wenzelm
added basic task timing;
2011-01-31, by wenzelm
some notes on Cygwin;
2011-01-31, by wenzelm
more platform hints;
2011-01-31, by wenzelm
merged
2011-01-31, by wenzelm
tuned;
2011-01-31, by wenzelm
back to post-release mode;
2011-01-31, by wenzelm
removed obsolete test tags;
2011-01-30, by wenzelm
removed Florian's email from isatest (bounces)
2011-01-28, by kleing
merged
2011-01-25, by hoelzl
use pre-image measure, instead of image
2011-01-24, by hoelzl
use AE_mp in AE_conjI proof
2011-01-21, by hoelzl
tuned proof
2011-01-19, by hoelzl
merged
2011-01-21, by haftmann
moved theorem
2011-01-21, by haftmann
restructured theory;
2011-01-21, by haftmann
merged
2011-01-19, by hoelzl
Gauge measure removed
2011-01-18, by hoelzl
merged
2011-01-18, by haftmann
report mutabelle log in mira configuration
2011-01-18, by haftmann
back to post-release mode;
2011-01-17, by wenzelm
delete .elc files unconditionally -- they cause too many incompatibilities;
2011-01-30, by wenzelm
Added tag Isabelle2011 for changeset 6d736d983d5c
2011-01-30, by wenzelm
clarified example settings for Proof General;
Isabelle2011
2011-01-30, by wenzelm
adhoc patches relative to ProofGeneral-4.1pre101216, which has setprefs working;
2011-01-28, by wenzelm
more precise stats;
2011-01-28, by wenzelm
some adhoc patches for ProofGeneral-4.1pre110112;
2011-01-28, by wenzelm
enforce STIXGeneral, which is preferred by PG 4.1;
2011-01-28, by wenzelm
default UTF-8 locale, to work with funny base directory (e.g. Chinese);
2011-01-28, by wenzelm
enforce fonts;
2011-01-28, by wenzelm
added option -f FONT;
2011-01-27, by wenzelm
Proof General 4.x interface wrapper;
2011-01-27, by wenzelm
old Proof General patches;
2011-01-27, by wenzelm
Added tag isa2011-test3 for changeset 55a45051b220
2011-01-27, by wenzelm
Tuned definition of sdiv.
2011-01-27, by berghofe
CRITICAL markup for critical poking with unsynchronized references;
2011-01-27, by wenzelm
Replaced smod by standard mod operator to reflect actual behaviour
2011-01-26, by berghofe
cancel document execution before editing, to improve reactivity on systems with few cores;
2011-01-27, by wenzelm
tuned isatest settings (for Poly/ML SVN 1278);
2011-01-25, by wenzelm
merged
2011-01-25, by wenzelm
do not restore old files on startup, which is potentially slow due to automatic rechecking;
2011-01-25, by wenzelm
singleton (sequential) execution, to avoid race conditions in theory loader state (e.g. when multiple independent theories import the same theory);
2011-01-25, by wenzelm
workaround for odd x86_64 problem in Poly/ML 5.4.0 (actually SVN 1151?), which causes unexpected nontermination of Isabelle/Scala document editing;
2011-01-25, by wenzelm
improved README -- Isabelle symbols and fonts;
2011-01-24, by wenzelm
delete compiled .elc files to improve portability on Linux, notably for GNU Emacs 23.1.x instead of 23.2.x;
2011-01-24, by wenzelm
do not overwrite proof-shell-quit-timeout by default (final PG 4.1 supposedly gets it right);
2011-01-23, by wenzelm
Added tag isa2011-test2 for changeset 237328506a42
2011-01-23, by wenzelm
Documented unused_thms
2011-01-23, by berghofe
JVM/Windows: more robust treatment of unicode in file names;
2011-01-21, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip