src/Pure/simplifier.ML
Tue, 21 Apr 2020 07:28:17 +0000 haftmann hooks for foundational terms: protection of foundational terms during simplification
Thu, 05 Dec 2019 09:24:34 +0000 haftmann more direct accessors for simpset
Tue, 20 Aug 2019 11:01:05 +0200 wenzelm clarified signature;
Mon, 03 Jun 2019 15:40:08 +0200 wenzelm clarified signature;
Fri, 04 Jan 2019 21:49:06 +0100 wenzelm support for isabelle update -u control_cartouches;
Tue, 27 Nov 2018 21:07:39 +0100 wenzelm more accurate positions for "name" (quoted string) and "embedded" (cartouche): refer to content without delimiters, which is e.g. relevant for systematic selection/renaming of scope groups;
Wed, 06 Jun 2018 18:19:55 +0200 nipkow reorient -> split; documented split
Thu, 26 Apr 2018 19:51:32 +0200 nipkow new simp modifier: reorient
Thu, 01 Feb 2018 15:31:25 +0100 wenzelm clarified signature: prefer proper order operation;
Wed, 06 Dec 2017 18:59:33 +0100 wenzelm prefer control symbol antiquotations;
Wed, 06 Dec 2017 15:46:35 +0100 wenzelm more embedded cartouche arguments;
Tue, 13 Dec 2016 11:51:42 +0100 wenzelm more symbols;
Wed, 20 Jul 2016 22:36:10 +0200 wenzelm provide Pure.simp/simp_all, which only know about meta-equality;
Thu, 02 Jun 2016 16:23:10 +0200 wenzelm avoid warnings on duplicate rules in the given list;
Fri, 08 Apr 2016 20:15:20 +0200 wenzelm eliminated unused simproc identifier;
Wed, 16 Dec 2015 16:31:36 +0100 wenzelm rule_attribute and declaration_attribute implicitly support abstract closure, but mixed_attribute implementations need to be aware of Thm.is_free_dummy;
Sun, 13 Dec 2015 21:56:15 +0100 wenzelm more general types Proof.method / context_tactic;
Fri, 25 Sep 2015 20:37:59 +0200 wenzelm moved remaining display.ML to more_thm.ML;
Wed, 09 Sep 2015 23:01:27 +0200 wenzelm clarified declaration flags, like 'declaration' command;
Wed, 09 Sep 2015 20:57:21 +0200 wenzelm simplified simproc programming interfaces;
Wed, 02 Sep 2015 23:31:41 +0200 wenzelm eliminated pointless cterms;
Fri, 03 Apr 2015 19:56:51 +0200 wenzelm more uniform "verbose" option to print name space;
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Sun, 01 Mar 2015 23:35:41 +0100 wenzelm added Proof_Context.cterm_of/ctyp_of convenience;
Tue, 10 Feb 2015 14:48:26 +0100 wenzelm proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
Mon, 10 Nov 2014 21:49:48 +0100 wenzelm proper context for assume_tac (atac remains as fall-back without context);
Sun, 09 Nov 2014 17:04:14 +0100 wenzelm proper context for match_tac etc.;
Wed, 27 Aug 2014 14:54:32 +0200 wenzelm more explicit Method.modifier with reported position;
Tue, 19 Aug 2014 17:00:44 +0200 wenzelm added PARALLEL_ALLGOALS convenience;
Thu, 10 Apr 2014 12:22:29 +0200 wenzelm added simproc markup, which also indicates legacy simprocs outside the name space;
Tue, 18 Mar 2014 15:29:58 +0100 wenzelm more antiquotations;
Wed, 12 Mar 2014 22:57:50 +0100 wenzelm tuned signature -- clarified module name;
Sun, 12 Jan 2014 18:34:00 +0100 wenzelm proper context for clear_simpset: preserve dounds, depth;
Thu, 12 Dec 2013 22:38:25 +0100 wenzelm clarified Trace_Ops: global theory data avoids init of simpset in Pure.thy, which is important to act as neutral element in merge;
Thu, 12 Dec 2013 21:14:33 +0100 wenzelm generic trace operations for main steps of Simplifier;
Thu, 12 Dec 2013 17:34:50 +0100 wenzelm tuned signature;
Mon, 11 Nov 2013 20:50:12 +0100 wenzelm tuned signature -- removed obsolete Addsimprocs, Delsimprocs;
Fri, 23 Aug 2013 20:35:50 +0200 wenzelm added Theory.setup convenience;
Wed, 26 Jun 2013 21:48:23 +0200 wenzelm less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Wed, 10 Apr 2013 17:27:38 +0200 wenzelm obsolete -- tools should refer to proper Proof.context;
Sat, 30 Mar 2013 17:13:21 +0100 wenzelm more formal cong_name;
Sat, 30 Mar 2013 13:40:19 +0100 wenzelm more item markup;
Fri, 29 Mar 2013 22:14:27 +0100 wenzelm Pretty.item markup for improved readability of lists of items;
Sat, 17 Nov 2012 17:55:52 +0100 wenzelm tuned signature;
Sat, 11 Aug 2012 22:17:46 +0200 wenzelm faster compilation of ML with antiquotations: static ML_context is bound once in auxiliary structure Isabelle;
Sat, 14 Apr 2012 17:15:57 +0200 wenzelm outermost SELECT_GOAL potentially improves performance;
Sat, 31 Mar 2012 19:26:23 +0200 wenzelm tuned signature;
Sun, 18 Mar 2012 13:04:22 +0100 wenzelm maintain generic context naming in structure Name_Space (NB: empty = default_naming, init = local_naming);
Sat, 17 Mar 2012 23:55:03 +0100 wenzelm proper naming of simprocs according to actual target context;
Sat, 03 Mar 2012 21:52:15 +0100 wenzelm tuned;
Tue, 14 Feb 2012 19:29:54 +0100 wenzelm tuned signature;
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;
Wed, 23 Nov 2011 22:59:39 +0100 wenzelm modernized some old-style infix operations, which were left over from the time of ML proof scripts;
Sun, 06 Nov 2011 21:51:46 +0100 wenzelm more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
Thu, 03 Nov 2011 22:15:47 +0100 wenzelm tuned -- Variable.declare_term is already part of Variable.auto_fixes;
Fri, 28 Oct 2011 22:17:30 +0200 wenzelm uniform Local_Theory.declaration with explicit params;
Fri, 28 Oct 2011 17:15:52 +0200 wenzelm tuned signature -- refined terminology;
Mon, 08 Aug 2011 17:23:15 +0200 wenzelm misc tuning -- eliminated old-fashioned rep_thm;
Wed, 29 Jun 2011 21:34:16 +0200 wenzelm tuned signature;
Wed, 29 Jun 2011 20:39:41 +0200 wenzelm simplified/unified Simplifier.mk_solver;
Mon, 27 Jun 2011 16:53:31 +0200 wenzelm ML antiquotations are managed as theory data, with proper name space and entity markup;
Fri, 13 May 2011 23:58:40 +0200 wenzelm clarified map_simpset versus Simplifier.map_simpset_global;
Fri, 13 May 2011 22:55:00 +0200 wenzelm proper Proof.context for classical tactics;
Sat, 23 Apr 2011 17:02:12 +0200 wenzelm added Name_Space.check/get convenience;
Sat, 23 Apr 2011 16:30:00 +0200 wenzelm clarified check_simproc (with report) vs. the_simproc;
Sat, 23 Apr 2011 13:53:09 +0200 wenzelm proper binding/report of defined simprocs;
Sun, 17 Apr 2011 19:54:04 +0200 wenzelm report Name_Space.declare/define, relatively to context;
Sat, 16 Apr 2011 23:41:25 +0200 wenzelm PARALLEL_GOALS for method "simp_all";
Sat, 16 Apr 2011 15:47:52 +0200 wenzelm modernized structure Proof_Context;
Wed, 22 Dec 2010 20:08:40 +0100 haftmann tuned comment
Fri, 17 Dec 2010 20:21:35 +0100 wenzelm more explicit references to structure Raw_Simplifier;
Fri, 17 Dec 2010 17:08:56 +0100 wenzelm renamed structure MetaSimplifier to raw_Simplifer, to emphasize its meaning;
Fri, 17 Dec 2010 14:09:37 +0100 wenzelm clarified exports of structure Simplifier;
Wed, 25 Aug 2010 18:36:22 +0200 wenzelm renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
Tue, 15 Jun 2010 14:28:08 +0200 haftmann tuned whitespace
Mon, 31 May 2010 21:06:57 +0200 wenzelm modernized some structure names, keeping a few legacy aliases;
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 23:33:42 +0200 wenzelm export Simplifier.with_context;
Fri, 30 Apr 2010 17:18:29 +0200 wenzelm conditional warnings: explicitly observe context visibility flag, not just accidental presence of a context;
Thu, 29 Apr 2010 22:56:32 +0200 wenzelm proper context for mksimps etc. -- via simpset of the running Simplifier;
Sat, 06 Mar 2010 15:39:16 +0100 wenzelm eliminated Args.bang_facts (legacy feature);
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;
Fri, 13 Nov 2009 21:11:15 +0100 wenzelm modernized structure Local_Theory;
Tue, 10 Nov 2009 15:32:43 +0100 wenzelm define simprocs: do not apply target_morphism prematurely, this is already done in LocalTheory.declaration;
Sun, 08 Nov 2009 16:30:41 +0100 wenzelm adapted Generic_Data, Proof_Data;
Thu, 05 Nov 2009 22:08:47 +0100 wenzelm adapted LocalTheory.declaration;
Sun, 25 Oct 2009 19:19:35 +0100 wenzelm LocalTheory.naming_of;
Sun, 25 Oct 2009 13:04:06 +0100 wenzelm make SML/NJ happy;
Sat, 24 Oct 2009 20:54:08 +0200 wenzelm maintain explicit name space kind;
Sat, 24 Oct 2009 19:47:37 +0200 wenzelm renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
Sat, 24 Oct 2009 19:20:03 +0200 wenzelm eliminated separate stamp -- NameSpace.define/merge etc. ensure uniqueness already;
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;
less more (0) -120 tip