src/HOL/BNF_Examples/Stream_Processor.thy
changeset 55076 1e73e090a514
parent 55075 b3d0a02a756d
child 55091 c43394c2e5ec
--- a/src/HOL/BNF_Examples/Stream_Processor.thy	Mon Jan 20 18:24:56 2014 +0100
+++ b/src/HOL/BNF_Examples/Stream_Processor.thy	Mon Jan 20 18:24:56 2014 +0100
@@ -9,7 +9,7 @@
 header {* Stream Processors *}
 
 theory Stream_Processor
-imports Stream "../BNF_Decl"
+imports Stream "~~/src/HOL/Library/BNF_Decl"
 begin
 
 section {* Continuous Functions on Streams *}