huffman [Thu, 04 Dec 2008 13:30:09 -0800] rev 28986
include iszero_simps in lemmas comp_arith
huffman [Thu, 04 Dec 2008 12:32:38 -0800] rev 28985
add named lemma lists: neg_simps and iszero_simps
huffman [Thu, 04 Dec 2008 11:14:24 -0800] rev 28984
change arith_special simps to avoid using neg
kleing [Fri, 05 Dec 2008 11:35:07 +1100] rev 28983
merged
kleing [Fri, 05 Dec 2008 11:33:03 +1100] rev 28982
run test for sunbroy2 on /tmp,
be careful about removing old test dir
wenzelm [Fri, 05 Dec 2008 00:23:37 +0100] rev 28981
merged
wenzelm [Thu, 04 Dec 2008 23:46:20 +0100] rev 28980
refined Future.fork interfaces, no longer export Future.future;
wenzelm [Thu, 04 Dec 2008 23:46:20 +0100] rev 28979
fork/map: no inheritance of group (structure is nested, not parallel);
removed group thread_data;
refined Future.fork interfaces, no longer export Future.future;
wenzelm [Thu, 04 Dec 2008 23:02:56 +0100] rev 28978
future proofs: pass actual futures to facilitate composite computations;
removed join_futures -- superceded by higher-level PureThy.force_proofs;
wenzelm [Thu, 04 Dec 2008 23:02:52 +0100] rev 28977
renamed type Lazy.T to lazy;
force_proofs: original order;