src/HOL/Library/Pocklington.thy
changeset 27487 c8a6ce181805
parent 27368 9f90ac19e32b
child 27668 6eb20b2cecf8
equal deleted inserted replaced
27486:c61507a98bff 27487:c8a6ce181805
     5 
     5 
     6 header {* Pocklington's Theorem for Primes *}
     6 header {* Pocklington's Theorem for Primes *}
     7 
     7 
     8 
     8 
     9 theory Pocklington
     9 theory Pocklington
    10 imports Plain List Primes
    10 imports Plain "~~/src/HOL/List" "~~/src/HOL/Primes"
    11 begin
    11 begin
    12 
    12 
    13 definition modeq:: "nat => nat => nat => bool"    ("(1[_ = _] '(mod _'))")
    13 definition modeq:: "nat => nat => nat => bool"    ("(1[_ = _] '(mod _'))")
    14   where "[a = b] (mod p) == ((a mod p) = (b mod p))"
    14   where "[a = b] (mod p) == ((a mod p) = (b mod p))"
    15 
    15