src/HOL/Fun.thy
changeset 12114 a8e860c86252
parent 11609 3f3d1add4d94
child 12258 5da24e7e9aba
--- a/src/HOL/Fun.thy	Fri Nov 09 00:06:15 2001 +0100
+++ b/src/HOL/Fun.thy	Fri Nov 09 00:09:47 2001 +0100
@@ -46,7 +46,7 @@
   inj_on :: ['a => 'b, 'a set] => bool
     "inj_on f A == ! x:A. ! y:A. f(x)=f(y) --> x=y"
 
-syntax (symbols)
+syntax (xsymbols)
   "op o"        :: "['b => 'c, 'a => 'b, 'a] => 'c"      (infixl "\\<circ>" 55)
 
 syntax
@@ -79,7 +79,7 @@
 
   (*Giving funcset the arrow syntax (namely ->) clashes with other theories*)
 
-syntax (symbols)
+syntax (xsymbols)
   "@Pi" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set"  ("(3\\<Pi> _\\<in>_./ _)"   10)
 
 translations