src/Pure/Isar/code.ML
Wed, 01 Jan 2014 01:05:30 +0100 haftmann uniform bookkeeping also in the case of deletion
Tue, 31 Dec 2013 22:18:31 +0100 haftmann dropped unused material
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
Thu, 28 Nov 2013 08:35:14 +0100 haftmann prefer sort-stripping const_typ over Sign.the_const_type whenever appropriate
Thu, 28 Nov 2013 08:34:52 +0100 haftmann prefer name-normalizing devarify over unvarifyT whenever appropriate
Fri, 23 Aug 2013 20:35:50 +0200 wenzelm added Theory.setup convenience;
Tue, 30 Jul 2013 15:09:25 +0200 wenzelm type theory is purely value-oriented;
Sun, 28 Jul 2013 05:32:02 +0200 haftmann silenced subsumption warnings for default code equations entirely
Sat, 13 Jul 2013 17:53:58 +0200 haftmann attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
Fri, 28 Jun 2013 21:07:42 +0200 haftmann sort out code equations headed by a projection of a abstract datatype
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Wed, 10 Apr 2013 15:30:19 +0200 wenzelm more standard module name Axclass (according to file name);
Sat, 30 Mar 2013 13:40:19 +0100 wenzelm more item markup;
Fri, 29 Mar 2013 22:14:27 +0100 wenzelm Pretty.item markup for improved readability of lists of items;
Wed, 27 Mar 2013 14:19:18 +0100 wenzelm tuned signature and module arrangement;
Thu, 07 Mar 2013 15:02:55 +0100 wenzelm tuned signature -- prefer terminology of Scala and Axiom;
Mon, 22 Oct 2012 19:02:36 +0200 haftmann close code theorems explicitly after preprocessing
Thu, 18 Oct 2012 09:17:00 +0200 haftmann no sort constraints on datatype constructors in internal bookkeeping
Wed, 10 Oct 2012 08:45:27 +0200 haftmann more consistent error messages on malformed code equations
Mon, 24 Sep 2012 19:11:35 +0200 haftmann made smlnj even happier
Sun, 23 Sep 2012 08:24:19 +0200 haftmann make smlnj happy
Sat, 22 Sep 2012 21:59:40 +0200 haftmann more strict typscheme_equiv check: must fix variables of more specific type;
Sat, 22 Sep 2012 21:59:40 +0200 haftmann cache should not contain material from descendant theory
Thu, 23 Aug 2012 13:03:29 +0200 wenzelm prefer classic take_prefix/take_suffix over chop_while (cf. 0659e84bdc5f);
Tue, 05 Jun 2012 10:12:54 +0200 haftmann apply preprocessing simpset also to rhs of abstract code equations
Sun, 03 Jun 2012 15:49:55 +0200 haftmann explicit check for correct number of arguments for abstract constructor
Wed, 18 Apr 2012 21:11:50 +0200 haftmann tuned
Thu, 12 Apr 2012 10:29:45 +0200 Andreas Lochbihler generalise case certificates to allow ignored parameters
Sat, 18 Feb 2012 11:31:35 +0100 haftmann more explicit error on malformed abstract equation; dropped dead code; tuned signature
Mon, 26 Dec 2011 18:32:43 +0100 haftmann dropped disfruitful `constant signatures`
Wed, 09 Nov 2011 21:36:18 +0100 wenzelm misc tuning;
Sat, 05 Nov 2011 15:00:49 +0100 wenzelm added Logic.varify_types_global/unvarify_types_global, which avoids somewhat expensive Term.map_types;
Wed, 19 Oct 2011 23:07:48 +0200 haftmann removed some remaining artefacts of ancient SML code generator
Wed, 06 Jul 2011 20:46:06 +0200 wenzelm prefer Synchronized.var;
Sat, 02 Jul 2011 10:37:35 +0200 haftmann correction: do not assume that case const index covered all cases
Fri, 01 Jul 2011 23:31:23 +0200 haftmann remove illegal case combinators after merge
Fri, 01 Jul 2011 23:10:27 +0200 haftmann corrected misunderstanding what `old functions` are supposed to be
Fri, 01 Jul 2011 23:07:06 +0200 haftmann centralized deletion of equations for constructors; corrected misunderstanding what `old functions` are supposed to be
Fri, 01 Jul 2011 19:57:41 +0200 haftmann index cases for constructors
Thu, 09 Jun 2011 20:22:22 +0200 wenzelm tuned signature: Name.invent and Name.invent_names;
Thu, 09 Jun 2011 17:51:49 +0200 wenzelm simplified Name.variant -- discontinued builtin fold_map;
Fri, 06 May 2011 11:57:21 +0200 bulwahn improving merge of code specifications by removing code equations of constructors after merging two theories
Sun, 17 Apr 2011 19:54:04 +0200 wenzelm report Name_Space.declare/define, relatively to context;
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;
Mon, 10 Jan 2011 16:45:28 +0100 wenzelm added merge_options convenience;
Sat, 08 Jan 2011 17:14:48 +0100 wenzelm misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
Wed, 01 Dec 2010 15:03:44 +0100 wenzelm more direct use of binder_types/body_type;
Mon, 29 Nov 2010 11:38:59 +0100 haftmann tuned
Sat, 27 Nov 2010 22:01:27 +0100 haftmann typscheme with signatures is inappropriate when building empty certificate;
Sat, 27 Nov 2010 19:41:28 +0100 haftmann corrected: use canonical variables of type scheme uniformly
Fri, 26 Nov 2010 23:49:49 +0100 haftmann consider sort constraints for datatype constructors when constructing the empty equation certificate;
Fri, 26 Nov 2010 22:33:21 +0100 haftmann keep type variable arguments of datatype constructors in bookkeeping
Tue, 16 Nov 2010 10:33:36 +0100 haftmann added forall2 predicate lifter
Thu, 04 Nov 2010 17:27:38 +0100 haftmann Code.check_const etc.: reject too specific types
Wed, 03 Nov 2010 11:06:22 +0100 wenzelm replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
Tue, 26 Oct 2010 15:00:42 +0200 haftmann more general treatment of type argument in code certificates for operations on abstract types
Fri, 01 Oct 2010 10:25:36 +0200 haftmann chop_while replace drop_while and take_while
Thu, 30 Sep 2010 18:37:29 +0200 haftmann take_while, drop_while
Thu, 30 Sep 2010 08:50:45 +0200 haftmann corrected subsumption check: arguments have been reversed; addition of default equations to non-default equations is identity
less more (0) -100 -60 tip