src/HOL/Library/ExecutableSet.thy
changeset 18757 f0d901bc0686
parent 18702 7dc7dcd63224
child 18772 f0dd51087eb3
equal deleted inserted replaced
18756:5eb3df798405 18757:f0d901bc0686
    27 and gen_set aG i = gen_set' aG i i;
    27 and gen_set aG i = gen_set' aG i i;
    28 *}
    28 *}
    29 
    29 
    30 code_syntax_tyco set
    30 code_syntax_tyco set
    31   ml ("_ list")
    31   ml ("_ list")
    32   haskell (atom "[_]")
    32   haskell (target_atom "[_]")
    33 
    33 
    34 code_syntax_const "{}"
    34 code_syntax_const "{}"
    35   ml (atom "[]")
    35   ml (target_atom "[]")
    36   haskell (atom "[]")
    36   haskell (target_atom "[]")
    37 
    37 
    38 consts_code
    38 consts_code
    39   "{}"      ("[]")
    39   "{}"      ("[]")
    40   "insert"  ("(_ ins _)")
    40   "insert"  ("(_ ins _)")
    41   "op Un"   ("(_ union _)")
    41   "op Un"   ("(_ union _)")