src/Pure/simplifier.ML
Wed, 30 Sep 2009 22:25:50 +0200 wenzelm eliminated dead code;
Tue, 29 Sep 2009 11:49:22 +0200 wenzelm explicit indication of Unsynchronized.ref;
Thu, 23 Jul 2009 18:44:08 +0200 wenzelm renamed simpset_of to global_simpset_of, and local_simpset_of to simpset_of -- same for claset and clasimpset;
Tue, 21 Jul 2009 01:03:18 +0200 wenzelm proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
Sat, 30 May 2009 12:53:11 +0200 wenzelm modernized method setup;
Fri, 20 Mar 2009 17:12:37 +0100 wenzelm Disposed old declarations, tactics, tactic combinators that refer to the simpset or claset of an implicit theory;
Sun, 15 Mar 2009 15:59:44 +0100 wenzelm simplified attribute setup;
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;
Thu, 12 Mar 2009 11:10:02 +0100 wenzelm renamed NameSpace.bind to NameSpace.define;
Sun, 08 Mar 2009 12:15:58 +0100 wenzelm added dest_ss;
Sat, 07 Mar 2009 11:45:56 +0100 wenzelm renamed rep_ss to MetaSimplifier.internal_ss;
Wed, 21 Jan 2009 23:21:44 +0100 wenzelm removed Ids;
Fri, 05 Dec 2008 08:04:53 +0100 haftmann dropped NameSpace.declare_base
Thu, 04 Dec 2008 14:43:33 +0100 haftmann cleaned up binding module and related code
Thu, 20 Nov 2008 19:06:02 +0100 haftmann dropped legacy naming code
Fri, 14 Nov 2008 08:50:10 +0100 haftmann namify and name_decl combinators
Thu, 13 Nov 2008 14:19:09 +0100 haftmann consider prefixes for name bindings of simprocs (a first approximation)
Tue, 02 Sep 2008 14:10:19 +0200 wenzelm name/var morphism operates on Name.binding;
Tue, 24 Jun 2008 19:43:14 +0200 wenzelm ML_Antiquote.value;
Thu, 29 May 2008 23:46:43 +0200 wenzelm proper context for attribute simplified;
Tue, 15 Apr 2008 16:12:05 +0200 wenzelm Thm.forall_elim_var(s);
Sat, 29 Mar 2008 22:55:57 +0100 wenzelm purely functional setup of claset/simpset/clasimpset;
Fri, 28 Mar 2008 20:02:04 +0100 wenzelm Context.>> : operate on Context.generic;
Thu, 27 Mar 2008 15:32:15 +0100 wenzelm eliminated delayed theory setup
Thu, 27 Mar 2008 14:41:10 +0100 wenzelm renamed ML_Context.the_context to ML_Context.the_global_context;
Sat, 01 Sep 2007 15:47:01 +0200 wenzelm replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
Thu, 02 Aug 2007 12:06:27 +0200 wenzelm turned simp_depth_limit into configuration option;
Sat, 28 Jul 2007 20:40:30 +0200 wenzelm added attribute "simproc";
Sun, 08 Jul 2007 19:51:58 +0200 wenzelm replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
Thu, 05 Jul 2007 20:01:35 +0200 wenzelm tuned;
Tue, 03 Jul 2007 17:17:11 +0200 wenzelm moved (asm_)rewrite_goal_tac from goal.ML to meta_simplifier.ML (no longer depends on SELECT_GOAL);
Thu, 24 May 2007 08:37:37 +0200 haftmann tuned Pure/General/name_space.ML
Mon, 07 May 2007 00:49:59 +0200 wenzelm simplified DataFun interfaces;
Mon, 23 Apr 2007 20:44:09 +0200 wenzelm def_simproc(_i): proper ProofContext.read/cert_terms;
Mon, 16 Apr 2007 16:11:03 +0200 haftmann canonical merge operations
Sun, 15 Apr 2007 23:25:50 +0200 wenzelm removed obsolete TypeInfer.logicT -- use dummyT;
Wed, 28 Feb 2007 22:05:44 +0100 wenzelm exported get_ss, map_ss;
Sun, 04 Feb 2007 22:02:16 +0100 wenzelm def_simproc(_i): tuned interface;
Mon, 29 Jan 2007 19:58:14 +0100 wenzelm added get_simproc, @{simproc};
Sun, 28 Jan 2007 23:29:15 +0100 wenzelm added def_simproc(_i) -- define named simprocs;
Sat, 20 Jan 2007 14:09:17 +0100 wenzelm added @{simpset};
Fri, 19 Jan 2007 22:08:02 +0100 wenzelm moved ML context stuff to from Context to ML_Context;
Thu, 07 Dec 2006 23:16:55 +0100 wenzelm reorganized structure Tactic vs. MetaSimplifier;
Thu, 07 Dec 2006 00:42:04 +0100 wenzelm reorganized structure Goal vs. Tactic;
Fri, 10 Nov 2006 07:44:47 +0100 haftmann introduces canonical AList functions for loop_tacs
Sat, 07 Oct 2006 01:30:58 +0200 wenzelm tuned;
Fri, 10 Feb 2006 02:22:16 +0100 wenzelm Args/Attrib syntax: Context.generic;
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 22:25:34 +0100 wenzelm generic attributes;
Tue, 10 Jan 2006 19:33:27 +0100 wenzelm Attrib.rule;
Fri, 28 Oct 2005 22:28:02 +0200 wenzelm export cong_modifiers, simp_modifiers';
Fri, 21 Oct 2005 18:14:47 +0200 wenzelm added simplification tactics and rules (from meta_simplifier.ML);
Tue, 18 Oct 2005 17:59:31 +0200 wenzelm renamed set_context to context;
Mon, 17 Oct 2005 23:10:21 +0200 wenzelm removed obsolete/experimental context components (superceded by Simplifier.the_context);
Thu, 29 Sep 2005 15:50:46 +0200 wenzelm export debug_bounds;
Tue, 02 Aug 2005 19:47:14 +0200 wenzelm export clear_ss;
Mon, 01 Aug 2005 19:20:43 +0200 wenzelm export MataSimplifier.inherit_bounds;
Wed, 13 Jul 2005 16:07:27 +0200 wenzelm removed obsolete delta stuff;
less more (0) -60 tip