src/HOL/MicroJava/BV/Typing_Framework_err.thy
changeset 15425 6356d2523f73
parent 13224 6f0928a942d1
child 16417 9bc16273c2d4
equal deleted inserted replaced
15424:7a91490c1b04 15425:6356d2523f73
    20 
    20 
    21 map_snd :: "('b \<Rightarrow> 'c) \<Rightarrow> ('a \<times> 'b) list \<Rightarrow> ('a \<times> 'c) list"
    21 map_snd :: "('b \<Rightarrow> 'c) \<Rightarrow> ('a \<times> 'b) list \<Rightarrow> ('a \<times> 'c) list"
    22 "map_snd f \<equiv> map (\<lambda>(x,y). (x, f y))"
    22 "map_snd f \<equiv> map (\<lambda>(x,y). (x, f y))"
    23 
    23 
    24 error :: "nat \<Rightarrow> (nat \<times> 'a err) list"
    24 error :: "nat \<Rightarrow> (nat \<times> 'a err) list"
    25 "error n \<equiv> map (\<lambda>x. (x,Err)) [0..n(]"
    25 "error n \<equiv> map (\<lambda>x. (x,Err)) [0..<n]"
    26 
    26 
    27 err_step :: "nat \<Rightarrow> (nat \<Rightarrow> 's \<Rightarrow> bool) \<Rightarrow> 's step_type \<Rightarrow> 's err step_type"
    27 err_step :: "nat \<Rightarrow> (nat \<Rightarrow> 's \<Rightarrow> bool) \<Rightarrow> 's step_type \<Rightarrow> 's err step_type"
    28 "err_step n app step p t \<equiv> 
    28 "err_step n app step p t \<equiv> 
    29   case t of 
    29   case t of 
    30     Err   \<Rightarrow> error n
    30     Err   \<Rightarrow> error n