src/HOL/Modelcheck/MuckeSyn.thy
changeset 14854 61bdf2ae4dc5
parent 12662 a9bbba3473f3
child 17272 c63e5220ed77
equal deleted inserted replaced
14853:8d710bece29f 14854:61bdf2ae4dc5
    30   "! " 		:: [idts, bool] => bool			("'((3forall _./ _)')" [0, 10] 10)
    30   "! " 		:: [idts, bool] => bool			("'((3forall _./ _)')" [0, 10] 10)
    31   "? "		:: [idts, bool] => bool			("'((3exists _./ _)')" [0, 10] 10)
    31   "? "		:: [idts, bool] => bool			("'((3exists _./ _)')" [0, 10] 10)
    32   "ALL "        :: [idts, bool] => bool                 ("'((3forall _./ _)')" [0, 10] 10)
    32   "ALL "        :: [idts, bool] => bool                 ("'((3forall _./ _)')" [0, 10] 10)
    33   "EX "         :: [idts, bool] => bool                 ("'((3exists _./ _)')" [0, 10] 10)
    33   "EX "         :: [idts, bool] => bool                 ("'((3exists _./ _)')" [0, 10] 10)
    34 
    34 
    35   "_lambda"	:: [idts, 'a::logic] => 'b::logic	("(3L _./ _)" 10)
    35   "_lambda"	:: [idts, 'a] => 'b  			("(3L _./ _)" 10)
    36   "_applC"	:: [('b => 'a), cargs] => aprop		("(1_/ '(_'))" [1000,1000] 999)
    36   "_applC"	:: [('b => 'a), cargs] => aprop		("(1_/ '(_'))" [1000,1000] 999)
    37   "_cargs" 	:: ['a, cargs] => cargs         	("_,/ _" [1000,1000] 1000)
    37   "_cargs" 	:: ['a, cargs] => cargs         	("_,/ _" [1000,1000] 1000)
    38 
    38 
    39   "_idts"     	:: [idt, idts] => idts		        ("_,/ _" [1, 0] 0)
    39   "_idts"     	:: [idt, idts] => idts		        ("_,/ _" [1, 0] 0)
    40 
    40