src/HOL/Proofs.thy
author boehmes
Tue, 23 Jul 2013 18:36:23 +0200
changeset 52722 2c81f7baf8c4
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
removed obsolete HOL-Boogie session; keep examples that also test SMT solvers, using a minimal version of the old Boogie loader

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end