src/Pure/Pure.thy
changeset 58868 c5e1cce7ace3
parent 58860 fee7cfa69c50
child 58918 8d36bc5eaed3
equal deleted inserted replaced
58867:911addd19e9f 58868:c5e1cce7ace3
    12     "attach" "begin" "binder" "constrains" "defines" "fixes" "for"
    12     "attach" "begin" "binder" "constrains" "defines" "fixes" "for"
    13     "identifier" "if" "imports" "in" "includes" "infix" "infixl"
    13     "identifier" "if" "imports" "in" "includes" "infix" "infixl"
    14     "infixr" "is" "keywords" "notes" "obtains" "open" "output"
    14     "infixr" "is" "keywords" "notes" "obtains" "open" "output"
    15     "overloaded" "pervasive" "shows" "structure" "unchecked" "where" "|"
    15     "overloaded" "pervasive" "shows" "structure" "unchecked" "where" "|"
    16   and "theory" :: thy_begin % "theory"
    16   and "theory" :: thy_begin % "theory"
    17   and "header" :: diag
    17   and "header" :: heading
    18   and "chapter" :: thy_heading1
    18   and "chapter" :: heading
    19   and "section" :: thy_heading2
    19   and "section" :: heading
    20   and "subsection" :: thy_heading3
    20   and "subsection" :: heading
    21   and "subsubsection" :: thy_heading4
    21   and "subsubsection" :: heading
    22   and "text" "text_raw" :: thy_decl
    22   and "text" "text_raw" :: thy_decl
    23   and "sect" :: prf_heading2 % "proof"
       
    24   and "subsect" :: prf_heading3 % "proof"
       
    25   and "subsubsect" :: prf_heading4 % "proof"
       
    26   and "txt" "txt_raw" :: prf_decl % "proof"
    23   and "txt" "txt_raw" :: prf_decl % "proof"
    27   and "default_sort" :: thy_decl == ""
    24   and "default_sort" :: thy_decl == ""
    28   and "typedecl" "type_synonym" "nonterminal" "judgment"
    25   and "typedecl" "type_synonym" "nonterminal" "judgment"
    29     "consts" "syntax" "no_syntax" "translations" "no_translations" "defs"
    26     "consts" "syntax" "no_syntax" "translations" "no_translations" "defs"
    30     "definition" "abbreviation" "type_notation" "no_type_notation" "notation"
    27     "definition" "abbreviation" "type_notation" "no_type_notation" "notation"