src/HOL/MicroJava/J/JListExample.thy
changeset 46506 c7faa011bfa7
parent 45827 66c68453455c
child 46512 4f9f61f9b535
equal deleted inserted replaced
46505:cefceb54c656 46506:c7faa011bfa7
     6 
     6 
     7 theory JListExample
     7 theory JListExample
     8 imports Eval
     8 imports Eval
     9 begin
     9 begin
    10 
    10 
    11 declare [[syntax_ambiguity_level = 100000]]
    11 declare [[syntax_ambiguity = ignore]]
    12 
    12 
    13 consts
    13 consts
    14   list_nam :: cnam
    14   list_nam :: cnam
    15   append_name :: mname
    15   append_name :: mname
    16 
    16