diff -r 0a28cf866d5d -r dc59f147b27d src/HOL/BNF_Examples/Stream_Processor.thy --- 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 ("\(_,/ _)\") definition \ :: "('p,'a) F * 'b \ ('p,'a * 'b) F" where - "\ xb = F id a. (snd xb)> (fst xb)" + "\ xb = F id \id, \ a. (snd xb)\ (fst xb)" (* The strength laws for \: *) lemma \_natural: "F id (map_prod f g) o \ = \ o map_prod (F id f) g"