src/HOL/Proofs.thy
author paulson <lp15@cam.ac.uk>
Fri, 02 Oct 2015 15:07:41 +0100
changeset 61306 9dd394c866fc
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
New theorems about connected sets. And pairwise moved to Set.thy.

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end