src/Sequents/ILL/ILL_predlog.thy
author wenzelm
Tue, 30 May 2000 16:08:38 +0200
changeset 9000 c20d58286a51
parent 6252 935f183bf406
child 14854 61bdf2ae4dc5
permissions -rw-r--r--
cleaned up;

(* 
    File:	 /Nfs/toton/usr20/sk/isa_files/ll/NEW/pred_log.thy
    Theory Name: pred_log
    Logic Image: HOL
*)

ILL_predlog  =  ILL +

types

    plf
    
arities

    plf :: logic
    
consts

  "&"   :: "[plf,plf] => plf"   (infixr 35)
  "|"   :: "[plf,plf] => plf"   (infixr 35)
  ">"   :: "[plf,plf] => plf"   (infixr 35)
  "="   :: "[plf,plf] => plf"   (infixr 35)
  "@NG" :: "plf => plf"   ("- _ " [50] 55)
  ff    :: "plf"
  
  PL    :: "plf => o"      ("[* / _ / *]" [] 100)


translations

  "[* A & B *]" == "[*A*] && [*B*]" 
  "[* A | B *]" == "![*A*] ++ ![*B*]"
  "[* - A *]"   == "[*A > ff*]"
  "[* ff *]"    == "0"
  "[* A = B *]" => "[* (A > B) & (B > A) *]"
  
  "[* A > B *]" == "![*A*] -o [*B*]"
  
(* another translations for linear implication:
  "[* A > B *]" == "!([*A*] -o [*B*])" *)

end