src/HOL/Tools/Sledgehammer/sledgehammer.ML
Thu, 04 Nov 2010 14:59:44 +0100 blanchet cosmetics
Thu, 04 Nov 2010 14:59:44 +0100 blanchet use the SMT integration's official list of built-ins
Wed, 03 Nov 2010 22:26:53 +0100 blanchet standardize on seconds for Nitpick and Sledgehammer timeouts
Thu, 28 Oct 2010 09:36:51 +0200 blanchet clear identification;
Tue, 26 Oct 2010 21:51:04 +0200 blanchet adapted SMT solver error handling to reflect latest changes in "SMT_Solver"
Tue, 26 Oct 2010 21:43:50 +0200 blanchet better list of irrelevant SMT constants
Tue, 26 Oct 2010 21:34:01 +0200 blanchet if "debug" is on, print list of relevant facts (poweruser request);
Tue, 26 Oct 2010 21:01:28 +0200 blanchet standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module
Tue, 26 Oct 2010 20:09:38 +0200 blanchet merge
Tue, 26 Oct 2010 16:56:54 +0200 blanchet remove needless context argument;
Tue, 26 Oct 2010 17:35:51 +0200 boehmes capture out-of-memory warnings of Z3 and turn them into proper exceptions; be more precise about SMT solver run-time: return NONE instead of ~1
Tue, 26 Oct 2010 14:48:55 +0200 blanchet tuning
Tue, 26 Oct 2010 13:50:57 +0200 blanchet proper error handling for SMT solvers in Sledgehammer
Tue, 26 Oct 2010 13:16:43 +0200 blanchet integrated "smt" proof method with Sledgehammer
Mon, 25 Oct 2010 21:06:56 +0200 wenzelm renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
Fri, 22 Oct 2010 18:31:45 +0200 blanchet tuning
Fri, 22 Oct 2010 16:11:43 +0200 blanchet more robust handling of "remote_" vs. non-"remote_" provers
Fri, 22 Oct 2010 15:02:27 +0200 blanchet generalized the relevance filter so that it takes the list of "irrelevant constants" as argument (since the ATP and SMT preprocessing are different)
Fri, 22 Oct 2010 14:47:43 +0200 blanchet replaced references with proper record that's threaded through
Fri, 22 Oct 2010 14:10:32 +0200 blanchet fixed signature of "is_smt_solver_installed";
Fri, 22 Oct 2010 13:57:54 +0200 blanchet renamed modules
Fri, 22 Oct 2010 13:48:21 +0200 blanchet remove more needless code ("run_smt_solvers");
Fri, 22 Oct 2010 12:15:31 +0200 blanchet got rid of duplicate functionality ("run_smt_solver_somehow");
Fri, 22 Oct 2010 11:58:33 +0200 blanchet bring ATPs and SMT solvers more in line with each other
Fri, 22 Oct 2010 11:11:34 +0200 blanchet make Sledgehammer minimizer fully work with SMT
Fri, 22 Oct 2010 09:50:18 +0200 blanchet generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well
Thu, 21 Oct 2010 16:25:40 +0200 blanchet first step in adding support for an SMT backend to Sledgehammer
Thu, 21 Oct 2010 14:55:09 +0200 blanchet use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
Thu, 16 Sep 2010 16:12:02 +0200 blanchet rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
Thu, 16 Sep 2010 15:38:46 +0200 blanchet move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
Thu, 16 Sep 2010 15:28:16 +0200 blanchet skip some "important" messages
Thu, 16 Sep 2010 15:16:08 +0200 blanchet refactoring: move ATP proof and error extraction code to "ATP_Proof" module
Thu, 16 Sep 2010 11:59:45 +0200 blanchet use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
Thu, 16 Sep 2010 11:12:08 +0200 blanchet factored out TSTP/SPASS/Vampire proof parsing;
Tue, 14 Sep 2010 23:01:29 +0200 blanchet finish support for E 1.2 proof reconstruction;
Tue, 14 Sep 2010 19:40:19 +0200 blanchet clarify message
Tue, 14 Sep 2010 19:38:44 +0200 blanchet use same hack as in "Async_Manager" to work around Proof General bug
Tue, 14 Sep 2010 16:34:26 +0200 blanchet handle relevance filter corner cases more gracefully;
Tue, 14 Sep 2010 15:39:57 +0200 blanchet Sledgehammer should be called in "prove" mode;
Mon, 13 Sep 2010 14:29:53 +0200 blanchet tuning
Sat, 11 Sep 2010 12:31:42 +0200 blanchet tuning
Sat, 11 Sep 2010 10:21:52 +0200 blanchet implemented Auto Sledgehammer
Thu, 09 Sep 2010 16:27:36 +0200 blanchet more precise error messages when Vampire is interrupted or SPASS runs into an internal bug
Thu, 09 Sep 2010 16:06:11 +0200 blanchet better error reporting when the Sledgehammer minimizer is interrupted
Wed, 08 Sep 2010 16:01:06 +0200 blanchet merge
Mon, 06 Sep 2010 16:50:29 +0200 blanchet use Future.fork rather than Thread.fork, so that the thread is part of the global thread management
Mon, 06 Sep 2010 13:06:27 +0200 wenzelm some results of concurrency code inspection;
Thu, 02 Sep 2010 22:50:16 +0200 blanchet show the number of facts for each prover in "verbose" mode
Thu, 02 Sep 2010 22:15:20 +0200 blanchet 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 blanchet 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 blanchet show real CPU time
Wed, 01 Sep 2010 23:55:59 +0200 blanchet factor out code shared by all ATPs so that it's run only once
Wed, 01 Sep 2010 23:47:05 +0200 blanchet handle all whitespace, not just ASCII 32
Wed, 01 Sep 2010 23:41:31 +0200 blanchet speed up SPASS hack + output time information in "blocking" mode
Wed, 01 Sep 2010 23:10:01 +0200 blanchet minor refactoring
Wed, 01 Sep 2010 23:04:47 +0200 blanchet translate the axioms to FOF once and for all ATPs
Wed, 01 Sep 2010 22:33:31 +0200 blanchet run relevance filter in a thread, to avoid blocking
Wed, 01 Sep 2010 18:47:07 +0200 blanchet only kill ATP threads in nonblocking mode
Wed, 01 Sep 2010 18:41:23 +0200 blanchet share the relevance filter among the provers
Wed, 01 Sep 2010 17:27:10 +0200 blanchet got rid of the "theory_relevant" option;
less more (0) -100 -60 tip