src/HOL/Integ/NatSimprocs.thy
author nipkow
Tue, 29 Oct 2002 11:32:52 +0100
changeset 13685 0b8fbcf65d73
parent 10536 8f34ecae1446
child 14128 fd6d20c2371c
permissions -rw-r--r--
added induction thms

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

setup nat_simprocs_setup

end