src/HOL/Proofs.thy
author blanchet
Wed, 23 Apr 2014 10:23:27 +0200
changeset 56650 1f9ab71d43a5
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
no need to make 'size' generation an interpretation -- overkill

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end