test: use SkipProof.make_thm instead of Thm.assume;
authorwenzelm
Fri, 12 Oct 2001 12:06:54 +0200
changeset 11727 a27150cc8fa5
parent 11726 2b2a45abe876
child 11728 b5f6963b193c
test: use SkipProof.make_thm instead of Thm.assume;
src/HOL/Tools/typedef_package.ML
--- a/src/HOL/Tools/typedef_package.ML	Fri Oct 12 12:06:23 2001 +0200
+++ b/src/HOL/Tools/typedef_package.ML	Fri Oct 12 12:06:54 2001 +0200
@@ -147,9 +147,9 @@
       |> (if no_def then I else (#1 oo (PureThy.add_defs_i false o map Thm.no_attributes))
        [Logic.mk_defpair (setC, set)])
       |> PureThy.add_axioms_i [((typedef_name, typedef_prop),
-          [apsnd (fn cond_axm => standard (nonempty RS cond_axm))])]
+          [apsnd (fn cond_axm => Drule.standard (nonempty RS cond_axm))])]
       |> (fn (theory', axm) =>
-        let fun make th = standard (th OF axm) in
+        let fun make th = Drule.standard (th OF axm) in
           rpair (hd axm) (theory'
           |> (#1 oo PureThy.add_thms)
             ([((Rep_name, make Rep), []),
@@ -193,8 +193,8 @@
 
     (*test theory errors now!*)
     val test_thy = Theory.copy thy;
-    val test_sign = Theory.sign_of test_thy;
-    val _ = (test_thy, Thm.assume (Thm.cterm_of test_sign goal)) |> typedef_att;
+    val _ = (test_thy,
+      setmp quick_and_dirty true (SkipProof.make_thm test_thy) goal) |> typedef_att;
 
   in (cset, goal, goal_pat, typedef_att) end
   handle ERROR => err_in_typedef name;