src/HOL/Main.thy
author berghofe
Fri, 31 Aug 2001 16:28:26 +0200
changeset 11533 0c0d2332e8f0
parent 11483 f4d10044a2cd
child 12024 b3661262541e
permissions -rw-r--r--
Added code generator setup.

(*  Title:      HOL/Main.thy
    ID:         $Id$
    Author:     Tobias Nipkow
    Copyright   2000 TU Muenchen

Theory Main includes everything.
Note that theory PreList already includes most HOL theories.
*)

theory Main = Map + String + Hilbert_Choice:

(*belongs to theory List*)
declare lists_mono [mono]
declare map_cong [recdef_cong]
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