src/ZF/List_ZF.thy
changeset 67443 3abf6a722518
parent 61798 27f3c10b0b50
--- a/src/ZF/List_ZF.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/ZF/List_ZF.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -98,7 +98,7 @@
 
 definition
   nth :: "[i, i]=>i"  where
-  \<comment>\<open>returns the (n+1)th element of a list, or 0 if the
+  \<comment> \<open>returns the (n+1)th element of a list, or 0 if the
    list is too short.\<close>
   "nth(n, as) == list_rec(\<lambda>n\<in>nat. 0,
                           %a l r. \<lambda>n\<in>nat. nat_case(a, %m. r`m, n), as) ` n"