src/HOL/Number_Theory/Euclidean_Algorithm.thy
changeset 64911 f0e07600de47
parent 64850 fc9265882329
child 65398 a14fa655b48c
--- a/src/HOL/Number_Theory/Euclidean_Algorithm.thy	Tue Jan 17 11:26:21 2017 +0100
+++ b/src/HOL/Number_Theory/Euclidean_Algorithm.thy	Tue Jan 17 13:59:10 2017 +0100
@@ -187,7 +187,7 @@
 proof -
   show "class.factorial_semiring divide plus minus zero times one
      unit_factor normalize"
-  proof (standard, rule factorial_semiring_altI_aux) -- \<open>FIXME rule\<close>
+  proof (standard, rule factorial_semiring_altI_aux) \<comment> \<open>FIXME rule\<close>
     fix x assume "x \<noteq> 0"
     thus "finite {p. p dvd x \<and> normalize p = p}"
     proof (induction "euclidean_size x" arbitrary: x rule: less_induct)