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.
move lemma Inf to usage point
2013-03-05, by hoelzl
tuned proof of Edelstein fixed point theorem (use continuity of dist and attains_sup)
2013-03-05, by hoelzl
tuned proofs (used continuity of infdist, dist and continuous_attains_sup)
2013-03-05, by hoelzl
generalized continuous/compact_attains_inf/sup from real to linorder_topology
2013-03-05, by hoelzl
continuity of pair operations
2013-03-05, by hoelzl
use generate_topology for second countable topologies, does not require intersection stable basis
2013-03-05, by hoelzl
generalized isGlb_unique
2013-03-05, by hoelzl
complete_linorder is also a complete_distrib_lattice
2013-03-05, by hoelzl
move Liminf / Limsup lemmas on complete_lattices to its own file
2013-03-05, by hoelzl
merged
2013-03-05, by nipkow
New theory of infinity-extended types; should replace Extended_xyz eventually
2013-03-05, by nipkow
Avoid ML warning about unreferenced identifier.
2013-03-05, by webertj
polymorphic SPASS is also SPASS
2013-03-05, by blanchet
allow more general coercion maps; tuned;
2013-03-05, by traytel
more lemmas about intervals
2013-03-05, by nipkow
merged
2013-03-04, by wenzelm
refined parallel_proofs = 2: fork whole Isar sub-proofs, not just terminal ones;
2013-03-04, by wenzelm
join all proofs before scheduling present phase (ordered according to weight);
2013-03-04, by wenzelm
more explicit datatype result;
2013-03-04, by wenzelm
split dense into inner_dense_order and no_top/no_bot
2013-02-20, by hoelzl
move auxiliary lemmas from Library/Extended_Reals to HOL image
2013-02-20, by hoelzl
tuned (extend datatype to inline option)
2013-03-04, by traytel
prefer more systematic Future.flat;
2013-03-03, by wenzelm
more uniform Future.map: always internalize failure;
2013-03-03, by wenzelm
uniform treatment of global/local proofs;
2013-03-03, by wenzelm
tuned;
2013-03-03, by wenzelm
clarified Toplevel.element_result wrt. Toplevel.is_ignored;
2013-03-03, by wenzelm
more Thy_Syntax.element operations;
2013-03-03, by wenzelm
coercion-invariant arguments at work
2013-03-01, by traytel
constants with coercion-invariant arguments (possibility to disable/reenable
2013-03-01, by traytel
simplified Proof.future_proof;
2013-02-28, by wenzelm
provide explicit dummy names (cf. dfe469293eb4);
2013-02-28, by wenzelm
discontinued empty name bindings in 'axiomatization';
2013-02-28, by wenzelm
provide common HOLogic.conj_conv and HOLogic.eq_conv;
2013-02-28, by wenzelm
just one HOLogic.Trueprop_conv, with regular exception CTERM;
2013-02-28, by wenzelm
discontinued obsolete 'axioms' command;
2013-02-28, by wenzelm
more robust build error handling, e.g. missing outer syntax commands;
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
eliminated legacy 'axioms';
2013-02-28, by wenzelm
marginalized historic strip_tac;
2013-02-28, by wenzelm
tuned proof;
2013-02-28, by wenzelm
tuned whitespace and indentation;
2013-02-28, by wenzelm
simplified imports;
2013-02-28, by wenzelm
load timings in parallel for improved performance;
2013-02-28, by wenzelm
proper place for cancel_div_mod.ML (see also ee729dbd1b7f and ec7f10155389);
2013-02-28, by wenzelm
parallel dep.load_files saves approx. 1s on 4 cores;
2013-02-27, by wenzelm
eliminated pointless re-ified errors;
2013-02-27, by wenzelm
merged
2013-02-27, by wenzelm
discontinued redundant 'use' command;
2013-02-27, by wenzelm
discontinued obsolete header "files" -- these are loaded explicitly after exploring dependencies;
2013-02-27, by wenzelm
discontinued obsolete 'uses' within theory header;
2013-02-27, by wenzelm
use lemma from Big_Operators
2013-02-27, by Andreas Lochbihler
add inclusion/exclusion lemma
2013-02-27, by Andreas Lochbihler
added lemma
2013-02-27, by Andreas Lochbihler
merged
2013-02-27, by Andreas Lochbihler
add wellorder instance for Numeral_Type (suggested by Jesus Aransay)
2013-02-27, by Andreas Lochbihler
updated Toplevel.command_exception;
2013-02-26, by wenzelm
tuned;
2013-02-26, by wenzelm
tuned signature;
2013-02-26, by wenzelm
fork diagnostic commands (theory loader and PIDE interaction);
2013-02-26, by wenzelm
disallow shutdown from worker, which would lead to deadlock since the scheduler cannot terminate;
2013-02-26, by wenzelm
tuned 2464ba6e6fc9 -- NB: approximative_id is NONE for PIDE document transactions;
2013-02-26, by wenzelm
signal work_available should be sufficient to initiate daisy-chained workers, and lead to separate broadcast work_finished eventually -- NB: broadcasting all worker threads tends to burn parallel CPU cycles;
2013-02-26, by wenzelm
less eventful shutdown: merely wait for scheduler to terminate;
2013-02-26, by wenzelm
tuned messages;
2013-02-26, by wenzelm
tuned;
2013-02-26, by wenzelm
merged;
2013-02-25, by wenzelm
more explicit Goal.shutdown_futures;
2013-02-25, by wenzelm
reconsider 'export_code' as "thy_decl" command due to its global side-effect on the file-system;
2013-02-25, by wenzelm
discontinued pointless command category "thy_schematic_goal" -- this is checked dynamically;
2013-02-25, by wenzelm
clarified Toplevel.element_result: scheduling policies happen here;
2013-02-25, by wenzelm
prefer stateless 'ML_val' for tests;
2013-02-25, by wenzelm
tuned comment;
2013-02-25, by wenzelm
reconsider 'pretty_setmargin' as "control" command (instead of "diag") -- it is stateful and Proof General legacy;
2013-02-25, by wenzelm
merged;
2013-02-25, by wenzelm
simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
2013-02-24, by wenzelm
tuned;
2013-02-24, by wenzelm
unified Command.is_proper in ML with Scala (see also 123be08eed88);
2013-02-24, by wenzelm
tuned order of modules;
2013-02-25, by wenzelm
fixed document;
2013-02-25, by wenzelm
turned example into library for comparing growth of functions
2013-02-24, by haftmann
corrected reference
2013-02-24, by haftmann
improved orderings
2013-02-24, by nipkow
tuned agressiveness of isar compression
2013-02-24, by smolkas
eliminated isize in favour of size + type coercion
2013-02-24, by kleing
make SML/NJ happy;
2013-02-23, by wenzelm
basic setup for appbundler-1.0 for Mac OS X and Java 7;
2013-02-23, by wenzelm
more robust handling of repeated interrupts while terminating managed process;
2013-02-23, by wenzelm
more friendly message for spurious InterruptedException, which might still occur due to JVM oddities;
2013-02-23, by wenzelm
more explicit GUI components for dynamic actions;
2013-02-23, by wenzelm
clarified Progress.stopped: rising edge only;
2013-02-23, by wenzelm
more explicit console interrupt handling;
2013-02-23, by wenzelm
more permissive File.read_lines, which is relevant for Managed_Process join/kill;
2013-02-23, by wenzelm
support for POSIX interrupts (bypassed on Windows);
2013-02-23, by wenzelm
merged
2013-02-22, by traytel
tuned error messages
2013-02-22, by traytel
Coercion_Examples defines required coercions itself (no Complex_Main needed)
2013-02-22, by traytel
apply unifying substitution before building the constraint graph
2013-02-22, by traytel
more abstract intervals
2013-02-22, by nipkow
more robust load_timings: ignore XML.Decode errors as well;
2013-02-22, by wenzelm
make SML/NJ happy;
2013-02-22, by wenzelm
identify exceptions more robustly, to allow SML/NJ report toplevel errors without crash;
2013-02-22, by wenzelm
make SML/NJ happy;
2013-02-22, by wenzelm
updated headers;
2013-02-22, by wenzelm
eliminated hard tabs;
2013-02-22, by wenzelm
discontinued obsolete src/HOL/IsaMakefile;
2013-02-22, by wenzelm
merged
2013-02-21, by wenzelm
more explicit session dependency, for improved parallel performance of HOL-UNITY test session -- NB: separate 'theories' sections are sequential;
2013-02-21, by wenzelm
merged
2013-02-21, by wenzelm
removed obsolete tags;
2013-02-21, by wenzelm
highest priority for proofs with unknown / very short timing -- recover original scheduling with parallel_proofs_reuse_timing = false;
2013-02-21, by wenzelm
tuned misleading message
2013-02-21, by blanchet
merged
2013-02-21, by wenzelm
option parallel_proofs_reuse_timing controls reuse of log information -- since it is not always beneficial for performance;
2013-02-20, by wenzelm
prefer outdegree in comparison again (cf. 88c96e836ed6) -- NB: big jobs might hide behind small ones in this naive queuing scheme;
2013-02-20, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip