src/ZF/equalities.ML
changeset 6068 2d8f3e1f1151
parent 5325 f7a5e06adea1
child 6288 694c9c1910e8
equal deleted inserted replaced
6067:0f8ab32093ae 6068:2d8f3e1f1151
   600 
   600 
   601 Goal "Collect(A - B, P) = Collect(A,P) - Collect(B,P)";
   601 Goal "Collect(A - B, P) = Collect(A,P) - Collect(B,P)";
   602 by (Blast_tac 1);
   602 by (Blast_tac 1);
   603 qed "Collect_Diff";
   603 qed "Collect_Diff";
   604 
   604 
   605 Goal "{x:cons(a,B). P(x)} = if(P(a), cons(a, {x:B. P(x)}), {x:B. P(x)})";
   605 Goal "{x:cons(a,B). P(x)} = \
       
   606 \     (if P(a) then cons(a, {x:B. P(x)}) else {x:B. P(x)})";
   606 by (simp_tac (simpset() addsplits [split_if]) 1);
   607 by (simp_tac (simpset() addsplits [split_if]) 1);
   607 by (Blast_tac 1);
   608 by (Blast_tac 1);
   608 qed "Collect_cons";
   609 qed "Collect_cons";
   609 
   610