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