src/Sequents/ILL_predlog.thy
changeset 35252 24c466b2cdc8
parent 35054 a5db9779b026
child 35762 af3ff2ba4c54
--- a/src/Sequents/ILL_predlog.thy	Sun Feb 21 20:54:07 2010 +0100
+++ b/src/Sequents/ILL_predlog.thy	Sun Feb 21 20:54:40 2010 +0100
@@ -11,7 +11,7 @@
   disj :: "[plf,plf] => plf"   (infixr "|" 35)
   impl :: "[plf,plf] => plf"   (infixr ">" 35)
   eq :: "[plf,plf] => plf"   (infixr "=" 35)
-  ff    :: "plf"
+  ff :: "plf"    ("ff")
 
   PL    :: "plf => o"      ("[* / _ / *]" [] 100)
 
@@ -22,8 +22,8 @@
 
   "[* A & B *]" == "[*A*] && [*B*]"
   "[* A | B *]" == "![*A*] ++ ![*B*]"
-  "[* - A *]"   == "[*A > CONST ff*]"
-  "[* XCONST ff *]" == "0"
+  "[* - A *]" == "[*A > ff*]"
+  "[* ff *]" == "0"
   "[* A = B *]" => "[* (A > B) & (B > A) *]"
 
   "[* A > B *]" == "![*A*] -o [*B*]"