src/HOL/Proofs.thy
author haftmann
Sat, 12 Mar 2016 22:04:52 +0100
changeset 62597 b3f2b8c906a6
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
model characters directly as range 0..255 * * * operate on syntax terms rather than asts

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end