src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
Tue, 07 Jun 2011 14:38:42 +0200 blanchet prioritize more relevant facts for monomorphization
Tue, 07 Jun 2011 14:17:35 +0200 blanchet more suitable implementation of "schematic_consts_of" for monomorphizer, for ATPs
Tue, 07 Jun 2011 14:17:35 +0200 blanchet workaround current "max_new_instances" semantics
Tue, 07 Jun 2011 11:13:52 +0200 blanchet move away from old SMT monomorphizer
Tue, 07 Jun 2011 11:05:09 +0200 blanchet merged
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
Tue, 07 Jun 2011 10:46:09 +0200 blanchet removed "verbose" option -- there won't be any verbosity in there, according to Sascha (yeah)
Tue, 07 Jun 2011 10:43:18 +0200 blanchet nicely thread monomorphism verbosity in Metis and Sledgehammer
Tue, 07 Jun 2011 10:24:16 +0200 boehmes clarified meaning of monomorphization configuration option by renaming it
Tue, 07 Jun 2011 08:52:35 +0200 blanchet 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 blanchet use new monomorphization code
Tue, 07 Jun 2011 07:06:24 +0200 blanchet renamed ML function
Tue, 07 Jun 2011 06:58:52 +0200 blanchet pass props not thms to ATP translator
Mon, 06 Jun 2011 23:43:28 +0200 blanchet removed confusing slicing logic
Mon, 06 Jun 2011 23:26:40 +0200 blanchet suggest first reconstructor that timed out, not last (i.e. metis not metisFT in most cases)
Mon, 06 Jun 2011 23:11:14 +0200 blanchet effectively reenable slices for SPASS and Vampire -- they were disabled by mistake
Mon, 06 Jun 2011 20:56:06 +0200 blanchet removed old optimization that isn't one anyone
Mon, 06 Jun 2011 20:56:06 +0200 blanchet Metis code cleanup
Mon, 06 Jun 2011 20:36:36 +0200 blanchet enable new Metis
Mon, 06 Jun 2011 20:36:35 +0200 blanchet more preparations towards hijacking Metis
Mon, 06 Jun 2011 20:36:35 +0200 blanchet 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 blanchet make "metisX"'s default more like old "metis"
Mon, 06 Jun 2011 20:36:34 +0200 blanchet temporarily added "MetisX" as reconstructor and minimizer
Mon, 06 Jun 2011 20:36:34 +0200 blanchet show what failed to play
Wed, 01 Jun 2011 10:29:43 +0200 blanchet tuned names
Tue, 31 May 2011 16:38:36 +0200 blanchet tuned name
Tue, 31 May 2011 16:38:36 +0200 blanchet make "prepare_atp_problem" more robust w.r.t. choice of type system
Tue, 31 May 2011 16:38:36 +0200 blanchet don't preprocess twice
Tue, 31 May 2011 16:38:36 +0200 blanchet more work on new metis that exploits the powerful new type encodings
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 don't slice if there are too few facts
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
Mon, 30 May 2011 17:00:38 +0200 blanchet support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
Sun, 29 May 2011 19:40:56 +0200 blanchet 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 blanchet cleanup proof text generation code
Fri, 27 May 2011 10:30:08 +0200 blanchet try both "metis" and (on failure) "metisFT" in replay
Fri, 27 May 2011 10:30:08 +0200 blanchet show time taken for reconstruction
Fri, 27 May 2011 10:30:08 +0200 blanchet more concise output
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 renamed "metis_timeout" to "preplay_timeout" and continued implementation
Fri, 27 May 2011 10:30:07 +0200 blanchet added syntax for specifying Metis timeout (currently used only by SMT solvers)
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
Fri, 27 May 2011 10:30:07 +0200 blanchet fully support all type system encodings in typed formats (TFF, THF)
Fri, 27 May 2011 10:30:07 +0200 blanchet towards supporting non-simply-typed encodings for TFF and THF (for orthogonality and experiments)
Tue, 24 May 2011 17:04:35 +0200 blanchet respect user's intention better when setting the CNF_UEQ type system (esp. w.r.t. "erased")
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 00:01:33 +0200 blanchet slightly gracefuller handling of LEO-II and Satallax output
Tue, 24 May 2011 00:01:33 +0200 blanchet identify HOL functions with THF functions
Tue, 24 May 2011 00:01:33 +0200 blanchet started adding support for THF output (but no lambdas)
Tue, 24 May 2011 00:01:33 +0200 blanchet filter Waldmeister facts better -- and don't encode type classes as predicates, since it doesn't like conditional equations
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
Sun, 22 May 2011 14:51:41 +0200 blanchet fish out axioms in Waldmeister output
Sun, 22 May 2011 14:51:01 +0200 blanchet added support for remote Waldmeister
Sun, 22 May 2011 14:49:35 +0200 blanchet reorganized ATP formats a little bit
Fri, 20 May 2011 12:47:59 +0200 blanchet make sure the Vampire incomplete proof detection code kicks in
Fri, 20 May 2011 12:47:59 +0200 blanchet automatically use "metisFT" when typed helpers are necessary
Fri, 20 May 2011 12:47:58 +0200 blanchet more informative message when Sledgehammer finds an unsound proof
Thu, 19 May 2011 10:24:13 +0200 blanchet tweaked ATP type systems further based on Judgment Day
Thu, 19 May 2011 10:24:13 +0200 blanchet reintroduce TFF workaround for limitations of actual TFF implementations (ToFoF, SNARK)
Tue, 17 May 2011 15:11:36 +0200 blanchet renamed thin to light, fat to heavy
Tue, 17 May 2011 15:11:36 +0200 blanchet run blacklist algorithm only if slicing is on
Tue, 17 May 2011 15:11:36 +0200 blanchet renamed "shallow" to "thin" and make it the default
Tue, 17 May 2011 15:11:36 +0200 blanchet added syntax for "shallow" encodings
Fri, 13 May 2011 10:10:43 +0200 blanchet tuned comment
Fri, 13 May 2011 10:10:43 +0200 blanchet fixed off-by-one bug
Thu, 12 May 2011 15:29:19 +0200 blanchet robustly detect how many type args were passed to the ATP, even if some of them were omitted
Thu, 12 May 2011 15:29:19 +0200 blanchet further lower penalty associated with existentials in Sledgehammer's relevance filter, so that "exhaust" facts are picked up
Thu, 12 May 2011 15:29:19 +0200 blanchet renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
Thu, 12 May 2011 15:29:19 +0200 blanchet remove unused parameter
Thu, 12 May 2011 15:29:19 +0200 blanchet reduced penalty associated with existential quantifiers
Thu, 12 May 2011 15:29:19 +0200 blanchet fine-tuned the relevance filter, so that equations of the form "c = (%x. _)" and constants occurring in chained facts are not unduely penalized
Thu, 12 May 2011 15:29:19 +0200 blanchet improve detection of quantifications over dangerous types by leveraging "is_type_surely_finite" predicate and added "prop" to the list of surely finite types
Thu, 12 May 2011 15:29:19 +0200 blanchet tune whitespace
Thu, 12 May 2011 15:29:18 +0200 blanchet added "max_mono_instances" option to Sledgehammer and renamed old "monomorphize_limit" option
Thu, 12 May 2011 15:29:18 +0200 blanchet allow each slice to have its own type system
Thu, 12 May 2011 15:29:18 +0200 blanchet renamed type systems for more consistency
Fri, 06 May 2011 13:34:59 +0200 blanchet allow each prover to specify its own formula kind for symbols occurring in the conjecture
Thu, 05 May 2011 12:40:48 +0200 blanchet no lies in debug output (e.g. "slice 2 of 1")
Wed, 04 May 2011 22:56:33 +0200 blanchet renamed "many_typed" to "simple" (as in simple types)
Wed, 04 May 2011 22:47:13 +0200 blanchet added type homogenization, whereby all (isomorphic) infinite types are mapped to the same type (to reduce the number of different predicates/TFF-types)
Tue, 03 May 2011 21:46:49 +0200 blanchet fixed per-ATP dangerous axiom detection -- embarrassing bugs introduced in change a7a30721767a
Tue, 03 May 2011 01:04:03 +0200 blanchet no need to generate fact numbers for polymorphic type systems -- this confuses the TPTP exporter
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 17:43:42 +0200 wenzelm merged
Mon, 02 May 2011 16:33:21 +0200 wenzelm added Attrib.setup_config_XXX conveniences, with implicit setup of the background theory;
Mon, 02 May 2011 15:01:36 +0200 blanchet make "debug" more verbose and "verbose" less verbose
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
Mon, 02 May 2011 14:10:09 +0200 blanchet fixed random number invocation
Sun, 01 May 2011 22:36:58 +0200 blanchet use "metis", not "metisFT", to reconstruct proofs found in fully-typed mode -- "metisFT" is just too slow...
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 take "partial_types" option with a grain of salt
Sun, 01 May 2011 18:37:25 +0200 blanchet fixed SPASS fact offset calculation and report unexpected unsound proofs with so-called sound encodings
Sun, 01 May 2011 18:37:25 +0200 blanchet implement the new ATP type system in Sledgehammer
Sun, 01 May 2011 18:37:25 +0200 blanchet define type system in ATP module so that ATPs can suggest a type system
Sun, 01 May 2011 18:37:25 +0200 blanchet made the format (TFF or FOF) of the TPTP problem a global argument of the problem again and have the ATPs report which formats they support
Sun, 01 May 2011 18:37:24 +0200 blanchet no needless "fequal" proxies if "explicit_apply" is set + always have readable names
Sun, 01 May 2011 18:37:24 +0200 blanchet make sure the minimizer monomorphizes when it should
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
Sun, 01 May 2011 18:37:24 +0200 blanchet move type declarations to the front, for TFF-compliance
Sun, 01 May 2011 18:37:24 +0200 blanchet added (without implementation yet) new type encodings for Sledgehammer/ATP
Sun, 01 May 2011 18:37:23 +0200 blanchet get rid of "explicit_forall" prover-specific option, even if that means some clutter -- foralls will be necessary to attach types to variables
Fri, 22 Apr 2011 00:57:59 +0200 blanchet iterate the unsound-fact-set removal process to recover even more unsound proofs
Fri, 22 Apr 2011 00:00:05 +0200 blanchet automatically remove offending facts when faced with an unsound proof -- instead of using the highly inefficient "full_types" option
Thu, 21 Apr 2011 22:32:00 +0200 blanchet automatically retry with full-types upon unsound proof
Thu, 21 Apr 2011 22:18:28 +0200 blanchet detect some unsound proofs before showing them to the user
Thu, 21 Apr 2011 21:14:06 +0200 blanchet tuning -- local semicolon consistency
Thu, 21 Apr 2011 18:51:22 +0200 blanchet tuning
Thu, 21 Apr 2011 18:39:22 +0200 blanchet fixed interaction between monomorphization and slicing for ATPs
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;
Fri, 01 Apr 2011 13:21:21 +0200 blanchet remove workaround 8f25605e646c, which is no longer necessary thanks to 173b0f488428
Fri, 01 Apr 2011 11:54:51 +0200 boehmes make configuration of (SMT) full monomorphization more flexible: turn boolean argument into a configuration option
less more (0) -120 tip