tuned imports
authorblanchet
Wed, 03 Sep 2014 00:06:26 +0200
changeset 58154 47c3c7019b97
parent 58153 ca7ea280e906
child 58155 14dda84afbb3
tuned imports
src/HOL/Main.thy
src/HOL/Num.thy
src/HOL/Option.thy
--- 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 =