Skip to content

Commit

Permalink
chore(analysis/seminorm): Weaken typeclasses on convex and `locally…
Browse files Browse the repository at this point in the history
…_convex` lemmas (#12645)

Generalize type-classes `normed_linearly_ordered_field` to `normed_field` (otherwise it would not work over complex numbers).
  • Loading branch information
mcdoll committed Mar 15, 2022
1 parent 53f6d68 commit b7978f3
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions src/analysis/seminorm.lean
Expand Up @@ -559,8 +559,8 @@ set.ext $ λ _, by rw [mem_preimage, mem_ball, mem_ball,

end normed_field

section normed_linear_ordered_field
variables [normed_linear_ordered_field 𝕜] [add_comm_group E] [normed_space ℝ 𝕜] [module 𝕜 E]
section convex
variables [normed_field 𝕜] [add_comm_group E] [normed_space ℝ 𝕜] [module 𝕜 E]

section has_scalar
variables [has_scalar ℝ E] [is_scalar_tower ℝ 𝕜 E] (p : seminorm 𝕜 E)
Expand Down Expand Up @@ -592,7 +592,7 @@ begin
end

end module
end normed_linear_ordered_field
end convex
end seminorm

/-! ### The norm as a seminorm -/
Expand Down Expand Up @@ -933,7 +933,7 @@ section locally_convex_space

open locally_convex_space

variables [nonempty ι] [normed_linear_ordered_field 𝕜] [normed_space ℝ 𝕜]
variables [nonempty ι] [normed_field 𝕜] [normed_space ℝ 𝕜]
[add_comm_group E] [module 𝕜 E] [module ℝ E] [is_scalar_tower ℝ 𝕜 E] [topological_space E]
[topological_add_group E]

Expand All @@ -956,7 +956,7 @@ end seminorm

section normed_space

variables (𝕜) [normed_linear_ordered_field 𝕜] [normed_space ℝ 𝕜] [semi_normed_group E]
variables (𝕜) [normed_field 𝕜] [normed_space ℝ 𝕜] [semi_normed_group E]

/-- Not an instance since `𝕜` can't be inferred. See `normed_space.to_locally_convex_space` for a
slightly weaker instance version. -/
Expand Down

0 comments on commit b7978f3

Please sign in to comment.