src/Pure/ML-Systems/smlnj-basis-compat.ML
author wenzelm
Fri, 06 Jan 2006 18:18:16 +0100
changeset 18598 94d658871c98
parent 17514 1d7771a659f6
permissions -rw-r--r--
prep_meta_eq: reuse mk_rews of local simpset; adapted ML code to common conventions; tuned;

(*  Title:      Pure/ML-Systems/smlnj-basis-compat.ML
    ID:         $Id$
    Author:     Sebastian Skalberg (TU Muenchen)

Compatibility file for Standard ML of New Jersey 110.44 or later. Here
signatures that have changed to adhere to the SML Basis Library are
changed back to their old values.
*)

structure TextIO =
struct
  open TextIO;

  fun inputLine is =
    (case TextIO.inputLine is of
      SOME str => str
    | NONE => "")
    handle IO.Io _ => raise Interrupt;
end;