src/HOL/Algebra/ringsimp.ML
changeset 67560 0fa87bd86566
parent 58811 19382bbfa93a
child 67561 f0b11413f1c9
--- a/src/HOL/Algebra/ringsimp.ML	Thu Feb 01 13:55:10 2018 +0100
+++ b/src/HOL/Algebra/ringsimp.ML	Thu Feb 01 15:12:57 2018 +0100
@@ -47,7 +47,7 @@
     val ops = map (fst o Term.strip_comb) ts;
     fun ord (Const (a, _)) = find_index (fn (Const (b, _)) => a=b | _ => false) ops
       | ord (Free (a, _)) = find_index (fn (Free (b, _)) => a=b | _ => false) ops;
-    fun less (a, b) = (Term_Ord.term_lpo ord (a, b) = LESS);
+    val less = is_less o Term_Ord.term_lpo ord;
   in asm_full_simp_tac (put_simpset HOL_ss ctxt addsimps simps |> Simplifier.set_termless less) end;
 
 fun algebra_tac ctxt =