wenzelm [Fri, 25 Jul 1997 14:31:48 +0200] rev 3581
removed split_paired_Ex;
fixed proc args;
nipkow [Fri, 25 Jul 1997 13:59:15 +0200] rev 3580
new simproc
wenzelm [Fri, 25 Jul 1997 13:20:12 +0200] rev 3579
*** empty log message ***
wenzelm [Fri, 25 Jul 1997 13:18:45 +0200] rev 3578
load simplifier.ML (again);
wenzelm [Fri, 25 Jul 1997 13:18:09 +0200] rev 3577
added prems argument to simplification procedures;
wenzelm [Fri, 25 Jul 1997 13:17:14 +0200] rev 3576
remove references to simplifier.ML;
wenzelm [Fri, 25 Jul 1997 11:47:09 +0200] rev 3575
improved rewrite_thm / rewrite_goals to handle conditional eqns;
nipkow [Thu, 24 Jul 1997 15:25:29 +0200] rev 3574
Added a few lemmas.
nipkow [Thu, 24 Jul 1997 11:20:12 +0200] rev 3573
Deleted comment.
nipkow [Thu, 24 Jul 1997 11:13:12 +0200] rev 3572
Replaced clumsy rewriting by the new function simplify on thms.
nipkow [Thu, 24 Jul 1997 11:12:18 +0200] rev 3571
List.ML: added lemmas by Stefan Merz.
simpodata.ML: removed rules about ? now subsumed by simplification proc.
paulson [Thu, 24 Jul 1997 10:46:32 +0200] rev 3570
set_of_list -> set
nipkow [Wed, 23 Jul 1997 17:44:15 +0200] rev 3569
Simplified a few proofs because of improved simplification.
nipkow [Wed, 23 Jul 1997 17:43:42 +0200] rev 3568
Prod.ML: Added split_paired_EX and lots of comments about failed attempts to
automate reasoning about products.
simpdata.ML: added simplification procedure for simplifying existential
statements of the form ? x. ... & x = t & ...
wenzelm [Wed, 23 Jul 1997 16:03:19 +0200] rev 3567
added simplification meta rules;