src/Sequents/LK0.thy
changeset 35417 47ee18b6ae32
parent 35355 613e133966ea
parent 35416 d8d7d1b785af
child 36452 d37c6eed8117
equal deleted inserted replaced
35415:1810b1ade437 35417:47ee18b6ae32
   120   (*Descriptions*)
   120   (*Descriptions*)
   121 
   121 
   122   The: "[| $H |- $E, P(a), $F;  !!x.$H, P(x) |- $E, x=a, $F |] ==>
   122   The: "[| $H |- $E, P(a), $F;  !!x.$H, P(x) |- $E, x=a, $F |] ==>
   123           $H |- $E, P(THE x. P(x)), $F"
   123           $H |- $E, P(THE x. P(x)), $F"
   124 
   124 
   125 constdefs
   125 definition If :: "[o, 'a, 'a] => 'a" ("(if (_)/ then (_)/ else (_))" 10) where 
   126   If :: "[o, 'a, 'a] => 'a"   ("(if (_)/ then (_)/ else (_))" 10)
       
   127    "If(P,x,y) == THE z::'a. (P --> z=x) & (~P --> z=y)"
   126    "If(P,x,y) == THE z::'a. (P --> z=x) & (~P --> z=y)"
   128 
   127 
   129 
   128 
   130 (** Structural Rules on formulas **)
   129 (** Structural Rules on formulas **)
   131 
   130