src/HOL/NumberTheory/WilsonBij.thy
author paulson
Mon, 07 Aug 2000 10:27:35 +0200
changeset 9545 c1d9500e2927
parent 9508 4d01dbf6ded7
child 11049 7eef34adb852
permissions -rw-r--r--
tidied

(*  Title:	WilsonBij.thy
    ID:         $Id$
    Author:	Thomas M. Rasmussen
    Copyright	2000  University of Cambridge
*)

WilsonBij = BijectionRel + IntFact +

consts
  reciR  :: "int => [int,int] => bool"
  inv    :: "[int,int] => int"

defs
  reciR_def "reciR p == (%a b. zcong (a*b) #1 p & 
                               #1<a & a<p-#1 & #1<b & b<p-#1)"
  inv_def   "inv p a == (if p:zprime & #0<a & a<p then
                           (@x. #0<=x & x<p & zcong (a*x) #1 p)
                         else #0)"

end