src/ZF/IntArith.thy
author nipkow
Wed, 06 Jun 2007 19:12:07 +0200
changeset 23279 e39dd93161d9
parent 23146 0bc590051d95
child 27237 c94eefffc3a5
permissions -rw-r--r--
tuned list comprehension, changed filter syntax from : to <-
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
23146
0bc590051d95 moved Integ files to canonical place;
wenzelm
parents:
diff changeset
     1
0bc590051d95 moved Integ files to canonical place;
wenzelm
parents:
diff changeset
     2
theory IntArith imports Bin
0bc590051d95 moved Integ files to canonical place;
wenzelm
parents:
diff changeset
     3
uses "int_arith.ML" begin
0bc590051d95 moved Integ files to canonical place;
wenzelm
parents:
diff changeset
     4
0bc590051d95 moved Integ files to canonical place;
wenzelm
parents:
diff changeset
     5
end