src/HOL/Corec_Examples/Tests/Stream_Friends.thy
changeset 66453 cc19f7ca2ed6
parent 62732 bf31fd0231ba
--- a/src/HOL/Corec_Examples/Tests/Stream_Friends.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Corec_Examples/Tests/Stream_Friends.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -9,7 +9,7 @@
 section \<open>Friendly Functions on Streams\<close>
 
 theory Stream_Friends
-imports "~~/src/HOL/Library/BNF_Corec"
+imports "HOL-Library.BNF_Corec"
 begin
 
 codatatype 'a stream = SCons (shd: 'a) (stl: "'a stream")