src/FOL/IFOL.thy
changeset 18813 fc35dcc2558b
parent 18708 4b3dadb4fe33
child 18861 38269ef5175a
equal deleted inserted replaced
18812:a4554848b59e 18813:fc35dcc2558b
   237 next
   237 next
   238   assume "x = y"
   238   assume "x = y"
   239   thus "x == y" by (rule eq_reflection)
   239   thus "x == y" by (rule eq_reflection)
   240 qed
   240 qed
   241 
   241 
       
   242 lemma atomize_iff [atomize]: "(A == B) == Trueprop (A <-> B)"
       
   243 proof
       
   244   assume "A == B"
       
   245   show "A <-> B" by (unfold prems) (rule iff_refl)
       
   246 next
       
   247   assume "A <-> B"
       
   248   thus "A == B" by (rule iff_reflection)
       
   249 qed
       
   250 
   242 lemma atomize_conj [atomize]:
   251 lemma atomize_conj [atomize]:
   243   "(!!C. (A ==> B ==> PROP C) ==> PROP C) == Trueprop (A & B)"
   252   "(!!C. (A ==> B ==> PROP C) ==> PROP C) == Trueprop (A & B)"
   244 proof
   253 proof
   245   assume "!!C. (A ==> B ==> PROP C) ==> PROP C"
   254   assume "!!C. (A ==> B ==> PROP C) ==> PROP C"
   246   show "A & B" by (rule conjI)
   255   show "A & B" by (rule conjI)