src/HOL/Import/shuffler.ML
changeset 35845 e5980f0ad025
parent 35408 b48ab741683b
child 36543 0e7fc5bf38de
--- a/src/HOL/Import/shuffler.ML	Sat Mar 20 02:23:41 2010 +0100
+++ b/src/HOL/Import/shuffler.ML	Sat Mar 20 17:33:11 2010 +0100
@@ -265,7 +265,7 @@
     let
         val cU = ctyp_of thy U
         val tfrees = OldTerm.add_term_tfrees (prop_of thm,[])
-        val (rens, thm') = Thm.varifyT'
+        val (rens, thm') = Thm.varifyT_global'
     (remove (op = o apsnd fst) name tfrees) thm
         val mid =
             case rens of
@@ -592,7 +592,7 @@
         fun process [] = NONE
           | process ((name,th)::thms) =
             let
-                val norm_th = Thm.varifyT (norm_thm thy (close_thm (Thm.transfer thy th)))
+                val norm_th = Thm.varifyT_global (norm_thm thy (close_thm (Thm.transfer thy th)))
                 val triv_th = trivial rhs
                 val _ = message ("Shuffler.set_prop: Gluing together " ^ (string_of_thm norm_th) ^ " and " ^ (string_of_thm triv_th))
                 val mod_th = case Seq.pull (Thm.bicompose false (*true*) (false,norm_th,0) 1 triv_th) of