Sat, 14 May 2011 13:32:33 +0200 simplified BLAST_DATA;
wenzelm [Sat, 14 May 2011 13:32:33 +0200] rev 42802
simplified BLAST_DATA;
Sat, 14 May 2011 13:26:55 +0200 proper Proof.context -- eliminated global operations;
wenzelm [Sat, 14 May 2011 13:26:55 +0200] rev 42801
proper Proof.context -- eliminated global operations;
Sat, 14 May 2011 12:40:11 +0200 just one universal Proof.context -- discontinued claset/clasimpset;
wenzelm [Sat, 14 May 2011 12:40:11 +0200] rev 42800
just one universal Proof.context -- discontinued claset/clasimpset;
Sat, 14 May 2011 11:42:43 +0200 modernized functor names;
wenzelm [Sat, 14 May 2011 11:42:43 +0200] rev 42799
modernized functor names; tuned;
Sat, 14 May 2011 00:32:16 +0200 method "deepen" with optional limit;
wenzelm [Sat, 14 May 2011 00:32:16 +0200] rev 42798
method "deepen" with optional limit;
Fri, 13 May 2011 23:59:48 +0200 merged
wenzelm [Fri, 13 May 2011 23:59:48 +0200] rev 42797
merged
Fri, 13 May 2011 21:36:01 +0200 removed redundant type annotations and duplicate examples
krauss [Fri, 13 May 2011 21:36:01 +0200] rev 42796
removed redundant type annotations and duplicate examples
Fri, 13 May 2011 23:58:40 +0200 clarified map_simpset versus Simplifier.map_simpset_global;
wenzelm [Fri, 13 May 2011 23:58:40 +0200] rev 42795
clarified map_simpset versus Simplifier.map_simpset_global;
Fri, 13 May 2011 23:24:06 +0200 make ZF_cs snapshot after final setup;
wenzelm [Fri, 13 May 2011 23:24:06 +0200] rev 42794
make ZF_cs snapshot after final setup;
Fri, 13 May 2011 22:55:00 +0200 proper Proof.context for classical tactics;
wenzelm [Fri, 13 May 2011 22:55:00 +0200] rev 42793
proper Proof.context for classical tactics; reduced claset to snapshot of classical context; discontinued clasimpset;
Fri, 13 May 2011 16:03:03 +0200 do not open ML structures;
wenzelm [Fri, 13 May 2011 16:03:03 +0200] rev 42792
do not open ML structures;
Fri, 13 May 2011 15:55:32 +0200 eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm [Fri, 13 May 2011 15:55:32 +0200] rev 42791
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
Fri, 13 May 2011 15:47:54 +0200 misc tuning and simplification;
wenzelm [Fri, 13 May 2011 15:47:54 +0200] rev 42790
misc tuning and simplification;
Fri, 13 May 2011 14:39:55 +0200 tuned proof;
wenzelm [Fri, 13 May 2011 14:39:55 +0200] rev 42789
tuned proof;
Fri, 13 May 2011 14:26:51 +0200 tuned proof;
wenzelm [Fri, 13 May 2011 14:26:51 +0200] rev 42788
tuned proof;
Fri, 13 May 2011 14:25:35 +0200 proper method_setup;
wenzelm [Fri, 13 May 2011 14:25:35 +0200] rev 42787
proper method_setup;
Fri, 13 May 2011 14:16:46 +0200 proper method_setup "split_idle";
wenzelm [Fri, 13 May 2011 14:16:46 +0200] rev 42786
proper method_setup "split_idle";
Fri, 13 May 2011 14:04:47 +0200 proper method_setup "enabled";
wenzelm [Fri, 13 May 2011 14:04:47 +0200] rev 42785
proper method_setup "enabled";
Fri, 13 May 2011 13:45:20 +0200 simplified clasimpset declarations -- prefer attributes;
wenzelm [Fri, 13 May 2011 13:45:20 +0200] rev 42784
simplified clasimpset declarations -- prefer attributes;
Fri, 13 May 2011 10:10:44 +0200 reduce the number of mono iterations to prevent the mono code from going berserk
blanchet [Fri, 13 May 2011 10:10:44 +0200] rev 42783
reduce the number of mono iterations to prevent the mono code from going berserk
Fri, 13 May 2011 10:10:43 +0200 tuned comment
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42782
tuned comment
Fri, 13 May 2011 10:10:43 +0200 optimized a common case
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42781
optimized a common case
Fri, 13 May 2011 10:10:43 +0200 avoid "UnequalLengths" exception for special constant "fequal" -- and optimize code in the common case where no type arguments are needed
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42780
avoid "UnequalLengths" exception for special constant "fequal" -- and optimize code in the common case where no type arguments are needed
Fri, 13 May 2011 10:10:43 +0200 tweak E slices
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42779
tweak E slices
Fri, 13 May 2011 10:10:43 +0200 make SML/NJ happy
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42778
make SML/NJ happy
Fri, 13 May 2011 10:10:43 +0200 fixed off-by-one bug
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42777
fixed off-by-one bug
Fri, 13 May 2011 10:10:43 +0200 added convenience syntax
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42776
added convenience syntax
Thu, 12 May 2011 23:23:48 +0200 prefer Proof.context over old-style claset/simpset;
wenzelm [Thu, 12 May 2011 23:23:48 +0200] rev 42775
prefer Proof.context over old-style claset/simpset; canonical argument order;
Thu, 12 May 2011 22:46:21 +0200 prefer plain simpset operations;
wenzelm [Thu, 12 May 2011 22:46:21 +0200] rev 42774
prefer plain simpset operations;
Thu, 12 May 2011 22:37:31 +0200 removed obsolete old-style cs/css;
wenzelm [Thu, 12 May 2011 22:37:31 +0200] rev 42773
removed obsolete old-style cs/css;
Thu, 12 May 2011 22:35:15 +0200 modernized dead code;
wenzelm [Thu, 12 May 2011 22:35:15 +0200] rev 42772
modernized dead code;
Thu, 12 May 2011 22:33:38 +0200 eliminated old-style MI_fast_css -- replaced by fast_solver with config option;
wenzelm [Thu, 12 May 2011 22:33:38 +0200] rev 42771
eliminated old-style MI_fast_css -- replaced by fast_solver with config option;
Thu, 12 May 2011 22:11:16 +0200 eliminated obsolete MI_css -- use current context directly;
wenzelm [Thu, 12 May 2011 22:11:16 +0200] rev 42770
eliminated obsolete MI_css -- use current context directly;
Thu, 12 May 2011 22:07:30 +0200 proper method_setup;
wenzelm [Thu, 12 May 2011 22:07:30 +0200] rev 42769
proper method_setup;
Thu, 12 May 2011 21:14:03 +0200 modernized simproc_setup;
wenzelm [Thu, 12 May 2011 21:14:03 +0200] rev 42768
modernized simproc_setup; misc tuning and simplification;
Thu, 12 May 2011 18:18:06 +0200 prefer Proof.context over old-style clasimpset;
wenzelm [Thu, 12 May 2011 18:18:06 +0200] rev 42767
prefer Proof.context over old-style clasimpset;
Thu, 12 May 2011 18:17:32 +0200 modernized dead code;
wenzelm [Thu, 12 May 2011 18:17:32 +0200] rev 42766
modernized dead code;
Thu, 12 May 2011 17:17:57 +0200 modernized specifications;
wenzelm [Thu, 12 May 2011 17:17:57 +0200] rev 42765
modernized specifications;
Thu, 12 May 2011 16:58:55 +0200 merged
wenzelm [Thu, 12 May 2011 16:58:55 +0200] rev 42764
merged
Thu, 12 May 2011 16:48:23 +0200 added hints and FAQs
blanchet [Thu, 12 May 2011 16:48:23 +0200] rev 42763
added hints and FAQs
Thu, 12 May 2011 15:29:19 +0200 prove one more lemma using Sledgehammer, with some guidance, and replace clumsy old proof that relied on old extensionality behavior
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42762
prove one more lemma using Sledgehammer, with some guidance, and replace clumsy old proof that relied on old extensionality behavior
Thu, 12 May 2011 15:29:19 +0200 fixed several bugs in Isar proof reconstruction, in particular w.r.t. mangled types and hAPP
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42761
fixed several bugs in Isar proof reconstruction, in particular w.r.t. mangled types and hAPP
Thu, 12 May 2011 15:29:19 +0200 another concession to backward compatibility
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42760
another concession to backward compatibility
Thu, 12 May 2011 15:29:19 +0200 no need to use metisFT for Isar proofs -- metis falls back on it anyway
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42759
no need to use metisFT for Isar proofs -- metis falls back on it anyway
Thu, 12 May 2011 15:29:19 +0200 handle equality proxy in a more backward-compatible way
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42758
handle equality proxy in a more backward-compatible way
Thu, 12 May 2011 15:29:19 +0200 remove problematic Isar proof
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42757
remove problematic Isar proof
Thu, 12 May 2011 15:29:19 +0200 added two mildly higher-order examples contributed by TN, removed references to obsoleted type systems, and moved things around
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42756
added two mildly higher-order examples contributed by TN, removed references to obsoleted type systems, and moved things around
Thu, 12 May 2011 15:29:19 +0200 robustly detect how many type args were passed to the ATP, even if some of them were omitted
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42755
robustly detect how many type args were passed to the ATP, even if some of them were omitted
Thu, 12 May 2011 15:29:19 +0200 make sure "simple_types_query" and "simple_types_bang" symbols are declared with the proper types
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42754
make sure "simple_types_query" and "simple_types_bang" symbols are declared with the proper types
Thu, 12 May 2011 15:29:19 +0200 drop some type arguments to constants in unsound type systems + remove a few type systems that make no sense from the circulation
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42753
drop some type arguments to constants in unsound type systems + remove a few type systems that make no sense from the circulation
Thu, 12 May 2011 15:29:19 +0200 tuning
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42752
tuning
Thu, 12 May 2011 15:29:19 +0200 fixed conjecture resolution bug for Vampire 1.0's TSTP output
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42751
fixed conjecture resolution bug for Vampire 1.0's TSTP output
Thu, 12 May 2011 15:29:19 +0200 ensure Set.member isn't introduced by Meson's preprocessing if it's supposed to be unfolded
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42750
ensure Set.member isn't introduced by Meson's preprocessing if it's supposed to be unfolded
Thu, 12 May 2011 15:29:19 +0200 Metis doesn't find an old proof in acceptable time now that higher-order equality reasoning is supported -- tuned proof script to help it
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42749
Metis doesn't find an old proof in acceptable time now that higher-order equality reasoning is supported -- tuned proof script to help it
Thu, 12 May 2011 15:29:19 +0200 drop support for Vampire's native output format -- it has too many undocumented oddities, e.g. "BDD definition:" lines
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42748
drop support for Vampire's native output format -- it has too many undocumented oddities, e.g. "BDD definition:" lines
Thu, 12 May 2011 15:29:19 +0200 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.
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42747
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.
Thu, 12 May 2011 15:29:19 +0200 further lower penalty associated with existentials in Sledgehammer's relevance filter, so that "exhaust" facts are picked up
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42746
further lower penalty associated with existentials in Sledgehammer's relevance filter, so that "exhaust" facts are picked up
Thu, 12 May 2011 15:29:19 +0200 reenabled equality proxy in Metis for higher-order reasoning
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42745
reenabled equality proxy in Metis for higher-order reasoning
Thu, 12 May 2011 15:29:19 +0200 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
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42744
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
Thu, 12 May 2011 15:29:19 +0200 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
blanchet [Thu, 12 May 2011 15:29:19 +0200] rev 42743
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
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip