src/ZF/Trancl.thy
changeset 69587 53982d5ec0bb
parent 60770 240563fbf41d
child 76213 e44d86131648
--- a/src/ZF/Trancl.thy	Thu Jan 03 21:06:39 2019 +0100
+++ b/src/ZF/Trancl.thy	Thu Jan 03 21:15:52 2019 +0100
@@ -32,16 +32,16 @@
     "trans(r) == \<forall>x y z. <x,y>: r \<longrightarrow> <y,z>: r \<longrightarrow> <x,z>: r"
 
 definition
-  trans_on :: "[i,i]=>o"  ("trans[_]'(_')")  where
+  trans_on :: "[i,i]=>o"  (\<open>trans[_]'(_')\<close>)  where
     "trans[A](r) == \<forall>x\<in>A. \<forall>y\<in>A. \<forall>z\<in>A.
                           <x,y>: r \<longrightarrow> <y,z>: r \<longrightarrow> <x,z>: r"
 
 definition
-  rtrancl :: "i=>i"  ("(_^*)" [100] 100)  (*refl/transitive closure*)  where
+  rtrancl :: "i=>i"  (\<open>(_^*)\<close> [100] 100)  (*refl/transitive closure*)  where
     "r^* == lfp(field(r)*field(r), %s. id(field(r)) \<union> (r O s))"
 
 definition
-  trancl  :: "i=>i"  ("(_^+)" [100] 100)  (*transitive closure*)  where
+  trancl  :: "i=>i"  (\<open>(_^+)\<close> [100] 100)  (*transitive closure*)  where
     "r^+ == r O r^*"
 
 definition