Admin/Isabelle2005-polyml-5.0/src/Pure/ML-Systems/polyml-5.0.ML
author wenzelm
Tue, 24 Jul 2007 19:44:32 +0200
changeset 23961 9e7e1e309ebd
parent 21688 e5287f12f1e1
permissions -rw-r--r--
Multithreading in Poly/ML (version 5.1).

(*  Title:      Pure/ML-Systems/polyml-5.0.ML
    ID:         $Id$

Compatibility wrapper for Poly/ML 5.0 -- version for Isabelle2005.
*)

structure Posix =
struct
  open Posix;
  structure IO =
  struct
    open IO;
    val mkReader = mkTextReader;
    val mkWriter = mkTextWriter;
  end;
end;

structure TextIO =
struct
  open TextIO;
  fun inputLine is = Option.getOpt (TextIO.inputLine is, "");
end;

structure Substring =
struct
  open Substring;
  val all = full;
end;


use "ML-Systems/polyml.ML";

val pointer_eq = PolyML.pointerEq;