src/HOL/Decision_Procs/Approximation.thy
changeset 41413 64cd30d6b0b8
parent 41024 ba961a606c67
child 42361 23f352990944
--- a/src/HOL/Decision_Procs/Approximation.thy	Wed Dec 29 13:51:17 2010 +0100
+++ b/src/HOL/Decision_Procs/Approximation.thy	Wed Dec 29 17:34:41 2010 +0100
@@ -4,7 +4,12 @@
 header {* Prove Real Valued Inequalities by Computation *}
 
 theory Approximation
-imports Complex_Main Float Reflection "~~/src/HOL/Decision_Procs/Dense_Linear_Order" Efficient_Nat
+imports
+  Complex_Main
+  "~~/src/HOL/Library/Float"
+  "~~/src/HOL/Library/Reflection"
+  "~~/src/HOL/Decision_Procs/Dense_Linear_Order"
+  "~~/src/HOL/Library/Efficient_Nat"
 begin
 
 section "Horner Scheme"