src/HOL/Prolog/HOHH.thy
author wenzelm
Fri, 10 Mar 2006 19:49:58 +0100
changeset 19240 3a73cb17a707
parent 17311 5b1d47d920ce
child 21425 c11ab38b78a7
permissions -rw-r--r--
tuned;

(*  Title:    HOL/Prolog/HOHH.thy
    ID:       $Id$
    Author:   David von Oheimb (based on a lecture on Lambda Prolog by Nadathur)
*)

header {* Higher-order hereditary Harrop formulas *}

theory HOHH
imports HOL
begin

consts

(* D-formulas (programs):  D ::= !x. D | D .. D | D :- G | A            *)
  "Dand"        :: "[bool, bool] => bool"         (infixr ".." 28)
  ":-"          :: "[bool, bool] => bool"         (infixl 29)

(* G-formulas (goals):     G ::= A | G & G | G | G | ? x. G
                               | True | !x. G | D => G                  *)
(*","           :: "[bool, bool] => bool"         (infixr 35)*)
  "=>"          :: "[bool, bool] => bool"         (infixr 27)

translations

  "D :- G"      =>      "G --> D"
  "D1 .. D2"    =>      "D1 & D2"
(*"G1 , G2"     =>      "G1 & G2"*)
  "D => G"      =>      "D --> G"

end