src/ZF/func.thy
changeset 69587 53982d5ec0bb
parent 63901 4ce989e962e0
child 69593 3dda49e08b9d
--- a/src/ZF/func.thy	Thu Jan 03 21:06:39 2019 +0100
+++ b/src/ZF/func.thy	Thu Jan 03 21:15:52 2019 +0100
@@ -451,10 +451,10 @@
 
   (* Let expressions *)
 
-  "_updbind"    :: "[i, i] => updbind"               ("(2_ :=/ _)")
-  ""            :: "updbind => updbinds"             ("_")
-  "_updbinds"   :: "[updbind, updbinds] => updbinds" ("_,/ _")
-  "_Update"     :: "[i, updbinds] => i"              ("_/'((_)')" [900,0] 900)
+  "_updbind"    :: "[i, i] => updbind"               (\<open>(2_ :=/ _)\<close>)
+  ""            :: "updbind => updbinds"             (\<open>_\<close>)
+  "_updbinds"   :: "[updbind, updbinds] => updbinds" (\<open>_,/ _\<close>)
+  "_Update"     :: "[i, updbinds] => i"              (\<open>_/'((_)')\<close> [900,0] 900)
 
 translations
   "_Update (f, _updbinds(b,bs))"  == "_Update (_Update(f,b), bs)"