src/ZF/Coind/Values.thy
changeset 76215 a642599ffdea
parent 76213 e44d86131648
child 76216 9fc34f76b4e8
--- a/src/ZF/Coind/Values.thy	Tue Sep 27 17:03:23 2022 +0100
+++ b/src/ZF/Coind/Values.thy	Tue Sep 27 17:46:52 2022 +0100
@@ -21,9 +21,9 @@
   type_intros  A_into_univ mapQU
 
 consts
-  ve_owr :: "[i,i,i] => i"
-  ve_dom :: "i=>i"
-  ve_app :: "[i,i] => i"
+  ve_owr :: "[i,i,i] \<Rightarrow> i"
+  ve_dom :: "i\<Rightarrow>i"
+  ve_app :: "[i,i] \<Rightarrow> i"
 
 
 primrec "ve_owr(ve_mk(m), x, v) = ve_mk(map_owr(m,x,v))"