equal
deleted
inserted
replaced
226 Addsimps[Un_UNIV_right]; |
226 Addsimps[Un_UNIV_right]; |
227 |
227 |
228 goal Set.thy "(insert a B) Un C = insert a (B Un C)"; |
228 goal Set.thy "(insert a B) Un C = insert a (B Un C)"; |
229 by (Blast_tac 1); |
229 by (Blast_tac 1); |
230 qed "Un_insert_left"; |
230 qed "Un_insert_left"; |
|
231 Addsimps[Un_insert_left]; |
231 |
232 |
232 goal Set.thy "A Un (insert a B) = insert a (A Un B)"; |
233 goal Set.thy "A Un (insert a B) = insert a (A Un B)"; |
233 by (Blast_tac 1); |
234 by (Blast_tac 1); |
234 qed "Un_insert_right"; |
235 qed "Un_insert_right"; |
|
236 Addsimps[Un_insert_right]; |
235 |
237 |
236 goal Set.thy "(insert a B) Int C = (if a:C then insert a (B Int C) \ |
238 goal Set.thy "(insert a B) Int C = (if a:C then insert a (B Int C) \ |
237 \ else B Int C)"; |
239 \ else B Int C)"; |
238 by (simp_tac (!simpset setloop split_tac [expand_if]) 1); |
240 by (simp_tac (!simpset setloop split_tac [expand_if]) 1); |
239 by (Blast_tac 1); |
241 by (Blast_tac 1); |