src/Pure/meta_simplifier.ML
changeset 28839 32d498cf7595
parent 28620 9846d772b306
child 29269 5c25a2012975
--- a/src/Pure/meta_simplifier.ML	Tue Nov 18 18:25:10 2008 +0100
+++ b/src/Pure/meta_simplifier.ML	Tue Nov 18 18:25:42 2008 +0100
@@ -79,12 +79,10 @@
   val rewrite_rule: thm list -> thm -> thm
   val rewrite_goals_rule: thm list -> thm -> thm
   val rewrite_goals_tac: thm list -> tactic
-  val rewrite_tac: thm list -> tactic
   val rewrite_goal_tac: thm list -> int -> tactic
   val rewtac: thm -> tactic
   val prune_params_tac: tactic
   val fold_rule: thm list -> thm -> thm
-  val fold_tac: thm list -> tactic
   val fold_goals_tac: thm list -> tactic
 end;
 
@@ -1285,14 +1283,11 @@
 
 (** meta-rewriting tactics **)
 
-(*Rewrite throughout proof state. *)
-fun rewrite_tac defs = PRIMITIVE (rewrite_rule defs);
-
-(*Rewrite subgoals only, not main goal. *)
+(*Rewrite all subgoals*)
 fun rewrite_goals_tac defs = PRIMITIVE (rewrite_goals_rule defs);
 fun rewtac def = rewrite_goals_tac [def];
 
-(*Rewrite subgoal i only.*)
+(*Rewrite one subgoal*)
 fun asm_rewrite_goal_tac mode prover_tac ss i thm =
   if 0 < i andalso i <= Thm.nprems_of thm then
     Seq.single (Conv.gconv_rule (rewrite_cterm mode (SINGLE o prover_tac) ss) i thm)
@@ -1329,7 +1324,6 @@
 val rev_defs = sort_lhs_depths o map symmetric;
 
 fun fold_rule defs = fold rewrite_rule (rev_defs defs);
-fun fold_tac defs = EVERY (map rewrite_tac (rev_defs defs));
 fun fold_goals_tac defs = EVERY (map rewrite_goals_tac (rev_defs defs));