src/HOL/Proofs.thy
author wenzelm
Thu, 03 Sep 2015 19:27:45 +0200
changeset 61109 1c98bfc5d743
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
proper restore_naming after global qed, which is important to make Name_Space.transform_naming work properly, e.g. for "private typedef";

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end