Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-1920
+1920
+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.
generate 'set_cases' theorem for (co)datatypes
2014-08-12, by desharna
document property 'set_intros'
2014-08-12, by desharna
generate 'set_intros' theorem for (co)datatypes
2014-08-12, by desharna
use Goal.prove_sorry instead of Goal.prove where possible (= no schematics in goal and tactic is expected to succeed)
2014-08-11, by traytel
reduced warnings;
2014-08-10, by wenzelm
some localization;
2014-08-10, by wenzelm
support aliases within the facts space;
2014-08-10, by wenzelm
support for named collections of theorems in canonical order;
2014-08-10, by wenzelm
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
tuned;
2014-07-27, by wenzelm
no -optimise -- produces bad bytecode;
2014-07-26, by wenzelm
output state first -- avoid fluctuation wrt. warnings, errors, etc.;
2014-07-26, by wenzelm
tuned comment;
2014-07-25, by wenzelm
updated to polyml-5.5.2-1 which addresses two hard crashes;
2014-07-25, by wenzelm
updated to cygwin-20140725, which is presumably close to Cygwin 1.7.31-1;
2014-07-25, by wenzelm
added more functions and lemmas
2014-07-25, by nipkow
proper mkdir;
2014-07-25, by wenzelm
proper option -O;
2014-07-25, by wenzelm
some reshuffling of Poly/ML version to evade failing tests;
2014-07-25, by wenzelm
old 'defs' is legacy --- slightly odd side-entry that bypasses regular Local_Theory.define interface;
2014-07-25, by wenzelm
proper volume name, such that background image is found in /Volumes/Isabelle/.background;
2014-07-25, by wenzelm
tuned;
2014-07-25, by wenzelm
tuned message;
2014-07-25, by wenzelm
setup for drag-and-drop DMG;
2014-07-25, by wenzelm
merge
2014-07-25, by blanchet
reordered provers
2014-07-25, by blanchet
compile
2014-07-25, by blanchet
faster minimization by not adding facts that are already in the simpset
2014-07-25, by blanchet
added missing facts to proof method
2014-07-25, by blanchet
don't lose 'minimize' flag before it reaches Isar proof text generation
2014-07-25, by blanchet
tuning
2014-07-25, by blanchet
avoid 'eproof' and 'eproof_ram' scripts if possible (i.e. if 'eprover' can produce reasonable enough proofs for one-liner reconstruction)
2014-07-25, by blanchet
compile
2014-07-25, by blanchet
more robustness in Isar proof construction
2014-07-25, by blanchet
tuning
2014-07-25, by blanchet
merged
2014-07-24, by wenzelm
more elementary exception handling: evade hard crash of (Runtime.thread true undefined) on Poly/ML 5.5.1 and 5.5.2;
2014-07-24, by wenzelm
tuned code
2014-07-24, by blanchet
having extra assumptions (typically from a context) means there is no chance to have a valid code equation => skip decoding and registration of the code equations
2014-07-24, by kuncar
store explicitly quotient types with no_code => more precise registration of code equations
2014-07-24, by kuncar
don't needlessly regenerate entire file when the time stamps are equal
2014-07-24, by blanchet
eliminated source of 'DUP's in MaSh
2014-07-24, by blanchet
fixed sorting (broken since 9cc802a8ab06)
2014-07-24, by blanchet
reenabled MaSh for Isabelle2014 release (hopefully)
2014-07-24, by blanchet
beware of duplicate fact names
2014-07-24, by blanchet
refined filter for ATP steps to avoid 'have True' steps in E proofs
2014-07-24, by blanchet
filter out 'theory(...)' from dependencies early on
2014-07-24, by blanchet
introduce fact chaining also under first step
2014-07-24, by blanchet
'shift_quantors' is not an E skolemization rule (cf. 3ab503b04bdb)
2014-07-24, by blanchet
merged
2014-07-24, by wenzelm
proper perl;
2014-07-24, by wenzelm
less warnings -- ignore potential prover startup/shutdown races;
2014-07-24, by wenzelm
tuned spelling;
2014-07-24, by wenzelm
further distinction of Isabelle distribution: alert for identified release candidates;
2014-07-24, by wenzelm
updated to scala-2.11.2;
2014-07-24, by wenzelm
clarified file names;
2014-07-24, by wenzelm
less ambitious isatest, avoid "Exception- InternalError: Backing up too far (32bit) raised while compiling" in polyml-5.4.1;
2014-07-24, by wenzelm
tuned imports;
2014-07-24, by wenzelm
proper scope of comments;
2014-07-24, by wenzelm
make SML/NJ happy;
2014-07-24, by wenzelm
prevent beta-contraction in proving extra assumptions for abs_eq
2014-07-24, by kuncar
more robust notation BNF_Def.convol, which is private to main HOL, but may cause syntax ambiguities nonetheless (e.g. List.thy);
2014-07-24, by wenzelm
reconfirm continuous checking on startup, to address common trap of disabling it accidentally;
2014-07-24, by wenzelm
tuned;
2014-07-24, by wenzelm
less authentic SHA1.digest: trust Scala side on blobs and avoid re-calculation via Foreign Language Interface, which might be a cause of problems;
2014-07-24, by wenzelm
updated NEWS according to d38a98f496dd (see also bdc2c6b40bf2);
2014-07-24, by wenzelm
stick to external proofs when invoking E, because they are more detailed and do not merge steps
2014-07-24, by blanchet
more robust handling of types for skolems (modeled as Frees)
2014-07-24, by blanchet
tuning
2014-07-24, by blanchet
repaired named derivations
2014-07-24, by blanchet
use the noted theorems in 'BNF_Comp'
2014-07-24, by blanchet
use the noted theorem whenever possible, also in 'BNF_Def'
2014-07-24, by blanchet
use termtab instead of (perhaps overly sensitive) thmtab
2014-07-24, by blanchet
use the noted theorem whenever possible, because it has a named derivation (leading to cleaner proof terms)
2014-07-24, by blanchet
tuned message;
2014-07-23, by wenzelm
added action "isabelle.options" (despite problems with initial window size);
2014-07-23, by wenzelm
more official Thy_Info.script_thy;
2014-07-23, by wenzelm
more frugal edits;
2014-07-23, by wenzelm
enable hires explictly, as seen for other high-end Java applications on the Web;
2014-07-23, by wenzelm
more markup;
2014-07-23, by wenzelm
another attempt at more aggressive auto-loading (amending af28fdd50690) -- hidden buffers are now suppressed;
2014-07-23, by wenzelm
more frugal edits;
2014-07-23, by wenzelm
more explicit treatment of cleared nodes (removal is implicit);
2014-07-23, by wenzelm
clarified display;
2014-07-23, by wenzelm
more workarounds for scalac;
2014-07-23, by wenzelm
clarified display;
2014-07-23, by wenzelm
avoid redundant data structure;
2014-07-23, by wenzelm
more explicit discrimination of empty nodes -- suppress from Theories panel;
2014-07-23, by wenzelm
tuned;
2014-07-23, by wenzelm
tuned comments;
2014-07-23, by wenzelm
clarified module name: facilitate alternative GUI frameworks;
2014-07-23, by wenzelm
proper change of perspective for removed nodes (stemming from closed buffers);
2014-07-23, by wenzelm
tuned signature;
2014-07-23, by wenzelm
some robustification of console output;
2014-07-22, by wenzelm
updated ErrorList.jar;
2014-07-22, by wenzelm
discontinued presumable workarounds for extra inter-theory space, which are obsolete since 0e5fa27d3293;
2014-07-22, by wenzelm
evade problems with MikTeX on Windows;
2014-07-22, by wenzelm
tuned messages;
2014-07-22, by wenzelm
support multiple selected print operations instead of slightly odd "menu";
2014-07-22, by wenzelm
more default imports;
2014-07-22, by wenzelm
no keyword completion within word context -- especially avoid its odd visual rendering;
2014-07-22, by wenzelm
merged
2014-07-22, by Andreas Lochbihler
merged
2014-07-21, by Andreas Lochbihler
add parametricity lemmas
2014-07-21, by Andreas Lochbihler
add lemma
2014-07-21, by Andreas Lochbihler
merged
2014-07-21, by wenzelm
refer to Simplifier Trace panel on first invocation;
2014-07-21, by wenzelm
removed unused markup (cf. 2f7d91242b99);
2014-07-21, by wenzelm
regular message to refer to Simplifier Trace panel (unused);
2014-07-21, by wenzelm
proper Swing buttons instead of active areas within text (by Lars Hupel);
2014-07-21, by wenzelm
misc tuning and simplification;
2014-07-21, by wenzelm
clarified "simp_trace_new" and corresponding isar-ref section;
2014-07-21, by wenzelm
more on "Simplifier trace" (by Lars Hupel);
2014-07-21, by wenzelm
always complete explicit symbols;
2014-07-21, by wenzelm
discontinued unfinished attempts at syntactic word context (see 2e1398b484aa, 08a1c860bc12, 7f229b0212fe) -- back to more basic completion of Isabelle2013-2;
2014-07-21, by wenzelm
updated to jdk-7u65;
2014-07-21, by wenzelm
regression test for datatypes defined in IsaFoR
2014-07-21, by traytel
ghc mac installation repaired; test back on.
2014-07-21, by kleing
proper condition wrt. ISABELLE_GHC (cf. 8840fa17e17c);
2014-07-20, by wenzelm
updated to jdk-8u11 (inactive);
2014-07-20, by wenzelm
avoid delay_load overrun;
2014-07-20, by wenzelm
provide explicit options file -- avoid multiple Scala/JVM invocation;
2014-07-20, by wenzelm
check and build Isabelle session for console tool -- avoid multiple Scala/JVM invocation;
2014-07-20, by wenzelm
attempt to run without ISABELLE_GHC setting again on mac-poly
2014-07-19, by kleing
apparently, setting ISABELLE_GHC makes ghc unusable
2014-07-19, by kleing
reverse induction over nonempty lists
2014-07-19, by haftmann
more appropriate postprocessing of rational numbers: extract sign to front of fraction
2014-07-19, by haftmann
doc fixes (contributed by Christian Sternagel)
2014-07-19, by blanchet
made SML/NJ happier
2014-07-19, by blanchet
avoid duplicate fact name
2014-07-18, by kleing
afp-poly runs on macbroy2 (different ghc)
2014-07-18, by kleing
reinstated popular add_ac and mult_ac to avoid needless incompatibilities in user space
2014-07-18, by nipkow
tuned
2014-07-18, by nipkow
register tree with datatype_compat ot support QuickCheck
2014-07-17, by hoelzl
fix bug caused by bad context
2014-07-17, by desharna
add mk_Trueprop_mem utility function
2014-07-17, by desharna
disabled MaSh for the Isabelle2014 release, due to a couple of issues
2014-07-16, by blanchet
refactor commonly used functions
2014-07-16, by desharna
document property 'rel_sel'
2014-07-16, by desharna
generate 'rel_sel' theorem for (co)datatypes
2014-07-16, by desharna
fix rel_cases
2014-07-16, by desharna
made SML/NJ happier
2014-07-15, by blanchet
add ISABELLE_GHC settings for isatest
2014-07-15, by kleing
mira.py: building jEdit plugin is required for makeall
2014-07-14, by noschinl
took out 'rel_cases' for now because of failing tactic
2014-07-15, by blanchet
record MaSh algorithm in spying data
2014-07-15, by blanchet
tuned whitespace (also in strings)
2014-07-15, by blanchet
also learn when 'fact_filter =' is set explicitly
2014-07-15, by blanchet
no warning in case MaSh is disabled
2014-07-15, by blanchet
don't generate a 'set-logic' command when generating problems in a non-standard (but Z3-supported) union-of-everything logic
2014-07-15, by blanchet
no need for 'mash' subdirectory after removal of Python program
2014-07-15, by blanchet
fix typo
2014-07-14, by panny
throw error for bad input
2014-07-14, by panny
catch "not found" case
2014-07-14, by panny
merge
2014-07-12, by blanchet
don't generate TPTP THF 'Definition's, because they complicate reconstruction for AgsyHOL and Satallax
2014-07-12, by blanchet
tuning
2014-07-12, by blanchet
made SML/NJ happier
2014-07-12, by blanchet
reactivate session Quickcheck_Examples
2014-07-11, by Andreas Lochbihler
adapt and reactivate Quickcheck_Types and add two test cases
2014-07-11, by Andreas Lochbihler
more docs
2014-07-11, by blanchet
lambda-lifting for Z3 Isar proofs
2014-07-10, by blanchet
append instead of prepend lambda-lifted definitions -- this eases reconstruction in veriT (outside repository)
2014-07-10, by blanchet
avoid loop in 'all_class_pairs' (caused by e.g. loading the 'Ceta' theory and calling Sledgehammer with the two facts 'fun_of_map.cases' and 'Lattices.bounded_lattice_top_class.sup_top_left' with a polymorphic type encoding)
2014-07-10, by blanchet
merged
2014-07-09, by nipkow
added lemmas
2014-07-09, by nipkow
improved docs
2014-07-09, by blanchet
made SML/NJ happier
2014-07-09, by blanchet
got rid of a pointer equality
2014-07-09, by blanchet
get rid of some pointer equalities
2014-07-09, by blanchet
tuned terminology
2014-07-09, by blanchet
improvements to the machine learning algos (due to Cezary K.)
2014-07-09, by blanchet
added lemma
2014-07-07, by nipkow
refactor some tactics
2014-07-07, by desharna
refactor some tactics
2014-07-07, by desharna
add helper function map_prod
2014-07-07, by desharna
document property 'rel_cases'
2014-07-07, by desharna
generate 'rel_cases' theorem for (co)datatypes
2014-07-07, by desharna
update for release;
2014-07-05, by wenzelm
Added tag Isabelle2014-RC0 for changeset 251ef0202e71
2014-07-05, by wenzelm
merged
2014-07-05, by wenzelm
modernized definitions;
2014-07-05, by wenzelm
proper plain_args to ensure that multi-argument overloading cannot escape pattern restriction (despite more liberal structural containment before 3ae3cc4b1eac);
2014-07-05, by wenzelm
CONTRIBUTORS
2014-07-05, by haftmann
refrain from auxiliary abbreviation: be more explicit to the reader in situations where syntax translation does not apply;
2014-07-05, by haftmann
misc tuning for release;
2014-07-05, by wenzelm
tuned;
2014-07-05, by wenzelm
NEWS
2014-07-05, by haftmann
prefer ac_simps collections over separate name bindings for add and mult
2014-07-05, by haftmann
added Tom's hyp_subst update
2014-07-05, by kleing
reduced name variants for assoc and commute on plus and mult
2014-07-04, by haftmann
tuned;
2014-07-04, by wenzelm
insist in explicit overloading;
2014-07-04, by wenzelm
more uniform names;
2014-07-04, by wenzelm
misc tuning for release;
2014-07-04, by wenzelm
revived unchecked theory (see cebaf814ca6e);
2014-07-04, by wenzelm
suppress completion of obscure keyword;
2014-07-04, by wenzelm
tuned;
2014-07-04, by wenzelm
misc tuning for release;
2014-07-04, by wenzelm
NEWS;
2014-07-04, by wenzelm
Tail recursion no longer supported by "function".
2014-07-03, by nipkow
merged
2014-07-03, by haftmann
weaker assumption for "list_emb_trans"; added lemma
2014-07-03, by Christian Sternagel
added monotonicity lemma for list embedding
2014-07-03, by Christian Sternagel
no built-in reflexivity of list embedding (which is more standard; now embedding is reflexive whenever the base-order is)
2014-07-03, by Christian Sternagel
renamed "list_hembeq" into slightly shorter "list_emb"
2014-07-03, by Christian Sternagel
misc tuning;
2014-07-03, by wenzelm
merge
2014-07-03, by desharna
document property 'rel_intros'
2014-07-03, by desharna
generate 'rel_intros' theorem for (co)datatypes
2014-07-03, by desharna
Hypsubst preserves equality hypotheses
2014-06-11, by Thomas Sewell
tuned grammar and spelling (cf. 0cf15843b82f);
2014-07-02, by wenzelm
document property 'corec_code'
2014-07-02, by desharna
generate 'corec_code' theorem for codatatypes
2014-07-02, by desharna
modernized definitions;
2014-07-02, by wenzelm
misc tuning and clarification;
2014-07-02, by wenzelm
check 'case' variable bindings as for 'fix', which means internal names are rejected as usual;
2014-07-02, by wenzelm
optional exit hook for theory-like targets
2014-07-02, by haftmann
restore exactly named target, prevent non-named targets to participate in the ad-hoc switch game
2014-07-02, by haftmann
centralized (ad-hoc) switching of targets in named_target.ML
2014-07-02, by haftmann
add lemmas: polynomial div/mod distribute over addition
2014-07-01, by huffman
reverted 9512b867259c -- appears to break 'metis'
2014-07-01, by blanchet
clarified "axiomatization" -- minor rewording of this delicate concept;
2014-07-01, by wenzelm
tuned;
2014-07-01, by wenzelm
more on ML options;
2014-07-01, by wenzelm
redundant error position, to ensure the message is attached somewhere, despite the distortion of positions due to glued tokens;
2014-07-01, by wenzelm
overdue NEWS concerning c4daa97ac57a
2014-07-01, by immler
Merge
2014-07-01, by paulson
for new release
2014-07-01, by paulson
merge
2014-07-01, by desharna
document property 'rel_induct'
2014-07-01, by desharna
generate 'rel_induct' theorem for datatypes
2014-07-01, by desharna
fixed soundness bug in monotonicity-based type encodings -- the helper facts must be considered too
2014-07-01, by blanchet
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
2014-07-01, by blanchet
whitespace tuning
2014-07-01, by blanchet
robustness in the face of ill-typed "unchecked" terms (e.g. case expressions)
2014-07-01, by blanchet
use context instead of theory
2014-07-01, by blanchet
fine-tuned methods
2014-07-01, by blanchet
tuned message
2014-07-01, by blanchet
updated docs
2014-07-01, by blanchet
changed default MaSh engine
2014-07-01, by blanchet
removed needless code
2014-07-01, by blanchet
speed up MaSh a bit
2014-07-01, by blanchet
mix NB and kNN
2014-07-01, by blanchet
tuned (reordered) code
2014-07-01, by blanchet
clean up MaSh export a bit
2014-07-01, by blanchet
clean up MaSh evaluation driver
2014-07-01, by blanchet
merged
2014-07-01, by wenzelm
tuned;
2014-07-01, by wenzelm
clarified quasi-generic PIDE;
2014-07-01, by wenzelm
misc updates for release;
2014-07-01, by wenzelm
more release notes;
2014-07-01, by wenzelm
Library/Tree: bst is preferred to be a function
2014-07-01, by hoelzl
Library/Tree: use datatype_new, bst is an inductive predicate
2014-07-01, by hoelzl
more equalities of topological filters; strengthen dependent_nat_choice; tuned a couple of proofs
2014-06-30, by hoelzl
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
2014-06-30, by hoelzl
some lemmas about the indicator function; removed lemma sums_def2
2014-06-30, by hoelzl
generate type correct terms in uncheck phase
2014-07-01, by traytel
updated to sumatra_pdf-2.5.2;
2014-06-30, by wenzelm
ProofGeneral-4.2-2 is optional component (including the traditional helper scripts);
2014-06-30, by wenzelm
removed obsolete Isar system commands -- raw ML console is normally used for system tinkering;
2014-06-30, by wenzelm
tuned comments;
2014-06-30, by wenzelm
updated README;
2014-06-30, by wenzelm
"isabelle tty" is superseded by "isabelle console";
2014-06-30, by wenzelm
tuned description: fit into 80 chars terminal;
2014-06-30, by wenzelm
qualified String.explode and String.implode
2014-06-30, by haftmann
removed non-existing MaSh component from list
2014-06-29, by blanchet
modernized diagnostic options
2014-06-29, by haftmann
use SMT2
2014-06-29, by blanchet
compile
2014-06-29, by blanchet
tuning
2014-06-29, by blanchet
killed Python version of MaSh, now that the SML version works adequately
2014-06-29, by blanchet
tracing facilities for the code generator preprocessor
2014-06-28, by haftmann
tuned interface
2014-06-28, by haftmann
corrected handled exception
2014-06-28, by haftmann
proper trading of variables;
2014-06-28, by haftmann
modernized
2014-06-28, by haftmann
jedit_completion_immediate is enabled by default: let all users participate in slightly more ambitious symbol insertion;
2014-06-28, by wenzelm
removed slightly odd fall-back on complete-word (NB: connection to default menu action is unclear);
2014-06-28, by wenzelm
updated NEWS -- removed material that is already in the manual;
2014-06-28, by wenzelm
merged
2014-06-28, by wenzelm
misc tuning;
2014-06-28, by wenzelm
misc tuning;
2014-06-28, by wenzelm
CONTRIBUTORS
2014-06-28, by haftmann
fact consolidation
2014-06-28, by haftmann
more tight Mailbox: single list is sufficient for single receiver, reverse outside critical section;
2014-06-27, by wenzelm
merged
2014-06-27, by wenzelm
command 'print_term_bindings' supersedes 'print_binds';
2014-06-27, by wenzelm
Proof General legacy;
2014-06-27, by wenzelm
removed obsolete "isabelle unsymbolize";
2014-06-27, by wenzelm
minor renovation of slightly odd and old README;
2014-06-27, by wenzelm
sane environment defaults for Mac OS X, based on former App1/script -- e.g. relevant for MacTeX PATH;
2014-06-27, by wenzelm
tweaking
2014-06-27, by blanchet
correctly take weights into consideration
2014-06-27, by blanchet
tuned whitespace and parentheses
2014-06-27, by blanchet
use right theory name for theorems in evaluation driver
2014-06-27, by blanchet
killed dead code
2014-06-27, by blanchet
reintroduced 'extra features' + only print message in verbose mode
2014-06-27, by blanchet
got rid of hard-coded weights, now that we have TFIDF
2014-06-27, by blanchet
tuning
2014-06-27, by blanchet
tuning
2014-06-27, by blanchet
reintroduced 'extra features' but with lower weight than before (to account for tfidf)
2014-06-27, by blanchet
resolution modulo double negation
2014-06-27, by blanchet
compile
2014-06-27, by blanchet
merged two small theory files
2014-06-27, by blanchet
tuned variable names
2014-06-27, by blanchet
whitespace tuning
2014-06-27, by blanchet
repaired BNF 'size' generation tactic for datatypes mixng old- and new-style datatypes on the right-hand side
2014-06-27, by blanchet
tiny refinements
2014-06-27, by paulson
suppress documentation "how_to_prove_it" for now, notably for release;
2014-06-26, by wenzelm
updated to jdk-7u60 -- back to stable Java 7 for Isabelle2014 release;
2014-06-26, by wenzelm
updated generated file;
2014-06-26, by wenzelm
merged
2014-06-26, by wenzelm
updated cygwin on server;
2014-06-26, by wenzelm
tuning
2014-06-26, by blanchet
reintroduced MaSh hints, this time as persistent creatures
2014-06-26, by blanchet
always expand all paths
2014-06-26, by blanchet
tuned output
2014-06-26, by blanchet
tuned output
2014-06-26, by blanchet
right array indexing
2014-06-26, by blanchet
incremental learning when learing several facts
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
more incremental learning of single fact
2014-06-26, by blanchet
avoid needless (trivial) reordering on load
2014-06-26, by blanchet
recompute learning data at learning time, not query time
2014-06-26, by blanchet
imported patch killed_num_known_facts0
2014-06-26, by blanchet
refactoring
2014-06-26, by blanchet
renamed experimental learning engines
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
refactoring
2014-06-26, by blanchet
removed experimental machine learning engine
2014-06-26, by blanchet
store string-to-index tables in memory
2014-06-26, by blanchet
disable 'extra' feature tainting for now
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
honor visible in SML naive Bayes
2014-06-26, by blanchet
honor visibility in SML k-NN
2014-06-26, by blanchet
got rid of a few experimental options
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
killed dead code
2014-06-26, by blanchet
avoid subscripting array with ~1
2014-06-26, by blanchet
killed dead data
2014-06-26, by blanchet
new version of adaptive k-NN with TFIDF
2014-06-26, by blanchet
refactoring
2014-06-26, by blanchet
tuning
2014-06-26, by blanchet
refactoring
2014-06-26, by blanchet
adaptive k-NN
2014-06-26, by blanchet
avoid parallelism, since it confuses the global state and leads to cheating (with 'sml_xxx' engines)
2014-06-26, by blanchet
generate right dependencies in MaSh driver
2014-06-26, by blanchet
more on "Futures";
2014-06-23, by wenzelm
more on "Futures";
2014-06-23, by wenzelm
more on "Future values";
2014-06-21, by wenzelm
more on "Lazy evaluation";
2014-06-21, by wenzelm
more on syntax phases;
2014-06-20, by wenzelm
more on syntax phases;
2014-06-19, by wenzelm
tuned;
2014-06-19, by wenzelm
tuned;
2014-06-19, by wenzelm
tuned;
2014-06-19, by wenzelm
tuned;
2014-06-19, by wenzelm
tuned;
2014-06-19, by wenzelm
added screenshot;
2014-06-18, by wenzelm
tuned;
2014-06-18, by wenzelm
misc tuning;
2014-06-18, by wenzelm
added screenshot;
2014-06-17, by wenzelm
misc tuning;
2014-06-17, by wenzelm
formal check of jEdit actions;
2014-06-16, by wenzelm
more on "Completion";
2014-06-16, by wenzelm
more on "Completion";
2014-06-16, by wenzelm
tuned;
2014-06-16, by wenzelm
clarified role of old user interfaces as misc tools;
2014-06-16, by wenzelm
added Index;
2014-06-16, by wenzelm
more on "Completion";
2014-06-14, by wenzelm
more on "Completion";
2014-06-13, by wenzelm
tuned;
2014-06-13, by wenzelm
more on "Completion";
2014-06-13, by wenzelm
more on "Completion";
2014-06-12, by wenzelm
more on "Auxiliary files";
2014-06-11, by wenzelm
more on "Document model";
2014-06-11, by wenzelm
suppress index;
2014-06-09, by wenzelm
more on command-line invocation -- moved material from system manual;
2014-06-09, by wenzelm
clarified section structure;
2014-06-09, by wenzelm
clarified section structure;
2014-06-09, by wenzelm
clarified section structure;
2014-06-09, by wenzelm
more on dockable windows;
2014-06-09, by wenzelm
clarified section structure;
2014-06-09, by wenzelm
tuned;
2014-06-06, by wenzelm
more on Query panel;
2014-06-06, by wenzelm
updated screenshots;
2014-06-06, by wenzelm
more on Query panel -- updated Find Theorems;
2014-06-05, by wenzelm
misc tuning and updates;
2014-06-04, by wenzelm
merged
2014-06-25, by Andreas Lochbihler
add lemma
2014-06-24, by Andreas Lochbihler
tuning
2014-06-24, by blanchet
optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
2014-06-24, by blanchet
minor table access optimization
2014-06-24, by blanchet
document property 'rel_coinduct'
2014-06-24, by desharna
tune the implementation of 'rel_coinduct'
2014-06-24, by desharna
generate 'rel_coinduct' theorem for codatatypes
2014-06-24, by desharna
generate 'rel_coinduct0' theorem for codatatypes
2014-06-24, by desharna
added parentheses around type arguments in THF
2014-06-24, by blanchet
optimize log
2014-06-24, by blanchet
enable TF-IDF
2014-06-24, by blanchet
added another experimental engine
2014-06-24, by blanchet
tweaked experimental setup
2014-06-24, by blanchet
changed order of facts so that 'name_tabs' has the same order everywhere (which affects unaliasing)
2014-06-24, by blanchet
use strings to communicate with external process, to ease debugging
2014-06-24, by blanchet
added 'dummy_thf_ml' prover for experiments with HOLyHammer
2014-06-24, by blanchet
phantoms may also occur in THF1
2014-06-24, by blanchet
added experimental MaSh engine
2014-06-24, by blanchet
move method silencing code closer to the methods it is trying to silence, to reduce bad side-effects
2014-06-24, by blanchet
help reconstruction of Z3 skolemization by weakening formulas a bit
2014-06-24, by blanchet
supports gradual skolemization (cf. Z3) by threading context through correctly
2014-06-24, by blanchet
given two one-liners, only show the best of the two
2014-06-24, by blanchet
don't generate Isar proof skeleton for what amounts to a one-line proof
2014-06-24, by blanchet
don't accidentally transform 'show' into 'obtains' (in general, more 'obtain's could be turned into 'have's, but this is not necessary for the correctness of the proof)
2014-06-24, by blanchet
r_into_(r)trancl should not be [simp]: helps little and comlicates some AFP proofs
2014-06-22, by nipkow
added [simp]
2014-06-21, by nipkow
Two basic lemmas on bij_betw.
2014-06-21, by ballarin
changed default MaSh parameters based on (in vitro) evaluation
2014-06-20, by blanchet
made 'tptp_graph' more liberal (why reject TFF?)
2014-06-20, by blanchet
made tactic more robust in the face of 'primcorec' specifications containing 'case_sum'
2014-06-18, by blanchet
more MaSh engine variations, for evaluations
2014-06-18, by blanchet
split parameter into two
2014-06-18, by blanchet
filters are easier to define with INF on filters.
2014-06-18, by hoelzl
moved lemmas from the proof of the Central Limit Theorem by Jeremy Avigad and Luke Serafin
2014-06-18, by hoelzl
more generous formula -- there are lots of duplicates out there
2014-06-18, by blanchet
automatically learn MaSh facts also in 'blocking' mode
2014-06-18, by blanchet
enabled MaSh by default -- set 'MaSh' to 'none' in Isabelle Plugin Options to disable
2014-06-18, by blanchet
Lemmas contributed by Joachim Breitner.
2014-06-17, by ballarin
reintroduce atomize in Waldmeister code
2014-06-17, by blanchet
changed type encoding for new Waldmeister, to trigger filtering of 'dangerous' lemmas
2014-06-17, by blanchet
compile
2014-06-16, by blanchet
integrated new Waldmeister code with 'sledgehammer' command
2014-06-16, by blanchet
fixed parsing of one-argument 'file()' in TSTP files
2014-06-16, by blanchet
use right delimiters for Waldmeister proofs
2014-06-16, by blanchet
added 'waldmeister_new' as ATP
2014-06-16, by blanchet
simplified code
2014-06-16, by blanchet
moved code around
2014-06-16, by blanchet
give Z3 TPTP proofs a chance
2014-06-16, by blanchet
fixed postprocessing of 'coinduct' formula to obtain right property format (without needless hypotheses)
2014-06-16, by blanchet
add more derivative and continuity rules for complex-values functions
2014-06-16, by hoelzl
Moving the remote prefix deleting on Sledgehammer's side
2014-06-16, by fleury
Correcting the type parser
2014-06-16, by fleury
imported patch leo2_skolem_simplication
2014-06-16, by fleury
add support for Isar reconstruction for thf1 ATP provers like Leo-II.
2014-06-16, by fleury
lemmas about the moments of the normal distribution
2014-06-16, by hoelzl
NEWS
2014-06-13, by paulson
properties of normal distributed random variables (by Sudeep Kanav)
2014-06-13, by hoelzl
announce Tree
2014-06-13, by nipkow
new theory of binary trees
2014-06-12, by nipkow
formal variable name: IVar NONE is strictly spoken not supported on lhs of function definitions, e.g. in Scala
2014-06-12, by haftmann
merged
2014-06-12, by nipkow
added [simp]
2014-06-12, by nipkow
tuning
2014-06-12, by blanchet
renamed Sledgehammer options
2014-06-12, by blanchet
removed dead code
2014-06-12, by blanchet
reintroduced vital 'Thm.transfer'
2014-06-12, by blanchet
tuned dependencies
2014-06-12, by blanchet
updated docs
2014-06-12, by blanchet
added support for CVC4 in SMT2
2014-06-12, by blanchet
don't ask proof-disabled solvers to do proofs
2014-06-12, by blanchet
tuning
2014-06-12, by blanchet
took out broken support for Yices from SMT2 stack -- see 'NEWS' for rationale
2014-06-12, by blanchet
made CVC3 work with SMT2 stack
2014-06-12, by blanchet
properties of Erlang and exponentially distributed random variables (by Sudeep Kanav)
2014-06-12, by hoelzl
clean up ContNotDenum; add lemmas by Jeremy Avigad and Luke Serafin
2014-06-11, by hoelzl
uniform treatment of trivial unit instances: simplify by default, unfold in code preprocessor
2014-06-12, by haftmann
adapted examples to changes in SMT triggers
2014-06-12, by blanchet
reduces Sledgehammer dependencies
2014-06-12, by blanchet
eliminate dependency of SMT2 module on 'list'
2014-06-12, by blanchet
tuning
2014-06-12, by blanchet
removed subsumed record-related code, now that records are registered as 'ctr_sugar'
2014-06-12, by blanchet
made lookup more robust in the face of missing (dummy) case constant
2014-06-12, by blanchet
use 'ctr_sugar' abstraction in SMT(2)
2014-06-12, by blanchet
register record extensions as freely generated types
2014-06-12, by blanchet
mixin definitions are within scope of "for"s of import expression
2014-06-11, by haftmann
proper proof context transfer wrt. background theory avoids ad-hoc restore operation
2014-06-11, by haftmann
refactoring
2014-06-11, by blanchet
moved generic code further up
2014-06-11, by blanchet
tuned code
2014-06-11, by blanchet
factor out SMT-LIB 2 type/term parsing from Z3-specific code
2014-06-11, by blanchet
simplify slightly ATP proof generated for Z3
2014-06-11, by blanchet
tuned whitespaces
2014-06-11, by steckerm
updated contributors to include students
2014-06-11, by blanchet
moved new highly experimental Waldmeister-specific code (authored by Albert Steckermeier) into Isabelle
2014-06-11, by blanchet
adapted SMT examples to new, corrected handling of 'typedef'
2014-06-11, by blanchet
fixed unsoundness in SMT(2) as oracle: don't register typedef Abs_x as constructor unless it is known to be injective
2014-06-11, by blanchet
updated NEWS slightly
2014-06-11, by blanchet
updated docs w.r.t. Z3
2014-06-11, by blanchet
rationalized CVC3 and Yices environment variable -- no need (unlike for Z3) to distinguish between old and new versions
2014-06-11, by blanchet
removed '_new' sufffix in SMT2 solver names (in some cases)
2014-06-11, by blanchet
removed old SMT module from Sledgehammer
2014-06-11, by blanchet
got rid of 'listF' example, which is now subsumed by the real 'list' type
2014-06-11, by blanchet
changed syntax of map: and rel: arguments to BNF-based datatypes
2014-06-10, by blanchet
tuning
2014-06-10, by blanchet
updated Z3 certificates
2014-06-10, by blanchet
generate ':named' attributes in SMT-LIB 2 problems, to facilitate reconstruction
2014-06-10, by blanchet
tuning
2014-06-10, by blanchet
add type class instances for unit
2014-06-10, by Andreas Lochbihler
use 'where' clause for selector default value syntax
2014-06-10, by blanchet
tuning
2014-06-10, by blanchet
added List.union
2014-06-09, by nipkow
Sup/Inf on functions decoupled from complete_lattice.
2014-06-09, by nipkow
tuned data structure
2014-06-08, by haftmann
recovered level-free fishing for locale, accidentally lost in dce365931721
2014-06-08, by haftmann
tuned terminology: emphasize stack-like nature of nested local theories
2014-06-08, by haftmann
self-contained locale_declaration operation
2014-06-08, by haftmann
yet another attempt for terminology: foo_target_bar denotes an operation bar operating solely on the target context of target foo, foo_bar denotes a whole stack of operations to accomplish bar for target foo
2014-06-08, by haftmann
tuned
2014-06-08, by haftmann
recovered structure of module, which got somehow convoluted due to incremental modifications
2014-06-08, by haftmann
re-unified approach towards class and locale consts, with refined terminology: foo_const_declaration denotes declaration for a particular logical layer, foo_const the full stack for a particular target
2014-06-08, by haftmann
revert effect of 63c7b29d29ac -- existing pervasive interpretation of class order for dvd etc. is too obstrusive at the moment
2014-06-08, by haftmann
less ad-hoc verision of educated guess: guess identity of declaration morphism wrt. canonical morphism rather than observing particular effects of declaration morphisms only;
2014-06-08, by haftmann
treat non-canonical interpretations of classes the same way as ordinary locale interpretations
2014-06-07, by haftmann
tuned
2014-06-07, by haftmann
avoid odd Named_Target.reinit altogether
2014-06-07, by haftmann
clarified terminology: toplevel is interwined with named targets in particular, not with local theories in general
2014-06-07, by haftmann
less baroque interface
2014-06-07, by haftmann
dropped obscure and unused ad-hoc before_exit hook for named targets
2014-06-06, by haftmann
added lemma
2014-06-06, by nipkow
mira: USER_HOME must exist for building JEdit documentation
2014-06-05, by noschinl
added lemmas
2014-06-06, by nipkow
sharpened criterion: bare named target is only at the bottom level
2014-06-05, by haftmann
tuned
2014-06-05, by haftmann
extended stream library
2014-06-05, by traytel
be more explicit: made sml/nj happy
2014-06-05, by haftmann
always refine interpretation morphism using canonical constant's definition theorem
2014-06-05, by haftmann
set USER_HOME to affect also ISABELLE_PATH et al
2014-06-04, by noschinl
merge
2014-06-03, by blanchet
updated SMT2 certificates
2014-06-03, by blanchet
tune
2014-06-03, by blanchet
disable hard-to-reconstruct Z3 feature
2014-06-03, by blanchet
new Z3 4.3.2 component, based on more recent repository version, and whose Mac binary was built on Mac OS X 10.7
2014-06-03, by blanchet
use 0 as integral-value for non-integrable functions, simplify a couple of rewrite rules
2014-06-03, by hoelzl
removed SMT weights -- their impact was very inconclusive anyway
2014-06-03, by blanchet
make SMT code less dependent on Z3 proofs
2014-06-03, by blanchet
tuning
2014-06-03, by blanchet
avoid division by 0
2014-06-02, by blanchet
formal treatment of dangling parameters for class abbrevs analogously to class consts
2014-06-02, by haftmann
explicit passing of params
2014-06-02, by haftmann
refactored Z3 to Isar proof construction code
2014-06-02, by blanchet
simplified counterexample handling
2014-06-02, by blanchet
split replay and proof parsing for Z3
2014-06-02, by blanchet
removed counterexample parser (obsolete and useless in practice)
2014-06-02, by blanchet
remove superfluous assumption
2014-06-02, by hoelzl
basic setup for zipperposition prover
2014-06-02, by fleury
document property 'sel_set'
2014-06-02, by desharna
generate 'sel_set' theorem for (co)datatypes
2014-06-02, by desharna
removed some spurious warnings in new (co)datatype package
2014-06-02, by blanchet
add option to keep duplicates, for more precise evaluation of relevance filters
2014-06-02, by blanchet
tuned whitespace
2014-06-02, by blanchet
definition in class: provide explicit auxiliary abbreviation carrying potential mixfix syntax in presence of dangling parameters
2014-06-01, by haftmann
tuned
2014-06-01, by haftmann
merged
2014-05-31, by boehmes
tuned
2014-05-31, by boehmes
more complete proof replay for Z3: support universally quantified rewrite steps
2014-05-31, by boehmes
postpone const declarations for nested context after canonical const declarations: keep const declarations stemming from interpretation together
2014-05-31, by haftmann
tuned
2014-05-31, by haftmann
explicit is better than implicit
2014-05-31, by haftmann
tuned names
2014-05-31, by haftmann
dropped accidental duplicate application of morphism
2014-05-31, by haftmann
generalizd measurability on restricted space; rule for integrability on compact sets
2014-05-30, by hoelzl
better support for restrict_space
2014-05-30, by hoelzl
must not cancel common factors on both sides of (in)equations in linear arithmetic decicision procedure
2014-05-30, by nipkow
merged
2014-05-30, by wenzelm
updated cygwin -- include perl_vendor for libwww-perl;
2014-05-30, by wenzelm
made 'Kuehlwein-style' be really like Python code, we now think
2014-05-30, by blanchet
make SML code closer to Python code when 'nb_kuehlwein_style' is true
2014-05-30, by blanchet
merge
2014-05-30, by blanchet
added sleep to give time for the server to shut down -- this is a hack, but it's only in experimental code that will hopefully soon go away
2014-05-30, by blanchet
introduce more powerful reindexing rules for big operators
2014-05-30, by hoelzl
merged
2014-05-30, by wenzelm
make double-sure that old popup is dismissed, before replacing it;
2014-05-30, by wenzelm
more robust bold_style, e.g. relevant for accidental \<^bold> before keyword;
2014-05-30, by wenzelm
added another way of invoking Python code, for experiments
2014-05-30, by blanchet
make SML naive Bayes closer to Python version
2014-05-30, by blanchet
tuned whitespace, to make datatype definitions slightly less intimidating
2014-05-30, by blanchet
more work on exporter
2014-05-30, by blanchet
got rid of 'linearize' option
2014-05-30, by blanchet
extend exporter with new versions of MaSh
2014-05-30, by blanchet
tuned
2014-05-30, by haftmann
tuned signature
2014-05-30, by haftmann
terminating code equations
2014-05-30, by haftmann
more direct passing of right-hand side
2014-05-29, by haftmann
even more uniform treatment of result after 95e5a633a18f
2014-05-29, by haftmann
Merge
2014-05-29, by paulson
New theorems to enable the simplification of certain functions when applied to specific natural number constants (such as 4)
2014-05-29, by paulson
removed Kleene_Algebra because of superior AFP entry; authors agreed
2014-05-29, by nipkow
typo
2014-05-29, by nipkow
uniform treatmen of result
2014-05-28, by haftmann
tuned variable names
2014-05-28, by haftmann
more generous max number of suggestions, for more safety
2014-05-28, by blanchet
changed MaSh to use SML version instead of Python version of naive Bayes by default (i.e. if MASH=yes in the settings, or 'fact_filter=mash' with no other explicit setting)
2014-05-28, by blanchet
export more ML functions, for experimentation
2014-05-28, by blanchet
tuned signature;
2014-05-28, by wenzelm
disabled IDF for now -- empirical evidence points the wrong way (as usual)
2014-05-28, by blanchet
tuning
2014-05-28, by blanchet
tuning
2014-05-28, by blanchet
optimized computation
2014-05-28, by blanchet
enabled IDF for naive Bayes ML
2014-05-28, by blanchet
tuning
2014-05-28, by blanchet
repaired subscript problem in SML kNN
2014-05-28, by blanchet
tuning
2014-05-28, by blanchet
always remove duplicates in meshing + use weights for Naive Bayes
2014-05-28, by blanchet
updated naive Bayes
2014-05-27, by blanchet
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
2014-05-27, by blanchet
don't conceal (co)datatypes
2014-05-26, by blanchet
changed '-:' to 'dead' in BNF
2014-05-26, by blanchet
got rid of '=:' squiggly
2014-05-26, by blanchet
use '%x. x = C' as default discriminator for nullary constructor C, instead of relying on odd '=:' syntax
2014-05-26, by blanchet
renamed 'MaSh' option
2014-05-26, by blanchet
document '=:' syntax better
2014-05-26, by blanchet
capitalize even more carefully (see 5ac67041ccf8), e.g. relevant for option "z3_non_commercial" and prospective "MaSh";
2014-05-26, by wenzelm
tuned;
2014-05-25, by wenzelm
clarified copy_file: allow to rename base name, e.g. relevant for 'display_drafts';
2014-05-24, by wenzelm
support for regular Windows TeX installation;
2014-05-24, by wenzelm
more portable file names;
2014-05-24, by wenzelm
more portable -- accomodate MiKTeX on Windows;
2014-05-24, by wenzelm
receovered alternative abbrevs for \<open> \<close> from 8e8243975860, to accommodate national keyboard layouts where "`" might be hard to produce;
2014-05-24, by wenzelm
strip trailing white space, to avoid notorious problems of jEdit with last line;
2014-05-24, by wenzelm
added fifth member to BNF team
2014-05-23, by blanchet
removed noise
2014-05-23, by blanchet
fixed semantics of 'linearize'
2014-05-23, by blanchet
automatically reload state file when it changes on disk
2014-05-23, by blanchet
tuned
2014-05-22, by haftmann
tuned names
2014-05-22, by haftmann
tuned signature
2014-05-22, by haftmann
moved const declaration further down in bootstrap hierarchy: keep Named_Target free of low-level stuff
2014-05-22, by haftmann
unused
2014-05-22, by haftmann
tuned
2014-05-22, by haftmann
more uniform order of operations;
2014-05-22, by haftmann
common background_abbrev operation
2014-05-22, by haftmann
tuned signature
2014-05-22, by haftmann
tuned: prefer separate function trails for locales and classes rather than ad-hoc case distinction
2014-05-22, by haftmann
compactified
2014-05-22, by haftmann
include Nominal2 keywords -- Proof General legacy;
2014-05-22, by wenzelm
another attempt to revive isatest -- reverting 801c01004a21;
2014-05-22, by wenzelm
avoid slow inspection of proof terms now that dependencies are stored in 'state'
2014-05-22, by blanchet
properly mark relearns as dirty
2014-05-22, by blanchet
disable weights that cause more harm than they help in kNN
2014-05-22, by blanchet
add self dependency to naive Bayes
2014-05-22, by blanchet
make MaSh Python the default when passing 'fact_filter = mash' without enabling the 'maSh' Isabelle system option
2014-05-22, by blanchet
compactified level discriminator
2014-05-22, by haftmann
properly reconstruct helpers in Z3 proofs
2014-05-22, by blanchet
reverted '|' features in MaSh -- these sounded like a good idea but never really worked
2014-05-22, by blanchet
tuning
2014-05-22, by blanchet
shorten Sledgehammer output, as suggested by Andrei Popescu
2014-05-22, by blanchet
until naive Bayes supports weights, don't incorporate 'extra' low-weight features
2014-05-22, by blanchet
spell-checker completion is restricted to explicit mode, to avoid odd effects with immediate edits vs. delayed language context markup, and occasional delays due to dictionary lookup of many variants;
2014-05-21, by wenzelm
merged
2014-05-21, by wenzelm
updated to scala-2.11.1, with full uncensored classpath;
2014-05-21, by wenzelm
updated cygwin more thoroughly;
2014-05-21, by wenzelm
document property 'sel_map'
2014-05-21, by desharna
generate 'sel_map[simp]' theorem for (co)datatypes and tuning 'disc_map_iff'
2014-05-21, by desharna
merged
2014-05-21, by wenzelm
more uniform Font_Info.Zoom_Box;
2014-05-21, by wenzelm
added zoom box, like for outer output windows;
2014-05-21, by wenzelm
tuned signature;
2014-05-21, by wenzelm
consolidate "break_thm" and "break_term" attributes into "simp_break";
2014-05-21, by Lars Hupel
docs
2014-05-21, by blanchet
added comment
2014-05-21, by blanchet
move exhaust first, for technical reasons
2014-05-21, by blanchet
avoid markup-generating @{make_string}
2014-05-21, by blanchet
generalized Bochner integral over infinite sums
2014-05-21, by hoelzl
unused;
2014-05-21, by wenzelm
obsolete;
2014-05-21, by wenzelm
approximative update of versions;
2014-05-21, by wenzelm
incorporate isabelle.graphview into Pure.jar, which saves 20..30s build time;
2014-05-21, by wenzelm
remove stray println;
2014-05-21, by Lars Hupel
CONTRIBUTORS
2014-05-20, by blanchet
added naive Bayes ML implementation, due to Cezary Kaliszyk (like k-NN)
2014-05-20, by blanchet
added Isabelle system option 'mash'
2014-05-20, by blanchet
updated cygwin;
2014-05-20, by wenzelm
afford strict check (see also AFP/a8e08d947f0a);
2014-05-20, by wenzelm
add various lemmas
2014-05-20, by hoelzl
merged
2014-05-20, by wenzelm
merged
2014-05-20, by wenzelm
adhoc move to lxbroy10, which has 120 GB more memory than lxbroy2;
2014-05-20, by wenzelm
explicit treatment of unfinished cartouches, which is important for Thy_Syntax.consolidate_spans;
2014-05-20, by wenzelm
news
2014-05-20, by blanchet
updated docs
2014-05-20, by blanchet
more flexible environment variable
2014-05-20, by blanchet
tuning
2014-05-20, by blanchet
added unit :: linorder
2014-05-20, by nipkow
added lemma
2014-05-20, by nipkow
implemented MaSh/SML hints
2014-05-20, by blanchet
better way to take invisible facts into account than 'island' business
2014-05-20, by blanchet
cleaner handling of learned proofs
2014-05-20, by blanchet
implemented learning of single proofs in SML MaSh
2014-05-20, by blanchet
take weights into consideration in knn
2014-05-19, by blanchet
added SML implementation of MaSh
2014-05-19, by blanchet
use E 1.8's auto scheduler option
2014-05-19, by blanchet
started work on MaSh/SML
2014-05-19, by blanchet
tune
2014-05-19, by blanchet
store all MaSh data on the Isabelle side, in preparation for replacing 'mash.py' with ML solution
2014-05-19, by blanchet
trace windows uses search feature of Pretty_Text_Area;
2014-05-19, by Lars Hupel
obsolete -- always pdf;
2014-05-19, by wenzelm
prefer T1 with searchable underscore (requires proper cm-super fonts);
2014-05-19, by wenzelm
merged
2014-05-19, by wenzelm
some adhoc event handling to unify L&F button focus behavior, e.g. Mac OS X vs. Nimbus;
2014-05-19, by wenzelm
re-focus target explicity, e.g. relevant for Sledgehammer panel;
2014-05-19, by wenzelm
clarified is_text in accordance to ML version (7e0178c84994), e.g. relevant for 'header' syntax in PIDE front-end;
2014-05-19, by wenzelm
more explicit identification for more robust adhoc change of environment /home/isatest/.isabelle/etc/settings -- notably for $ISABELLE_PLATFORM64;
2014-05-19, by wenzelm
renamed positive_integral to nn_integral
2014-05-19, by hoelzl
hide more consts to beautify documentation
2014-05-19, by blanchet
fixed document generation for HOL-Probability
2014-05-19, by hoelzl
introduce Bochner integral: generalizes Lebesgue integral from real-valued function to functions on real-normed vector spaces
2014-05-19, by hoelzl
document property 'disc_map_iff'
2014-05-19, by desharna
generate 'disc_map_iff[simp]' theorem for (co)datatypes
2014-05-15, by desharna
fix 'set_empty' theorem when the discriminator is 'op ='
2014-05-19, by desharna
typos
2014-05-18, by nipkow
tuned comments;
2014-05-18, by wenzelm
clarified dependencies -- Mavericks presently does not work;
2014-05-18, by wenzelm
clarified docking layout, amending 9c2ca698690e;
2014-05-18, by wenzelm
correctly add extra facts to lemmas (cf. conjecture and hypotheses) in Z3 Isar proofs
2014-05-16, by blanchet
removed needless transfer
2014-05-16, by blanchet
use 'simp add:' syntax in Sledgehammer rather than 'using'
2014-05-16, by blanchet
silence methods even better
2014-05-16, by blanchet
honor original format of conjecture or hypotheses in Z3-to-Isar proofs
2014-05-16, by blanchet
proper priority for error over warning, which got mixed up in 0546e036d1c0 and 4df2727a0b5f;
2014-05-16, by wenzelm
added lemmas for -1
2014-05-16, by noschinl
proper handling of 'ctor_dtor' for mutual corecursive cases where not all type variables are present in all low-level constructors (cf. 'coind_wit1' etc. in 'Misc_Codatatypes.thy')
2014-05-16, by blanchet
new syntax for card, normalized spacing for #
2014-05-16, by nipkow
clarified stylized status of sandwich algebra
2014-05-15, by haftmann
dropped dead code
2014-05-15, by haftmann
accurate separation of static and dynamic context
2014-05-15, by haftmann
syntactic means to prevent accidental mixup of static and dynamic context
2014-05-15, by haftmann
proper separation of static and dynamic context
2014-05-15, by haftmann
optimization for trivial cases
2014-05-15, by haftmann
modernized setup
2014-05-15, by haftmann
dropped obsolete hand-waving adjustion of type variables: safely done in preprocessor
2014-05-15, by haftmann
unified approach toward conversions and simple term rewriting in preprocessor by means of sandwiches
2014-05-15, by haftmann
normalize type variables of evaluation term by conversion
2014-05-15, by haftmann
more aggressive nested size handling in the absence of 'size_o_map' theorems (+ unrelated pattern matching fix)
2014-05-15, by blanchet
new approach to silence proof methods, to avoid weird theory/context mismatches
2014-05-15, by blanchet
type
2014-05-15, by haftmann
merged
2014-05-14, by wenzelm
restrict default docking layout to bare minimum -- NB: Simplifier Trace still needs fine-tuning to show up on demand;
2014-05-14, by wenzelm
updated isatest;
2014-05-14, by wenzelm
updated to polyml-5.5.2;
2014-05-14, by wenzelm
practically obsolete: plain "poly" should work, except for Linux without libgmp installed;
2014-05-14, by wenzelm
updated to polyml-5.5.2;
2014-05-14, by wenzelm
document 'set_empty'
2014-05-14, by desharna
generate 'set_empty' theorem for BNFs
2014-05-12, by desharna
document 'map_id0'
2014-05-08, by desharna
note map_id0 more often
2014-05-08, by desharna
added lemma
2014-05-14, by nipkow
added lemmas
2014-05-13, by nipkow
transfer theorems since 'silence_methods' may change the theory
2014-05-13, by blanchet
add mono rules for diff
2014-05-13, by hoelzl
clean up Lebesgue integration
2014-05-13, by hoelzl
more bnf_decl -> bnf_axiomatization
2014-05-13, by blanchet
tuned docs
2014-05-13, by blanchet
hide more internal names
2014-05-13, by blanchet
tuning
2014-05-13, by blanchet
no reset for 'end' -- e.g. relevant for 'notepad';
2014-05-13, by wenzelm
updated keywords
2014-05-13, by traytel
bnf_decl -> bnf_axiomatization
2014-05-13, by traytel
tuned signature to make axiomatizations more easy to spot in the source, via "add_axioms" or "axiomatization";
2014-05-12, by wenzelm
Replaced refute with nitpick.
2014-05-12, by webertj
NEWS;
2014-05-12, by wenzelm
tuned message;
2014-05-12, by wenzelm
smarter recovery from toplevel type error;
2014-05-12, by wenzelm
more direct patch of public interface DockableWindowContainer -- avoid package org.gjt.sp.jedit.gui intrusion;
2014-05-11, by wenzelm
updated keywords;
2014-05-09, by wenzelm
merged
2014-05-09, by wenzelm
more markup;
2014-05-09, by wenzelm
more position markup to help locating the query context, e.g. from "Info" dockable;
2014-05-09, by wenzelm
always bounce focus back to main text area, unless explicit focus component is given here (see also 7b65f4da136d);
2014-05-09, by wenzelm
tuned signature;
2014-05-09, by wenzelm
delete attribute for code abbrev
2014-05-09, by haftmann
dropped term_of obfuscation -- not really required;
2014-05-09, by haftmann
hardcoded nbe and sml into value command
2014-05-09, by haftmann
modernized setups
2014-05-09, by haftmann
degeneralized value command into HOL
2014-05-09, by haftmann
dimiss simplified as evaluator due to little practical relevance
2014-05-09, by haftmann
prefer separate command for approximation
2014-05-09, by haftmann
removed junk from library theory
2014-05-09, by haftmann
note of_class rule for type classes in theory: useful to promote class instance proofs to locale interpretation proofs
2014-05-09, by haftmann
normalizing of type variables before evaluation with explicit resubstitution function: make nbe work with funny type variables like \<AA>;
2014-05-09, by haftmann
tuned GUI;
2014-05-08, by wenzelm
clarified detach_operation: ignore empty output;
2014-05-08, by wenzelm
bounce focus back to main text area -- Output is for output, not query input;
2014-05-08, by wenzelm
update for release;
2014-05-08, by wenzelm
merged
2014-05-08, by wenzelm
tuned message;
2014-05-08, by wenzelm
no qualifier for now, to avoid confusion concerning loaded_theories in PIDE interaction;
2014-05-08, by wenzelm
some position markup to help locating the query context, e.g. from "Info" dockable;
2014-05-08, by wenzelm
tuned GUI;
2014-05-08, by wenzelm
tuned GUI;
2014-05-08, by wenzelm
tuned GUI;
2014-05-08, by wenzelm
tuned message: more compact, imitate actual command line;
2014-05-08, by wenzelm
enable "PIDE" docking framework by default, and rely on its "Detach" menu item;
2014-05-08, by wenzelm
some odd tricks to provide "Detach" menu item, via "PIDE" docking framework;
2014-05-08, by wenzelm
untyped, unscoped, unchecked access to JVM objects;
2014-05-08, by wenzelm
Documented new property
2014-05-08, by desharna
generate 'map_ident' theorem for BNFs
2014-05-08, by desharna
explicit option to build library, which takes most of the time;
2014-05-07, by wenzelm
NEWS;
2014-05-07, by wenzelm
merged
2014-05-07, by wenzelm
more symbols;
2014-05-07, by wenzelm
tuned message: "step" goes back to TTY mode before Proof General, while "depth" is more informative but sometimes confusing due to implementation details;
2014-05-07, by wenzelm
print results as "state", to avoid intrusion into the source text;
2014-05-07, by wenzelm
run commands as interactive, again after long history of fluctuation (9e196062bf88, 173974e07dea, e07dacec79e7) and quite different infrastructure for print tasks;
2014-05-07, by wenzelm
discontinued Toplevel.print flag -- print uniformly according to Keyword.is_printed;
2014-05-07, by wenzelm
more emphatic output for Proof General;
2014-05-07, by wenzelm
tuned;
2014-05-07, by wenzelm
tuned defaults;
2014-05-07, by wenzelm
tuned message -- more context for detached window etc.;
2014-05-07, by wenzelm
tuned signature;
2014-05-07, by wenzelm
avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.
2014-05-07, by hoelzl
tuned GUI for Windows L&F;
2014-05-06, by wenzelm
clarified print_state, which goes back to TTY loop before Proof General, and before separate print_context;
2014-05-06, by wenzelm
tuned GUI layout;
2014-05-06, by wenzelm
clarified GUI events, e.g. relevant for insert via completion;
2014-05-06, by wenzelm
more robust line_range, according to usual jEdit confusion at end of last line (see also 71c5d1f516c0);
2014-05-06, by wenzelm
common support for search field, which is actually a light-weight Highlighter;
2014-05-06, by wenzelm
clarified GUI focus;
2014-05-06, by wenzelm
more uniform detach button;
2014-05-06, by wenzelm
tuned signature;
2014-05-06, by wenzelm
renamed "Find" to "Query", with more general operations;
2014-05-06, by wenzelm
hardwired default_frequency to avoid fluctuation of popup content;
2014-05-06, by wenzelm
more visual feedback on path_completion, at the risk of file-system access in GUI painting;
2014-05-06, by wenzelm
tuned;
2014-05-06, by wenzelm
explicit option parallel_print to downgrade parallel scheduling, which might occasionally help for big and heavy "scripts";
2014-05-06, by wenzelm
tuned GUI layout;
2014-05-06, by wenzelm
tuned;
2014-05-06, by wenzelm
some complication with ListView.Renderer to get tooltips;
2014-05-05, by wenzelm
expose interrupts more like ML version, but not in managed bash processes of Build;
2014-05-05, by wenzelm
merged
2014-05-05, by wenzelm
uniform Toplevel.print for all proof commands;
2014-05-05, by wenzelm
clarified print operations for "terms" and "theorems";
2014-05-05, by wenzelm
more print operations;
2014-05-05, by wenzelm
tuned GUI;
2014-05-05, by wenzelm
more decisive change of focus;
2014-05-05, by wenzelm
support print operations as asynchronous query;
2014-05-05, by wenzelm
allow empty original, e.g. path "";
2014-05-05, by wenzelm
more robust process kill -- postpone interrupts on current thread;
2014-05-05, by wenzelm
tuned signature;
2014-05-05, by wenzelm
tuned signature;
2014-05-05, by wenzelm
tuned comment
2014-05-05, by blanchet
simplify selectors in code views
2014-05-05, by blanchet
note correct induction schemes in 'primrec' (for N2M)
2014-05-05, by blanchet
use right meson tactic for preplaying
2014-05-04, by blanchet
simplify unused universally quantified variables in Z3 proofs
2014-05-04, by blanchet
fixed Waldmeister endgame w.r.t. "Trueprop"
2014-05-04, by blanchet
tuned structure name
2014-05-04, by blanchet
added 'satx' to Sledgehammer's portfolio (cf. 'isar_try0')
2014-05-04, by blanchet
renamed 'dpll_p' to 'cdclite', to avoid confusion with the old 'dpll' and to reflect the idea that the new prover implements some ideas from CDCL not in DPLL -- this follows its author's, Sascha B.'s, wish
2014-05-04, by blanchet
added 'satx' proof method to Try0
2014-05-04, by blanchet
make 'dpll_p' the default SAT solver, rather than the hard-to-get zChaff-with-proofs
2014-05-04, by blanchet
added missing space between command-line options
2014-05-04, by blanchet
improved whitelist (cf. be1874de8344)
2014-05-04, by blanchet
renamed 'xxx_size' to 'size_xxx' for old datatype package
2014-05-04, by blanchet
removed obsolete internal SAT solvers
2014-05-04, by boehmes
standardize to implode_short form;
2014-05-03, by wenzelm
support for path completion based on file-system content;
2014-05-03, by wenzelm
yet another completion option, to imitate old less ambitious behavior;
2014-05-03, by wenzelm
reduced cluttering of popups;
2014-05-03, by wenzelm
propagate more events, notably after hide_popup (e.g. LEFT, RIGHT);
2014-05-03, by wenzelm
merged
2014-05-02, by wenzelm
NEWS;
2014-05-02, by wenzelm
more robust interrupt handling for Scala_Console, which uses JVM Thread.interrupt instead of POSIX SIGINT;
2014-05-02, by wenzelm
more sensible interrupt of interpreter, when the user pushes Cancel button;
2014-05-02, by wenzelm
obsolete in scala-2.11.0;
2014-05-02, by wenzelm
fork Scala interpreter thread, independently of Swing_Thread;
2014-05-02, by wenzelm
clarified synchronization and exception handling;
2014-05-02, by wenzelm
more redirection;
2014-05-02, by wenzelm
prefer scala.Console with its support for thread-local redirection;
2014-05-02, by wenzelm
tuned signature -- channels for diagnostic output for system tools means stderr;
2014-05-02, by wenzelm
proper tool wrap-up;
2014-05-02, by wenzelm
tuned spelling;
2014-05-02, by wenzelm
avoid deprecated Scala syntax;
2014-05-02, by wenzelm
enforce case of identifiers only to accomodate strict language requirements (or clear separation of constructors from variables in the case of SML)
2014-05-02, by haftmann
more standard doc session specification;
2014-05-02, by wenzelm
discontinued adhoc check (see also ea8343187225);
2014-05-02, by wenzelm
more frugal access to theory text via Reader, reduced costs for I/O text decoding;
2014-05-02, by wenzelm
support URLs as well;
2014-05-02, by wenzelm
reclaimed Byte_Reader from 51560e392e1b;
2014-05-02, by wenzelm
new documentation: How to Prove it
2014-05-02, by nipkow
disable bad Z3 proof
2014-05-01, by boehmes
use SMT2 for Boogie examples
2014-05-01, by boehmes
less verbose SAT tactic
2014-05-01, by boehmes
use internal proof-producing SAT solver for more efficient SMT proof replay
2014-05-01, by boehmes
added internal proof-producing SAT solver
2014-05-01, by boehmes
tuned output;
2014-05-01, by wenzelm
separate ML module
2014-05-01, by haftmann
centralized upper/lowercase name mangling
2014-05-01, by haftmann
optional case enforcement
2014-05-01, by haftmann
obsolete: no symbol identifiers remaining in Pure
2014-05-01, by haftmann
prevent subscription in nested contexts explicitly -- at foundational and user level
2014-05-01, by haftmann
cleanup
2014-05-01, by haftmann
NEWS
2014-05-01, by haftmann
use qualified name (was interpreted as a catch-all variable name)
2014-05-01, by panny
add additional check to avoid selector formula right-hand side consisting of a nullary constructor getting interpreted as a discriminator formula
2014-05-01, by panny
updated keywords;
2014-05-01, by wenzelm
clarified signature: load_file is still required internally;
2014-04-30, by wenzelm
merged
2014-04-30, by wenzelm
some support for session-qualified theories: allow to refer to resources via qualified name instead of odd file-system path;
2014-04-30, by wenzelm
support for long names in Scala;
2014-04-30, by wenzelm
tuned;
2014-04-30, by wenzelm
Discontinued old spark_open; spark_open_siv is now spark_open
2014-04-30, by berghofe
suppress slightly odd completions of "real";
2014-04-29, by wenzelm
tuned proofs;
2014-04-29, by wenzelm
tuned proofs;
2014-04-29, by wenzelm
clarified exit sequence: prover is reset afterwards, no more output messages;
2014-04-29, by wenzelm
more synchronized treatment of prover process, which might emit more messages before shutdown and requires manager to accept them;
2014-04-29, by wenzelm
tuned;
2014-04-29, by wenzelm
some sanity checks for Isabelle sources;
2014-04-29, by wenzelm
prefer plain ASCII / latex over not-so-universal Unicode;
2014-04-29, by wenzelm
tuned whitespace;
2014-04-29, by wenzelm
proper Unix line termination;
2014-04-29, by wenzelm
require explicit 'document_files';
2014-04-29, by wenzelm
updated mkroot;
2014-04-29, by wenzelm
basic support for Mercurial command line tools;
2014-04-29, by wenzelm
clarified;
2014-04-29, by wenzelm
ignore malformed file names outright, e.g. .class files with dollar;
2014-04-29, by wenzelm
more systematic Isabelle output, like in classic Isabelle/ML (without markup);
2014-04-29, by wenzelm
systematic replacement of 'files' by 'document_files';
2014-04-29, by wenzelm
tuned signature -- accomodate operations of ROOT files;
2014-04-29, by wenzelm
tuned -- prefer Isabelle/Scala operations;
2014-04-29, by wenzelm
tuned proofs;
2014-04-28, by wenzelm
tuned;
2014-04-28, by wenzelm
tuned proofs;
2014-04-28, by wenzelm
improved syslog performance -- avoid denial-of-service e.g. with threads_trace = 5 and active Syslog dockable;
2014-04-28, by wenzelm
tuned -- fewer aliases of critical operations;
2014-04-28, by wenzelm
removed dead code;
2014-04-28, by wenzelm
tuned comments;
2014-04-28, by wenzelm
more systematic delay_first discipline for change_buffer and prune_history;
2014-04-28, by wenzelm
mane delayed events outside of Swing thread -- triggers no longer require Swing_Thread.later;
2014-04-28, by wenzelm
tuned;
2014-04-28, by wenzelm
added Scala version of module Event_Timer;
2014-04-28, by wenzelm
restored naming trick
2014-04-28, by blanchet
more reliable 'name_of_bnf'
2014-04-28, by blanchet
cleaner 'rel_inject' theorems
2014-04-28, by blanchet
modernized Isabelle classpath for graphview;
2014-04-27, by wenzelm
tuned;
2014-04-27, by wenzelm
merged
2014-04-26, by wenzelm
NEWS;
2014-04-26, by wenzelm
tuned message;
2014-04-26, by wenzelm
proper handling of shared zoom component: update layout dynamically;
2014-04-26, by wenzelm
PIDE support for find_consts;
2014-04-26, by wenzelm
some rearrangements to support multiple find operations;
2014-04-26, by wenzelm
tuned;
2014-04-26, by wenzelm
clarified GUI focus;
2014-04-26, by wenzelm
actually observe search limit;
2014-04-26, by wenzelm
misc tuning;
2014-04-26, by wenzelm
uniform focus traversal via TAB / Shift-TAB for all fields, in contrast to Java defaults, but in accordance to occasional jEdit practice;
2014-04-26, by wenzelm
tuned GUI events;
2014-04-26, by wenzelm
tuned;
2014-04-26, by wenzelm
tuned spelling;
2014-04-26, by wenzelm
clarified PIDE modules;
2014-04-26, by wenzelm
clarified;
2014-04-26, by wenzelm
tuned signature;
2014-04-26, by wenzelm
tuned imports;
2014-04-26, by wenzelm
tuned headers;
2014-04-26, by wenzelm
tuned signature;
2014-04-26, by wenzelm
more complete classical rules for Inf and Sup, modelled after theiry counterparts on Inter and Union (and INF and SUP)
2014-04-26, by haftmann
subsumed by existing default simp rules for functions and booleans
2014-04-26, by haftmann
tuned
2014-04-26, by haftmann
avoid non-standard simp default rule
2014-04-26, by haftmann
retired wwwfind
2014-04-26, by kleing
use right set of variables for recursive check
2014-04-26, by blanchet
merged
2014-04-26, by wenzelm
tuned -- potentially more robust;
2014-04-26, by wenzelm
suppress potential dangerous option (see 1baa5d19ac44);
2014-04-25, by wenzelm
manager is direct receiver of prover output -- discontinued old performance tuning (329320fc88df, 1baa5d19ac44);
2014-04-25, by wenzelm
modernized theory setup;
2014-04-25, by wenzelm
just one default thread pool (which is hardwired to Runtime.availableProcessors);
2014-04-25, by wenzelm
tuned signature -- separate pool for JFuture tasks, which can be canceled;
2014-04-25, by wenzelm
prefer Isabelle/Scala operations;
2014-04-25, by wenzelm
unused;
2014-04-25, by wenzelm
use Z3 4.3.2 to fix most FIXMEs
2014-04-25, by blanchet
added Z3 4.3.2 (unstable) component
2014-04-25, by blanchet
updated Z3 version number
2014-04-25, by blanchet
use Z3 4.3.2 syntax
2014-04-25, by blanchet
subscription as target-specific implementation device
2014-04-25, by haftmann
make SML/NJ happier;
2014-04-25, by wenzelm
merged
2014-04-25, by wenzelm
updated properties for scala.concurrent.ExecutionContext.Implicits.global (future task farm), similar to Isabelle/ML;
2014-04-25, by wenzelm
simplified change_buffer (again, see 937826d702d5): no thread, just timer, rely on asynchronous commands_changed.post;
2014-04-25, by wenzelm
replaced manager Actor by Consumer_Thread, which is lazy to defer its start to actual Handler init time;
2014-04-25, by wenzelm
tuned whitespace;
2014-04-25, by wenzelm
obsolete;
2014-04-25, by wenzelm
clarified Session.Consumer, with Session.Outlet managed by dispatcher thread;
2014-04-25, by wenzelm
tuned comments;
2014-04-25, by wenzelm
more robust prover termination;
2014-04-25, by wenzelm
more explicit checks;
2014-04-25, by wenzelm
tuned signature;
2014-04-24, by wenzelm
more uniform warning/error handling, potentially with propagation to send_wait caller;
2014-04-24, by wenzelm
more careful shutdown (amending f2f53f7046f4);
2014-04-24, by wenzelm
misc tuning;
2014-04-24, by wenzelm
obsolete;
2014-04-24, by wenzelm
converted main session manager to Consumer_Thread: messages need to be consumed immediately, postponed_changes replaces implicit actor mailbox scanning;
2014-04-24, by wenzelm
simplified commands_changed_buffer (in contrast to a8331fb5c959): rely on better performance of Consumer_Thread/Mailbox and more direct Timer (like session_actor.receiver);
2014-04-24, by wenzelm
simplified -- prefer Consumer_Thread over Actor;
2014-04-24, by wenzelm
tuned imports;
2014-04-24, by wenzelm
support for requests with explicit acknowledgment (and exception propagation);
2014-04-24, by wenzelm
more robust thread: continue after failure;
2014-04-24, by wenzelm
clarified command_input: Consumer_Thread;
2014-04-24, by wenzelm
further robustification wrt. unclear ranges;
2014-04-24, by wenzelm
allow more control of main loop;
2014-04-24, by wenzelm
eliminated pointless output actors;
2014-04-24, by wenzelm
more robust shutdown;
2014-04-24, by wenzelm
consumer thread with unbounded queueing of requests (similar to Message_Channel in ML);
2014-04-24, by wenzelm
proper signaling after each state update (NB: ML version does this uniformly via timed_access);
2014-04-24, by wenzelm
added Mailbox, as in ML;
2014-04-24, by wenzelm
synchronized access, similar to ML version;
2014-04-24, by wenzelm
tuned signature, in accordance to ML version;
2014-04-24, by wenzelm
eliminated redundant Volatile;
2014-04-24, by wenzelm
retain canonical reverse order;
2014-04-24, by wenzelm
more canonical list operations;
2014-04-24, by wenzelm
tuned signature in accordance to ML version;
2014-04-24, by wenzelm
canonical list operations, as in ML;
2014-04-24, by wenzelm
more uniform synchronized variables;
2014-04-24, by wenzelm
more unfolding and more folding in size equations, to look more natural in the nested case
2014-04-25, by blanchet
reintroduced '...' (nonexhaustive) syntax for SPASS-Pirate
2014-04-25, by blanchet
really unfold
2014-04-24, by blanchet
avoid non-standard simp default rule
2014-04-24, by haftmann
now covered by AFP 3ddac3e572cf
2014-04-24, by haftmann
avoid name shadowing
2014-04-24, by blanchet
spelling
2014-04-24, by blanchet
predicator simplification rules: support also partially specialized types e.g. 'a * nat
2014-04-23, by kuncar
all BNF tests can be part of a normal session because they are much faster now
2014-04-23, by kuncar
merged
2014-04-23, by wenzelm
tuned;
2014-04-23, by wenzelm
modernized Future/Promise implementation, bypassing old actors;
2014-04-23, by wenzelm
updated according to scala-2.11.0 recommendations;
2014-04-23, by wenzelm
explicit Exn.error_message in accordance to Output.error_message in ML;
2014-04-23, by wenzelm
detect nested interrupts;
2014-04-23, by wenzelm
clarified message and return code, in accordance to ML version;
2014-04-23, by wenzelm
interruptible dependencies, which can take a few seconds;
2014-04-23, by wenzelm
more abstract Exn.Interrupt and POSIX return code;
2014-04-23, by wenzelm
avoid accidental use of scala.language.reflectiveCalls;
2014-04-23, by wenzelm
tuned options for scalac;
2014-04-23, by wenzelm
updated workaround;
2014-04-23, by wenzelm
avoid "Adaptation of argument list by inserting ()" -- deprecated in scala-2.11.0;
2014-04-22, by wenzelm
avoid "Adaptation of argument list by inserting ()" -- deprecated in scala-2.11.0;
2014-04-22, by wenzelm
avoid octal escape literals -- deprecated in scala-2.11.0;
2014-04-22, by wenzelm
updated to scala-2.11.0 with classpath provided by its etc/settings;
2014-04-22, by wenzelm
no need to copy jars, after regular use of classpath in 793a429c63e7;
2014-04-22, by wenzelm
accomodate scala-2.11.0: evade somewhat erratic fix of ImmutableSetFactory in Scala/bfa70315d72d;
2014-04-22, by wenzelm
made SML/NJ happier
2014-04-23, by blanchet
size function for multisets
2014-04-23, by blanchet
updated BNF docs
2014-04-23, by blanchet
qualify name
2014-04-23, by blanchet
tuned doc comment
2014-04-23, by blanchet
updated NEWS
2014-04-23, by blanchet
localize new size function generation code
2014-04-23, by blanchet
no need to make 'size' generation an interpretation -- overkill
2014-04-23, by blanchet
put theorems in right slot
2014-04-23, by blanchet
manual merge + added 'rel_distincts' field to record for symmetry
2014-04-23, by blanchet
pick up all 'nesting' theorems
2014-04-23, by blanchet
added 'size' of finite sets
2014-04-23, by blanchet
prevent tactic failures by detecting and ignoring BNFs with no 'size' functions early
2014-04-23, by blanchet
updated docs
2014-04-23, by blanchet
move size hooks together, with new one preceding old one and sharing same theory data
2014-04-23, by blanchet
allow registration of custom size functions for BNF-based datatypes
2014-04-23, by blanchet
reverted rb458558cbcc2 -- better to keep 'case' and 'rec' distinct, otherwise we lose the connection between 'ctor_rec' (the low-level recursor) and 'rec'
2014-04-23, by blanchet
generate 'rec_o_map' and 'size_o_map' in size extension
2014-04-23, by blanchet
made old-style 'size' interpretation hook more robust in case 'size' is already specified (either by the user or by the new datatype package)
2014-04-23, by blanchet
generate size instances for new-style datatypes
2014-04-23, by blanchet
invoke 'fp_sugar' interpretation hook on mutually recursive clique
2014-04-23, by blanchet
declare 'bool' and its proxies as a datatype for SPASS-Pirate
2014-04-23, by blanchet
added 'inj_map' as auxiliary BNF theorem
2014-04-23, by blanchet
tuned whitespace
2014-04-23, by blanchet
remove add_eq_zero_iff, it is replaced by add_nonneg_eq_0_iff; also removes it from the simpset
2014-04-23, by hoelzl
favorites for jEdit file browser, although an expanded directory path is expected here, not environment variables;
2014-04-22, by wenzelm
tuned;
2014-04-22, by wenzelm
clarified exit code for the rare situation where Runtime.exn_error_message might fail;
2014-04-22, by wenzelm
tuned;
2014-04-22, by wenzelm
tuned -- avoid warning about catch-all handler;
2014-04-22, by wenzelm
more general exit;
2014-04-22, by wenzelm
swap with qualifier;
2014-04-21, by haftmann
sos accepts False, returns apply command
2014-04-20, by paulson
clarified actor plumbing;
2014-04-19, by wenzelm
more elementary option sledgehammer_provers, avoiding complications of defaults from ML side (NB: guessing at number of cores does not make sense in PIDE);
2014-04-19, by wenzelm
clarified tooltip_lines: HTML.encode already takes care of newline (but not space);
2014-04-19, by wenzelm
removed odd context argument: Thy_Info.get_theory does not fit into PIDE document model;
2014-04-19, by wenzelm
obsolete for release;
2014-04-19, by wenzelm
obsolete since polyml-5.5.0;
2014-04-19, by wenzelm
added command 'SML_export' and 'SML_import' for exchange of toplevel bindings;
2014-04-19, by wenzelm
reintroduced process interrupt for the sake of synchronous protocol commands like "use_theories" (see also 27930cf6f0f7);
2014-04-17, by wenzelm
added protocol command "use_theories", with core functionality of batch build;
2014-04-17, by wenzelm
tuned comments;
2014-04-17, by wenzelm
tuned;
2014-04-17, by wenzelm
tuned option name;
2014-04-17, by wenzelm
tuned;
2014-04-17, by wenzelm
proper tooltip_lines for multi-line text;
2014-04-17, by wenzelm
unused;
2014-04-17, by wenzelm
capitalize more carefully, e.g. relevant for option "ML_exception_trace";
2014-04-17, by wenzelm
more simp rules for Fun.swap
2014-04-16, by haftmann
updated to jdk-8u5;
2014-04-16, by wenzelm
avoid ooddity: invoke intended function instead of java.awt.Container.invalidate();
2014-04-16, by wenzelm
tuned;
2014-04-16, by wenzelm
tuned spelling;
2014-04-16, by wenzelm
more uniform treatment of word case for check / complete;
2014-04-16, by wenzelm
capitalize fully (like in Emacs);
2014-04-16, by wenzelm
clarified word case;
2014-04-16, by wenzelm
more specific support for sequence of words;
2014-04-16, by wenzelm
tuned signature -- separate module Word;
2014-04-16, by wenzelm
more NEWS;
2014-04-15, by wenzelm
tuned default: melange of all "en" dialects;
2014-04-15, by wenzelm
updated to jortho-1.0-2: added dictionary "en-CA", changed dictionary "en" to be the union of all dialects instead of intersection;
2014-04-15, by wenzelm
more context-sensitivity;
2014-04-15, by wenzelm
tuned spelling;
2014-04-15, by wenzelm
back to unrestricted before_caret_range, which is important for quick editing at the end of line (amending 83777a91f5de);
2014-04-15, by wenzelm
prefer direct caret_range for update_dictionary actions, which usually happen outside the flow of editing;
2014-04-15, by wenzelm
clarified abbreviations for cartouche delimiters, to work in any context;
2014-04-15, by wenzelm
clarified treatment of markup ranges wrt. revert/convert: inflate_singularity allows to retrieve information like language_context more reliably during editing;
2014-04-15, by wenzelm
more robust JEdit_Lib.line_range, according to usual jEdit confusion at end of last line;
2014-04-15, by wenzelm
avoid conflict of Isabelle/jEdit popups with jEdit context menu;
2014-04-15, by wenzelm
clarified before_caret_range: prevent continuation on next line;
2014-04-15, by wenzelm
explicit menu action to complete word;
2014-04-15, by wenzelm
common context menu for Isabelle/jEdit;
2014-04-15, by wenzelm
tuned;
2014-04-15, by wenzelm
tuned;
2014-04-15, by wenzelm
tuned spelling;
2014-04-15, by wenzelm
tuned menu;
2014-04-15, by wenzelm
NEWS;
2014-04-15, by wenzelm
tuned spelling;
2014-04-15, by wenzelm
proper signature for dynamic BeanShell action;
2014-04-14, by wenzelm
tuned;
2014-04-14, by wenzelm
added context menu for spell checker actions;
2014-04-14, by wenzelm
full repaint after dictionary update;
2014-04-14, by wenzelm
some actions to maintain spell-checker dictionary;
2014-04-14, by wenzelm
more explicit user declarations for main dictionary;
2014-04-14, by wenzelm
Removed old experiment (broken since b458b4ac570f resp 4159caa18f85)
2014-04-14, by noschinl
added divide_nonneg_nonneg and co; made it a simp rule
2014-04-14, by hoelzl
support for persistent user dictionaries;
2014-04-14, by wenzelm
tuned;
2014-04-14, by wenzelm
eliminated somewhat pointless locale parameter;
2014-04-14, by wenzelm
tuned;
2014-04-13, by wenzelm
clarified complete: participate in case-mangling of check;
2014-04-13, by wenzelm
tuned;
2014-04-13, by wenzelm
added spell-checker completion dialog, without counting frequency of items due to empty name;
2014-04-13, by wenzelm
tuned signature;
2014-04-13, by wenzelm
special treatment for '' ligature in TeX, which counts as word separator
2014-04-13, by wenzelm
more elementary notion of "word" (similar to VoxSpell) -- treat hyphen as separator;
2014-04-13, by wenzelm
tuned rendering -- avoid overlap with squiggly underline;
2014-04-13, by wenzelm
added dictionaries_selector GUI;
2014-04-13, by wenzelm
tuned signature -- explicit Spell_Checker_Variable;
2014-04-13, by wenzelm
updated to jortho-1.0-1: dictionaries from SCOWL 7.1, with parameters like aspell;
2014-04-13, by wenzelm
clarified according to ML version;
2014-04-13, by wenzelm
merged
2014-04-12, by wenzelm
NEWS;
2014-04-12, by wenzelm
more spell_checker_elements;
2014-04-12, by wenzelm
some case-mangling;
2014-04-12, by wenzelm
more general spell_checker_elements;
2014-04-12, by wenzelm
added spell-checker options;
2014-04-12, by wenzelm
added bad_words;
2014-04-12, by wenzelm
markup for prose words within formal comments;
2014-04-12, by wenzelm
added spell-checker based on jortho-1.0;
2014-04-11, by wenzelm
prefere standard Isabelle/Scala operation, with fixed locale;
2014-04-11, by wenzelm
more operations and lemmas
2014-04-12, by haftmann
made mult_pos_pos a simp rule
2014-04-12, by nipkow
bi_unique and co. rules from the BNF hook must be introduced after bi_unique op= and co. rules are introduced
2014-04-11, by kuncar
merged
2014-04-11, by nipkow
made divide_pos_pos a simp rule
2014-04-11, by nipkow
fix the reflexivity prover
2014-04-11, by kuncar
merged
2014-04-11, by kuncar
observe also DEADID BNFs and associate the conjunction in rel_inject to the right
2014-04-11, by kuncar
made ereal_add_nonneg_nonneg a simp rule
2014-04-11, by nipkow
made mult_nonneg_nonneg a simp rule
2014-04-11, by nipkow
merged
2014-04-11, by wenzelm
more formal dependencies via 'document_files';
2014-04-11, by wenzelm
explicit 'document_files' in session ROOT specifications;
2014-04-11, by wenzelm
tuned message, to accommodate extra brackets produced by Scala parsers;
2014-04-11, by wenzelm
tuned;
2014-04-10, by wenzelm
removed obsolete doc_dump option (see also 892061142ba6);
2014-04-10, by wenzelm
restoring notion of primitive vs. derived operations in terms of generated code;
2014-04-09, by haftmann
removed duplication and tuned
2014-04-09, by haftmann
make list_all an abbreviation of pred_list - prevent duplication
2014-04-10, by kuncar
add pred_inject for product and sum because these theorems are not generated automatically because prod and sum are not in FP sugar for bootstrapping reasons
2014-04-10, by kuncar
simplify and fix theories thanks to 356a5efdb278
2014-04-10, by kuncar
setup for Transfer and Lifting from BNF; tuned thm names
2014-04-10, by kuncar
revert idiomatic handling of namings from 5a93b8f928a2 because in combination with Named_Target.theory_init global names are sometimes created
2014-04-10, by kuncar
don't forget to init Interpretation and transfer theorems in the interpretation hook
2014-04-10, by kuncar
export theorems
2014-04-10, by kuncar
abstract Domainp in relator_domain rules => more natural statement of the rule
2014-04-10, by kuncar
more appropriate name (Lifting.invariant -> eq_onp)
2014-04-10, by kuncar
left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
2014-04-10, by kuncar
tuned
2014-04-10, by kuncar
more accurate type arguments for intermeadiate typedefs
2014-04-10, by traytel
merged
2014-04-10, by wenzelm
ignore other_id reports for now (see 8eda56033203): massive amounts of redirections to 'class' etc. makes it difficult to edit main HOL;
2014-04-10, by wenzelm
more standard names;
2014-04-10, by wenzelm
modernized simproc_setup;
2014-04-10, by wenzelm
modernized theory setup;
2014-04-10, by wenzelm
added simproc markup, which also indicates legacy simprocs outside the name space;
2014-04-10, by wenzelm
modernized simproc_setup;
2014-04-10, by wenzelm
misc tuning;
2014-04-10, by wenzelm
more contributors;
2014-04-10, by wenzelm
tuned;
2014-04-10, by wenzelm
NEWS;
2014-04-10, by wenzelm
tuned error -- allow user to click on hyperlink to open remote file;
2014-04-10, by wenzelm
no comment -- File.read_stream already enforces UTF8 (like HTML5) and HTTP servers often produce a wrong charset encoding;
2014-04-10, by wenzelm
improved support for external URLs, based on standard Java network operations;
2014-04-09, by wenzelm
basic URL operations (with Isabelle/Scala error handling);
2014-04-09, by wenzelm
proper Args.name vs. Args.text as documented (in contrast to adhoc union in 75aaee32893d, which had to cope with more limited Args.T);
2014-04-09, by wenzelm
allow text cartouches in regular outer syntax categories "text" and "altstring";
2014-04-09, by wenzelm
tuned comments (see Scala version);
2014-04-09, by wenzelm
dismiss popups more carefully (amending 7e8c11011fdf), notably allow mouse dragging within some tooltip, e.g. for text selection;
2014-04-09, by wenzelm
clarifed results range;
2014-04-09, by wenzelm
more explicit message discrimination;
2014-04-09, by wenzelm
avoid confusion about pointless cursor movement with external links;
2014-04-09, by wenzelm
prefer regular Goal_Display.pretty_goals, without censorship of options;
2014-04-09, by wenzelm
more standard names;
2014-04-09, by wenzelm
proper context for print_tac;
2014-04-09, by wenzelm
more conventional tactic programming;
2014-04-09, by wenzelm
tuned;
2014-04-09, by wenzelm
reintroduce example (cf. 39281b3e4fac)
2014-04-10, by traytel
use mutual clique information (cf. c451cf8b29c8) to make N2M more robust
2014-04-10, by traytel
made N2M tactic more robust
2014-04-10, by traytel
generate cliques for 'prim(co)rec' N2M
2014-04-09, by blanchet
thread mutual cliques through
2014-04-09, by blanchet
generalize ln/log_powr; add log_base_powr/pow
2014-04-09, by hoelzl
parametricity transfer rule for INFIMUM, SUPREMUM
2014-04-09, by haftmann
add divide_simps
2014-04-09, by hoelzl
field_simps: better support for negation and division, and power
2014-04-09, by hoelzl
revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
2014-04-09, by hoelzl
merged
2014-04-08, by wenzelm
more native rm_tree, using Java 7 facilities;
2014-04-08, by wenzelm
expose more bad cases;
2014-04-08, by wenzelm
tuned signature;
2014-04-08, by wenzelm
more direct interpretation of "warned" status, like "failed" and independently of "finished", e.g. relevant for Rendering.overview_color of aux. files where main command status is unavailable (amending 0546e036d1c0);
2014-04-08, by wenzelm
simplified Text.Chunk -- eliminated ooddities;
2014-04-08, by wenzelm
tuned;
2014-04-08, by wenzelm
more frugal Symbol.Index -- no need to waste space on mostly empty arrays;
2014-04-08, by wenzelm
accumulate markup reports for "other" command ids, which are later retargeted and merged for rendering (in erratic order);
2014-04-08, by wenzelm
avoid data redundancy;
2014-04-08, by wenzelm
tuned signature -- moved Command.Chunk to Text.Chunk;
2014-04-08, by wenzelm
more uniform ML/document antiquotations;
2014-04-08, by wenzelm
obsolete;
2014-04-08, by wenzelm
more positions and markup;
2014-04-08, by wenzelm
more precise token positions;
2014-04-08, by wenzelm
more uniform Command.Chunk operations;
2014-04-08, by wenzelm
more explicit Command.Chunk types, less ooddities;
2014-04-08, by wenzelm
tuned;
2014-04-08, by wenzelm
ignore deps_changed (again) -- avoid proactive load attempts of unfinished header specification while the user is typing;
2014-04-08, by wenzelm
no report for position singularity, notably for aux. file, especially empty one;
2014-04-08, by wenzelm
simplified blob again (amending 1e77ed11f2f7): only store file node name, i.e. the raw editor file name;
2014-04-07, by wenzelm
tuned signature -- prefer static type Document.Node.Name;
2014-04-07, by wenzelm
commented out example that triggers a bug
2014-04-08, by blanchet
allow arguments to 'datatype_compat' in disorder
2014-04-08, by blanchet
added 'datatype_compat' examples/tests
2014-04-08, by blanchet
support deeply nested datatypes in 'datatype_compat'
2014-04-08, by blanchet
preserve user type variable names to avoid mismatches/confusion
2014-04-08, by blanchet
even more standardized doc session names after #b266e7a86485
2014-04-08, by haftmann
refrain from changing jEdit default shortcuts, due to potential for conflicts and actually not working on Mac OS X;
2014-04-07, by wenzelm
support for URL as file name, similar to treatment in jEdit.java;
2014-04-07, by wenzelm
provide old-style ISABELLE_SCALA_SCRIPT for uniformity;
2014-04-07, by wenzelm
separate file_node vs. file_path, e.g. relevant on Windows for hyperlink to the latter;
2014-04-07, by wenzelm
merged
2014-04-06, by nipkow
tuned lemmas: more general class
2014-04-06, by nipkow
tuned proofs;
2014-04-06, by wenzelm
removed abbrev "<-" again (see c771f0fe28d1) due to conflict with important "<->" and "<-->";
2014-04-06, by wenzelm
merged
2014-04-06, by nipkow
made field_simps "more complete"
2014-04-06, by nipkow
shell functions for all Isabelle executables;
2014-04-06, by wenzelm
renamed "isabelle-process" to "isabelle_process", with shell function to avoid dynamic path lookups;
2014-04-06, by wenzelm
more source positions;
2014-04-06, by wenzelm
clarified position: no offset here;
2014-04-06, by wenzelm
more source positions;
2014-04-06, by wenzelm
approximate ML antiquotation @{here} for Isabelle/Pure bootstrap;
2014-04-06, by wenzelm
clarified ML bootstrap;
2014-04-06, by wenzelm
prepare "back" position for Navigator, before following hyperlink;
2014-04-06, by wenzelm
tuned;
2014-04-05, by wenzelm
merged
2014-04-05, by wenzelm
more uniform build options;
2014-04-05, by wenzelm
re-implemented build_doc in Isabelle/Scala;
2014-04-05, by wenzelm
more standard Isabelle_System.tmp_file and tmp_dir operations, in accordance to ML version;
2014-04-05, by wenzelm
more standard hash-bang (python *is* canonical according to Admin/PLATFORMS);
2014-04-05, by wenzelm
tuned -- just one qualification of sections ("!");
2014-04-05, by wenzelm
tuned error;
2014-04-05, by wenzelm
proper settings instead of hard-wired information;
2014-04-05, by wenzelm
explicit indication of important doc sections ("!"), which are expanded in the tree view;
2014-04-05, by wenzelm
clarified Doc entry: more explicit path;
2014-04-05, by wenzelm
updated to jedit_build-20140405: Code2HTML.jar, CommonControls.jar, Console.jar, kappalayout.jar, Navigator.jar, SideKick.jar, doc with jEdit manuals (ant dist-manuals);
2014-04-05, by wenzelm
closer correspondence of document and session names, while maintaining document names for external reference
2014-04-05, by haftmann
ignore jedit mark files
2014-04-05, by paulson
avoid romanism
2014-04-05, by haftmann
churning pie charts (with non-canonical prerequisites!)
2014-04-05, by haftmann
CONTRIBUTORS
2014-04-05, by haftmann
proper inclusion into library
2014-04-05, by haftmann
A single [simp] to handle the case -a/-b.
2014-04-05, by paulson
support for jEdit Navigator plugin;
2014-04-04, by wenzelm
more permissive Session.update_options: this is wired to jEdit PropertiesChanged, which may occur before the prover is started;
2014-04-04, by wenzelm
added option to Mirabelle
2014-04-04, by blanchet
divide_minus_left divide_minus_right are in field_simps but are not default simprules
2014-04-04, by paulson
removing simprule status for divide_minus_left and divide_minus_right
2014-04-03, by paulson
merged;
2014-04-04, by wenzelm
tuned rendering -- take 1px line border into account;
2014-04-04, by wenzelm
revert ce37fcb30cf2 for the sake of Mac OS X -- let some event listeners of jEdit reset the cursor;
2014-04-04, by wenzelm
tuned white space;
2014-04-04, by wenzelm
use Z3 TPTP cores rather than proofs since the latter are somewhat broken
2014-04-04, by blanchet
tuned spaces
2014-04-04, by blanchet
merged
2014-04-04, by Andreas Lochbihler
add missing adaptation for narrowing to work with variables of type integer => integer
2014-04-04, by Andreas Lochbihler
merged
2014-04-04, by wenzelm
added ML antiquotation @{print};
2014-04-04, by wenzelm
afford larger full_index, to save a few milliseconds during rendering (notably text_overview);
2014-04-04, by wenzelm
improved parsing of "z3_tptp" proofs
2014-04-04, by blanchet
merged
2014-04-03, by wenzelm
more direct warning within persistent Protocol.Status;
2014-04-03, by wenzelm
clarified Version.syntax -- avoid guessing initial situation;
2014-04-03, by wenzelm
more abstract Prover.Syntax, as proposed by Carst Tankink;
2014-04-03, by wenzelm
tuned signature (see also 0850d43cb355);
2014-04-03, by wenzelm
slightly more readable protocol trace (NB1: prover input is always marked as <prover_command/>; NB2: adding indentation would invalidate the XML);
2014-04-03, by wenzelm
recovered public command_line from d92eb5c3960d, which is important for alternative prover processes;
2014-04-03, by wenzelm
tuned rendering for 5 different look-and-feels;
2014-04-03, by wenzelm
more symbol abbrevs, e.g. relevant for list comprehension in HOL/List.thy or HOL/Library/Monad_Syntax.thy;
2014-04-03, by wenzelm
more general prover operations;
2014-04-03, by wenzelm
tuned signature -- pro forma;
2014-04-03, by wenzelm
more general prover operations;
2014-04-03, by wenzelm
Merge
2014-04-03, by paulson
Cleaned up some messy proofs
2014-04-03, by paulson
fix #0556204bc230
2014-04-03, by hoelzl
merged DERIV_intros, has_derivative_intros into derivative_intros
2014-04-03, by hoelzl
don't pass Vampire option that doesn't exist anymore (and that wasn't strictly necessary with older Vampires)
2014-04-03, by blanchet
use Alt-Ergo 0.95.2, the latest and greatest version
2014-04-03, by blanchet
updated Z3 TPTP to 4.3.1+
2014-04-03, by blanchet
updated Why3 version in docs
2014-04-03, by blanchet
added same idiomatic handling of namings for Ctr_Sugar/BNF-related interpretation hooks as for typedef and (old-style) datatypes
2014-04-03, by blanchet
use same idiom as used for datatype 'size' function to name constants and theorems emerging from various type interpretations -- reduces the chances of name clashes on theory merges
2014-04-03, by blanchet
removed clone (cf. 300f613060b0)
2014-04-03, by blanchet
tuned signature -- more explicit iterator terminology;
2014-04-02, by wenzelm
more explicit iterator terminology, in accordance to Scala 2.8 library;
2014-04-02, by wenzelm
extend continuous_intros; remove continuous_on_intros and isCont_intros
2014-04-02, by hoelzl
reorder Complex_Analysis_Basics; rename DD to deriv
2014-04-02, by hoelzl
moved generic theorems from Complex_Analysis_Basic; fixed some theorem names
2014-04-02, by hoelzl
merged;
2014-04-02, by wenzelm
tuned rendering;
2014-04-02, by wenzelm
new theorem about zero limits
2014-04-02, by paulson
New theorems for extracting quotients
2014-04-02, by paulson
more contributors;
2014-04-02, by wenzelm
document value generation for quickcheck's testers
2014-04-01, by Andreas Lochbihler
tuned whitespace;
2014-04-02, by wenzelm
suppress slightly odd completion of "simp";
2014-04-02, by wenzelm
observe extra line spacing for output as well;
2014-04-02, by wenzelm
persistent protocol_status, to improve performance of node_status a little;
2014-04-02, by wenzelm
more uniform painting of caret, which also improves visibility in invisible state;
2014-04-02, by wenzelm
tuned rendering -- visual indication of the status range, to make more clear when information might is out of view;
2014-04-02, by wenzelm
tuned for-comprehensions -- less structure mapping;
2014-04-01, by wenzelm
some rephrasing to ensure that this becomes cheap "foreach" and not expensive "map" (cf. 0fc032898b05);
2014-04-01, by wenzelm
more direct command states -- merge_results is hardly ever needed;
2014-04-01, by wenzelm
unused;
2014-04-01, by wenzelm
more frugal command_status, which is often used in a tight loop;
2014-04-01, by wenzelm
simplified using "value class";
2014-04-01, by wenzelm
more precise BNF bound for datatypes
2014-04-01, by traytel
compile
2014-04-01, by blanchet
tuning
2014-04-01, by blanchet
added new-style (co)datatype interpretation hook
2014-04-01, by blanchet
added BNF interpretation hook
2014-04-01, by blanchet
added 'ctr_sugar' interpretation hook
2014-04-01, by blanchet
tuned
2014-04-01, by traytel
merged
2014-03-31, by wenzelm
cumulative NEWS;
2014-03-31, by wenzelm
observe focus change for all tooltips, e.g. relevant for focus change to unrelated components;
2014-03-31, by wenzelm
clear active areas (notably mouse pointer) before changing context (e.g. via hyperlink);
2014-03-31, by wenzelm
reset mouse pointer more decisively, for the sake of Mac OS X (despite the builtin policie of jEdit);
2014-03-31, by wenzelm
proper structural hashCode, which is required for Command.File equals (NB: Array has physical object identity);
2014-03-31, by wenzelm
tuned output;
2014-03-31, by wenzelm
tuned signature -- more static typing;
2014-03-31, by wenzelm
store blob content within document node: aux. files that were once open are made persistent;
2014-03-31, by wenzelm
some shortcuts for chunks, which sometimes avoid bulky string output;
2014-03-31, by wenzelm
support bulk messages consisting of small string segments, which are more healthy to the Poly/ML RTS and might prevent spurious GC crashes such as MTGCProcessMarkPointers::ScanAddressesInObject;
2014-03-31, by wenzelm
tuned proofs
2014-03-31, by hoelzl
add complex_of_real coercion
2014-03-31, by hoelzl
add limits of power at top and bot
2014-03-31, by hoelzl
add connected_local_const
2014-03-31, by hoelzl
add rules about infinity of intervals
2014-03-31, by hoelzl
tuned proofs;
2014-03-30, by wenzelm
immediate completion even with delay, which is the default according to 638b29331549;
2014-03-30, by wenzelm
special treatment for various kinds of selections: imitate normal flow of editing;
2014-03-30, by wenzelm
merged
2014-03-29, by wenzelm
do not absorb vacuous copy operation, e.g. relevant when tooltip has focus but no selection, while the main text area has a selection but no focus;
2014-03-29, by wenzelm
check global mouse status before opening tooltip, e.g. relevant when the mouse has moved outside the window and mouse events are no longer seen by this component;
2014-03-29, by wenzelm
dismiss all popups on mouse drags, e.g. to avoid conflict of C-hover of Isabelle/jEdit and C-selection of jEdit;
2014-03-29, by wenzelm
tuned proofs
2014-03-28, by huffman
minimized imports
2014-03-28, by huffman
merged
2014-03-29, by wenzelm
tuned rendering -- change mouse pointer for active areas;
2014-03-29, by wenzelm
propagate deps_changed, to resolve missing files without requiring jEdit events (e.g. buffer load/save);
2014-03-29, by wenzelm
tuned signature;
2014-03-29, by wenzelm
tuned signature;
2014-03-29, by wenzelm
tuned -- see Text.Range.overlaps(Range);
2014-03-29, by wenzelm
tuned
2014-03-29, by nipkow
tuned;
2014-03-28, by wenzelm
merged
2014-03-27, by wenzelm
tuned -- avoid code duplication;
2014-03-27, by wenzelm
tuned;
2014-03-27, by wenzelm
more frugal merge of markup trees: restrict to expected range before checking trivial cases, e.g. relevant for sporadic warnings (eval_exec) within big ML reports (print_exec);
2014-03-27, by wenzelm
back to cumulative treatment of command status, which is important for total accounting (amending 8201790fdeb9);
2014-03-27, by wenzelm
tuned;
2014-03-27, by wenzelm
redirect ML_Compiler reports more directly: only the (big) parse tree report is deferred via Execution.print (NB: this does not work for asynchronous "diag" commands);
2014-03-27, by wenzelm
clarified Isabelle/ML bootstrap, such that Execution does not require ML_Compiler;
2014-03-27, by wenzelm
more frugal merge of markup trees: non-overlapping tree counts as empty;
2014-03-27, by wenzelm
more frugal merge of markup trees: filter wrt. subsequent query;
2014-03-27, by wenzelm
tuned signature;
2014-03-27, by wenzelm
more careful treatment of multiple command states (eval + prints): merge content that is actually required;
2014-03-27, by wenzelm
tuned signature -- expose less intermediate information;
2014-03-26, by wenzelm
support to redirect report on asynchronous / non-strict print function (NB: not scalable due to bulky merge of markup trees);
2014-03-26, by wenzelm
less markup by default -- this is stored persistently in Isabelle/Scala;
2014-03-26, by wenzelm
clarified valid_id: always standardize towards static command.id;
2014-03-26, by wenzelm
prefer Context_Position where a context is available;
2014-03-26, by wenzelm
unused;
2014-03-26, by wenzelm
more uniform Execution.fork vs. Execution.print;
2014-03-26, by wenzelm
added Execution.print: accumulate print operations for some command execution, which are applied later and print time;
2014-03-26, by wenzelm
tuned proofs
2014-03-26, by huffman
Some useful lemmas
2014-03-26, by paulson
tuned comments;
2014-03-26, by wenzelm
tuned load order;
2014-03-26, by wenzelm
superseded by (provide_)parse_files;
2014-03-26, by wenzelm
tuned;
2014-03-26, by wenzelm
merged
2014-03-25, by wenzelm
more warnings for recent versions of Poly/ML (see also fe1f6a1707f7);
2014-03-25, by wenzelm
eliminated dead code;
2014-03-25, by wenzelm
proper configuration option "ML_print_depth";
2014-03-25, by wenzelm
removed junk;
2014-03-25, by wenzelm
clarified options ML_source_trace and ML_exception_trace (NB: the latter needs to be a system option, since the context is sometimes not available, e.g. for 'theory' command);
2014-03-25, by wenzelm
separate tokenization and language context for SML: no symbols, no antiquotes;
2014-03-25, by wenzelm
separate "sml" mode, suppress old "ml" mode altogether;
2014-03-25, by wenzelm
some SML examples;
2014-03-25, by wenzelm
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
2014-03-25, by wenzelm
updated to scala-2.10.4;
2014-03-25, by wenzelm
cleanup auxiliary proofs for Brouwer fixpoint theorem (removes ~2400 lines)
2014-03-25, by hoelzl
prove theorems with fixed variables (export afterwards)
2014-03-25, by traytel
generalized theorems about derivatives of limits of sequences of funtions
2014-03-24, by huffman
removed unused 'ax_specification', to give 'specification' a chance to become localized;
2014-03-24, by wenzelm
merged;
2014-03-24, by wenzelm
merged
2014-03-24, by wenzelm
proper Sign.full_name to get internal name (like Sign.add_consts);
2014-03-24, by wenzelm
formal check of user input, avoiding direct references of interal names;
2014-03-24, by wenzelm
discontinued Toplevel.debug in favour of system option "exception_trace";
2014-03-24, by wenzelm
tuned proofs
2014-03-20, by huffman
made tactic more robust
2014-03-24, by traytel
inline helper function
2014-03-24, by traytel
rearranging some deriv theorems
2014-03-24, by paulson
modernized approximation, avoiding bad name binding;
2014-03-23, by wenzelm
more sensible treatment of quasi-local variables (NB: Variable.add_fixes is only for term variables, while Variable.declare takes care of types within given terms);
2014-03-23, by wenzelm
merged
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
tuned message;
2014-03-22, by wenzelm
more antiquotations;
2014-03-22, by wenzelm
avoid hard-wired theory names;
2014-03-22, by wenzelm
generalized and strengthened cong rules on compound operators, similar to 1ed737a98198
2014-03-22, by haftmann
added splash screen for jvm boot, which is important for initial encounter to avoid multiple copies running against each other;
2014-03-21, by wenzelm
merged
2014-03-21, by wenzelm
more qualified names;
2014-03-21, by wenzelm
more qualified names;
2014-03-21, by wenzelm
more qualified names;
2014-03-21, by wenzelm
tuned;
2014-03-21, by wenzelm
more qualified names;
2014-03-21, by wenzelm
tuned signature;
2014-03-21, by wenzelm
tuned signature;
2014-03-21, by wenzelm
a few new lemmas and generalisations of old ones
2014-03-21, by paulson
simplified internal datatype construction
2014-03-21, by traytel
merged
2014-03-20, by wenzelm
merged
2014-03-20, by wenzelm
produce qualified names more directly;
2014-03-20, by wenzelm
more symbols;
2014-03-20, by wenzelm
more static checking of proof methods;
2014-03-20, by wenzelm
enforce subgoal boundaries via SUBGOAL/SUBGOAL_CASES -- clean tactical failure if out-of-range;
2014-03-20, by wenzelm
more standard method_setup;
2014-03-20, by wenzelm
tuned error, according to "use" in General/secure.ML;
2014-03-20, by wenzelm
tuned proofs;
2014-03-20, by wenzelm
generalize more theorems
2014-03-20, by huffman
generalize some theorems
2014-03-20, by huffman
fixing messy proofs
2014-03-20, by paulson
pointer to the other proof direction
2014-03-20, by kleing
generalize theory of operator norms to work with class real_normed_vector
2014-03-19, by huffman
tuned -- no need for slightly obscure "local" prefix;
2014-03-19, by wenzelm
accomodate word as part of schematic variable name;
2014-03-19, by wenzelm
more explicit Long_Name operations (NB: analyzing qualifiers is inherently fragile);
2014-03-19, by wenzelm
tuned proofs;
2014-03-19, by wenzelm
elongated INFI and SUPR, to reduced risk of confusing theorems names in the future while still being consistent with INTER and UNION
2014-03-19, by haftmann
Some rationalisation of basic lemmas
2014-03-19, by paulson
Merge
2014-03-19, by paulson
New complex analysis material
2014-03-19, by paulson
NEWS
2014-03-19, by hoelzl
further renaming in Series
2014-03-19, by hoelzl
consolidated theorem names containing INFI and SUPR: have INF and SUP instead uniformly
2014-03-18, by haftmann
merged;
2014-03-18, by wenzelm
clarified module arrangement;
2014-03-18, by wenzelm
simplified (despite 70898d016538);
2014-03-18, by wenzelm
clarifed module name;
2014-03-18, by wenzelm
tuned proofs;
2014-03-18, by wenzelm
clarified module arrangement;
2014-03-18, by wenzelm
clarified modules;
2014-03-18, by wenzelm
more antiquotations;
2014-03-18, by wenzelm
clarified bootstrap process: switch to ML with context and antiquotations earlier;
2014-03-18, by wenzelm
more markup for improper elements;
2014-03-18, by wenzelm
tuned signature;
2014-03-18, by wenzelm
unused;
2014-03-18, by wenzelm
tuned signature -- rearranged modules;
2014-03-18, by wenzelm
tuned proofs;
2014-03-18, by wenzelm
back to KeyEventInterceptor (see 423e29f1f304), but without focus change, which helps to avoid loosing key events due to quick opening and closing of popups;
2014-03-17, by wenzelm
remove unnecessary finiteness assumptions from lemmas about setsum
2014-03-18, by huffman
adapt to Isabelle/c726ecfb22b6
2014-03-18, by huffman
fix HOL-NSA; move lemmas
2014-03-18, by hoelzl
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
2014-03-18, by hoelzl
changed policy when to define constants
2014-03-18, by traytel
tuned proofs; removed duplicated facts
2014-03-18, by traytel
additional lemmas
2014-03-18, by immler
removed dependencies on theory Ordered_Euclidean_Space
2014-03-18, by immler
use cbox to relax class constraints
2014-03-18, by immler
merged
2014-03-17, by wenzelm
tuned;
2014-03-17, by wenzelm
more antiquotations;
2014-03-17, by wenzelm
more robust machine-generated ML sources: constructors for typ and term sometimes occur elsewhere;
2014-03-17, by wenzelm
remove sums_seq, it is not used
2014-03-17, by hoelzl
update syntax of has_*derivative to infix 50; fixed proofs
2014-03-17, by hoelzl
unify syntax for has_derivative and differentiable
2014-03-17, by hoelzl
tuned proofs
2014-03-17, by haftmann
tuned internal construction
2014-03-17, by traytel
a few new theorems
2014-03-17, by paulson
proper flags for main action (amending 638b29331549);
2014-03-17, by wenzelm
tuned rendering -- avoid flashing background of aux. files that are disconnected from the document model;
2014-03-17, by wenzelm
merge semantic and syntax completion;
2014-03-17, by wenzelm
tuned;
2014-03-17, by wenzelm
tuned signature;
2014-03-17, by wenzelm
tuned signature;
2014-03-17, by wenzelm
clarified key event propagation, in accordance to outer_key_listener;
2014-03-17, by wenzelm
allow implicit semantic completion, notably after delay that exceeds usual round-trip time;
2014-03-17, by wenzelm
reject internal names, notably from Term.free_dummy_patterns;
2014-03-17, by wenzelm
more uniform alias vs. hide: proper check, allow to hide global names as well;
2014-03-17, by wenzelm
tuned proofs
2014-03-16, by huffman
normalising simp rules for compound operators
2014-03-16, by haftmann
tuned markup;
2014-03-15, by wenzelm
minor tuning;
2014-03-15, by wenzelm
more markup;
2014-03-15, by wenzelm
clarified completion ordering: prefer local names;
2014-03-15, by wenzelm
tuned signature;
2014-03-15, by wenzelm
tuned -- avoid vacuous reports;
2014-03-15, by wenzelm
clarified local facts;
2014-03-15, by wenzelm
more explicit treatment of verbose mode, which includes concealed entries;
2014-03-15, by wenzelm
removed dead code;
2014-03-15, by wenzelm
clarified retrieve_generic: local error takes precedence, which is relevant for completion;
2014-03-15, by wenzelm
clarified print_local_facts;
2014-03-15, by wenzelm
more complete set of lemmas wrt. image and composition
2014-03-15, by haftmann
merge
2014-03-15, by panny
add error messages for invalid inputs
2014-03-15, by panny
add lemmas about nhds filter; tuned proof
2014-03-14, by huffman
remove unused lemma which was a direct consequence of tendsto_intros
2014-03-14, by huffman
merged
2014-03-14, by wenzelm
merged
2014-03-14, by wenzelm
prefer more robust Synchronized.var;
2014-03-14, by wenzelm
discontinued somewhat pointless "thy_script" keyword kind;
2014-03-14, by wenzelm
conceal improper cases, e.g. relevant for completion (and potentially for markup);
2014-03-14, by wenzelm
conceal somewhat obscure internal facts, e.g. relevant for 'print_theorems', 'find_theorems';
2014-03-14, by wenzelm
more accurate resolution of hybrid facts, which actually changes the sort order of results;
2014-03-14, by wenzelm
tuned -- command 'text' was localized some years ago;
2014-03-14, by wenzelm
back to a form of hybrid facts, to reduce performance impact of ed92ce2ac88e;
2014-03-14, by wenzelm
just one cumulative Proof_Context.facts, with uniform retrieval (including PIDE markup, completion etc.);
2014-03-14, by wenzelm
more frugal recording of changes: join merely requires information from one side;
2014-03-13, by wenzelm
do not test details of error messages;
2014-03-13, by wenzelm
minor tuning -- NB: props are usually empty for global facts;
2014-03-13, by wenzelm
even smarter Path.smart_implode;
2014-03-13, by wenzelm
added ML antiquotation @{path};
2014-03-13, by wenzelm
clarified Path.smart_implode;
2014-03-13, by wenzelm
generalization of differential_zero_maxmin to class real_normed_vector
2014-03-14, by huffman
delayed construction of command (and of noncommercial check) + tuning
2014-03-14, by blanchet
tuning
2014-03-14, by blanchet
consolidate consecutive steps that prove the same formula
2014-03-14, by blanchet
remove '__' skolem suffixes before showing terms to users
2014-03-14, by blanchet
undo rewrite rules (e.g. for 'fun_app') in Isar
2014-03-14, by blanchet
debugging stuff
2014-03-14, by blanchet
more simplification of trivial steps
2014-03-14, by blanchet
tuning
2014-03-14, by blanchet
tuned wording (pun)
2014-03-14, by blanchet
document the new 'nonexhaustive' option (cf. 52e8f110fec3)
2014-03-14, by blanchet
made SML/NJ happier
2014-03-14, by blanchet
print warning if some constructors are missing;
2014-03-14, by panny
updated Sledgehammer docs w.r.t. 'smt2' and 'z3_new'
2014-03-14, by blanchet
updated documentation w.r.t. 'z3_non_commercial' option in Isabelle/jEdit
2014-03-14, by blanchet
updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
2014-03-14, by blanchet
remove ordered_euclidean_space constraint from brouwer/derivative lemmas;
2014-03-13, by huffman
typos
2014-03-13, by nipkow
merged
2014-03-13, by traytel
tuned tactics
2014-03-13, by traytel
simplified internal codatatype construction
2014-03-13, by traytel
updated SMT2 examples and certificates
2014-03-13, by blanchet
updated SMT2 certificates
2014-03-13, by blanchet
added Z3 4.3.0 as component (for use with 'smt2' method)
2014-03-13, by blanchet
updated SMT example certificates
2014-03-13, by blanchet
added 'smt2_status' to keywords
2014-03-13, by blanchet
avoid name clash
2014-03-13, by blanchet
simplify index handling
2014-03-13, by blanchet
more robust indices
2014-03-13, by blanchet
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
2014-03-13, by blanchet
move lemmas to theory file, towards textual proof reconstruction
2014-03-13, by blanchet
simpler translation of 'div' and 'mod' for Z3
2014-03-13, by blanchet
tuning
2014-03-13, by blanchet
tuning
2014-03-13, by blanchet
thread through step IDs from Z3 to Sledgehammer
2014-03-13, by blanchet
adapted to ML structure renaming
2014-03-13, by blanchet
tuning
2014-03-13, by blanchet
avoid names that may clash with Z3's output (e.g. '')
2014-03-13, by blanchet
do less work in 'filter' mode
2014-03-13, by blanchet
let exception pass through in debug mode
2014-03-13, by blanchet
simplified preplaying information
2014-03-13, by blanchet
renamed (hardly used) 'prod_pred' and 'option_pred' to 'pred_prod' and 'pred_option'
2014-03-13, by blanchet
simplified solution parsing
2014-03-13, by blanchet
adapted to renamed ML files
2014-03-13, by blanchet
renamed ML files
2014-03-13, by blanchet
reintroduced old model reconstruction code -- still needs to be ported
2014-03-13, by blanchet
slacker error code policy for Z3
2014-03-13, by blanchet
repaired 'if' logic
2014-03-13, by blanchet
killed a few 'metis' calls
2014-03-13, by blanchet
honor the fact that the new Z3 can generate Isar proofs
2014-03-13, by blanchet
have Sledgehammer generate Isar proofs from Z3 proofs
2014-03-13, by blanchet
tuned ML interface
2014-03-13, by blanchet
integrate SMT2 with Sledgehammer
2014-03-13, by blanchet
removed tracing output
2014-03-13, by blanchet
use 'smt2' in SMT examples as much as currently possible
2014-03-13, by blanchet
moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
2014-03-13, by blanchet
tuned proofs
2014-03-13, by haftmann
dropped redundant theorems
2014-03-13, by haftmann
tuned
2014-03-13, by haftmann
monotonicity in complete lattices
2014-03-13, by haftmann
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
2014-03-13, by nipkow
tuned signature -- clarified module name;
2014-03-12, by wenzelm
added ML antiquotation @{here};
2014-03-12, by wenzelm
ML_Context.check_antiquotation still required;
2014-03-12, by wenzelm
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
2014-03-12, by wenzelm
proper base comparison;
2014-03-12, by wenzelm
tuned;
2014-03-12, by wenzelm
tuned proofs;
2014-03-12, by wenzelm
more explicit markup and explanation of the improper status of 'back', following the AFP style-guide;
2014-03-12, by wenzelm
clarified Markup.operator vs. Markup.delimiter;
2014-03-12, by wenzelm
more explicit markup for Token.Literal;
2014-03-12, by wenzelm
tuned signature;
2014-03-12, by wenzelm
modernized setup;
2014-03-12, by wenzelm
tuned;
2014-03-12, by wenzelm
some document antiquotations for Isabelle/jEdit elements;
2014-03-12, by wenzelm
merged
2014-03-12, by wenzelm
more explicit Sign.change_check -- detect structural mistakes where they emerge, not at later theory merges;
2014-03-12, by wenzelm
more efficient local theory operations, by imposing a linear change discipline on the main types/consts tables, in order to speed-up Proof_Context.transfer_syntax required for Local_Theory.raw_theory_result;
2014-03-11, by wenzelm
slightly more rubust (and opportunistic) exit for old-fashioned theory_to_proof, which is used by global 'sublocale' with Named_Target.init but without proper exit;
2014-03-11, by wenzelm
more standard internal data integrity;
2014-03-11, by wenzelm
tables with changes relative to some common base version -- support for efficient join/merge of big global tables with small local updates;
2014-03-11, by wenzelm
tuned signature;
2014-03-11, by wenzelm
tuned comment;
2014-03-11, by wenzelm
minor performance tuning via fast matching filter;
2014-03-11, by wenzelm
added missing theorems to unfolding set
2014-03-11, by blanchet
moved 'Quickcheck_Narrowing' further down the theory graph
2014-03-11, by blanchet
make it possible to load Quickcheck exhaustive & narrowing in parallel
2014-03-11, by blanchet
full path
2014-03-11, by blanchet
measurable_lfp/gfp: indirection not necessary
2014-03-11, by hoelzl
merged
2014-03-10, by wenzelm
tuned proofs;
2014-03-10, by wenzelm
proper Char comparison, despite weakly-typed Scala (cf. 5ff5208de089);
2014-03-10, by wenzelm
tuned message;
2014-03-10, by wenzelm
tuned message;
2014-03-10, by wenzelm
include long identifiers in the reckoning of words (e.g. "integer.lifting" vs. 'lifting_update');
2014-03-10, by wenzelm
tuned messages -- in accordance to Isabelle/Scala;
2014-03-10, by wenzelm
tuned;
2014-03-10, by wenzelm
enabled test in PIDE interaction;
2014-03-10, by wenzelm
proper Args.syntax for slightly odd bundle trickery;
2014-03-10, by wenzelm
some Markup.language_path to prevent completion of symbols (notably "~") -- always "delimited" for simplicity in contrast to 42ac3cfb89f6;
2014-03-10, by wenzelm
more markup;
2014-03-10, by wenzelm
clarified Args.check_src: retain name space information for error output;
2014-03-10, by wenzelm
tuned;
2014-03-10, by wenzelm
modernized data managed via Name_Space.table;
2014-03-10, by wenzelm
clarified Args.src: more abstract type, position refers to name only;
2014-03-10, by wenzelm
tuned signature;
2014-03-10, by wenzelm
prefer Name_Space.pretty with its builtin markup;
2014-03-10, by wenzelm
tuned signature -- prefer Name_Space.get with its builtin error;
2014-03-10, by wenzelm
abstract type Name_Space.table;
2014-03-10, by wenzelm
more structured order;
2014-03-10, by wenzelm
more direct Long_Name.qualification;
2014-03-10, by wenzelm
more restrictive completion: intern/extern stability;
2014-03-10, by wenzelm
add measurability rule for (co)inductive predicates
2014-03-10, by hoelzl
introduced antimono; incseq, decseq are now abbreviations for mono and antimono; renamed Library/Continuity to Library/Order_Continuity; removed up_cont; renamed down_cont to down_continuity and generalized to complete_lattices
2014-03-10, by hoelzl
hide implementation details
2014-03-10, by kuncar
copy-paste typo
2014-03-10, by traytel
tuned tactic
2014-03-10, by traytel
unfold intermediate definitions after sealing the bnf
2014-03-10, by traytel
bootstrap fundamental Fun theory immediately after Set theory, without dependency on complete lattices
2014-03-09, by haftmann
tuned;
2014-03-09, by haftmann
more careful unfolding of internal constants
2014-03-09, by traytel
made typedef for the type of the bound optional (size-based)
2014-03-09, by traytel
made natLe{q,ss} constants (yields smaller terms in composition)
2014-03-07, by traytel
removed junk
2014-03-07, by traytel
tuned proofs;
2014-03-09, by wenzelm
unused;
2014-03-09, by wenzelm
tuned;
2014-03-09, by wenzelm
more formal read_root;
2014-03-09, by wenzelm
simplified / modernized hide commands: proper outer parsers and PIDE markup via check;
2014-03-09, by wenzelm
removed dead code;
2014-03-09, by wenzelm
check fact names with PIDE markup;
2014-03-09, by wenzelm
tuned signature;
2014-03-09, by wenzelm
do allow replacement of words where this is appropriate, notably symbol abbrevs and keyword templates (see also 1c42ebdb3a58);
2014-03-09, by wenzelm
tuned proofs;
2014-03-08, by wenzelm
tuned proofs;
2014-03-08, by wenzelm
keep current context visibility for PIDE markup and completion (in contrast to 8e3e004f1c31): Attrib.check_src of 9dc5ce83202c should intern/report attributes once, which happens for local_theory in the (visible) auxiliary context;
2014-03-08, by wenzelm
modernized Attrib.check_name/check_src similar to methods (see also a989bdaf8121);
2014-03-08, by wenzelm
allow suffix of underscores for words (notably keywords), similar to semantic completion;
2014-03-08, by wenzelm
back to polyml-svn, with more threads to avoid problems with HOL-Proofs (see f376f18fd0b7);
2014-03-08, by wenzelm
no completion for complete keywords, to avoid confusion of 'assume' ~> 'assumes' etc.;
2014-03-08, by wenzelm
clarified description;
2014-03-08, by wenzelm
tuned;
2014-03-08, by wenzelm
tuned proofs;
2014-03-07, by wenzelm
more antiquotations;
2014-03-07, by wenzelm
ignore special names that are treated differently for various sub-languages (main wild-card is identifier "__");
2014-03-07, by wenzelm
merged
2014-03-07, by wenzelm
misc tuning;
2014-03-07, by wenzelm
more strict discrimination: symbols vs. keywords could overlap;
2014-03-07, by wenzelm
tuned;
2014-03-07, by wenzelm
more accurate description;
2014-03-07, by wenzelm
misc tuning and clarification;
2014-03-07, by wenzelm
more accurate description;
2014-03-07, by wenzelm
tuned proofs;
2014-03-07, by wenzelm
tuned;
2014-03-07, by wenzelm
tuned message: reveal ambiguity where Syntax_Phases.decode_term fails and thus reduces proper_results beforehand, e.g. term "f(x := y)" in ~~/src/HOL/Hoare/Hoare_Logic.thy;
2014-03-07, by wenzelm
tuned description and its rendering;
2014-03-07, by wenzelm
more detailed description of completion items;
2014-03-07, by wenzelm
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
2014-03-07, by wenzelm
no completion of concealed names;
2014-03-07, by wenzelm
more official const syntax: avoid educated guessing by Syntax_Phases.decode_term;
2014-03-07, by wenzelm
less
more
|
(0)
-30000
-10000
-1920
+1920
+10000
tip