src/Sequents/ILL_predlog.thy
changeset 80914 d97fdabd9e2b
parent 61386 0a29a984a91b
child 81213 d1170873976e
equal deleted inserted replaced
80913:46f59511b7bb 80914:d97fdabd9e2b
     3 begin
     3 begin
     4 
     4 
     5 typedecl plf
     5 typedecl plf
     6 
     6 
     7 consts
     7 consts
     8   conj :: "[plf,plf] \<Rightarrow> plf"   (infixr "&" 35)
     8   conj :: "[plf,plf] \<Rightarrow> plf"   (infixr \<open>&\<close> 35)
     9   disj :: "[plf,plf] \<Rightarrow> plf"   (infixr "|" 35)
     9   disj :: "[plf,plf] \<Rightarrow> plf"   (infixr \<open>|\<close> 35)
    10   impl :: "[plf,plf] \<Rightarrow> plf"   (infixr ">" 35)
    10   impl :: "[plf,plf] \<Rightarrow> plf"   (infixr \<open>>\<close> 35)
    11   eq :: "[plf,plf] \<Rightarrow> plf"   (infixr "=" 35)
    11   eq :: "[plf,plf] \<Rightarrow> plf"   (infixr \<open>=\<close> 35)
    12   ff :: "plf"    ("ff")
    12   ff :: "plf"    (\<open>ff\<close>)
    13 
    13 
    14   PL    :: "plf \<Rightarrow> o"      ("[* / _ / *]" [] 100)
    14   PL    :: "plf \<Rightarrow> o"      (\<open>[* / _ / *]\<close> [] 100)
    15 
    15 
    16 syntax
    16 syntax
    17   "_NG" :: "plf \<Rightarrow> plf"   ("- _ " [50] 55)
    17   "_NG" :: "plf \<Rightarrow> plf"   (\<open>- _ \<close> [50] 55)
    18 
    18 
    19 translations
    19 translations
    20   "[* A & B *]" \<rightleftharpoons> "[*A*] && [*B*]"
    20   "[* A & B *]" \<rightleftharpoons> "[*A*] && [*B*]"
    21   "[* A | B *]" \<rightleftharpoons> "![*A*] ++ ![*B*]"
    21   "[* A | B *]" \<rightleftharpoons> "![*A*] ++ ![*B*]"
    22   "[* - A *]" \<rightleftharpoons> "[*A > ff*]"
    22   "[* - A *]" \<rightleftharpoons> "[*A > ff*]"