src/HOL/Library/Stirling.thy
changeset 65552 f533820e7248
parent 64267 b9a1486e79be
child 66655 e9be3d6995f9
equal deleted inserted replaced
65551:d164c4fc0d2c 65552:f533820e7248
     6 *)
     6 *)
     7 
     7 
     8 section \<open>Stirling numbers of first and second kind\<close>
     8 section \<open>Stirling numbers of first and second kind\<close>
     9 
     9 
    10 theory Stirling
    10 theory Stirling
    11 imports Binomial
    11 imports Main
    12 begin
    12 begin
    13 
    13 
    14 subsection \<open>Stirling numbers of the second kind\<close>
    14 subsection \<open>Stirling numbers of the second kind\<close>
    15 
    15 
    16 fun Stirling :: "nat \<Rightarrow> nat \<Rightarrow> nat"
    16 fun Stirling :: "nat \<Rightarrow> nat \<Rightarrow> nat"