src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
Fri, 01 Jul 2011 15:53:38 +0200 renamed "type_sys" to "type_enc", which is more accurate
Thu, 30 Jun 2011 13:21:41 +0200 standardized use of Path operations;
Mon, 27 Jun 2011 14:56:35 +0200 clarify minimizer output
Mon, 27 Jun 2011 14:56:28 +0200 added "sound" option to force Sledgehammer to be pedantically sound
Mon, 27 Jun 2011 13:52:47 +0200 removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
Tue, 21 Jun 2011 17:17:39 +0200 generate type predicates for existentials/skolems, otherwise some problems might not be provable
Mon, 20 Jun 2011 12:13:43 +0200 clean up SPASS FLOTTER hack
Mon, 20 Jun 2011 11:42:41 +0200 remove automatic recovery from (some) unsound proofs, now that we use sound encodings for all the interesting provers
Mon, 20 Jun 2011 10:41:02 +0200 deal with ATP time slices in a more flexible/robust fashion
Fri, 10 Jun 2011 17:52:09 +0200 name tuning
Fri, 10 Jun 2011 17:52:09 +0200 don't trim proofs in debug mode
Fri, 10 Jun 2011 12:01:15 +0200 pass --trim option to "eproof" script to speed up proof reconstruction
Thu, 09 Jun 2011 00:16:28 +0200 cleaner fact freshening, which also works in corner cases, e.g. if two backquoted facts have the same name (but have different variable indices)
Thu, 09 Jun 2011 00:16:28 +0200 added a really fully typed translation as a fallback for Metis, in rare cases where Metis correctly proves a theorem but has type-unsound steps in it (which is likelier to happen with some of the lighter translations)
Wed, 08 Jun 2011 08:47:43 +0200 exploit new semantics of "max_new_instances"
Wed, 08 Jun 2011 08:47:43 +0200 make sure that the message tail (timing + TPTP important message) is preserved upon automatic minimization
Wed, 08 Jun 2011 08:47:43 +0200 killed "explicit_apply" option in Sledgehammer -- the "smart" default is about as lightweight as "false" and just as complete as "true"
Tue, 07 Jun 2011 14:38:42 +0200 prioritize more relevant facts for monomorphization
Tue, 07 Jun 2011 14:17:35 +0200 more suitable implementation of "schematic_consts_of" for monomorphizer, for ATPs
Tue, 07 Jun 2011 14:17:35 +0200 workaround current "max_new_instances" semantics
Tue, 07 Jun 2011 11:13:52 +0200 move away from old SMT monomorphizer
Tue, 07 Jun 2011 11:05:09 +0200 merged
Tue, 07 Jun 2011 11:04:17 +0200 use the proper prover name, e.g. metis_full_types, not metis (full_types), for minimizing
Tue, 07 Jun 2011 10:46:09 +0200 removed "verbose" option -- there won't be any verbosity in there, according to Sascha (yeah)
Tue, 07 Jun 2011 10:43:18 +0200 nicely thread monomorphism verbosity in Metis and Sledgehammer
Tue, 07 Jun 2011 10:24:16 +0200 clarified meaning of monomorphization configuration option by renaming it
Tue, 07 Jun 2011 08:52:35 +0200 obsoleted "metisFT", and added "no_types" version of Metis as fallback to Sledgehammer after noticing how useful it can be
Tue, 07 Jun 2011 07:45:12 +0200 use new monomorphization code
Tue, 07 Jun 2011 07:06:24 +0200 renamed ML function
Tue, 07 Jun 2011 06:58:52 +0200 pass props not thms to ATP translator
Mon, 06 Jun 2011 23:43:28 +0200 removed confusing slicing logic
Mon, 06 Jun 2011 23:26:40 +0200 suggest first reconstructor that timed out, not last (i.e. metis not metisFT in most cases)
Mon, 06 Jun 2011 23:11:14 +0200 effectively reenable slices for SPASS and Vampire -- they were disabled by mistake
Mon, 06 Jun 2011 20:56:06 +0200 removed old optimization that isn't one anyone
Mon, 06 Jun 2011 20:56:06 +0200 Metis code cleanup
Mon, 06 Jun 2011 20:36:36 +0200 enable new Metis
Mon, 06 Jun 2011 20:36:35 +0200 more preparations towards hijacking Metis
Mon, 06 Jun 2011 20:36:35 +0200 remove more occurrences of "metisX", preparing for the D Day when it will silently hijack "metis" and "metisFT"
Mon, 06 Jun 2011 20:36:35 +0200 make "metisX"'s default more like old "metis"
Mon, 06 Jun 2011 20:36:34 +0200 temporarily added "MetisX" as reconstructor and minimizer
Mon, 06 Jun 2011 20:36:34 +0200 show what failed to play
Wed, 01 Jun 2011 10:29:43 +0200 tuned names
Tue, 31 May 2011 16:38:36 +0200 tuned name
Tue, 31 May 2011 16:38:36 +0200 make "prepare_atp_problem" more robust w.r.t. choice of type system
Tue, 31 May 2011 16:38:36 +0200 don't preprocess twice
Tue, 31 May 2011 16:38:36 +0200 more work on new metis that exploits the powerful new type encodings
Tue, 31 May 2011 16:38:36 +0200 first step in sharing more code between ATP and Metis translation
Mon, 30 May 2011 17:00:38 +0200 don't slice if there are too few facts
Mon, 30 May 2011 17:00:38 +0200 automatically minimize with Metis when this can be done within a few seconds
Mon, 30 May 2011 17:00:38 +0200 minimize with Metis if possible
Mon, 30 May 2011 17:00:38 +0200 support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
Sun, 29 May 2011 19:40:56 +0200 always check plain "metis" even if the ATP proof seems to require "metisFT" -- maybe the proof is needlessly complicated
Fri, 27 May 2011 10:30:08 +0200 cleanup proof text generation code
Fri, 27 May 2011 10:30:08 +0200 try both "metis" and (on failure) "metisFT" in replay
Fri, 27 May 2011 10:30:08 +0200 show time taken for reconstruction
Fri, 27 May 2011 10:30:08 +0200 more concise output
Fri, 27 May 2011 10:30:08 +0200 handle non-auto try case of Sledgehammer better
Fri, 27 May 2011 10:30:08 +0200 renamed "metis_timeout" to "preplay_timeout" and continued implementation
Fri, 27 May 2011 10:30:07 +0200 added syntax for specifying Metis timeout (currently used only by SMT solvers)
Fri, 27 May 2011 10:30:07 +0200 make output more concise