Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+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;
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
tip