src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
Thu, 30 Jan 2014 21:56:25 +0100 blanchet got rid of one of two Metis variants
Thu, 30 Jan 2014 21:02:19 +0100 blanchet tuning
Thu, 30 Jan 2014 18:37:08 +0100 blanchet killed needless pass
Thu, 30 Jan 2014 17:34:42 +0100 blanchet don't forget the last inference(s) after conjecture skolemization
Thu, 30 Jan 2014 15:01:40 +0100 blanchet keep formula right before skolemization, because the universal variables might be different (or differently ordered) as in the original axiom or negated conjecture from which it was skolemized
Thu, 30 Jan 2014 14:37:53 +0100 blanchet renamed Sledgehammer options for symmetry between positive and negative versions
Wed, 29 Jan 2014 23:24:34 +0100 blanchet proper 'show' detection
Wed, 29 Jan 2014 22:34:34 +0100 blanchet correctly handle exceptions arising from (experimental) Isar proof code
Fri, 20 Dec 2013 20:36:38 +0100 blanchet reconstruct SPASS-Pirate steps of the form 'x ~= C x' (or more complicated)
Fri, 20 Dec 2013 14:27:07 +0100 blanchet recognize datatype reasoning in SPASS-Pirate
Thu, 19 Dec 2013 20:07:06 +0100 blanchet tuning
Thu, 19 Dec 2013 19:16:44 +0100 blanchet don't do 'isar_try0' if preplaying is off
Thu, 19 Dec 2013 18:39:54 +0100 blanchet more data structure refactoring
Thu, 19 Dec 2013 17:52:58 +0100 blanchet refactored preplaying outcome data structure
Thu, 19 Dec 2013 17:24:17 +0100 blanchet distinguish not preplayed & timed out
Thu, 19 Dec 2013 13:43:21 +0100 blanchet made timeouts in Sledgehammer not be 'option's -- simplified lots of code
Thu, 19 Dec 2013 09:28:20 +0100 blanchet tuning
Wed, 18 Dec 2013 16:50:14 +0100 blanchet try 'auto' first -- more likely to succeed
Wed, 18 Dec 2013 16:50:14 +0100 blanchet tuning
Mon, 16 Dec 2013 23:05:16 +0100 blanchet handle Skolems gracefully for SPASS as well
Mon, 16 Dec 2013 20:43:04 +0100 blanchet move some Z3 specifics out (and into private repository with the rest of the Z3-specific code)
Mon, 16 Dec 2013 20:24:13 +0100 blanchet reverse Skolem function arguments
Mon, 16 Dec 2013 17:58:31 +0100 blanchet correcly recognize E skolemization steps that are wrapped in a 'shift_quantors' inference
Mon, 16 Dec 2013 17:18:52 +0100 blanchet fixed confusion between 'prop' and 'bool' introduced in 4960647932ec
Mon, 16 Dec 2013 14:49:18 +0100 blanchet generalize method list further to list of list (clustering preferred methods together)
Mon, 16 Dec 2013 12:26:18 +0100 blanchet store alternative proof methods in Isar data structure
Mon, 16 Dec 2013 12:02:28 +0100 blanchet tuning
Mon, 16 Dec 2013 09:40:02 +0100 blanchet tuning
Sun, 15 Dec 2013 22:03:12 +0100 blanchet generate proper succedent for cases with trivial branches
Sun, 15 Dec 2013 20:31:25 +0100 blanchet tuning
Sun, 15 Dec 2013 20:09:13 +0100 blanchet simplify generated propositions
Sun, 15 Dec 2013 19:01:06 +0100 blanchet use 'prop' rather than 'bool' systematically in Isar reconstruction code
Sun, 15 Dec 2013 18:54:26 +0100 blanchet tuning
Sun, 15 Dec 2013 18:01:38 +0100 blanchet use 'arith' when appropriate in Z3 proofs
Sun, 15 Dec 2013 18:01:38 +0100 blanchet robustness in degenerate case + tuning
Sun, 15 Dec 2013 18:01:38 +0100 blanchet use simplifier for rewrite
Sun, 15 Dec 2013 18:01:38 +0100 blanchet implemented Z3 skolemization
Sun, 15 Dec 2013 18:01:38 +0100 blanchet inline Z3 hypotheses
Sat, 14 Dec 2013 07:26:45 +0800 blanchet better handling of Z3 proof blocks
Wed, 11 Dec 2013 22:53:32 +0800 blanchet reverse order in which lines are selected, to ensure that the number of dependencies is accurate
Wed, 11 Dec 2013 22:23:42 +0800 blanchet truncate proof once False is hit to avoid confusing the rest of the code (no idea why Z3 goes on)
Tue, 10 Dec 2013 15:24:17 +0800 blanchet more work on Z3 Isar proofs
Mon, 09 Dec 2013 06:33:46 +0100 blanchet adapted code for Z3 proof reconstruction
Mon, 09 Dec 2013 05:06:48 +0100 blanchet useful debugging info
Wed, 20 Nov 2013 18:08:02 +0100 blanchet support Negated_Conjecture as a TPTP role as well (e.g. for SMT proofs)
Tue, 19 Nov 2013 22:20:01 +0100 blanchet whitespace tuning
Tue, 19 Nov 2013 19:36:24 +0100 blanchet more refactoring to accommodate SMT proofs
Tue, 19 Nov 2013 18:34:04 +0100 blanchet tuning
Tue, 19 Nov 2013 18:11:52 +0100 blanchet simplified old code
Tue, 19 Nov 2013 17:37:35 +0100 blanchet refactoring
Tue, 19 Nov 2013 17:12:58 +0100 blanchet refactoring
Tue, 19 Nov 2013 16:48:50 +0100 blanchet refactored
Wed, 09 Oct 2013 16:40:03 +0200 blanchet no isar proofs if preplay was not attempted
Fri, 20 Sep 2013 22:39:30 +0200 blanchet merged "isar_try0" and "isar_minimize" options
Fri, 20 Sep 2013 22:39:30 +0200 blanchet hardcoded obscure option
Fri, 20 Sep 2013 22:39:30 +0200 blanchet hard-coded an obscure option
Fri, 20 Sep 2013 22:39:30 +0200 blanchet use configuration mechanism for low-level tracing
Thu, 12 Sep 2013 22:10:57 +0200 blanchet prefixed types and some functions with "atp_" for disambiguation
Sat, 17 Aug 2013 19:13:28 +0200 wenzelm sledgehammer sendback always uses Markup.padding_command: sensible default for most practical applications -- old-style in-line replacement is superseded by auto mode or panel;
Sat, 17 Aug 2013 11:34:50 +0200 wenzelm more explicit sendback propertries based on mode;
Mon, 29 Jul 2013 16:13:35 +0200 blanchet parse nonnumeric identifiers in E proofs correctly
Thu, 18 Jul 2013 20:53:22 +0200 wenzelm explicit padding on command boundary for "auto" generated sendback -- do not replace the corresponding goal command, but append to it;
Fri, 12 Jul 2013 22:41:25 +0200 smolkas added sledgehammer parameters isar_try0 and isar_minimize and their negative aliases
Fri, 12 Jul 2013 19:03:08 +0200 smolkas cleaner preplay interface
Fri, 12 Jul 2013 14:18:06 +0200 smolkas minimize dependencies (used facts) of Isar proof steps; remove unreferenced steps
Thu, 11 Jul 2013 20:08:06 +0200 smolkas optimize isar-proofs by trying different proof methods
Tue, 09 Jul 2013 18:45:06 +0200 smolkas completely rewrote SH compress; added two parameters for experimentation/fine grained control
Tue, 09 Jul 2013 18:44:59 +0200 smolkas moved code -> easier debugging
Wed, 26 Jun 2013 18:26:00 +0200 smolkas tuned: cleaned up data structure
Wed, 26 Jun 2013 18:25:13 +0200 smolkas simplified data structure
Thu, 13 Jun 2013 16:58:20 -0400 blanchet tuning
Tue, 11 Jun 2013 19:58:09 -0400 smolkas uncheck terms before annotation to avoid awkward syntax
Tue, 11 Jun 2013 16:13:19 -0400 smolkas make use of show_type_emphasis instead of using hack; make sure global configurations don't affect proof script creation
Tue, 28 May 2013 08:52:41 +0200 blanchet redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
Sun, 26 May 2013 12:56:37 +0200 blanchet handle lambda-lifted problems in Isar construction code
Fri, 24 May 2013 16:43:37 +0200 blanchet improved handling of free variables' types in Isar proofs
Mon, 20 May 2013 13:07:31 +0200 blanchet parse agsyHOL proofs (as unsat cores)
Thu, 16 May 2013 14:58:30 +0200 blanchet correctly 'repair' the monomorphization context for SMT solvers from Sledgehammer
Thu, 16 May 2013 13:34:13 +0200 blanchet tuning -- renamed '_from_' to '_of_' in Sledgehammer
Wed, 15 May 2013 17:43:42 +0200 blanchet renamed Sledgehammer functions with 'for' in their names to 'of'
Tue, 14 May 2013 09:49:03 +0200 blanchet generate valid direct Isar proof also if the facts are contradictory
Mon, 06 May 2013 11:03:08 +0200 smolkas added preplay tracing
Tue, 23 Apr 2013 16:30:30 +0200 blanchet tuning
Sat, 23 Feb 2013 22:00:12 +0100 wenzelm make SML/NJ happy;
Thu, 21 Feb 2013 12:22:26 +0100 blanchet generate Isar proof if Metis appears to be too slow
Wed, 20 Feb 2013 17:42:20 +0100 blanchet ensure all conjecture clauses are in the graph -- to prevent exceptions later
Wed, 20 Feb 2013 17:05:24 +0100 blanchet remove needless steps from refutation graph -- these confuse the proof redirection algorithm (and are needless)
Wed, 20 Feb 2013 14:47:19 +0100 blanchet trust preplayed proof in Mirabelle
Wed, 20 Feb 2013 14:44:00 +0100 blanchet added case taken out by mistake
Wed, 20 Feb 2013 14:21:17 +0100 blanchet tuning (removed redundant datatype)
Wed, 20 Feb 2013 14:10:51 +0100 blanchet minimize SMT proofs with E if Isar proofs are desired and Metis managed to preplay
Wed, 20 Feb 2013 10:54:13 +0100 blanchet got rid of rump support for Vampire definitions
Wed, 20 Feb 2013 08:56:34 +0100 blanchet tuning
Wed, 20 Feb 2013 08:44:24 +0100 blanchet use new skolemizer only if some skolems have two or more arguments -- otherwise the old skolemizer cannot get the arg order wrong
Wed, 20 Feb 2013 08:44:24 +0100 blanchet slacker comparison for Skolems, to avoid trivial equations
Wed, 20 Feb 2013 08:44:24 +0100 blanchet made "isar_proofs" a 3-way option, to provide a way to totally disable isar_proofs if desired
Tue, 19 Feb 2013 17:01:06 +0100 blanchet avoid using "smt" for minimization -- better use the prover itself, since then Sledgehammer gets to try metis again and gives the opportunity to output an Isar proof -- and show Isar proof as fallback for SMT proofs
Mon, 18 Feb 2013 12:16:27 +0100 smolkas split isar_step into isar_step, fix, assms; made isar_proof explicit; register fixed variables in ctxt and auto_fix terms to avoid superfluous annotations
Mon, 18 Feb 2013 12:16:02 +0100 smolkas simplified byline, isar_qualifier
Fri, 15 Feb 2013 16:53:39 +0100 blanchet tuning
Fri, 15 Feb 2013 16:40:39 +0100 blanchet repaired collateral damage from 4f0147ed8bcb
Fri, 15 Feb 2013 13:54:54 +0100 blanchet annotate obtains with types
Fri, 15 Feb 2013 13:37:37 +0100 blanchet made check for conjecture skolemization sound
Fri, 15 Feb 2013 11:27:15 +0100 blanchet skolemize conjecture properly in Isar proof
Fri, 15 Feb 2013 10:48:06 +0100 blanchet tuning -- refactoring in preparation for handling skolemization of conjecture
Fri, 15 Feb 2013 10:18:44 +0100 blanchet removed dead weight from data structure
Fri, 15 Feb 2013 10:13:04 +0100 blanchet tuned code
Fri, 15 Feb 2013 10:00:25 +0100 blanchet tuned code
Thu, 14 Feb 2013 22:49:22 +0100 smolkas renamed sledgehammer_shrink to sledgehammer_compress
Thu, 14 Feb 2013 22:49:22 +0100 smolkas dont skolemize conjecture
Thu, 14 Feb 2013 22:49:22 +0100 smolkas introduced subblock in isar_step datatype for conjecture herbrandization
Thu, 07 Feb 2013 18:39:24 +0100 blanchet more robustness in Isar proof reconstruction (cf. bug report by Ondrej)
Thu, 07 Feb 2013 14:05:33 +0100 blanchet tuned indent
Thu, 17 Jan 2013 11:56:34 +0100 smolkas changed type of preplay time; tuned preplaying
Tue, 15 Jan 2013 20:51:30 +0100 blanchet more improvements to Isar proof reconstructions
Thu, 03 Jan 2013 17:28:55 +0100 blanchet use new skolemizer for reconstructing skolemization steps in Isar proofs (because the old skolemizer messes up the order of the Skolem arguments)
Wed, 02 Jan 2013 20:52:39 +0100 smolkas removed whitespace
Wed, 02 Jan 2013 20:35:49 +0100 smolkas use rpair to avoid swap
Wed, 02 Jan 2013 19:59:06 +0100 blanchet generate "obtain" steps corresponding to skolemization inferences
Wed, 02 Jan 2013 16:32:40 +0100 blanchet keep E's and Vampire's skolemization steps
Wed, 02 Jan 2013 16:02:33 +0100 blanchet tuning
Wed, 02 Jan 2013 15:54:38 +0100 blanchet fixed oversensitive Skolem handling (cf. eaa540986291)
Wed, 02 Jan 2013 15:44:00 +0100 blanchet added "obtain" to Isar proof construction data structure
Wed, 02 Jan 2013 13:31:13 +0100 blanchet tuning
Wed, 02 Jan 2013 13:14:47 +0100 blanchet properly take the existential closure of skolems
Sat, 15 Dec 2012 19:57:12 +0100 blanchet thread no timeout properly
Mon, 10 Dec 2012 13:52:33 +0100 wenzelm generalized notion of active area, where sendback is just one application;
Thu, 06 Dec 2012 23:01:49 +0100 wenzelm proper Sendback.markup, as required for standard Prover IDE protocol (see also c62ce309dc26);
Wed, 28 Nov 2012 12:25:43 +0100 smolkas tweaked calculation of sledgehammer messages
Wed, 28 Nov 2012 12:25:43 +0100 smolkas adapted sledgehammer warnings
Wed, 28 Nov 2012 12:25:43 +0100 smolkas fixed preplaying of case splits; incorperated new name of structure: Isabelle_Markup -> Markup
Wed, 28 Nov 2012 12:25:43 +0100 smolkas added warning when shrinking proof without preplaying
Wed, 28 Nov 2012 12:25:43 +0100 smolkas deal with the case that metis does not time out, but fails instead
Wed, 28 Nov 2012 12:25:43 +0100 smolkas renaming, minor tweaks, added signature
Wed, 28 Nov 2012 12:25:43 +0100 smolkas moved thms_of_name to Sledgehammer_Util and removed copies, updated references
Wed, 28 Nov 2012 12:25:43 +0100 smolkas removed duplicate decleration
Wed, 28 Nov 2012 12:25:43 +0100 smolkas renamed sledgehammer_isar_reconstruct to sledgehammer_proof
Wed, 28 Nov 2012 12:25:43 +0100 smolkas fixed problem with fact names
Wed, 28 Nov 2012 12:25:06 +0100 smolkas remove hack and generalize code slightly
Wed, 28 Nov 2012 12:23:44 +0100 smolkas simplified isar_qualifiers and qs merging
Wed, 28 Nov 2012 12:22:17 +0100 smolkas put shrink in own structure
Wed, 28 Nov 2012 12:22:05 +0100 smolkas put annotate in own structure
Wed, 28 Nov 2012 12:21:42 +0100 smolkas support assumptions as facts for preplaying
Wed, 28 Nov 2012 12:20:06 +0100 smolkas some minor improvements in shrink_proof
Mon, 26 Nov 2012 21:46:04 +0100 wenzelm tuned signature;
Mon, 26 Nov 2012 11:45:12 +0100 blanchet distinguish declated tfrees from other tfrees -- only the later can be optimized away
Thu, 22 Nov 2012 13:21:02 +0100 wenzelm more abstract Sendback operations, with explicit id/exec_id properties;
Fri, 16 Nov 2012 16:59:56 +0100 wenzelm made SML/NJ happy;
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
Tue, 06 Nov 2012 15:15:33 +0100 blanchet renamed Sledgehammer option
Tue, 06 Nov 2012 15:12:31 +0100 blanchet always show timing for structured proofs
Tue, 06 Nov 2012 14:46:21 +0100 blanchet use implications rather than disjunctions to improve readability
Tue, 06 Nov 2012 13:47:51 +0100 blanchet avoid name clashes
Tue, 06 Nov 2012 13:09:02 +0100 blanchet fixed more "Trueprop" issues
Tue, 06 Nov 2012 12:38:45 +0100 blanchet removed needless sort
Tue, 06 Nov 2012 11:24:48 +0100 blanchet avoid double "Trueprop"s
Tue, 06 Nov 2012 11:20:56 +0100 blanchet use original formulas for hypotheses and conclusion to avoid mismatches
Tue, 06 Nov 2012 11:20:56 +0100 blanchet track formula roles in proofs and use that to determine whether the conjecture should be negated or not
Tue, 06 Nov 2012 11:20:56 +0100 blanchet proper handling of assumptions arising from the goal's being expressed in rule format, for Isar proof construction
Fri, 02 Nov 2012 16:16:48 +0100 blanchet handle non-unit clauses gracefully
Fri, 02 Nov 2012 16:16:48 +0100 blanchet several improvements to Isar proof reconstruction, by Steffen Smolka (step merging in case splits, time measurements, etc.)
Wed, 31 Oct 2012 11:23:21 +0100 blanchet fixed bool vs. prop mismatch
Wed, 31 Oct 2012 11:23:21 +0100 blanchet took out "using only ..." comments in Sledgehammer generated metis/smt calls, until these can be generated soundly
Wed, 31 Oct 2012 11:23:21 +0100 blanchet use metaquantification when possible in Isar proofs
Wed, 31 Oct 2012 11:23:21 +0100 blanchet tuning
Fri, 19 Oct 2012 17:52:21 +0200 wenzelm made SML/NJ happy;
Thu, 18 Oct 2012 15:41:15 +0200 blanchet tuned Isar output
Thu, 18 Oct 2012 15:05:17 +0200 blanchet renamed Isar-proof related options + changed semantics of Isar shrinking
Thu, 18 Oct 2012 14:26:45 +0200 blanchet tuning
Thu, 18 Oct 2012 13:46:24 +0200 blanchet fixed theorem lookup code in Isar proof reconstruction
Thu, 18 Oct 2012 13:37:53 +0200 blanchet tuning
Thu, 18 Oct 2012 13:19:44 +0200 blanchet refactor code
Thu, 18 Oct 2012 11:59:45 +0200 blanchet tuning
Tue, 16 Oct 2012 20:31:08 +0200 blanchet added missing file
Fri, 22 Oct 2010 12:15:31 +0200 blanchet got rid of duplicate functionality ("run_smt_solver_somehow");
Thu, 21 Oct 2010 16:25:40 +0200 blanchet first step in adding support for an SMT backend to Sledgehammer
Tue, 05 Oct 2010 11:45:10 +0200 blanchet hide uninteresting MESON/Metis constants and facts and remove "meson_" prefix to (now hidden) fact names
Sat, 25 Sep 2010 10:32:14 +0200 blanchet make SML/NJ happy
Fri, 17 Sep 2010 01:22:01 +0200 blanchet move functions around
Thu, 16 Sep 2010 16:24:23 +0200 blanchet added new "Metis_Reconstruct" module, temporarily empty
Thu, 16 Sep 2010 16:12:02 +0200 blanchet rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"
Thu, 16 Sep 2010 15:38:46 +0200 blanchet move SPASS's Flotter hack to "Sledgehammer_Reconstruct"
Thu, 16 Sep 2010 13:52:17 +0200 blanchet merge constructors
Thu, 16 Sep 2010 13:44:41 +0200 blanchet factor out the inverse of "nice_atp_problem"
Thu, 16 Sep 2010 11:59:45 +0200 blanchet use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
Thu, 16 Sep 2010 11:12:08 +0200 blanchet factored out TSTP/SPASS/Vampire proof parsing;
Wed, 15 Sep 2010 18:27:29 +0200 blanchet fix parsing of higher-order formulas;
Tue, 14 Sep 2010 23:36:23 +0200 blanchet fix splitting of proof lines for one-line metis calls;
Tue, 14 Sep 2010 23:01:29 +0200 blanchet finish support for E 1.2 proof reconstruction;
Tue, 14 Sep 2010 20:07:18 +0200 blanchet first step in generalizing to nonnumeric proof step names (e.g. remote Vampire 0.6)
Tue, 14 Sep 2010 19:38:44 +0200 blanchet use same hack as in "Async_Manager" to work around Proof General bug
Tue, 14 Sep 2010 17:36:27 +0200 blanchet generalize proof reconstruction code;
Mon, 13 Sep 2010 21:24:10 +0200 blanchet merged
Sat, 11 Sep 2010 12:31:42 +0200 blanchet tuning
Sun, 12 Sep 2010 19:04:02 +0200 wenzelm eliminated aliases of Type.constraint;
Sun, 05 Sep 2010 21:41:24 +0200 wenzelm turned show_sorts/show_types into proper configuration options;
Fri, 03 Sep 2010 15:54:03 +0200 wenzelm turned show_no_free_types into proper configuration option show_free_types, with flipped polarity;
Thu, 02 Sep 2010 22:02:48 +0200 blanchet fix trivial "x = x" fact detection
Tue, 31 Aug 2010 23:50:59 +0200 blanchet finished renaming
Tue, 31 Aug 2010 23:46:23 +0200 blanchet shorten a few file names
less more (0) tip