--- a/src/HOL/Main.thy Wed Sep 03 00:06:25 2014 +0200
+++ b/src/HOL/Main.thy Wed Sep 03 00:06:26 2014 +0200
@@ -2,7 +2,7 @@
theory Main
imports Predicate_Compile Quickcheck_Narrowing Extraction Lifting_Sum Coinduction Nitpick
- BNF_Greatest_Fixpoint
+ BNF_Greatest_Fixpoint Old_Datatype
begin
text {*
--- a/src/HOL/Num.thy Wed Sep 03 00:06:25 2014 +0200
+++ b/src/HOL/Num.thy Wed Sep 03 00:06:26 2014 +0200
@@ -6,7 +6,7 @@
header {* Binary Numerals *}
theory Num
-imports BNF_Least_Fixpoint Old_Datatype
+imports BNF_Least_Fixpoint
begin
subsection {* The @{text num} type *}
--- a/src/HOL/Option.thy Wed Sep 03 00:06:25 2014 +0200
+++ b/src/HOL/Option.thy Wed Sep 03 00:06:26 2014 +0200
@@ -5,7 +5,7 @@
header {* Datatype option *}
theory Option
-imports BNF_Least_Fixpoint Old_Datatype Finite_Set
+imports BNF_Least_Fixpoint Finite_Set
begin
datatype_new 'a option =