src/HOL/Integ/IntArith.thy
author wenzelm
Sat, 03 Nov 2001 01:33:54 +0100
changeset 12023 d982f98e0f0d
parent 11868 56db9f3a6b3e
child 13575 ecb6ecd9af13
permissions -rw-r--r--
tuned;


header {* Integer arithmetic *}

theory IntArith = Bin
files ("int_arith1.ML") ("int_arith2.ML"):

use "int_arith1.ML"
setup int_arith_setup
use "int_arith2.ML"
declare zabs_split [arith_split]

end