src/HOL/Proofs.thy
author fleury <Mathias.Fleury@mpi-inf.mpg.de>
Tue, 12 Jul 2016 13:55:35 +0200
changeset 63456 3365c8ec67bd
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
sharing simp rules between ordered monoids and rings

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end