src/HOL/Integ/NatSimprocs.thy
author berghofe
Fri, 09 Nov 2001 10:25:10 +0100
changeset 12125 316d11f760f7
parent 10536 8f34ecae1446
child 14128 fd6d20c2371c
permissions -rw-r--r--
Commands prf and full_prf can now also be used to display proof term of current proof state.

(*Loading further simprocs*)
theory NatSimprocs = NatBin
files "int_factor_simprocs.ML" "nat_simprocs.ML":

setup nat_simprocs_setup

end