src/HOL/Library/Sum_of_Squares/sum_of_squares.ML
changeset 46497 89ccf66aa73d
parent 44469 266dfd7f4e82
child 47108 2a1953f0d20d
--- a/src/HOL/Library/Sum_of_Squares/sum_of_squares.ML	Wed Feb 15 22:44:31 2012 +0100
+++ b/src/HOL/Library/Sum_of_Squares/sum_of_squares.ML	Wed Feb 15 23:19:30 2012 +0100
@@ -772,7 +772,7 @@
   (* FIXME : This is very bad!!!*)
 fun subst_conv eqs t =
  let
-  val t' = fold (Thm.cabs o Thm.lhs_of) eqs t
+  val t' = fold (Thm.lambda o Thm.lhs_of) eqs t
  in Conv.fconv_rule (Thm.beta_conversion true) (fold (C Thm.combination) eqs (Thm.reflexive t'))
  end
 
@@ -819,7 +819,7 @@
   fun make_substitution th =
    let
     val (c,v) = substitutable_monomial [] (Thm.dest_arg1(concl th))
-    val th1 = Drule.arg_cong_rule (Thm.capply @{cterm "op * :: real => _"} (RealArith.cterm_of_rat (Rat.inv c))) (mk_meta_eq th)
+    val th1 = Drule.arg_cong_rule (Thm.apply @{cterm "op * :: real => _"} (RealArith.cterm_of_rat (Rat.inv c))) (mk_meta_eq th)
     val th2 = fconv_rule (binop_conv real_poly_mul_conv) th1
    in fconv_rule (arg_conv real_poly_conv) (isolate_variable v th2)
    end