src/HOL/Library/State_Monad.thy
changeset 25595 6c48275f9c76
parent 24253 3d7f74fd9fd9
child 25765 49580bd58a21
--- a/src/HOL/Library/State_Monad.thy	Mon Dec 10 11:24:09 2007 +0100
+++ b/src/HOL/Library/State_Monad.thy	Mon Dec 10 11:24:12 2007 +0100
@@ -6,7 +6,7 @@
 header {* Combinators syntax for generic, open state monads (single threaded monads) *}
 
 theory State_Monad
-imports Main
+imports List
 begin
 
 subsection {* Motivation *}