src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML
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 00:01:33 +0200 blanchet detect inappropriate problems and crashes better in Waldmeister
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 improved Waldmeister support -- even run it by default on unit equational goals
Thu, 12 May 2011 15:29:18 +0200 blanchet added "force_sos" options to control SPASS's and Vampire's use of SOS in experiments + added corresponding Mirabelle options
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
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
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:51 +0200 blanchet added support for "dest:" to "try"
Fri, 18 Mar 2011 22:55:28 +0100 blanchet added "simp:", "intro:", and "elim:" to "try" command
Fri, 11 Feb 2011 11:54:24 +0100 blanchet added option to Mirabelle Sledgehammer
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 10:18:56 +0100 blanchet added "sledgehammer_tac" as possible reconstructor in Mirabelle
Tue, 21 Dec 2010 06:53:20 +0100 blanchet avoid weird symbols in path
Tue, 21 Dec 2010 06:06:28 +0100 blanchet mechanism to keep SMT input and output files around in Mirabelle
Sat, 18 Dec 2010 23:31:22 +0100 blanchet two layers of timeouts seem to be less reliable than a single layer
Sat, 18 Dec 2010 22:15:39 +0100 blanchet move relevance filter into hard timeout
Sat, 18 Dec 2010 21:24:34 +0100 blanchet handle timeouts in Mirabelle more gracefully
Sat, 18 Dec 2010 13:48:24 +0100 blanchet higher hard timeout
Sat, 18 Dec 2010 13:38:14 +0100 blanchet compile
Sat, 18 Dec 2010 12:55:33 +0100 blanchet use minimizing prover in Mirabelle
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 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:20:02 +0100 blanchet compile
Thu, 16 Dec 2010 15:44:32 +0100 blanchet removed unused variable
Thu, 16 Dec 2010 15:12:17 +0100 blanchet tuning
Wed, 15 Dec 2010 11:26:29 +0100 blanchet added support for "type_sys" option to Mirabelle
Wed, 15 Dec 2010 11:26:29 +0100 blanchet honor "metisFT" in Mirabelle
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 split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
Mon, 06 Dec 2010 11:41:24 +0100 blanchet handle "max_relevant" uniformly
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
Thu, 25 Nov 2010 14:13:48 +0100 blanchet reverted c059d550afec -- the triviality check had apparently nothing to do with spontaneous Interrupt exceptions
Tue, 23 Nov 2010 23:10:13 +0100 blanchet disable triviality checking -- it might be the source of the spurious Interrupt exceptions that make it almost impossible to run Judgement Day
Tue, 23 Nov 2010 19:01:21 +0100 blanchet make Mirabelle take into consideration whether the SMT solver proof should be reconstructed with Metis or SMT
Sat, 20 Nov 2010 00:53:26 +0100 wenzelm renamed raw "explode" function to "raw_explode" to emphasize its meaning;
Mon, 15 Nov 2010 18:56:30 +0100 blanchet turn on Sledgehammer verbosity so we can track down crashes
Sat, 13 Nov 2010 19:55:45 +0100 wenzelm total Symbol.source;
Sun, 07 Nov 2010 18:19:04 +0100 blanchet always use a hard timeout in Mirabelle
Sun, 07 Nov 2010 18:15:13 +0100 blanchet use "smt" (rather than "metis") to reconstruct SMT proofs
Fri, 05 Nov 2010 09:05:22 +0100 blanchet make Mirabelle work correctly if the prover (e.g. the SMT solver) returns no timing information
Thu, 04 Nov 2010 15:30:48 +0100 blanchet remove " s" suffix since seconds are now implicit
Thu, 04 Nov 2010 14:59:44 +0100 blanchet use the SMT integration's official list of built-ins
Tue, 02 Nov 2010 20:55:12 +0100 wenzelm simplified some time constants;
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
Fri, 22 Oct 2010 18:31:45 +0200 blanchet tuning
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";
less more (0) -100 -60 tip