src/FOL/IFOL.thy
changeset 52230 1105b3b5aa77
parent 51798 ad3a241def73
child 52241 5f6e885382e9
equal deleted inserted replaced
52228:ee8e3eaad24c 52230:1105b3b5aa77
   222    apply (erule impI)
   222    apply (erule impI)
   223   apply (erule impI)
   223   apply (erule impI)
   224   done
   224   done
   225 
   225 
   226 
   226 
   227 (*Observe use of rewrite_rule to unfold "<->" in meta-assumptions (prems) *)
       
   228 lemma iffE:
   227 lemma iffE:
   229   assumes major: "P <-> Q"
   228   assumes major: "P <-> Q"
   230     and r: "P-->Q ==> Q-->P ==> R"
   229     and r: "P-->Q ==> Q-->P ==> R"
   231   shows R
   230   shows R
   232   apply (insert major, unfold iff_def)
   231   apply (insert major, unfold iff_def)