src/HOL/Proofs.thy
author paulson <lp15@cam.ac.uk>
Wed, 01 Apr 2015 16:04:21 +0100
changeset 59872 db4000b71fdb
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
Theorem "arctan" is no longer a default simprule

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end