src/HOL/Main.thy
changeset 12439 e90a4f5a27f0
parent 12024 b3661262541e
child 12554 671b4d632c34
equal deleted inserted replaced
12438:afd41635dcf9 12439:e90a4f5a27f0
    94 
    94 
    95 subsection {* Configuration of the code generator *}
    95 subsection {* Configuration of the code generator *}
    96 
    96 
    97 types_code
    97 types_code
    98   "bool"  ("bool")
    98   "bool"  ("bool")
    99   "*"     ("prod")
    99   "*"     ("(_ */ _)")
   100   "list"  ("list")
   100   "list"  ("_ list")
   101 
   101 
   102 consts_code
   102 consts_code
   103   "op ="    ("(_ =/ _)")
   103   "op ="    ("(_ =/ _)")
   104 
   104 
   105   "True"    ("true")
   105   "True"    ("true")
   113   "fst"     ("fst")
   113   "fst"     ("fst")
   114   "snd"     ("snd")
   114   "snd"     ("snd")
   115 
   115 
   116   "Nil"     ("[]")
   116   "Nil"     ("[]")
   117   "Cons"    ("(_ ::/ _)")
   117   "Cons"    ("(_ ::/ _)")
   118   
   118 
   119 end
   119 end