src/HOL/Tools/groebner.ML
changeset 67405 e9ab4ad7bd15
parent 67399 eab6ce8368fa
child 67559 833d154ab189
--- a/src/HOL/Tools/groebner.ML	Thu Jan 11 12:32:07 2018 +0100
+++ b/src/HOL/Tools/groebner.ML	Thu Jan 11 13:48:17 2018 +0100
@@ -601,7 +601,7 @@
     else tm::acc ;
 
 fun grobify_term vars tm =
-((if not (member (aconvc) vars tm) then raise CTERM ("Not a variable", [tm]) else
+((if not (member (op aconvc) vars tm) then raise CTERM ("Not a variable", [tm]) else
      [(@1, map (fn i => if i aconvc tm then 1 else 0) vars)])
 handle  CTERM _ =>
  ((let val x = dest_const tm
@@ -823,7 +823,7 @@
   val th1 = (the (get_first (try (isolate_variable vars)) cjs)
              handle Option.Option => raise CTERM ("unwind_polys_conv",[tm]))
   val eq = Thm.lhs_of th1
-  val bod' = list_mk_binop \<^cterm>\<open>HOL.conj\<close> (eq::(remove (aconvc) eq cjs))
+  val bod' = list_mk_binop \<^cterm>\<open>HOL.conj\<close> (eq::(remove (op aconvc) eq cjs))
   val th2 = conj_ac_rule (mk_eq bod bod')
   val th3 =
     Thm.transitive th2