Skip to content

Commit

Permalink
bump to nightly-2023-04-06-10
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Apr 6, 2023
1 parent a30809a commit 678d4ff
Show file tree
Hide file tree
Showing 11 changed files with 205 additions and 57 deletions.
6 changes: 3 additions & 3 deletions Mathbin/Analysis/LocallyConvex/AbsConvex.lean
Expand Up @@ -167,9 +167,9 @@ variable [TopologicalAddGroup E] [ContinuousSMul π•œ E]
variable [SMulCommClass ℝ π•œ E] [LocallyConvexSpace ℝ E]

/-- The topology of a locally convex space is induced by the gauge seminorm family. -/
theorem withGaugeSeminormFamily : WithSeminorms (gaugeSeminormFamily π•œ E) :=
theorem with_gaugeSeminormFamily : WithSeminorms (gaugeSeminormFamily π•œ E) :=
by
refine' SeminormFamily.withSeminormsOfHasBasis _ _
refine' SeminormFamily.withSeminorms_of_hasBasis _ _
refine' (nhds_basis_abs_convex_open π•œ E).to_hasBasis (fun s hs => _) fun s hs => _
· refine' ⟨s, ⟨_, rfl.subset⟩⟩
convert(gaugeSeminormFamily _ _).basisSets_singleton_mem ⟨s, hs⟩ one_pos
Expand All @@ -189,5 +189,5 @@ theorem withGaugeSeminormFamily : WithSeminorms (gaugeSeminormFamily π•œ E) :=
have hr'' : (r : π•œ) β‰  0 := by simp [hr.ne']
rw [hr', ← Seminorm.smul_ball_zero hr'', gaugeSeminormFamily_ball]
exact S.coe_is_open.smulβ‚€ hr''
#align with_gauge_seminorm_family withGaugeSeminormFamily
#align with_gauge_seminorm_family with_gaugeSeminormFamily

8 changes: 4 additions & 4 deletions Mathbin/Analysis/LocallyConvex/WeakDual.lean
Expand Up @@ -145,10 +145,10 @@ theorem LinearMap.hasBasis_weakBilin (B : E β†’β‚—[π•œ] F β†’β‚—[π•œ] π•œ) :
exact hx y hy
#align linear_map.has_basis_weak_bilin LinearMap.hasBasis_weakBilin

theorem LinearMap.weakBilinWithSeminorms (B : E β†’β‚—[π•œ] F β†’β‚—[π•œ] π•œ) :
theorem LinearMap.weakBilin_withSeminorms (B : E β†’β‚—[π•œ] F β†’β‚—[π•œ] π•œ) :
WithSeminorms (LinearMap.toSeminormFamily B : F β†’ Seminorm π•œ (WeakBilin B)) :=
SeminormFamily.withSeminormsOfHasBasis _ B.hasBasis_weakBilin
#align linear_map.weak_bilin_with_seminorms LinearMap.weakBilinWithSeminorms
SeminormFamily.withSeminorms_of_hasBasis _ B.hasBasis_weakBilin
#align linear_map.weak_bilin_with_seminorms LinearMap.weakBilin_withSeminorms

end Topology

Expand All @@ -159,7 +159,7 @@ variable [NormedField π•œ] [AddCommGroup E] [Module π•œ E] [AddCommGroup F] [M
variable [Nonempty ΞΉ] [NormedSpace ℝ π•œ] [Module ℝ E] [IsScalarTower ℝ π•œ E]

instance {B : E β†’β‚—[π•œ] F β†’β‚—[π•œ] π•œ} : LocallyConvexSpace ℝ (WeakBilin B) :=
B.weakBilinWithSeminorms.toLocallyConvexSpace
B.weakBilin_withSeminorms.toLocallyConvexSpace

end LocallyConvex

28 changes: 14 additions & 14 deletions Mathbin/Analysis/LocallyConvex/WithSeminorms.lean
Expand Up @@ -298,7 +298,7 @@ variable {p : SeminormFamily π•œ E ΞΉ}
theorem WithSeminorms.topologicalAddGroup (hp : WithSeminorms p) : TopologicalAddGroup E :=
by
rw [hp.with_seminorms_eq]
exact AddGroupFilterBasis.is_topological_add_group _
exact AddGroupFilterBasis.isTopologicalAddGroup _
#align with_seminorms.topological_add_group WithSeminorms.topologicalAddGroup

theorem WithSeminorms.hasBasis (hp : WithSeminorms p) :
Expand Down Expand Up @@ -432,20 +432,20 @@ variable [Nonempty ΞΉ]

include t

theorem SeminormFamily.withSeminormsOfNhds (p : SeminormFamily π•œ E ΞΉ)
theorem SeminormFamily.withSeminorms_of_nhds (p : SeminormFamily π•œ E ΞΉ)
(h : 𝓝 (0 : E) = p.ModuleFilterBasis.toFilterBasis.filterβ‚“) : WithSeminorms p :=
by
refine'
⟨TopologicalAddGroup.ext inferInstance p.add_group_filter_basis.is_topological_add_group _⟩
rw [AddGroupFilterBasis.nhds_zero_eq]
exact h
#align seminorm_family.with_seminorms_of_nhds SeminormFamily.withSeminormsOfNhds
#align seminorm_family.with_seminorms_of_nhds SeminormFamily.withSeminorms_of_nhds

theorem SeminormFamily.withSeminormsOfHasBasis (p : SeminormFamily π•œ E ΞΉ)
theorem SeminormFamily.withSeminorms_of_hasBasis (p : SeminormFamily π•œ E ΞΉ)
(h : (𝓝 (0 : E)).HasBasis (fun s : Set E => s ∈ p.basis_sets) id) : WithSeminorms p :=
p.withSeminormsOfNhds <|
p.withSeminorms_of_nhds <|
Filter.HasBasis.eq_of_same_basis h p.AddGroupFilterBasis.toFilterBasis.HasBasis
#align seminorm_family.with_seminorms_of_has_basis SeminormFamily.withSeminormsOfHasBasis
#align seminorm_family.with_seminorms_of_has_basis SeminormFamily.withSeminorms_of_hasBasis

theorem SeminormFamily.withSeminorms_iff_nhds_eq_infα΅’ (p : SeminormFamily π•œ E ΞΉ) :
WithSeminorms p ↔ (𝓝 0 : Filter E) = β¨… i, (𝓝 0).comap (p i) :=
Expand Down Expand Up @@ -505,7 +505,7 @@ end TopologicalAddGroup
section NormedSpace

/-- The topology of a `normed_space π•œ E` is induced by the seminorm `norm_seminorm π•œ E`. -/
theorem normWithSeminorms (π•œ E) [NormedField π•œ] [SeminormedAddCommGroup E] [NormedSpace π•œ E] :
theorem norm_withSeminorms (π•œ E) [NormedField π•œ] [SeminormedAddCommGroup E] [NormedSpace π•œ E] :
WithSeminorms fun _ : Fin 1 => normSeminorm π•œ E :=
by
let p : SeminormFamily π•œ E (Fin 1) := fun _ => normSeminorm π•œ E
Expand All @@ -525,7 +525,7 @@ theorem normWithSeminorms (π•œ E) [NormedField π•œ] [SeminormedAddCommGroup E]
Β· rw [Finset.sup_const h]
rw [finset.not_nonempty_iff_eq_empty.mp h, Finset.sup_empty, ball_bot _ hr]
exact Set.subset_univ _
#align norm_with_seminorms normWithSeminorms
#align norm_with_seminorms norm_withSeminorms

end NormedSpace

Expand Down Expand Up @@ -661,15 +661,15 @@ theorem cont_withSeminorms_normedSpace (F) [SeminormedAddCommGroup F] [NormedSpa
(f : E β†’β‚›β‚—[τ₁₂] F) (hf : βˆƒ (s : Finset ΞΉ)(C : ℝβ‰₯0), (normSeminorm 𝕝₂ F).comp f ≀ C β€’ s.sup p) :
Continuous f := by
rw [← Seminorm.isBounded_const (Fin 1)] at hf
exact continuous_from_bounded hp (normWithSeminorms 𝕝₂ F) f hf
exact continuous_from_bounded hp (norm_withSeminorms 𝕝₂ F) f hf
#align seminorm.cont_with_seminorms_normed_space Seminorm.cont_withSeminorms_normedSpace

theorem cont_normedSpace_to_withSeminorms (E) [SeminormedAddCommGroup E] [NormedSpace 𝕝 E]
[UniformSpace F] [UniformAddGroup F] {q : ΞΉ β†’ Seminorm 𝕝₂ F} (hq : WithSeminorms q)
(f : E β†’β‚›β‚—[τ₁₂] F) (hf : βˆ€ i : ΞΉ, βˆƒ C : ℝβ‰₯0, (q i).comp f ≀ C β€’ normSeminorm 𝕝 E) :
Continuous f := by
rw [← Seminorm.const_isBounded (Fin 1)] at hf
exact continuous_from_bounded (normWithSeminorms 𝕝 E) hq f hf
exact continuous_from_bounded (norm_withSeminorms 𝕝 E) hq f hf
#align seminorm.cont_normed_space_to_with_seminorms Seminorm.cont_normedSpace_to_withSeminorms

end Seminorm
Expand All @@ -687,7 +687,7 @@ theorem WithSeminorms.toLocallyConvexSpace {p : SeminormFamily π•œ E ΞΉ} (hp :
LocallyConvexSpace ℝ E :=
by
apply of_basis_zero ℝ E id fun s => s ∈ p.basis_sets
Β· rw [hp.1, AddGroupFilterBasis.nhds_eq _, AddGroupFilterBasis.n_zero]
Β· rw [hp.1, AddGroupFilterBasis.nhds_eq _, AddGroupFilterBasis.N_zero]
exact FilterBasis.hasBasis _
Β· intro s hs
change s ∈ Set.unionᡒ _ at hs
Expand All @@ -706,7 +706,7 @@ variable (π•œ) [NormedField π•œ] [NormedSpace ℝ π•œ] [SeminormedAddCommGrou
slightly weaker instance version. -/
theorem NormedSpace.toLocallyConvexSpace' [NormedSpace π•œ E] [Module ℝ E] [IsScalarTower ℝ π•œ E] :
LocallyConvexSpace ℝ E :=
(normWithSeminorms π•œ E).toLocallyConvexSpace
(norm_withSeminorms π•œ E).toLocallyConvexSpace
#align normed_space.to_locally_convex_space' NormedSpace.toLocallyConvexSpace'

/-- See `normed_space.to_locally_convex_space'` for a slightly stronger version which is not an
Expand Down Expand Up @@ -745,7 +745,7 @@ theorem SeminormFamily.finset_sup_comp (q : SeminormFamily π•œβ‚‚ F ΞΉ) (s : Fi

variable [TopologicalSpace F] [TopologicalAddGroup F]

theorem LinearMap.withSeminormsInduced [hΞΉ : Nonempty ΞΉ] {q : SeminormFamily π•œβ‚‚ F ΞΉ}
theorem LinearMap.withSeminorms_induced [hΞΉ : Nonempty ΞΉ] {q : SeminormFamily π•œβ‚‚ F ΞΉ}
(hq : WithSeminorms q) (f : E β†’β‚›β‚—[σ₁₂] F) :
@WithSeminorms π•œ E ΞΉ _ _ _ _ (q.comp f) (induced f inferInstance) :=
by
Expand All @@ -755,7 +755,7 @@ theorem LinearMap.withSeminormsInduced [hΞΉ : Nonempty ΞΉ] {q : SeminormFamily
q.with_seminorms_iff_nhds_eq_infi.mp hq, Filter.comap_infα΅’]
refine' infα΅’_congr fun i => _
exact Filter.comap_comap
#align linear_map.with_seminorms_induced LinearMap.withSeminormsInduced
#align linear_map.with_seminorms_induced LinearMap.withSeminorms_induced

theorem Inducing.withSeminorms [hΞΉ : Nonempty ΞΉ] {q : SeminormFamily π•œβ‚‚ F ΞΉ} (hq : WithSeminorms q)
[TopologicalSpace E] {f : E β†’β‚›β‚—[σ₁₂] F} (hf : Inducing f) : WithSeminorms (q.comp f) :=
Expand Down
20 changes: 10 additions & 10 deletions Mathbin/Analysis/SchwartzSpace.lean
Expand Up @@ -504,23 +504,23 @@ theorem schwartzSeminormFamily_apply_zero :
instance : TopologicalSpace 𝓒(E, F) :=
(schwartzSeminormFamily ℝ E F).ModuleFilterBasis.topology'

theorem schwartzWithSeminorms : WithSeminorms (schwartzSeminormFamily π•œ E F) :=
theorem schwartz_withSeminorms : WithSeminorms (schwartzSeminormFamily π•œ E F) :=
by
have A : WithSeminorms (schwartzSeminormFamily ℝ E F) := ⟨rfl⟩
rw [SeminormFamily.withSeminorms_iff_nhds_eq_infᡒ] at A⊒
rw [A]
rfl
#align schwartz_with_seminorms schwartzWithSeminorms
#align schwartz_with_seminorms schwartz_withSeminorms

variable {π•œ E F}

instance : ContinuousSMul π•œ 𝓒(E, F) :=
by
rw [(schwartzWithSeminorms π•œ E F).withSeminorms_eq]
rw [(schwartz_withSeminorms π•œ E F).withSeminorms_eq]
exact (schwartzSeminormFamily π•œ E F).ModuleFilterBasis.ContinuousSMul

instance : TopologicalAddGroup 𝓒(E, F) :=
(schwartzSeminormFamily ℝ E F).AddGroupFilterBasis.is_topological_add_group
(schwartzSeminormFamily ℝ E F).AddGroupFilterBasis.isTopologicalAddGroup

instance : UniformSpace 𝓒(E, F) :=
(schwartzSeminormFamily ℝ E F).AddGroupFilterBasis.UniformSpace
Expand All @@ -529,10 +529,10 @@ instance : UniformAddGroup 𝓒(E, F) :=
(schwartzSeminormFamily ℝ E F).AddGroupFilterBasis.UniformAddGroup

instance : LocallyConvexSpace ℝ 𝓒(E, F) :=
(schwartzWithSeminorms ℝ E F).toLocallyConvexSpace
(schwartz_withSeminorms ℝ E F).toLocallyConvexSpace

instance : TopologicalSpace.FirstCountableTopology 𝓒(E, F) :=
(schwartzWithSeminorms ℝ E F).first_countable
(schwartz_withSeminorms ℝ E F).first_countable

end Topology

Expand Down Expand Up @@ -594,8 +594,8 @@ def mkClm [RingHomIsometric Οƒ] (A : (D β†’ E) β†’ F β†’ G)
cont := by
change Continuous (mk_lm A hadd hsmul hsmooth hbound : 𝓒(D, E) β†’β‚›β‚—[Οƒ] 𝓒(F, G))
refine'
Seminorm.continuous_from_bounded (schwartzWithSeminorms π•œ D E) (schwartzWithSeminorms π•œ' F G)
_ fun n => _
Seminorm.continuous_from_bounded (schwartz_withSeminorms π•œ D E)
(schwartz_withSeminorms π•œ' F G) _ fun n => _
rcases hbound n with ⟨s, C, hC, h⟩
refine' ⟨s, ⟨C, hC⟩, fun f => _⟩
simp only [Seminorm.comp_apply, Seminorm.smul_apply, NNReal.smul_def, Algebra.id.smul_eq_mul,
Expand Down Expand Up @@ -686,8 +686,8 @@ def toBoundedContinuousFunctionClm : 𝓒(E, F) β†’L[π•œ] E →ᡇ F :=
cont := by
change Continuous (to_bounded_continuous_function_lm π•œ E F)
refine'
Seminorm.continuous_from_bounded (schwartzWithSeminorms π•œ E F)
(normWithSeminorms π•œ (E →ᡇ F)) _ fun i => ⟨{0}, 1, fun f => _⟩
Seminorm.continuous_from_bounded (schwartz_withSeminorms π•œ E F)
(norm_withSeminorms π•œ (E →ᡇ F)) _ fun i => ⟨{0}, 1, fun f => _⟩
rw [Finset.sup_singleton, one_smul, Seminorm.comp_apply, coe_normSeminorm,
schwartz_seminorm_family_apply_zero, BoundedContinuousFunction.norm_le (map_nonneg _ _)]
intro x
Expand Down
2 changes: 1 addition & 1 deletion Mathbin/FieldTheory/KrullTopology.lean
Expand Up @@ -211,7 +211,7 @@ instance krullTopology (K L : Type _) [Field K] [Field L] [Algebra K L] :

/-- For a field extension `L/K`, the Krull topology on `L ≃ₐ[K] L` makes it a topological group. -/
instance (K L : Type _) [Field K] [Field L] [Algebra K L] : TopologicalGroup (L ≃ₐ[K] L) :=
GroupFilterBasis.is_topologicalGroup (galGroupBasis K L)
GroupFilterBasis.isTopologicalGroup (galGroupBasis K L)

section KrullT2

Expand Down

0 comments on commit 678d4ff

Please sign in to comment.