src/HOL/Proofs.thy
author haftmann
Sat, 31 Dec 2016 08:12:31 +0100
changeset 64715 33d5fa0ce6e5
parent 52488 cd65ee49a8ba
permissions -rw-r--r--
more elementary rules about div / mod on int

theory Proofs
imports Pure
begin

ML "Proofterm.proofs := 2"

end