src/HOL/Finite_Set.thy
changeset 49806 acb6fa98e310
parent 49764 9979d64b8016
parent 49756 28e37eab4e6f
child 51290 c48477e76de5
equal deleted inserted replaced
49805:9a2a53be24a2 49806:acb6fa98e310
  1755 subsubsection {* The image case with fixed function and idempotency *}
  1755 subsubsection {* The image case with fixed function and idempotency *}
  1756 
  1756 
  1757 locale folding_image_simple_idem = folding_image_simple +
  1757 locale folding_image_simple_idem = folding_image_simple +
  1758   assumes idem: "x * x = x"
  1758   assumes idem: "x * x = x"
  1759 
  1759 
  1760 sublocale folding_image_simple_idem < semilattice proof
  1760 sublocale folding_image_simple_idem < semilattice: semilattice proof
  1761 qed (fact idem)
  1761 qed (fact idem)
  1762 
  1762 
  1763 context folding_image_simple_idem
  1763 context folding_image_simple_idem
  1764 begin
  1764 begin
  1765 
  1765 
  1896 subsubsection {* The neutral-less case with idempotency *}
  1896 subsubsection {* The neutral-less case with idempotency *}
  1897 
  1897 
  1898 locale folding_one_idem = folding_one +
  1898 locale folding_one_idem = folding_one +
  1899   assumes idem: "x * x = x"
  1899   assumes idem: "x * x = x"
  1900 
  1900 
  1901 sublocale folding_one_idem < semilattice proof
  1901 sublocale folding_one_idem < semilattice: semilattice proof
  1902 qed (fact idem)
  1902 qed (fact idem)
  1903 
  1903 
  1904 context folding_one_idem
  1904 context folding_one_idem
  1905 begin
  1905 begin
  1906 
  1906