src/HOL/ex/Ballot.thy
changeset 61609 77b453bd616f
parent 61343 5b5656a63bd6
child 63040 eb4ddd18d635
--- a/src/HOL/ex/Ballot.thy	Tue Nov 03 11:20:21 2015 +0100
+++ b/src/HOL/ex/Ballot.thy	Tue Nov 10 14:18:41 2015 +0000
@@ -266,7 +266,7 @@
 proof -
   from main_nat[of a b] \<open>b < a\<close> have
     "(real a + real b) * real (valid_countings a b) = (real a - real b) * real (all_countings a b)"
-    by (simp only: real_of_nat_add[symmetric] real_of_nat_mult[symmetric]) auto
+    by (simp only: of_nat_add[symmetric] of_nat_mult[symmetric]) auto
   from this \<open>b < a\<close> show ?thesis
     by (subst mult_left_cancel[of "real a + real b", symmetric]) auto
 qed