Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+1000
+3000
+10000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
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
tuned whitespace;
2014-03-07, by wenzelm
removed dead code;
2014-03-07, by wenzelm
modernized theory setup;
2014-03-07, by wenzelm
Some new proofs. Tidying up, esp to remove "apply rule".
2014-03-07, by paulson
use balanced tuples in 'primcorec'
2014-03-07, by blanchet
tuning
2014-03-07, by blanchet
a few new lemmas
2014-03-07, by paulson
balance tuples that represent curried functions
2014-03-07, by blanchet
merged
2014-03-06, by wenzelm
tuned proofs;
2014-03-06, by wenzelm
some NEWS;
2014-03-06, by wenzelm
special identifier "__" (i.e. empty name with internal suffix) serves as wild-card for completion;
2014-03-06, by wenzelm
completion is part of error (not report) and thus not subject to context visibility -- e.g. relevant for 'fixes' in long statements;
2014-03-06, by wenzelm
proper position for decode_pos, which is relevant for completion;
2014-03-06, by wenzelm
more decisive commitment to get_free vs. the_const;
2014-03-06, by wenzelm
more rigid const demands, based on educated guesses about the tools involved here;
2014-03-06, by wenzelm
more compact Markup.markup_report: message body may consist of multiple elements;
2014-03-06, by wenzelm
reject internal term names outright, and complete consts instead;
2014-03-06, by wenzelm
eliminated odd type constraint for read_const (see also 79c1d2bbe5a9);
2014-03-06, by wenzelm
more uniform check_const/read_const;
2014-03-06, by wenzelm
tuned;
2014-03-06, by wenzelm
more rigid type_name demands, based on educated guesses about the tools involved here;
2014-03-06, by wenzelm
tuned signature -- more uniform check_type_name/read_type_name;
2014-03-06, by wenzelm
clarified treatment of consts -- prefer value-oriented reports;
2014-03-06, by wenzelm
clarified check of internal names;
2014-03-06, by wenzelm
tuned signature;
2014-03-06, by wenzelm
tuned;
2014-03-06, by wenzelm
tuned
2014-03-06, by Lars Hupel
renamed 'fun_rel' to 'rel_fun'
2014-03-06, by blanchet
renamed 'prod_rel' to 'rel_prod'
2014-03-06, by blanchet
renamed 'sum_rel' to 'rel_sum'
2014-03-06, by blanchet
renamed 'filter_rel' to 'rel_filter'
2014-03-06, by blanchet
renamed 'endofun_rel' to 'rel_endofun'
2014-03-06, by blanchet
renamed 'vset_rel' to 'rel_vset'
2014-03-06, by blanchet
fixed NEWS
2014-03-06, by blanchet
renamed 'set_rel' to 'rel_set'
2014-03-06, by blanchet
tuned
2014-03-06, by traytel
rationalized imports
2014-03-06, by traytel
move special BNFs used for composition only to BNF_Comp;
2014-03-06, by traytel
renamed 'cset_rel' to 'rel_cset'
2014-03-06, by blanchet
renamed 'fset_rel' to 'rel_fset'
2014-03-06, by blanchet
renamed 'map_pair' to 'map_prod'
2014-03-06, by blanchet
renamed 'map_sum' to 'sum_map'
2014-03-06, by blanchet
more careful simplification of sets (cf. abf91ebd0820)---yields smaller terms
2014-03-06, by traytel
remove lemmas in favor of more general ones: convex(_hull)_set_{plus,setsum}
2014-03-05, by huffman
generalize lemma closure_sum
2014-03-05, by huffman
generalize lemmas
2014-03-05, by huffman
more symbols;
2014-03-05, by wenzelm
tuned proofs;
2014-03-05, by wenzelm
tuned color (cf. jEdit FUNCTION);
2014-03-05, by wenzelm
tuned;
2014-03-05, by wenzelm
more markup for inner syntax class/type names (notably for completion);
2014-03-05, by wenzelm
tuned proofs;
2014-03-05, by wenzelm
back to stable polyml-5.5.1, due to problems with Poly/ML SVN 1913 and HOL-Proofs (Fail "Insufficient memory");
2014-03-05, by wenzelm
more explicit quasi_keyword markup, for Args.$$$ material, which is somewhere in between of outer and inner syntax;
2014-03-05, by wenzelm
unused;
2014-03-05, by wenzelm
special treatment of method combinators like Args.$$$ keywords, although parsed via Parse.$$$;
2014-03-05, by wenzelm
more thorough (potentially duplicate) markup, e.g. relevant for embedded Args syntax within antiquotations;
2014-03-05, by wenzelm
suppress short abbreviations more uniformly, for outer and quasi-outer syntax;
2014-03-05, by wenzelm
clarified init_assignable: make double-sure that initial values are reset;
2014-03-05, by wenzelm
proper UTF-8;
2014-03-05, by wenzelm
fix typo
2014-03-04, by huffman
remove simp rules made redundant by the replacement of neg_numeral with negated numerals
2014-03-04, by huffman
tuned proof
2014-03-04, by huffman
tuned proof script
2014-03-04, by huffman
no 'sorry' so that the schematic variable gets instantiated
2014-03-04, by blanchet
removed junk
2014-03-04, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+1000
+3000
+10000
tip