Wed, 09 Oct 2013 16:40:03 +0200 |
blanchet |
no isar proofs if preplay was not attempted
|
file |
diff |
annotate
|
Fri, 20 Sep 2013 22:39:30 +0200 |
blanchet |
merged "isar_try0" and "isar_minimize" options
|
file |
diff |
annotate
|
Fri, 20 Sep 2013 22:39:30 +0200 |
blanchet |
hardcoded obscure option
|
file |
diff |
annotate
|
Fri, 20 Sep 2013 22:39:30 +0200 |
blanchet |
hard-coded an obscure option
|
file |
diff |
annotate
|
Fri, 20 Sep 2013 22:39:30 +0200 |
blanchet |
use configuration mechanism for low-level tracing
|
file |
diff |
annotate
|
Thu, 12 Sep 2013 22:10:57 +0200 |
blanchet |
prefixed types and some functions with "atp_" for disambiguation
|
file |
diff |
annotate
|
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;
|
file |
diff |
annotate
|
Sat, 17 Aug 2013 11:34:50 +0200 |
wenzelm |
more explicit sendback propertries based on mode;
|
file |
diff |
annotate
|
Mon, 29 Jul 2013 16:13:35 +0200 |
blanchet |
parse nonnumeric identifiers in E proofs correctly
|
file |
diff |
annotate
|
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;
|
file |
diff |
annotate
|
Fri, 12 Jul 2013 22:41:25 +0200 |
smolkas |
added sledgehammer parameters isar_try0 and isar_minimize and their negative aliases
|
file |
diff |
annotate
|
Fri, 12 Jul 2013 19:03:08 +0200 |
smolkas |
cleaner preplay interface
|
file |
diff |
annotate
|
Fri, 12 Jul 2013 14:18:06 +0200 |
smolkas |
minimize dependencies (used facts) of Isar proof steps; remove unreferenced steps
|
file |
diff |
annotate
|
Thu, 11 Jul 2013 20:08:06 +0200 |
smolkas |
optimize isar-proofs by trying different proof methods
|
file |
diff |
annotate
|
Tue, 09 Jul 2013 18:45:06 +0200 |
smolkas |
completely rewrote SH compress; added two parameters for experimentation/fine grained control
|
file |
diff |
annotate
|
Tue, 09 Jul 2013 18:44:59 +0200 |
smolkas |
moved code -> easier debugging
|
file |
diff |
annotate
|
Wed, 26 Jun 2013 18:26:00 +0200 |
smolkas |
tuned: cleaned up data structure
|
file |
diff |
annotate
|
Wed, 26 Jun 2013 18:25:13 +0200 |
smolkas |
simplified data structure
|
file |
diff |
annotate
|
Thu, 13 Jun 2013 16:58:20 -0400 |
blanchet |
tuning
|
file |
diff |
annotate
|
Tue, 11 Jun 2013 19:58:09 -0400 |
smolkas |
uncheck terms before annotation to avoid awkward syntax
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
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])
|
file |
diff |
annotate
|
Sun, 26 May 2013 12:56:37 +0200 |
blanchet |
handle lambda-lifted problems in Isar construction code
|
file |
diff |
annotate
|
Fri, 24 May 2013 16:43:37 +0200 |
blanchet |
improved handling of free variables' types in Isar proofs
|
file |
diff |
annotate
|
Mon, 20 May 2013 13:07:31 +0200 |
blanchet |
parse agsyHOL proofs (as unsat cores)
|
file |
diff |
annotate
|
Thu, 16 May 2013 14:58:30 +0200 |
blanchet |
correctly 'repair' the monomorphization context for SMT solvers from Sledgehammer
|
file |
diff |
annotate
|
Thu, 16 May 2013 13:34:13 +0200 |
blanchet |
tuning -- renamed '_from_' to '_of_' in Sledgehammer
|
file |
diff |
annotate
|
Wed, 15 May 2013 17:43:42 +0200 |
blanchet |
renamed Sledgehammer functions with 'for' in their names to 'of'
|
file |
diff |
annotate
|
Tue, 14 May 2013 09:49:03 +0200 |
blanchet |
generate valid direct Isar proof also if the facts are contradictory
|
file |
diff |
annotate
|
Mon, 06 May 2013 11:03:08 +0200 |
smolkas |
added preplay tracing
|
file |
diff |
annotate
|
Tue, 23 Apr 2013 16:30:30 +0200 |
blanchet |
tuning
|
file |
diff |
annotate
|
Sat, 23 Feb 2013 22:00:12 +0100 |
wenzelm |
make SML/NJ happy;
|
file |
diff |
annotate
|
Thu, 21 Feb 2013 12:22:26 +0100 |
blanchet |
generate Isar proof if Metis appears to be too slow
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 17:42:20 +0100 |
blanchet |
ensure all conjecture clauses are in the graph -- to prevent exceptions later
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 17:05:24 +0100 |
blanchet |
remove needless steps from refutation graph -- these confuse the proof redirection algorithm (and are needless)
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 14:47:19 +0100 |
blanchet |
trust preplayed proof in Mirabelle
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 14:44:00 +0100 |
blanchet |
added case taken out by mistake
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 14:21:17 +0100 |
blanchet |
tuning (removed redundant datatype)
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 14:10:51 +0100 |
blanchet |
minimize SMT proofs with E if Isar proofs are desired and Metis managed to preplay
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 10:54:13 +0100 |
blanchet |
got rid of rump support for Vampire definitions
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 08:56:34 +0100 |
blanchet |
tuning
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 08:44:24 +0100 |
blanchet |
slacker comparison for Skolems, to avoid trivial equations
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
Mon, 18 Feb 2013 12:16:02 +0100 |
smolkas |
simplified byline, isar_qualifier
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 16:53:39 +0100 |
blanchet |
tuning
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 16:40:39 +0100 |
blanchet |
repaired collateral damage from 4f0147ed8bcb
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 13:54:54 +0100 |
blanchet |
annotate obtains with types
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 13:37:37 +0100 |
blanchet |
made check for conjecture skolemization sound
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 11:27:15 +0100 |
blanchet |
skolemize conjecture properly in Isar proof
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 10:48:06 +0100 |
blanchet |
tuning -- refactoring in preparation for handling skolemization of conjecture
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 10:18:44 +0100 |
blanchet |
removed dead weight from data structure
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 10:13:04 +0100 |
blanchet |
tuned code
|
file |
diff |
annotate
|
Fri, 15 Feb 2013 10:00:25 +0100 |
blanchet |
tuned code
|
file |
diff |
annotate
|
Thu, 14 Feb 2013 22:49:22 +0100 |
smolkas |
renamed sledgehammer_shrink to sledgehammer_compress
|
file |
diff |
annotate
|
Thu, 14 Feb 2013 22:49:22 +0100 |
smolkas |
dont skolemize conjecture
|
file |
diff |
annotate
|
Thu, 14 Feb 2013 22:49:22 +0100 |
smolkas |
introduced subblock in isar_step datatype for conjecture herbrandization
|
file |
diff |
annotate
|
Thu, 07 Feb 2013 18:39:24 +0100 |
blanchet |
more robustness in Isar proof reconstruction (cf. bug report by Ondrej)
|
file |
diff |
annotate
|