Thu, 12 May 2011 22:35:15 +0200 |
wenzelm |
modernized dead code;
|
changeset |
files
|
Thu, 12 May 2011 22:33:38 +0200 |
wenzelm |
eliminated old-style MI_fast_css -- replaced by fast_solver with config option;
|
changeset |
files
|
Thu, 12 May 2011 22:11:16 +0200 |
wenzelm |
eliminated obsolete MI_css -- use current context directly;
|
changeset |
files
|
Thu, 12 May 2011 22:07:30 +0200 |
wenzelm |
proper method_setup;
|
changeset |
files
|
Thu, 12 May 2011 21:14:03 +0200 |
wenzelm |
modernized simproc_setup;
|
changeset |
files
|
Thu, 12 May 2011 18:18:06 +0200 |
wenzelm |
prefer Proof.context over old-style clasimpset;
|
changeset |
files
|
Thu, 12 May 2011 18:17:32 +0200 |
wenzelm |
modernized dead code;
|
changeset |
files
|
Thu, 12 May 2011 17:17:57 +0200 |
wenzelm |
modernized specifications;
|
changeset |
files
|
Thu, 12 May 2011 16:58:55 +0200 |
wenzelm |
merged
|
changeset |
files
|
Thu, 12 May 2011 16:48:23 +0200 |
blanchet |
added hints and FAQs
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
prove one more lemma using Sledgehammer, with some guidance, and replace clumsy old proof that relied on old extensionality behavior
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
fixed several bugs in Isar proof reconstruction, in particular w.r.t. mangled types and hAPP
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
another concession to backward compatibility
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
no need to use metisFT for Isar proofs -- metis falls back on it anyway
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
handle equality proxy in a more backward-compatible way
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
remove problematic Isar proof
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
added two mildly higher-order examples contributed by TN, removed references to obsoleted type systems, and moved things around
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
robustly detect how many type args were passed to the ATP, even if some of them were omitted
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
make sure "simple_types_query" and "simple_types_bang" symbols are declared with the proper types
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
drop some type arguments to constants in unsound type systems + remove a few type systems that make no sense from the circulation
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
tuning
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
fixed conjecture resolution bug for Vampire 1.0's TSTP output
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
ensure Set.member isn't introduced by Meson's preprocessing if it's supposed to be unfolded
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
Metis doesn't find an old proof in acceptable time now that higher-order equality reasoning is supported -- tuned proof script to help it
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
drop support for Vampire's native output format -- it has too many undocumented oddities, e.g. "BDD definition:" lines
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
use the same code for extensionalization in Metis and Sledgehammer and generalize that code so that it gracefully handles negations (e.g. negated conjecture), formulas of the form (%x. t) = u, etc.
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
further lower penalty associated with existentials in Sledgehammer's relevance filter, so that "exhaust" facts are picked up
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
reenabled equality proxy in Metis for higher-order reasoning
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
added "SMT." qualifier for constant to make it possible to reload "smt_monomorph.ML" from outside the "SMT" theory (for experiments) -- this is also consistent with the other SMT constants mentioned in this source file
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
reflect option renaming in doc + do not document the type systems poly_preds? and poly_tags?, since they are virtually identical to the non-? versions
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
unfold set constants in Sledgehammer/ATP as well if Metis does it too
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
do not pollute relevance filter facts with too many facts about the boring set constants Collect and mem_def, which we might anyway unfold depending on Meson's settings
|
changeset |
files
|