Skip to content

Commit

Permalink
chore(data/finset/pointwise): {a} • t = a • t (#17072)
Browse files Browse the repository at this point in the history
Change `singleton_smul` so that it uses the `•` spelling on the RHS.
  • Loading branch information
YaelDillies committed Oct 23, 2022
1 parent 3798ca1 commit a2a1963
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/data/finset/pointwise.lean
Expand Up @@ -659,9 +659,7 @@ nonempty.of_image₂_left
nonempty.of_image₂_right
@[to_additive] lemma smul_singleton (b : β) : s • ({b} : finset β) = s.image (• b) :=
image₂_singleton_right
@[to_additive] lemma singleton_smul (a : α) : ({a} : finset α) • t = t.image ((•) a) :=
image₂_singleton_left
@[simp, to_additive] lemma singleton_smul_singleton (a : α) (b : β) :
@[to_additive] lemma singleton_smul_singleton (a : α) (b : β) :
({a} : finset α) • ({b} : finset β) = {a • b} :=
image₂_singleton

Expand Down Expand Up @@ -782,6 +780,8 @@ lemma coe_smul_finset (a : α) (s : finset β) : (↑(a • s) : set β) = a •
@[simp, to_additive] lemma smul_finset_nonempty : (a • s).nonempty ↔ s.nonempty :=
nonempty.image_iff _
@[to_additive] lemma nonempty.smul_finset (hs : s.nonempty) : (a • s).nonempty := hs.image _
@[simp, to_additive] lemma singleton_smul (a : α) : ({a} : finset α) • t = a • t :=
image₂_singleton_left

@[to_additive, mono]
lemma smul_finset_subset_smul_finset : s ⊆ t → a • s ⊆ a • t := image_subset_image
Expand Down

0 comments on commit a2a1963

Please sign in to comment.