diff -r 5d8faadf3ecf -r 0bc590051d95 src/ZF/IntArith.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/ZF/IntArith.thy Thu May 31 12:06:31 2007 +0200 @@ -0,0 +1,5 @@ + +theory IntArith imports Bin +uses "int_arith.ML" begin + +end