src/HOL/Number_Theory/Primes.thy
changeset 33718 06e9aff51d17
parent 32479 521cc9bf2958
child 33946 fcc20072df9a
equal deleted inserted replaced
33717:c03edebe7408 33718:06e9aff51d17
    14 The original theory "IntPrimes" was by Thomas M. Rasmussen, and
    14 The original theory "IntPrimes" was by Thomas M. Rasmussen, and
    15 extended gcd, lcm, primes to the integers. Amine Chaieb provided
    15 extended gcd, lcm, primes to the integers. Amine Chaieb provided
    16 another extension of the notions to the integers, and added a number
    16 another extension of the notions to the integers, and added a number
    17 of results to "Primes" and "GCD". IntPrimes also defined and developed
    17 of results to "Primes" and "GCD". IntPrimes also defined and developed
    18 the congruence relations on the integers. The notion was extended to
    18 the congruence relations on the integers. The notion was extended to
    19 the natural numbers by Chiaeb.
    19 the natural numbers by Chaieb.
    20 
    20 
    21 Jeremy Avigad combined all of these, made everything uniform for the
    21 Jeremy Avigad combined all of these, made everything uniform for the
    22 natural numbers and the integers, and added a number of new theorems.
    22 natural numbers and the integers, and added a number of new theorems.
    23 
    23 
    24 Tobias Nipkow cleaned up a lot.
    24 Tobias Nipkow cleaned up a lot.