src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
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
less more (0) -60 tip