src/ZF/IntArith.thy
author wenzelm
Thu, 14 Jun 2007 23:04:36 +0200
changeset 23393 31781b2de73d
parent 23146 0bc590051d95
child 27237 c94eefffc3a5
permissions -rw-r--r--
tuned proofs: avoid implicit prems;


theory IntArith imports Bin
uses "int_arith.ML" begin

end