src/HOL/Multivariate_Analysis/normarith.ML
changeset 43333 2bdec7f430d3
parent 42793 88bee9f6eec7
child 44454 6f28f96a09bf
--- a/src/HOL/Multivariate_Analysis/normarith.ML	Thu Jun 09 22:25:25 2011 +0200
+++ b/src/HOL/Multivariate_Analysis/normarith.ML	Thu Jun 09 23:12:02 2011 +0200
@@ -306,7 +306,7 @@
         (fn t => null (FuncUtil.Ctermfunc.dom (vector_lincomb t))) (map snd rawdests)
 
   in fst (RealArith.real_linear_prover translator
-        (map (fn t => instantiate ([(tv_n, ctyp_of_term t)],[]) pth_zero)
+        (map (fn t => Drule.instantiate_normalize ([(tv_n, ctyp_of_term t)],[]) pth_zero)
             zerodests,
         map (fconv_rule (try_conv (Conv.top_sweep_conv (K norm_canon_conv) ctxt) then_conv
                        arg_conv (arg_conv real_poly_conv))) ges',
@@ -343,7 +343,7 @@
   val shs = filter (member (fn (t,th) => t aconvc cprop_of th) asl) (#hyps (crep_thm th1))
   val th11 = hd (Variable.export ctxt' ctxt [fold Thm.implies_intr shs th1])
   val cps = map (swap o Thm.dest_equals) (cprems_of th11)
-  val th12 = instantiate ([], cps) th11
+  val th12 = Drule.instantiate_normalize ([], cps) th11
   val th13 = fold Thm.elim_implies (map (Thm.reflexive o snd) cps) th12;
  in hd (Variable.export ctxt' ctxt [th13])
  end