src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML
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";
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:12:02 +0200 blanchet rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
Tue, 14 Sep 2010 23:38:36 +0200 blanchet tuning
Tue, 14 Sep 2010 16:34:26 +0200 blanchet handle relevance filter corner cases more gracefully;
Tue, 14 Sep 2010 14:47:53 +0200 blanchet added a timeout around "try" call in Mirabelle
Mon, 13 Sep 2010 15:11:10 +0200 blanchet indicate triviality in the list of proved things
Mon, 13 Sep 2010 15:01:31 +0200 blanchet indicate which goals are trivial
Mon, 13 Sep 2010 14:29:05 +0200 blanchet keep track of trivial vs. nontrivial calls using "try" for 30 seconds
Sat, 11 Sep 2010 10:24:57 +0200 blanchet make Mirabelle happy
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 22:33:31 +0200 blanchet run relevance filter in a thread, to avoid blocking
Wed, 01 Sep 2010 18:41:23 +0200 blanchet share the relevance filter among the provers
Tue, 31 Aug 2010 23:50:59 +0200 blanchet finished renaming
Fri, 27 Aug 2010 15:37:03 +0200 blanchet drop chained facts
Thu, 26 Aug 2010 10:42:06 +0200 blanchet consider "locality" when assigning weights to facts
Tue, 24 Aug 2010 19:55:34 +0200 blanchet make Mirabelle happy
Wed, 18 Aug 2010 17:16:37 +0200 blanchet get rid of "minimize_timeout", now that there's an automatic adaptive timeout mechanism in "minimize"
Mon, 09 Aug 2010 12:05:48 +0200 blanchet move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
Thu, 29 Jul 2010 23:37:10 +0200 blanchet fix Mirabelle timeout
Thu, 29 Jul 2010 23:24:07 +0200 blanchet make Mirabelle happy
Thu, 29 Jul 2010 14:42:09 +0200 blanchet "axiom_clauses" -> "axioms" (these are no longer clauses)
Tue, 27 Jul 2010 20:16:03 +0200 blanchet compile
Tue, 27 Jul 2010 17:04:09 +0200 blanchet implemented "sublinear" minimization algorithm
Mon, 26 Jul 2010 14:14:24 +0200 blanchet make TPTP generator accept full first-order formulas
Tue, 29 Jun 2010 11:20:05 +0200 blanchet compile
Tue, 29 Jun 2010 11:14:52 +0200 blanchet compile
Mon, 28 Jun 2010 11:04:02 +0200 blanchet compile
Fri, 25 Jun 2010 17:08:39 +0200 blanchet renamed "Sledgehammer_FOL_Clauses" to "Metis_Clauses", so that Metis doesn't depend on Sledgehammer
Fri, 25 Jun 2010 16:42:06 +0200 blanchet merge "Sledgehammer_{F,H}OL_Clause", as requested by a FIXME
Tue, 22 Jun 2010 19:08:25 +0200 blanchet turn on "natural form" filtering in the Mirabelle tests, to see how it performs
Mon, 17 May 2010 23:54:15 +0200 wenzelm prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
Mon, 17 May 2010 15:11:25 +0200 wenzelm renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
Sun, 16 May 2010 00:02:11 +0200 wenzelm prefer structure Parse_Spec;
Wed, 28 Apr 2010 16:56:03 +0200 blanchet make Mirabelle happy
Mon, 26 Apr 2010 21:50:36 +0200 blanchet compile
Fri, 23 Apr 2010 16:55:51 +0200 blanchet move some sledgehammer stuff out of "atp_manager.ML"
Fri, 23 Apr 2010 12:24:30 +0200 blanchet compile
Mon, 19 Apr 2010 15:15:21 +0200 blanchet make Sledgehammer's minimizer also minimize Isar proofs
Thu, 01 Apr 2010 11:12:08 +0200 blanchet add missing goal argument
Thu, 25 Mar 2010 17:55:55 +0100 blanchet make Mirabelle happy again
Mon, 22 Mar 2010 10:38:28 +0100 blanchet remove the iteration counter from Sledgehammer's minimizer
Fri, 19 Mar 2010 15:33:18 +0100 blanchet move all ATP setup code into ATP_Wrapper
Fri, 19 Mar 2010 15:07:44 +0100 blanchet move the Sledgehammer Isar commands together into one file;
Thu, 18 Mar 2010 13:43:50 +0100 blanchet fix Mirabelle after renaming Sledgehammer structures
Fri, 05 Mar 2010 23:51:32 +0100 wenzelm use regular Proof.goal (which is what methods usually see) and prevent sledgehammer from crashing;
Thu, 10 Dec 2009 18:10:59 +0100 boehmes only invoke metisFT if metis failed
less more (0) -100 -60 tip