src/HOL/Corec_Examples/Stream_Processor.thy
changeset 62726 5b2a7caa855b
parent 62698 9d706e37ddab
child 66453 cc19f7ca2ed6
--- a/src/HOL/Corec_Examples/Stream_Processor.thy	Mon Mar 28 12:05:47 2016 +0200
+++ b/src/HOL/Corec_Examples/Stream_Processor.thy	Mon Mar 28 12:05:47 2016 +0200
@@ -7,7 +7,7 @@
 Stream processors---a syntactic representation of continuous functions on streams.
 *)
 
-section {* Stream Processors---A Syntactic Representation of Continuous Functions on Streams *}
+section \<open>Stream Processors---A Syntactic Representation of Continuous Functions on Streams\<close>
 
 theory Stream_Processor
 imports "~~/src/HOL/Library/BNF_Corec" "~~/src/HOL/Library/Stream"