src/HOL/Fun.thy
changeset 26588 d83271bfaba5
parent 26357 19b153ebda0b
child 27106 ff27dc6e7d05
--- a/src/HOL/Fun.thy	Wed Apr 09 08:10:09 2008 +0200
+++ b/src/HOL/Fun.thy	Wed Apr 09 08:10:11 2008 +0200
@@ -82,19 +82,13 @@
 by (unfold comp_def, blast)
 
 
-subsection {* The Forward Composition Operator @{text "f \<circ>> g"} *}
+subsection {* The Forward Composition Operator @{text fcomp} *}
 
 definition
   fcomp :: "('a \<Rightarrow> 'b) \<Rightarrow> ('b \<Rightarrow> 'c) \<Rightarrow> 'a \<Rightarrow> 'c" (infixl "o>" 60)
 where
   "f o> g = (\<lambda>x. g (f x))"
 
-notation (xsymbols)
-  fcomp  (infixl "\<circ>>" 60)
-
-notation (HTML output)
-  fcomp  (infixl "\<circ>>" 60)
-
 lemma fcomp_apply:  "(f o> g) x = g (f x)"
   by (simp add: fcomp_def)
 
@@ -107,6 +101,8 @@
 lemma fcomp_id [simp]: "f o> id = f"
   by (simp add: fcomp_def)
 
+no_notation fcomp (infixl "o>" 60)
+
 
 subsection {* Injectivity and Surjectivity *}