src/Pure/raw_simplifier.ML
changeset 46460 68cf3d3550b5
parent 46186 9ae331a1d8c5
child 46462 9b3f6767d175
--- a/src/Pure/raw_simplifier.ML	Tue Feb 14 17:11:33 2012 +0100
+++ b/src/Pure/raw_simplifier.ML	Tue Feb 14 17:26:35 2012 +0100
@@ -55,7 +55,6 @@
   val rewrite_goals_rule: thm list -> thm -> thm
   val rewrite_goals_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_goals_tac: thm list -> tactic
@@ -1305,7 +1304,6 @@
 
 (*Rewrite all subgoals*)
 fun rewrite_goals_tac defs = PRIMITIVE (rewrite_goals_rule defs);
-fun rewtac def = rewrite_goals_tac [def];
 
 (*Rewrite one subgoal*)
 fun asm_rewrite_goal_tac mode prover_tac ss i thm =