src/HOL/Proofs/Extraction/Euclid.thy
changeset 76987 4c275405faae
parent 67320 6afba546f0e5
--- a/src/HOL/Proofs/Extraction/Euclid.thy	Sun Jan 15 16:28:03 2023 +0100
+++ b/src/HOL/Proofs/Extraction/Euclid.thy	Sun Jan 15 18:30:18 2023 +0100
@@ -16,7 +16,7 @@
 
 text \<open>
   A constructive version of the proof of Euclid's theorem by
-  Markus Wenzel and Freek Wiedijk @{cite "Wenzel-Wiedijk-JAR2002"}.
+  Markus Wenzel and Freek Wiedijk \<^cite>\<open>"Wenzel-Wiedijk-JAR2002"\<close>.
 \<close>
 
 lemma factor_greater_one1: "n = m * k \<Longrightarrow> m < n \<Longrightarrow> k < n \<Longrightarrow> Suc 0 < m"