src/HOL/Library/Open_State_Syntax.thy
changeset 67399 eab6ce8368fa
parent 66270 403d84138c5c
child 68224 1f7308050349
--- a/src/HOL/Library/Open_State_Syntax.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Library/Open_State_Syntax.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -60,12 +60,12 @@
 
 text \<open>
   Given two transformations @{term f} and @{term g}, they may be
-  directly composed using the @{term "op \<circ>>"} combinator, forming a
+  directly composed using the @{term "(\<circ>>)"} combinator, forming a
   forward composition: @{prop "(f \<circ>> g) s = f (g s)"}.
 
   After any yielding transformation, we bind the side result
   immediately using a lambda abstraction.  This is the purpose of the
-  @{term "op \<circ>\<rightarrow>"} combinator: @{prop "(f \<circ>\<rightarrow> (\<lambda>x. g)) s = (let (x, s')
+  @{term "(\<circ>\<rightarrow>)"} combinator: @{prop "(f \<circ>\<rightarrow> (\<lambda>x. g)) s = (let (x, s')
   = f s in g s')"}.
 
   For queries, the existing @{term "Let"} is appropriate.