src/ZF/CardinalArith.thy
changeset 69587 53982d5ec0bb
parent 67443 3abf6a722518
child 69593 3dda49e08b9d
--- a/src/ZF/CardinalArith.thy	Thu Jan 03 21:06:39 2019 +0100
+++ b/src/ZF/CardinalArith.thy	Thu Jan 03 21:15:52 2019 +0100
@@ -12,11 +12,11 @@
     "InfCard(i) == Card(i) & nat \<le> i"
 
 definition
-  cmult         :: "[i,i]=>i"       (infixl "\<otimes>" 70)  where
+  cmult         :: "[i,i]=>i"       (infixl \<open>\<otimes>\<close> 70)  where
     "i \<otimes> j == |i*j|"
 
 definition
-  cadd          :: "[i,i]=>i"       (infixl "\<oplus>" 65)  where
+  cadd          :: "[i,i]=>i"       (infixl \<open>\<oplus>\<close> 65)  where
     "i \<oplus> j == |i+j|"
 
 definition