src/HOL/Tools/SMT2/z3_new_proof.ML
changeset 56245 84fc7dfa3cd4
parent 56122 40f7b45b2472
child 56811 b66639331db5
--- a/src/HOL/Tools/SMT2/z3_new_proof.ML	Fri Mar 21 15:12:03 2014 +0100
+++ b/src/HOL/Tools/SMT2/z3_new_proof.ML	Fri Mar 21 20:33:56 2014 +0100
@@ -463,7 +463,7 @@
     val match = Sign.typ_match (Proof_Context.theory_of ctxt)
 
     val t' = singleton (Variable.polymorphic ctxt) t
-    val patTs = map snd (Term.strip_qnt_vars @{const_name all} t')
+    val patTs = map snd (Term.strip_qnt_vars @{const_name Pure.all} t')
     val objTs = map (the o Symtab.lookup env) bounds
     val subst = subst_of (fold match (patTs ~~ objTs) Vartab.empty)
   in Same.commit (Term_Subst.map_types_same (substTs_same subst)) t' end
@@ -501,7 +501,7 @@
     SOME (tyenv, _) => subst_of tyenv
   | NONE => strip_match ctxt pat (i + 1) (dest_quant i obj))
 
-fun dest_all i (Const (@{const_name all}, _) $ (a as Abs (_, T, _))) =
+fun dest_all i (Const (@{const_name Pure.all}, _) $ (a as Abs (_, T, _))) =
       dest_all (i + 1) (Term.betapply (a, Var (("", i), T)))
   | dest_all i t = (i, t)
 
@@ -517,7 +517,7 @@
     | SOME subst =>
         let
           val applyT = Same.commit (substTs_same subst)
-          val patTs = map snd (Term.strip_qnt_vars @{const_name all} t'')
+          val patTs = map snd (Term.strip_qnt_vars @{const_name Pure.all} t'')
         in SOME (Symtab.make (bs' ~~ map applyT patTs)) end)
   end