diff -r 5efaa884ac6c -r 256fc20716f2 src/Doc/Isar_Ref/Document_Preparation.thy --- a/src/Doc/Isar_Ref/Document_Preparation.thy Thu Aug 11 18:26:16 2016 +0200 +++ b/src/Doc/Isar_Ref/Document_Preparation.thy Thu Aug 11 18:26:44 2016 +0200 @@ -195,8 +195,9 @@ @@{antiquotation emph} options @{syntax text} | @@{antiquotation bold} options @{syntax text} | @@{antiquotation verbatim} options @{syntax text} | + @@{antiquotation path} options @{syntax name} | @@{antiquotation "file"} options @{syntax name} | - @@{antiquotation file_unchecked} options @{syntax name} | + @@{antiquotation dir} options @{syntax name} | @@{antiquotation url} options @{syntax embedded} | @@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and') ; @@ -283,11 +284,13 @@ \<^descr> \@{verbatim s}\ prints uninterpreted source text literally as ASCII characters, using some type-writer font style. - \<^descr> \@{file path}\ checks that \path\ refers to a file (or directory) and - prints it verbatim. + \<^descr> \@{path name}\ prints the file-system path name verbatim. - \<^descr> \@{file_unchecked path}\ is like \@{file path}\, but does not check the - existence of the \path\ within the file-system. + \<^descr> \@{file name}\ is like \@{path name}\, but ensures that \name\ refers to a + plain file. + + \<^descr> \@{dir name}\ is like \@{path name}\, but ensures that \name\ refers to a + directory. \<^descr> \@{url name}\ produces markup for the given URL, which results in an active hyperlink within the text.