thys/MyFirst.thy
changeset 15 bdabf71fa35b
parent 14 5c6f9325327f
child 16 a92c10af61bd
equal deleted inserted replaced
14:5c6f9325327f 15:bdabf71fa35b
    89 value "trip 2"
    89 value "trip 2"
    90 
    90 
    91 fun mull :: "nat \<Rightarrow> nat \<Rightarrow> nat" where
    91 fun mull :: "nat \<Rightarrow> nat \<Rightarrow> nat" where
    92 "mull 0 0 = 0" |
    92 "mull 0 0 = 0" |
    93 "mull m 0 = 0" |
    93 "mull m 0 = 0" |
    94 "mull m 1 = m" |
    94 (**"mull m 1 = m" | **)
    95 "mull m n = 0" 
    95 "mull m n = m*n" 
    96 
    96 
    97 (**
    97 (**
    98 fun count :: "'a\<Rightarrow>'a list\<Rightarrow>nat" where
    98 fun count :: "'a\<Rightarrow>'a list\<Rightarrow>nat" where
    99 "count  "
    99 "count  "
   100 **)
   100 **)