src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML
changeset 36692 54b64d4ad524
parent 36556 81dc2c20f052
child 36966 adc11fb3f3aa
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML	Wed May 05 09:24:42 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML	Wed May 05 18:25:34 2010 +0200
@@ -410,7 +410,7 @@
   | arity_clause dfg seen n (tcons, ("HOL.type",_)::ars) =  (*ignore*)
       arity_clause dfg seen n (tcons,ars)
   | arity_clause dfg seen n (tcons, (ar as (class,_)) :: ars) =
-      if class mem_string seen then (*multiple arities for the same tycon, class pair*)
+      if member (op =) seen class then (*multiple arities for the same tycon, class pair*)
           make_axiom_arity_clause dfg (tcons, lookup_type_const dfg tcons ^ "_" ^ class ^ "_" ^ Int.toString n, ar) ::
           arity_clause dfg seen (n+1) (tcons,ars)
       else