src/Pure/Isar/isar_cmd.ML
Fri, 23 Aug 2013 20:35:50 +0200 wenzelm added Theory.setup convenience;
Sun, 07 Jul 2013 18:34:29 +0200 wenzelm discontinued command 'print_drafts';
Sat, 25 May 2013 15:37:53 +0200 wenzelm syntax translations always depend on context;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Sat, 30 Mar 2013 12:13:39 +0100 wenzelm item markup for Proof_Context.pretty_fact;
Sat, 05 Jan 2013 16:16:22 +0100 wenzelm tuned -- less indirection;
Wed, 17 Oct 2012 13:20:08 +0200 wenzelm more method position information, notably finished_pos after end of previous text;
Tue, 16 Oct 2012 20:23:00 +0200 wenzelm more proof method text position information;
Wed, 26 Sep 2012 14:23:33 +0200 wenzelm tuned pretty_locale/print_locale, with more basic pretty_locale_deps based on that;
Tue, 25 Sep 2012 15:40:41 +0200 wenzelm separate module Graph_Display;
Thu, 30 Aug 2012 21:23:04 +0200 wenzelm refined treatment of forked proofs at transaction boundaries, including proof commands (see also 7ee000ce5390);
Fri, 24 Aug 2012 12:35:39 +0200 wenzelm check side-comments of command spans (normally filtered out in Outer_Syntax.toplevel_source);
Wed, 22 Aug 2012 12:47:49 +0200 wenzelm clarified Parse.path vs. Parse.explode -- prefer errors in proper transaction context;
Tue, 14 Aug 2012 11:43:08 +0200 wenzelm support for 'typ' with explicit sort constraint;
Sat, 11 Aug 2012 22:17:46 +0200 wenzelm faster compilation of ML with antiquotations: static ML_context is bound once in auxiliary structure Isabelle;
Fri, 27 Apr 2012 22:47:30 +0200 wenzelm clarified signature;
Wed, 14 Mar 2012 17:52:38 +0100 wenzelm source positions for locale and class expressions;
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, 28 Oct 2011 22:17:30 +0200 wenzelm uniform Local_Theory.declaration with explicit params;
Sat, 20 Aug 2011 23:35:30 +0200 wenzelm refined Graph implementation: more abstract/scalable Graph.Keys instead of plain lists -- order of adjacency is now standardized wrt. Key.ord;
Mon, 27 Jun 2011 22:20:49 +0200 wenzelm document antiquotations are managed as theory data, with proper name space and entity markup;
Mon, 27 Jun 2011 16:53:31 +0200 wenzelm ML antiquotations are managed as theory data, with proper name space and entity markup;
Sat, 23 Apr 2011 13:53:09 +0200 wenzelm proper binding/report of defined simprocs;
Wed, 20 Apr 2011 13:54:07 +0200 wenzelm added Theory.nodes_of convenience;
Sat, 16 Apr 2011 15:47:52 +0200 wenzelm modernized structure Proof_Context;
Sat, 16 Apr 2011 15:25:25 +0200 wenzelm prefer local name spaces;
Sat, 16 Apr 2011 13:48:45 +0200 wenzelm Name_Space: proper configuration options long_names, short_names, unique_names instead of former unsynchronized references;
Wed, 06 Apr 2011 13:33:46 +0200 wenzelm typed_print_translation: discontinued show_sorts argument;
Wed, 06 Apr 2011 10:59:43 +0200 wenzelm renamed Standard_Syntax to Syntax_Phases;
Tue, 05 Apr 2011 23:14:41 +0200 wenzelm moved decode/parse operations to standard_syntax.ML;
Tue, 05 Apr 2011 14:25:18 +0200 wenzelm discontinued special treatment of structure Ast: no pervasive content, no inclusion in structure Syntax;
Sun, 03 Apr 2011 21:59:33 +0200 wenzelm added Position.reports convenience;
Thu, 06 Jan 2011 21:06:18 +0100 ballarin Diagnostic command to show locale dependencies.
Sun, 28 Nov 2010 16:15:31 +0100 wenzelm added 'syntax_declaration' command;
Sat, 27 Nov 2010 15:28:00 +0100 wenzelm more explicit Isabelle_System operations;
Sat, 06 Nov 2010 19:36:54 +0100 wenzelm mark 'cd' and 'commit' as control command -- not usable in asynchronous document model, likely to cause confusion in Proof General;
Mon, 20 Sep 2010 16:05:25 +0200 wenzelm renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
Fri, 17 Sep 2010 20:18:27 +0200 wenzelm tuned signature of (Context_)Position.report variants;
Mon, 06 Sep 2010 22:31:54 +0200 wenzelm discontinued obsolete ProofContext.prems_limit;
Fri, 03 Sep 2010 21:13:53 +0200 wenzelm pretty_goals: turned some global references and function arguments into configuration options (goals_limit = 10, goals_total = true, show_main_goal = false) depending on the context;
Mon, 30 Aug 2010 11:17:05 +0200 wenzelm tuned;
Wed, 11 Aug 2010 17:29:54 +0200 wenzelm prefer plain Attrib.eval_thms with plain Proof.context instead of Proof.state;
Tue, 03 Aug 2010 18:13:57 +0200 wenzelm eliminated Thy_Info.thy_ord, which is not really stable in interactive mode, since it depends on the somewhat accidental load order;
Sat, 31 Jul 2010 21:14:20 +0200 ballarin print_interps shows interpretations in proofs.
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;
Sun, 25 Jul 2010 12:57:29 +0200 wenzelm Thy_Load.check_loaded via Theory.at_end;
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;
Wed, 21 Jul 2010 15:23:46 +0200 wenzelm thm_deps/unused_thms: Context.get_theory based on proper theory ancestry, not accidental theory loader state;
Wed, 21 Jul 2010 13:55:44 +0200 wenzelm thy_deps: more direct comparison of sessions, which is presumably what "unfold" is meant to indicate here -- also avoid referring to accidental theory loader state;
Thu, 03 Jun 2010 22:17:36 +0200 wenzelm diagnostic commands 'ML_val' and 'ML_command' may refer to antiquotations @{Isar.state} and @{Isar.goal};
Mon, 31 May 2010 21:06:57 +0200 wenzelm modernized some structure names, keeping a few legacy aliases;
Sun, 30 May 2010 21:34:19 +0200 wenzelm replaced ML_Lex.read_antiq by more concise ML_Lex.read, which includes full read/report with explicit position information;
Thu, 27 May 2010 18:10:37 +0200 wenzelm renamed structure PrintMode to Print_Mode, keeping the old name as legacy alias for some time;
Sat, 15 May 2010 23:16:32 +0200 wenzelm refer directly to structure Keyword and Parse;
Sat, 08 May 2010 19:14:13 +0200 wenzelm unified/simplified Pretty.margin_default;
Sun, 25 Apr 2010 21:18:04 +0200 wenzelm replaced Sorts.rep_algebra by slightly more abstract selectors classes_of/arities_of;
Sun, 25 Apr 2010 15:52:03 +0200 wenzelm modernized naming conventions of main Isar proof elements;
Fri, 16 Apr 2010 22:18:59 +0200 wenzelm keep localized 'types' as regular non-old-style version -- 'type_abbrev' as 'type' just causes too many problems, e.g. clash with "type" in translations or "type:" argument syntax;
less more (0) -100 -60 tip