src/HOL/Code_Evaluation.thy
changeset 50055 94041d602ecb
parent 48891 c0eafbd55de3
child 51112 da97167e03f7
--- a/src/HOL/Code_Evaluation.thy	Mon Nov 12 18:42:49 2012 +0100
+++ b/src/HOL/Code_Evaluation.thy	Mon Nov 12 23:24:40 2012 +0100
@@ -5,7 +5,7 @@
 header {* Term evaluation using the generic code generator *}
 
 theory Code_Evaluation
-imports Plain Typerep Code_Numeral Predicate
+imports Plain Typerep New_DSequence
 begin
 
 subsection {* Term representation *}