Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
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.
insist in proper 'document_files';
2014-08-10, by wenzelm
tuned -- avoid confusion with @{assert} for system failures (exception Fail);
2014-08-10, by wenzelm
tuned -- eliminated redundant check (see 1f77110c94ef);
2014-08-10, by wenzelm
merged -- with manual conflict resolution for src/HOL/SMT_Examples/SMT_Examples.certs2, src/HOL/SMT_Examples/SMT_Word_Examples.certs2, src/Doc/Prog_Prove/document/intro-isabelle.tex;
2014-08-10, by wenzelm
updated URL (anticipate merge with 85b8cc142384);
2014-08-10, by wenzelm
Added tag Isabelle2014-RC3 for changeset 91e188508bc9
2014-08-10, by wenzelm
proper layered_pane for JDialog, e.g. relevant for floating dockables in jEdit, for completion popup in text field;
2014-08-10, by wenzelm
follow link to originating command, to ensure that Simplifier_Trace_Dockable displays its results (via current_command);
2014-08-10, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned comments;
2014-08-09, by wenzelm
clarified synchronized scope;
2014-08-09, by wenzelm
tuned comments;
2014-08-09, by wenzelm
application manifest for Windows 8/8.1 dpi scaling;
2014-08-08, by wenzelm
observe context visibility -- less redundant warnings;
2014-08-08, by wenzelm
improved monitor panel;
2014-08-08, by wenzelm
protocol command for heap management, e.g. in Isabelle/jEdit/Scala console: PIDE.session.protocol_command("ML_System.share_common_data");
2014-08-05, by wenzelm
added system option editor_output_delay: lower value might help big sessions under low-memory situations;
2014-08-05, by wenzelm
obsolete (see f7700146678d);
2014-08-05, by wenzelm
tuned proofs -- fewer warnings;
2014-08-05, by wenzelm
clarified Element.init vs. Element.init' -- the latter also avoids redundant warnings due to declatations when preparing locale expressions / interpretations;
2014-08-05, by wenzelm
avoid duplication of warnings stemming from simp/intro declarations etc.;
2014-08-05, by wenzelm
tuned proofs;
2014-08-05, by wenzelm
restrict edit_command (for sendback) to current node -- no attempt to goto target buffer first, which might not be loaded;
2014-08-05, by wenzelm
tuned;
2014-08-05, by wenzelm
more careful treatment of context visibility for rule declarations (see also 39d9c7f175e0, e639d91d9073) -- avoid duplicate warnings;
2014-08-05, by wenzelm
refined context visibility again (amending f5f9fad3321c, 8e3e004f1c31): avoid spurious warning due to global config options;
2014-08-05, by wenzelm
even more thorough reset on mouse drag (see also 0c63f3538639, 7e8c11011fdf);
2014-08-04, by wenzelm
tuned;
2014-08-04, by wenzelm
tuned;
2014-08-04, by wenzelm
Added tag Isabelle2014-RC2 for changeset ee908fccabc2
2014-08-04, by wenzelm
more user aliases;
2014-08-04, by wenzelm
registered Haskabelle-2014
2014-08-04, by noschinl
tuned, so codegen runs with current isabelle again
2014-08-01, by Lars Noschinski
tuned whitespace;
2014-08-03, by wenzelm
more robust popup geometry vs. formatted margin;
2014-08-03, by wenzelm
tuned message;
2014-08-03, by wenzelm
updated URL;
2014-08-02, by wenzelm
tuned;
2014-08-02, by wenzelm
updated URL;
2014-08-02, by wenzelm
more emphatic warning via error_message (violating historic TTY protocol);
2014-08-02, by wenzelm
proper priority for error over warning also for node_status (see 9c5220e05e04);
2014-08-02, by wenzelm
more direct access to persistent blobs (see also 8953d4cc060a), avoiding fragile digest lookup from later version (which might have removed unused blobs already);
2014-08-02, by wenzelm
always resolve symlinks for local files, e.g. relevant for ML_file to load proper source via editor instead of stored file via prover;
2014-08-02, by wenzelm
tuned output;
2014-08-02, by wenzelm
prefer non-strict Execution.print, e.g relevant for redirected ML compiler reports after error (see also e79f76a48449 and 40274e4f5ebf);
2014-08-01, by wenzelm
careful when calling 'Thm.proof_body_of' -- it can throw exceptions
2014-08-01, by blanchet
removed unused stuff;
2014-08-01, by wenzelm
agree on keyword categories with ML;
2014-08-01, by wenzelm
more keyword categories (as in ML);
2014-08-01, by wenzelm
prefer dynamic ML_print_depth if context happens to be available;
2014-07-31, by wenzelm
completion popup supports both ENTER and TAB (default);
2014-07-31, by wenzelm
clarified compile-time use of ML_print_depth;
2014-07-31, by wenzelm
more general notion of "user error" including empty message -- NB: Output.error_message needs non-empty string to emit anything;
2014-07-31, by wenzelm
correctly resolve selector names in default value equations
2014-07-30, by blanchet
update documentation for Lifting/Transfer
2014-07-30, by kuncar
add Isabelle Datatype Manual to the bibliography
2014-07-30, by kuncar
CONTRIBUTORS;
2014-07-30, by wenzelm
NEWS
2014-07-30, by kuncar
better ordering of positive_integral renaming to nn_integral in NEWS
2014-07-29, by hoelzl
made tactic more robust w.r.t. dead variables; tuned;
2014-07-28, by desharna
do not embed 'nat' into 'int's in 'smt2' method -- this is highly inefficient and decreases the Sledgehammer success rate significantly
2014-07-27, by blanchet
some actual workaround to remove document nodes;
2014-07-28, by wenzelm
Added tag Isabelle2014-RC1 for changeset c0fd03d13d28
2014-07-27, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned
2014-08-09, by nipkow
add complete_lattice instances for Enum.finite_* types such that quickcheck deals with lattice class operations
2014-08-08, by Andreas Lochbihler
tuned
2014-08-08, by nipkow
no need for 'set_simps' now that 'datatype_new' generates the desired 'set' property
2014-08-07, by blanchet
generate nicer 'set' theorems for (co)datatypes
2014-08-07, by blanchet
compile
2014-08-07, by blanchet
took out test driver
2014-08-07, by blanchet
make TPTP tools work on polymorphic (TFF1) problems as well
2014-08-07, by blanchet
put comments between TPTP lines to comply with TPTP BNF
2014-08-07, by blanchet
test driver
2014-08-07, by blanchet
treat variables as frees in 'conjecture's
2014-08-07, by blanchet
support TFF1 in TPTP parser/interpreter
2014-08-07, by blanchet
tuning
2014-08-07, by blanchet
tuned
2014-08-07, by traytel
tuned
2014-08-07, by nipkow
tuned
2014-08-07, by nipkow
merged
2014-08-06, by traytel
handle deep nesting in N2M
2014-08-06, by traytel
made tactic more robust
2014-08-06, by traytel
added lemma
2014-08-06, by nipkow
replaced misleading - by _
2014-08-06, by nipkow
more correct clique computation for N2M
2014-08-05, by blanchet
regenerated ML-Lex/Yacc files
2014-08-05, by blanchet
correctly interpret arithmetic types
2014-08-05, by blanchet
added 'datatype_compat' tests
2014-08-05, by blanchet
tuning whitespace
2014-08-05, by blanchet
tuned skolemization
2014-08-05, by blanchet
rationalize Skolem names
2014-08-05, by blanchet
tuning
2014-08-05, by blanchet
tuned code
2014-08-05, by blanchet
don't rename variables which will be renamed later anyway
2014-08-05, by blanchet
normalize skolem argument variable names so that they coincide when taking the conjunction
2014-08-05, by blanchet
tuning
2014-08-05, by blanchet
tuned comments
2014-08-04, by blanchet
deal with E definitions
2014-08-04, by blanchet
updated 'compress' docs
2014-08-04, by blanchet
cleaner 'compress' option
2014-08-04, by blanchet
renamed 'sh_minimize' to 'minimize'; compile;
2014-08-04, by blanchet
restored more sorting
2014-08-04, by blanchet
tuned terminology (cf. 'isar_proofs' option)
2014-08-04, by blanchet
sort facts in minimizer as well
2014-08-04, by blanchet
default on 'metis' for ATPs if preplaying is disabled
2014-08-04, by blanchet
more informative preplay failures
2014-08-04, by blanchet
rationalized sorting of facts -- so that preplaying (almost always) coincides with the real thing, preventing odd failures
2014-08-04, by blanchet
slightly earlier exit from preplaying
2014-08-04, by blanchet
honor 'dont_minimize' option when preplaying one-liner proof
2014-08-04, by blanchet
Metis is being used to emulate E steps;
2014-06-22, by sultana
updated application of print_tac to take context parameter;
2014-06-22, by sultana
better duplicate detection
2014-08-02, by blanchet
normalize conjectures vs. negated conjectures when comparing terms
2014-08-01, by blanchet
tweaked 'clone' formula detection
2014-08-01, by blanchet
fine-tuned Isar reconstruction, esp. boolean simplifications
2014-08-01, by blanchet
centralized boolean simplification so that e.g. LEO-II benefits from it
2014-08-01, by blanchet
careful when compressing 'obtains'
2014-08-01, by blanchet
better handling of variable names
2014-08-01, by blanchet
try to get rid of skolems first
2014-08-01, by blanchet
nicer generated variable names
2014-08-01, by blanchet
tuning
2014-08-01, by blanchet
tuning
2014-08-01, by blanchet
no need to 'obtain' variables not in formula
2014-08-01, by blanchet
more precise handling of LEO-II skolemization
2014-08-01, by blanchet
beware of 'skolem' rules that do not skolemize (e.g. LEO-II)
2014-08-01, by blanchet
tuning
2014-08-01, by blanchet
peek instead of joining -- is perhaps less risky
2014-08-01, by blanchet
export ML function
2014-08-01, by blanchet
compile
2014-08-01, by blanchet
removed 'metisFT' support in Mirabelle
2014-08-01, by blanchet
removed Mirabelle minimization code
2014-08-01, by blanchet
modernized Mirabelle (a bit) and made it compile
2014-08-01, by blanchet
restored a bit of laziness
2014-08-01, by blanchet
reorder quantifiers to ease Z3 skolemization
2014-08-01, by blanchet
tuned order of arguments
2014-08-01, by blanchet
tuned name context code
2014-08-01, by blanchet
tuned whitespace
2014-08-01, by blanchet
more rational unskolemizing of names
2014-08-01, by blanchet
added appropriate method for skolemization of Z3 steps to the mix
2014-08-01, by blanchet
pushing skolems under 'iff' sometimes breaks things further down the proof (as was to be feared)
2014-08-01, by blanchet
honor 'try0' also for one-liners
2014-08-01, by blanchet
tentatively took out 'fastforce' from the set of tried methods -- it seems to be largely subsumed and is hard to silence
2014-08-01, by blanchet
further minimize one-liner
2014-08-01, by blanchet
tuning
2014-08-01, by blanchet
eliminated needlessly complex message tail
2014-08-01, by blanchet
updated NEWS
2014-08-01, by blanchet
update documentation after removal of 'min' subcommand
2014-08-01, by blanchet
eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)
2014-08-01, by blanchet
rationalized preplaying by eliminating (now superfluous) laziness
2014-08-01, by blanchet
removed proof methods as provers from docs
2014-08-01, by blanchet
simplified minimization logic
2014-08-01, by blanchet
tuning
2014-08-01, by blanchet
remove lambda-lifting related assumptions from generated Isar proofs
2014-08-01, by blanchet
whitespace tuning
2014-08-01, by blanchet
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
2014-08-01, by blanchet
generate backquotes without markup, since this confuses preplay; bump up spying version identifier;
2014-08-01, by blanchet
simplified tactics slightly
2014-07-31, by traytel
cascading timeout in parallel evaluation, to rapidly find optimum
2014-07-31, by blanchet
put faster proof methods first
2014-07-30, by blanchet
use parallel preplay machinery also for one-line proofs
2014-07-30, by blanchet
updated docs
2014-07-30, by blanchet
always minimize Sledgehammer results by default
2014-07-30, by blanchet
tuned ML function name
2014-07-30, by blanchet
reduced preplay timeout to 1 s
2014-07-30, by blanchet
added more proof methods for one-liners
2014-07-30, by blanchet
unlift before uncombine, because the definition of a lambda-lifted symbol might have an SK combinator in it (in hybrid encodings)
2014-07-30, by blanchet
Improving robustness and indentation corrections.
2014-07-30, by fleury
Skolemization for tmp_ite_elim rule in the SMT solver veriT.
2014-07-30, by fleury
Changing the role of rule "tmp_ite_elim" of the SMT solver veriT to Lemma.
2014-07-30, by fleury
Whitespace and indentation correction.
2014-07-30, by fleury
Simplifying the labels in the proof of the SMT solver veriT.
2014-07-30, by fleury
Changing ~ into - for unuary minus (not supported by veriT)
2014-07-30, by fleury
imported patch satallax_skolemization_in_tree_part
2014-07-30, by fleury
imported patch hilbert_choice_support
2014-07-30, by fleury
veriT changes for lifted terms, and ite_elim rules.
2014-07-30, by fleury
imported patch satallax_proof_support_Sledgehammer
2014-07-30, by fleury
Basic support for the higher-order ATP Satallax.
2014-07-30, by fleury
Subproofs for the SMT solver veriT.
2014-07-30, by fleury
Basic support for the SMT prover veriT.
2014-07-30, by fleury
removing the '= True' generated by Leo-II.
2014-07-30, by fleury
Skolemization support for leo-II and Zipperposition.
2014-07-30, by fleury
document property 'set_induct'
2014-07-30, by desharna
generate 'set_induct' theorem for codatatypes
2014-07-30, by desharna
also try 'metis' with 'full_types'
2014-07-30, by blanchet
header tuning
2014-07-29, by blanchet
correctly translate THF functions from terms to types
2014-07-28, by blanchet
do not embed 'nat' into 'int's in 'smt2' method -- this is highly inefficient and decreases the Sledgehammer success rate significantly
2014-07-27, by blanchet
back to post-release mode -- after fork point;
2014-07-27, by wenzelm
tuned;
2014-07-27, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
tip