src/HOL/Integ/IntArith.thy
author wenzelm
Mon, 11 Feb 2002 10:56:33 +0100
changeset 12873 d7f8dfaad46d
parent 12023 d982f98e0f0d
child 13575 ecb6ecd9af13
permissions -rw-r--r--
include SVC_Test;


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