src/HOL/Tools/Sledgehammer/sledgehammer.ML
Mon, 06 Sep 2010 13:06:27 +0200 some results of concurrency code inspection;
Thu, 02 Sep 2010 22:50:16 +0200 show the number of facts for each prover in "verbose" mode
Thu, 02 Sep 2010 22:15:20 +0200 make sure "Unknown ATP" errors reach the users -- i.e. don't generate them from a thread
Thu, 02 Sep 2010 22:03:25 +0200 If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
Thu, 02 Sep 2010 00:15:53 +0200 show real CPU time
Wed, 01 Sep 2010 23:55:59 +0200 factor out code shared by all ATPs so that it's run only once
Wed, 01 Sep 2010 23:47:05 +0200 handle all whitespace, not just ASCII 32
Wed, 01 Sep 2010 23:41:31 +0200 speed up SPASS hack + output time information in "blocking" mode
Wed, 01 Sep 2010 23:10:01 +0200 minor refactoring
Wed, 01 Sep 2010 23:04:47 +0200 translate the axioms to FOF once and for all ATPs
Wed, 01 Sep 2010 22:33:31 +0200 run relevance filter in a thread, to avoid blocking
Wed, 01 Sep 2010 18:47:07 +0200 only kill ATP threads in nonblocking mode
Wed, 01 Sep 2010 18:41:23 +0200 share the relevance filter among the provers
Wed, 01 Sep 2010 17:27:10 +0200 got rid of the "theory_relevant" option;
Wed, 01 Sep 2010 00:07:31 +0200 rename sledgehammer config attributes
Tue, 31 Aug 2010 23:50:59 +0200 finished renaming
Tue, 31 Aug 2010 23:43:23 +0200 added "expect" feature of Nitpick to Sledgehammer, for regression testing
Tue, 31 Aug 2010 22:27:33 +0200 added "blocking" option to Sledgehammer to run in synchronous mode;
Mon, 30 Aug 2010 11:10:44 +0200 remove useless var
Mon, 30 Aug 2010 09:41:59 +0200 remove needless parameter
Thu, 26 Aug 2010 14:05:22 +0200 improve SPASS hack, when a clause comes from several facts
Thu, 26 Aug 2010 10:42:06 +0200 consider "locality" when assigning weights to facts
Thu, 26 Aug 2010 00:49:38 +0200 renaming
Wed, 25 Aug 2010 19:41:18 +0200 reorganize options regarding to the relevance threshold and decay
Wed, 25 Aug 2010 17:49:52 +0200 make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
Wed, 25 Aug 2010 09:32:43 +0200 get rid of "defs_relevant" feature;
Wed, 25 Aug 2010 09:02:07 +0200 renamed "relevance_convergence" to "relevance_decay"
Tue, 24 Aug 2010 22:57:22 +0200 make sure that "undo_ascii_of" is the inverse of "ascii_of", also for non-printable characters -- and avoid those in ``-style facts
Tue, 24 Aug 2010 18:03:43 +0200 clean handling of whether a fact is chained or not;
Mon, 23 Aug 2010 18:25:49 +0200 weed out junk in relevance filter
Sun, 22 Aug 2010 22:47:03 +0200 be more generous towards SPASS's -SOS mode
Sun, 22 Aug 2010 09:43:10 +0200 prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
Thu, 19 Aug 2010 11:30:48 +0200 tuning
Thu, 19 Aug 2010 11:02:59 +0200 no spurious trailing "\n" at the end of Sledgehammer's output
Wed, 18 Aug 2010 17:16:37 +0200 get rid of "minimize_timeout", now that there's an automatic adaptive timeout mechanism in "minimize"
Wed, 18 Aug 2010 17:09:05 +0200 added "max_relevant_per_iter" option to Sledgehammer
Wed, 18 Aug 2010 09:38:50 +0200 improve SPASS clause numbering hack
Mon, 16 Aug 2010 16:58:45 +0200 more debug output
Mon, 09 Aug 2010 14:08:30 +0200 prevent ATP thread for staying around for 1 minute if an exception occurred earlier;
Mon, 09 Aug 2010 12:05:48 +0200 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
Mon, 09 Aug 2010 10:13:18 +0200 reintroduced old code that removed axioms from the conjecture assumptions, ported to FOF
Mon, 09 Aug 2010 09:57:38 +0200 fix embarrassing bug in elim rule handling, introduced during the port to FOF
Thu, 05 Aug 2010 12:40:12 +0200 fix bug in Nitpick's "equationalize" function (the prems were ignored) + make it do some basic extensionalization
Fri, 30 Jul 2010 00:02:25 +0200 don't choke on synonyms when parsing SPASS's Flotter output + renamings;
Thu, 29 Jul 2010 23:11:35 +0200 fix bug in the newly introduced "bound concealing" code
Thu, 29 Jul 2010 22:43:46 +0200 use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
Thu, 29 Jul 2010 21:20:24 +0200 handle schematic vars the same way in Sledgehammer as in Metis, to avoid unreplayable proofs
Thu, 29 Jul 2010 18:45:41 +0200 speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
Thu, 29 Jul 2010 17:45:22 +0200 work around atomization failures
Thu, 29 Jul 2010 16:41:32 +0200 perform the presimplification done by Metis.make_nnf in Sledgehammer again, to deal with "If" and similar constructs
Thu, 29 Jul 2010 16:11:02 +0200 fix bug with "=" vs. "fequal" introduced by last change (dddb8ba3a1ce)
Thu, 29 Jul 2010 15:50:26 +0200 generate correct names for "$true" and "$false";
Thu, 29 Jul 2010 15:37:27 +0200 don't assume canonical rule format
Thu, 29 Jul 2010 14:53:55 +0200 avoid "clause" and "cnf" terminology where it no longer makes sense
Thu, 29 Jul 2010 14:42:09 +0200 "axiom_clauses" -> "axioms" (these are no longer clauses)
Thu, 29 Jul 2010 14:39:43 +0200 remove the "extra_clauses" business introduced in 19a5f1c8a844;
Wed, 28 Jul 2010 23:01:27 +0200 handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
Wed, 28 Jul 2010 18:54:18 +0200 minor refactoring
Wed, 28 Jul 2010 18:07:25 +0200 fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
Wed, 28 Jul 2010 17:38:40 +0200 revive "e" and "remote_e"'s fact extraction so that it works with E 1.2 as well;