src/HOL/Datatype_Examples/Koenig.thy
changeset 58607 1f90ea1b4010
parent 58309 a09ec6daaa19
child 58889 5b7a9633cfa8
--- a/src/HOL/Datatype_Examples/Koenig.thy	Tue Oct 07 10:34:24 2014 +0200
+++ b/src/HOL/Datatype_Examples/Koenig.thy	Tue Oct 07 10:48:29 2014 +0200
@@ -9,7 +9,7 @@
 header {* Koenig's Lemma *}
 
 theory Koenig
-imports TreeFI Stream
+imports TreeFI "~~/src/HOL/Library/Stream"
 begin
 
 (* infinite trees: *)