src/HOL/Finite.ML
changeset 9736 332fab43628f
parent 9421 d8dfa816a368
child 9837 7b26f2d51ba4
equal deleted inserted replaced
9735:203e5552496b 9736:332fab43628f
   568 by (asm_simp_tac (simpset() addsimps [f_lcomm]) 1);
   568 by (asm_simp_tac (simpset() addsimps [f_lcomm]) 1);
   569 val lemma = result();
   569 val lemma = result();
   570 
   570 
   571 
   571 
   572 Goal "[| (A, x) : foldSet f e;  (A, y) : foldSet f e |] ==> y=x";
   572 Goal "[| (A, x) : foldSet f e;  (A, y) : foldSet f e |] ==> y=x";
   573 by (blast_tac (claset() addIs [normalize_thm [RSspec, RSmp] lemma]) 1);
   573 by (blast_tac (claset() addIs [rulify lemma]) 1);
   574 qed "foldSet_determ";
   574 qed "foldSet_determ";
   575 
   575 
   576 Goalw [fold_def] "(A,y) : foldSet f e ==> fold f e A = y";
   576 Goalw [fold_def] "(A,y) : foldSet f e ==> fold f e A = y";
   577 by (blast_tac (claset() addIs [foldSet_determ]) 1);
   577 by (blast_tac (claset() addIs [foldSet_determ]) 1);
   578 qed "fold_equality";
   578 qed "fold_equality";