src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
Tue, 08 Feb 2011 16:10:06 +0100 blanchet enable SMT weights and triggers, since they lead to slight improvements according to the Judgment Day suite
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 04:33:17 +0100 blanchet proper handling of the arguments of SMT builtins -- for numerals, ignore the arguments (Pls, Bit0, Bit1, ..), for functions, consider them;
Tue, 21 Dec 2010 03:56:51 +0100 blanchet added "smt_triggers" option to experiment with triggers in Sledgehammer;
Mon, 20 Dec 2010 14:55:24 +0100 blanchet run SPASS and Vampire in SOS mode only if >= 50 facts are passed -- otherwise we are probably minimizing and then it's better if the prover is run only once with a full strategy
Mon, 20 Dec 2010 14:09:45 +0100 blanchet remove spurious line
Mon, 20 Dec 2010 12:12:35 +0100 blanchet optionally supply constant weights to E -- turned off by default until properly parameterized
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 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 15:30:43 +0100 blanchet run the SMT relevance filter only once, then run the normalization/monomorphization code once _per class_ of SMT solvers
Fri, 17 Dec 2010 12:10:08 +0100 blanchet make timeout part of the SMT filter's tail
Fri, 17 Dec 2010 12:02:46 +0100 blanchet split "smt_filter" into head and tail
Fri, 17 Dec 2010 09:56:04 +0100 blanchet trap one more Z3 error
Fri, 17 Dec 2010 00:27:40 +0100 blanchet more precise/correct SMT error handling
Thu, 16 Dec 2010 22:45:02 +0100 blanchet discriminate SMT errors a bit better
Thu, 16 Dec 2010 15:46:54 +0100 blanchet no need to do a super-duper atomization if Metis fails afterwards anyway
Thu, 16 Dec 2010 15:12:17 +0100 blanchet robustly handle SMT exceptions in Sledgehammer
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 18:10:32 +0100 blanchet facilitate debugging
Wed, 15 Dec 2010 17:14:44 +0100 blanchet clean up fudge factors a little bit
Wed, 15 Dec 2010 16:42:07 +0100 blanchet added weights to SMT problems
Wed, 15 Dec 2010 12:08:41 +0100 blanchet honor "overlord" option for SMT solvers as well and don't pass "ext" to them
Wed, 15 Dec 2010 11:26:29 +0100 blanchet crank up Metis's timeout for SMT solvers, since users love Metis
Wed, 15 Dec 2010 11:26:29 +0100 blanchet generate a "using [[smt_solver = ...]]" command if a proof is found by another SMT solver than the current one, to ensure it's also used for reconstruction
Wed, 15 Dec 2010 11:26:28 +0100 blanchet added Sledgehammer support for higher-order propositional reasoning
Wed, 15 Dec 2010 11:26:28 +0100 blanchet implemented partially-typed "tags" type encoding
Wed, 15 Dec 2010 11:26:28 +0100 blanchet implemented new type system encoding "overload_args", which is more lightweight than "const_args" (the unsound default) and hopefully almost as sound
Wed, 15 Dec 2010 11:26:28 +0100 blanchet added "type_sys" option to Sledgehammer
Wed, 15 Dec 2010 08:39:24 +0100 boehmes re-ordered SMT normalization code (eta-normalization, lambda abstractions and partial functions will be dealt with on the term level);
Fri, 10 Dec 2010 09:18:17 +0100 krauss made smlnj happy
Wed, 08 Dec 2010 22:18:37 +0100 blanchet lower fudge factor
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