doc-src/IsarImplementation/Thy/base.thy
author wenzelm
Thu, 06 Mar 2008 20:44:54 +0100
changeset 26223 f4a1a96cc07c
parent 21374 27ae6bc4102a
child 26957 e3f04fdd994d
permissions -rw-r--r--
specific system_out (MosML lacks structure Posix); dummy implementation of Posix.ProcEnv.getpid;


(* $Id$ *)

theory base
imports CPure
uses "../../antiquote_setup.ML"
begin

end