Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-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.
merged
2013-03-13, by wenzelm
clarified parallel_subproofs_saturation (blind guess) vs. parallel_subproofs_threshold (precient timing estimate);
2013-03-13, by wenzelm
proper formatting, to facilitate line-based diff;
2013-03-13, by wenzelm
more uniform session descriptions, which show up in chapter index;
2013-03-13, by wenzelm
proper index for HOL-Proofs, which is also in chapter "HOL";
2013-03-13, by wenzelm
include only README.html, not historic README, which tends towards surprises like src/HOL/SPARK/Examples/README;
2013-03-13, by wenzelm
more accurate handling of global browser info at the very end (without races), subject to no_build and info.browser_info;
2013-03-13, by wenzelm
sessions may be organized via 'chapter' in ROOT;
2013-03-13, by wenzelm
do not absorb I/O errors;
2013-03-13, by wenzelm
show expanded path, to avoid odd /foo/bar/$ISABELLE_BROWSER_INFO/baz;
2013-03-13, by wenzelm
new lemma subset_decode_imp_le
2013-03-13, by paulson
merged
2013-03-13, by kleing
more IMP snippets
2013-03-13, by kleing
rename fset_member to fmember and prove parametricity
2013-03-13, by kuncar
BNF uses fset defined via Lifting/Transfer rather than Quotient
2013-03-13, by traytel
nitpick setup and code generation for streams
2013-03-13, by traytel
merged
2013-03-13, by nipkow
tuned
2013-03-13, by nipkow
proper path -- I/O was hidden due to permissiveness;
2013-03-12, by wenzelm
merged
2013-03-12, by wenzelm
removed odd cvs artifacts;
2013-03-12, by wenzelm
refurbished some old README.html files as session descriptions, which show up in chapter index;
2013-03-12, by wenzelm
include session description in chapter index;
2013-03-12, by wenzelm
tuned;
2013-03-12, by wenzelm
more accurate theory links;
2013-03-12, by wenzelm
discontinued "isabelle usedir" option -r (reset session path);
2013-03-12, by wenzelm
discontinued "isabelle usedir" option -P (remote path);
2013-03-11, by wenzelm
support for 'chapter' specifications within session ROOT;
2013-03-11, by wenzelm
added latex markup
2013-03-12, by nipkow
merged
2013-03-12, by kleing
more snippets
2013-03-12, by kleing
added pairs
2013-03-12, by nipkow
extended set comprehension notation with {pttrn : A . P}
2013-03-12, by nipkow
tuned
2013-03-11, by nipkow
more factorisation of Step & Co
2013-03-11, by nipkow
factored out Step
2013-03-10, by nipkow
merged
2013-03-10, by nipkow
stepwise instantiation is more modular
2013-03-10, by nipkow
generalized subclass relation;
2013-03-10, by haftmann
termination proof for narrowing: fewer assumptions
2013-03-10, by nipkow
accomodate encrypted file-system on linux;
2013-03-09, by wenzelm
tuned;
2013-03-09, by wenzelm
discontinued theory src/HOL/Library/Eval_Witness -- assumptions do not longer hold in presence of abstract types
2013-03-09, by haftmann
updated keywords (cf. 84d01fd733cf);
2013-03-08, by wenzelm
proper type inference for default values
2013-03-08, by blanchet
convert mappings to parametric lifting
2013-03-08, by kuncar
setup_lifting doesn't support a type variable as a raw type
2013-03-08, by kuncar
add [relator_mono] and [relator_distr] rules
2013-03-08, by kuncar
simplify Lift_FSet because we have parametricity in Lifting now
2013-03-08, by kuncar
patch Isabelle ditribution to conform to changes regarding the parametricity
2013-03-08, by kuncar
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
2013-03-08, by kuncar
merged
2013-03-08, by nipkow
simplified basic termination proof
2013-03-08, by nipkow
some simp rules for fset
2013-03-08, by traytel
avoid -Infinity which confuses JFreeChart histogram;
2013-03-07, by wenzelm
tuned proofs -- more structure, less warnings;
2013-03-07, by wenzelm
tuned signature -- prefer terminology of Scala and Axiom;
2013-03-07, by wenzelm
better message (type-unsoundnesses are becoming rare, usually the issue is elsewhere, e.g. in the TSTP proof parser)
2013-03-07, by blanchet
avoid using Arith_Data.dest_sum in extended-nat simprocs (it treats 'x - y' as 'x + - y', which is not valid for enat)
2013-03-06, by huffman
netlimit is abbreviation for Lim
2013-03-06, by hoelzl
tuned proofs
2013-03-06, by hoelzl
changed has_derivative_intros into a named theorems collection
2013-03-06, by hoelzl
changed continuous_on_intros into a named theorems collection
2013-03-06, by hoelzl
changed continuous_intros into a named theorems collection
2013-03-06, by hoelzl
add tendsto_eq_intros: they add an additional rewriting step at the rhs of --->
2013-03-06, by hoelzl
major redesign: order instead of preorder, new definition of intervals as quotients
2013-03-06, by nipkow
added lemma
2013-03-06, by nipkow
extended numerals
2013-03-06, by nipkow
merged
2013-03-05, by wenzelm
merged
2013-03-05, by wenzelm
removed unused Future.flat, while leaving its influence of Future.map (see bcd6b1aa4db5);
2013-03-05, by wenzelm
extended stream library a little more
2013-03-05, by traytel
extended stream library
2013-03-05, by traytel
generalized lemmas in Extended_Real_Limits
2013-03-05, by hoelzl
eventually nhds represented using sequentially
2013-03-05, by hoelzl
generalized compact_Times to topological_space
2013-03-05, by hoelzl
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
more tight representation of command timing;
2013-02-20, by wenzelm
prefer comparison of session timing, if this is known already;
2013-02-20, by wenzelm
proper check of Proof.is_relevant (again, cf. c3e99efacb67 and df8fc0567a3d);
2013-02-20, by wenzelm
support nested Thy_Syntax.element;
2013-02-20, by wenzelm
back to non-schematic 'sublocale' and 'interpretation' (despite df8fc0567a3d) for more potential parallelism;
2013-02-19, by wenzelm
help JVM to cope with large symbolic structures;
2013-02-19, by wenzelm
improved scheduling of forked proofs, based on elapsed time estimate (from last run via session log file);
2013-02-19, by wenzelm
read logs from failed sessions as well;
2013-02-19, by wenzelm
recover timing information from old log files;
2013-02-19, by wenzelm
suppress timing message in full PIDE protocol -- this is for batch build;
2013-02-19, by wenzelm
support for build passing timings from Scala to ML;
2013-02-19, by wenzelm
support for prescient timing information within command transactions;
2013-02-19, by wenzelm
emit command_timing properties into build log;
2013-02-19, by wenzelm
generate Isar proof if Metis appears to be too slow
2013-02-21, by blanchet
swap slices so that the last slice is more complete (for minimization)
2013-02-21, by blanchet
tuning
2013-02-21, by blanchet
ensure all conjecture clauses are in the graph -- to prevent exceptions later
2013-02-20, by blanchet
generalize syntax of SPASS proofs
2013-02-20, by blanchet
tweaked hack some more
2013-02-20, by blanchet
more simplifying constructors
2013-02-20, by blanchet
remove needless steps from refutation graph -- these confuse the proof redirection algorithm (and are needless)
2013-02-20, by blanchet
more precise error
2013-02-20, by blanchet
improved hack
2013-02-20, by blanchet
upgraded to Alt-Ergo 0.95
2013-02-20, by blanchet
don't pass chained facts directly to SMT solvers -- this breaks various invariants and is never necessary
2013-02-20, by blanchet
trust preplayed proof in Mirabelle
2013-02-20, by blanchet
added case taken out by mistake
2013-02-20, by blanchet
tuning (removed redundant datatype)
2013-02-20, by blanchet
minimize SMT proofs with E if Isar proofs are desired and Metis managed to preplay
2013-02-20, by blanchet
honor linearization option also in the evaluation driver
2013-02-20, by blanchet
got rid of rump support for Vampire definitions
2013-02-20, by blanchet
optimize Isar output some more
2013-02-20, by blanchet
turn off more evil Vampire options to facilitate Isar proof generation
2013-02-20, by blanchet
fixed typo in option name
2013-02-20, by blanchet
tuning
2013-02-20, by blanchet
use new skolemizer only if some skolems have two or more arguments -- otherwise the old skolemizer cannot get the arg order wrong
2013-02-20, by blanchet
slacker comparison for Skolems, to avoid trivial equations
2013-02-20, by blanchet
auto-minimizer should respect "isar_proofs = true"
2013-02-20, by blanchet
made "isar_proofs" a 3-way option, to provide a way to totally disable isar_proofs if desired
2013-02-20, by blanchet
alias for people like me
2013-02-20, by blanchet
dropped spurious left-over from 0a2371e7ced3
2013-02-19, by haftmann
avoid using "smt" for minimization -- better use the prover itself, since then Sledgehammer gets to try metis again and gives the opportunity to output an Isar proof -- and show Isar proof as fallback for SMT proofs
2013-02-19, by blanchet
interpret "max_facts" argument in a slice-dependent fashion, instead of forcing the same number of facts to all slices
2013-02-19, by blanchet
delete also predicates on relations when hiding an implementation of an abstract type
2013-02-19, by kuncar
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip