src/HOL/Proofs.thy
author blanchet
Mon, 08 Sep 2014 14:03:40 +0200
changeset 58223 ba7a2d19880c
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
export useful functions for users of (co)recursors

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end