src/HOL/Integ/NatSimprocs.thy
author berghofe
Fri, 28 Jun 2002 19:51:19 +0200
changeset 13256 cf85c4f7dcf2
parent 10536 8f34ecae1446
child 14128 fd6d20c2371c
permissions -rw-r--r--
Added function prop_of' taking assumption context as an argument.

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

setup nat_simprocs_setup

end