src/HOL/Finite.ML
changeset 6024 cb87f103d114
parent 5782 7559f116cb10
child 6141 a6922171b396
equal deleted inserted replaced
6023:832b9269dedd 6024:cb87f103d114
   673 (* Delete rules to do with foldSet relation: obsolete *)
   673 (* Delete rules to do with foldSet relation: obsolete *)
   674 Delsimps [foldSet_imp_finite];
   674 Delsimps [foldSet_imp_finite];
   675 Delrules [empty_foldSetE];
   675 Delrules [empty_foldSetE];
   676 Delrules foldSet.intrs;
   676 Delrules foldSet.intrs;
   677 
   677 
   678 Close_locale();
   678 Close_locale "LC";
   679 
   679 
   680 Open_locale "ACe"; 
   680 Open_locale "ACe"; 
   681 
   681 
   682 val f_ident   = thm "ident";
   682 val f_ident   = thm "ident";
   683 val f_commute = thm "commute";
   683 val f_commute = thm "commute";
   720 by (simp_tac (simpset() addsimps f_idents) 1);
   720 by (simp_tac (simpset() addsimps f_idents) 1);
   721 by (asm_full_simp_tac (simpset() addsimps f_ac @ f_idents @
   721 by (asm_full_simp_tac (simpset() addsimps f_ac @ f_idents @
   722            [export fold_insert,insert_absorb, Int_insert_left]) 1);
   722            [export fold_insert,insert_absorb, Int_insert_left]) 1);
   723 qed "fold_Un_disjoint2";
   723 qed "fold_Un_disjoint2";
   724 
   724 
   725 Close_locale();
   725 Close_locale "ACe";
   726 
   726 
   727 Delrules ([empty_foldSetE] @ foldSet.intrs);
   727 Delrules ([empty_foldSetE] @ foldSet.intrs);
   728 Delsimps [foldSet_imp_finite];
   728 Delsimps [foldSet_imp_finite];
   729 
   729 
   730 (*** setsum ***)
   730 (*** setsum ***)