doc-src/ZF/If.thy
changeset 19792 e8e3da6d3ff7
parent 16417 9bc16273c2d4
child 35416 d8d7d1b785af
equal deleted inserted replaced
19791:ab326de16ad5 19792:e8e3da6d3ff7
     7 *)
     7 *)
     8 
     8 
     9 theory If imports FOL begin
     9 theory If imports FOL begin
    10 
    10 
    11 constdefs
    11 constdefs
    12   if :: "[o,o,o]=>o"
    12   "if" :: "[o,o,o]=>o"
    13    "if(P,Q,R) == P&Q | ~P&R"
    13   "if(P,Q,R) == P&Q | ~P&R"
    14 
    14 
    15 lemma ifI:
    15 lemma ifI:
    16     "[| P ==> Q; ~P ==> R |] ==> if(P,Q,R)"
    16     "[| P ==> Q; ~P ==> R |] ==> if(P,Q,R)"
    17   --{* @{subgoals[display,indent=0,margin=65]} *}
    17   --{* @{subgoals[display,indent=0,margin=65]} *}
    18 apply (simp add: if_def)
    18 apply (simp add: if_def)