src/Tools/Code/code_thingol.ML
Wed, 07 Sep 2011 13:51:39 +0200 bulwahn removing previously used function locally_monomorphic in the code generator
Wed, 07 Sep 2011 13:51:38 +0200 bulwahn setting const_sorts to false in the type inference of the code generator
Wed, 07 Sep 2011 13:51:36 +0200 bulwahn removing previous crude approximation to add type annotations to disambiguate types
Wed, 07 Sep 2011 13:51:35 +0200 bulwahn adding minimalistic implementation for printing the type annotations
Wed, 07 Sep 2011 13:51:34 +0200 bulwahn adding call to disambiguation annotations
Wed, 07 Sep 2011 13:51:34 +0200 bulwahn adding type inference for disambiguation annotations in code equation
Wed, 07 Sep 2011 13:51:32 +0200 bulwahn adding the body type as well to the code generation for constants as it is required for type annotations of constants
Wed, 07 Sep 2011 13:51:30 +0200 bulwahn changing const type to pass along if typing annotations are necessary for disambigous terms
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;
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;
Mon, 30 May 2011 13:58:00 +0200 bulwahn improving heuristics of type annotations in contravariant positions for the special case with instances of the class partial_term_of
Mon, 18 Apr 2011 12:04:21 +0200 wenzelm simplified Sorts.class_error: plain Proof.context;
Mon, 18 Apr 2011 11:13:29 +0200 wenzelm simplified pretty printing context, which is only required for certain kernel operations;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Sat, 16 Apr 2011 15:25:25 +0200 wenzelm prefer local name spaces;
Fri, 08 Apr 2011 13:31:16 +0200 wenzelm explicit structure Syntax_Trans;
Thu, 17 Feb 2011 09:31:29 +0100 haftmann added is_IAbs; tuned brackets and comments
Tue, 21 Dec 2010 15:15:55 +0100 haftmann proper static closures
Tue, 21 Dec 2010 09:18:29 +0100 haftmann canonical handling of theory context argument
Wed, 15 Dec 2010 09:47:12 +0100 haftmann simplified evaluation function names
Mon, 13 Dec 2010 22:54:47 +0100 haftmann separated dictionary weakning into separate type
Thu, 09 Dec 2010 17:25:43 +0100 haftmann dictionary constants must permit explicit weakening of classes;
Wed, 01 Dec 2010 15:03:44 +0100 wenzelm more direct use of binder_types/body_type;
Fri, 26 Nov 2010 22:33:21 +0100 haftmann keep type variable arguments of datatype constructors in bookkeeping
Fri, 26 Nov 2010 12:03:18 +0100 haftmann globbing constant expressions use more idiomatic underscore rather than star
Mon, 20 Sep 2010 18:43:18 +0200 haftmann Pure equality is a regular cpde operation
Fri, 17 Sep 2010 11:05:53 +0200 haftmann proper closures for static evaluation; no need for FIXMEs any longer
Thu, 16 Sep 2010 16:51:34 +0200 haftmann separation of static and dynamic thy context
Wed, 15 Sep 2010 15:11:39 +0200 haftmann ignore code cache optionally
Tue, 07 Sep 2010 16:05:20 +0200 haftmann dropped outdated substitution
Fri, 27 Aug 2010 10:56:46 +0200 haftmann formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
Mon, 23 Aug 2010 11:51:32 +0200 haftmann preliminary versions of static_eval_conv(_simple)
Mon, 23 Aug 2010 11:09:49 +0200 haftmann refined and unified naming convention for dynamic code evaluation techniques
Wed, 21 Jul 2010 15:31:38 +0200 wenzelm replaced Thy_Info.the_theory by Context.this_theory -- avoid referring to accidental theory loader state;
Fri, 16 Jul 2010 13:57:46 +0200 haftmann don't fail gracefully
Thu, 08 Jul 2010 16:19:24 +0200 haftmann tuned titles
Mon, 05 Jul 2010 10:39:49 +0200 haftmann dropped passed irregular names
Fri, 02 Jul 2010 16:20:56 +0200 haftmann reverted to verion from fc27be4c6b1c
Fri, 02 Jul 2010 16:15:49 +0200 haftmann traceback for error messages
Wed, 30 Jun 2010 11:38:51 +0200 haftmann unfold_fun_n
Thu, 17 Jun 2010 15:59:46 +0200 haftmann explicit type variable arguments for constructors
Thu, 17 Jun 2010 11:33:04 +0200 haftmann transitive superclasses were also only a misunderstanding
Thu, 17 Jun 2010 10:57:00 +0200 haftmann formal introduction of transitive superclasses
Thu, 17 Jun 2010 10:51:38 +0200 haftmann dropped obscure type argument weakening mapping -- was only a misunderstanding
Tue, 15 Jun 2010 11:38:40 +0200 haftmann maintain cong rules for case combinators; more precise permissiveness
Tue, 15 Jun 2010 08:32:32 +0200 haftmann formal introduction of case cong
Mon, 14 Jun 2010 16:00:47 +0200 haftmann teaked naming of superclass projections
Mon, 07 Jun 2010 13:42:38 +0200 haftmann more consistent naming aroud type classes and instances
Mon, 31 May 2010 21:06:57 +0200 wenzelm modernized some structure names, keeping a few legacy aliases;
Mon, 17 May 2010 23:54:15 +0200 wenzelm prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
Wed, 21 Apr 2010 15:20:59 +0200 haftmann optionally ignore errors during translation of equations; tuned representation of abstraction points
Mon, 19 Apr 2010 15:31:58 +0200 haftmann more appropriate representation of valid positions for abstractors
Sun, 11 Apr 2010 13:08:14 +0200 wenzelm of_sort_derivation: pass-through full type information -- following the version by krauss/schropp;
Thu, 25 Mar 2010 21:27:04 +0100 wenzelm Sorts.of_sort_derivation: do not use slow Graph.irreducible_paths here, which not always needed (SUBTLE CHANGE IN SEMANTICS);
Sat, 20 Mar 2010 17:33:11 +0100 wenzelm renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
Mon, 22 Feb 2010 11:10:20 +0100 haftmann proper distinction of code datatypes and abstypes
Fri, 19 Feb 2010 11:06:21 +0100 haftmann a simple concept for datatype invariants
Wed, 13 Jan 2010 12:20:37 +0100 haftmann explicit abstract type of code certificates
Tue, 12 Jan 2010 16:27:42 +0100 haftmann code certificates as integral part of code generation
less more (0) -60 tip