Thu, 10 Apr 2014 17:48:17 +0200 kuncar revert idiomatic handling of namings from 5a93b8f928a2 because in combination with Named_Target.theory_init global names are sometimes created
Thu, 10 Apr 2014 17:48:16 +0200 kuncar don't forget to init Interpretation and transfer theorems in the interpretation hook
Thu, 10 Apr 2014 17:48:16 +0200 kuncar export theorems
Thu, 10 Apr 2014 17:48:15 +0200 kuncar abstract Domainp in relator_domain rules => more natural statement of the rule
Thu, 10 Apr 2014 17:48:15 +0200 kuncar more appropriate name (Lifting.invariant -> eq_onp)
Thu, 10 Apr 2014 17:48:14 +0200 kuncar left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
Thu, 10 Apr 2014 17:48:13 +0200 kuncar tuned
Thu, 10 Apr 2014 15:14:38 +0200 traytel more accurate type arguments for intermeadiate typedefs
Thu, 10 Apr 2014 14:40:11 +0200 wenzelm merged
Thu, 10 Apr 2014 14:36:29 +0200 wenzelm ignore other_id reports for now (see 8eda56033203): massive amounts of redirections to 'class' etc. makes it difficult to edit main HOL;
Thu, 10 Apr 2014 14:27:35 +0200 wenzelm more standard names;
Thu, 10 Apr 2014 12:48:01 +0200 wenzelm modernized simproc_setup;
Thu, 10 Apr 2014 12:30:02 +0200 wenzelm modernized theory setup;
Thu, 10 Apr 2014 12:22:29 +0200 wenzelm added simproc markup, which also indicates legacy simprocs outside the name space;
Thu, 10 Apr 2014 12:00:25 +0200 wenzelm modernized simproc_setup;
Thu, 10 Apr 2014 11:24:58 +0200 wenzelm misc tuning;
Thu, 10 Apr 2014 11:06:45 +0200 wenzelm more contributors;
Thu, 10 Apr 2014 10:36:29 +0200 wenzelm tuned;
Thu, 10 Apr 2014 10:30:32 +0200 wenzelm NEWS;
Thu, 10 Apr 2014 10:27:29 +0200 wenzelm tuned error -- allow user to click on hyperlink to open remote file;
Thu, 10 Apr 2014 10:06:54 +0200 wenzelm no comment -- File.read_stream already enforces UTF8 (like HTML5) and HTTP servers often produce a wrong charset encoding;
Wed, 09 Apr 2014 23:22:58 +0200 wenzelm improved support for external URLs, based on standard Java network operations;
Wed, 09 Apr 2014 23:04:20 +0200 wenzelm basic URL operations (with Isabelle/Scala error handling);
Wed, 09 Apr 2014 20:58:32 +0200 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);
Wed, 09 Apr 2014 17:54:09 +0200 wenzelm allow text cartouches in regular outer syntax categories "text" and "altstring";
Wed, 09 Apr 2014 17:29:37 +0200 wenzelm tuned comments (see Scala version);
Wed, 09 Apr 2014 16:22:06 +0200 wenzelm dismiss popups more carefully (amending 7e8c11011fdf), notably allow mouse dragging within some tooltip, e.g. for text selection;
Wed, 09 Apr 2014 15:19:22 +0200 wenzelm clarifed results range;
Wed, 09 Apr 2014 15:03:07 +0200 wenzelm more explicit message discrimination;
Wed, 09 Apr 2014 13:32:34 +0200 wenzelm avoid confusion about pointless cursor movement with external links;
Wed, 09 Apr 2014 12:33:02 +0200 wenzelm prefer regular Goal_Display.pretty_goals, without censorship of options;
Wed, 09 Apr 2014 12:28:24 +0200 wenzelm more standard names;
Wed, 09 Apr 2014 12:22:57 +0200 wenzelm proper context for print_tac;
Wed, 09 Apr 2014 11:32:41 +0200 wenzelm more conventional tactic programming;
Wed, 09 Apr 2014 10:44:06 +0200 wenzelm tuned;
Thu, 10 Apr 2014 11:34:55 +0200 traytel reintroduce example (cf. 39281b3e4fac)
Thu, 10 Apr 2014 10:52:48 +0200 traytel use mutual clique information (cf. c451cf8b29c8) to make N2M more robust
Thu, 10 Apr 2014 09:38:38 +0200 traytel made N2M tactic more robust
Wed, 09 Apr 2014 18:40:21 +0200 blanchet generate cliques for 'prim(co)rec' N2M
Wed, 09 Apr 2014 18:22:11 +0200 blanchet thread mutual cliques through
Wed, 09 Apr 2014 13:15:21 +0200 hoelzl generalize ln/log_powr; add log_base_powr/pow
Wed, 09 Apr 2014 10:04:31 +0200 haftmann parametricity transfer rule for INFIMUM, SUPREMUM
Wed, 09 Apr 2014 09:37:49 +0200 hoelzl add divide_simps
Wed, 09 Apr 2014 09:37:48 +0200 hoelzl field_simps: better support for negation and division, and power
Wed, 09 Apr 2014 09:37:47 +0200 hoelzl revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
Tue, 08 Apr 2014 23:16:00 +0200 wenzelm merged
Tue, 08 Apr 2014 23:05:21 +0200 wenzelm more native rm_tree, using Java 7 facilities;
Tue, 08 Apr 2014 22:24:00 +0200 wenzelm expose more bad cases;
Tue, 08 Apr 2014 22:01:08 +0200 wenzelm tuned signature;
Tue, 08 Apr 2014 21:48:09 +0200 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);
Tue, 08 Apr 2014 20:03:00 +0200 wenzelm simplified Text.Chunk -- eliminated ooddities;
Tue, 08 Apr 2014 20:00:53 +0200 wenzelm tuned;
Tue, 08 Apr 2014 19:35:50 +0200 wenzelm more frugal Symbol.Index -- no need to waste space on mostly empty arrays;
Tue, 08 Apr 2014 19:17:28 +0200 wenzelm accumulate markup reports for "other" command ids, which are later retargeted and merged for rendering (in erratic order);
Tue, 08 Apr 2014 16:07:02 +0200 wenzelm avoid data redundancy;
Tue, 08 Apr 2014 15:12:54 +0200 wenzelm tuned signature -- moved Command.Chunk to Text.Chunk;
Tue, 08 Apr 2014 14:59:36 +0200 wenzelm more uniform ML/document antiquotations;
Tue, 08 Apr 2014 14:56:55 +0200 wenzelm obsolete;
Tue, 08 Apr 2014 14:15:48 +0200 wenzelm more positions and markup;
Tue, 08 Apr 2014 13:24:08 +0200 wenzelm more precise token positions;
Tue, 08 Apr 2014 12:31:17 +0200 wenzelm more uniform Command.Chunk operations;
Tue, 08 Apr 2014 12:19:33 +0200 wenzelm more explicit Command.Chunk types, less ooddities;
Tue, 08 Apr 2014 10:24:42 +0200 wenzelm tuned;
Tue, 08 Apr 2014 09:48:38 +0200 wenzelm ignore deps_changed (again) -- avoid proactive load attempts of unfinished header specification while the user is typing;
Tue, 08 Apr 2014 09:45:13 +0200 wenzelm no report for position singularity, notably for aux. file, especially empty one;
Mon, 07 Apr 2014 23:02:29 +0200 wenzelm simplified blob again (amending 1e77ed11f2f7): only store file node name, i.e. the raw editor file name;
Mon, 07 Apr 2014 21:23:02 +0200 wenzelm tuned signature -- prefer static type Document.Node.Name;
Tue, 08 Apr 2014 18:48:10 +0200 blanchet commented out example that triggers a bug
Tue, 08 Apr 2014 18:16:47 +0200 blanchet allow arguments to 'datatype_compat' in disorder
Tue, 08 Apr 2014 18:06:21 +0200 blanchet added 'datatype_compat' examples/tests
Tue, 08 Apr 2014 17:49:03 +0200 blanchet support deeply nested datatypes in 'datatype_compat'
Tue, 08 Apr 2014 13:47:27 +0200 blanchet preserve user type variable names to avoid mismatches/confusion
Tue, 08 Apr 2014 12:46:38 +0200 haftmann even more standardized doc session names after #b266e7a86485
Mon, 07 Apr 2014 16:37:57 +0200 wenzelm refrain from changing jEdit default shortcuts, due to potential for conflicts and actually not working on Mac OS X;
Mon, 07 Apr 2014 13:55:12 +0200 wenzelm support for URL as file name, similar to treatment in jEdit.java;
Mon, 07 Apr 2014 13:11:31 +0200 wenzelm provide old-style ISABELLE_SCALA_SCRIPT for uniformity;
Mon, 07 Apr 2014 13:06:34 +0200 wenzelm separate file_node vs. file_path, e.g. relevant on Windows for hyperlink to the latter;
Sun, 06 Apr 2014 21:01:45 +0200 nipkow merged
Sun, 06 Apr 2014 21:01:33 +0200 nipkow tuned lemmas: more general class
Sun, 06 Apr 2014 19:35:35 +0200 wenzelm tuned proofs;
Sun, 06 Apr 2014 19:16:34 +0200 wenzelm removed abbrev "<-" again (see c771f0fe28d1) due to conflict with important "<->" and "<-->";
Sun, 06 Apr 2014 17:19:08 +0200 nipkow merged
Sun, 06 Apr 2014 17:18:57 +0200 nipkow made field_simps "more complete"
Sun, 06 Apr 2014 17:09:32 +0200 wenzelm shell functions for all Isabelle executables;
Sun, 06 Apr 2014 16:59:41 +0200 wenzelm renamed "isabelle-process" to "isabelle_process", with shell function to avoid dynamic path lookups;
Sun, 06 Apr 2014 16:36:28 +0200 wenzelm more source positions;
Sun, 06 Apr 2014 15:51:02 +0200 wenzelm clarified position: no offset here;
Sun, 06 Apr 2014 15:43:45 +0200 wenzelm more source positions;
Sun, 06 Apr 2014 15:38:54 +0200 wenzelm approximate ML antiquotation @{here} for Isabelle/Pure bootstrap;
Sun, 06 Apr 2014 15:19:22 +0200 wenzelm clarified ML bootstrap;
Sun, 06 Apr 2014 14:30:26 +0200 wenzelm prepare "back" position for Navigator, before following hyperlink;
Sat, 05 Apr 2014 23:56:21 +0200 wenzelm tuned;
Sat, 05 Apr 2014 23:42:30 +0200 wenzelm merged
Sat, 05 Apr 2014 23:36:00 +0200 wenzelm more uniform build options;
Sat, 05 Apr 2014 23:17:30 +0200 wenzelm re-implemented build_doc in Isabelle/Scala;
Sat, 05 Apr 2014 22:37:17 +0200 wenzelm more standard Isabelle_System.tmp_file and tmp_dir operations, in accordance to ML version;
Sat, 05 Apr 2014 20:08:00 +0200 wenzelm more standard hash-bang (python *is* canonical according to Admin/PLATFORMS);
Sat, 05 Apr 2014 19:16:44 +0200 wenzelm tuned -- just one qualification of sections ("!");
Sat, 05 Apr 2014 19:16:16 +0200 wenzelm tuned error;
Sat, 05 Apr 2014 19:07:05 +0200 wenzelm proper settings instead of hard-wired information;
Sat, 05 Apr 2014 18:52:03 +0200 wenzelm explicit indication of important doc sections ("!"), which are expanded in the tree view;
Sat, 05 Apr 2014 18:14:54 +0200 wenzelm clarified Doc entry: more explicit path;
Sat, 05 Apr 2014 15:03:40 +0200 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);
Sat, 05 Apr 2014 11:37:00 +0200 haftmann closer correspondence of document and session names, while maintaining document names for external reference
Sat, 05 Apr 2014 17:52:29 +0100 paulson ignore jedit mark files
Sat, 05 Apr 2014 10:12:51 +0200 haftmann avoid romanism
Sat, 05 Apr 2014 10:03:04 +0200 haftmann churning pie charts (with non-canonical prerequisites!)
Sat, 05 Apr 2014 10:03:03 +0200 haftmann CONTRIBUTORS
Sat, 05 Apr 2014 10:01:07 +0200 haftmann proper inclusion into library
Sat, 05 Apr 2014 01:04:46 +0100 paulson A single [simp] to handle the case -a/-b.
Fri, 04 Apr 2014 22:51:22 +0200 wenzelm support for jEdit Navigator plugin;
Fri, 04 Apr 2014 22:21:46 +0200 wenzelm more permissive Session.update_options: this is wired to jEdit PropertiesChanged, which may occur before the prover is started;
Fri, 04 Apr 2014 19:09:56 +0200 blanchet added option to Mirabelle
Fri, 04 Apr 2014 17:58:25 +0100 paulson divide_minus_left divide_minus_right are in field_simps but are not default simprules
Thu, 03 Apr 2014 23:51:52 +0100 paulson removing simprule status for divide_minus_left and divide_minus_right
Fri, 04 Apr 2014 16:43:47 +0200 wenzelm merged;
Fri, 04 Apr 2014 15:58:20 +0200 wenzelm tuned rendering -- take 1px line border into account;
Fri, 04 Apr 2014 14:31:31 +0200 wenzelm revert ce37fcb30cf2 for the sake of Mac OS X -- let some event listeners of jEdit reset the cursor;
Fri, 04 Apr 2014 13:12:16 +0200 wenzelm tuned white space;
Fri, 04 Apr 2014 15:56:40 +0200 blanchet use Z3 TPTP cores rather than proofs since the latter are somewhat broken
Fri, 04 Apr 2014 14:44:51 +0200 blanchet tuned spaces
Fri, 04 Apr 2014 13:22:26 +0200 Andreas Lochbihler merged
Fri, 04 Apr 2014 13:22:15 +0200 Andreas Lochbihler add missing adaptation for narrowing to work with variables of type integer => integer
Fri, 04 Apr 2014 12:37:57 +0200 wenzelm merged
Fri, 04 Apr 2014 12:07:48 +0200 wenzelm added ML antiquotation @{print};
Fri, 04 Apr 2014 10:41:53 +0200 wenzelm afford larger full_index, to save a few milliseconds during rendering (notably text_overview);
Fri, 04 Apr 2014 11:49:47 +0200 blanchet improved parsing of "z3_tptp" proofs
Thu, 03 Apr 2014 22:04:57 +0200 wenzelm merged
Thu, 03 Apr 2014 21:55:48 +0200 wenzelm more direct warning within persistent Protocol.Status;
Thu, 03 Apr 2014 21:08:00 +0200 wenzelm clarified Version.syntax -- avoid guessing initial situation;
Thu, 03 Apr 2014 20:53:35 +0200 wenzelm more abstract Prover.Syntax, as proposed by Carst Tankink;
Thu, 03 Apr 2014 20:17:12 +0200 wenzelm tuned signature (see also 0850d43cb355);
Thu, 03 Apr 2014 19:49:53 +0200 wenzelm slightly more readable protocol trace (NB1: prover input is always marked as <prover_command/>; NB2: adding indentation would invalidate the XML);
Thu, 03 Apr 2014 19:26:39 +0200 wenzelm recovered public command_line from d92eb5c3960d, which is important for alternative prover processes;
Thu, 03 Apr 2014 18:39:42 +0200 wenzelm tuned rendering for 5 different look-and-feels;
Thu, 03 Apr 2014 15:40:31 +0200 wenzelm more symbol abbrevs, e.g. relevant for list comprehension in HOL/List.thy or HOL/Library/Monad_Syntax.thy;
Thu, 03 Apr 2014 14:54:17 +0200 wenzelm more general prover operations;
Thu, 03 Apr 2014 13:49:37 +0200 wenzelm tuned signature -- pro forma;
Thu, 03 Apr 2014 13:46:18 +0200 wenzelm more general prover operations;
Thu, 03 Apr 2014 17:26:45 +0100 paulson Merge
Thu, 03 Apr 2014 17:26:04 +0100 paulson Cleaned up some messy proofs
Thu, 03 Apr 2014 18:24:08 +0200 hoelzl fix #0556204bc230
Thu, 03 Apr 2014 17:56:08 +0200 hoelzl merged DERIV_intros, has_derivative_intros into derivative_intros
Thu, 03 Apr 2014 17:16:02 +0200 blanchet don't pass Vampire option that doesn't exist anymore (and that wasn't strictly necessary with older Vampires)
Thu, 03 Apr 2014 17:00:14 +0200 blanchet use Alt-Ergo 0.95.2, the latest and greatest version
Thu, 03 Apr 2014 16:57:19 +0200 blanchet updated Z3 TPTP to 4.3.1+
Thu, 03 Apr 2014 13:29:58 +0200 blanchet updated Why3 version in docs
Thu, 03 Apr 2014 10:51:24 +0200 blanchet added same idiomatic handling of namings for Ctr_Sugar/BNF-related interpretation hooks as for typedef and (old-style) datatypes
Thu, 03 Apr 2014 10:51:22 +0200 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
Thu, 03 Apr 2014 10:51:20 +0200 blanchet removed clone (cf. 300f613060b0)
Wed, 02 Apr 2014 20:41:44 +0200 wenzelm tuned signature -- more explicit iterator terminology;
Wed, 02 Apr 2014 20:22:12 +0200 wenzelm more explicit iterator terminology, in accordance to Scala 2.8 library;
Wed, 02 Apr 2014 18:35:07 +0200 hoelzl extend continuous_intros; remove continuous_on_intros and isCont_intros
Wed, 02 Apr 2014 18:35:02 +0200 hoelzl reorder Complex_Analysis_Basics; rename DD to deriv
Wed, 02 Apr 2014 18:35:01 +0200 hoelzl moved generic theorems from Complex_Analysis_Basic; fixed some theorem names
Wed, 02 Apr 2014 17:47:56 +0200 wenzelm merged;
Wed, 02 Apr 2014 17:39:47 +0200 wenzelm tuned rendering;
Wed, 02 Apr 2014 16:45:31 +0100 paulson new theorem about zero limits
Wed, 02 Apr 2014 16:34:37 +0100 paulson New theorems for extracting quotients
Wed, 02 Apr 2014 17:11:44 +0200 wenzelm more contributors;
Tue, 01 Apr 2014 14:24:28 +0200 Andreas Lochbihler document value generation for quickcheck's testers
Wed, 02 Apr 2014 13:53:32 +0200 wenzelm tuned whitespace;
Wed, 02 Apr 2014 13:54:50 +0200 wenzelm suppress slightly odd completion of "simp";
Wed, 02 Apr 2014 13:03:01 +0200 wenzelm observe extra line spacing for output as well;
Wed, 02 Apr 2014 12:26:11 +0200 wenzelm persistent protocol_status, to improve performance of node_status a little;
Wed, 02 Apr 2014 11:55:37 +0200 wenzelm more uniform painting of caret, which also improves visibility in invisible state;
Wed, 02 Apr 2014 11:08:16 +0200 wenzelm tuned rendering -- visual indication of the status range, to make more clear when information might is out of view;
Tue, 01 Apr 2014 23:04:22 +0200 wenzelm tuned for-comprehensions -- less structure mapping;
Tue, 01 Apr 2014 22:25:01 +0200 wenzelm some rephrasing to ensure that this becomes cheap "foreach" and not expensive "map" (cf. 0fc032898b05);
Tue, 01 Apr 2014 20:22:25 +0200 wenzelm more direct command states -- merge_results is hardly ever needed;
Tue, 01 Apr 2014 17:29:47 +0200 wenzelm unused;
Tue, 01 Apr 2014 17:26:32 +0200 wenzelm more frugal command_status, which is often used in a tight loop;
Tue, 01 Apr 2014 16:16:25 +0200 wenzelm simplified using "value class";
Tue, 01 Apr 2014 11:02:40 +0200 traytel more precise BNF bound for datatypes
Tue, 01 Apr 2014 10:51:29 +0200 blanchet compile
Tue, 01 Apr 2014 10:51:29 +0200 blanchet tuning
Tue, 01 Apr 2014 10:51:29 +0200 blanchet added new-style (co)datatype interpretation hook
Tue, 01 Apr 2014 10:51:29 +0200 blanchet added BNF interpretation hook
Tue, 01 Apr 2014 10:51:29 +0200 blanchet added 'ctr_sugar' interpretation hook
Tue, 01 Apr 2014 10:04:05 +0200 traytel tuned
Mon, 31 Mar 2014 21:15:26 +0200 wenzelm merged
Mon, 31 Mar 2014 21:13:51 +0200 wenzelm cumulative NEWS;
Mon, 31 Mar 2014 20:45:30 +0200 wenzelm observe focus change for all tooltips, e.g. relevant for focus change to unrelated components;
Mon, 31 Mar 2014 20:07:59 +0200 wenzelm clear active areas (notably mouse pointer) before changing context (e.g. via hyperlink);
Mon, 31 Mar 2014 18:28:35 +0200 wenzelm reset mouse pointer more decisively, for the sake of Mac OS X (despite the builtin policie of jEdit);
Mon, 31 Mar 2014 17:41:45 +0200 wenzelm proper structural hashCode, which is required for Command.File equals (NB: Array has physical object identity);
Mon, 31 Mar 2014 15:34:37 +0200 wenzelm tuned output;
Mon, 31 Mar 2014 15:28:14 +0200 wenzelm tuned signature -- more static typing;
Mon, 31 Mar 2014 15:05:24 +0200 wenzelm store blob content within document node: aux. files that were once open are made persistent;
Mon, 31 Mar 2014 12:35:39 +0200 wenzelm some shortcuts for chunks, which sometimes avoid bulky string output;
Mon, 31 Mar 2014 10:28:08 +0200 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;
Mon, 31 Mar 2014 17:17:37 +0200 hoelzl tuned proofs
Mon, 31 Mar 2014 12:32:15 +0200 hoelzl add complex_of_real coercion
Mon, 31 Mar 2014 12:16:39 +0200 hoelzl add limits of power at top and bot
Mon, 31 Mar 2014 12:16:37 +0200 hoelzl add connected_local_const
Mon, 31 Mar 2014 12:16:35 +0200 hoelzl add rules about infinity of intervals
Sun, 30 Mar 2014 21:24:59 +0200 wenzelm tuned proofs;
Sun, 30 Mar 2014 21:03:40 +0200 wenzelm immediate completion even with delay, which is the default according to 638b29331549;
Sun, 30 Mar 2014 20:23:26 +0200 wenzelm special treatment for various kinds of selections: imitate normal flow of editing;
Sat, 29 Mar 2014 21:26:11 +0100 wenzelm merged
Sat, 29 Mar 2014 20:41:50 +0100 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;
Sat, 29 Mar 2014 20:22:38 +0100 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;
Sat, 29 Mar 2014 12:42:24 +0100 wenzelm dismiss all popups on mouse drags, e.g. to avoid conflict of C-hover of Isabelle/jEdit and C-selection of jEdit;
Fri, 28 Mar 2014 18:21:07 -0700 huffman tuned proofs
Fri, 28 Mar 2014 18:21:20 -0700 huffman minimized imports
Sat, 29 Mar 2014 12:05:24 +0100 wenzelm merged
Sat, 29 Mar 2014 11:29:42 +0100 wenzelm tuned rendering -- change mouse pointer for active areas;
Sat, 29 Mar 2014 10:49:32 +0100 wenzelm propagate deps_changed, to resolve missing files without requiring jEdit events (e.g. buffer load/save);
Sat, 29 Mar 2014 10:17:09 +0100 wenzelm tuned signature;
Sat, 29 Mar 2014 09:34:51 +0100 wenzelm tuned signature;
Sat, 29 Mar 2014 09:24:39 +0100 wenzelm tuned -- see Text.Range.overlaps(Range);
Sat, 29 Mar 2014 11:41:39 +0100 nipkow tuned
Fri, 28 Mar 2014 21:17:47 +0100 wenzelm tuned;
Thu, 27 Mar 2014 21:38:45 +0100 wenzelm merged
Thu, 27 Mar 2014 21:18:14 +0100 wenzelm tuned -- avoid code duplication;
Thu, 27 Mar 2014 21:16:08 +0100 wenzelm tuned;
Thu, 27 Mar 2014 20:28:19 +0100 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);
Thu, 27 Mar 2014 19:47:30 +0100 wenzelm back to cumulative treatment of command status, which is important for total accounting (amending 8201790fdeb9);
Thu, 27 Mar 2014 18:42:53 +0100 wenzelm tuned;
Thu, 27 Mar 2014 17:56:13 +0100 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);
Thu, 27 Mar 2014 17:12:40 +0100 wenzelm clarified Isabelle/ML bootstrap, such that Execution does not require ML_Compiler;
Thu, 27 Mar 2014 13:00:40 +0100 wenzelm more frugal merge of markup trees: non-overlapping tree counts as empty;
Thu, 27 Mar 2014 12:11:32 +0100 wenzelm more frugal merge of markup trees: filter wrt. subsequent query;
Thu, 27 Mar 2014 11:19:31 +0100 wenzelm tuned signature;
Thu, 27 Mar 2014 10:43:43 +0100 wenzelm more careful treatment of multiple command states (eval + prints): merge content that is actually required;
Wed, 26 Mar 2014 21:01:09 +0100 wenzelm tuned signature -- expose less intermediate information;
Wed, 26 Mar 2014 20:32:15 +0100 wenzelm support to redirect report on asynchronous / non-strict print function (NB: not scalable due to bulky merge of markup trees);
Wed, 26 Mar 2014 20:08:07 +0100 wenzelm less markup by default -- this is stored persistently in Isabelle/Scala;
Wed, 26 Mar 2014 19:42:16 +0100 wenzelm clarified valid_id: always standardize towards static command.id;
Wed, 26 Mar 2014 14:41:52 +0100 wenzelm prefer Context_Position where a context is available;
Wed, 26 Mar 2014 14:15:34 +0100 wenzelm unused;
Wed, 26 Mar 2014 12:32:51 +0100 wenzelm more uniform Execution.fork vs. Execution.print;
Wed, 26 Mar 2014 12:15:42 +0100 wenzelm added Execution.print: accumulate print operations for some command execution, which are applied later and print time;
Wed, 26 Mar 2014 11:05:25 -0700 huffman tuned proofs
Wed, 26 Mar 2014 14:00:37 +0000 paulson Some useful lemmas
Wed, 26 Mar 2014 09:19:04 +0100 wenzelm tuned comments;
Wed, 26 Mar 2014 09:13:38 +0100 wenzelm tuned load order;
Wed, 26 Mar 2014 09:07:31 +0100 wenzelm superseded by (provide_)parse_files;
Wed, 26 Mar 2014 08:59:53 +0100 wenzelm tuned;
Tue, 25 Mar 2014 20:12:53 +0100 wenzelm merged
(0) -30000 -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 tip