Fixes for new isabelle
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Thu, 06 May 2010 14:09:21 +0200
changeset 2069 2b6ba4d4e19a
parent 2068 79b733010bc5
child 2070 ff69913e2608
Fixes for new isabelle
Nominal-General/nominal_eqvt.ML
Nominal-General/nominal_permeq.ML
--- a/Nominal-General/nominal_eqvt.ML	Thu May 06 13:25:37 2010 +0200
+++ b/Nominal-General/nominal_eqvt.ML	Thu May 06 14:09:21 2010 +0200
@@ -77,7 +77,7 @@
 let
   fun split_conj names (Const ("op &", _) $ f1 $ f2) = 
       (case head_of f1 of
-         Const (name, _) => if name mem names then SOME f2 else NONE
+         Const (name, _) => if member (op =) names name then SOME f2 else NONE
        | _ => NONE)
   | split_conj _ _ = NONE;
 in
@@ -178,4 +178,4 @@
       K.thy_decl (P.xname >> equivariance);
 end;
 
-end (* structure *)
\ No newline at end of file
+end (* structure *)
--- a/Nominal-General/nominal_permeq.ML	Thu May 06 13:25:37 2010 +0200
+++ b/Nominal-General/nominal_permeq.ML	Thu May 06 14:09:21 2010 +0200
@@ -117,7 +117,7 @@
     let
       val hd = head_of trm
     in 
-      if is_Const hd andalso (fst (dest_Const hd)) mem bad_hds then ()
+      if is_Const hd andalso member (op =) bad_hds (fst (dest_Const hd)) then ()
       else (if strict_flag then error else warning) 
              ("Cannot solve equivariance for " ^ (Syntax.string_of_term ctxt trm))
     end
@@ -183,4 +183,4 @@
 fun perm_strict_simp_meth (thms, consts) ctxt = 
   SIMPLE_METHOD (HEADGOAL (eqvt_strict_tac ctxt thms consts))
 
-end; (* structure *)
\ No newline at end of file
+end; (* structure *)