diff -r b044a06ad0d6 -r d997c7ba3305 src/Doc/Isar_Ref/Spec.thy --- a/src/Doc/Isar_Ref/Spec.thy Fri Aug 23 21:08:27 2019 +0200 +++ b/src/Doc/Isar_Ref/Spec.thy Sat Aug 24 12:03:00 2019 +0200 @@ -501,7 +501,7 @@ subsection \Locale declarations\ text \ - \begin{matharray}{rcl} + \begin{tabular}{rcll} @{command_def "locale"} & : & \theory \ local_theory\ \\ @{command_def "experiment"} & : & \theory \ local_theory\ \\ @{command_def "print_locale"}\\<^sup>*\ & : & \context \\ \\ @@ -509,7 +509,8 @@ @{command_def "locale_deps"}\\<^sup>*\ & : & \context \\ \\ @{method_def intro_locales} & : & \method\ \\ @{method_def unfold_locales} & : & \method\ \\ - \end{matharray} + @{attribute_def trace_locales} & : & \attribute\ & default \false\ \\ + \end{tabular} \indexisarelem{fixes}\indexisarelem{constrains}\indexisarelem{assumes} \indexisarelem{defines}\indexisarelem{notes} @@ -627,6 +628,11 @@ specifications entailed by the context, both from target statements, and from interpretations (see below). New goals that are entailed by the current context are discharged automatically. + + \<^descr> @{attribute trace_locales}, when set to + \true\, prints the locale instances activated during + roundup. Useful for understanding local theories created by complex + locale hierarchies. \