src/HOL/Fun.thy
changeset 61955 e96292f32c3c
parent 61799 4cf66f21b764
child 62390 842917225d56
--- a/src/HOL/Fun.thy	Mon Dec 28 19:23:15 2015 +0100
+++ b/src/HOL/Fun.thy	Mon Dec 28 21:47:32 2015 +0100
@@ -42,11 +42,11 @@
 
 subsection \<open>The Composition Operator \<open>f \<circ> g\<close>\<close>
 
-definition comp :: "('b \<Rightarrow> 'c) \<Rightarrow> ('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'c" (infixl "o" 55) where
-  "f o g = (\<lambda>x. f (g x))"
+definition comp :: "('b \<Rightarrow> 'c) \<Rightarrow> ('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'c"  (infixl "\<circ>" 55)
+  where "f \<circ> g = (\<lambda>x. f (g x))"
 
-notation (xsymbols)
-  comp  (infixl "\<circ>" 55)
+notation (ASCII)
+  comp  (infixl "o" 55)
 
 lemma comp_apply [simp]: "(f o g) x = f (g x)"
   by (simp add: comp_def)