dropped essentially ineffective tuning
authorhaftmann
Mon, 19 Jul 2010 16:09:43 +0200
changeset 37885 c43805c80eb6
parent 37884 314a88278715
child 37886 2f9d3fc1a8ac
dropped essentially ineffective tuning
src/HOL/ex/Lagrange.thy
--- a/src/HOL/ex/Lagrange.thy	Mon Jul 19 16:09:43 2010 +0200
+++ b/src/HOL/ex/Lagrange.thy	Mon Jul 19 16:09:43 2010 +0200
@@ -22,12 +22,6 @@
 However, this is an abstract theorem about commutative rings.  It has,
 a priori, nothing to do with nat. *}
 
-(* These two simprocs are even less efficient than ordered rewriting
-   and kill the second example: *)
-ML {*
-  Delsimprocs [ab_group_add_cancel.sum_conv, ab_group_add_cancel.rel_conv]
-*}
-
 lemma Lagrange_lemma: fixes x1 :: "'a::comm_ring" shows
   "(sq x1 + sq x2 + sq x3 + sq x4) * (sq y1 + sq y2 + sq y3 + sq y4) =
    sq (x1*y1 - x2*y2 - x3*y3 - x4*y4)  +