Skip to content

Commit

Permalink
Balanced.mulActionHom_preimage
Browse files Browse the repository at this point in the history
  • Loading branch information
mans0954 committed Jan 22, 2025
1 parent 461b0d5 commit eb50959
Showing 1 changed file with 6 additions and 1 deletion.
7 changes: 6 additions & 1 deletion Mathlib/Analysis/LocallyConvex/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -42,7 +42,7 @@ open Set

open Pointwise Topology

variable {π•œ 𝕝 E : Type*} {ΞΉ : Sort*} {ΞΊ : ΞΉ β†’ Sort*}
variable {π•œ 𝕝 E F : Type*} {ΞΉ : Sort*} {ΞΊ : ΞΉ β†’ Sort*}

section SeminormedRing

Expand Down Expand Up @@ -105,6 +105,11 @@ theorem balanced_iInterβ‚‚ {f : βˆ€ i, ΞΊ i β†’ Set E} (h : βˆ€ i j, Balanced
Balanced π•œ (β‹‚ (i) (j), f i j) :=
balanced_iInter fun _ => balanced_iInter <| h _

theorem Balanced.mulActionHom_preimage [SMul π•œ F] {s : Set F} (hs : Balanced π•œ s)
(f : MulActionHom (RingHom.id π•œ) E F) : Balanced π•œ (f ⁻¹' s) := fun a ha x ⟨y,⟨hy₁,hyβ‚‚βŸ©βŸ© => by
rw [mem_preimage, ← hyβ‚‚, map_smul]
exact hs a ha (smul_mem_smul_set hy₁)

variable [SMul 𝕝 E] [SMulCommClass π•œ 𝕝 E]

theorem Balanced.smul (a : 𝕝) (hs : Balanced π•œ s) : Balanced π•œ (a β€’ s) := fun _b hb =>
Expand Down

0 comments on commit eb50959

Please sign in to comment.