src/HOL/Algebra/abstract/Ring2.thy
changeset 45625 750c5a47400b
parent 42814 5af15f1e2ef6
child 50108 f171b5240c31
--- a/src/HOL/Algebra/abstract/Ring2.thy	Thu Nov 24 20:45:34 2011 +0100
+++ b/src/HOL/Algebra/abstract/Ring2.thy	Thu Nov 24 21:01:06 2011 +0100
@@ -210,7 +210,9 @@
 
 fun termless_ring (a, b) = (Term_Ord.term_lpo ring_ord (a, b) = LESS);
 
-val ring_ss = HOL_basic_ss settermless termless_ring addsimps
+val ring_ss =
+  (HOL_basic_ss |> Simplifier.set_termless termless_ring)
+  addsimps
   [@{thm a_assoc}, @{thm l_zero}, @{thm l_neg}, @{thm a_comm}, @{thm m_assoc},
    @{thm l_one}, @{thm l_distr}, @{thm m_comm}, @{thm minus_def},
    @{thm r_zero}, @{thm r_neg}, @{thm r_neg2}, @{thm r_neg1}, @{thm minus_add},