src/HOL/Main.thy
changeset 11533 0c0d2332e8f0
parent 11483 f4d10044a2cd
child 12024 b3661262541e
equal deleted inserted replaced
11532:da74db1373ea 11533:0c0d2332e8f0
    13 declare lists_mono [mono]
    13 declare lists_mono [mono]
    14 declare map_cong [recdef_cong]
    14 declare map_cong [recdef_cong]
    15 lemmas rev_induct [case_names Nil snoc] = rev_induct
    15 lemmas rev_induct [case_names Nil snoc] = rev_induct
    16   and rev_cases [case_names Nil snoc] = rev_exhaust
    16   and rev_cases [case_names Nil snoc] = rev_exhaust
    17 
    17 
       
    18 (** configuration of code generator **)
       
    19 
       
    20 types_code
       
    21   "bool"  ("bool")
       
    22   "*"     ("prod")
       
    23   "list"  ("list")
       
    24 
       
    25 consts_code
       
    26   "op ="    ("(_ =/ _)")
       
    27 
       
    28   "True"    ("true")
       
    29   "False"   ("false")
       
    30   "Not"     ("not")
       
    31   "op |"    ("(_ orelse/ _)")
       
    32   "op &"    ("(_ andalso/ _)")
       
    33   "If"      ("(if _/ then _/ else _)")
       
    34 
       
    35   "Pair"    ("(_,/ _)")
       
    36   "fst"     ("fst")
       
    37   "snd"     ("snd")
       
    38 
       
    39   "Nil"     ("[]")
       
    40   "Cons"    ("(_ ::/ _)")
       
    41   
    18 end
    42 end