src/Tools/eqsubst.ML
changeset 52239 6a6033fa507c
parent 52238 d84ff5a93764
child 52240 066c2ff17f7c
--- a/src/Tools/eqsubst.ML	Thu May 30 15:51:55 2013 +0200
+++ b/src/Tools/eqsubst.ML	Thu May 30 16:11:14 2013 +0200
@@ -247,7 +247,7 @@
 fun apply_subst_in_concl ctxt i st (cfvs, conclthm) rule m =
   RWInst.rw ctxt m rule conclthm
   |> IsaND.unfix_frees cfvs
-  |> RWInst.beta_eta_contract
+  |> Conv.fconv_rule Drule.beta_eta_conversion
   |> (fn r => Tactic.rtac r i st);
 
 (* substitute within the conclusion of goal i of gth, using a meta
@@ -327,7 +327,7 @@
       |> (Seq.hd o prune_params_tac)
       |> Thm.permute_prems 0 ~1 (* put old asm first *)
       |> IsaND.unfix_frees cfvs (* unfix any global params *)
-      |> RWInst.beta_eta_contract; (* normal form *)
+      |> Conv.fconv_rule Drule.beta_eta_conversion; (* normal form *)
   in
     (* ~j because new asm starts at back, thus we subtract 1 *)
     Seq.map (Thm.rotate_rule (~ j) (Thm.nprems_of rule + i))