src/HOL/Fact.thy
changeset 57113 7e95523302e6
parent 50240 019d642d422d
child 57129 7edb7550663e
equal deleted inserted replaced
57111:de33f3965ca6 57113:7e95523302e6
   322     by (subst setprod_insert[symmetric]) (auto simp: atLeastAtMost_insertL)
   322     by (subst setprod_insert[symmetric]) (auto simp: atLeastAtMost_insertL)
   323   with assms show ?thesis
   323   with assms show ?thesis
   324     by (induct r rule: nat.induct) (auto simp add: fact_div_fact Suc_diff_Suc mult_le_mono)
   324     by (induct r rule: nat.induct) (auto simp add: fact_div_fact Suc_diff_Suc mult_le_mono)
   325 qed
   325 qed
   326 
   326 
       
   327 lemma fact_numeral:  --{*Evaluation for specific numerals*}
       
   328   "fact (numeral k) = (numeral k) * (fact (pred_numeral k))"
       
   329   by (simp add: numeral_eq_Suc)
       
   330 
   327 end
   331 end