src/HOL/Library/Eval.thy
changeset 25691 8f8d83af100a
parent 25666 f46ed5b333fd
child 25763 474f8ba9dfa9
--- a/src/HOL/Library/Eval.thy	Tue Dec 18 12:26:24 2007 +0100
+++ b/src/HOL/Library/Eval.thy	Tue Dec 18 14:37:00 2007 +0100
@@ -6,7 +6,7 @@
 header {* A simple term evaluation mechanism *}
 
 theory Eval
-imports PreList Pure_term
+imports ATP_Linkup Pure_term
 begin
 
 subsection {* @{text typ_of} class *}