src/HOL/Power.thy
changeset 7843 077d305615df
parent 5183 89f162de39cf
child 8844 db71c334e854
--- a/src/HOL/Power.thy	Wed Oct 13 12:07:03 1999 +0200
+++ b/src/HOL/Power.thy	Wed Oct 13 12:07:23 1999 +0200
@@ -9,7 +9,7 @@
 
 Power = Divides + 
 consts
-  binomial :: "[nat,nat] => nat"      ("'(_ choose _')" [50,50])
+  binomial :: "[nat,nat] => nat"      (infixl "choose" 65)
 
 primrec
   "p ^ 0 = 1"