Sun, 18 Aug 2013 17:00:10 +0200 |
wenzelm |
merged
|
changeset |
files
|
Sun, 18 Aug 2013 15:59:48 +0200 |
wenzelm |
load_theories if continuous_checking;
|
changeset |
files
|
Sun, 18 Aug 2013 15:33:26 +0200 |
wenzelm |
discontinued redundant abbreviations -- Isabelle/jEdit provides keyboard shortcuts already;
|
changeset |
files
|
Sun, 18 Aug 2013 15:31:12 +0200 |
wenzelm |
prefer plain subscript;
|
changeset |
files
|
Sun, 18 Aug 2013 15:10:18 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Sun, 18 Aug 2013 15:35:01 +0200 |
haftmann |
spelling and typos
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
relaxed preconditions
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
type class for generic division algorithm on numerals
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
added lemma
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
added lemma
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
generalized sort constraint of lemmas
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
explicit conversion from and to bool, and into algebraic structures with 0 and 1
|
changeset |
files
|
Sun, 18 Aug 2013 15:29:50 +0200 |
haftmann |
some vague grouping of related theorems, with slight tuning of headings and sorting out of dubious lemmas into separate theory
|
changeset |
files
|
Sun, 18 Aug 2013 13:58:33 +0200 |
wenzelm |
more markup;
|
changeset |
files
|
Sun, 18 Aug 2013 13:28:06 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Sun, 18 Aug 2013 13:25:31 +0200 |
wenzelm |
updated identifier syntax;
|
changeset |
files
|
Sat, 17 Aug 2013 22:58:48 +0200 |
wenzelm |
Sledgehammer is docked on startup;
|
changeset |
files
|
Sat, 17 Aug 2013 22:45:48 +0200 |
wenzelm |
prefer system option sledgehammer_timeout, with standard GUI in jEdit Plugin Options;
|
changeset |
files
|
Sat, 17 Aug 2013 22:27:41 +0200 |
wenzelm |
more robust startup;
|
changeset |
files
|
Sat, 17 Aug 2013 22:15:45 +0200 |
wenzelm |
some protocol to determine provers according to ML;
|
changeset |
files
|
Sat, 17 Aug 2013 22:08:21 +0200 |
wenzelm |
public access for protocol handlers and protocol commands -- to be used within reason;
|
changeset |
files
|
Sat, 17 Aug 2013 19:54:16 +0200 |
wenzelm |
always enable "minimize" to simplify interaction model;
|
changeset |
files
|
Sat, 17 Aug 2013 19:13:28 +0200 |
wenzelm |
sledgehammer sendback always uses Markup.padding_command: sensible default for most practical applications -- old-style in-line replacement is superseded by auto mode or panel;
|
changeset |
files
|
Sat, 17 Aug 2013 14:13:18 +0200 |
wenzelm |
recovered Locale.intern from d51bac27d4a0 (still used in AFP/Simp);
|
changeset |
files
|
Sat, 17 Aug 2013 12:25:26 +0200 |
wenzelm |
NEWS;
|
changeset |
files
|
Sat, 17 Aug 2013 12:21:25 +0200 |
wenzelm |
eliminated pointless subgoal argument;
|
changeset |
files
|
Sat, 17 Aug 2013 12:13:53 +0200 |
wenzelm |
more direct sledgehammer configuration via mode = Normal_Result and output_result;
|
changeset |
files
|
Sat, 17 Aug 2013 11:34:50 +0200 |
wenzelm |
more explicit sendback propertries based on mode;
|
changeset |
files
|
Fri, 16 Aug 2013 23:11:51 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Fri, 16 Aug 2013 22:57:16 +0200 |
wenzelm |
check_tool wrt. official ISABELLE_TOOLS;
|
changeset |
files
|
Fri, 16 Aug 2013 22:39:31 +0200 |
wenzelm |
more markup via Name_Space.check;
|
changeset |
files
|
Fri, 16 Aug 2013 21:33:36 +0200 |
wenzelm |
more standard attribute_setup / method_setup -- export key ML operations instead of parsers;
|
changeset |
files
|
Fri, 16 Aug 2013 21:28:05 +0200 |
wenzelm |
standardized aliases;
|
changeset |
files
|
Fri, 16 Aug 2013 20:58:15 +0200 |
wenzelm |
more markup -- avoid old Locale.extern;
|
changeset |
files
|
Fri, 16 Aug 2013 19:03:31 +0200 |
blanchet |
renamed function
|
changeset |
files
|
Fri, 16 Aug 2013 18:56:33 +0200 |
blanchet |
eliminate quasi-duplicate function
|
changeset |
files
|
Fri, 16 Aug 2013 18:45:57 +0200 |
blanchet |
generalized "mk_permute"
|
changeset |
files
|
Fri, 16 Aug 2013 18:36:55 +0200 |
blanchet |
tuning
|
changeset |
files
|
Fri, 16 Aug 2013 18:14:58 +0200 |
blanchet |
added more functions to BNF library
|
changeset |
files
|
Fri, 16 Aug 2013 18:06:37 +0200 |
blanchet |
moved function to where it seems to belong
|
changeset |
files
|
Fri, 16 Aug 2013 18:04:39 +0200 |
blanchet |
moved library function where it belongs, and used Dmitriy's inside-out implementation
|
changeset |
files
|
Fri, 16 Aug 2013 16:48:46 +0200 |
blanchet |
added useful library function
|
changeset |
files
|
Fri, 16 Aug 2013 15:49:16 +0200 |
traytel |
tuned
|
changeset |
files
|
Fri, 16 Aug 2013 15:35:47 +0200 |
blanchet |
moved useful library functions upstream
|
changeset |
files
|
Fri, 16 Aug 2013 15:33:24 +0200 |
blanchet |
merge
|
changeset |
files
|
Wed, 14 Aug 2013 14:05:54 +0200 |
blanchet |
added fixme
|
changeset |
files
|
Wed, 14 Aug 2013 13:15:28 +0200 |
blanchet |
more (co)datatype documentation
|
changeset |
files
|
Wed, 14 Aug 2013 17:45:16 +0200 |
Andreas Lochbihler |
use nat_of_integer for term reconstruction instead of abstract constructor to allow reconstructed terms being fed back to the code generator
|
changeset |
files
|
Tue, 13 Aug 2013 18:22:55 +0200 |
traytel |
got rid of the dependency of Lifting_* on the function package; use the original rel constants for basic BNFs;
|
changeset |
files
|
Wed, 14 Aug 2013 00:15:03 +0200 |
blanchet |
more work on (co)datatype docs
|
changeset |
files
|
Tue, 13 Aug 2013 22:37:58 +0200 |
wenzelm |
more symbolic notation;
|
changeset |
files
|
Tue, 13 Aug 2013 22:25:24 +0200 |
wenzelm |
Completion popup based on javax.swing.PopupFactory, which has better cross-platform chances than JWindow (cf. org/gjt/jedit/gui/CompletionPopup.java);
|
changeset |
files
|
Tue, 13 Aug 2013 20:35:45 +0200 |
wenzelm |
merged
|
changeset |
files
|
Tue, 13 Aug 2013 20:34:46 +0200 |
wenzelm |
discontinued special treatment of \<^isub> and \<^isup> in rendering or editor front-end;
|
changeset |
files
|
Tue, 13 Aug 2013 19:52:12 +0200 |
wenzelm |
merged
|
changeset |
files
|
Tue, 13 Aug 2013 16:15:31 +0200 |
wenzelm |
more general window_geometry;
|
changeset |
files
|
Tue, 13 Aug 2013 19:57:57 +0200 |
blanchet |
added rail diagram
|
changeset |
files
|
Tue, 13 Aug 2013 17:45:22 +0200 |
wenzelm |
merged
|
changeset |
files
|
Tue, 13 Aug 2013 17:26:22 +0200 |
wenzelm |
disable old identifier syntax by default, legacy_isub_isup := true may be used temporarily as fall-back;
|
changeset |
files
|