src/HOL/Proofs.thy
author blanchet
Mon, 18 Nov 2013 18:04:45 +0100
changeset 54481 5c9819d7713b
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
compile

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end