src/HOL/Number_Theory/Residues.thy
changeset 66453 cc19f7ca2ed6
parent 66305 7454317f883c
child 66817 0b12755ccbb2
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     8 section \<open>Residue rings\<close>
     8 section \<open>Residue rings\<close>
     9 
     9 
    10 theory Residues
    10 theory Residues
    11 imports
    11 imports
    12   Cong
    12   Cong
    13   "~~/src/HOL/Algebra/More_Group"
    13   "HOL-Algebra.More_Group"
    14   "~~/src/HOL/Algebra/More_Ring"
    14   "HOL-Algebra.More_Ring"
    15   "~~/src/HOL/Algebra/More_Finite_Product"
    15   "HOL-Algebra.More_Finite_Product"
    16   "~~/src/HOL/Algebra/Multiplicative_Group"
    16   "HOL-Algebra.Multiplicative_Group"
    17   Totient
    17   Totient
    18 begin
    18 begin
    19 
    19 
    20 definition QuadRes :: "int \<Rightarrow> int \<Rightarrow> bool"
    20 definition QuadRes :: "int \<Rightarrow> int \<Rightarrow> bool"
    21   where "QuadRes p a = (\<exists>y. ([y^2 = a] (mod p)))"
    21   where "QuadRes p a = (\<exists>y. ([y^2 = a] (mod p)))"