doc-src/Codegen/Thy/Further.thy
changeset 46520 a0abc2ea815e
parent 46514 4f7780086991
equal deleted inserted replaced
46519:17dde5feea4b 46520:a0abc2ea815e
    16     \item @{text Scala} prefers tupled syntax over curried syntax.
    16     \item @{text Scala} prefers tupled syntax over curried syntax.
    17 
    17 
    18     \item @{text Scala} sacrifices Hindely-Milner type inference for a
    18     \item @{text Scala} sacrifices Hindely-Milner type inference for a
    19       much more rich type system with subtyping etc.  For this reason
    19       much more rich type system with subtyping etc.  For this reason
    20       type arguments sometimes have to be given explicitly in square
    20       type arguments sometimes have to be given explicitly in square
    21       brackets (mimicing System F syntax).
    21       brackets (mimicking System F syntax).
    22 
    22 
    23     \item In contrast to @{text Haskell} where most specialities of
    23     \item In contrast to @{text Haskell} where most specialities of
    24       the type system are implemented using \emph{type classes},
    24       the type system are implemented using \emph{type classes},
    25       @{text Scala} provides a sophisticated system of \emph{implicit
    25       @{text Scala} provides a sophisticated system of \emph{implicit
    26       arguments}.
    26       arguments}.