src/HOL/Codegenerator_Test/Code_Lazy_Test.thy
changeset 81091 c007e6d9941d
parent 81090 843dba3d307a
child 81182 fc5066122e68
equal deleted inserted replaced
81090:843dba3d307a 81091:c007e6d9941d
    23 code_lazy_type llist
    23 code_lazy_type llist
    24 
    24 
    25 no_notation lazy_llist (\<open>_\<close>)
    25 no_notation lazy_llist (\<open>_\<close>)
    26 syntax
    26 syntax
    27   "_llist" :: "args => 'a list"  (\<open>(\<open>indent=1 notation=\<open>mixfix lazy list enumeration\<close>\<close>\<^bold>[_\<^bold>])\<close>)
    27   "_llist" :: "args => 'a list"  (\<open>(\<open>indent=1 notation=\<open>mixfix lazy list enumeration\<close>\<close>\<^bold>[_\<^bold>])\<close>)
    28 syntax_consts
       
    29   lazy_llist
       
    30 translations
    28 translations
    31   "\<^bold>[x, xs\<^bold>]" == "x\<^bold>#\<^bold>[xs\<^bold>]"
    29   "\<^bold>[x, xs\<^bold>]" == "x\<^bold>#\<^bold>[xs\<^bold>]"
    32   "\<^bold>[x\<^bold>]" == "x\<^bold>#\<^bold>[\<^bold>]"
    30   "\<^bold>[x\<^bold>]" == "x\<^bold>#\<^bold>[\<^bold>]"
    33   "\<^bold>[x\<^bold>]" == "CONST lazy_llist x"
    31   "\<^bold>[x\<^bold>]" == "CONST lazy_llist x"
    34 
    32