Nominal/FSet.thy
changeset 1951 a0c7290a4e27
parent 1913 39951d71bfce
child 1952 27cdc0a3a763
--- a/Nominal/FSet.thy	Wed Apr 21 10:24:39 2010 +0200
+++ b/Nominal/FSet.thy	Wed Apr 21 12:25:52 2010 +0200
@@ -370,7 +370,7 @@
   "{|x|}"     == "CONST finsert x {||}"
 
 quotient_definition
-  fin ("_ |\<in>| _" [50, 51] 50)
+  fin (infix "|\<in>|" 50)
 where
   "fin :: 'a \<Rightarrow> 'a fset \<Rightarrow> bool" is "memb"