src/ZF/ex/NatSum.thy
changeset 76219 cf7db6353322
parent 76215 a642599ffdea
--- a/src/ZF/ex/NatSum.thy	Tue Sep 27 22:57:30 2022 +0100
+++ b/src/ZF/ex/NatSum.thy	Wed Sep 28 11:00:13 2022 +0200
@@ -1,5 +1,5 @@
 (*  Title:      ZF/ex/NatSum.thy
-    Author:     Tobias Nipkow \<and> Lawrence C Paulson
+    Author:     Tobias Nipkow & Lawrence C Paulson
 
 A summation operator. sum(f,n+1) is the sum of all f(i), i=0...n.