src/HOL/SMT.thy
changeset 57226 c22ad39c3b4b
parent 57213 9daec42f6784
child 57229 489083abce44
--- 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 Record
+imports List
 keywords "smt_status" :: diag
 begin