src/HOL/Nominal/nominal_inductive2.ML
changeset 36692 54b64d4ad524
parent 36428 874843c1e96e
child 36960 01594f816e3a
--- a/src/HOL/Nominal/nominal_inductive2.ML	Wed May 05 09:24:42 2010 +0200
+++ b/src/HOL/Nominal/nominal_inductive2.ML	Wed May 05 18:25:34 2010 +0200
@@ -46,7 +46,7 @@
 fun mk_perm_bool_simproc names = Simplifier.simproc_i
   (theory_of_thm perm_bool) "perm_bool" [@{term "perm pi x"}] (fn thy => fn ss =>
     fn Const ("Nominal.perm", _) $ _ $ t =>
-         if the_default "" (try (head_of #> dest_Const #> fst) t) mem names
+         if member (op =) names (the_default "" (try (head_of #> dest_Const #> fst) t))
          then SOME perm_bool else NONE
      | _ => NONE);
 
@@ -77,7 +77,7 @@
 
 fun split_conj f names (Const ("op &", _) $ p $ q) _ = (case head_of p of
       Const (name, _) =>
-        if name mem names then SOME (f p q) else NONE
+        if member (op =) names name then SOME (f p q) else NONE
     | _ => NONE)
   | split_conj _ _ _ _ = NONE;
 
@@ -96,7 +96,7 @@
 fun inst_conj_all names ps pis (Const ("op &", _) $ p $ q) _ =
       (case head_of p of
          Const (name, _) =>
-           if name mem names then SOME (HOLogic.mk_conj (p,
+           if member (op =) names name then SOME (HOLogic.mk_conj (p,
              Const ("Fun.id", HOLogic.boolT --> HOLogic.boolT) $
                (subst_bounds (pis, strip_all pis q))))
            else NONE
@@ -239,7 +239,7 @@
     fun lift_prem (t as (f $ u)) =
           let val (p, ts) = strip_comb t
           in
-            if p mem ps then
+            if member (op =) ps p then
               Const (inductive_forall_name,
                 (fsT --> HOLogic.boolT) --> HOLogic.boolT) $
                   Abs ("z", fsT, lift_pred p (map (incr_boundvars 1) ts))