src/Pure/Isar/locale.ML
changeset 21708 45e7491bea47
parent 21701 627c90b310c1
child 21962 279b129498b6
--- a/src/Pure/Isar/locale.ML	Thu Dec 07 21:44:13 2006 +0100
+++ b/src/Pure/Isar/locale.ML	Thu Dec 07 23:16:55 2006 +0100
@@ -1648,17 +1648,17 @@
     val cert = Thm.cterm_of defs_thy;
 
     val intro = Goal.prove_global defs_thy [] norm_ts statement (fn _ =>
-      Tactic.rewrite_goals_tac [pred_def] THEN
+      MetaSimplifier.rewrite_goals_tac [pred_def] THEN
       Tactic.compose_tac (false, body_eq RS Drule.equal_elim_rule1, 1) 1 THEN
       Tactic.compose_tac (false, Conjunction.intr_list (map (Thm.assume o cert) norm_ts), 0) 1);
 
     val conjuncts =
       (Drule.equal_elim_rule2 OF [body_eq,
-        Tactic.rewrite_rule [pred_def] (Thm.assume (cert statement))])
+        MetaSimplifier.rewrite_rule [pred_def] (Thm.assume (cert statement))])
       |> Conjunction.elim_precise [length ts] |> hd;
     val axioms = ts ~~ conjuncts |> map (fn (t, ax) =>
       Element.prove_witness defs_ctxt t
-       (Tactic.rewrite_goals_tac defs THEN
+       (MetaSimplifier.rewrite_goals_tac defs THEN
         Tactic.compose_tac (false, ax, 0) 1));
   in ((statement, intro, axioms), defs_thy) end;