src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
Thu, 09 Jun 2011 00:16:28 +0200 blanchet tuning
Wed, 08 Jun 2011 16:20:18 +0200 blanchet don't launch the automatic minimizer for zero facts
Wed, 08 Jun 2011 16:20:18 +0200 blanchet renamed option to avoid talking about seconds, since this is now the default Isabelle unit
Wed, 08 Jun 2011 08:47:43 +0200 blanchet make sure that the message tail (timing + TPTP important message) is preserved upon automatic minimization
Tue, 07 Jun 2011 11:04:17 +0200 blanchet use the proper prover name, e.g. metis_full_types, not metis (full_types), for minimizing
Mon, 06 Jun 2011 20:36:34 +0200 blanchet refined auto minimization code: don't use Metis if Isar proofs are desired, and fall back on prover if Metis is too slow
Mon, 06 Jun 2011 20:36:34 +0200 blanchet tuning
Tue, 31 May 2011 16:38:36 +0200 blanchet first step in sharing more code between ATP and Metis translation
Mon, 30 May 2011 17:00:38 +0200 blanchet made "explicit_apply" smarter -- no need to force explicit applications in minimizer on all constants, better do it more fine granularly
Mon, 30 May 2011 17:00:38 +0200 blanchet make all messages urgent in verbose mode
Mon, 30 May 2011 17:00:38 +0200 blanchet minimize automatically even if Metis failed, if the external prover was really fast
Mon, 30 May 2011 17:00:38 +0200 blanchet automatically minimize with Metis when this can be done within a few seconds
Mon, 30 May 2011 17:00:38 +0200 blanchet minimize with Metis if possible
Sun, 29 May 2011 19:40:56 +0200 blanchet normalize indices in chained facts to make sure that backtick facts (which often result in different names) are recognized + changed definition of urgent messages
Fri, 27 May 2011 10:30:08 +0200 blanchet cleanup proof text generation code
Fri, 27 May 2011 10:30:08 +0200 blanchet make Sledgehammer a little bit less verbose in "try"
Fri, 27 May 2011 10:30:08 +0200 blanchet handle non-auto try case of Sledgehammer better
Fri, 27 May 2011 10:30:08 +0200 blanchet added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
Fri, 27 May 2011 10:30:07 +0200 blanchet make output more concise
Fri, 27 May 2011 10:30:07 +0200 blanchet merge timeout messages from several ATPs into one message to avoid clutter
Fri, 27 May 2011 10:30:07 +0200 blanchet fix soundness bug in Sledgehammer: distinguish params in goals from fixed variables in context
Tue, 24 May 2011 10:01:03 +0200 blanchet more work on parsing LEO-II proofs and extracting uses of extensionality
Tue, 24 May 2011 10:00:38 +0200 blanchet more work on parsing LEO-II proofs without lambdas
Tue, 24 May 2011 00:01:33 +0200 blanchet tuning -- the "appropriate" terminology is inspired from TPTP
Sun, 22 May 2011 14:51:42 +0200 blanchet added message when Waldmeister isn't run
Sun, 22 May 2011 14:51:42 +0200 blanchet improved Waldmeister support -- even run it by default on unit equational goals
Thu, 19 May 2011 10:24:13 +0200 blanchet distinguish between a soft timeout (30 s by defalt) and a hard timeout (60 s), to let minimization-based provers (such as CVC3, Yices, and occasionally the other provers) do their job
Tue, 03 May 2011 00:10:22 +0200 blanchet replaced some Unsynchronized.refs with Config.Ts
Mon, 02 May 2011 22:52:15 +0200 blanchet tuning
Mon, 02 May 2011 22:52:15 +0200 blanchet have each ATP filter out dangerous facts for themselves, based on their type system
Mon, 02 May 2011 14:40:57 +0200 blanchet use strings to encode type systems in ATP module, to reduce the amount of out-of-place information and also to make it easier to print the type system used
Sun, 01 May 2011 18:37:25 +0200 blanchet restructured type systems some more -- the old naming schemes had "argshg diff |less" and "tagshg diff |less" as equivalent and didn't support a monomorphic version of "tags"
Sun, 01 May 2011 18:37:25 +0200 blanchet implement the new ATP type system in Sledgehammer
Sun, 01 May 2011 18:37:24 +0200 blanchet reimplemented the hAPP introduction code so that it's done earlier, when the types are still available
Sun, 01 May 2011 18:37:24 +0200 blanchet perform constant mangling and/or removal of its type args in an earlier phase, so that the rest of the code doesn't need to worry about it
Thu, 21 Apr 2011 22:18:28 +0200 blanchet detect some unsound proofs before showing them to the user
Thu, 21 Apr 2011 18:39:22 +0200 blanchet cleanup: get rid of "may_slice" arguments without changing semantics
Thu, 21 Apr 2011 18:39:22 +0200 blanchet implemented general slicing for ATPs, especially E 1.2w and above
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Thu, 31 Mar 2011 11:16:52 +0200 blanchet added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
Thu, 17 Mar 2011 11:18:31 +0100 blanchet add option to function to keep trivial ATP formulas, needed for some experiments
Mon, 21 Feb 2011 10:29:00 +0100 blanchet added a timeout around SMT preprocessing (notably monomorphization)
Fri, 18 Feb 2011 16:30:44 +0100 blanchet gracious timeout in "blocking" mode
Thu, 10 Feb 2011 16:15:43 +0100 blanchet run all provers in blocking mode, even if a proof was already found -- this behavior is less confusing to the user
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
less more (0) -60 tip