src/HOL/SMT.thy
changeset 57229 489083abce44
parent 57226 c22ad39c3b4b
child 57231 dca8d06ecbba
--- a/src/HOL/SMT.thy	Thu Jun 12 01:00:49 2014 +0200
+++ b/src/HOL/SMT.thy	Thu Jun 12 01:00:49 2014 +0200
@@ -5,7 +5,7 @@
 header {* Bindings to Satisfiability Modulo Theories (SMT) solvers *}
 
 theory SMT
-imports List
+imports ATP
 keywords "smt_status" :: diag
 begin