src/HOL/Tools/Sledgehammer/sledgehammer_proof_reconstruct.ML
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
Fri, 27 Aug 2010 16:05:46 +0200 blanchet merged
Thu, 26 Aug 2010 14:05:22 +0200 blanchet improve SPASS hack, when a clause comes from several facts
Fri, 27 Aug 2010 10:56:46 +0200 haftmann formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
Thu, 26 Aug 2010 20:51:17 +0200 haftmann formerly unnamed infix impliciation now named HOL.implies
Thu, 26 Aug 2010 10:42:06 +0200 blanchet consider "locality" when assigning weights to facts
Thu, 26 Aug 2010 00:49:38 +0200 blanchet renaming
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")
Thu, 19 Aug 2010 11:30:32 +0200 blanchet parse SNARK proofs
Thu, 19 Aug 2010 11:02:59 +0200 blanchet no spurious trailing "\n" at the end of Sledgehammer's output
Tue, 17 Aug 2010 16:47:40 +0200 blanchet tuning
Tue, 17 Aug 2010 14:37:16 +0200 blanchet handle E's Skolem constants more gracefully
Mon, 09 Aug 2010 12:05:48 +0200 blanchet move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
Fri, 30 Jul 2010 00:02:25 +0200 blanchet don't choke on synonyms when parsing SPASS's Flotter output + renamings;
Thu, 29 Jul 2010 14:53:55 +0200 blanchet avoid "clause" and "cnf" terminology where it no longer makes sense
Thu, 29 Jul 2010 09:47:23 +0200 blanchet kill polymorphic "val"s
Wed, 28 Jul 2010 18:07:25 +0200 blanchet fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
Wed, 28 Jul 2010 17:38:40 +0200 blanchet revive "e" and "remote_e"'s fact extraction so that it works with E 1.2 as well;
Wed, 28 Jul 2010 16:54:12 +0200 blanchet more robust proof reconstruction
Wed, 28 Jul 2010 15:53:52 +0200 blanchet fix remote_vampire's proof reconstruction
Wed, 28 Jul 2010 15:34:10 +0200 blanchet fix proof reconstruction for latest Vampire
Wed, 28 Jul 2010 10:45:49 +0200 blanchet renaming
Wed, 28 Jul 2010 10:06:06 +0200 blanchet support latest version of Vampire (1.0) locally
Tue, 27 Jul 2010 19:41:19 +0200 blanchet minor refactoring
Tue, 27 Jul 2010 19:17:15 +0200 blanchet standardize "Author" tags
Tue, 27 Jul 2010 17:43:11 +0200 blanchet complete renaming of "Sledgehammer_TPTP_Format" to "ATP_Problem"
Tue, 27 Jul 2010 17:32:10 +0200 blanchet move Sledgehammer-specific code out of "Sledgehammer_TPTP_Format"
Tue, 27 Jul 2010 17:04:09 +0200 blanchet implemented "sublinear" minimization algorithm
Tue, 27 Jul 2010 15:28:23 +0200 blanchet extract sort constraints from FOFs properly;
Tue, 27 Jul 2010 12:01:02 +0200 blanchet handle Vampire's equality proxy axiom correctly
Mon, 26 Jul 2010 17:22:39 +0200 blanchet remove more Skolemization-aware code
Mon, 26 Jul 2010 17:09:10 +0200 blanchet simplify "conjecture_shape" business, as a result of using FOF instead of CNF
Mon, 26 Jul 2010 17:03:21 +0200 blanchet generate full first-order formulas (FOF) in Sledgehammer
Mon, 26 Jul 2010 14:14:24 +0200 blanchet make TPTP generator accept full first-order formulas
Mon, 26 Jul 2010 11:21:11 +0200 blanchet proof reconstruction for full FOF terms
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;
Fri, 23 Jul 2010 15:04:49 +0200 blanchet first step in using "fof" rather than "cnf" in TPTP problems
Wed, 21 Jul 2010 21:15:07 +0200 blanchet renamings + only need second component of name pool to reconstruct proofs
Wed, 30 Jun 2010 18:03:34 +0200 blanchet rewrote the TPTP problem generation code more or less from scratch;
Tue, 29 Jun 2010 09:19:16 +0200 blanchet move "nice names" from Metis to TPTP format
Mon, 28 Jun 2010 17:31:38 +0200 blanchet always perform relevance filtering on original formulas
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
Fri, 25 Jun 2010 16:15:03 +0200 blanchet renamed "Sledgehammer_Fact_Preprocessor" to "Clausifier";
Fri, 25 Jun 2010 15:59:13 +0200 blanchet more intra-module dependency cleanup + merge "const" and "type_const" tables, since this is safe
Tue, 22 Jun 2010 14:28:22 +0200 blanchet removed Sledgehammer's support for the DFG syntax;
Mon, 21 Jun 2010 12:31:41 +0200 blanchet try to improve Sledgehammer/Metis's behavior in full_types mode, e.g. by handing True, False, and If better
Mon, 14 Jun 2010 10:36:01 +0200 blanchet adjusted the polymorphism handling of Skolem constants so that proof reconstruction doesn't fail in "equality_inf"
Fri, 11 Jun 2010 17:10:23 +0200 blanchet proper polymorphic Skolemization of uncached facts + synchronization of caching and relevance filter
Fri, 04 Jun 2010 14:08:23 +0200 blanchet fix bugs in Sledgehammer's Isar proof "redirection" code
Wed, 02 Jun 2010 17:19:44 +0200 blanchet handle Vampire's definitions smoothly
Wed, 02 Jun 2010 17:06:28 +0200 blanchet fix bug in direct Isar proofs, which was exhibited by the "BigO" example
Wed, 02 Jun 2010 14:35:52 +0200 blanchet show types in Isar proofs, but not for free variables;
Fri, 28 May 2010 17:00:38 +0200 blanchet merged
Fri, 28 May 2010 13:49:21 +0200 blanchet make sure chained facts appear in Isar proofs generated by Sledgehammer -- otherwise the proof won't work
Thu, 27 May 2010 18:10:37 +0200 wenzelm renamed structure PrintMode to Print_Mode, keeping the old name as legacy alias for some time;
Thu, 27 May 2010 17:41:27 +0200 wenzelm renamed structure TypeInfer to Type_Infer, keeping the old name as legacy alias for some time;
Mon, 17 May 2010 15:21:11 +0200 blanchet make sure chained facts don't pop up in the metis proof
less more (0) -100 -60 tip