src/HOL/BNF_Examples/Compat.thy
changeset 58112 8081087096ad
parent 57634 efc00b9b8680
child 58124 c60617a84c1d
--- a/src/HOL/BNF_Examples/Compat.thy	Mon Sep 01 16:17:46 2014 +0200
+++ b/src/HOL/BNF_Examples/Compat.thy	Mon Sep 01 16:17:46 2014 +0200
@@ -80,6 +80,6 @@
 datatype_new tree = Tree "tree foo"
 datatype_compat tree
 
-ML {* Datatype_Data.get_info @{theory} @{type_name tree} *}
+ML {* Old_Datatype_Data.get_info @{theory} @{type_name tree} *}
 
 end