src/HOL/Tools/typedef_package.ML
Fri, 30 Nov 2007 20:13:07 +0100 haftmann interpretation for typedefs
Wed, 28 Nov 2007 16:44:20 +0100 wenzelm ObjectLogic.typedecl;
Fri, 23 Nov 2007 21:09:30 +0100 haftmann separated typedecl module, providing typedecl command with interpretation
Tue, 09 Oct 2007 17:10:34 +0200 wenzelm AxClass.axiomatize: renamed XXX_i to XXX, and XXX to XXX_cmd;
Tue, 09 Oct 2007 00:20:13 +0200 wenzelm generic Syntax.pretty/string_of operations;
Sat, 06 Oct 2007 16:50:04 +0200 wenzelm simplified interfaces for outer syntax;
Fri, 05 Oct 2007 22:00:15 +0200 wenzelm tuned Induct interface: prefer pred'' over set'';
Thu, 04 Oct 2007 14:42:47 +0200 wenzelm moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
Tue, 25 Sep 2007 17:06:14 +0200 wenzelm proper Sign operations instead of Theory aliases;
Sat, 01 Sep 2007 15:47:01 +0200 wenzelm replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
Tue, 14 Aug 2007 13:20:12 +0200 wenzelm PrimitiveDefs.mk_defpair;
Mon, 07 May 2007 00:49:59 +0200 wenzelm simplified DataFun interfaces;
Tue, 28 Nov 2006 00:35:18 +0100 wenzelm simplified '?' operator;
Tue, 21 Nov 2006 18:07:30 +0100 wenzelm simplified Proof.theorem(_i);
Tue, 14 Nov 2006 15:29:52 +0100 wenzelm simplified Proof.theorem(_i) interface;
Tue, 14 Nov 2006 00:15:42 +0100 wenzelm removed legacy read/cert/string_of;
Wed, 06 Sep 2006 10:01:04 +0200 haftmann TypedefPackage.add_typedef_* now yields name of introduced type constructor
Fri, 01 Sep 2006 23:18:01 +0200 wenzelm signature: do not export private stuff;
Tue, 08 Aug 2006 08:20:24 +0200 haftmann fixed code generator theorem generation
Sat, 08 Jul 2006 12:54:33 +0200 wenzelm Goal.prove_global;
Wed, 24 May 2006 01:04:57 +0200 wenzelm simplified info/get_info;
Thu, 11 May 2006 19:19:31 +0200 wenzelm avoid raw equality on type thm;
Sun, 07 May 2006 00:22:05 +0200 wenzelm removed 'concl is' patterns;
Sun, 30 Apr 2006 22:50:03 +0200 wenzelm AxClass.axiomatize_arity_i;
Wed, 26 Apr 2006 22:38:05 +0200 wenzelm tuned;
Mon, 24 Apr 2006 16:37:52 +0200 haftmann seperated typedef codegen from main code
Mon, 10 Apr 2006 00:33:49 +0200 wenzelm Term.itselfT;
Thu, 06 Apr 2006 16:09:20 +0200 haftmann added functions for definitional code generation
Tue, 07 Feb 2006 19:56:45 +0100 wenzelm renamed gen_duplicates to duplicates;
Mon, 06 Feb 2006 11:01:28 +0100 haftmann subsituted gen_duplicates / has_duplicates for duplicates whenever appropriate
Fri, 27 Jan 2006 19:03:02 +0100 wenzelm moved theorem tags from Drule to PureThy;
Sat, 21 Jan 2006 23:02:14 +0100 wenzelm simplified type attribute;
Thu, 19 Jan 2006 21:22:08 +0100 wenzelm setup: theory -> theory;
Sat, 14 Jan 2006 17:14:06 +0100 wenzelm sane ERROR handling;
Tue, 10 Jan 2006 19:34:04 +0100 wenzelm generic attributes;
Fri, 09 Dec 2005 09:06:45 +0100 haftmann oriented result pairs in PureThy
Tue, 06 Dec 2005 09:04:09 +0100 haftmann re-oriented some result tuples in PureThy
Fri, 21 Oct 2005 18:14:34 +0200 wenzelm Goal.prove;
Wed, 19 Oct 2005 21:52:34 +0200 wenzelm removed obsolete add_typedef_x;
Thu, 15 Sep 2005 17:16:56 +0200 wenzelm TableFun/Symtab: curried lookup and update;
Tue, 13 Sep 2005 22:19:23 +0200 wenzelm tuned Isar interfaces;
Tue, 06 Sep 2005 16:59:55 +0200 wenzelm proper treatment of polymorphic sets;
Mon, 05 Sep 2005 17:38:18 +0200 wenzelm curried_lookup/update;
Thu, 25 Aug 2005 16:10:16 +0200 berghofe Implemented incremental code generation.
Tue, 16 Aug 2005 13:42:26 +0200 wenzelm OuterKeyword;
Fri, 01 Jul 2005 14:13:40 +0200 berghofe Adapted to modular code generation.
Mon, 20 Jun 2005 22:13:59 +0200 wenzelm get_thm(s): Name;
Fri, 17 Jun 2005 18:35:27 +0200 wenzelm accomodate change of TheoryDataFun;
Tue, 31 May 2005 11:53:17 +0200 wenzelm fixed outer syntax: allow type_args with parentheses;
Thu, 03 Mar 2005 12:43:01 +0100 skalberg Move towards standard functions.
Sun, 13 Feb 2005 17:15:14 +0100 skalberg Deleted Library.option type.
Mon, 24 Jan 2005 17:59:48 +0100 berghofe Adapted to modified interface of PureThy.get_thm(s).
Wed, 27 Oct 2004 10:30:07 +0200 berghofe Added type constraint to make SML/NJ happy.
Tue, 26 Oct 2004 16:30:32 +0200 berghofe Added simple code generator.
Mon, 21 Jun 2004 10:25:57 +0200 kleing Merged in license change from Isabelle2004
Sat, 29 May 2004 14:58:44 +0200 wenzelm Library.read_int;
Thu, 15 Apr 2004 20:30:50 +0200 wenzelm finalconsts RepC AbsC;
Fri, 02 Aug 2002 11:49:55 +0200 wenzelm typedef: "open" option;
Wed, 24 Jul 2002 00:11:24 +0200 wenzelm adapted fact names;
Tue, 12 Feb 2002 20:28:27 +0100 wenzelm got rid of explicit marginal comments (now stripped earlier from input);
Thu, 10 Jan 2002 01:11:43 +0100 wenzelm simplified IsarThy.theorem_i;
Thu, 03 Jan 2002 17:56:15 +0100 wenzelm tuned msg;
Sat, 01 Dec 2001 18:52:32 +0100 wenzelm renamed class "term" to "type" (actually "HOL.type");
Sun, 04 Nov 2001 20:56:59 +0100 wenzelm IsarThy.theorem_i (None, []);
Wed, 31 Oct 2001 21:59:07 +0100 wenzelm IsarThy.theorem_i: no locale;
Sat, 27 Oct 2001 23:17:46 +0200 wenzelm use Tactic.prove;
Thu, 18 Oct 2001 21:01:59 +0200 wenzelm sane internal interface for add_typedef(_i);
Wed, 17 Oct 2001 20:25:19 +0200 wenzelm improved internal interface of typedef;
Tue, 16 Oct 2001 17:55:53 +0200 wenzelm typedef: export result;
Sat, 13 Oct 2001 21:44:58 +0200 wenzelm 'morphisms' spec;
Sat, 13 Oct 2001 20:31:34 +0200 wenzelm IsarThy.theorem_i Drule.internalK;
Fri, 12 Oct 2001 12:06:54 +0200 wenzelm test: use SkipProof.make_thm instead of Thm.assume;
Thu, 27 Sep 2001 22:26:00 +0200 wenzelm renamed theory "subset" to "Typedef";
Sun, 15 Jul 2001 14:48:36 +0200 wenzelm abtract non-emptiness statements (no longer use Eps);
Tue, 19 Dec 2000 13:06:49 +0100 wenzelm improved errors;
Thu, 14 Dec 2000 19:38:37 +0100 wenzelm 'typedef': present result theorem "type_definition Rep Abs A";
Wed, 06 Dec 2000 20:45:08 +0100 wenzelm less rude treatment of "no_def";
Mon, 13 Nov 2000 21:59:49 +0100 wenzelm tuned IsarThy.theorem_i;
Thu, 19 Oct 2000 21:25:15 +0200 wenzelm provide more theorems (see subset.thy);
Fri, 15 Sep 2000 12:39:57 +0200 paulson renamed (most of...) the select rules
Thu, 13 Jul 2000 23:13:10 +0200 wenzelm adapted PureThy.add_defs_i;
Sat, 01 Jul 2000 19:55:22 +0200 wenzelm GPLed;
Mon, 13 Mar 2000 13:16:57 +0100 wenzelm adapted to new PureThy.add_thms etc.;
Tue, 25 Jan 2000 20:22:57 +0100 wenzelm fallback on PureThy version;
Wed, 05 Jan 2000 11:56:04 +0100 wenzelm replaced HOLogic.termTVar by HOLogic.termT;
Sat, 04 Sep 1999 21:13:55 +0200 wenzelm goal_nonempty: Ex goal for new-style version;
Mon, 02 Aug 1999 17:58:23 +0200 wenzelm tuned outer syntax;
Thu, 08 Jul 1999 18:36:09 +0200 wenzelm propp: 'concl' patterns;
Tue, 25 May 1999 20:24:10 +0200 wenzelm formal comments (still dummy);
Mon, 24 May 1999 21:57:13 +0200 wenzelm outer syntax keyword classification;
Fri, 21 May 1999 11:48:42 +0200 wenzelm typedef_proof: pass interactive flag;
Wed, 17 Mar 1999 13:49:14 +0100 wenzelm actually check non-emptiness theorem;
Thu, 11 Mar 1999 21:57:34 +0100 wenzelm named witnesses: PureThy.get_thmss;
Tue, 12 Jan 1999 13:54:51 +0100 wenzelm eliminated tthm type and Attribute structure;
Tue, 20 Oct 1998 16:37:02 +0200 wenzelm quiet_mode, message;
Fri, 24 Jul 1998 12:55:05 +0200 berghofe Added new function add_typedef_i_no_def which doesn't add
Wed, 01 Jul 1998 11:20:32 +0200 wenzelm added add_typedecls;
Wed, 27 May 1998 12:21:39 +0200 paulson Changed require to requires for MLWorks
Fri, 15 May 1998 11:34:12 +0200 wenzelm PureThy.add_typedecls;
Wed, 29 Apr 1998 11:39:52 +0200 wenzelm renamed from typedef.ML;
less more (0) tip