src/Tools/eqsubst.ML
Thu, 11 Sep 2014 21:11:03 +0200 blanchet fixed some spelling mistakes
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
Fri, 23 Aug 2013 17:01:12 +0200 wenzelm tuned signature;
Sat, 27 Jul 2013 16:35:51 +0200 wenzelm standardized aliases;
Thu, 30 May 2013 17:26:01 +0200 wenzelm tuned signature;
Thu, 30 May 2013 16:53:32 +0200 wenzelm more standard fold/fold_rev;
Thu, 30 May 2013 16:31:53 +0200 wenzelm misc tuning;
Thu, 30 May 2013 16:11:14 +0200 wenzelm prefer existing beta_eta_conversion;
Thu, 30 May 2013 15:51:55 +0200 wenzelm more standard names;
Thu, 30 May 2013 15:02:33 +0200 wenzelm simplified method setup;
Thu, 30 May 2013 14:37:06 +0200 wenzelm tuned -- prefer terminology of tactic / goal state;
Thu, 30 May 2013 14:17:56 +0200 wenzelm tuned;
Thu, 30 May 2013 13:59:38 +0200 wenzelm misc tuning;
Wed, 29 May 2013 18:25:11 +0200 wenzelm tuned signature -- more explicit flags for low-level Thm.bicompose;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Wed, 12 Sep 2012 23:18:26 +0200 wenzelm observe context more carefully when producing "fresh" variables -- for increased chances that method "subst" works in local context (including that of forked proofs);
Wed, 12 Sep 2012 22:00:29 +0200 wenzelm eliminated some old material that is unused in the visible universe;
Tue, 09 Aug 2011 15:50:13 +0200 wenzelm misc tuning and simplification;
Thu, 09 Jun 2011 16:34:49 +0200 wenzelm discontinued Name.variant to emphasize that this is old-style / indirect;
Wed, 15 Dec 2010 15:11:56 +0100 wenzelm avoid ML structure aliases (especially single-letter abbreviations);
Fri, 26 Nov 2010 22:29:41 +0100 wenzelm make two copies (!) of Library.UnequalLengths coincide with ListPair.UnequalLengths;
Mon, 17 May 2010 23:54:15 +0200 wenzelm prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
Tue, 27 Oct 2009 17:34:00 +0100 wenzelm normalized basic type abbreviations;
Sat, 17 Oct 2009 14:43:18 +0200 wenzelm eliminated hard tabulators, guessing at each author's individual tab-width;
Tue, 29 Sep 2009 16:24:36 +0200 wenzelm explicit indication of Unsynchronized.ref;
Thu, 23 Jul 2009 18:44:09 +0200 wenzelm renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
Fri, 17 Jul 2009 21:33:00 +0200 wenzelm tuned/modernized Envir operations;
Sat, 30 May 2009 13:12:15 +0200 wenzelm minimal signature cleanup;
Fri, 13 Mar 2009 21:25:15 +0100 wenzelm eliminated type Args.T;
Fri, 13 Mar 2009 19:58:26 +0100 wenzelm unified type Proof.method and pervasive METHOD combinators;
Fri, 06 Mar 2009 22:32:27 +0100 wenzelm replaced archaic use of rep_ss by Simplifier.mksimps;
Sat, 28 Feb 2009 14:02:12 +0100 wenzelm moved some generic tools to src/Tools/ -- src/Provers is essentially obsolete;
less more (0) tip