src/Pure/thm.ML
changeset 46217 7b19666f0e3d
parent 45443 c8a9a5e577bd
child 46218 ecf6375e2abb
--- a/src/Pure/thm.ML	Sat Jan 14 18:18:06 2012 +0100
+++ b/src/Pure/thm.ML	Sat Jan 14 19:06:05 2012 +0100
@@ -753,7 +753,7 @@
         shyps = Sorts.union sorts shyps,
         hyps = hyps,
         tpairs = tpairs,
-        prop = Term.all T $ Abs (a, T, abstract_over (x, prop))});
+        prop = Logic.all_const T $ Abs (a, T, abstract_over (x, prop))});
     fun check_occs a x ts =
       if exists (fn t => Logic.occs (x, t)) ts then
         raise THM ("forall_intr: variable " ^ quote a ^ " free in assumptions", 0, [th])
@@ -1588,7 +1588,7 @@
         val T' = Envir.subst_type (Envir.type_env env) T
         (*Must instantiate types of parameters because they are flattened;
           this could be a NEW parameter*)
-      in Term.all T' $ Abs (a, T', norm_term_skip env n t) end
+      in Logic.all_const T' $ Abs (a, T', norm_term_skip env n t) end
   | norm_term_skip env n (Const ("==>", _) $ A $ B) =
       Logic.mk_implies (A, norm_term_skip env (n - 1) B)
   | norm_term_skip _ _ _ = error "norm_term_skip: too few assumptions??";