src/HOL/Proofs.thy
author wenzelm
Sun, 24 Jan 2016 15:25:39 +0100
changeset 62242 a4e6ea45f416
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
guard sessions that no longer work with SML/NJ -- memory problems;

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end