src/ZF/Integ/IntArith.thy
author schirmer
Mon, 26 Jan 2004 10:34:02 +0100
changeset 14361 ad2f5da643b4
parent 9570 e16e168984e1
child 16417 9bc16273c2d4
permissions -rw-r--r--
* Support for raw latex output in control symbols: \<^raw...> * Symbols may only start with one backslash: \<...>. \\<...> is no longer accepted by the scanner. - Adapted some Isar-theories to fit to this policy
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
9570
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents:
diff changeset
     1
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents:
diff changeset
     2
theory IntArith = Bin
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents:
diff changeset
     3
files "int_arith.ML":
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