tuned operator precedence
authortraytel
Mon, 29 Apr 2013 10:03:35 +0200
changeset 51806 5c53d40a8eed
parent 51805 67757f1d5e71
child 51807 d694233adeae
tuned operator precedence
src/HOL/Cardinals/Cardinal_Arithmetic.thy
--- a/src/HOL/Cardinals/Cardinal_Arithmetic.thy	Mon Apr 29 09:45:14 2013 +0200
+++ b/src/HOL/Cardinals/Cardinal_Arithmetic.thy	Mon Apr 29 10:03:35 2013 +0200
@@ -366,10 +366,10 @@
 
 subsection {* Exponentiation *}
 
-definition cexp (infixr "^c" 80) where
+definition cexp (infixr "^c" 90) where
   "r1 ^c r2 \<equiv> |Func (Field r2) (Field r1)|"
 
-definition ccexp (infixr "^^c" 80) where
+definition ccexp (infixr "^^c" 90) where
   "r1 ^^c r2 \<equiv> |Pfunc (Field r2) (Field r1)|"
 
 lemma cexp_ordLeq_ccexp: "r1 ^c r2 \<le>o r1 ^^c r2"