src/HOL/Library/Ramsey.thy
changeset 81142 6ad2c917dd2e
parent 80914 d97fdabd9e2b
child 81332 f94b30fa2b6c
--- a/src/HOL/Library/Ramsey.thy	Wed Oct 09 22:01:33 2024 +0200
+++ b/src/HOL/Library/Ramsey.thy	Wed Oct 09 23:38:29 2024 +0200
@@ -15,7 +15,7 @@
 
 subsubsection \<open>The $n$-element subsets of a set $A$\<close>
 
-definition nsets :: "['a set, nat] \<Rightarrow> 'a set set" (\<open>([_]\<^bsup>_\<^esup>)\<close> [0,999] 999)
+definition nsets :: "['a set, nat] \<Rightarrow> 'a set set" (\<open>(\<open>notation=\<open>mixfix nsets\<close>\<close>[_]\<^bsup>_\<^esup>)\<close> [0,999] 999)
   where "nsets A n \<equiv> {N. N \<subseteq> A \<and> finite N \<and> card N = n}"
 
 lemma finite_imp_finite_nsets: "finite A \<Longrightarrow> finite ([A]\<^bsup>k\<^esup>)"