equal
deleted
inserted
replaced
280 qed |
280 qed |
281 |
281 |
282 lemma finite_deflation_ssum_map: |
282 lemma finite_deflation_ssum_map: |
283 assumes "finite_deflation d1" and "finite_deflation d2" |
283 assumes "finite_deflation d1" and "finite_deflation d2" |
284 shows "finite_deflation (ssum_map\<cdot>d1\<cdot>d2)" |
284 shows "finite_deflation (ssum_map\<cdot>d1\<cdot>d2)" |
285 proof (intro finite_deflation.intro finite_deflation_axioms.intro) |
285 proof (rule finite_deflation_intro) |
286 interpret d1: finite_deflation d1 by fact |
286 interpret d1: finite_deflation d1 by fact |
287 interpret d2: finite_deflation d2 by fact |
287 interpret d2: finite_deflation d2 by fact |
288 have "deflation d1" and "deflation d2" by fact+ |
288 have "deflation d1" and "deflation d2" by fact+ |
289 thus "deflation (ssum_map\<cdot>d1\<cdot>d2)" by (rule deflation_ssum_map) |
289 thus "deflation (ssum_map\<cdot>d1\<cdot>d2)" by (rule deflation_ssum_map) |
290 have "{x. ssum_map\<cdot>d1\<cdot>d2\<cdot>x = x} \<subseteq> |
290 have "{x. ssum_map\<cdot>d1\<cdot>d2\<cdot>x = x} \<subseteq> |