src/HOL/Proofs/Extraction/Euclid.thy
changeset 58622 aa99568f56de
parent 57514 bdc2c6b40bf2
child 58889 5b7a9633cfa8
equal deleted inserted replaced
58621:7a2c567061b3 58622:aa99568f56de
    13   "~~/src/HOL/Library/Code_Target_Numeral"
    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"}.
    19 *}
    19 *}
    20 
    20 
    21 lemma factor_greater_one1: "n = m * k \<Longrightarrow> m < n \<Longrightarrow> k < n \<Longrightarrow> Suc 0 < m"
    21 lemma factor_greater_one1: "n = m * k \<Longrightarrow> m < n \<Longrightarrow> k < n \<Longrightarrow> Suc 0 < m"
    22   by (induct m) auto
    22   by (induct m) auto
    23 
    23