src/HOL/Proofs.thy
author wenzelm
Mon, 22 Sep 2014 16:28:24 +0200
changeset 58419 593917a7ad02
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
examples for local CSDP executable;

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end