src/HOL/Number_Theory/Pocklington.thy
changeset 67345 debef21cbed6
parent 67091 1393c2340eec
child 67399 eab6ce8368fa
--- a/src/HOL/Number_Theory/Pocklington.thy	Sat Jan 06 10:08:11 2018 +0100
+++ b/src/HOL/Number_Theory/Pocklington.thy	Sat Jan 06 13:05:25 2018 +0100
@@ -372,7 +372,7 @@
     have eqo: "[(a^?o)^?q = 1] (mod n)"
       using cong_pow ord_works by fastforce
     from H have onz: "?o \<noteq> 0" by (simp add: ord_eq_0)
-    then have op: "?o > 0" by simp
+    then have opos: "?o > 0" by simp
     from div_mult_mod_eq[of d "ord n a"] \<open>?lhs\<close>
     have "[a^(?o*?q + ?r) = 1] (mod n)"
       by (simp add: cong_def mult.commute)
@@ -387,7 +387,7 @@
       then show ?thesis by (simp add: dvd_eq_mod_eq_0)
     next
       case False
-      with mod_less_divisor[OF op, of d] have r0o:"?r >0 \<and> ?r < ?o" by simp
+      with mod_less_divisor[OF opos, of d] have r0o:"?r >0 \<and> ?r < ?o" by simp
       from conjunct2[OF ord_works[of a n], rule_format, OF r0o] th
       show ?thesis by blast
     qed