src/ZF/upair.thy
changeset 32960 69916a850301
parent 24893 b8ef7afe3a6b
child 45602 2a858377c3d2
equal deleted inserted replaced
32959:23a8c5ac35f8 32960:69916a850301
     1 (*  Title:      ZF/upair.thy
     1 (*  Title:      ZF/upair.thy
     2     ID:         $Id$
       
     3     Author:     Lawrence C Paulson and Martin D Coen, CU Computer Laboratory
     2     Author:     Lawrence C Paulson and Martin D Coen, CU Computer Laboratory
     4     Copyright   1993  University of Cambridge
     3     Copyright   1993  University of Cambridge
     5 
     4 
     6 Observe the order of dependence:
     5 Observe the order of dependence:
     7     Upair is defined in terms of Replace
     6     Upair is defined in terms of Replace
   224 lemma split_if [split]:
   223 lemma split_if [split]:
   225      "P(if Q then x else y) <-> ((Q --> P(x)) & (~Q --> P(y)))"
   224      "P(if Q then x else y) <-> ((Q --> P(x)) & (~Q --> P(y)))"
   226 by (case_tac Q, simp_all)
   225 by (case_tac Q, simp_all)
   227 
   226 
   228 (** Rewrite rules for boolean case-splitting: faster than 
   227 (** Rewrite rules for boolean case-splitting: faster than 
   229 	addsplits[split_if]
   228         addsplits[split_if]
   230 **)
   229 **)
   231 
   230 
   232 lemmas split_if_eq1 = split_if [of "%x. x = b", standard]
   231 lemmas split_if_eq1 = split_if [of "%x. x = b", standard]
   233 lemmas split_if_eq2 = split_if [of "%x. a = x", standard]
   232 lemmas split_if_eq2 = split_if [of "%x. a = x", standard]
   234 
   233