src/HOL/Proofs.thy
author kuncar
Sat, 15 Feb 2014 00:11:17 +0100
changeset 55487 6380313b8ed5
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
abstract type must be a type constructor; check it

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end