src/HOL/Inductive.thy
Thu, 11 Feb 2010 23:00:22 +0100 wenzelm modernized translations;
Mon, 30 Nov 2009 11:42:49 +0100 haftmann modernized structures and tuned headers of datatype package modules; joined former datatype.ML and datatype_rep_proofs.ML
Mon, 30 Nov 2009 08:08:31 +0100 haftmann merged
Fri, 27 Nov 2009 08:41:10 +0100 haftmann renamed former datatype.ML to datatype_data.ML; datatype.ML provides uniform view on datatype.ML and datatype_rep_proofs.ML
Wed, 25 Nov 2009 11:16:57 +0100 haftmann bootstrap datatype_rep_proofs in Datatype.thy (avoids unchecked dynamic name references)
Fri, 27 Nov 2009 16:26:04 +0100 berghofe Streamlined setup for monotonicity rules (no longer requires classical rules).
Wed, 23 Sep 2009 14:00:43 +0200 haftmann merged
Sat, 19 Sep 2009 07:38:03 +0200 haftmann inter and union are mere abbreviations for inf and sup
Wed, 23 Sep 2009 12:03:47 +0200 haftmann stripped legacy ML bindings
Wed, 16 Sep 2009 13:43:05 +0200 haftmann Inter and Union are mere abbreviations for Inf and Sup
Mon, 06 Jul 2009 14:19:13 +0200 haftmann moved Inductive.myinv to Fun.inv; tuned
Tue, 23 Jun 2009 16:27:12 +0200 haftmann tuned interfaces of datatype module
Tue, 23 Jun 2009 12:09:30 +0200 haftmann uniformly capitialized names for subdirectories
Fri, 19 Jun 2009 17:23:21 +0200 haftmann discontinued ancient tradition to suffix certain ML module names with "_package"
Wed, 10 Jun 2009 15:04:33 +0200 haftmann separate directory for datatype package
Wed, 31 Dec 2008 20:31:36 +0100 wenzelm eliminated OldTerm.add_term_free_names;
Wed, 31 Dec 2008 18:53:16 +0100 wenzelm moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
Wed, 07 May 2008 10:56:35 +0200 berghofe Instantiated some rules to avoid problems with HO unification.
Wed, 30 Jan 2008 10:57:44 +0100 haftmann Theorem Inductive.lfp_ordinal_induct generalized to complete lattices
Thu, 06 Dec 2007 15:10:09 +0100 haftmann added new primrec package
Wed, 05 Dec 2007 14:15:45 +0100 haftmann simplified infrastructure for code generator operational equality
Fri, 30 Nov 2007 20:13:03 +0100 haftmann adjustions to due to instance target
Mon, 08 Oct 2007 22:03:25 +0200 haftmann integrated FixedPoint into Inductive
Thu, 04 Oct 2007 19:54:46 +0200 haftmann tuned datatype_codegen setup
Wed, 26 Sep 2007 19:17:55 +0200 wenzelm removed dead code;
Tue, 25 Sep 2007 12:16:08 +0200 haftmann datatype interpretators for size and datatype_realizer
Tue, 18 Sep 2007 07:46:00 +0200 haftmann introduced generic concepts for theory interpretators
Tue, 18 Sep 2007 07:36:38 +0200 haftmann separated code for inductive sequences from inductive_codegen.ML
Mon, 20 Aug 2007 18:10:13 +0200 nipkow Final mods for list comprehension
Wed, 11 Jul 2007 10:59:23 +0200 berghofe Added new package for inductive sets.
Tue, 10 Jul 2007 17:30:49 +0200 haftmann clarified import
Tue, 03 Jul 2007 15:23:11 +0200 nipkow Fixed problem with patterns in lambdas
Mon, 02 Jul 2007 23:14:06 +0200 nipkow Added pattern maatching for lambda abstraction
Thu, 14 Jun 2007 18:33:31 +0200 wenzelm tuned proofs: avoid implicit prems;
Wed, 09 May 2007 07:53:06 +0200 haftmann moved recfun_codegen.ML to Code_Generator.thy
Mon, 07 May 2007 00:49:59 +0200 wenzelm simplified DataFun interfaces;
Tue, 24 Apr 2007 15:18:42 +0200 berghofe Added datatype_case.
Wed, 31 Jan 2007 16:05:10 +0100 haftmann dropped lemma duplicates in HOL.thy
Fri, 13 Oct 2006 18:12:58 +0200 berghofe Added new package for inductive definitions, moved old package
Tue, 19 Sep 2006 15:22:35 +0200 haftmann added auxiliary lemma for code generation 2
Tue, 09 May 2006 10:09:37 +0200 haftmann added DatatypeHooks
Thu, 22 Dec 2005 00:28:34 +0100 wenzelm updated auxiliary facts for induct method;
Wed, 03 Aug 2005 14:48:13 +0200 avigad import FixedPoint instead of Gfp
Fri, 17 Jun 2005 16:12:49 +0200 haftmann migrated theory headers to new format
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 nipkow New theory header syntax.
Mon, 21 Jun 2004 10:25:57 +0200 kleing Merged in license change from Isabelle2004
Wed, 13 Nov 2002 15:25:17 +0100 berghofe Added InductiveRealizer package.
Wed, 07 Aug 2002 16:48:20 +0200 berghofe Added file Tools/datatype_realizer.ML
Thu, 21 Feb 2002 20:09:48 +0100 wenzelm include theory Record (tuned dependencies);
Mon, 10 Dec 2001 15:17:49 +0100 berghofe Moved code generator setup from Recdef to Inductive.
Sat, 03 Nov 2001 01:33:54 +0100 wenzelm tuned;
Wed, 31 Oct 2001 01:21:01 +0100 wenzelm use induct_rulify2;
Thu, 18 Oct 2001 20:59:59 +0200 wenzelm moved InductMethod.setup to theory HOL;
Thu, 04 Oct 2001 15:43:17 +0200 wenzelm generic induct_method.ML;
Sun, 22 Jul 2001 21:30:21 +0200 wenzelm tuned;
Fri, 20 Jul 2001 22:00:06 +0200 wenzelm private "myinv" (uses "The" instead of "Eps");
Tue, 22 May 2001 15:10:06 +0200 berghofe Inductive definitions are now introduced earlier in the theory hierarchy.
Tue, 30 Jan 2001 18:57:24 +0100 oheimb added if_def2
Fri, 22 Dec 2000 18:23:41 +0100 wenzelm added inductive_conj;
less more (0) -60 tip