src/HOL/Proofs.thy
author blanchet
Fri, 16 May 2014 12:56:39 +0200
changeset 56978 0c1b4987e6b2
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
proper handling of 'ctor_dtor' for mutual corecursive cases where not all type variables are present in all low-level constructors (cf. 'coind_wit1' etc. in 'Misc_Codatatypes.thy')

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end