src/Pure/Pure.thy
changeset 67446 1f4d167b6ac9
parent 67386 998e01d6f8fd
child 67450 b0ae74b86ef3
equal deleted inserted replaced
67445:4311845b0412 67446:1f4d167b6ac9
     4 The Pure theory, with definitions of Isar commands and some lemmas.
     4 The Pure theory, with definitions of Isar commands and some lemmas.
     5 *)
     5 *)
     6 
     6 
     7 theory Pure
     7 theory Pure
     8 keywords
     8 keywords
     9     "!!" "!" "+" "--" ":" ";" "<" "<=" "==" "=>" "?" "[" "\<comment>" "\<equiv>" "\<leftharpoondown>" "\<rightharpoonup>" "\<rightleftharpoons>"
     9     "!!" "!" "+" ":" ";" "<" "<=" "==" "=>" "?" "[" "\<comment>" "\<equiv>" "\<leftharpoondown>" "\<rightharpoonup>" "\<rightleftharpoons>"
    10     "\<subseteq>" "]" "attach" "binder" "in" "infix" "infixl" "infixr" "is" "open" "output"
    10     "\<subseteq>" "]" "attach" "binder" "in" "infix" "infixl" "infixr" "is" "open" "output"
    11     "overloaded" "pervasive" "premises" "structure" "unchecked"
    11     "overloaded" "pervasive" "premises" "structure" "unchecked"
    12   and "private" "qualified" :: before_command
    12   and "private" "qualified" :: before_command
    13   and "assumes" "constrains" "defines" "fixes" "for" "if" "includes" "notes" "rewrites"
    13   and "assumes" "constrains" "defines" "fixes" "for" "if" "includes" "notes" "rewrites"
    14     "obtains" "shows" "when" "where" "|" :: quasi_command
    14     "obtains" "shows" "when" "where" "|" :: quasi_command