src/HOL/Proofs.thy
author wenzelm
Tue, 08 Sep 2015 15:37:13 +0200
changeset 61134 80ac5e17772d
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
clarified Java runtime options for 32 vs. 64 bit;

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end