fixed indentation
authorpaulson <lp15@cam.ac.uk>
Mon, 03 Feb 2014 00:22:48 +0000
changeset 55262 16724746ad89
parent 55261 ad3604df6bc6
child 55263 4d63fffcde8d
fixed indentation
src/HOL/Number_Theory/Residues.thy
--- a/src/HOL/Number_Theory/Residues.thy	Sun Feb 02 21:48:28 2014 +0000
+++ b/src/HOL/Number_Theory/Residues.thy	Mon Feb 03 00:22:48 2014 +0000
@@ -312,9 +312,9 @@
       done
     with `x dvd p` `1 < x` have "False" by auto }
   then show ?thesis 
-    using `2 \<le> p` apply (simp add: prime_def)
-by (metis One_nat_def dvd_pos_nat nat_dvd_not_less nat_neq_iff not_gr0 
-  not_numeral_le_zero one_dvd)
+    using `2 \<le> p` 
+    by (simp add: prime_def)
+       (metis One_nat_def dvd_pos_nat nat_dvd_not_less nat_neq_iff not_gr0 not_numeral_le_zero one_dvd)
 qed
 
 lemma phi_zero [simp]: "phi 0 = 0"