src/Pure/Pure.thy
changeset 58868 c5e1cce7ace3
parent 58860 fee7cfa69c50
child 58918 8d36bc5eaed3
--- a/src/Pure/Pure.thy	Sun Nov 02 13:26:20 2014 +0100
+++ b/src/Pure/Pure.thy	Sun Nov 02 15:27:37 2014 +0100
@@ -14,15 +14,12 @@
     "infixr" "is" "keywords" "notes" "obtains" "open" "output"
     "overloaded" "pervasive" "shows" "structure" "unchecked" "where" "|"
   and "theory" :: thy_begin % "theory"
-  and "header" :: diag
-  and "chapter" :: thy_heading1
-  and "section" :: thy_heading2
-  and "subsection" :: thy_heading3
-  and "subsubsection" :: thy_heading4
+  and "header" :: heading
+  and "chapter" :: heading
+  and "section" :: heading
+  and "subsection" :: heading
+  and "subsubsection" :: heading
   and "text" "text_raw" :: thy_decl
-  and "sect" :: prf_heading2 % "proof"
-  and "subsect" :: prf_heading3 % "proof"
-  and "subsubsect" :: prf_heading4 % "proof"
   and "txt" "txt_raw" :: prf_decl % "proof"
   and "default_sort" :: thy_decl == ""
   and "typedecl" "type_synonym" "nonterminal" "judgment"