Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+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.
updated to named_theorems;
2014-08-16, by wenzelm
updated to named_theorems;
2014-08-16, by wenzelm
modernized module name and setup;
2014-08-16, by wenzelm
updated syntax for localized commands;
2014-08-16, by wenzelm
updated documentation concerning 'named_theorems';
2014-08-16, by wenzelm
prefer 'named_theorems' over Named_Thms, with subtle change of semantics due to visual order vs. internal reverse order;
2014-08-16, by wenzelm
more informative Token.Name with history of morphisms;
2014-08-15, by wenzelm
merged
2014-08-14, by wenzelm
more informative Token.Fact: retain name of dynamic fact (without selection);
2014-08-14, by wenzelm
localized command 'method_setup' and 'attribute_setup';
2014-08-14, by wenzelm
T1 font encoding with searchable underscore (requires proper cm-super fonts);
2014-08-14, by wenzelm
prefer high-level change of \isabellestyle;
2014-08-14, by wenzelm
tuned;
2014-08-14, by wenzelm
tuned;
2014-08-14, by wenzelm
tuned signature;
2014-08-14, by wenzelm
localized method definitions (see also f14c1248d064);
2014-08-14, by wenzelm
tuned signature -- prefer self-contained user-space tool;
2014-08-14, by wenzelm
document property 'rel_map'
2014-08-14, by desharna
generate 'rel_map' theorem for BNFs
2014-08-14, by desharna
tuned;
2014-08-13, by wenzelm
merged
2014-08-13, by wenzelm
tuned signature -- proper Local_Theory.add_thms_dynamic;
2014-08-13, by wenzelm
transfer result of Global_Theory.add_thms_dynamic to context stack;
2014-08-13, by wenzelm
localized attribute definitions;
2014-08-13, by wenzelm
load local_theory.ML before attrib.ML, with subtle change of semantics due to canonical Local_Theory.map_contexts instead of private Local_Theory.map_top;
2014-08-13, by wenzelm
clarified terminology: first is top (amending d110b0d1bc12);
2014-08-13, by wenzelm
tuned whitespace;
2014-08-13, by wenzelm
tuned comments;
2014-08-13, by wenzelm
add algebraic type class instances for Enum.finite* types
2014-08-13, by Andreas Lochbihler
Quickcheck_Types is no longer needed due to 51aa30c9ee4e
2014-08-13, by Andreas Lochbihler
clarified focus and key handling -- more like SideKick;
2014-08-12, by wenzelm
merged
2014-08-12, by wenzelm
tuned signature according to Scala version -- prefer explicit argument;
2014-08-12, by wenzelm
tuned signature;
2014-08-12, by wenzelm
generic process wrapping in Prover;
2014-08-12, by wenzelm
more abstract Prover.System_Process, which allows to bypass Isabelle_System.Managed_Process;
2014-08-12, by wenzelm
allow hyperlinks without offset, just in case the prover emits such reports, despite Position.is_reported;
2014-08-12, by wenzelm
more frugal standard message properties;
2014-08-12, by wenzelm
tuned;
2014-08-12, by wenzelm
clarified Position.Identified: do not require range from prover, default to command position;
2014-08-12, by wenzelm
maintain Command_Range position as in ML;
2014-08-12, by wenzelm
more compact representation of special string values;
2014-08-12, by wenzelm
separate Java FX modules -- no need to include jfxrt.jar by default;
2014-08-12, by wenzelm
tuned signature;
2014-08-12, by wenzelm
tuned signature;
2014-08-12, by wenzelm
separate module Command_Span: mostly syntactic representation;
2014-08-12, by wenzelm
tuned signature;
2014-08-11, by wenzelm
clarified Command_Span in accordance to Scala (see also c2c1e5944536);
2014-08-11, by wenzelm
tuned output, in accordance to transaction name in ML;
2014-08-11, by wenzelm
more explicit type Span in Scala, according to ML version;
2014-08-11, by wenzelm
clarified modules;
2014-08-11, by wenzelm
clarified signature: entity serial number is not position id;
2014-08-11, by wenzelm
avoid needless (and wrong w.r.t. sorts) generation of type variables; tuned whitespaces;
2014-08-12, by blanchet
improved unfolding of 'let's
2014-08-12, by blanchet
tuned whitespace
2014-08-12, by blanchet
less aggressive unfolding; removed debugging;
2014-08-12, by blanchet
document property 'set_cases'
2014-08-12, by desharna
generate 'set_cases' theorem for (co)datatypes
2014-08-12, by desharna
document property 'set_intros'
2014-08-12, by desharna
generate 'set_intros' theorem for (co)datatypes
2014-08-12, by desharna
use Goal.prove_sorry instead of Goal.prove where possible (= no schematics in goal and tactic is expected to succeed)
2014-08-11, by traytel
reduced warnings;
2014-08-10, by wenzelm
some localization;
2014-08-10, by wenzelm
support aliases within the facts space;
2014-08-10, by wenzelm
support for named collections of theorems in canonical order;
2014-08-10, by wenzelm
insist in proper 'document_files';
2014-08-10, by wenzelm
tuned -- avoid confusion with @{assert} for system failures (exception Fail);
2014-08-10, by wenzelm
tuned -- eliminated redundant check (see 1f77110c94ef);
2014-08-10, by wenzelm
merged -- with manual conflict resolution for src/HOL/SMT_Examples/SMT_Examples.certs2, src/HOL/SMT_Examples/SMT_Word_Examples.certs2, src/Doc/Prog_Prove/document/intro-isabelle.tex;
2014-08-10, by wenzelm
updated URL (anticipate merge with 85b8cc142384);
2014-08-10, by wenzelm
Added tag Isabelle2014-RC3 for changeset 91e188508bc9
2014-08-10, by wenzelm
proper layered_pane for JDialog, e.g. relevant for floating dockables in jEdit, for completion popup in text field;
2014-08-10, by wenzelm
follow link to originating command, to ensure that Simplifier_Trace_Dockable displays its results (via current_command);
2014-08-10, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned;
2014-08-09, by wenzelm
tuned comments;
2014-08-09, by wenzelm
clarified synchronized scope;
2014-08-09, by wenzelm
tuned comments;
2014-08-09, by wenzelm
application manifest for Windows 8/8.1 dpi scaling;
2014-08-08, by wenzelm
observe context visibility -- less redundant warnings;
2014-08-08, by wenzelm
improved monitor panel;
2014-08-08, by wenzelm
protocol command for heap management, e.g. in Isabelle/jEdit/Scala console: PIDE.session.protocol_command("ML_System.share_common_data");
2014-08-05, by wenzelm
added system option editor_output_delay: lower value might help big sessions under low-memory situations;
2014-08-05, by wenzelm
obsolete (see f7700146678d);
2014-08-05, by wenzelm
tuned proofs -- fewer warnings;
2014-08-05, by wenzelm
clarified Element.init vs. Element.init' -- the latter also avoids redundant warnings due to declatations when preparing locale expressions / interpretations;
2014-08-05, by wenzelm
avoid duplication of warnings stemming from simp/intro declarations etc.;
2014-08-05, by wenzelm
tuned proofs;
2014-08-05, by wenzelm
restrict edit_command (for sendback) to current node -- no attempt to goto target buffer first, which might not be loaded;
2014-08-05, by wenzelm
tuned;
2014-08-05, by wenzelm
more careful treatment of context visibility for rule declarations (see also 39d9c7f175e0, e639d91d9073) -- avoid duplicate warnings;
2014-08-05, by wenzelm
refined context visibility again (amending f5f9fad3321c, 8e3e004f1c31): avoid spurious warning due to global config options;
2014-08-05, by wenzelm
even more thorough reset on mouse drag (see also 0c63f3538639, 7e8c11011fdf);
2014-08-04, by wenzelm
tuned;
2014-08-04, by wenzelm
tuned;
2014-08-04, by wenzelm
Added tag Isabelle2014-RC2 for changeset ee908fccabc2
2014-08-04, by wenzelm
more user aliases;
2014-08-04, by wenzelm
registered Haskabelle-2014
2014-08-04, by noschinl
tuned, so codegen runs with current isabelle again
2014-08-01, by Lars Noschinski
tuned whitespace;
2014-08-03, by wenzelm
more robust popup geometry vs. formatted margin;
2014-08-03, by wenzelm
tuned message;
2014-08-03, by wenzelm
updated URL;
2014-08-02, by wenzelm
tuned;
2014-08-02, by wenzelm
updated URL;
2014-08-02, by wenzelm
more emphatic warning via error_message (violating historic TTY protocol);
2014-08-02, by wenzelm
proper priority for error over warning also for node_status (see 9c5220e05e04);
2014-08-02, by wenzelm
more direct access to persistent blobs (see also 8953d4cc060a), avoiding fragile digest lookup from later version (which might have removed unused blobs already);
2014-08-02, by wenzelm
always resolve symlinks for local files, e.g. relevant for ML_file to load proper source via editor instead of stored file via prover;
2014-08-02, by wenzelm
tuned output;
2014-08-02, by wenzelm
prefer non-strict Execution.print, e.g relevant for redirected ML compiler reports after error (see also e79f76a48449 and 40274e4f5ebf);
2014-08-01, by wenzelm
careful when calling 'Thm.proof_body_of' -- it can throw exceptions
2014-08-01, by blanchet
removed unused stuff;
2014-08-01, by wenzelm
agree on keyword categories with ML;
2014-08-01, by wenzelm
more keyword categories (as in ML);
2014-08-01, by wenzelm
prefer dynamic ML_print_depth if context happens to be available;
2014-07-31, by wenzelm
completion popup supports both ENTER and TAB (default);
2014-07-31, by wenzelm
clarified compile-time use of ML_print_depth;
2014-07-31, by wenzelm
more general notion of "user error" including empty message -- NB: Output.error_message needs non-empty string to emit anything;
2014-07-31, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
tip