diff -r 5467858e9419 -r f6c88cb715db src/Doc/Isar_Ref/Document_Preparation.thy --- a/src/Doc/Isar_Ref/Document_Preparation.thy Sat Aug 25 20:48:16 2018 +0200 +++ b/src/Doc/Isar_Ref/Document_Preparation.thy Sat Aug 25 21:15:43 2018 +0200 @@ -94,6 +94,7 @@ @{antiquotation_def typ} & : & \antiquotation\ \\ @{antiquotation_def type} & : & \antiquotation\ \\ @{antiquotation_def class} & : & \antiquotation\ \\ + @{antiquotation_def locale} & : & \antiquotation\ \\ @{antiquotation_def "text"} & : & \antiquotation\ \\ @{antiquotation_def goals} & : & \antiquotation\ \\ @{antiquotation_def subgoals} & : & \antiquotation\ \\ @@ -180,6 +181,7 @@ @@{antiquotation typ} options @{syntax type} | @@{antiquotation type} options @{syntax embedded} | @@{antiquotation class} options @{syntax embedded} | + @@{antiquotation locale} options @{syntax embedded} | (@@{antiquotation command} | @@{antiquotation method} | @@{antiquotation attribute}) options @{syntax name} ; @@ -252,6 +254,8 @@ \<^descr> \@{class c}\ prints a class \c\. + \<^descr> \@{locale c}\ prints a locale \c\. + \<^descr> \@{command name}\, \@{method name}\, \@{attribute name}\ print checked entities of the Isar language.