src/HOL/Proofs.thy
author blanchet
Wed, 03 Sep 2014 00:06:24 +0200
changeset 58152 6fe60a9a5bad
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
use 'datatype_new' in 'Main'

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end