moved Drule.unvarify to Thm.unvarify (cf. more_thm.ML);
authorwenzelm
Thu, 11 Oct 2007 19:10:17 +0200
changeset 24976 821628d16552
parent 24975 592a5d8700a7
child 24977 9f98751c9628
moved Drule.unvarify to Thm.unvarify (cf. more_thm.ML);
src/HOL/Import/proof_kernel.ML
src/HOL/Tools/datatype_codegen.ML
src/Pure/conjunction.ML
src/Tools/code/code_package.ML
--- a/src/HOL/Import/proof_kernel.ML	Thu Oct 11 18:58:34 2007 +0200
+++ b/src/HOL/Import/proof_kernel.ML	Thu Oct 11 19:10:17 2007 +0200
@@ -2030,7 +2030,7 @@
 				 names'
 				 (thy1,th)
 	    val _ = ImportRecorder.add_specification names' th
-	    val res' = Drule.unvarify res
+	    val res' = Thm.unvarify res
 	    val hth = HOLThm(rens,res')
 	    val rew = rewrite_hol4_term (concl_of res') thy'
 	    val th  = equal_elim rew res'
--- a/src/HOL/Tools/datatype_codegen.ML	Thu Oct 11 18:58:34 2007 +0200
+++ b/src/HOL/Tools/datatype_codegen.ML	Thu Oct 11 19:10:17 2007 +0200
@@ -411,7 +411,7 @@
       (#case_rewrites o DatatypePackage.the_datatype thy) tyco;
     val thms as hd_thm :: _ = raw_thms
       |> Conjunction.intr_balanced
-      |> Drule.unvarify
+      |> Thm.unvarify
       |> Conjunction.elim_balanced (length raw_thms)
       |> map Simpdata.mk_meta_eq
       |> map Drule.zero_var_indexes
--- a/src/Pure/conjunction.ML	Thu Oct 11 18:58:34 2007 +0200
+++ b/src/Pure/conjunction.ML	Thu Oct 11 19:10:17 2007 +0200
@@ -69,7 +69,7 @@
 val ABC = read_prop "A ==> B ==> C";
 val A_B = read_prop "A && B";
 
-val conjunction_def = Drule.unvarify ProtoPure.conjunction_def;
+val conjunction_def = Thm.unvarify ProtoPure.conjunction_def;
 
 fun conjunctionD which =
   Drule.implies_intr_list [A, B] (Thm.assume (which (A, B))) COMP
--- a/src/Tools/code/code_package.ML	Thu Oct 11 18:58:34 2007 +0200
+++ b/src/Tools/code/code_package.ML	Thu Oct 11 19:10:17 2007 +0200
@@ -157,7 +157,7 @@
 
 fun mk_codeprops thy all_cs sel_cs =
   let
-    fun select (thmref, thm) = case try (Drule.unvarify o Drule.zero_var_indexes) thm
+    fun select (thmref, thm) = case try (Thm.unvarify o Drule.zero_var_indexes) thm
      of NONE => NONE
       | SOME thm => let
           val t = (ObjectLogic.drop_judgment thy o Thm.prop_of) thm;