Theory HOHH
section ‹Higher-order hereditary Harrop formulas›
theory HOHH
imports HOL.HOL
begin
ML_file ‹prolog.ML›
method_setup ptac =
‹Attrib.thms >> (fn thms => fn ctxt => SIMPLE_METHOD' (Prolog.ptac ctxt thms))›
"basic Lambda Prolog interpreter"
method_setup prolog =
‹Attrib.thms >> (fn thms => fn ctxt => SIMPLE_METHOD (Prolog.prolog_tac ctxt thms))›
"Lambda Prolog interpreter"
syntax
"_Dand" :: "[bool, bool] => bool" (infixr ‹..› 28)
"_Dif" :: "[bool, bool] => bool" (infixl ‹:-› 29)
"_Dimp" :: "[bool, bool] => bool" (infixr ‹=>› 27)
translations
"D :- G" => "G --> D"
"D1 .. D2" => "D1 & D2"
"D => G" => "D --> G"
end