src/HOL/Datatype_Examples/Koenig.thy
changeset 66453 cc19f7ca2ed6
parent 63167 0909deb8059b
--- a/src/HOL/Datatype_Examples/Koenig.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Datatype_Examples/Koenig.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -9,7 +9,7 @@
 section \<open>Koenig's Lemma\<close>
 
 theory Koenig
-imports TreeFI "~~/src/HOL/Library/Stream"
+imports TreeFI "HOL-Library.Stream"
 begin
 
 (* infinite trees: *)