src/HOL/Set.ML
changeset 4135 4830f1f5f6ea
parent 4089 96fba19bcbe2
child 4159 4aff9b7e5597
equal deleted inserted replaced
4134:5c6cb2a25816 4135:4830f1f5f6ea
   231   [ (blast_tac (claset() addIs [prem RS FalseE]) 1) ]);
   231   [ (blast_tac (claset() addIs [prem RS FalseE]) 1) ]);
   232 
   232 
   233 qed_goal "equals0D" Set.thy "!!a. [| A={};  a:A |] ==> P"
   233 qed_goal "equals0D" Set.thy "!!a. [| A={};  a:A |] ==> P"
   234  (fn _ => [ (Blast_tac 1) ]);
   234  (fn _ => [ (Blast_tac 1) ]);
   235 
   235 
   236 goal Set.thy "Ball {} P = True";
       
   237 by (simp_tac (HOL_ss addsimps [mem_Collect_eq, Ball_def, empty_def]) 1);
       
   238 qed "ball_empty";
       
   239 
       
   240 goal Set.thy "Bex {} P = False";
       
   241 by (simp_tac (HOL_ss addsimps [mem_Collect_eq, Bex_def, empty_def]) 1);
       
   242 qed "bex_empty";
       
   243 Addsimps [ball_empty, bex_empty];
       
   244 
       
   245 
   236 
   246 section "The Powerset operator -- Pow";
   237 section "The Powerset operator -- Pow";
   247 
   238 
   248 qed_goalw "Pow_iff" Set.thy [Pow_def] "(A : Pow(B)) = (A <= B)"
   239 qed_goalw "Pow_iff" Set.thy [Pow_def] "(A : Pow(B)) = (A <= B)"
   249  (fn _ => [ (Asm_simp_tac 1) ]);
   240  (fn _ => [ (Asm_simp_tac 1) ]);