src/HOL/Tools/Datatype/datatype.ML
changeset 32671 fbd224850767
parent 32374 62617ef2c0d0
child 32712 ec5976f4d3d8
--- a/src/HOL/Tools/Datatype/datatype.ML	Wed Sep 23 16:20:12 2009 +0200
+++ b/src/HOL/Tools/Datatype/datatype.ML	Wed Sep 23 16:20:12 2009 +0200
@@ -26,7 +26,7 @@
   val info_of_case : theory -> string -> info option
   val interpretation : (config -> string list -> theory -> theory) -> theory -> theory
   val distinct_simproc : simproc
-  val make_case :  Proof.context -> bool -> string list -> term ->
+  val make_case :  Proof.context -> DatatypeCase.config -> string list -> term ->
     (term * term) list -> term * (term * (int * bool)) list
   val strip_case : Proof.context -> bool -> term -> (term * (term * term) list) option
   val read_typ: theory ->