Function.thy revision eca83bf7d98670ee4fa52661d2f8222429a4f91a
theory Function
imports Real
begin
type_synonym real_vector = "nat \<Rightarrow> real"
fun maximum ::
"nat \<Rightarrow> real_vector \<Rightarrow> real" where
"maximum 0 _ = 0" |
"maximum (Suc n) y = max 0 (max (maximum n y) (y (Suc n)))"
fun testfun ::
"nat \<Rightarrow> real \<Rightarrow> real \<Rightarrow> real" where
"testfun _ _ _ = 0"
fun testfun1 ::
"nat \<Rightarrow> nat" where
"testfun1 _ = 0"
end