src/HOL/Main.thy
changeset 11533 0c0d2332e8f0
parent 11483 f4d10044a2cd
child 12024 b3661262541e
--- a/src/HOL/Main.thy	Fri Aug 31 16:27:43 2001 +0200
+++ b/src/HOL/Main.thy	Fri Aug 31 16:28:26 2001 +0200
@@ -15,4 +15,28 @@
 lemmas rev_induct [case_names Nil snoc] = rev_induct
   and rev_cases [case_names Nil snoc] = rev_exhaust
 
+(** configuration of code generator **)
+
+types_code
+  "bool"  ("bool")
+  "*"     ("prod")
+  "list"  ("list")
+
+consts_code
+  "op ="    ("(_ =/ _)")
+
+  "True"    ("true")
+  "False"   ("false")
+  "Not"     ("not")
+  "op |"    ("(_ orelse/ _)")
+  "op &"    ("(_ andalso/ _)")
+  "If"      ("(if _/ then _/ else _)")
+
+  "Pair"    ("(_,/ _)")
+  "fst"     ("fst")
+  "snd"     ("snd")
+
+  "Nil"     ("[]")
+  "Cons"    ("(_ ::/ _)")
+  
 end