src/HOL/Prolog/HOHH.thy
author kleing
Mon, 21 Jun 2004 10:25:57 +0200
changeset 14981 e73f8140af78
parent 13208 965f95a3abd9
child 17311 5b1d47d920ce
permissions -rw-r--r--
Merged in license change from Isabelle2004

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

higher-order hereditary Harrop formulas 
*)

HOHH = HOL +

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