src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML
Thu, 10 Feb 2011 16:05:33 +0100 blanchet remove pointless clutter
Thu, 10 Feb 2011 10:09:38 +0100 blanchet make minimizer verbose
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
Mon, 10 Jan 2011 15:45:46 +0100 wenzelm eliminated Int.toString;
Tue, 21 Dec 2010 03:56:51 +0100 blanchet added "smt_triggers" option to experiment with triggers in Sledgehammer;
Sun, 19 Dec 2010 00:13:25 +0100 blanchet reduce the minimizer slack and add verbose information
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)
Fri, 17 Dec 2010 22:15:08 +0100 blanchet more precise error messages in "verbose" (or "debug") mode, following this morning's permission debacle
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 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 11:26:28 +0100 blanchet implemented partially-typed "tags" type encoding
Wed, 15 Dec 2010 11:26:28 +0100 blanchet added "type_sys" option to Sledgehammer
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 split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
Mon, 06 Dec 2010 11:41:24 +0100 blanchet handle "max_relevant" uniformly
Mon, 06 Dec 2010 09:54:58 +0100 blanchet [mq]: sledge_binary_minimizer
Fri, 03 Dec 2010 18:29:14 +0100 blanchet replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
Mon, 15 Nov 2010 18:56:29 +0100 blanchet pick up SMT solver crashes and report them to the user/Mirabelle if desired
Wed, 03 Nov 2010 22:33:23 +0100 blanchet don't be overly verbose in Sledgehammer's minimizer
Wed, 03 Nov 2010 22:26:53 +0100 blanchet standardize on seconds for Nitpick and Sledgehammer timeouts
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 16:56:54 +0200 blanchet remove needless context argument;
Tue, 26 Oct 2010 13:50:57 +0200 blanchet proper error handling for SMT solvers in 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 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 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:54:42 +0200 blanchet got caught once again by SML's pattern maching (ctor vs. var)
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:12:08 +0200 blanchet factored out TSTP/SPASS/Vampire proof parsing;
Tue, 14 Sep 2010 16:34:26 +0200 blanchet handle relevance filter corner cases more gracefully;
Mon, 13 Sep 2010 14:30:21 +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:06:11 +0200 blanchet better error reporting when the Sledgehammer minimizer is interrupted
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 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;
Wed, 01 Sep 2010 16:46:11 +0200 blanchet generalize theorem argument parsing syntax
Tue, 31 Aug 2010 23:50:59 +0200 blanchet finished renaming
Tue, 31 Aug 2010 23:46:23 +0200 blanchet shorten a few file names
less more (0) tip