src/HOL/Tools/inductive_package.ML
Fri, 07 Apr 2006 17:27:53 +0200 berghofe Fixed bug that caused proof of induction rule to fail
Fri, 03 Feb 2006 23:12:28 +0100 wenzelm canonical member/insert/merge;
Fri, 27 Jan 2006 19:03:02 +0100 wenzelm moved theorem tags from Drule to PureThy;
Thu, 26 Jan 2006 15:37:14 +0100 berghofe Inductive sets with no introduction rules are now allowed as well.
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;
Thu, 22 Dec 2005 00:28:47 +0100 wenzelm actually produce projected rules;
Fri, 16 Dec 2005 09:00:11 +0100 haftmann re-arranged tuples (theory * 'a) to ('a * theory) in Pure
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, 02 Dec 2005 08:06:59 +0100 haftmann introduced new map2, fold
Wed, 23 Nov 2005 18:52:01 +0100 wenzelm RuleCases.case_conclusion;
Tue, 22 Nov 2005 19:34:40 +0100 wenzelm declare coinduct rule;
Tue, 25 Oct 2005 18:18:49 +0200 wenzelm avoid legacy goals;
Fri, 21 Oct 2005 18:14:38 +0200 wenzelm OldGoals;
Mon, 19 Sep 2005 16:38:35 +0200 haftmann introduced AList module
Thu, 15 Sep 2005 17:16:56 +0200 wenzelm TableFun/Symtab: curried lookup and update;
Mon, 12 Sep 2005 18:20:32 +0200 haftmann introduced new-style AList operations
Mon, 05 Sep 2005 17:38:18 +0200 wenzelm curried_lookup/update;
Tue, 16 Aug 2005 13:42:26 +0200 wenzelm OuterKeyword;
Wed, 03 Aug 2005 14:48:22 +0200 avigad changed reference to Lfp.lfp to FixedPint.lfp, ditto for gfp
Mon, 01 Aug 2005 19:20:29 +0200 wenzelm Sign.read_term;
Thu, 28 Jul 2005 15:19:49 +0200 wenzelm Sign.typ_unify;
Tue, 19 Jul 2005 17:21:47 +0200 wenzelm Logic.incr_tvar;
Fri, 15 Jul 2005 15:44:15 +0200 wenzelm tuned fold on terms;
Wed, 13 Jul 2005 10:48:21 +0200 haftmann (corrected wrong commit)
Wed, 13 Jul 2005 10:44:51 +0200 haftmann (intermediate commit)
Mon, 20 Jun 2005 22:13:59 +0200 wenzelm get_thm(s): Name;
Fri, 17 Jun 2005 18:33:17 +0200 wenzelm accomodate change of TheoryDataFun;
Sat, 11 Jun 2005 22:15:48 +0200 wenzelm refer to name spaces values instead of names;
Sun, 05 Jun 2005 23:07:25 +0200 wenzelm Type.freeze;
Tue, 31 May 2005 11:53:13 +0200 wenzelm renamed cond_extern to extern;
Thu, 21 Apr 2005 18:57:18 +0200 berghofe Adapted to new interface of instantiation and unification / matching functions.
Wed, 13 Apr 2005 18:45:25 +0200 wenzelm *** MESSAGE REFERS TO PREVIOUS VERSION ***
Wed, 13 Apr 2005 18:34:22 +0200 wenzelm *** empty log message ***
Fri, 04 Mar 2005 15:07:34 +0100 skalberg Removed practically all references to Library.foldr.
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.
Thu, 10 Feb 2005 18:51:54 +0100 nipkow HOL.order -> Orderings.order due to restructering
Mon, 24 Jan 2005 18:16:57 +0100 berghofe Adapted to modified interface of PureThy.get_thm(s).
Thu, 16 Dec 2004 14:34:23 +0100 paulson Further fix to a bug (involving equational premises) in inductive definitions
Thu, 09 Dec 2004 16:45:46 +0100 paulson converted Sum_Type to new-style theory: Inl, Inr are NO LONGER global
Sun, 11 Jul 2004 20:33:22 +0200 wenzelm local_cla/simpset_of;
Mon, 21 Jun 2004 10:25:57 +0200 kleing Merged in license change from Isabelle2004
Thu, 22 Apr 2004 10:52:32 +0200 wenzelm tuned;
Wed, 15 Oct 2003 11:02:28 +0200 berghofe Fixed bug in mk_ind_def that caused the inductive definition package to
Thu, 12 Dec 2002 11:38:18 +0100 paulson Better treatment of equality in premises of inductive definitions. Less
Wed, 13 Nov 2002 15:31:14 +0100 berghofe - No longer applies norm_hhf_rule
Mon, 21 Oct 2002 17:00:45 +0200 berghofe Now applies standard' to "unfold" theorem (due to flex-flex constraints).
Fri, 04 Oct 2002 15:23:12 +0200 paulson Fixed bug involving inductive definitions having equalities in the premises,
Fri, 31 May 2002 18:49:31 +0200 berghofe Changed interface of MetaSimplifier.rewrite_term.
Thu, 21 Feb 2002 20:10:34 +0100 wenzelm clarified internal theory dependencies;
Wed, 20 Feb 2002 00:53:53 +0100 wenzelm Symbol.bump_string;
Tue, 12 Feb 2002 20:28:27 +0100 wenzelm got rid of explicit marginal comments (now stripped earlier from input);
Thu, 17 Jan 2002 21:01:17 +0100 wenzelm MetaSimplifier.rewrite_term replaces slow Tactic.rewrite_cterm;
Fri, 11 Jan 2002 00:28:43 +0100 wenzelm IsarThy.theorems_i;
Sat, 29 Dec 2001 18:35:27 +0100 wenzelm 'inductive_cases': support 'and' form;
Tue, 18 Dec 2001 02:17:20 +0100 wenzelm tuned Type.unify;
Fri, 14 Dec 2001 11:50:38 +0100 wenzelm changed Type.varify;
Thu, 06 Dec 2001 00:40:56 +0100 wenzelm added the_mk_cases;
Sat, 01 Dec 2001 18:52:32 +0100 wenzelm renamed class "term" to "type" (actually "HOL.type");
Wed, 28 Nov 2001 00:46:26 +0100 wenzelm theory data: removed obsolete finish method;
Wed, 21 Nov 2001 00:34:06 +0100 wenzelm Set.vimage;
Wed, 14 Nov 2001 18:44:27 +0100 wenzelm inductive: removed con_defs;
Tue, 13 Nov 2001 22:18:46 +0100 wenzelm tuned;
Mon, 12 Nov 2001 23:27:04 +0100 wenzelm mutual rules declared as ``consumes 0'';
Fri, 09 Nov 2001 22:50:58 +0100 wenzelm tuned;
Thu, 08 Nov 2001 23:59:37 +0100 wenzelm theory data: finish method;
Wed, 31 Oct 2001 01:21:31 +0100 wenzelm use HOL.induct_XXX;
Mon, 22 Oct 2001 17:58:26 +0200 wenzelm quick_and_dirty_prove_goalw_cterm;
Thu, 18 Oct 2001 21:27:47 +0200 wenzelm GPLed;
Thu, 18 Oct 2001 21:05:35 +0200 wenzelm moved atomize stuff to theory HOL;
Mon, 15 Oct 2001 20:35:10 +0200 wenzelm Tactic.rewrite_cterm;
Sun, 14 Oct 2001 22:08:29 +0200 wenzelm moved rulify to ObjectLogic;
Sun, 14 Oct 2001 20:05:07 +0200 wenzelm "HOL.mono";
Sat, 13 Oct 2001 20:31:34 +0200 wenzelm IsarThy.theorem_i Drule.internalK;
Thu, 04 Oct 2001 15:39:43 +0200 wenzelm simp_case_tac is back again from induct_method.ML;
Fri, 28 Sep 2001 19:19:26 +0200 wenzelm inductive: no collective atts;
Thu, 16 Aug 2001 23:19:12 +0200 wenzelm prefer immediate monos;
Fri, 01 Jun 2001 11:03:50 +0200 paulson now checks for leading meta-quantifiers and complains, instead of
Fri, 02 Feb 2001 22:20:09 +0100 wenzelm use hol_simplify;
Wed, 31 Jan 2001 01:13:01 +0100 wenzelm more robust handling of rule cases hints;
Mon, 29 Jan 2001 13:26:04 +0100 berghofe Splitting of arguments of product types in induction rules is now less
Tue, 16 Jan 2001 00:32:38 +0100 wenzelm export inductive_forall_name, inductive_forall_def, rulify;
Sat, 06 Jan 2001 21:26:27 +0100 wenzelm Tactic.norm_hhf;
Wed, 27 Dec 2000 18:27:19 +0100 wenzelm Method.erule 0;
Sat, 23 Dec 2000 22:51:34 +0100 wenzelm simplified quick_and_dirty stuff;
Fri, 22 Dec 2000 18:24:39 +0100 wenzelm handle proper rules;
Fri, 01 Dec 2000 19:43:06 +0100 wenzelm ignore quick_and_dirty for coind;
Thu, 19 Oct 2000 21:23:47 +0200 wenzelm InductAttrib;
Thu, 12 Oct 2000 18:38:23 +0200 nipkow *** empty log message ***
Thu, 12 Oct 2000 13:01:19 +0200 nipkow induct -> lfp_induct
Wed, 11 Oct 2000 09:09:06 +0200 nipkow *** empty log message ***
Sat, 23 Sep 2000 16:08:23 +0200 paulson renaming the inverse image operator in HOL
Sun, 17 Sep 2000 22:21:31 +0200 wenzelm Display.pretty_thm_sg;
Tue, 12 Sep 2000 17:39:29 +0200 wenzelm tuned handling of "intros";
Thu, 07 Sep 2000 20:51:07 +0200 wenzelm tuned msg;
Mon, 04 Sep 2000 21:19:07 +0200 wenzelm tuned "mono" att setup;
Sat, 02 Sep 2000 21:50:38 +0200 wenzelm "inductive_cases": proper command;
Thu, 17 Aug 2000 21:07:25 +0200 wenzelm removed obsolete keyword;
Thu, 17 Aug 2000 10:37:33 +0200 wenzelm renamed 'mk_cases_tac' to 'ind_cases';
Mon, 14 Aug 2000 18:14:54 +0200 wenzelm raplaced "intrs" by "intrs" (new-style only);
Wed, 09 Aug 2000 20:46:58 +0200 wenzelm fixed mk_cases_i: TRYALL InductMethod.simp_case_tac;
Sat, 22 Jul 2000 12:58:12 +0200 wenzelm improved error msg;
Thu, 13 Jul 2000 23:13:10 +0200 wenzelm adapted PureThy.add_defs_i;
Thu, 13 Jul 2000 11:42:11 +0200 wenzelm use InductMethod.simp_case_tac;
Mon, 03 Jul 2000 11:13:08 +0200 wenzelm previde 'defs' field for quick_and_dirty;
Thu, 29 Jun 2000 22:38:30 +0200 wenzelm adapted args of IsarThy.have_theorems_i;
Fri, 23 Jun 2000 12:29:55 +0200 berghofe get_inductive now returns None instead of raising an exception.
Thu, 15 Jun 2000 16:02:12 +0200 berghofe Now also proves monotonicity when in quick_and_dirty mode.
Mon, 17 Apr 2000 13:57:55 +0200 wenzelm Pretty.chunks;
Fri, 31 Mar 2000 21:55:27 +0200 wenzelm use Attrib.add_del_args;
Mon, 13 Mar 2000 13:20:51 +0100 wenzelm adapted to new PureThy.add_thms etc.;
Fri, 10 Mar 2000 15:02:04 +0100 berghofe Type.unify now uses Vartab instead of association lists.
Thu, 09 Mar 2000 22:57:13 +0100 wenzelm more robust case names of induct;
Wed, 08 Mar 2000 23:45:37 +0100 wenzelm removed tune_names;
Wed, 08 Mar 2000 18:06:12 +0100 wenzelm mk_elims, add_cases_induct: name rule cases;
Fri, 03 Mar 2000 21:01:57 +0100 wenzelm mk_cases / inductive_cases: use InductMethod.con_elim_(solved_)tac;
less more (0) -120 tip