add upper bounds for factorial and binomial; add equation for binomial using nat-division (both from AFP/Girth_Chromatic)
(* Title: HOL/Imperative_HOL/Imperative_HOL.thy
Author: John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen
*)
header {* Entry point into monadic imperative HOL *}
theory Imperative_HOL
imports Array Ref Mrec
begin
end