src/Provers/hypsubst.ML
Fri, 04 Jul 2014 17:19:03 +0200 wenzelm more uniform names;
Wed, 11 Jun 2014 14:24:23 +1000 Thomas Sewell Hypsubst preserves equality hypotheses
Fri, 21 Mar 2014 20:33:56 +0100 wenzelm more qualified names;
Fri, 24 May 2013 17:00:46 +0200 wenzelm tuned signature;
Sat, 27 Apr 2013 20:50:20 +0200 wenzelm uniform Proof.context for hyp_subst_tac;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Thu, 08 Nov 2012 19:55:35 +0100 bulwahn hyp_subst_tac allows to pass an optional simpset to the internal simplifier call to avoid renamed bound variable warnings in the simplifier call
Tue, 19 Jun 2012 11:18:09 +0200 Rafal Kolanski Updated comment to reflect current state.
Sat, 14 Jan 2012 21:16:15 +0100 wenzelm discontinued old-style Term.list_abs in favour of plain Term.abs;
Mon, 28 Nov 2011 17:05:41 +0100 wenzelm avoid stepping outside of context -- plain zero_var_indexes should be sufficient;
Thu, 24 Nov 2011 21:01:06 +0100 wenzelm modernized some old-style infix operations, which were left over from the time of ML proof scripts;
Mon, 08 Aug 2011 17:23:15 +0200 wenzelm misc tuning -- eliminated old-fashioned rep_thm;
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;
Sat, 14 May 2011 11:42:43 +0200 wenzelm modernized functor names;
Sat, 16 Apr 2011 20:26:59 +0200 wenzelm more direct Thm.cprem_of (with exception THM instead of Subscript);
Sat, 16 Apr 2011 18:11:20 +0200 wenzelm eliminated old List.nth;
Thu, 24 Mar 2011 16:47:24 +0100 wenzelm more direct loose_bvar1;
Wed, 29 Sep 2010 11:02:24 +0200 krauss backed out my old attempt at single_hyp_subst_tac (67cd6ed76446)
Fri, 10 Sep 2010 23:56:35 +0200 krauss use eta-contracted version for occurrence check (avoids possible non-termination)
Sat, 15 May 2010 21:50:05 +0200 wenzelm less pervasive names from structure Thm;
Thu, 29 Apr 2010 22:56:32 +0200 wenzelm proper context for mksimps etc. -- via simpset of the running Simplifier;
Sat, 13 Mar 2010 16:44:12 +0100 wenzelm removed old CVS Ids;
Fri, 19 Feb 2010 16:11:45 +0100 wenzelm renamed Simplifier.theory_context to Simplifier.global_context to emphasize that this is not the real thing;
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, 17 Oct 2009 00:52:37 +0200 wenzelm explicitly qualify Drule.standard;
Fri, 13 Mar 2009 23:50:05 +0100 wenzelm simplified method setup;
Fri, 13 Mar 2009 19:58:26 +0100 wenzelm unified type Proof.method and pervasive METHOD combinators;
Mon, 04 Aug 2008 22:55:00 +0200 wenzelm meta_subst: xsymbols make it work with clean Pure;
Mon, 14 Jul 2008 17:47:18 +0200 krauss single_hyp(_meta)_subst_tac: Controlled substitution of a single hyp
Sat, 24 May 2008 23:52:35 +0200 wenzelm inst_subst_tac: match types -- no longer assume that subst rule has exactly one type argument;
less more (0) -50 -30 tip