src/HOL/BNF_Examples/Stream_Processor.thy
changeset 57641 dc59f147b27d
parent 57634 efc00b9b8680
--- a/src/HOL/BNF_Examples/Stream_Processor.thy	Thu Jul 24 11:51:22 2014 +0200
+++ b/src/HOL/BNF_Examples/Stream_Processor.thy	Thu Jul 24 11:54:15 2014 +0200
@@ -152,10 +152,10 @@
 
 bnf_axiomatization ('a, 'b) F for map: F
 
-notation BNF_Def.convol ("<_ , _>")
+notation BNF_Def.convol ("\<langle>(_,/ _)\<rangle>")
 
 definition \<theta> :: "('p,'a) F * 'b \<Rightarrow> ('p,'a * 'b) F" where
-  "\<theta> xb = F id <id, \<lambda> a. (snd xb)> (fst xb)"
+  "\<theta> xb = F id \<langle>id, \<lambda> a. (snd xb)\<rangle> (fst xb)"
 
 (* The strength laws for \<theta>: *)
 lemma \<theta>_natural: "F id (map_prod f g) o \<theta> = \<theta> o map_prod (F id f) g"