src/HOL/Inductive.thy
changeset 31784 bd3486c57ba3
parent 31775 2b04504fcb69
child 31949 3f933687fae9
--- a/src/HOL/Inductive.thy	Tue Jun 23 15:32:34 2009 +0200
+++ b/src/HOL/Inductive.thy	Tue Jun 23 16:27:12 2009 +0200
@@ -364,7 +364,7 @@
   fun fun_tr ctxt [cs] =
     let
       val x = Free (Name.variant (Term.add_free_names cs []) "x", dummyT);
-      val ft = DatatypeCase.case_tr true Datatype.datatype_of_constr
+      val ft = DatatypeCase.case_tr true Datatype.info_of_constr
                  ctxt [x, cs]
     in lambda x ft end
 in [("_lam_pats_syntax", fun_tr)] end