src/HOL/Proofs.thy
author blanchet
Tue, 31 May 2016 10:53:11 +0200
changeset 63188 38d6aabec460
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
more flexible parsing (towards type class support)

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end