src/HOL/Tools/Sledgehammer/sledgehammer_util.ML
Fri, 12 Jul 2013 14:18:07 +0200 smolkas added |>! and #>! for convenient printing of timing information
Tue, 09 Jul 2013 18:45:06 +0200 smolkas completely rewrote SH compress; added two parameters for experimentation/fine grained control
Sat, 11 May 2013 16:57:18 +0200 wenzelm prefer explicitly qualified exceptions, which is particular important for robust handlers;
Mon, 18 Feb 2013 18:34:55 +0100 blanchet implement (more) accurate computation of parents
Thu, 31 Jan 2013 17:54:05 +0100 blanchet tuned data structure
Thu, 31 Jan 2013 17:54:05 +0100 blanchet thread fact triple (MeSh, MePo, MaSh) to allow different filters in different slices
Fri, 04 Jan 2013 21:56:20 +0100 blanchet refined class handling, to prevent cycles in fact graph
Fri, 04 Jan 2013 21:56:19 +0100 blanchet learn from low-level, inside-class facts
Thu, 20 Dec 2012 15:51:27 +0100 blanchet better weight functions for MePo/MaSh etc.
Sat, 15 Dec 2012 19:57:12 +0100 blanchet thread no timeout properly
Wed, 12 Dec 2012 02:47:45 +0100 blanchet merge aliased theorems in MaSh dependencies, modulo symmetry of equality
Wed, 28 Nov 2012 12:25:43 +0100 smolkas moved thms_of_name to Sledgehammer_Util and removed copies, updated references
Mon, 12 Nov 2012 12:06:56 +0100 blanchet avoid messing too much with output of "string_of_term", so that it doesn't break the yxml encoding for jEdit
Mon, 12 Nov 2012 11:52:37 +0100 blanchet centralized term printing code
Fri, 03 Aug 2012 09:51:28 +0200 blanchet cleaner temporary file cleanup for MaSh, based on tried-and-trusted code
Fri, 20 Jul 2012 22:19:46 +0200 blanchet added "learn_from_atp" command to MaSh, for patient users
Fri, 20 Jul 2012 22:19:46 +0200 blanchet learn command in MaSh
Wed, 18 Jul 2012 08:44:04 +0200 blanchet more consolidation of MaSh code
Wed, 18 Jul 2012 08:44:04 +0200 blanchet drastic overhaul of MaSh data structures + fixed a few performance issues
Wed, 18 Jul 2012 08:44:03 +0200 blanchet more code rationalization in relevance filter
Wed, 11 Jul 2012 21:43:19 +0200 blanchet moved most of MaSh exporter code to Sledgehammer
Fri, 16 Mar 2012 11:26:55 +0100 wenzelm clarified Keyword.is_keyword: union of minor and major;
Tue, 31 May 2011 16:38:36 +0200 blanchet first step in sharing more code between ATP and Metis translation
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 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 use helpers and tweak Quickcheck's priority to it comes second (to give Solve Direct slightly more time before another prover runs)
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 00:01:33 +0200 blanchet eliminated more code duplication in Nitrox
Sun, 22 May 2011 14:51:42 +0200 blanchet improved Waldmeister support -- even run it by default on unit equational goals
Fri, 20 May 2011 12:47:59 +0200 blanchet improved "poly_preds_{bang,query}" by picking up good witnesses for the possible infinity of common type classes and ensuring that "?'a::type" doesn't ruin everything
Fri, 20 May 2011 12:47:59 +0200 blanchet reintroduced type encodings "poly_preds_{bang,query}", but this time being more liberal about type variables of known safe sorts
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, 05 May 2011 12:40:48 +0200 blanchet query typedefs as well for monotonicity
Wed, 04 May 2011 19:35:48 +0200 blanchet exploit inferred monotonicity
Fri, 08 Apr 2011 16:34:14 +0200 wenzelm discontinued special treatment of structure Lexicon;
Thu, 16 Dec 2010 15:46:54 +0100 blanchet no need to do a super-duper atomization if Metis fails afterwards anyway
Thu, 16 Dec 2010 15:12:17 +0100 blanchet instantiate induction rules automatically
Sat, 20 Nov 2010 00:53:26 +0100 wenzelm renamed raw "explode" function to "raw_explode" to emphasize its meaning;
Wed, 03 Nov 2010 22:26:53 +0100 blanchet standardize on seconds for Nitpick and Sledgehammer timeouts
Wed, 29 Sep 2010 23:30:10 +0200 blanchet finished renaming file and module
Mon, 27 Sep 2010 10:44:08 +0200 blanchet rename "Clausifier" to "Meson_Clausifier" and merge with "Meson_Tactic"
Mon, 20 Sep 2010 15:08:51 +0200 wenzelm added XML.content_of convenience -- cover XML.body, which is the general situation;
Fri, 17 Sep 2010 01:22:01 +0200 blanchet move functions around
Thu, 16 Sep 2010 14:24:48 +0200 blanchet avoid code duplication
Tue, 14 Sep 2010 11:18:40 +0200 blanchet speed up helper function
Sat, 11 Sep 2010 10:21:52 +0200 blanchet implemented Auto Sledgehammer
Thu, 26 Aug 2010 14:05:22 +0200 blanchet improve SPASS hack, when a clause comes from several facts
Thu, 26 Aug 2010 10:42:06 +0200 blanchet consider "locality" when assigning weights to facts
Tue, 24 Aug 2010 22:57:22 +0200 blanchet make sure that "undo_ascii_of" is the inverse of "ascii_of", also for non-printable characters -- and avoid those in ``-style facts
Tue, 24 Aug 2010 18:03:43 +0200 blanchet clean handling of whether a fact is chained or not;
Tue, 24 Aug 2010 16:24:11 +0200 blanchet quote facts whose names collide with a keyword or command name (cf. "subclass" in "Jinja/J/TypeSafe.thy")
Mon, 23 Aug 2010 14:54:17 +0200 blanchet perform eta-expansion of quantifier bodies in Sledgehammer translation when needed + transform elim rules later;
Fri, 20 Aug 2010 10:58:01 +0200 blanchet beta eta contract the Sledgehammer conjecture (and also the axioms, although this might not be needed), just like Metis does (implicitly);
Thu, 05 Aug 2010 12:40:12 +0200 blanchet fix bug in Nitpick's "equationalize" function (the prems were ignored) + make it do some basic extensionalization
Wed, 28 Jul 2010 18:54:18 +0200 blanchet minor refactoring
Tue, 27 Jul 2010 17:43:11 +0200 blanchet complete renaming of "Sledgehammer_TPTP_Format" to "ATP_Problem"
Mon, 26 Jul 2010 17:03:21 +0200 blanchet generate full first-order formulas (FOF) in Sledgehammer
Fri, 23 Jul 2010 21:29:29 +0200 blanchet keep track of clause numbers for SPASS now that we generate FOF rather than CNF problems;
less more (0) -60 tip