src/HOL/Tools/TFL/post.ML
Tue, 10 Feb 2015 14:48:26 +0100 wenzelm proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
Fri, 21 Mar 2014 20:33:56 +0100 wenzelm more qualified names;
Sat, 01 Feb 2014 18:42:46 +0100 wenzelm proper context for printing;
Sun, 26 Jan 2014 13:45:40 +0100 wenzelm tuned signature;
Sat, 25 Jan 2014 22:06:07 +0100 wenzelm explicit eigen-context for attributes "where", "of", and corresponding read_instantiate, instantiate_tac;
Sun, 12 Jan 2014 16:42:02 +0100 wenzelm clarified context;
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
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);
Mon, 12 Sep 2011 07:55:43 +0200 nipkow new fastforce replacing fastsimp - less confusing name
Fri, 13 May 2011 22:55:00 +0200 wenzelm proper Proof.context for classical tactics;
Thu, 12 May 2011 23:23:48 +0200 wenzelm prefer Proof.context over old-style claset/simpset;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Fri, 04 Mar 2011 11:43:20 +0100 krauss clarified
Wed, 15 Dec 2010 15:11:56 +0100 wenzelm avoid ML structure aliases (especially single-letter abbreviations);
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
Thu, 19 Aug 2010 11:02:14 +0200 haftmann use antiquotations for remaining unqualified constants in HOL
Mon, 03 May 2010 20:53:49 +0200 wenzelm replaced Thm.legacy_freezeT by Thm.unvarify_global -- these facts stem from closed definitions, i.e. there are no term Vars;
Mon, 03 May 2010 20:13:36 +0200 wenzelm renamed Thm.freezeT to Thm.legacy_freezeT -- it is based on Type.legacy_freeze;
Mon, 03 May 2010 14:25:56 +0200 wenzelm renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
Fri, 30 Apr 2010 18:06:29 +0200 wenzelm proper context for rule_by_tactic;
Mon, 15 Mar 2010 20:27:23 +0100 wenzelm preserve full const name more carefully, and avoid slightly odd Sign.intern_term;
Fri, 12 Mar 2010 12:14:30 +0100 bulwahn refining and adding Spec_Rules to definitional packages old_primrec, primrec, recdef, size and function
Sun, 07 Mar 2010 12:19:47 +0100 wenzelm modernized structure Object_Logic;
Thu, 25 Feb 2010 22:46:52 +0100 wenzelm modernized structure Split_Rule;
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, 29 Oct 2009 23:56:33 +0100 wenzelm eliminated some old folds;
Thu, 29 Oct 2009 17:58:26 +0100 wenzelm standardized filter/filter_out;
Tue, 27 Oct 2009 22:56:14 +0100 wenzelm eliminated some old folds;
less more (0) -30 tip