src/HOL/Integ/NatSimprocs.thy
author paulson
Fri, 16 Nov 2001 18:24:11 +0100
changeset 12224 02df7cbe7d25
parent 10536 8f34ecae1446
child 14128 fd6d20c2371c
permissions -rw-r--r--
even more theories from Jacques

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

setup nat_simprocs_setup

end