src/HOL/Codegenerator_Test/Candidates.thy
changeset 61130 8e736ce4c6f4
parent 61129 774752af4a1f
child 61227 19ee25fe9737
equal deleted inserted replaced
61129:774752af4a1f 61130:8e736ce4c6f4
    53 
    53 
    54 definition check_list :: unit
    54 definition check_list :: unit
    55 where
    55 where
    56   "check_list = (if funny_list = funny_list' then () else undefined)"
    56   "check_list = (if funny_list = funny_list' then () else undefined)"
    57 
    57 
       
    58 text \<open>Explicit check in @{text Scala} for correct bracketing of abstractions\<close>
       
    59 
       
    60 definition funny_funs :: "(bool \<Rightarrow> bool) list \<Rightarrow> (bool \<Rightarrow> bool) list"
       
    61 where
       
    62   "funny_funs fs = (\<lambda>x. x \<or> True) # (\<lambda>x. x \<or> False) # fs"
       
    63 
    58 end
    64 end