accomodate simplified Thm.lift_rule;
authorwenzelm
Fri, 28 Oct 2005 22:28:03 +0200
changeset 18034 5351a1538ea5
parent 18033 ab8803126f84
child 18035 eaae44affc9e
accomodate simplified Thm.lift_rule; tuned;
src/Pure/tactic.ML
--- a/src/Pure/tactic.ML	Fri Oct 28 22:28:02 2005 +0200
+++ b/src/Pure/tactic.ML	Fri Oct 28 22:28:03 2005 +0200
@@ -253,7 +253,7 @@
     fun liftpair (cv,ct) = (cterm_fun liftvar cv, cterm_fun liftterm ct)
     val lifttvar = pairself (ctyp_fun (Logic.incr_tvar inc))
 in Drule.instantiate (map lifttvar Tinsts, map liftpair insts)
-                     (lift_rule (st,i) rule)
+                     (Thm.lift_rule (Thm.cgoal_of st i) rule)
 end;
 
 fun lift_inst_rule (st, i, sinsts, rule) = lift_inst_rule'
@@ -285,7 +285,7 @@
       (ctyp_of thy (TVar ((a, i + inc), S)),
        ctyp_of thy (Logic.incr_tvar inc T))
 in Drule.instantiate (map liftTpair Tinsts, map liftpair insts)
-                     (lift_rule (st,i) rule)
+                     (Thm.lift_rule (Thm.cgoal_of st i) rule)
 end;
 
 (*** Resolve after lifting and instantation; may refer to parameters of the
@@ -636,7 +636,7 @@
 val conj_tac = SUBGOAL (fn (Const ("all", _) $ Abs (_, _, Const ("==>", _) $
       (Const ("==>", _) $ _ $ (Const ("==>", _) $ _ $ Bound 0)) $ Bound 0), i) =>
     (fn st =>
-      compose_tac (false, Drule.incr_indexes_wrt [] [] [] [st] Drule.conj_intr_thm, 2) i st)
+      compose_tac (false, Drule.incr_indexes st Drule.conj_intr_thm, 2) i st)
   | _ => no_tac);
 
 val conjunction_tac = ALLGOALS (REPEAT_ALL_NEW conj_tac);