src/ZF/IntArith.thy
author wenzelm
Tue, 18 Sep 2007 18:05:34 +0200
changeset 24633 0a3a02066244
parent 23146 0bc590051d95
child 27237 c94eefffc3a5
permissions -rw-r--r--
moved Tools/integer.ML to Pure/General/integer.ML;


theory IntArith imports Bin
uses "int_arith.ML" begin

end