src/HOL/Tools/Quickcheck/quickcheck_common.ML
changeset 58186 a6c3962ea907
parent 58145 3cfbb68ad2e0
child 58354 04ac60da613e
--- a/src/HOL/Tools/Quickcheck/quickcheck_common.ML	Fri Sep 05 00:41:00 2014 +0200
+++ b/src/HOL/Tools/Quickcheck/quickcheck_common.ML	Fri Sep 05 00:41:01 2014 +0200
@@ -32,7 +32,7 @@
     -> Old_Datatype_Aux.config -> string list -> theory -> theory
   val ensure_common_sort_datatype :
     (sort * instantiation) -> Old_Datatype_Aux.config -> string list -> theory -> theory
-  val datatype_interpretation : (sort * instantiation) -> theory -> theory
+  val datatype_interpretation : string -> sort * instantiation -> theory -> theory
   val gen_mk_parametric_generator_expr :
    (((Proof.context -> term * term list -> term) * term) * typ)
      -> Proof.context -> (term * term list) list -> term
@@ -422,8 +422,8 @@
   ensure_sort (((@{sort typerep}, @{sort term_of}), sort),
     (fn thy => BNF_LFP_Compat.the_descr thy BNF_LFP_Compat.Keep_Nesting, instantiate))
 
-val datatype_interpretation =
-  BNF_LFP_Compat.interpretation BNF_LFP_Compat.Keep_Nesting o ensure_common_sort_datatype
+fun datatype_interpretation name =
+  BNF_LFP_Compat.interpretation name BNF_LFP_Compat.Keep_Nesting o ensure_common_sort_datatype
   
 (** generic parametric compilation **)