src/HOL/HOL.thy
changeset 22444 fb80fedd192d
parent 22377 61610b1beedf
child 22445 e4fd2d02391d
equal deleted inserted replaced
22443:346729a55460 22444:fb80fedd192d
   723 proof -
   723 proof -
   724   from 2 and 1 have P .
   724   from 2 and 1 have P .
   725   with 1 show R by (rule notE)
   725   with 1 show R by (rule notE)
   726 qed
   726 qed
   727 
   727 
   728 lemmas [Pure.elim!] = disjE iffE FalseE conjE exE
   728 lemma TrueE: "True ==> P ==> P" .
       
   729 lemma notFalseE: "~ False ==> P ==> P" .
       
   730 
       
   731 lemmas [Pure.elim!] = disjE iffE FalseE conjE exE TrueE notFalseE
   729   and [Pure.intro!] = iffI conjI impI TrueI notI allI refl
   732   and [Pure.intro!] = iffI conjI impI TrueI notI allI refl
   730   and [Pure.elim 2] = allE notE' impE'
   733   and [Pure.elim 2] = allE notE' impE'
   731   and [Pure.intro] = exI disjI2 disjI1
   734   and [Pure.intro] = exI disjI2 disjI1
   732 
   735 
   733 lemmas [trans] = trans
   736 lemmas [trans] = trans