src/Doc/Isar_Ref/Misc.thy
changeset 58618 782f0b662cae
parent 58552 66fed99e874f
child 59917 9830c944670f
--- a/src/Doc/Isar_Ref/Misc.thy	Tue Oct 07 21:28:24 2014 +0200
+++ b/src/Doc/Isar_Ref/Misc.thy	Tue Oct 07 21:29:59 2014 +0200
@@ -2,11 +2,11 @@
 imports Base Main
 begin
 
-chapter {* Other commands *}
+chapter \<open>Other commands\<close>
 
-section {* Inspecting the context *}
+section \<open>Inspecting the context\<close>
 
-text {*
+text \<open>
   \begin{matharray}{rcl}
     @{command_def "print_theory"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
     @{command_def "print_methods"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
@@ -110,6 +110,6 @@
   only the unused theorems in the current theory are displayed.
   
   \end{description}
-*}
+\<close>
 
 end