src/HOL/ex/CodeEval.thy
changeset 21924 fe474e69e603
parent 21836 b2cbcf8a018e
child 22005 0faa5afd5d69
--- a/src/HOL/ex/CodeEval.thy	Fri Dec 29 03:57:01 2006 +0100
+++ b/src/HOL/ex/CodeEval.thy	Fri Dec 29 12:11:00 2006 +0100
@@ -40,9 +40,8 @@
   fun mk arities _ thy =
     (maps (fn ((tyco, asorts), _) => [(("", []), TypOf.mk_typ_of_def
       (Type (tyco, map TFree (Name.names Name.context "'a" asorts))))]) arities, thy);
-  fun tac _ = ClassPackage.intro_classes_tac [];
   fun hook specs =
-    DatatypeCodegen.prove_codetypes_arities tac
+    DatatypeCodegen.prove_codetypes_arities (ClassPackage.intro_classes_tac [])
       (map (fn (tyco, (is_dt, _)) => (tyco, is_dt)) specs)
       [TypOf.class_typ_of] mk ((K o K) I)
 in DatatypeCodegen.add_codetypes_hook_bootstrap hook end
@@ -101,11 +100,10 @@
       |> PrimrecPackage.gen_primrec thy_note thy_def "" defs'
       |> snd
     end;
-  fun tac _ = ClassPackage.intro_classes_tac [];
   fun hook specs =
     if (fst o hd) specs = (fst o dest_Type) Embed.typ_typ then I
     else
-      DatatypeCodegen.prove_codetypes_arities tac
+      DatatypeCodegen.prove_codetypes_arities (ClassPackage.intro_classes_tac [])
       (map (fn (tyco, (is_dt, _)) => (tyco, is_dt)) specs)
       [TermOf.class_term_of] ((K o K o pair) []) mk
 in DatatypeCodegen.add_codetypes_hook_bootstrap hook end