src/HOL/HOL.thy
changeset 81706 7beb0cf38292
parent 81595 ed264056f5dc
equal deleted inserted replaced
81705:53fea2ccab19 81706:7beb0cf38292
  2072 | constant True \<rightharpoonup>
  2072 | constant True \<rightharpoonup>
  2073     (SML) "true" and (OCaml) "true" and (Haskell) "True" and (Scala) "true"
  2073     (SML) "true" and (OCaml) "true" and (Haskell) "True" and (Scala) "true"
  2074 | constant False \<rightharpoonup>
  2074 | constant False \<rightharpoonup>
  2075     (SML) "false" and (OCaml) "false" and (Haskell) "False" and (Scala) "false"
  2075     (SML) "false" and (OCaml) "false" and (Haskell) "False" and (Scala) "false"
  2076 
  2076 
  2077 code_reserved SML
  2077 code_reserved
  2078   bool true false
  2078   (SML) bool true false
  2079 
  2079   and (OCaml) bool
  2080 code_reserved OCaml
  2080   and (Scala) Boolean
  2081   bool
       
  2082 
       
  2083 code_reserved Scala
       
  2084   Boolean
       
  2085 
  2081 
  2086 code_printing
  2082 code_printing
  2087   constant Not \<rightharpoonup>
  2083   constant Not \<rightharpoonup>
  2088     (SML) "not" and (OCaml) "not" and (Haskell) "not" and (Scala) "'! _"
  2084     (SML) "not" and (OCaml) "not" and (Haskell) "not" and (Scala) "'! _"
  2089 | constant HOL.conj \<rightharpoonup>
  2085 | constant HOL.conj \<rightharpoonup>
  2099     (SML) "!(if (_)/ then (_)/ else (_))"
  2095     (SML) "!(if (_)/ then (_)/ else (_))"
  2100     and (OCaml) "!(if (_)/ then (_)/ else (_))"
  2096     and (OCaml) "!(if (_)/ then (_)/ else (_))"
  2101     and (Haskell) "!(if (_)/ then (_)/ else (_))"
  2097     and (Haskell) "!(if (_)/ then (_)/ else (_))"
  2102     and (Scala) "!((_) match {/ case true => (_)/ case false => (_)/ })"
  2098     and (Scala) "!((_) match {/ case true => (_)/ case false => (_)/ })"
  2103 
  2099 
  2104 code_reserved SML
  2100 code_reserved
  2105   not
  2101   (SML) not
  2106 
  2102   and (OCaml) not
  2107 code_reserved OCaml
       
  2108   not
       
  2109 
  2103 
  2110 code_identifier
  2104 code_identifier
  2111   code_module Pure \<rightharpoonup>
  2105   code_module Pure \<rightharpoonup>
  2112     (SML) HOL and (OCaml) HOL and (Haskell) HOL and (Scala) HOL
  2106     (SML) HOL and (OCaml) HOL and (Haskell) HOL and (Scala) HOL
  2113 
  2107