Thu, 12 May 2011 22:37:31 +0200 |
wenzelm |
removed obsolete old-style cs/css;
|
changeset |
files
|
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
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
added unfold set constant functionality to Meson/Metis -- disabled by default for now
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
remove unused parameter
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
reduced penalty associated with existential quantifiers
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
ensure that Auto Sledgehammer is run with full type information
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
fine-tuned the relevance filter, so that equations of the form "c = (%x. _)" and constants occurring in chained facts are not unduely penalized
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
don't give weights to built-in symbols
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
more robust exception handling in Metis (also works if there are several subgoals)
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
no penality for constants that appear in chained facts
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
gracefully declare fTrue and fFalse proxies' types if the constants only appear in the helpers
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
improve detection of quantifications over dangerous types by leveraging "is_type_surely_finite" predicate and added "prop" to the list of surely finite types
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
tune whitespace
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
added configuration options for experimental features
|
changeset |
files
|
Thu, 12 May 2011 15:29:19 +0200 |
blanchet |
ensure type class predicates are generated in symbol declarations (for "poly_preds" and similar)
|
changeset |
files
|
Thu, 12 May 2011 15:29:18 +0200 |
blanchet |
avoid "Empty" exception by making sure that a certain optimization only is attempted when it makes sense
|
changeset |
files
|
Thu, 12 May 2011 15:29:18 +0200 |
blanchet |
added "force_sos" options to control SPASS's and Vampire's use of SOS in experiments + added corresponding Mirabelle options
|
changeset |
files
|
Thu, 12 May 2011 15:29:18 +0200 |
blanchet |
added "max_mono_instances" option to Sledgehammer and renamed old "monomorphize_limit" option
|
changeset |
files
|
Thu, 12 May 2011 15:29:18 +0200 |
blanchet |
allow each slice to have its own type system
|
changeset |
files
|
Thu, 12 May 2011 15:29:18 +0200 |
blanchet |
renamed type systems for more consistency
|
changeset |
files
|
Thu, 12 May 2011 16:46:49 +0200 |
wenzelm |
updated versions;
|
changeset |
files
|
Thu, 12 May 2011 16:46:21 +0200 |
wenzelm |
added toplevel isabelle package -- reduce warnings with scala-2.9.0.final;
|
changeset |
files
|
Thu, 12 May 2011 16:42:57 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Thu, 12 May 2011 16:28:46 +0200 |
wenzelm |
minor adaption for scala-2.9.0.final;
|
changeset |
files
|
Thu, 12 May 2011 16:23:13 +0200 |
wenzelm |
proper configuration options Proof_Context.debug and Proof_Context.verbose;
|
changeset |
files
|
Thu, 12 May 2011 16:00:48 +0200 |
wenzelm |
pretend that all versions of BSD are Linux, which might actually work due to binary compatibilty mode of these obsolete platforms;
|
changeset |
files
|
Thu, 12 May 2011 11:03:48 +0200 |
haftmann |
more uniform naming of lemma
|
changeset |
files
|
Mon, 09 May 2011 16:11:20 +0200 |
noschinl |
add a lemma about commutative append to List.thy
|
changeset |
files
|