src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML
Wed, 24 Aug 2011 11:17:33 +0200 more reliable "sledgehammer\_tac" reconstruction, by avoiding "insert_tac"
Mon, 22 Aug 2011 15:02:45 +0200 removed unused configuration option
Mon, 27 Jun 2011 22:44:44 +0200 merged
Mon, 27 Jun 2011 15:03:55 +0200 old gensym is now legacy -- global state is out of fashion, and its result is not guaranteed to be fresh;
Mon, 27 Jun 2011 14:56:33 +0200 don't export any metastrange or other nonatomizable formulas, since these don't help proving normal things, they are somewhat broken in the ATP output, and they are atypical
Tue, 21 Jun 2011 17:17:38 +0200 insert rather than append special facts to make it less likely that they're truncated away
Mon, 20 Jun 2011 10:41:02 +0200 respect "really_all" argument, which is used by "ATP_Export"
Thu, 16 Jun 2011 13:50:35 +0200 fixed soundness bug related to extensionality
Fri, 10 Jun 2011 12:01:15 +0200 compute the set of base facts only once (instead of three times in parallel) -- this saves about .5 s of CPU time, albeit much less clock wall time
Thu, 09 Jun 2011 16:34:49 +0200 discontinued Name.variant to emphasize that this is old-style / indirect;
Tue, 07 Jun 2011 14:17:35 +0200 optimized the relevance filter a little bit
Tue, 31 May 2011 16:38:36 +0200 first step in sharing more code between ATP and Metis translation
Mon, 30 May 2011 17:00:38 +0200 fixed bug in appending special facts introduced in be0e66ccebfa -- if several special facts were added, they overwrote each other
Tue, 24 May 2011 00:01:33 +0200 use "eq_thm_prop" for slacker comparison -- ensures that backtick-quoted chained facts are recognized in the minimizer, among other things
Tue, 24 May 2011 00:01:33 +0200 tuning -- the "appropriate" terminology is inspired from TPTP
Sun, 22 May 2011 14:51:42 +0200 improved Waldmeister support -- even run it by default on unit equational goals
Tue, 17 May 2011 15:11:36 +0200 append special boring facts rather than prepend them, to avoid confusing E's weighting mechanism
Sun, 15 May 2011 16:40:24 +0200 tuned signature;
Sat, 14 May 2011 21:42:17 +0200 slightly more efficient claset operations, using Item_Net to maintain rules in canonical order;
Thu, 12 May 2011 15:29:19 +0200 do not pollute relevance filter facts with too many facts about the boring set constants Collect and mem_def, which we might anyway unfold depending on Meson's settings
Thu, 12 May 2011 15:29:19 +0200 remove unused parameter
Thu, 12 May 2011 15:29:19 +0200 fine-tuned the relevance filter, so that equations of the form "c = (%x. _)" and constants occurring in chained facts are not unduely penalized
Thu, 12 May 2011 15:29:19 +0200 no penality for constants that appear in chained facts
Thu, 12 May 2011 15:29:19 +0200 improve detection of quantifications over dangerous types by leveraging "is_type_surely_finite" predicate and added "prop" to the list of surely finite types
Thu, 12 May 2011 15:29:19 +0200 tune whitespace
Thu, 12 May 2011 15:29:19 +0200 added configuration options for experimental features
Thu, 05 May 2011 14:18:58 +0200 tuning
Wed, 04 May 2011 19:35:48 +0200 exploit inferred monotonicity
Tue, 03 May 2011 21:46:49 +0200 fixed per-ATP dangerous axiom detection -- embarrassing bugs introduced in change a7a30721767a
Tue, 03 May 2011 00:10:22 +0200 replaced some Unsynchronized.refs with Config.Ts
Mon, 02 May 2011 22:52:15 +0200 recognize simplification rules even if they look a bit different from the theorems in the theories (meta equality, variable numbers)
Mon, 02 May 2011 22:52:15 +0200 have each ATP filter out dangerous facts for themselves, based on their type system
Sun, 01 May 2011 18:37:25 +0200 restructured type systems some more -- the old naming schemes had "argshg diff |less" and "tagshg diff |less" as equivalent and didn't support a monomorphic version of "tags"
Sun, 01 May 2011 18:37:25 +0200 implement the new ATP type system in Sledgehammer
Thu, 21 Apr 2011 22:18:28 +0200 detect some unsound proofs before showing them to the user
Sat, 16 Apr 2011 16:15:37 +0200 modernized structure Proof_Context;
Sat, 16 Apr 2011 13:48:45 +0200 Name_Space: proper configuration options long_names, short_names, unique_names instead of former unsynchronized references;
Fri, 08 Apr 2011 16:34:14 +0200 discontinued special treatment of structure Lexicon;
Fri, 18 Mar 2011 22:55:28 +0100 added "simp:", "intro:", and "elim:" to "try" command
Thu, 17 Mar 2011 11:18:31 +0100 add option to relevance filter's "all_facts" function to really get all facts (needed for some experiments)
Mon, 21 Feb 2011 10:31:48 +0100 give more weight to Frees than to Consts in relevance filter
Thu, 17 Feb 2011 12:14:47 +0100 export more functionality of Sledgehammer to applications (for experiments)
Wed, 16 Feb 2011 19:07:53 +0100 export useful function (needed in a Sledgehammer-related experiment)
Mon, 10 Jan 2011 15:45:46 +0100 eliminated Int.toString;
Tue, 21 Dec 2010 04:33:17 +0100 proper handling of the arguments of SMT builtins -- for numerals, ignore the arguments (Pls, Bit0, Bit1, ..), for functions, consider them;
Sun, 19 Dec 2010 13:25:18 +0100 escape backticks in altstrings
Sat, 18 Dec 2010 21:07:34 +0100 made the relevance filter treat unatomizable facts like "atomize_all" properly (these result in problems that get E spinning seemingly forever);
Thu, 16 Dec 2010 15:46:54 +0100 no need to do a super-duper atomization if Metis fails afterwards anyway
Thu, 16 Dec 2010 15:12:17 +0100 reintroduce the higher penalty for skolems
Thu, 16 Dec 2010 15:12:17 +0100 comment tuning
Thu, 16 Dec 2010 15:12:17 +0100 get rid of experimental feature of term patterns in relevance filter -- doesn't work well unless we take into consideration the equality theory entailed by the relevant facts
Thu, 16 Dec 2010 15:12:17 +0100 make it more likely that induction rules are picked up by Sledgehammer
Thu, 16 Dec 2010 15:12:17 +0100 add the current theory's constant to the goal to make theorems from the current theory more relevant on the first iteration already
Thu, 16 Dec 2010 15:12:17 +0100 instantiate induction rules automatically
Wed, 15 Dec 2010 16:42:06 +0100 move facts supplied with "add:" to the front, so that they get a better weight (SMT)
Wed, 15 Dec 2010 12:08:41 +0100 honor "overlord" option for SMT solvers as well and don't pass "ext" to them
Wed, 15 Dec 2010 11:26:29 +0100 make Sledgehammer's relevance filter include the "ext" rule when appropriate
Wed, 15 Dec 2010 11:26:28 +0100 added Sledgehammer support for higher-order propositional reasoning
Wed, 15 Dec 2010 11:26:28 +0100 implemented partially-typed "tags" type encoding
Tue, 07 Dec 2010 16:27:07 +0100 pass constant arguments to the built-in check function, cf. d2b1fc1b8e19