src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
Wed, 09 Feb 2011 17:18:58 +0100 blanchet tuning
Wed, 09 Feb 2011 17:18:58 +0100 blanchet automatically minimize Z3-as-an-ATP proofs (cf. CVC3 and Yices)
Wed, 09 Feb 2011 17:18:58 +0100 blanchet renamed field
Tue, 08 Feb 2011 16:10:10 +0100 blanchet available_provers ~> supported_provers (for clarity)
Thu, 06 Jan 2011 17:51:56 +0100 boehmes differentiate between local and remote SMT solvers (e.g., "z3" vs. "remote_z3");
Tue, 21 Dec 2010 03:56:51 +0100 blanchet added "smt_triggers" option to experiment with triggers in Sledgehammer;
Mon, 20 Dec 2010 14:10:40 +0100 blanchet make exceptions more transparent in "debug" mode
Sat, 18 Dec 2010 14:02:14 +0100 blanchet tuning
Sat, 18 Dec 2010 13:43:46 +0100 blanchet lower threshold where the binary algorithm kick in and use the same value for automatic minimization
Sat, 18 Dec 2010 13:34:32 +0100 blanchet let each prover minimizes its own stuff (rather than taking the first prover of the list to minimize every prover's stuff)
Sat, 18 Dec 2010 12:53:56 +0100 blanchet renamed function to run prover with minimizer and changed signature to clarify its semantics and make it a drop in replacement for "get_prover"
Sat, 18 Dec 2010 12:46:58 +0100 blanchet factored out running a prover with (optionally) an implicit minimizer phrase
Fri, 17 Dec 2010 23:09:53 +0100 blanchet remove option that doesn't work in Mirabelle anyway (Mirabelle uses Sledgehammer_Provers, not Sledgehammer_Run)
Fri, 17 Dec 2010 21:31:19 +0100 blanchet put the SMT weights back where they belong, so that they're also used by Mirabelle
Fri, 17 Dec 2010 18:23:56 +0100 blanchet added debugging option to find out how good the relevance filter was at identifying relevant facts
Fri, 17 Dec 2010 16:55:27 +0100 blanchet export experimental options
Fri, 17 Dec 2010 15:30:43 +0100 blanchet run the SMT relevance filter only once, then run the normalization/monomorphization code once _per class_ of SMT solvers
Thu, 16 Dec 2010 15:12:17 +0100 blanchet make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
Wed, 15 Dec 2010 19:41:24 +0100 blanchet make sure errors generated in a thread don't vanish in cyberspace (e.g., when invoking Sledgehammer with unknown facts)
Wed, 15 Dec 2010 18:10:32 +0100 blanchet facilitate debugging
Wed, 15 Dec 2010 11:26:28 +0100 blanchet weaken the "expect" flag so that it doesn't trigger errors if a prover is not installed
Wed, 15 Dec 2010 11:26:28 +0100 blanchet implemented partially-typed "tags" type encoding
Wed, 08 Dec 2010 22:17:53 +0100 blanchet implicitly call the minimizer for SMT solvers that don't return an unsat core
Wed, 08 Dec 2010 22:17:52 +0100 blanchet renamings
Wed, 08 Dec 2010 22:17:52 +0100 blanchet moved function to later module
Wed, 08 Dec 2010 22:17:52 +0100 blanchet clarified terminology
Wed, 08 Dec 2010 22:17:52 +0100 blanchet split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
less more (0) tip