src/HOL/Algebra/abstract/Ring2.thy
changeset 35408 b48ab741683b
parent 35330 e7eb254db165
child 35848 5443079512ea
--- a/src/HOL/Algebra/abstract/Ring2.thy	Sat Feb 27 22:52:25 2010 +0100
+++ b/src/HOL/Algebra/abstract/Ring2.thy	Sat Feb 27 23:13:01 2010 +0100
@@ -207,7 +207,7 @@
         @{const_name Groups.minus}, @{const_name Groups.one}, @{const_name Groups.times}]
   | ring_ord _ = ~1;
 
-fun termless_ring (a, b) = (TermOrd.term_lpo ring_ord (a, b) = LESS);
+fun termless_ring (a, b) = (Term_Ord.term_lpo ring_ord (a, b) = LESS);
 
 val ring_ss = HOL_basic_ss settermless termless_ring addsimps
   [thm "a_assoc", thm "l_zero", thm "l_neg", thm "a_comm", thm "m_assoc",