Skip to content

Commit

Permalink
feat(algebra/module/pointwise_pi): add a file with lemmas on smul_pi (#…
Browse files Browse the repository at this point in the history
…9369)

Make a new file rather than add an import to either of `algebra.pointwise` or `algebra.module.pi`.

From #2819
  • Loading branch information
alexjbest committed Sep 26, 2021
1 parent b3ca07f commit 865ad47
Showing 1 changed file with 50 additions and 0 deletions.
50 changes: 50 additions & 0 deletions src/algebra/module/pointwise_pi.lean
@@ -0,0 +1,50 @@
/-
Copyright (c) 2021 Alex J. Best. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Alex J. Best
-/
import algebra.pointwise
import algebra.module.pi

/-!
# Pointwise actions on sets in Pi types
This file contains lemmas about pointwise actions on sets in Pi types.
## Tags
set multiplication, set addition, pointwise addition, pointwise multiplication, pi
-/

open_locale pointwise
open set

variables {K ι : Type*} {R : ι → Type*}

@[to_additive]
lemma smul_pi_subset [∀ i, has_scalar K (R i)] (r : K) (s : set ι) (t : Π i, set (R i)) :
r • pi s t ⊆ pi s (r • t) :=
begin
rintros x ⟨y, h, rfl⟩ i hi,
exact smul_mem_smul_set (h i hi),
end

@[to_additive]
lemma smul_univ_pi [∀ i, has_scalar K (R i)] (r : K) (t : Π i, set (R i)) :
r • pi (univ : set ι) t = pi (univ : set ι) (r • t) :=
subset.antisymm (smul_pi_subset _ _ _) $ λ x h, begin
refine ⟨λ i, classical.some (h i $ set.mem_univ _), λ i hi, _, funext $ λ i, _⟩,
{ exact (classical.some_spec (h i _)).left, },
{ exact (classical.some_spec (h i _)).right, },
end

@[to_additive]
lemma smul_pi [group K] [∀ i, mul_action K (R i)] (r : K) (S : set ι) (t : Π i, set (R i)) :
r • S.pi t = S.pi (r • t) :=
subset.antisymm (smul_pi_subset _ _ _) $ λ x h,
⟨r⁻¹ • x, λ i hiS, mem_smul_set_iff_inv_smul_mem.mp (h i hiS), smul_inv_smul _ _⟩

lemma smul_pi' [group_with_zero K] [∀ i, mul_action K (R i)] {r : K} (S : set ι)
(t : Π i, set (R i)) (hr : r ≠ 0) : r • S.pi t = S.pi (r • t) :=
smul_pi (units.mk0 r hr) S t

0 comments on commit 865ad47

Please sign in to comment.