wenzelm [Sat, 14 May 2011 11:42:43 +0200] rev 42799
modernized functor names;
tuned;
wenzelm [Sat, 14 May 2011 00:32:16 +0200] rev 42798
method "deepen" with optional limit;
wenzelm [Fri, 13 May 2011 23:59:48 +0200] rev 42797
merged
krauss [Fri, 13 May 2011 21:36:01 +0200] rev 42796
removed redundant type annotations and duplicate examples
wenzelm [Fri, 13 May 2011 23:58:40 +0200] rev 42795
clarified map_simpset versus Simplifier.map_simpset_global;
wenzelm [Fri, 13 May 2011 23:24:06 +0200] rev 42794
make ZF_cs snapshot after final setup;
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;
wenzelm [Fri, 13 May 2011 16:03:03 +0200] rev 42792
do not open ML structures;
wenzelm [Fri, 13 May 2011 15:55:32 +0200] rev 42791
eliminated weight_ASTAR: int Unsynchronized.ref (astar_tac appears to be obsolete anyway);
wenzelm [Fri, 13 May 2011 15:47:54 +0200] rev 42790
misc tuning and simplification;
wenzelm [Fri, 13 May 2011 14:39:55 +0200] rev 42789
tuned proof;
wenzelm [Fri, 13 May 2011 14:26:51 +0200] rev 42788
tuned proof;
wenzelm [Fri, 13 May 2011 14:25:35 +0200] rev 42787
proper method_setup;
wenzelm [Fri, 13 May 2011 14:16:46 +0200] rev 42786
proper method_setup "split_idle";
wenzelm [Fri, 13 May 2011 14:04:47 +0200] rev 42785
proper method_setup "enabled";
wenzelm [Fri, 13 May 2011 13:45:20 +0200] rev 42784
simplified clasimpset declarations -- prefer attributes;
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
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42782
tuned comment
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42781
optimized a common case
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
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42779
tweak E slices
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42778
make SML/NJ happy
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42777
fixed off-by-one bug
blanchet [Fri, 13 May 2011 10:10:43 +0200] rev 42776
added convenience syntax
wenzelm [Thu, 12 May 2011 23:23:48 +0200] rev 42775
prefer Proof.context over old-style claset/simpset;
canonical argument order;
wenzelm [Thu, 12 May 2011 22:46:21 +0200] rev 42774
prefer plain simpset operations;
wenzelm [Thu, 12 May 2011 22:37:31 +0200] rev 42773
removed obsolete old-style cs/css;
wenzelm [Thu, 12 May 2011 22:35:15 +0200] rev 42772
modernized dead code;
wenzelm [Thu, 12 May 2011 22:33:38 +0200] rev 42771
eliminated old-style MI_fast_css -- replaced by fast_solver with config option;
wenzelm [Thu, 12 May 2011 22:11:16 +0200] rev 42770
eliminated obsolete MI_css -- use current context directly;