src/HOL/Integ/NatSimprocs.thy
author berghofe
Thu, 10 Oct 2002 14:19:17 +0200
changeset 13636 fdf7e9388be7
parent 10536 8f34ecae1446
child 14128 fd6d20c2371c
permissions -rw-r--r--
Removed obsolete function "Funs".

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

setup nat_simprocs_setup

end