src/HOL/Factorial.thy
changeset 67411 3f4b0c84630f
parent 67399 eab6ce8368fa
child 67969 83c8cafdebe8
--- a/src/HOL/Factorial.thy	Fri Jan 12 17:58:03 2018 +0100
+++ b/src/HOL/Factorial.thy	Sat Jan 13 09:18:54 2018 +0000
@@ -26,7 +26,7 @@
       atLeastLessThanSuc_atLeastAtMost)
 
 lemma fact_prod_rev: "fact n = of_nat (\<Prod>i = 0..<n. n - i)"
-  using prod.atLeast_atMost_rev [of "\<lambda>i. i" 1 n]
+  using prod.atLeastAtMost_rev [of "\<lambda>i. i" 1 n]
   by (cases n)
     (simp_all add: fact_prod_Suc prod.atLeast_Suc_atMost_Suc_shift
       atLeastLessThanSuc_atLeastAtMost)
@@ -191,7 +191,7 @@
   where pochhammer_prod: "pochhammer a n = prod (\<lambda>i. a + of_nat i) {0..<n}"
 
 lemma pochhammer_prod_rev: "pochhammer a n = prod (\<lambda>i. a + of_nat (n - i)) {1..n}"
-  using prod.atLeast_lessThan_rev_at_least_Suc_atMost [of "\<lambda>i. a + of_nat i" 0 n]
+  using prod.atLeastLessThan_rev_at_least_Suc_atMost [of "\<lambda>i. a + of_nat i" 0 n]
   by (simp add: pochhammer_prod)
 
 lemma pochhammer_Suc_prod: "pochhammer a (Suc n) = prod (\<lambda>i. a + of_nat i) {0..n}"