src/HOL/Proofs.thy
author wenzelm
Fri, 07 Mar 2014 22:19:52 +0100
changeset 55989 55827fc7c0dd
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
ignore special names that are treated differently for various sub-languages (main wild-card is identifier "__");

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end