src/HOL/Inductive.thy
Fri, 14 Mar 2014 15:41:29 +0100 wenzelm discontinued somewhat pointless "thy_script" keyword kind;
Thu, 20 Feb 2014 15:14:37 +0100 noschinl less flex-flex pairs
Wed, 19 Feb 2014 08:34:33 +0100 blanchet moved 'primrec' up (for real this time) and removed temporary 'old_primrec'
Mon, 17 Feb 2014 13:31:42 +0100 blanchet renamed old 'primrec' to 'old_primrec' (until the new 'primrec' can be moved above 'Nat' in the theory dependencies)
Mon, 02 Dec 2013 20:31:54 +0100 blanchet generalized datatype code generation code so that it works with old-style and new-style (co)datatypes (as long as they are not local)
Tue, 12 Nov 2013 13:47:24 +0100 blanchet moved 'Ctr_Sugar' further up the theory hierarchy, so that 'Datatype' can use it
Sat, 25 May 2013 15:37:53 +0200 wenzelm syntax translations always depend on context;
Wed, 10 Apr 2013 21:20:35 +0200 wenzelm tuned pretty layout: avoid nested Pretty.string_of, which merely happens to work with Isabelle/jEdit since formatting is delegated to Scala side;
Sat, 06 Apr 2013 01:42:07 +0200 traytel disallow coercions to interfere with case translations
Fri, 05 Apr 2013 22:08:42 +0200 traytel allow redundant cases in the list comprehension translation
Fri, 05 Apr 2013 22:08:42 +0200 traytel special constant to prevent eta-contraction of the check-phase syntax of case translations
Tue, 22 Jan 2013 14:33:45 +0100 traytel separate data used for case translation from the datatype package
Tue, 22 Jan 2013 13:32:41 +0100 berghofe case translations performed in a separate check phase (with adjustments by traytel)
Fri, 30 Nov 2012 22:55:02 +0100 wenzelm added 'print_inductives' command;
Wed, 22 Aug 2012 22:55:41 +0200 wenzelm prefer ML_file over old uses;
Thu, 19 Jul 2012 19:38:39 +0200 haftmann removed ML module DSeq which was a part of the ancient code generator (cf. 58e33a125f32)
Thu, 15 Mar 2012 22:08:53 +0100 wenzelm declare command keywords via theory header, including strict checking outside Pure;
Thu, 15 Mar 2012 19:02:34 +0100 wenzelm declare minor keywords via theory header;
Wed, 28 Dec 2011 20:03:13 +0100 wenzelm reverted some changes for set->predicate transition, according to "hg log -u berghofe -r Isabelle2007:Isabelle2008";
Sat, 17 Dec 2011 12:42:10 +0100 wenzelm clarified modules that contribute to datatype package;
Fri, 16 Dec 2011 12:03:33 +0100 wenzelm prefer Name.context operations;
Fri, 16 Dec 2011 10:52:35 +0100 wenzelm clarified modules that contribute to datatype package;
Thu, 15 Dec 2011 18:08:40 +0100 wenzelm clarified module dependencies: Datatype_Data, Datatype_Case, Rep_Datatype;
Thu, 15 Dec 2011 17:37:14 +0100 wenzelm separate rep_datatype.ML;
Sat, 10 Sep 2011 10:29:24 +0200 haftmann renamed theory Complete_Lattice to Complete_Lattices, in accordance with Lattices, Orderings etc.
Mon, 27 Jun 2011 17:04:04 +0200 krauss new Datatype.info_of_constr with strict behaviour wrt. to overloaded constructors -- side effect: function package correctly identifies 0::int as a non-constructor;
Thu, 09 Jun 2011 16:34:49 +0200 wenzelm discontinued Name.variant to emphasize that this is old-style / indirect;
Wed, 08 Dec 2010 14:52:23 +0100 haftmann tuned
Tue, 28 Sep 2010 15:39:59 +0200 haftmann dropped old primrec package
Thu, 10 Jun 2010 12:24:02 +0200 haftmann moved inductive_codegen to place where product type is available; tuned structure name
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.
less more (0) -100 -60 tip