Skip to content

Commit

Permalink
chore(topology/continuous_function/bounded): add an is_central_scalar…
Browse files Browse the repository at this point in the history
… instance (#12272)

This is only possible very recently now that `𝕜ᵐᵒᵖ` has a metric space instance.
  • Loading branch information
eric-wieser committed Feb 24, 2022
1 parent feb5473 commit f7518db
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/topology/continuous_function/bounded.lean
Expand Up @@ -834,6 +834,9 @@ instance : has_scalar 𝕜 (α →ᵇ β) :=
@[simp] lemma coe_smul (c : 𝕜) (f : α →ᵇ β) : ⇑(c • f) = λ x, c • (f x) := rfl
lemma smul_apply (c : 𝕜) (f : α →ᵇ β) (x : α) : (c • f) x = c • f x := rfl

instance [has_scalar 𝕜ᵐᵒᵖ β] [is_central_scalar 𝕜 β] : is_central_scalar 𝕜 (α →ᵇ β) :=
{ op_smul_eq_smul := λ _ _, ext $ λ _, op_smul_eq_smul _ _ }

instance : has_bounded_smul 𝕜 (α →ᵇ β) :=
{ dist_smul_pair' := λ c f₁ f₂, begin
rw dist_le (mul_nonneg dist_nonneg dist_nonneg),
Expand Down

0 comments on commit f7518db

Please sign in to comment.