src/HOL/HOL.thy
changeset 37877 d4a30d210220
parent 37781 2fbbf0a48cef
child 38525 324219de6ee3
equal deleted inserted replaced
37876:48116a1764c5 37877:d4a30d210220
  1926     and infixl 4 "&&" and infixl 2 "||"
  1926     and infixl 4 "&&" and infixl 2 "||"
  1927     and "!(if (_)/ then (_)/ else (_))")
  1927     and "!(if (_)/ then (_)/ else (_))")
  1928   (Haskell "True" and "False" and "not"
  1928   (Haskell "True" and "False" and "not"
  1929     and infixl 3 "&&" and infixl 2 "||"
  1929     and infixl 3 "&&" and infixl 2 "||"
  1930     and "!(if (_)/ then (_)/ else (_))")
  1930     and "!(if (_)/ then (_)/ else (_))")
  1931   (Scala "true" and "false" and "'! _"
  1931   (Scala "true" and "false" and "'!/ _"
  1932     and infixl 3 "&&" and infixl 1 "||"
  1932     and infixl 3 "&&" and infixl 1 "||"
  1933     and "!(if ((_))/ (_)/ else (_))")
  1933     and "!(if ((_))/ (_)/ else (_))")
  1934 
  1934 
  1935 code_reserved SML
  1935 code_reserved SML
  1936   bool true false not
  1936   bool true false not