src/HOL/Tools/recdef.ML
Mon, 06 Apr 2015 17:06:48 +0200 wenzelm @{command_spec} is superseded by @{command_keyword};
Tue, 31 Mar 2015 00:11:54 +0200 wenzelm tuned signature;
Fri, 07 Nov 2014 22:15:51 +0100 wenzelm eliminated pointless check -- command definitions are subject to theory context;
Wed, 29 Oct 2014 17:01:44 +0100 wenzelm modernized setup;
Wed, 27 Aug 2014 14:54:32 +0200 wenzelm more explicit Method.modifier with reported position;
Thu, 21 Aug 2014 22:48:39 +0200 wenzelm tuned signature -- define some elementary operations earlier;
Tue, 19 Aug 2014 23:17:51 +0200 wenzelm tuned signature -- moved type src to Token, without aliases;
Sat, 16 Aug 2014 22:14:57 +0200 wenzelm updated to named_theorems;
Sat, 22 Mar 2014 15:58:27 +0100 wenzelm avoid hard-wired theory names;
Tue, 18 Mar 2014 11:27:09 +0100 wenzelm tuned signature;
Mon, 10 Mar 2014 18:06:23 +0100 wenzelm clarified Args.check_src: retain name space information for error output;
Mon, 10 Mar 2014 16:30:07 +0100 wenzelm clarified Args.src: more abstract type, position refers to name only;
Sat, 08 Mar 2014 21:08:10 +0100 wenzelm modernized Attrib.check_name/check_src similar to methods (see also a989bdaf8121);
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Mon, 26 Nov 2012 14:43:28 +0100 wenzelm tuned command descriptions;
Fri, 27 Apr 2012 22:47:30 +0200 wenzelm clarified signature;
Wed, 21 Mar 2012 21:06:31 +0100 wenzelm optional 'includes' element for long theorem statements;
Fri, 16 Mar 2012 18:20:12 +0100 wenzelm outer syntax command definitions based on formal command_spec derived from theory header declarations;
Thu, 15 Mar 2012 20:07:00 +0100 wenzelm prefer formally checked @{keyword} parser;
Thu, 15 Mar 2012 19:02:34 +0100 wenzelm declare minor keywords via theory header;
Wed, 11 Jan 2012 16:23:59 +0100 wenzelm refer to imp_cong from HOL, not Drule (!) -- cf. 4ed94d92ae19;
Wed, 23 Nov 2011 22:59:39 +0100 wenzelm modernized some old-style infix operations, which were left over from the time of ML proof scripts;
Tue, 02 Aug 2011 10:36:50 +0200 krauss moved recdef package to HOL/Library/Old_Recdef.thy
Wed, 08 Jun 2011 15:56:57 +0200 wenzelm more robust exception pattern General.Subscript;
Fri, 13 May 2011 23:58:40 +0200 wenzelm clarified map_simpset versus Simplifier.map_simpset_global;
Thu, 12 May 2011 23:23:48 +0200 wenzelm prefer Proof.context over old-style claset/simpset;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
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;
Mon, 17 May 2010 23:54:15 +0200 wenzelm prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
Sun, 16 May 2010 00:02:11 +0200 wenzelm prefer structure Parse_Spec;
Wed, 12 May 2010 15:25:58 +0200 wenzelm updated/unified some legacy warnings;
Mon, 03 May 2010 14:25:56 +0200 wenzelm renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
Fri, 12 Mar 2010 12:14:30 +0100 bulwahn refining and adding Spec_Rules to definitional packages old_primrec, primrec, recdef, size and function
Wed, 10 Mar 2010 15:29:22 +0100 haftmann recdef is legacy
Thu, 21 Jan 2010 14:13:21 +0100 bulwahn corrected and simplified Spec_Rules registration in the Recdef package
Wed, 20 Jan 2010 18:02:22 +0100 bulwahn added registration of equational theorems from prim_rec and rec_def to Spec_Rules
Sun, 15 Nov 2009 19:44:29 +0100 wenzelm permissive AList.merge -- most likely setup for theory data (beware of spurious AList.DUP);
Thu, 12 Nov 2009 22:02:11 +0100 wenzelm eliminated obsolete "internal" kind -- collapsed to unspecific "";
Tue, 10 Nov 2009 15:33:35 +0100 wenzelm removed unused Quickcheck_RecFun_Simps;
Sun, 08 Nov 2009 18:43:42 +0100 wenzelm adapted Theory_Data;
Sun, 08 Nov 2009 16:30:41 +0100 wenzelm adapted Generic_Data, Proof_Data;
Wed, 28 Oct 2009 16:25:27 +0100 wenzelm conceal internal bindings;
Wed, 21 Oct 2009 17:34:35 +0200 blanchet renamed "nitpick_const_xxx" attributes to "nitpick_xxx" and "nitpick_ind_intros" to "nitpick_intros"
Thu, 15 Oct 2009 23:28:10 +0200 wenzelm replaced String.concat by implode;
Fri, 02 Oct 2009 23:15:36 +0200 wenzelm eliminated dead code;
Thu, 23 Jul 2009 18:44:09 +0200 wenzelm renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
Tue, 21 Jul 2009 01:03:18 +0200 wenzelm proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
Thu, 02 Jul 2009 17:34:14 +0200 wenzelm renamed NamedThmsFun to Named_Thms;
Fri, 19 Jun 2009 17:23:21 +0200 haftmann discontinued ancient tradition to suffix certain ML module names with "_package"
less more (0) tip