MetaSimplifier.SIMPLIFIER;
authorwenzelm
Fri, 02 Jan 2009 11:31:40 +0100
changeset 29306 2c764235e041
parent 29305 76af2a3c9d28
child 29307 3a0b38b7fbb4
child 29335 88d23c927e37
MetaSimplifier.SIMPLIFIER;
src/ZF/Tools/inductive_package.ML
--- a/src/ZF/Tools/inductive_package.ML	Fri Jan 02 11:31:07 2009 +0100
+++ b/src/ZF/Tools/inductive_package.ML	Fri Jan 02 11:31:40 2009 +0100
@@ -249,7 +249,7 @@
     |> ListPair.map (fn (t, tacs) =>
       Goal.prove_global thy1 [] [] t
         (fn _ => EVERY (rewrite_goals_tac part_rec_defs :: tacs)))
-    handle Simplifier.SIMPLIFIER (msg, thm) => (Display.print_thm thm; error msg);
+    handle MetaSimplifier.SIMPLIFIER (msg, thm) => (Display.print_thm thm; error msg);
 
   (********)
   val dummy = writeln "  Proving the elimination rule...";