src/Pure/Isar/toplevel.ML
Tue, 26 Feb 2013 19:44:26 +0100 wenzelm fork diagnostic commands (theory loader and PIDE interaction);
Tue, 26 Feb 2013 13:27:24 +0100 wenzelm tuned 2464ba6e6fc9 -- NB: approximative_id is NONE for PIDE document transactions;
Tue, 26 Feb 2013 11:57:19 +0100 wenzelm tuned;
Mon, 25 Feb 2013 13:29:19 +0100 wenzelm discontinued pointless command category "thy_schematic_goal" -- this is checked dynamically;
Mon, 25 Feb 2013 12:52:27 +0100 wenzelm clarified Toplevel.element_result: scheduling policies happen here;
Sun, 24 Feb 2013 17:29:55 +0100 wenzelm simplified Outer_Syntax.read_span: internalized Toplevel.is_ignored;
Fri, 22 Feb 2013 16:52:10 +0100 wenzelm make SML/NJ happy;
Fri, 22 Feb 2013 14:38:52 +0100 wenzelm eliminated hard tabs;
Thu, 21 Feb 2013 10:52:14 +0100 wenzelm highest priority for proofs with unknown / very short timing -- recover original scheduling with parallel_proofs_reuse_timing = false;
Wed, 20 Feb 2013 15:22:22 +0100 wenzelm more tight representation of command timing;
Wed, 20 Feb 2013 11:40:30 +0100 wenzelm proper check of Proof.is_relevant (again, cf. c3e99efacb67 and df8fc0567a3d);
Tue, 19 Feb 2013 17:55:26 +0100 wenzelm improved scheduling of forked proofs, based on elapsed time estimate (from last run via session log file);
Tue, 19 Feb 2013 14:47:57 +0100 wenzelm suppress timing message in full PIDE protocol -- this is for batch build;
Tue, 19 Feb 2013 12:58:32 +0100 wenzelm support for prescient timing information within command transactions;
Tue, 19 Feb 2013 10:55:11 +0100 wenzelm emit command_timing properties into build log;
Wed, 16 Jan 2013 21:49:56 +0100 wenzelm tuned signature;
Sat, 05 Jan 2013 17:38:54 +0100 wenzelm more precise Local_Theory.level: 1 really means main target and >= 2 nested context;
Sun, 25 Nov 2012 19:49:24 +0100 wenzelm Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
Tue, 16 Oct 2012 15:14:12 +0200 wenzelm more informative errors for 'proof' and 'apply' steps;
Sat, 01 Sep 2012 19:43:18 +0200 wenzelm discontinued complicated/unreliable notion of recent proofs within context;
Fri, 31 Aug 2012 16:35:30 +0200 wenzelm more precise register_proofs for local goals;
Thu, 30 Aug 2012 21:23:04 +0200 wenzelm refined treatment of forked proofs at transaction boundaries, including proof commands (see also 7ee000ce5390);
Thu, 30 Aug 2012 19:18:49 +0200 wenzelm some support for registering forked proofs within Proof.state, using its bottom context;
Thu, 30 Aug 2012 16:39:50 +0200 wenzelm tuned signature;
Wed, 29 Aug 2012 12:07:45 +0200 wenzelm tuned signature;
Wed, 29 Aug 2012 11:48:45 +0200 wenzelm renamed Position.str_of to Position.here;
Sat, 11 Aug 2012 19:34:36 +0200 wenzelm vacuous execution after first malformed command;
Wed, 01 Aug 2012 15:33:08 +0200 wenzelm recovered comination of Toplevel.skip_proofs and Goal.parallel_proofs from 9679bab23f93 (NB: skip_proofs leads to failure of Toplevel.proof_of);
Thu, 17 May 2012 15:23:00 +0200 wenzelm tuned error -- reduce potential for confusion in a higher-level context, e.g. partial checking of theory sub-graph;
Wed, 11 Apr 2012 15:02:48 +0200 wenzelm clarified proof_result: finish proof formally via head tr, not end_tr;
Tue, 10 Apr 2012 22:53:41 +0200 wenzelm misc tuning and simplification;
Tue, 10 Apr 2012 21:31:05 +0200 wenzelm static relevance of proof via syntax keywords;
Mon, 02 Apr 2012 19:10:52 +0200 wenzelm misc tuning and simplification;
Wed, 21 Mar 2012 23:26:35 +0100 wenzelm more explicit Toplevel.open_target/close_target;
Fri, 16 Mar 2012 14:42:11 +0100 wenzelm defer actual parsing of command spans and thus allow new commands to be used in the same theory where defined;
Mon, 28 Nov 2011 22:05:32 +0100 wenzelm separate module for concrete Isabelle markup;
Mon, 14 Nov 2011 16:52:19 +0100 wenzelm pass positions for named targets, for formal links in the document model;
Fri, 19 Aug 2011 23:25:47 +0200 wenzelm maintain recent future proofs at transaction boundaries;
Thu, 18 Aug 2011 17:53:32 +0200 wenzelm more careful treatment of exception serial numbers, with propagation to message channel;
Mon, 15 Aug 2011 20:38:16 +0200 wenzelm tuned error message;
Sat, 13 Aug 2011 21:06:01 +0200 wenzelm clarified Toplevel.end_theory;
Sat, 13 Aug 2011 20:49:41 +0200 wenzelm simplified Toplevel.init_theory: discontinued special name argument;
Sat, 13 Aug 2011 20:41:29 +0200 wenzelm simplified Toplevel.init_theory: discontinued special master argument;
Sat, 13 Aug 2011 20:20:36 +0200 wenzelm provide node header via Scala layer;
Tue, 05 Jul 2011 20:36:49 +0200 wenzelm get theory from last executation state;
Tue, 05 Jul 2011 19:45:59 +0200 wenzelm explicit exit_transaction with Theory.end_theory (which could include sanity checks as in HOL-SPARK for example);
Tue, 05 Jul 2011 11:16:37 +0200 wenzelm tuned signature;
Sat, 16 Apr 2011 15:47:52 +0200 wenzelm modernized structure Proof_Context;
Sat, 26 Mar 2011 21:45:29 +0100 wenzelm present theory content as future, depending on intermediate proof state futures -- potential to reduce memory requirements and improve parallelization;
Sun, 20 Mar 2011 21:28:11 +0100 wenzelm structure Timing: covers former start_timing/end_timing and Output.timeit etc;
Fri, 04 Feb 2011 17:11:00 +0100 wenzelm parallelization of nested Isar proofs is subject to Goal.parallel_proofs_threshold;
Mon, 31 Jan 2011 23:02:53 +0100 wenzelm tuned signature;
Mon, 31 Jan 2011 22:57:01 +0100 wenzelm support named tasks, for improved tracing;
Thu, 13 Jan 2011 17:34:45 +0100 wenzelm Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
Sat, 04 Dec 2010 21:26:55 +0100 wenzelm formal notepad without any result;
Mon, 25 Oct 2010 21:06:56 +0200 wenzelm renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
Fri, 17 Sep 2010 22:17:57 +0200 wenzelm discontinued Output.debug, which belongs to early PGIP experiments (b6788dbd2ef9) and causes just too many problems (like spamming the message channel if it is used by more than one module);
Fri, 10 Sep 2010 23:11:58 +0200 wenzelm avoid extra wrapping for interrupts;
Thu, 09 Sep 2010 18:18:34 +0200 wenzelm removed dead code;
Thu, 09 Sep 2010 17:20:27 +0200 wenzelm more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
Tue, 31 Aug 2010 23:46:49 +0200 wenzelm moved Toplevel.run_command to Pure/PIDE/document.ML;
Mon, 30 Aug 2010 16:49:41 +0200 wenzelm Toplevel.run_command: more careful treatment of interrupts stemming from nested multi-exceptions etc.;
Mon, 30 Aug 2010 15:19:39 +0200 wenzelm tuned messages: discontinued spurious full-stops (messages are occasionally composed unexpectedly);
Wed, 25 Aug 2010 21:31:22 +0200 wenzelm added some proof state markup, notably number of subgoals (e.g. for indentation);
Thu, 12 Aug 2010 13:42:13 +0200 haftmann named target is optional; explicit Name_Target.reinit
Thu, 12 Aug 2010 13:28:18 +0200 haftmann Named_Target.init: empty string represents theory target
Thu, 12 Aug 2010 13:23:46 +0200 haftmann Named_Target.theory_init
Wed, 11 Aug 2010 20:25:44 +0200 haftmann merged
Wed, 11 Aug 2010 17:16:02 +0200 haftmann avoid arcane Local_Theory.reinit entirely
Wed, 11 Aug 2010 18:17:53 +0200 wenzelm merged
Wed, 11 Aug 2010 14:45:38 +0200 haftmann renamed Theory_Target to the more appropriate Named_Target
Wed, 11 Aug 2010 18:11:07 +0200 wenzelm removed obsolete Toplevel.enter_proof_body;
Sun, 08 Aug 2010 19:36:31 +0200 wenzelm explicitly distinguish Output.status (essential feedback) vs. Output.report (useful markup);
Tue, 27 Jul 2010 22:00:26 +0200 wenzelm simplified/clarified theory loader: more explicit task management, kill old versions at start, commit results only in the very end, non-optional master dependency, do not store text in deps;
Sun, 25 Jul 2010 14:41:48 +0200 wenzelm simplified handling of theory begin/end wrt. toplevel and theory loader;
Sat, 24 Jul 2010 21:40:48 +0200 wenzelm tuned;
Sat, 24 Jul 2010 21:22:21 +0200 wenzelm moved basic thy file name operations from Thy_Load to Thy_Header;
Sat, 24 Jul 2010 12:14:53 +0200 wenzelm moved management of auxiliary theory source files to Thy_Load -- as theory data instead of accidental loader state;
Thu, 22 Jul 2010 20:36:41 +0200 wenzelm tuned signature;
Thu, 22 Jul 2010 14:59:27 +0200 wenzelm eliminated some unreferenced identifiers;
Thu, 22 Jul 2010 14:01:43 +0200 wenzelm tuned;
Wed, 21 Jul 2010 13:25:14 +0200 wenzelm clarified/exported Future.worker_subgroup, which is already the default for Future.fork;
Tue, 20 Jul 2010 21:07:23 +0200 wenzelm avoid duplicate printing of 'theory' state (cf. 173974e07dea);
Tue, 20 Jul 2010 20:56:28 +0200 wenzelm toplevel pp for Proof.state and Toplevel.state;
Tue, 20 Jul 2010 18:33:19 +0200 wenzelm Topelevel.run_command: interactive mode for initial 'theory' ensures that Thy_Info.begin_theory loads parent theories;
Tue, 20 Jul 2010 14:44:33 +0200 wenzelm eliminated old-style sys_error/SYS_ERROR in favour of exception Fail -- after careful checking that there is no overlap with existing handling of that;
Mon, 05 Jul 2010 20:36:39 +0200 wenzelm async_state: report within proper transaction context;
Sun, 04 Jul 2010 21:01:22 +0200 wenzelm general Future.report -- also for Toplevel.async_state;
Sat, 03 Jul 2010 23:24:36 +0200 wenzelm run_command: actually observe "print" flag;
Sat, 03 Jul 2010 22:33:10 +0200 wenzelm Toplevel.run_command: asynchronous state output, as an attempt to address potentially slow pretty printing (e.g. in HOL/Bali);
Mon, 31 May 2010 21:06:57 +0200 wenzelm modernized some structure names, keeping a few legacy aliases;
Mon, 31 May 2010 16:45:48 +0200 wenzelm Toplevel.run_command: reraise Interrupt, to terminate the Isar_Document.execution and not store a failed attempt;
Sat, 15 May 2010 23:16:32 +0200 wenzelm refer directly to structure Keyword and Parse;
Mon, 26 Apr 2010 21:36:44 +0200 wenzelm proofs that are discontinued via 'oops' are treated as relevant --- for improved robustness of the final join of all proofs, which is hooked to results that are missing here;
Fri, 23 Apr 2010 21:00:28 +0200 wenzelm added keyword category "schematic goal", which prevents any attempt to fork the proof;
Thu, 18 Feb 2010 23:41:01 +0100 wenzelm removed unused Theory_Target.begin;
Tue, 17 Nov 2009 15:53:35 +0100 wenzelm init_theory: Runtime.controlled_execution for proper exception trace etc.;
Tue, 17 Nov 2009 14:51:32 +0100 wenzelm implicit name space grouping for theory/local_theory transactions;
Fri, 13 Nov 2009 21:11:15 +0100 wenzelm modernized structure Local_Theory;
Tue, 10 Nov 2009 23:18:03 +0100 wenzelm Toplevel.thread provides Isar-style exception output;
Tue, 10 Nov 2009 16:04:57 +0100 wenzelm modernized structure Theory_Target;
Sun, 08 Nov 2009 16:30:41 +0100 wenzelm adapted Generic_Data, Proof_Data;
Mon, 02 Nov 2009 21:03:41 +0100 wenzelm modernized structure Proof_Node;
Tue, 27 Oct 2009 13:16:16 +0100 wenzelm non-critical atomic accesses;
Wed, 30 Sep 2009 23:13:18 +0200 wenzelm eliminated dead code;
Tue, 29 Sep 2009 11:49:22 +0200 wenzelm explicit indication of Unsynchronized.ref;
Mon, 20 Jul 2009 00:37:39 +0200 wenzelm Proof.future_proof: declare all assumptions as well;
Sun, 19 Jul 2009 18:02:40 +0200 wenzelm more abstract Future.is_worker;
Sat, 06 Jun 2009 21:11:22 +0200 wenzelm moved Isar toplevel runtime support to runtime.ML, which is loaded early (before ml_compiler.ML);
Thu, 04 Jun 2009 17:31:39 +0200 wenzelm exn_message/raised: ML_Compiler.exception_position;
Mon, 30 Mar 2009 22:38:37 +0200 wenzelm added Toplevel.previous_node_of;
Sat, 21 Mar 2009 13:11:12 +0100 wenzelm restricted interrupts for tasks running as future worker thread -- attempt to prevent interrupt race conditions;
Wed, 18 Mar 2009 19:11:26 +0100 wenzelm reduced verbosity;
Wed, 11 Mar 2009 20:54:03 +0100 wenzelm debugging: special handling of EXCURSION_FAIL;
Tue, 10 Mar 2009 21:43:19 +0100 wenzelm controlled_execution/debugging: special handling of UNDEF to prevent it to appear in exception_trace;
Mon, 09 Mar 2009 21:26:13 +0100 wenzelm simplified presentation_context_of;
Sun, 08 Mar 2009 20:31:01 +0100 wenzelm simplified presentation: built into transaction, pass state directly;
Fri, 16 Jan 2009 15:20:31 +0100 wenzelm run_command: check theory name for init;
Thu, 15 Jan 2009 00:41:53 +0100 wenzelm added run_command (from isar_document.ML);
Sun, 11 Jan 2009 18:18:35 +0100 wenzelm added Goal.future_enabled abstraction -- now also checks that this is already
less more (0) -120 tip