src/Pure/drule.ML
Tue, 15 Dec 2015 16:57:10 +0100 wenzelm tuned signature -- clarified modules;
Sun, 16 Aug 2015 21:55:11 +0200 wenzelm produce certified vars without access to theory_of_thm, and without context;
Sun, 16 Aug 2015 19:25:08 +0200 wenzelm added Thm.chyps_of;
Tue, 28 Jul 2015 21:47:03 +0200 wenzelm more explicit context;
Tue, 28 Jul 2015 21:10:41 +0200 wenzelm clarified Variable.gen_all;
Tue, 28 Jul 2015 20:59:39 +0200 wenzelm more explicit context;
Tue, 28 Jul 2015 19:49:54 +0200 wenzelm more direct access to atomic cterms;
Mon, 27 Jul 2015 23:40:39 +0200 wenzelm tuned signature;
Mon, 27 Jul 2015 17:44:55 +0200 wenzelm tuned signature;
Mon, 27 Jul 2015 15:13:05 +0200 wenzelm more explicit checks -- improved errors;
Mon, 27 Jul 2015 14:56:06 +0200 wenzelm eliminated cterm_instantiate;
Mon, 27 Jul 2015 11:30:10 +0200 wenzelm tuned signature;
Mon, 27 Jul 2015 00:17:18 +0200 wenzelm added infer_instantiate_vars, which allows inconsistent types for variables, as required for Metis proof reconstruction;
Sun, 26 Jul 2015 20:54:02 +0200 wenzelm ignore non-existant variables, like other instantiate rules;
Sun, 26 Jul 2015 12:24:16 +0200 wenzelm added infer_instantiate';
Sun, 26 Jul 2015 11:08:57 +0200 wenzelm more uniform exceptions, like cterm_instantiate;
Sat, 25 Jul 2015 23:15:37 +0200 wenzelm more accurate maxidx;
Sat, 25 Jul 2015 21:54:09 +0200 wenzelm clarified error;
Sat, 25 Jul 2015 21:37:09 +0200 wenzelm added infer_instantiate, which is meant to supersede cterm_instantiate;
Sun, 05 Jul 2015 15:02:30 +0200 wenzelm simplified Thm.instantiate and derivatives: the LHS refers to non-certified variables -- this merely serves as index into already certified structures (or is ignored);
Wed, 03 Jun 2015 19:25:05 +0200 wenzelm clarified context;
Sun, 31 May 2015 00:20:35 +0200 wenzelm obsolete;
Sun, 31 May 2015 00:11:12 +0200 wenzelm tuned;
Sat, 30 May 2015 23:58:06 +0200 wenzelm standardize towards Thm.eta_long_conversion, which just does eta_long conversion;
Sat, 30 May 2015 22:04:15 +0200 wenzelm tuned;
Sat, 30 May 2015 21:52:37 +0200 wenzelm more explicit context;
Sat, 30 May 2015 21:28:01 +0200 wenzelm obsolete;
Sat, 30 May 2015 20:21:53 +0200 wenzelm tuned -- more direct Thm.renamed_prop;
Sun, 03 May 2015 16:44:38 +0200 wenzelm suppress formal sort-constraints, in accordance to norm_hhf_eqs;
Fri, 10 Apr 2015 11:29:12 +0200 wenzelm tuned;
Tue, 31 Mar 2015 00:11:54 +0200 wenzelm tuned signature;
Sun, 22 Mar 2015 12:38:41 +0100 wenzelm tuned;
Fri, 20 Mar 2015 11:09:08 +0100 wenzelm tuned -- prepare instantiation more uniformly;
Sat, 07 Mar 2015 21:32:31 +0100 wenzelm clarified Drule.gen_all: observe context more carefully;
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Thu, 05 Mar 2015 13:28:04 +0100 wenzelm tuned -- more explicit use of context;
Wed, 04 Mar 2015 23:21:09 +0100 wenzelm tuned signature;
Wed, 04 Mar 2015 22:05:01 +0100 wenzelm clarified signature;
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Wed, 26 Nov 2014 20:05:34 +0100 wenzelm renamed "pairself" to "apply2", in accordance to @{apply 2};
Sat, 08 Nov 2014 21:31:51 +0100 wenzelm optional proof context for unify operations, for the sake of proper local options;
Sun, 06 Apr 2014 15:43:45 +0200 wenzelm more source positions;
Fri, 21 Mar 2014 20:33:56 +0100 wenzelm more qualified names;
Thu, 27 Jun 2013 17:06:22 +0200 wenzelm tuned signature;
Thu, 27 Jun 2013 11:33:42 +0200 wenzelm tuned signature;
Wed, 29 May 2013 18:52:35 +0200 wenzelm more precise "incremented" indication, which might be relevant in corner cases, e.g. instantiation of leading to vars with different types (which is a potential problem nonetheless);
Wed, 29 May 2013 18:25:11 +0200 wenzelm tuned signature -- more explicit flags for low-level Thm.bicompose;
Fri, 24 May 2013 17:00:46 +0200 wenzelm tuned signature;
Mon, 25 Jun 2012 17:50:05 +0200 wenzelm eliminated obsolete swap_prems_rl -- rotate_prems usually does the job more directly;
Wed, 11 Apr 2012 21:40:46 +0200 wenzelm rule composition via attribute "OF" (or ML functions OF/MRS) is more tolerant against multiple unifiers;
Sat, 31 Mar 2012 19:26:23 +0200 wenzelm tuned signature;
Mon, 19 Mar 2012 21:10:33 +0100 wenzelm moved some legacy stuff;
Wed, 15 Feb 2012 23:19:30 +0100 wenzelm renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
Wed, 15 Feb 2012 22:44:31 +0100 wenzelm discontinued Drule.term_rule, which tends to cause confusion due to builtin cterm_of (NB: the standard morphisms already provide a separate term component);
Tue, 14 Feb 2012 20:57:05 +0100 wenzelm discontinued unused MRL -- in correspondence with section "2.4.2 Rule composition" in the implementation manual;
Sat, 14 Jan 2012 16:58:29 +0100 wenzelm tuned;
Wed, 11 Jan 2012 16:25:34 +0100 wenzelm more qualified names;
Sat, 05 Nov 2011 20:32:12 +0100 wenzelm tuned cterm_instantiate: avoid somewhat expensive Term.map_types and cterm_of;
Sat, 05 Nov 2011 20:07:38 +0100 wenzelm misc tuning and modernization;
Sun, 16 Oct 2011 18:48:30 +0200 wenzelm added Term.dummy_pattern conveniences;
Wed, 10 Aug 2011 19:45:41 +0200 wenzelm avoid OldTerm operations -- with subtle changes of semantics;
Mon, 27 Jun 2011 15:03:55 +0200 wenzelm old gensym is now legacy -- global state is out of fashion, and its result is not guaranteed to be fresh;
Thu, 09 Jun 2011 23:12:02 +0200 wenzelm renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
Thu, 09 Jun 2011 20:56:08 +0200 wenzelm clarified special incr_type_indexes;
Thu, 09 Jun 2011 16:34:49 +0200 wenzelm discontinued Name.variant to emphasize that this is old-style / indirect;
Sat, 23 Apr 2011 19:41:53 +0200 wenzelm hardwired mapping "_" -> "Pure.asm_rl" avoids legacy binding;
Fri, 26 Nov 2010 22:29:41 +0100 wenzelm make two copies (!) of Library.UnequalLengths coincide with ListPair.UnequalLengths;
Mon, 20 Sep 2010 16:05:25 +0200 wenzelm renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
Wed, 25 Aug 2010 15:12:49 +0200 wenzelm structure Thm: less pervasive names;
Sat, 15 May 2010 21:41:32 +0200 wenzelm less pervasive names from structure Thm;
Mon, 03 May 2010 20:13:36 +0200 wenzelm renamed Thm.freezeT to Thm.legacy_freezeT -- it is based on Type.legacy_freeze;
Sun, 25 Apr 2010 23:09:32 +0200 wenzelm renamed Drule.unconstrainTs to Thm.unconstrain_allTs to accomdate the version by krauss/schropp;
Sat, 27 Mar 2010 15:20:31 +0100 wenzelm moved Drule.forall_intr_frees to Thm.forall_intr_frees (in more_thm.ML, which is loaded before pure_thy.ML);
Mon, 22 Mar 2010 19:29:11 +0100 wenzelm eliminated old-style Drule.add_axiom in favour of Specification.axiom, with explicit Drule.export_without_context to imitate the old behaviour;
Mon, 22 Mar 2010 00:48:56 +0100 wenzelm replaced PureThy.add_axioms by more basic Drule.add_axiom, which is old-style nonetheless;
Sat, 20 Mar 2010 17:33:11 +0100 wenzelm renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
Fri, 19 Feb 2010 20:39:48 +0100 wenzelm moved ancient Drule.get_def to OldGoals.get_def;
Sun, 07 Feb 2010 19:33:34 +0100 wenzelm renamed old-style Drule.standard to Drule.export_without_context, to emphasize that this is in no way a standard operation;
Sat, 21 Nov 2009 15:49:29 +0100 wenzelm explicitly mark some legacy freeze operations;
Thu, 12 Nov 2009 22:02:11 +0100 wenzelm eliminated obsolete "internal" kind -- collapsed to unspecific "";
Mon, 02 Nov 2009 20:34:59 +0100 wenzelm modernized structure Simple_Syntax;
Wed, 28 Oct 2009 16:25:26 +0100 wenzelm Drule.store: proper binding;
Sat, 24 Oct 2009 19:47:37 +0200 wenzelm renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
Sat, 17 Oct 2009 00:53:18 +0200 wenzelm legacy Drule.standard is no longer pervasive;
Thu, 09 Jul 2009 22:48:12 +0200 wenzelm renamed structure TermSubst to Term_Subst;
Mon, 06 Jul 2009 21:24:30 +0200 wenzelm structure Thm: less pervasive names;
Thu, 02 Jul 2009 21:26:18 +0200 wenzelm renamed Drule.sort_triv to Thm.sort_triv (cf. more_thm.ML);
Mon, 16 Mar 2009 23:39:44 +0100 wenzelm refined is_norm_hhf: reject beta-redexes (rules based on term nets or could_unify assume normal form), also potentially faster by avoiding expensive Envir.beta_eta_contract;
Sat, 07 Mar 2009 22:04:59 +0100 wenzelm moved Thm.def_name(_optional) to more_thm.ML;
Wed, 21 Jan 2009 16:47:04 +0100 haftmann binding replaces bstring
Sun, 04 Jan 2009 15:28:09 +0100 wenzelm added comp_no_flatten;
Wed, 31 Dec 2008 18:53:16 +0100 wenzelm moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
Wed, 31 Dec 2008 00:08:13 +0100 wenzelm moved old add_term_vars, add_term_frees etc. to structure OldTerm;
Fri, 31 Oct 2008 10:39:04 +0100 berghofe Theorem "_" is now stored with open derivation.
Thu, 23 Oct 2008 15:28:01 +0200 wenzelm renamed Thm.get_axiom_i to Thm.axiom;
Thu, 16 Oct 2008 22:44:27 +0200 wenzelm added rules for sort_constraint, include in norm_hhf_eqs;
Thu, 14 Aug 2008 16:52:46 +0200 wenzelm moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
Mon, 23 Jun 2008 23:45:46 +0200 wenzelm Logic.implies;
Thu, 19 Jun 2008 20:48:03 +0200 wenzelm moved add_used to Isar/rule_insts.ML;
Mon, 16 Jun 2008 22:13:47 +0200 wenzelm removed obsolete global read_insts/read_instantiate (cf. Isar/rule_insts.ML);
Wed, 11 Jun 2008 18:03:14 +0200 wenzelm qualified types_sorts, read_insts etc.;
Sun, 18 May 2008 15:04:09 +0200 wenzelm moved global pretty/string_of functions from Sign to Syntax;
Tue, 15 Apr 2008 16:12:05 +0200 wenzelm Thm.forall_elim_var(s);
Sat, 12 Apr 2008 17:00:38 +0200 wenzelm rep_cterm/rep_thm: no longer dereference theory_ref;
Sat, 29 Mar 2008 19:14:09 +0100 wenzelm certify wrt. dynamic context;
Thu, 27 Mar 2008 14:41:09 +0100 wenzelm eliminated theory ProtoPure;
Tue, 27 Nov 2007 15:43:31 +0100 berghofe Better error messages for cterm_instantiate.
Thu, 11 Oct 2007 19:10:20 +0200 wenzelm moved Drule.unvarify to Thm.unvarify (cf. more_thm.ML);
Wed, 10 Oct 2007 17:31:54 +0200 wenzelm improved abs_def: only abstract over outermost (unique) Vars;
Thu, 04 Oct 2007 20:29:24 +0200 wenzelm replaced literal 'a by Name.aT;
Fri, 24 Aug 2007 14:17:54 +0200 paulson new derived rule: incr_type_indexes
Mon, 13 Aug 2007 18:10:18 +0200 wenzelm SimpleSyntax.read_prop;
Sun, 29 Jul 2007 14:30:04 +0200 wenzelm moved Drule.add/del/merge_rules to Thm.add/del/merge_thms;
Fri, 27 Jul 2007 20:11:48 +0200 wenzelm added dummy_thm, is_dummy_thm;
Wed, 04 Jul 2007 16:49:36 +0200 wenzelm added binop_cong_rule;
Tue, 03 Jul 2007 17:17:11 +0200 wenzelm tuned rotate_prems;
Wed, 20 Jun 2007 17:32:53 +0200 paulson A more robust flexflex_unique
Tue, 19 Jun 2007 23:15:51 +0200 wenzelm added with_subgoal;
Thu, 31 May 2007 23:47:36 +0200 wenzelm simplified/unified list fold;
Fri, 11 May 2007 18:49:15 +0200 wenzelm proper type for fun/arg_cong_rule;
Fri, 11 May 2007 18:47:08 +0200 wenzelm added fun/arg_cong_rule;
Thu, 10 May 2007 00:39:52 +0200 wenzelm moved some operations to more_thm.ML and conv.ML;
Sun, 15 Apr 2007 14:31:53 +0200 wenzelm moved Drule.plain_prop_of, Drule.fold_terms to more_thm.ML;
Sat, 14 Apr 2007 17:36:09 +0200 wenzelm cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
Mon, 02 Apr 2007 11:31:08 +0200 paulson optimizing the null instantiation case
Mon, 26 Feb 2007 23:18:24 +0100 wenzelm moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
Tue, 13 Feb 2007 16:37:14 +0100 paulson COMP now performs a distinctness check on the multiple results before failing
Sat, 10 Feb 2007 16:43:23 +0100 paulson Completing the bug fix from the previous update: the result of unifying type
Thu, 08 Feb 2007 18:14:13 +0100 paulson cterm_instantiate was calling a type instantiation function that works only for matching,
Fri, 19 Jan 2007 22:08:18 +0100 wenzelm moved inst from drule.ML to old_goals.ML;
Tue, 05 Dec 2006 00:30:38 +0100 wenzelm thm/prf: separate official name vs. additional tags;
Thu, 30 Nov 2006 14:17:27 +0100 wenzelm added zero_var_indexes_list;
Wed, 29 Nov 2006 23:33:09 +0100 wenzelm *** bad commit -- reverted to previous version ***
Wed, 29 Nov 2006 23:28:08 +0100 wenzelm added INCR_COMP, COMP_INCR;
Wed, 29 Nov 2006 04:11:11 +0100 wenzelm added INCR_COMP, COMP_INCR;
Tue, 28 Nov 2006 00:35:21 +0100 wenzelm dest_term: strip_imp_concl;
Fri, 24 Nov 2006 22:05:15 +0100 wenzelm added cterm_rule;
Tue, 21 Nov 2006 18:07:33 +0100 wenzelm moved theorem kinds from PureThy to Thm;
Mon, 09 Oct 2006 02:19:56 +0200 wenzelm added dest_equals_lhs;
Sat, 07 Oct 2006 01:31:09 +0200 wenzelm added term_rule;
Thu, 05 Oct 2006 10:40:12 +0200 paulson a few new functions on thms and cterms
Thu, 21 Sep 2006 19:04:55 +0200 wenzelm added dest_equals_rhs;
Mon, 18 Sep 2006 19:39:07 +0200 wenzelm Thm.dest_arg;
Tue, 12 Sep 2006 12:12:46 +0200 wenzelm moved term subst functions to TermSubst;
Thu, 03 Aug 2006 17:30:37 +0200 wenzelm tuned types_sorts, add_used;
Wed, 02 Aug 2006 22:26:52 +0200 wenzelm removed obsolete frees/vars_of etc.;
Sun, 30 Jul 2006 21:28:52 +0200 wenzelm Thm.adjust_maxidx;
Thu, 27 Jul 2006 13:43:05 +0200 wenzelm removed obsolete equal_abs_elim(_list);
Tue, 11 Jul 2006 12:17:02 +0200 wenzelm replaced Term.variant(list) by Name.variant(_list);
Tue, 04 Jul 2006 19:49:50 +0200 wenzelm added generalize;
Sat, 17 Jun 2006 19:37:47 +0200 wenzelm Term.internal;
Tue, 13 Jun 2006 23:41:44 +0200 wenzelm removed weak_eq_thm;
Mon, 12 Jun 2006 21:19:00 +0200 wenzelm tuned Seq/Envir/Unify interfaces;
Sun, 11 Jun 2006 21:59:21 +0200 wenzelm outer_params: Syntax.dest_internal;
Mon, 05 Jun 2006 21:54:21 +0200 wenzelm support embedded terms;
Thu, 01 Jun 2006 14:51:37 +0200 paulson Tiny code cleanup
Fri, 26 May 2006 22:20:05 +0200 wenzelm forall_intr_list: do not ignore errors;
Mon, 01 May 2006 17:05:11 +0200 wenzelm added sort_triv;
Sat, 29 Apr 2006 23:16:46 +0200 wenzelm added unconstrainTs;
Thu, 27 Apr 2006 15:06:35 +0200 wenzelm tuned basic list operators (flat, maps, map_filter);
Thu, 13 Apr 2006 12:00:59 +0200 wenzelm added equal_elim_rule2;
Sat, 04 Mar 2006 21:10:07 +0100 wenzelm added mk_conjunction;
Wed, 22 Feb 2006 22:18:38 +0100 wenzelm removed rename_indexes_wrt;
Wed, 15 Feb 2006 21:35:02 +0100 wenzelm added distinct_prems_rl;
Mon, 06 Feb 2006 20:58:54 +0100 wenzelm Envir.(beta_)eta_contract;
Fri, 03 Feb 2006 23:12:30 +0100 wenzelm removed add/del_rules;
Sat, 28 Jan 2006 17:28:54 +0100 wenzelm added equals_cong;
Fri, 27 Jan 2006 19:03:02 +0100 wenzelm moved theorem tags from Drule to PureThy;
Wed, 25 Jan 2006 00:21:35 +0100 wenzelm abs_def: improved error;
Sat, 21 Jan 2006 23:02:24 +0100 wenzelm simplified type attribute;
Tue, 10 Jan 2006 19:33:32 +0100 wenzelm added declaration_attribute;
Sat, 31 Dec 2005 21:49:43 +0100 wenzelm tuned forall_intr_vars;
Fri, 23 Dec 2005 15:16:46 +0100 wenzelm conj_elim_precise: proper treatment of nested conjunctions;
Thu, 22 Dec 2005 00:28:54 +0100 wenzelm fixed has_internal;
Thu, 08 Dec 2005 20:16:10 +0100 wenzelm removed Syntax.deskolem;
Fri, 02 Dec 2005 22:54:45 +0100 wenzelm abs_def: beta/eta contract lhs;
Fri, 25 Nov 2005 18:58:37 +0100 wenzelm forall_conv: limit prefix;
Tue, 22 Nov 2005 19:34:44 +0100 wenzelm export map_tags;
Sat, 19 Nov 2005 14:21:03 +0100 wenzelm removed conj_mono;
Wed, 16 Nov 2005 17:45:25 +0100 wenzelm added protect_cong, cong_mono_thm;
Wed, 09 Nov 2005 16:26:44 +0100 wenzelm added fold_terms;
Tue, 08 Nov 2005 10:43:09 +0100 wenzelm removed impose_hyps, satisfy_hyps;
Fri, 28 Oct 2005 22:27:52 +0200 wenzelm added incr_indexes;
Fri, 21 Oct 2005 18:14:44 +0200 wenzelm renamed triv_goal to goalI, rev_triv_goal to goalD;
Thu, 29 Sep 2005 12:30:30 +0200 berghofe Optimized and exported flexflex_unique.
Mon, 26 Sep 2005 19:19:14 +0200 wenzelm moved disambiguate_frees to ProofKernel;
Mon, 26 Sep 2005 02:06:44 +0200 obua added Drule.disambiguate_frees : thm -> thm
Mon, 12 Sep 2005 18:20:32 +0200 haftmann introduced new-style AList operations
Wed, 31 Aug 2005 15:46:40 +0200 wenzelm refer to theory instead of low-level tsig;
Mon, 01 Aug 2005 19:20:37 +0200 wenzelm replaced atless by term_ord;
Thu, 28 Jul 2005 15:20:06 +0200 wenzelm tuned gen_all, forall_elim_list, implies_intr_list, standard;
Fri, 15 Jul 2005 15:44:15 +0200 wenzelm tuned fold on terms;
Wed, 13 Jul 2005 11:30:37 +0200 haftmann (fix for an accidental commit)
Wed, 13 Jul 2005 11:16:34 +0200 haftmann (intermediate commit)
Wed, 06 Jul 2005 20:00:25 +0200 wenzelm Thm.full_prop_of;
Mon, 04 Jul 2005 17:08:19 +0200 wenzelm tuned;
Wed, 29 Jun 2005 15:13:25 +0200 wenzelm added implies_intr_hyps (from thm.ML);
Fri, 17 Jun 2005 18:33:08 +0200 wenzelm accomodate identification of type Sign.sg and theory;
Tue, 10 May 2005 18:37:43 +0200 paulson new cterm primitives
Wed, 04 May 2005 18:50:21 +0200 berghofe Added eta_long_conversion.
Thu, 28 Apr 2005 21:35:47 +0200 wenzelm added plain_prop_of;
Thu, 21 Apr 2005 19:12:03 +0200 berghofe - Eliminated nodup_vars check.
Thu, 07 Apr 2005 09:27:20 +0200 wenzelm added add_used; include tpairs;
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.
Tue, 22 Feb 2005 18:42:22 +0100 dixon Lucas - fixed bug in zero_var_indexes: it was ignoring vars in the flex-flex pairs. These are now taken into account.
Sun, 13 Feb 2005 17:15:14 +0100 skalberg Deleted Library.option type.
Thu, 03 Feb 2005 16:06:19 +0100 paulson new treatment of demodulation in proof reconstruction
Tue, 18 Jan 2005 14:34:24 +0100 berghofe Added variants of instantiation functions that operate on pairs of type
Tue, 26 Oct 2004 16:33:09 +0200 berghofe Added function strip_type (for ctyps).
Wed, 23 Jun 2004 14:44:22 +0200 skalberg Moved conversion rules from MetaSimplifier to Drule. refl_implies removed
Tue, 01 Jun 2004 12:33:50 +0200 wenzelm removed obsolete sort 'logic';
Sat, 29 May 2004 15:00:52 +0200 wenzelm improved output;
Thu, 22 Apr 2004 10:52:32 +0200 wenzelm tuned;
Thu, 19 Feb 2004 10:37:15 +0100 paulson comments!!
Tue, 17 Feb 2004 17:41:30 +0100 berghofe Moved application of flexflex_unique from standard' to standard.
Sun, 15 Feb 2004 10:46:37 +0100 paulson Polymorphic treatment of binary arithmetic using axclasses
Tue, 06 Jan 2004 10:38:14 +0100 paulson correction to cterm_instantiate by Christoph Leuth
Sun, 29 Jun 2003 21:28:13 +0200 berghofe Added functions for renaming bound variables.
Mon, 21 Oct 2002 17:07:27 +0200 berghofe Removed obsolete functions dealing with flex-flex constraints.
Thu, 17 Oct 2002 10:52:59 +0200 paulson fixing the cut_tac method to work when there are no instantiations and the
Mon, 30 Sep 2002 16:37:44 +0200 berghofe Removed nRS again because extract_rews now takes care of preserving names.
Thu, 19 Sep 2002 16:01:29 +0200 nipkow drule: added nRS
Thu, 18 Jul 2002 12:05:51 +0200 wenzelm added satisfy_hyps;
Tue, 16 Jul 2002 18:37:03 +0200 wenzelm added equal_elim_rule1;
Tue, 09 Jul 2002 18:03:26 +0200 berghofe Added function abs_def.
Fri, 31 May 2002 18:50:03 +0200 berghofe Changed interface of Pattern.rewrite_term.
Tue, 07 May 2002 14:26:32 +0200 wenzelm use eq_thm_prop instead of slightly inadequate eq_thm;
Wed, 20 Feb 2002 16:00:32 +0100 berghofe New function strip_comb (cterm version of Term.strip_comb).
Thu, 17 Jan 2002 21:02:52 +0100 wenzelm added is_norm_hhf (from logic.ML);
Tue, 15 Jan 2002 00:09:29 +0100 wenzelm conj_intr_list and conj_elim_precise: cover 0 conjuncts;
Sat, 12 Jan 2002 16:37:58 +0100 wenzelm renamed forall_elim_vars_safe to gen_all;
Fri, 11 Jan 2002 14:53:05 +0100 wenzelm improved forall_elim_vars_safe (no longer invents new indexes);
Fri, 11 Jan 2002 00:29:25 +0100 wenzelm kind: ignore "";
Tue, 18 Dec 2001 02:17:20 +0100 wenzelm tuned Type.unify;
Fri, 14 Dec 2001 11:51:01 +0100 wenzelm export add_tvarsT etc.;
Wed, 05 Dec 2001 03:09:21 +0100 wenzelm added add_rule, del_rule;
Mon, 26 Nov 2001 18:33:21 +0100 wenzelm added remdups_rl;
Sat, 24 Nov 2001 16:55:00 +0100 wenzelm gen_merge_lists';
Fri, 16 Nov 2001 15:24:09 +0100 wenzelm local_standard: plain strip_shyps instead of strip_shyps_warning;
less more (0) -240 tip