Isabelle_DOF/examples/technical_report/IsaDof_Manual/IsaDofManual.thy

22 lines
280 B
Plaintext

(*<*)
theory IsaDofManual
imports "06_Conclusion"
begin
(*<*)
text*[bib::bibliography]\<open>References\<close>
(*<*)
close_monitor*[this]
check_doc_global
text\<open>Resulting trace in doc\_item ''this'': \<close>
ML\<open>@{trace_attribute this}\<close>
end
(*>*)