src/ZF/ex/Ring.thy
changeset 69587 53982d5ec0bb
parent 67398 5eb932e604a2
child 76213 e44d86131648
--- a/src/ZF/ex/Ring.thy	Thu Jan 03 21:06:39 2019 +0100
+++ b/src/ZF/ex/Ring.thy	Thu Jan 03 21:15:52 2019 +0100
@@ -7,8 +7,8 @@
 theory Ring imports Group begin
 
 no_notation
-  cadd  (infixl "\<oplus>" 65) and
-  cmult  (infixl "\<otimes>" 70)
+  cadd  (infixl \<open>\<oplus>\<close> 65) and
+  cmult  (infixl \<open>\<otimes>\<close> 70)
 
 (*First, we must simulate a record declaration:
 record ring = monoid +
@@ -21,11 +21,11 @@
   "add_field(M) = fst(snd(snd(snd(M))))"
 
 definition
-  ring_add :: "[i, i, i] => i" (infixl "\<oplus>\<index>" 65) where
+  ring_add :: "[i, i, i] => i" (infixl \<open>\<oplus>\<index>\<close> 65) where
   "ring_add(M,x,y) = add_field(M) ` <x,y>"
 
 definition
-  zero :: "i => i" ("\<zero>\<index>") where
+  zero :: "i => i" (\<open>\<zero>\<index>\<close>) where
   "zero(M) = fst(snd(snd(snd(snd(M)))))"
 
 
@@ -42,11 +42,11 @@
 text \<open>Derived operations.\<close>
 
 definition
-  a_inv :: "[i,i] => i" ("\<ominus>\<index> _" [81] 80) where
+  a_inv :: "[i,i] => i" (\<open>\<ominus>\<index> _\<close> [81] 80) where
   "a_inv(R) == m_inv (<carrier(R), add_field(R), zero(R), 0>)"
 
 definition
-  minus :: "[i,i,i] => i" ("(_ \<ominus>\<index> _)" [65,66] 65) where
+  minus :: "[i,i,i] => i" (\<open>(_ \<ominus>\<index> _)\<close> [65,66] 65) where
   "\<lbrakk>x \<in> carrier(R); y \<in> carrier(R)\<rbrakk> \<Longrightarrow> x \<ominus>\<^bsub>R\<^esub> y = x \<oplus>\<^bsub>R\<^esub> (\<ominus>\<^bsub>R\<^esub> y)"
 
 locale abelian_monoid = fixes G (structure)