src/HOL/Proofs.thy
author wenzelm
Sun, 28 Dec 2014 22:03:11 +0100
changeset 59194 b51489b75bb9
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
proper sequential version;

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end