tuned assoc;
authorwenzelm
Fri, 15 Jul 2005 15:44:21 +0200
changeset 16866 cde0b6864924
parent 16865 fb39dcfc1c24
child 16867 cf7d61d56acf
tuned assoc;
src/Pure/Proof/proof_syntax.ML
--- a/src/Pure/Proof/proof_syntax.ML	Fri Jul 15 15:44:20 2005 +0200
+++ b/src/Pure/Proof/proof_syntax.ML	Fri Jul 15 15:44:21 2005 +0200
@@ -92,10 +92,10 @@
 fun disambiguate_names thy prf =
   let
     val thms = thms_of_proof Symtab.empty prf;
-    val thms' = map (apsnd (#prop o rep_thm)) (PureThy.all_thms_of thy);
+    val thms' = map (apsnd Thm.full_prop_of) (PureThy.all_thms_of thy);
 
     val tab = Symtab.foldl (fn (tab, (key, ps)) =>
-      let val prop = getOpt (assoc (thms', key), Bound 0)
+      let val prop = getOpt (assoc_string (thms', key), Bound 0)
       in fst (foldr (fn ((prop', prf), x as (tab, i)) =>
         if prop <> prop' then
           (Symtab.update ((key ^ "_" ^ string_of_int i, prf), tab), i+1)
@@ -108,7 +108,7 @@
       | rename (prf % t) = rename prf % t
       | rename (prf' as PThm ((s, tags), prf, prop, Ts)) =
           let
-            val prop' = getOpt (assoc (thms', s), Bound 0);
+            val prop' = getOpt (assoc_string (thms', s), Bound 0);
             val ps = map fst (valOf (Symtab.lookup (thms, s))) \ prop'
           in if prop = prop' then prf' else
             PThm ((s ^ "_" ^ string_of_int (length ps - find_index_eq prop ps), tags),
@@ -136,13 +136,13 @@
                "axm" :: xs =>
                  let
                    val name = NameSpace.pack xs;
-                   val prop = (case assoc (axms, name) of
+                   val prop = (case assoc_string (axms, name) of
                        SOME prop => prop
                      | NONE => error ("Unknown axiom " ^ quote name))
                  in PAxm (name, prop, NONE) end
              | "thm" :: xs =>
                  let val name = NameSpace.pack xs;
-                 in (case assoc (thms, name) of
+                 in (case assoc_string (thms, name) of
                      SOME thm => fst (strip_combt (Thm.proof_of thm))
                    | NONE => (case Symtab.lookup (tab, name) of
                          SOME prf => prf