src/ZF/Integ/IntArith.thy
author wenzelm
Wed, 02 Aug 2006 22:27:02 +0200
changeset 20308 ddb7e7129481
parent 16417 9bc16273c2d4
permissions -rw-r--r--
added tactical result; simplified obtain_export: no Seq.seq, no lifting of result prems; tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
9570
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents:
diff changeset
     1
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 9570
diff changeset
     2
theory IntArith imports Bin
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 9570
diff changeset
     3
uses "int_arith.ML" begin
9570
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents:
diff changeset
     4
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents:
diff changeset
     5
end