doc-src/IsarAdvanced/Codegen/Thy/ML.thy
author wenzelm
Wed, 17 Sep 2008 21:27:38 +0200
changeset 28273 17f6aa02ded3
parent 28213 b52f9205a02d
child 28419 f65e8b318581
permissions -rw-r--r--
simplified ML_Context.eval_in -- expect immutable Proof.context value;

theory "ML"
imports Setup
begin

section {* ML system interfaces *}

end