Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+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.
duplicate "relpow" facts for "relpowp" (to emphasize that both worlds exist and obtain better search results with "find_theorems")
2012-04-16, by Christian Sternagel
updated for release;
2012-04-16, by wenzelm
more precise handling of java failure, due to missing ISABELLE_JDK_HOME;
2012-04-16, by wenzelm
tuned some proofs;
2012-04-16, by huffman
centralized enriched_type declaration, thanks to in-situ available Isar commands
2012-04-15, by haftmann
tuned whitespace
2012-04-15, by haftmann
replace locale 'UFT' with new un-named context block feature;
2012-04-15, by huffman
more CONTRIBUTORS;
2012-04-15, by wenzelm
some coverage of bundled declarations;
2012-04-15, by wenzelm
more uniform outline;
2012-04-15, by wenzelm
some coverage of unnamed contexts, which can be nested within other targets;
2012-04-15, by wenzelm
gathered mirabelle_sledgehammer's hardcoded defaults
2012-04-14, by sultana
Mirabelle's 'usage' description relating to Sledgehammer now synchs with the ML code of the Mirabelle-Sledgehammer action
2012-04-14, by sultana
Mirabelle now gives usage info when no arguments given
2012-04-14, by sultana
switched from using sed to perl in mirabelle tool
2012-04-14, by sultana
renamed mirabelle Tools directory to Actions, to make consistent with 'usage' description;
2012-04-14, by sultana
refined Cooper.tac / "presburger" method: Subgoal.FOCUS_PARAMS allows to solve more problems with outer quantifiers, e.g "!!x. [| 0 <= (x::int); x div 2 < f x |] ==> x < f x * 2";
2012-04-14, by wenzelm
merged;
2012-04-14, by wenzelm
removed HOL/ex/Set_Algebras -- outdated clone, obsolete as example
2012-04-14, by krauss
aligned tptp_graph dependencies to Isabelle conventions;
2012-04-14, by sultana
more ambitious isatest settings using polyml-svn (e.g. 1487);
2012-04-14, by wenzelm
use official TextArea.isCaretVisible and thus follow the "blink" flag;
2012-04-14, by wenzelm
display more memory;
2012-04-14, by wenzelm
keyword ";" is declared via prover (as "minor", not "diag");
2012-04-14, by wenzelm
outermost SELECT_GOAL potentially improves performance;
2012-04-14, by wenzelm
report ISABELLE_HOME_WINDOWS;
2012-04-14, by wenzelm
chmod +x;
2012-04-14, by wenzelm
more robust invocation via ISABELLE_JDK_HOME and SCALA_HOME;
2012-04-14, by wenzelm
misc tuning for release;
2012-04-14, by wenzelm
revert changes of already published NEWS;
2012-04-14, by wenzelm
some updates for release;
2012-04-14, by wenzelm
more robust treatment of ISABELLE_HOME on windows: eliminate spaces and funny unicode characters in directory name via DOS~1 notation;
2012-04-14, by wenzelm
updated Scala/JVM versions;
2012-04-14, by wenzelm
include trailing comments in proper_command range;
2012-04-13, by wenzelm
minimal support for x86-mingw;
2012-04-13, by wenzelm
recognize MacOS on modern Java implementations, notably OpenJDK 1.7;
2012-04-13, by wenzelm
updated to Scala 2.9.2;
2012-04-13, by wenzelm
updated headers;
2012-04-13, by wenzelm
eliminated hard tabs;
2012-04-13, by wenzelm
Automated merge with ssh://macbroy25.informatik.tu-muenchen.de//home/isabelle-repository/repos/isabelle
2012-04-13, by Andreas Lochbihler
NEWS
2012-04-13, by Andreas Lochbihler
adapt to changes in RBT_Impl
2012-04-13, by Andreas Lochbihler
move RBT implementation into type class contexts
2012-04-13, by Andreas Lochbihler
misc tuning;
2012-04-13, by wenzelm
NEWS
2012-04-13, by bulwahn
merged
2012-04-12, by krauss
distributivity of * over Un and UNION
2012-04-12, by krauss
Set_Algebras: removed syntax \<oplus> and \<otimes>, in favour of plain + and *
2012-04-12, by krauss
removed "setsum_set", now subsumed by generic setsum
2012-04-12, by krauss
backported Set_Algebras to use type classes (basically reverting b3e8d5ec721d from 2008)
2012-04-12, by krauss
tuned README;
2012-04-12, by wenzelm
direct scala toplevel tools to ISABELLE_JDK_HOME;
2012-04-12, by wenzelm
simplified component structure;
2012-04-12, by wenzelm
merged
2012-04-12, by wenzelm
merged
2012-04-12, by Andreas Lochbihler
generalise case certificates to allow ignored parameters
2012-04-12, by Andreas Lochbihler
merged
2012-04-12, by bulwahn
manual merge
2012-04-04, by griff
dropped abbreviation "pred_comp"; introduced infix notation "P OO Q" for "relcompp P Q"
2012-04-03, by griff
renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
2012-04-03, by griff
more standard method setup;
2012-04-12, by wenzelm
more precise declaration of goal_tfrees in forked proof state;
2012-04-12, by wenzelm
partial revert of 8a179a0493e3 -- expose failure status of result (potentially via group) instead of isolated interrupt;
2012-04-12, by wenzelm
multiset operations are defined with lift_definitions;
2012-04-12, by bulwahn
remove outdated comment
2012-04-12, by huffman
rule composition via attribute "OF" (or ML functions OF/MRS) is more tolerant against multiple unifiers;
2012-04-11, by wenzelm
standardized ML aliases;
2012-04-11, by wenzelm
clarified proof_result: finish proof formally via head tr, not end_tr;
2012-04-11, by wenzelm
tuned;
2012-04-11, by wenzelm
more robust Future.fulfill wrt. duplicate assignment and interrupt;
2012-04-11, by wenzelm
tuned message;
2012-04-11, by wenzelm
always signal after cancel_group: passive tasks may have become active;
2012-04-11, by wenzelm
just one dedicated execution per document version -- NB: non-monotonicity of cancel always requires fresh update;
2012-04-11, by wenzelm
merged
2012-04-10, by wenzelm
moved lift_raw_const wrapper out of the Quotient-package into Nominal2
2012-04-10, by Christian Urban
misc tuning and simplification;
2012-04-10, by wenzelm
static relevance of proof via syntax keywords;
2012-04-10, by wenzelm
tuned future priorities: print 0, goal ~1, execute ~2;
2012-04-10, by wenzelm
updated for Poly/ML SVN 1476;
2012-04-10, by wenzelm
some coverage of HOL/TPTP;
2012-04-10, by wenzelm
added graph-conversion utility for TPTP files
2012-04-10, by sultana
moved non-interpret-specific code to different module
2012-04-10, by sultana
disable parallel proofs (again) -- still suffering from instabilites wrt. interrupts;
2012-04-09, by wenzelm
tuned proofs;
2012-04-09, by wenzelm
slightly faster default compilation of Isabelle/Scala;
2012-04-09, by wenzelm
more explicit last exec result;
2012-04-09, by wenzelm
dynamic propagation of node "updated" status, which is required to propagate edits and re-assigments and allow direct memo_result;
2012-04-09, by wenzelm
tuned;
2012-04-09, by wenzelm
simplified Future.cancel/cancel_group (again) -- running threads only;
2012-04-09, by wenzelm
added ML pretty-printing;
2012-04-09, by wenzelm
merged
2012-04-07, by wenzelm
merged
2012-04-07, by wenzelm
explicit constructor Nat leaves nat_of as conversion
2012-04-07, by haftmann
abandoned almost redundant *_foldr lemmas
2012-04-06, by haftmann
tuned
2012-04-06, by haftmann
no preference wrt. fold(l/r); prefer fold rather than foldr for iterating over lists in generated code
2012-04-06, by haftmann
enable parallel proofs (cf. e8552cba702d), only affects packages so far;
2012-04-07, by wenzelm
added static command status markup, to emphasize accepted but unassigned/unparsed commands (notably in overview panel);
2012-04-07, by wenzelm
tuned proofs;
2012-04-07, by wenzelm
more robust update_perspective, e.g. required after reload of buffer that is not at start position;
2012-04-07, by wenzelm
tuned imports;
2012-04-07, by wenzelm
updated header keywords;
2012-04-07, by wenzelm
init message not bad;
2012-04-07, by wenzelm
explicit checks stable_finished_theory/stable_command allow parallel asynchronous command transactions;
2012-04-07, by wenzelm
discontinued obsolete last_execs (cf. cd3ab7625519);
2012-04-06, by wenzelm
remove now-unnecessary type annotations from lift_definition commands
2012-04-06, by huffman
more robust generation of quotient rules using tactics
2012-04-06, by huffman
merged
2012-04-06, by huffman
add function dest_Quotient
2012-04-06, by huffman
standardized alias;
2012-04-06, by wenzelm
fixed document;
2012-04-06, by wenzelm
merged
2012-04-06, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip