src/HOL/HOL.thy
Mon, 02 Mar 2009 16:58:39 +0100 reduced confusion code_funcgr vs. code_wellsorted
Sat, 28 Feb 2009 14:52:21 +0100 moved generic intuitionistic prover to src/Tools/intuitionistic.ML;
Sat, 28 Feb 2009 14:02:12 +0100 moved some generic tools to src/Tools/ -- src/Provers is essentially obsolete;
Sun, 22 Feb 2009 22:32:50 +0100 experimental switch to new well-sorting algorithm
Sun, 22 Feb 2009 10:22:29 +0100 formal dependency on newly emerging algorithm
Fri, 20 Feb 2009 14:49:24 +0100 reverted to old wellsorting algorithm
Fri, 20 Feb 2009 10:14:31 +0100 experimental inclusion of new wellsorting algorithm for code equations
Wed, 18 Feb 2009 19:18:31 +0100 do not drop arguments to 0, 1
Tue, 10 Feb 2009 14:02:45 +0100 Renamed descriptions of Nitpick (and ATP) attributes, so that they fit well with the rest of the sentence in ProofGeneral.
Mon, 09 Feb 2009 12:31:36 +0100 Reintroduced nitpick_ind_intro attribute.
Mon, 09 Feb 2009 10:37:59 +0100 Added Nitpick_Const_Psimp attribute, dropped the 's' in Nitpick_Const_Simps, and killed the Nitpick_Ind_Intros attribute.
Fri, 06 Feb 2009 15:57:47 +0100 Added "nitpick_const_simps" and "nitpick_ind_intros" attributes for theorems;
Wed, 21 Jan 2009 23:40:23 +0100 no base sort in class import
Fri, 16 Jan 2009 08:29:11 +0100 added HOL-Base image
Mon, 15 Dec 2008 09:58:45 +0100 moved value.ML to src/Tools
Wed, 03 Dec 2008 15:58:44 +0100 made repository layout more coherent with logical distribution structure; stripped some $Id$s
Thu, 20 Nov 2008 00:03:47 +0100 Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
Thu, 13 Nov 2008 15:58:38 +0100 simproc for let
Tue, 28 Oct 2008 11:03:07 +0100 Removed 'includes meta_term_syntax' and 'includes meta_conjunction_syntax'.
Fri, 24 Oct 2008 17:48:34 +0200 "arbitrary" merely abbreviates undefined
Wed, 22 Oct 2008 14:15:45 +0200 code identifier namings are no longer imperative
Fri, 10 Oct 2008 06:45:53 +0200 `code func` now just `code`
Tue, 07 Oct 2008 16:07:16 +0200 re-introduces axiom subst
Mon, 29 Sep 2008 12:31:57 +0200 polished code generator setup
Thu, 25 Sep 2008 09:28:03 +0200 discontinued special treatment of op = vs. eq_class.eq
Mon, 22 Sep 2008 23:00:15 +0200 Added setup for coherent logic prover.
Tue, 16 Sep 2008 09:21:22 +0200 generic value command
Thu, 28 Aug 2008 22:09:20 +0200 restructured and split code serializer module
Wed, 27 Aug 2008 11:24:29 +0200 tuned code generator setup
Mon, 14 Jul 2008 17:47:18 +0200 single_hyp(_meta)_subst_tac: Controlled substitution of a single hyp
Tue, 24 Jun 2008 19:43:14 +0200 ML_Antiquote.value;
Mon, 23 Jun 2008 15:51:38 +0200 moved src/HOL/Tools/induct_tacs.ML to src/Tools/induct_tacs.ML;
Sat, 14 Jun 2008 23:20:03 +0200 removed obsolete case_split_tac -- cannot work without;
Tue, 10 Jun 2008 19:15:19 +0200 eliminated obsolete case_split_thm -- use case_split;
Tue, 10 Jun 2008 15:30:58 +0200 localized Least in Orderings.thy
Sun, 18 May 2008 17:03:20 +0200 eliminated theory CPure;
Thu, 24 Apr 2008 16:53:04 +0200 moved 'trivial classes' to foundation of code generator
Tue, 22 Apr 2008 22:00:25 +0200 different handling of eq class for nbe
Tue, 22 Apr 2008 08:33:16 +0200 constant HOL.eq now qualified
Tue, 15 Apr 2008 18:49:13 +0200 Sign.hide_const;
Tue, 08 Apr 2008 18:30:40 +0200 Generic conversion and tactic "atomize_elim" to convert elimination rules
Fri, 04 Apr 2008 13:40:21 +0200 postprocessing of equality
Wed, 02 Apr 2008 15:58:32 +0200 explicit class "eq" for operational equality
Sat, 29 Mar 2008 22:55:49 +0100 purely functional setup of claset/simpset/clasimpset;
Wed, 26 Mar 2008 22:40:01 +0100 pass imp_elim, swap to classical prover;
Fri, 25 Jan 2008 14:54:44 +0100 dropped superfluous code theorems
Wed, 02 Jan 2008 15:14:02 +0100 splitted class uminus from class minus
Sat, 22 Dec 2007 14:10:22 +0100 use random_word.ML earlier;
Wed, 05 Dec 2007 14:15:45 +0100 simplified infrastructure for code generator operational equality
Wed, 28 Nov 2007 16:44:18 +0100 replaced typedecl interpretation by ObjectLogic.typedecl (based on base_sort);
Fri, 23 Nov 2007 21:09:33 +0100 interpretation of typedecls: instantiation to class type
Sun, 11 Nov 2007 14:00:05 +0100 tuned specifications of 'notation';
Mon, 05 Nov 2007 22:50:00 +0100 move itself into HOL types
Tue, 16 Oct 2007 23:12:45 +0200 global class syntax
Mon, 08 Oct 2007 08:04:28 +0200 added first version of user-space type system for class target
Thu, 04 Oct 2007 19:54:44 +0200 certificates for code generator case expressions
Thu, 04 Oct 2007 19:42:03 +0200 clarified declarations in class ord
Thu, 04 Oct 2007 14:42:47 +0200 moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
Sat, 29 Sep 2007 08:58:51 +0200 proper syntax during class specification
Tue, 18 Sep 2007 18:05:34 +0200 moved Tools/integer.ML to Pure/General/integer.ML;