src/HOL/Proofs/Extraction/Euclid.thy
changeset 51143 0a2371e7ced3
parent 45170 7dd207fe7b6e
child 57512 cc97b347b301
equal deleted inserted replaced
51142:ac9e909fe55d 51143:0a2371e7ced3
     8 
     8 
     9 theory Euclid
     9 theory Euclid
    10 imports
    10 imports
    11   "~~/src/HOL/Number_Theory/UniqueFactorization"
    11   "~~/src/HOL/Number_Theory/UniqueFactorization"
    12   Util
    12   Util
    13   "~~/src/HOL/Library/Efficient_Nat"
    13   "~~/src/HOL/Library/Code_Target_Numeral"
    14 begin
    14 begin
    15 
    15 
    16 text {*
    16 text {*
    17 A constructive version of the proof of Euclid's theorem by
    17 A constructive version of the proof of Euclid's theorem by
    18 Markus Wenzel and Freek Wiedijk \cite{Wenzel-Wiedijk-JAR2002}.
    18 Markus Wenzel and Freek Wiedijk \cite{Wenzel-Wiedijk-JAR2002}.