src/HOL/HOL.thy
Sat, 15 May 2010 21:50:05 +0200 wenzelm less pervasive names from structure Thm;
Sat, 15 May 2010 17:59:06 +0200 wenzelm incorporated further conversions and conversionals, after some minor tuning;
Sun, 09 May 2010 19:15:21 +0200 wenzelm just one version of Thm.unconstrainT, which affects all variables;
Wed, 05 May 2010 18:25:34 +0200 haftmann farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
Tue, 04 May 2010 14:10:42 +0200 berghofe merged
Tue, 04 May 2010 12:26:46 +0200 berghofe induct_true_def and induct_false_def are already contained in induct_rulify_fallback.
Tue, 04 May 2010 08:55:43 +0200 haftmann locale predicates of classes carry a mandatory "class" prefix
Thu, 29 Apr 2010 22:56:32 +0200 wenzelm proper context for mksimps etc. -- via simpset of the running Simplifier;
Thu, 29 Apr 2010 15:00:41 +0200 haftmann avoid popular infixes
Wed, 28 Apr 2010 12:07:52 +0200 wenzelm renamed command 'defaultsort' to 'default_sort';
Mon, 26 Apr 2010 09:45:22 -0700 huffman merged
Mon, 26 Apr 2010 09:26:31 -0700 huffman syntax precedence for If and Let
Sun, 25 Apr 2010 23:09:32 +0200 wenzelm renamed Drule.unconstrainTs to Thm.unconstrain_allTs to accomdate the version by krauss/schropp;
Fri, 23 Apr 2010 19:36:04 +0200 wenzelm removed obsolete Named_Thm_Set -- Named_Thms provides efficient member operation;
Wed, 21 Apr 2010 12:10:52 +0200 bulwahn added peephole optimisations to the predicate compiler; added structure Predicate_Compile_Simps for peephole optimisations
Fri, 16 Apr 2010 21:28:09 +0200 wenzelm replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
Mon, 29 Mar 2010 14:49:53 +0200 blanchet reintroduce efficient set structure to collect "no_atp" theorems
Thu, 18 Mar 2010 12:58:52 +0100 blanchet now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
Wed, 17 Mar 2010 12:01:01 +0100 blanchet fix typo in "nitpick_choice_spec" attribute name (singular, not plural)
Wed, 17 Mar 2010 09:14:43 +0100 blanchet added support for "specification" and "ax_specification" constructs to Nitpick
Sun, 07 Mar 2010 12:19:47 +0100 wenzelm modernized structure Object_Logic;
Mon, 01 Mar 2010 13:42:31 +0100 haftmann merged
Mon, 01 Mar 2010 13:40:23 +0100 haftmann replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
Fri, 26 Feb 2010 21:43:26 +0100 wenzelm tuned hyp_subst_tac';
Thu, 25 Feb 2010 22:32:09 +0100 wenzelm more antiquotations;
Thu, 11 Feb 2010 23:00:22 +0100 wenzelm modernized translations;
Sun, 31 Jan 2010 15:22:40 +0100 berghofe merged
Sat, 30 Jan 2010 16:59:49 +0100 berghofe Added setup for simplification of equality constraints in cases rules.
Thu, 28 Jan 2010 11:48:49 +0100 haftmann new theory Algebras.thy for generic algebraic structures
Fri, 15 Jan 2010 14:43:00 +0100 berghofe merged
Sun, 10 Jan 2010 18:03:20 +0100 berghofe Added setup for simplification of equality constraints in induction rules.
Wed, 13 Jan 2010 08:56:15 +0100 haftmann some syntax setup for Scala
Mon, 11 Jan 2010 16:45:02 +0100 haftmann tuned code equations
Fri, 08 Jan 2010 14:34:17 +0100 haftmann boolean operators for scala
Fri, 08 Jan 2010 12:25:15 +0100 haftmann a primitive scala serializer
Wed, 30 Dec 2009 10:24:53 +0100 krauss killed a few warnings
Mon, 07 Dec 2009 16:27:48 +0100 haftmann split off evaluation mechanisms in separte module Code_Eval
Tue, 24 Nov 2009 17:19:33 +0100 wenzelm some rearangement of load order to keep preferences adjacent -- slightly fragile;
Thu, 19 Nov 2009 08:25:57 +0100 bulwahn replacing Predicate_Compile_Preproc_Const_Defs by more general Spec_Rules
Tue, 10 Nov 2009 15:33:35 +0100 wenzelm removed unused Quickcheck_RecFun_Simps;
Sun, 08 Nov 2009 19:15:37 +0100 wenzelm modernized structure Reorient_Proc;
Sun, 01 Nov 2009 15:44:26 +0100 wenzelm modernized structure Context_Rules;
Fri, 30 Oct 2009 18:32:40 +0100 haftmann tuned code setup
Thu, 29 Oct 2009 16:59:12 +0100 wenzelm modernized some structure names;
Thu, 29 Oct 2009 16:06:15 +0100 wenzelm separate ResBlacklist, based on scalable persistent data -- avoids inefficient hashing later on;
Mon, 26 Oct 2009 10:51:41 +0100 haftmann tuned code setup for primitive boolean connectors
Fri, 23 Oct 2009 17:12:36 +0200 haftmann turned off old quickcheck
Wed, 21 Oct 2009 17:34:35 +0200 blanchet renamed "nitpick_const_xxx" attributes to "nitpick_xxx" and "nitpick_ind_intros" to "nitpick_intros"
Tue, 20 Oct 2009 15:02:48 +0100 paulson Removal of the unused atpset concept, the atp attribute and some related code.
Tue, 29 Sep 2009 16:24:36 +0200 wenzelm explicit indication of Unsynchronized.ref;
Mon, 28 Sep 2009 23:13:37 +0200 wenzelm misc tuning and modernization;
Mon, 28 Sep 2009 22:47:34 +0200 wenzelm moved generic cong_tac from HOL/Tools/datatype_aux.ML to Tools/cong_tac.ML, proper subgoal selection (failure, not exception);
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn added first prototype of the extended predicate compiler
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn experimenting to add some useful interface for definitions
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn added predicate compile preprocessing structure for definitional thms -- probably is replaced by hooking the theorem command differently
Wed, 09 Sep 2009 11:31:20 +0200 haftmann moved eq handling in nbe into separate oracle
Wed, 26 Aug 2009 11:40:28 +0200 boehmes added further conversions and conversionals
Fri, 24 Jul 2009 21:21:45 +0200 wenzelm renamed functor BlastFun to Blast, require explicit theory;
Fri, 24 Jul 2009 18:58:58 +0200 wenzelm renamed functor ProjectRuleFun to Project_Rule;
Fri, 24 Jul 2009 12:33:00 +0200 wenzelm renamed functor InductFun to Induct;
less more (0) -300 -100 -60 tip