formal
stringlengths
41
427k
informal
stringclasses
1 value
nhdsWithin_pos_comap_mul_left ** 𝕜 : Type u_1 α : Type u_2 inst✝² : LinearOrderedField 𝕜 inst✝¹ : TopologicalSpace 𝕜 inst✝ : OrderTopology 𝕜 l : Filter α f g : α → 𝕜 x : 𝕜 hx : 0 < x ⊢ comap (fun x_1 => x * x_1) (𝓝[Ioi 0] 0) = 𝓝[Ioi 0] 0 ** rw [nhdsWithin, comap_inf, comap_principal, preimage_const_mul_Ioi _ hx, zero_div] ** 𝕜 : Type u_1 α : Type u_2 inst✝² : LinearOrderedField 𝕜 inst✝¹ : TopologicalSpace 𝕜 inst✝ : OrderTopology 𝕜 l : Filter α f g : α → 𝕜 x : 𝕜 hx : 0 < x ⊢ comap (fun x_1 => x * x_1) (𝓝 0) ⊓ 𝓟 (Ioi 0) = 𝓝 0 ⊓ 𝓟 (Ioi 0) ** congr 1 ** case e_a 𝕜 : Type u_1 α : Type u_2 inst✝² : LinearOrderedField 𝕜 inst✝¹ : TopologicalSpace 𝕜 inst✝ : OrderTopology 𝕜 l : Filter α f g : α → 𝕜 x : 𝕜 hx : 0 < x ⊢ comap (fun x_1 => x * x_1) (𝓝 0) = 𝓝 0 ** refine ((Homeomorph.mulLeft₀ x hx.ne').comap_nhds_eq _).trans ?_ ** case e_a 𝕜 : Type u_1 α : Type u_2 inst✝² : LinearOrderedField 𝕜 inst✝¹ : TopologicalSpace 𝕜 inst✝ : OrderTopology 𝕜 l : Filter α f g : α → 𝕜 x : 𝕜 hx : 0 < x ⊢ 𝓝 (↑(Homeomorph.symm (Homeomorph.mulLeft₀ x (_ : x ≠ 0))) 0) = 𝓝 0 ** simp ** Qed
eventually_nhdsWithin_pos_mul_left ** 𝕜 : Type u_1 α : Type u_2 inst✝² : LinearOrderedField 𝕜 inst✝¹ : TopologicalSpace 𝕜 inst✝ : OrderTopology 𝕜 l : Filter α f g : α → 𝕜 x : 𝕜 hx : 0 < x p : 𝕜 → Prop h : ∀ᶠ (ε : 𝕜) in 𝓝[Ioi 0] 0, p ε ⊢ ∀ᶠ (ε : 𝕜) in 𝓝[Ioi 0] 0, p (x * ε) ** rw [← nhdsWithin_pos_comap_mul_left hx] ** 𝕜 : Type u_1 α : Type u_2 inst✝² : LinearOrderedField 𝕜 inst✝¹ : TopologicalSpace 𝕜 inst✝ : OrderTopology 𝕜 l : Filter α f g : α → 𝕜 x : 𝕜 hx : 0 < x p : 𝕜 → Prop h : ∀ᶠ (ε : 𝕜) in 𝓝[Ioi 0] 0, p ε ⊢ ∀ᶠ (ε : 𝕜) in comap (fun x_1 => x * x_1) (𝓝[Ioi 0] 0), p (x * ε) ** exact h.comap fun ε => x * ε ** Qed
Bornology.isBounded_compl_iff ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α ⊢ IsBounded sᶜ ↔ IsCobounded s ** rw [isBounded_def, isCobounded_def, compl_compl] ** Qed
Bornology.isBounded_empty ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α ⊢ IsBounded ∅ ** rw [isBounded_def, compl_empty] ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α ⊢ univ ∈ cobounded α ** exact univ_mem ** Qed
Bornology.isBounded_singleton ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α ⊢ IsBounded {x} ** rw [isBounded_def] ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α ⊢ {x}ᶜ ∈ cobounded α ** exact le_cofinite _ (finite_singleton x).compl_mem_cofinite ** Qed
Bornology.isBounded_iff_forall_mem ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α h : ∀ (x : α), x ∈ s → IsBounded s ⊢ IsBounded s ** rcases s.eq_empty_or_nonempty with rfl | ⟨x, hx⟩ ** case inl ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α t : Set α x : α h : ∀ (x : α), x ∈ ∅ → IsBounded ∅ ⊢ IsBounded ∅ case inr.intro ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x✝ : α h : ∀ (x : α), x ∈ s → IsBounded s x : α hx : x ∈ s ⊢ IsBounded s ** exacts [isBounded_empty, h x hx] ** Qed
Bornology.isBounded_union ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α s t : Set α x : α ⊢ IsBounded (s ∪ t) ↔ IsBounded s ∧ IsBounded t ** simp only [← isCobounded_compl_iff, compl_union, isCobounded_inter] ** Qed
Bornology.comap_cobounded_le_iff ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝¹ : Bornology α s t : Set α x : α inst✝ : Bornology β f : α → β ⊢ comap f (cobounded β) ≤ cobounded α ↔ ∀ ⦃s : Set α⦄, IsBounded s → IsBounded (f '' s) ** refine' ⟨fun h s hs => _, fun h t ht => ⟨(f '' tᶜ)ᶜ, h <| IsCobounded.compl ht, compl_subset_comm.1 <| subset_preimage_image _ _⟩⟩ ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝¹ : Bornology α s✝ t : Set α x : α inst✝ : Bornology β f : α → β h : comap f (cobounded β) ≤ cobounded α s : Set α hs : IsBounded s ⊢ IsBounded (f '' s) ** obtain ⟨t, ht, hts⟩ := h hs.compl ** case intro.intro ι : Type u_1 α : Type u_2 β : Type u_3 inst✝¹ : Bornology α s✝ t✝ : Set α x : α inst✝ : Bornology β f : α → β h : comap f (cobounded β) ≤ cobounded α s : Set α hs : IsBounded s t : Set β ht : t ∈ cobounded β hts : f ⁻¹' t ⊆ sᶜ ⊢ IsBounded (f '' s) ** rw [subset_compl_comm, ← preimage_compl] at hts ** case intro.intro ι : Type u_1 α : Type u_2 β : Type u_3 inst✝¹ : Bornology α s✝ t✝ : Set α x : α inst✝ : Bornology β f : α → β h : comap f (cobounded β) ≤ cobounded α s : Set α hs : IsBounded s t : Set β ht : t ∈ cobounded β hts : s ⊆ f ⁻¹' tᶜ ⊢ IsBounded (f '' s) ** exact (IsCobounded.compl ht).subset ((image_subset f hts).trans <| image_preimage_subset _ _) ** Qed
Bornology.isBounded_ofBounded_iff ** ι : Type u_1 α : Type u_2 β : Type u_3 s : Set α B : Set (Set α) empty_mem : ∅ ∈ B subset_mem : ∀ (s₁ : Set α), s₁ ∈ B → ∀ (s₂ : Set α), s₂ ⊆ s₁ → s₂ ∈ B union_mem : ∀ (s₁ : Set α), s₁ ∈ B → ∀ (s₂ : Set α), s₂ ∈ B → s₁ ∪ s₂ ∈ B sUnion_univ : ∀ (x : α), {x} ∈ B ⊢ IsBounded s ↔ s ∈ B ** rw [@isBounded_def _ (ofBounded B empty_mem subset_mem union_mem sUnion_univ), ← Filter.mem_sets, ofBounded_cobounded_sets, Set.mem_setOf_eq, compl_compl] ** Qed
Bornology.isBounded_biUnion ** ι : Type u_1 α : Type u_2 β : Type u_3 s✝ : Set α inst✝ : Bornology α s : Set ι f : ι → Set α hs : Set.Finite s ⊢ IsBounded (⋃ i ∈ s, f i) ↔ ∀ (i : ι), i ∈ s → IsBounded (f i) ** simp only [← isCobounded_compl_iff, compl_iUnion, isCobounded_biInter hs] ** Qed
Bornology.isBounded_sUnion ** ι : Type u_1 α : Type u_2 β : Type u_3 s : Set α inst✝ : Bornology α S : Set (Set α) hs : Set.Finite S ⊢ IsBounded (⋃₀ S) ↔ ∀ (s : Set α), s ∈ S → IsBounded s ** rw [sUnion_eq_biUnion, isBounded_biUnion hs] ** Qed
Bornology.isBounded_iUnion ** ι : Type u_1 α : Type u_2 β : Type u_3 s✝ : Set α inst✝¹ : Bornology α inst✝ : Finite ι s : ι → Set α ⊢ IsBounded (⋃ i, s i) ↔ ∀ (i : ι), IsBounded (s i) ** rw [← sUnion_range, isBounded_sUnion (finite_range s), forall_range_iff] ** Qed
Bornology.cobounded_eq_bot_iff ** ι : Type u_1 α : Type u_2 β : Type u_3 inst✝ : Bornology α ⊢ cobounded α = ⊥ ↔ BoundedSpace α ** rw [← isBounded_univ, isBounded_def, compl_univ, empty_mem_iff_bot] ** Qed
quotientMap_projIcc ** α : Type u_1 β : Type u_2 γ : Type u_3 inst✝⁴ : LinearOrder α inst✝³ : TopologicalSpace γ a b c : α h : a ≤ b inst✝² : TopologicalSpace α inst✝¹ : OrderTopology α inst✝ : TopologicalSpace β s : Set ↑(Icc a b) hs : IsOpen (projIcc a b h ⁻¹' s) ⊢ Subtype.val ⁻¹' (projIcc a b h ⁻¹' s) = s ** ext ** case h α : Type u_1 β : Type u_2 γ : Type u_3 inst✝⁴ : LinearOrder α inst✝³ : TopologicalSpace γ a b c : α h : a ≤ b inst✝² : TopologicalSpace α inst✝¹ : OrderTopology α inst✝ : TopologicalSpace β s : Set ↑(Icc a b) hs : IsOpen (projIcc a b h ⁻¹' s) x✝ : { x // x ∈ Icc a b } ⊢ x✝ ∈ Subtype.val ⁻¹' (projIcc a b h ⁻¹' s) ↔ x✝ ∈ s ** simp ** Qed
TopologicalSpace.IsSeparable.secondCountableTopology ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁴ : TopologicalSpace X inst✝³ : TopologicalSpace Y inst✝² : Finite ι inst✝¹ : (i : ι) → TopologicalSpace (π i) inst✝ : PseudoMetrizableSpace X s : Set X hs : IsSeparable s ⊢ SecondCountableTopology ↑s ** letI := pseudoMetrizableSpacePseudoMetric X ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁴ : TopologicalSpace X inst✝³ : TopologicalSpace Y inst✝² : Finite ι inst✝¹ : (i : ι) → TopologicalSpace (π i) inst✝ : PseudoMetrizableSpace X s : Set X hs : IsSeparable s this : PseudoMetricSpace X := pseudoMetrizableSpacePseudoMetric X ⊢ SecondCountableTopology ↑s ** have := hs.separableSpace ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁴ : TopologicalSpace X inst✝³ : TopologicalSpace Y inst✝² : Finite ι inst✝¹ : (i : ι) → TopologicalSpace (π i) inst✝ : PseudoMetrizableSpace X s : Set X hs : IsSeparable s this✝ : PseudoMetricSpace X := pseudoMetrizableSpacePseudoMetric X this : SeparableSpace ↑s ⊢ SecondCountableTopology ↑s ** exact UniformSpace.secondCountable_of_separable s ** Qed
TopologicalSpace.exists_embedding_l_infty ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X ⊢ ∃ f, Embedding f ** rcases exists_countable_basis X with ⟨B, hBc, -, hB⟩ ** case intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B ⊢ ∃ f, Embedding f ** let s : Set (Set X × Set X) := { UV ∈ B ×ˢ B | closure UV.1 ⊆ UV.2 } ** case intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} ⊢ ∃ f, Embedding f ** haveI : Encodable s := ((hBc.prod hBc).mono (inter_subset_left _ _)).toEncodable ** case intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this : Encodable ↑s ⊢ ∃ f, Embedding f ** letI : TopologicalSpace s := ⊥ ** case intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝ : Encodable ↑s this : TopologicalSpace ↑s := ⊥ ⊢ ∃ f, Embedding f ** haveI : DiscreteTopology s := ⟨rfl⟩ ** case intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s ⊢ ∃ f, Embedding f ** rsuffices ⟨f, hf⟩ : ∃ f : X → s →ᵇ ℝ, Embedding f ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s ⊢ ∃ f, Embedding f ** have hd : ∀ UV : s, Disjoint (closure UV.1.1) UV.1.2ᶜ := fun UV => disjoint_compl_right.mono_right (compl_subset_compl.2 UV.2.2) ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ⊢ ∃ f, Embedding f ** obtain ⟨ε, ε01, hε⟩ : ∃ ε : s → ℝ, (∀ UV, ε UV ∈ Ioc (0 : ℝ) 1) ∧ Tendsto ε cofinite (𝓝 0) := by rcases posSumOfEncodable zero_lt_one s with ⟨ε, ε0, c, hεc, hc1⟩ refine' ⟨ε, fun UV => ⟨ε0 UV, _⟩, hεc.summable.tendsto_cofinite_zero⟩ exact (le_hasSum hεc UV fun _ _ => (ε0 _).le).trans hc1 ** case intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) ⊢ ∃ f, Embedding f ** have : ∀ UV : s, ∃ f : C(X, ℝ), EqOn f 0 UV.1.1 ∧ EqOn f (fun _ => ε UV) UV.1.2ᶜ ∧ ∀ x, f x ∈ Icc 0 (ε UV) := by intro UV rcases exists_continuous_zero_one_of_closed isClosed_closure (hB.isOpen UV.2.1.2).isClosed_compl (hd UV) with ⟨f, hf₀, hf₁, hf01⟩ exact ⟨ε UV • f, fun x hx => by simp [hf₀ (subset_closure hx)], fun x hx => by simp [hf₁ hx], fun x => ⟨mul_nonneg (ε01 _).1.le (hf01 _).1, mul_le_of_le_one_right (ε01 _).1.le (hf01 _).2⟩⟩ ** case intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝² : Encodable ↑s this✝¹ : TopologicalSpace ↑s := ⊥ this✝ : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) this : ∀ (UV : ↑s), ∃ f, EqOn (↑f) 0 (↑UV).1 ∧ EqOn (↑f) (fun x => ε UV) (↑UV).2ᶜ ∧ ∀ (x : X), ↑f x ∈ Icc 0 (ε UV) ⊢ ∃ f, Embedding f ** choose f hf0 hfε hf0ε using this ** case intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) ⊢ ∃ f, Embedding f ** have hf01 : ∀ UV x, f UV x ∈ Icc (0 : ℝ) 1 := fun UV x => Icc_subset_Icc_right (ε01 _).2 (hf0ε _ _) ** case intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 ⊢ ∃ f, Embedding f ** set F : X → s →ᵇ ℝ := fun x => ⟨⟨fun UV => f UV x, continuous_of_discreteTopology⟩, 1, fun UV₁ UV₂ => Real.dist_le_of_mem_Icc_01 (hf01 _ _) (hf01 _ _)⟩ ** case intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } ⊢ ∃ f, Embedding f ** have hF : ∀ x UV, F x UV = f UV x := fun _ _ => rfl ** case intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x ⊢ ∃ f, Embedding f ** refine' ⟨F, Embedding.mk' _ (fun x y hxy => _) fun x => le_antisymm _ _⟩ ** case intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s f : X → ↑s →ᵇ ℝ hf : Embedding f ⊢ ∃ f, Embedding f ** exact ⟨fun x => (f x).extend (Encodable.encode' s) 0, (BoundedContinuousFunction.isometry_extend (Encodable.encode' s) (0 : ℕ →ᵇ ℝ)).embedding.comp hf⟩ ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ⊢ ∃ ε, (∀ (UV : ↑s), ε UV ∈ Ioc 0 1) ∧ Tendsto ε cofinite (𝓝 0) ** rcases posSumOfEncodable zero_lt_one s with ⟨ε, ε0, c, hεc, hc1⟩ ** case mk.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε0 : ∀ (i : ↑s), 0 < ε i c : ℝ hεc : HasSum ε c hc1 : c ≤ 1 ⊢ ∃ ε, (∀ (UV : ↑s), ε UV ∈ Ioc 0 1) ∧ Tendsto ε cofinite (𝓝 0) ** refine' ⟨ε, fun UV => ⟨ε0 UV, _⟩, hεc.summable.tendsto_cofinite_zero⟩ ** case mk.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε0 : ∀ (i : ↑s), 0 < ε i c : ℝ hεc : HasSum ε c hc1 : c ≤ 1 UV : ↑s ⊢ ε UV ≤ 1 ** exact (le_hasSum hεc UV fun _ _ => (ε0 _).le).trans hc1 ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) ⊢ ∀ (UV : ↑s), ∃ f, EqOn (↑f) 0 (↑UV).1 ∧ EqOn (↑f) (fun x => ε UV) (↑UV).2ᶜ ∧ ∀ (x : X), ↑f x ∈ Icc 0 (ε UV) ** intro UV ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) UV : ↑s ⊢ ∃ f, EqOn (↑f) 0 (↑UV).1 ∧ EqOn (↑f) (fun x => ε UV) (↑UV).2ᶜ ∧ ∀ (x : X), ↑f x ∈ Icc 0 (ε UV) ** rcases exists_continuous_zero_one_of_closed isClosed_closure (hB.isOpen UV.2.1.2).isClosed_compl (hd UV) with ⟨f, hf₀, hf₁, hf01⟩ ** case intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) UV : ↑s f : C(X, ℝ) hf₀ : EqOn (↑f) 0 (closure (↑UV).1) hf₁ : EqOn (↑f) 1 (↑UV).2ᶜ hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1 ⊢ ∃ f, EqOn (↑f) 0 (↑UV).1 ∧ EqOn (↑f) (fun x => ε UV) (↑UV).2ᶜ ∧ ∀ (x : X), ↑f x ∈ Icc 0 (ε UV) ** exact ⟨ε UV • f, fun x hx => by simp [hf₀ (subset_closure hx)], fun x hx => by simp [hf₁ hx], fun x => ⟨mul_nonneg (ε01 _).1.le (hf01 _).1, mul_le_of_le_one_right (ε01 _).1.le (hf01 _).2⟩⟩ ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) UV : ↑s f : C(X, ℝ) hf₀ : EqOn (↑f) 0 (closure (↑UV).1) hf₁ : EqOn (↑f) 1 (↑UV).2ᶜ hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1 x : X hx : x ∈ (↑UV).1 ⊢ ↑(ε UV • f) x = OfNat.ofNat 0 x ** simp [hf₀ (subset_closure hx)] ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) UV : ↑s f : C(X, ℝ) hf₀ : EqOn (↑f) 0 (closure (↑UV).1) hf₁ : EqOn (↑f) 1 (↑UV).2ᶜ hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1 x : X hx : x ∈ (↑UV).2ᶜ ⊢ ↑(ε UV • f) x = (fun x => ε UV) x ** simp [hf₁ hx] ** case intro.intro.refine'_1 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y ⊢ x = y ** by_contra Hne ** case intro.intro.refine'_1 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y Hne : ¬x = y ⊢ False ** rcases hB.mem_nhds_iff.1 (isOpen_ne.mem_nhds Hne) with ⟨V, hVB, hxV, hVy⟩ ** case intro.intro.refine'_1.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y Hne : ¬x = y V : Set X hVB : V ∈ B hxV : x ∈ V hVy : V ⊆ {y_1 | y_1 ≠ y} ⊢ False ** rcases hB.exists_closure_subset (hB.mem_nhds hVB hxV) with ⟨U, hUB, hxU, hUV⟩ ** case intro.intro.refine'_1.intro.intro.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y Hne : ¬x = y V : Set X hVB : V ∈ B hxV : x ∈ V hVy : V ⊆ {y_1 | y_1 ≠ y} U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V ⊢ False ** set UV : ↥s := ⟨(U, V), ⟨hUB, hVB⟩, hUV⟩ ** case intro.intro.refine'_1.intro.intro.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y Hne : ¬x = y V : Set X hVB : V ∈ B hxV : x ∈ V hVy : V ⊆ {y_1 | y_1 ≠ y} U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } ⊢ False ** apply (ε01 UV).1.ne ** case intro.intro.refine'_1.intro.intro.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y Hne : ¬x = y V : Set X hVB : V ∈ B hxV : x ∈ V hVy : V ⊆ {y_1 | y_1 ≠ y} U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } ⊢ 0 = ε UV ** calc (0 : ℝ) = F x UV := (hf0 UV hxU).symm _ = F y UV := by rw [hxy] _ = ε UV := hfε UV fun h : y ∈ V => hVy h rfl ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x y : X hxy : F x = F y Hne : ¬x = y V : Set X hVB : V ∈ B hxV : x ∈ V hVy : V ⊆ {y_1 | y_1 ≠ y} U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } ⊢ ↑(F x) UV = ↑(F y) UV ** rw [hxy] ** case intro.intro.refine'_2 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X ⊢ comap F (𝓝 (F x)) ≤ 𝓝 x ** refine' ((nhds_basis_ball.comap _).le_basis_iff hB.nhds_hasBasis).2 _ ** case intro.intro.refine'_2 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X ⊢ ∀ (i' : Set X), i' ∈ B ∧ x ∈ i' → ∃ i, 0 < i ∧ F ⁻¹' ball (F x) i ⊆ i' ** rintro V ⟨hVB, hxV⟩ ** case intro.intro.refine'_2.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V ⊢ ∃ i, 0 < i ∧ F ⁻¹' ball (F x) i ⊆ V ** rcases hB.exists_closure_subset (hB.mem_nhds hVB hxV) with ⟨U, hUB, hxU, hUV⟩ ** case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V ⊢ ∃ i, 0 < i ∧ F ⁻¹' ball (F x) i ⊆ V ** set UV : ↥s := ⟨(U, V), ⟨hUB, hVB⟩, hUV⟩ ** case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } ⊢ ∃ i, 0 < i ∧ F ⁻¹' ball (F x) i ⊆ V ** refine' ⟨ε UV, (ε01 UV).1, fun y (hy : dist (F y) (F x) < ε UV) => _⟩ ** case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } y : X hy : dist (F y) (F x) < ε UV ⊢ y ∈ V ** replace hy : dist (F y UV) (F x UV) < ε UV ** case hy ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } y : X hy : dist (F y) (F x) < ε UV ⊢ dist (↑(F y) UV) (↑(F x) UV) < ε UV case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } y : X hy : dist (↑(F y) UV) (↑(F x) UV) < ε UV ⊢ y ∈ V ** exact (BoundedContinuousFunction.dist_coe_le_dist _).trans_lt hy ** case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } y : X hy : dist (↑(F y) UV) (↑(F x) UV) < ε UV ⊢ y ∈ V ** contrapose! hy ** case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } y : X hy : ¬y ∈ V ⊢ ε UV ≤ dist (↑(F y) UV) (↑(F x) UV) ** rw [hF, hF, hfε UV hy, hf0 UV hxU, Pi.zero_apply, dist_zero_right] ** case intro.intro.refine'_2.intro.intro.intro.intro ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X V : Set X hVB : V ∈ B hxV : x ∈ V U : Set X hUB : U ∈ B hxU : x ∈ U hUV : closure U ⊆ V UV : ↑s := { val := (U, V), property := (_ : (U, V) ∈ B ×ˢ B ∧ closure (U, V).1 ⊆ (U, V).2) } y : X hy : ¬y ∈ V ⊢ ε UV ≤ ‖(fun x => ε UV) y‖ ** exact le_abs_self _ ** case intro.intro.refine'_3 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X ⊢ 𝓝 x ≤ comap F (𝓝 (F x)) ** refine' (nhds_basis_closedBall.comap _).ge_iff.2 fun δ δ0 => _ ** case intro.intro.refine'_3 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ ⊢ F ⁻¹' closedBall (F x) δ ∈ 𝓝 x ** have h_fin : { UV : s | δ ≤ ε UV }.Finite := by simpa only [← not_lt] using hε (gt_mem_nhds δ0) ** case intro.intro.refine'_3 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} ⊢ F ⁻¹' closedBall (F x) δ ∈ 𝓝 x ** have : ∀ᶠ y in 𝓝 x, ∀ UV, δ ≤ ε UV → dist (F y UV) (F x UV) ≤ δ := by refine' (eventually_all_finite h_fin).2 fun UV _ => _ exact (f UV).continuous.tendsto x (closedBall_mem_nhds _ δ0) ** case intro.intro.refine'_3 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝² : Encodable ↑s this✝¹ : TopologicalSpace ↑s := ⊥ this✝ : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} this : ∀ᶠ (y : X) in 𝓝 x, ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ ⊢ F ⁻¹' closedBall (F x) δ ∈ 𝓝 x ** refine' this.mono fun y hy => (BoundedContinuousFunction.dist_le δ0.le).2 fun UV => _ ** case intro.intro.refine'_3 ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝² : Encodable ↑s this✝¹ : TopologicalSpace ↑s := ⊥ this✝ : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} this : ∀ᶠ (y : X) in 𝓝 x, ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ y : X hy : ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ UV : ↑s ⊢ dist (↑(F y) UV) (↑(F x) UV) ≤ δ ** cases' le_total δ (ε UV) with hle hle ** case intro.intro.refine'_3.inl ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝² : Encodable ↑s this✝¹ : TopologicalSpace ↑s := ⊥ this✝ : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} this : ∀ᶠ (y : X) in 𝓝 x, ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ y : X hy : ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ UV : ↑s hle : δ ≤ ε UV ⊢ dist (↑(F y) UV) (↑(F x) UV) ≤ δ case intro.intro.refine'_3.inr ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝² : Encodable ↑s this✝¹ : TopologicalSpace ↑s := ⊥ this✝ : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} this : ∀ᶠ (y : X) in 𝓝 x, ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ y : X hy : ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ UV : ↑s hle : ε UV ≤ δ ⊢ dist (↑(F y) UV) (↑(F x) UV) ≤ δ ** exacts [hy _ hle, (Real.dist_le_of_mem_Icc (hf0ε _ _) (hf0ε _ _)).trans (by rwa [sub_zero])] ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ ⊢ Set.Finite {UV | δ ≤ ε UV} ** simpa only [← not_lt] using hε (gt_mem_nhds δ0) ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} ⊢ ∀ᶠ (y : X) in 𝓝 x, ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ ** refine' (eventually_all_finite h_fin).2 fun UV _ => _ ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝¹ : Encodable ↑s this✝ : TopologicalSpace ↑s := ⊥ this : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} UV : ↑s x✝ : UV ∈ {UV | δ ≤ ε UV} ⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (↑(F x_1) UV) (↑(F x) UV) ≤ δ ** exact (f UV).continuous.tendsto x (closedBall_mem_nhds _ δ0) ** ι : Type u_1 X : Type u_2 Y : Type u_3 π : ι → Type u_4 inst✝⁵ : TopologicalSpace X inst✝⁴ : TopologicalSpace Y inst✝³ : Finite ι inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : T3Space X inst✝ : SecondCountableTopology X B : Set (Set X) hBc : Set.Countable B hB : IsTopologicalBasis B s : Set (Set X × Set X) := {UV | UV ∈ B ×ˢ B ∧ closure UV.1 ⊆ UV.2} this✝² : Encodable ↑s this✝¹ : TopologicalSpace ↑s := ⊥ this✝ : DiscreteTopology ↑s hd : ∀ (UV : ↑s), Disjoint (closure (↑UV).1) (↑UV).2ᶜ ε : ↑s → ℝ ε01 : ∀ (UV : ↑s), ε UV ∈ Ioc 0 1 hε : Tendsto ε cofinite (𝓝 0) f : ↑s → C(X, ℝ) hf0 : ∀ (UV : ↑s), EqOn (↑(f UV)) 0 (↑UV).1 hfε : ∀ (UV : ↑s), EqOn (↑(f UV)) (fun x => ε UV) (↑UV).2ᶜ hf0ε : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 (ε UV) hf01 : ∀ (UV : ↑s) (x : X), ↑(f UV) x ∈ Icc 0 1 F : X → ↑s →ᵇ ℝ := fun x => { toContinuousMap := ContinuousMap.mk fun UV => ↑(f UV) x, map_bounded' := (_ : ∃ C, ∀ (x_1 y : ↑s), dist (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) x_1) (ContinuousMap.toFun (ContinuousMap.mk fun UV => ↑(f UV) x) y) ≤ C) } hF : ∀ (x : X) (UV : ↑s), ↑(F x) UV = ↑(f UV) x x : X δ : ℝ δ0 : 0 < δ h_fin : Set.Finite {UV | δ ≤ ε UV} this : ∀ᶠ (y : X) in 𝓝 x, ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ y : X hy : ∀ (UV : ↑s), δ ≤ ε UV → dist (↑(F y) UV) (↑(F x) UV) ≤ δ UV : ↑s hle : ε UV ≤ δ ⊢ ε UV - 0 ≤ δ ** rwa [sub_zero] ** Qed
CauSeq.tendsto_limit ** β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm ⊢ ∀ (s : Set β), IsOpen s → lim f ∈ s → ↑f ⁻¹' s ∈ atTop ** intro s os lfs ** β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ⊢ ↑f ⁻¹' s ∈ atTop ** suffices ∃ a : ℕ, ∀ b : ℕ, b ≥ a → f b ∈ s by simpa using this ** β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ⊢ ∃ a, ∀ (b : ℕ), b ≥ a → ↑f b ∈ s ** rcases Metric.isOpen_iff.1 os _ lfs with ⟨ε, ⟨hε, hεs⟩⟩ ** case intro.intro β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s ⊢ ∃ a, ∀ (b : ℕ), b ≥ a → ↑f b ∈ s ** cases' Setoid.symm (CauSeq.equiv_lim f) _ hε with N hN ** case intro.intro.intro β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ‖↑(const norm (lim f) - f) j‖ < ε ⊢ ∃ a, ∀ (b : ℕ), b ≥ a → ↑f b ∈ s ** exists N ** case intro.intro.intro β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ‖↑(const norm (lim f) - f) j‖ < ε ⊢ ∀ (b : ℕ), b ≥ N → ↑f b ∈ s ** intro b hb ** case intro.intro.intro β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ‖↑(const norm (lim f) - f) j‖ < ε b : ℕ hb : b ≥ N ⊢ ↑f b ∈ s ** apply hεs ** case intro.intro.intro.a β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ‖↑(const norm (lim f) - f) j‖ < ε b : ℕ hb : b ≥ N ⊢ ↑f b ∈ Metric.ball (lim f) ε ** dsimp [Metric.ball] ** case intro.intro.intro.a β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ‖↑(const norm (lim f) - f) j‖ < ε b : ℕ hb : b ≥ N ⊢ dist (↑f b) (lim f) < ε ** rw [dist_comm, dist_eq_norm] ** case intro.intro.intro.a β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s ε : ℝ hε : ε > 0 hεs : Metric.ball (lim f) ε ⊆ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ‖↑(const norm (lim f) - f) j‖ < ε b : ℕ hb : b ≥ N ⊢ ‖lim f - ↑f b‖ < ε ** solve_by_elim ** β : Type v inst✝¹ : NormedRing β hn : IsAbsoluteValue norm f : CauSeq β norm inst✝ : IsComplete β norm s : Set β os : IsOpen s lfs : lim f ∈ s this : ∃ a, ∀ (b : ℕ), b ≥ a → ↑f b ∈ s ⊢ ↑f ⁻¹' s ∈ atTop ** simpa using this ** Qed
CauchySeq.isCauSeq ** β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f ⊢ IsCauSeq norm f ** cases' cauchy_iff.1 hf with hf1 hf2 ** case intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ⊢ IsCauSeq norm f ** intro ε hε ** case intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 ⊢ ∃ i, ∀ (j : ℕ), j ≥ i → ‖f j - f i‖ < ε ** rcases hf2 { x | dist x.1 x.2 < ε } (dist_mem_uniformity hε) with ⟨t, ⟨ht, htsub⟩⟩ ** case intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β ht : t ∈ map f atTop htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} ⊢ ∃ i, ∀ (j : ℕ), j ≥ i → ‖f j - f i‖ < ε ** simp at ht ** case intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} ht : ∃ a, ∀ (b : ℕ), a ≤ b → f b ∈ t ⊢ ∃ i, ∀ (j : ℕ), j ≥ i → ‖f j - f i‖ < ε ** cases' ht with N hN ** case intro.intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} N : ℕ hN : ∀ (b : ℕ), N ≤ b → f b ∈ t ⊢ ∃ i, ∀ (j : ℕ), j ≥ i → ‖f j - f i‖ < ε ** exists N ** case intro.intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} N : ℕ hN : ∀ (b : ℕ), N ≤ b → f b ∈ t ⊢ ∀ (j : ℕ), j ≥ N → ‖f j - f N‖ < ε ** intro j hj ** case intro.intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} N : ℕ hN : ∀ (b : ℕ), N ≤ b → f b ∈ t j : ℕ hj : j ≥ N ⊢ ‖f j - f N‖ < ε ** rw [← dist_eq_norm] ** case intro.intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} N : ℕ hN : ∀ (b : ℕ), N ≤ b → f b ∈ t j : ℕ hj : j ≥ N ⊢ dist (f j) (f N) < ε ** apply @htsub (f j, f N) ** case intro.intro.intro.intro β : Type v inst✝ : NormedField β f : ℕ → β hf : CauchySeq f hf1 : NeBot (map f atTop) hf2 : ∀ (s : Set (β × β)), s ∈ uniformity β → ∃ t, t ∈ map f atTop ∧ t ×ˢ t ⊆ s ε : ℝ hε : ε > 0 t : Set β htsub : t ×ˢ t ⊆ {x | dist x.1 x.2 < ε} N : ℕ hN : ∀ (b : ℕ), N ≤ b → f b ∈ t j : ℕ hj : j ≥ N ⊢ (f j, f N) ∈ t ×ˢ t ** apply Set.mk_mem_prod <;> solve_by_elim [le_refl] ** Qed
CauSeq.cauchySeq ** β : Type v inst✝ : NormedField β f : CauSeq β norm ⊢ CauchySeq ↑f ** refine' cauchy_iff.2 ⟨by infer_instance, fun s hs => _⟩ ** β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ⊢ ∃ t, t ∈ map (↑f) atTop ∧ t ×ˢ t ⊆ s ** rcases mem_uniformity_dist.1 hs with ⟨ε, ⟨hε, hεs⟩⟩ ** case intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s ⊢ ∃ t, t ∈ map (↑f) atTop ∧ t ×ˢ t ⊆ s ** cases' CauSeq.cauchy₂ f hε with N hN ** case intro.intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε ⊢ ∃ t, t ∈ map (↑f) atTop ∧ t ×ˢ t ⊆ s ** exists { n | n ≥ N }.image f ** case intro.intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε ⊢ ↑f '' {n | n ≥ N} ∈ map (↑f) atTop ∧ (↑f '' {n | n ≥ N}) ×ˢ (↑f '' {n | n ≥ N}) ⊆ s ** simp only [exists_prop, mem_atTop_sets, mem_map, mem_image, ge_iff_le, mem_setOf_eq] ** case intro.intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε ⊢ (∃ a, ∀ (b : ℕ), a ≤ b → b ∈ ↑f ⁻¹' (↑f '' {n | N ≤ n})) ∧ (↑f '' {n | N ≤ n}) ×ˢ (↑f '' {n | N ≤ n}) ⊆ s ** constructor ** β : Type v inst✝ : NormedField β f : CauSeq β norm ⊢ NeBot (map (↑f) atTop) ** infer_instance ** case intro.intro.intro.left β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε ⊢ ∃ a, ∀ (b : ℕ), a ≤ b → b ∈ ↑f ⁻¹' (↑f '' {n | N ≤ n}) ** exists N ** case intro.intro.intro.left β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε ⊢ ∀ (b : ℕ), N ≤ b → b ∈ ↑f ⁻¹' (↑f '' {n | N ≤ n}) ** intro b hb ** case intro.intro.intro.left β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε b : ℕ hb : N ≤ b ⊢ b ∈ ↑f ⁻¹' (↑f '' {n | N ≤ n}) ** exists b ** case intro.intro.intro.right β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε ⊢ (↑f '' {n | N ≤ n}) ×ˢ (↑f '' {n | N ≤ n}) ⊆ s ** rintro ⟨a, b⟩ ⟨⟨a', ⟨ha'1, ha'2⟩⟩, ⟨b', ⟨hb'1, hb'2⟩⟩⟩ ** case intro.intro.intro.right.mk.intro.intro.intro.intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε a b : β a' : ℕ ha'1 : a' ∈ {n | N ≤ n} ha'2 : ↑f a' = (a, b).1 b' : ℕ hb'1 : b' ∈ {n | N ≤ n} hb'2 : ↑f b' = (a, b).2 ⊢ (a, b) ∈ s ** dsimp at ha'1 ha'2 hb'1 hb'2 ** case intro.intro.intro.right.mk.intro.intro.intro.intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε a b : β a' : ℕ ha'1 : N ≤ a' ha'2 : ↑f a' = a b' : ℕ hb'1 : N ≤ b' hb'2 : ↑f b' = b ⊢ (a, b) ∈ s ** rw [← ha'2, ← hb'2] ** case intro.intro.intro.right.mk.intro.intro.intro.intro.intro β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε a b : β a' : ℕ ha'1 : N ≤ a' ha'2 : ↑f a' = a b' : ℕ hb'1 : N ≤ b' hb'2 : ↑f b' = b ⊢ (↑f a', ↑f b') ∈ s ** apply hεs ** case intro.intro.intro.right.mk.intro.intro.intro.intro.intro.a β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε a b : β a' : ℕ ha'1 : N ≤ a' ha'2 : ↑f a' = a b' : ℕ hb'1 : N ≤ b' hb'2 : ↑f b' = b ⊢ dist (↑f a') (↑f b') < ε ** rw [dist_eq_norm] ** case intro.intro.intro.right.mk.intro.intro.intro.intro.intro.a β : Type v inst✝ : NormedField β f : CauSeq β norm s : Set (β × β) hs : s ∈ uniformity β ε : ℝ hε : ε > 0 hεs : ∀ {a b : β}, dist a b < ε → (a, b) ∈ s N : ℕ hN : ∀ (j : ℕ), j ≥ N → ∀ (k : ℕ), k ≥ N → ‖↑f j - ↑f k‖ < ε a b : β a' : ℕ ha'1 : N ≤ a' ha'2 : ↑f a' = a b' : ℕ hb'1 : N ≤ b' hb'2 : ↑f b' = b ⊢ ‖↑f a' - ↑f b'‖ < ε ** apply hN <;> assumption ** Qed
Metric.equicontinuousAt_iff_pair ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β ⊢ EquicontinuousAt F x₀ ↔ ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε ** rw [equicontinuousAt_iff_pair] ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β ⊢ (∀ (U : Set (α × α)), U ∈ 𝓤 α → ∃ V, V ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U) ↔ ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε ** constructor <;> intro H ** case mp α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β H : ∀ (U : Set (α × α)), U ∈ 𝓤 α → ∃ V, V ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U ⊢ ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε ** intro ε hε ** case mp α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β H : ∀ (U : Set (α × α)), U ∈ 𝓤 α → ∃ V, V ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U ε : ℝ hε : ε > 0 ⊢ ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε ** exact H _ (dist_mem_uniformity hε) ** case mpr α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β H : ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε ⊢ ∀ (U : Set (α × α)), U ∈ 𝓤 α → ∃ V, V ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U ** intro U hU ** case mpr α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β H : ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε U : Set (α × α) hU : U ∈ 𝓤 α ⊢ ∃ V, V ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U ** rcases mem_uniformity_dist.mp hU with ⟨ε, hε, hεU⟩ ** case mpr.intro.intro α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β H : ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε U : Set (α × α) hU : U ∈ 𝓤 α ε : ℝ hε : ε > 0 hεU : ∀ {a b : α}, dist a b < ε → (a, b) ∈ U ⊢ ∃ V, V ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U ** refine' Exists.imp (fun V => And.imp_right fun h => _) (H _ hε) ** case mpr.intro.intro α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β F : ι → β → α x₀ : β H : ∀ (ε : ℝ), ε > 0 → ∃ U, U ∈ 𝓝 x₀ ∧ ∀ (x : β), x ∈ U → ∀ (x' : β), x' ∈ U → ∀ (i : ι), dist (F i x) (F i x') < ε U : Set (α × α) hU : U ∈ 𝓤 α ε : ℝ hε : ε > 0 hεU : ∀ {a b : α}, dist a b < ε → (a, b) ∈ U V : Set β h : ∀ (x : β), x ∈ V → ∀ (x' : β), x' ∈ V → ∀ (i : ι), dist (F i x) (F i x') < ε ⊢ ∀ (x : β), x ∈ V → ∀ (y : β), y ∈ V → ∀ (i : ι), (F i x, F i y) ∈ U ** exact fun x hx x' hx' i => hεU (h _ hx _ hx' i) ** Qed
Metric.equicontinuousAt_of_continuity_modulus ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β x₀ : β b : β → ℝ b_lim : Tendsto b (𝓝 x₀) (𝓝 0) F : ι → β → α H : ∀ᶠ (x : β) in 𝓝 x₀, ∀ (i : ι), dist (F i x₀) (F i x) ≤ b x ⊢ EquicontinuousAt F x₀ ** rw [Metric.equicontinuousAt_iff_right] ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β x₀ : β b : β → ℝ b_lim : Tendsto b (𝓝 x₀) (𝓝 0) F : ι → β → α H : ∀ᶠ (x : β) in 𝓝 x₀, ∀ (i : ι), dist (F i x₀) (F i x) ≤ b x ⊢ ∀ (ε : ℝ), ε > 0 → ∀ᶠ (x : β) in 𝓝 x₀, ∀ (i : ι), dist (F i x₀) (F i x) < ε ** intro ε ε0 ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : TopologicalSpace β x₀ : β b : β → ℝ b_lim : Tendsto b (𝓝 x₀) (𝓝 0) F : ι → β → α H : ∀ᶠ (x : β) in 𝓝 x₀, ∀ (i : ι), dist (F i x₀) (F i x) ≤ b x ε : ℝ ε0 : ε > 0 ⊢ ∀ᶠ (x : β) in 𝓝 x₀, ∀ (i : ι), dist (F i x₀) (F i x) < ε ** filter_upwards [Filter.mem_map.mp <| b_lim (Iio_mem_nhds ε0), H] using fun x hx₁ hx₂ i => (hx₂ i).trans_lt hx₁ ** Qed
Metric.uniformEquicontinuous_of_continuity_modulus ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ⊢ UniformEquicontinuous F ** rw [Metric.uniformEquicontinuous_iff] ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ⊢ ∀ (ε : ℝ), ε > 0 → ∃ δ, δ > 0 ∧ ∀ (x y : β), dist x y < δ → ∀ (i : ι), dist (F i x) (F i y) < ε ** intro ε ε0 ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ε : ℝ ε0 : ε > 0 ⊢ ∃ δ, δ > 0 ∧ ∀ (x y : β), dist x y < δ → ∀ (i : ι), dist (F i x) (F i y) < ε ** rcases tendsto_nhds_nhds.1 b_lim ε ε0 with ⟨δ, δ0, hδ⟩ ** case intro.intro α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ε : ℝ ε0 : ε > 0 δ : ℝ δ0 : δ > 0 hδ : ∀ {x : ℝ}, dist x 0 < δ → dist (b x) 0 < ε ⊢ ∃ δ, δ > 0 ∧ ∀ (x y : β), dist x y < δ → ∀ (i : ι), dist (F i x) (F i y) < ε ** refine' ⟨δ, δ0, fun x y hxy i => _⟩ ** case intro.intro α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ε : ℝ ε0 : ε > 0 δ : ℝ δ0 : δ > 0 hδ : ∀ {x : ℝ}, dist x 0 < δ → dist (b x) 0 < ε x y : β hxy : dist x y < δ i : ι ⊢ dist (F i x) (F i y) < ε ** calc dist (F i x) (F i y) ≤ b (dist x y) := H x y i _ ≤ |b (dist x y)| := (le_abs_self _) _ = dist (b (dist x y)) 0 := by simp [Real.dist_eq] _ < ε := hδ (by simpa only [Real.dist_eq, tsub_zero, abs_dist] using hxy) ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ε : ℝ ε0 : ε > 0 δ : ℝ δ0 : δ > 0 hδ : ∀ {x : ℝ}, dist x 0 < δ → dist (b x) 0 < ε x y : β hxy : dist x y < δ i : ι ⊢ |b (dist x y)| = dist (b (dist x y)) 0 ** simp [Real.dist_eq] ** α : Type u_1 β : Type u_2 ι✝ : Type u_3 inst✝¹ : PseudoMetricSpace α ι : Type u_4 inst✝ : PseudoMetricSpace β b : ℝ → ℝ b_lim : Tendsto b (𝓝 0) (𝓝 0) F : ι → β → α H : ∀ (x y : β) (i : ι), dist (F i x) (F i y) ≤ b (dist x y) ε : ℝ ε0 : ε > 0 δ : ℝ δ0 : δ > 0 hδ : ∀ {x : ℝ}, dist x 0 < δ → dist (b x) 0 < ε x y : β hxy : dist x y < δ i : ι ⊢ dist (dist x y) 0 < δ ** simpa only [Real.dist_eq, tsub_zero, abs_dist] using hxy ** Qed
tendsto_atTop_isLUB ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f ha : IsLUB (range f) a ⊢ Tendsto f atTop (𝓝 a) ** suffices : Tendsto (rangeFactorization f) atTop atTop ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f ha : IsLUB (range f) a this : Tendsto (rangeFactorization f) atTop atTop ⊢ Tendsto f atTop (𝓝 a) case this α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f ha : IsLUB (range f) a ⊢ Tendsto (rangeFactorization f) atTop atTop ** exact (SupConvergenceClass.tendsto_coe_atTop_isLUB _ _ ha).comp this ** case this α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f ha : IsLUB (range f) a ⊢ Tendsto (rangeFactorization f) atTop atTop ** exact h_mono.rangeFactorization.tendsto_atTop_atTop fun b => b.2.imp fun a ha => ha.ge ** Qed
tendsto_atBot_isLUB ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : SupConvergenceClass α f : ι → α a : α h_anti : Antitone f ha : IsLUB (range f) a ⊢ Tendsto f atBot (𝓝 a) ** convert tendsto_atTop_isLUB h_anti.dual_left ha using 1 ** Qed
tendsto_atBot_isGLB ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : InfConvergenceClass α f : ι → α a : α h_mono : Monotone f ha : IsGLB (range f) a ⊢ Tendsto f atBot (𝓝 a) ** convert tendsto_atTop_isLUB h_mono.dual ha.dual using 1 ** Qed
tendsto_atTop_isGLB ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : InfConvergenceClass α f : ι → α a : α h_anti : Antitone f ha : IsGLB (range f) a ⊢ Tendsto f atTop (𝓝 a) ** convert tendsto_atBot_isLUB h_anti.dual ha.dual using 1 ** Qed
tendsto_atTop_ciSup ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : ConditionallyCompleteLattice α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f hbdd : BddAbove (range f) ⊢ Tendsto f atTop (𝓝 (⨆ i, f i)) ** cases isEmpty_or_nonempty ι ** case inl α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : ConditionallyCompleteLattice α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f hbdd : BddAbove (range f) h✝ : IsEmpty ι ⊢ Tendsto f atTop (𝓝 (⨆ i, f i)) case inr α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : ConditionallyCompleteLattice α inst✝ : SupConvergenceClass α f : ι → α a : α h_mono : Monotone f hbdd : BddAbove (range f) h✝ : Nonempty ι ⊢ Tendsto f atTop (𝓝 (⨆ i, f i)) ** exacts [tendsto_of_isEmpty, tendsto_atTop_isLUB h_mono (isLUB_ciSup hbdd)] ** Qed
tendsto_atBot_ciSup ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : ConditionallyCompleteLattice α inst✝ : SupConvergenceClass α f : ι → α a : α h_anti : Antitone f hbdd : BddAbove (range f) ⊢ Tendsto f atBot (𝓝 (⨆ i, f i)) ** convert tendsto_atTop_ciSup h_anti.dual hbdd.dual using 1 ** Qed
tendsto_atBot_ciInf ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : ConditionallyCompleteLattice α inst✝ : InfConvergenceClass α f : ι → α a : α h_mono : Monotone f hbdd : BddBelow (range f) ⊢ Tendsto f atBot (𝓝 (⨅ i, f i)) ** convert tendsto_atTop_ciSup h_mono.dual hbdd.dual using 1 ** Qed
tendsto_atTop_ciInf ** α : Type u_1 β : Type u_2 ι : Type u_3 inst✝³ : Preorder ι inst✝² : TopologicalSpace α inst✝¹ : ConditionallyCompleteLattice α inst✝ : InfConvergenceClass α f : ι → α a : α h_anti : Antitone f hbdd : BddBelow (range f) ⊢ Tendsto f atTop (𝓝 (⨅ i, f i)) ** convert tendsto_atBot_ciSup h_anti.dual hbdd.dual using 1 ** Qed
tendsto_iff_tendsto_subseq_of_monotone ** α✝ : Type u_1 β : Type u_2 ι₁ : Type u_3 ι₂ : Type u_4 α : Type u_5 inst✝⁶ : SemilatticeSup ι₁ inst✝⁵ : Preorder ι₂ inst✝⁴ : Nonempty ι₁ inst✝³ : TopologicalSpace α inst✝² : ConditionallyCompleteLinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α f : ι₂ → α φ : ι₁ → ι₂ l : α hf : Monotone f hg : Tendsto φ atTop atTop ⊢ Tendsto f atTop (𝓝 l) ↔ Tendsto (f ∘ φ) atTop (𝓝 l) ** constructor <;> intro h ** case mp α✝ : Type u_1 β : Type u_2 ι₁ : Type u_3 ι₂ : Type u_4 α : Type u_5 inst✝⁶ : SemilatticeSup ι₁ inst✝⁵ : Preorder ι₂ inst✝⁴ : Nonempty ι₁ inst✝³ : TopologicalSpace α inst✝² : ConditionallyCompleteLinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α f : ι₂ → α φ : ι₁ → ι₂ l : α hf : Monotone f hg : Tendsto φ atTop atTop h : Tendsto f atTop (𝓝 l) ⊢ Tendsto (f ∘ φ) atTop (𝓝 l) ** exact h.comp hg ** case mpr α✝ : Type u_1 β : Type u_2 ι₁ : Type u_3 ι₂ : Type u_4 α : Type u_5 inst✝⁶ : SemilatticeSup ι₁ inst✝⁵ : Preorder ι₂ inst✝⁴ : Nonempty ι₁ inst✝³ : TopologicalSpace α inst✝² : ConditionallyCompleteLinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α f : ι₂ → α φ : ι₁ → ι₂ l : α hf : Monotone f hg : Tendsto φ atTop atTop h : Tendsto (f ∘ φ) atTop (𝓝 l) ⊢ Tendsto f atTop (𝓝 l) ** rcases tendsto_of_monotone hf with (h' | ⟨l', hl'⟩) ** case mpr.inl α✝ : Type u_1 β : Type u_2 ι₁ : Type u_3 ι₂ : Type u_4 α : Type u_5 inst✝⁶ : SemilatticeSup ι₁ inst✝⁵ : Preorder ι₂ inst✝⁴ : Nonempty ι₁ inst✝³ : TopologicalSpace α inst✝² : ConditionallyCompleteLinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α f : ι₂ → α φ : ι₁ → ι₂ l : α hf : Monotone f hg : Tendsto φ atTop atTop h : Tendsto (f ∘ φ) atTop (𝓝 l) h' : Tendsto f atTop atTop ⊢ Tendsto f atTop (𝓝 l) ** exact (not_tendsto_atTop_of_tendsto_nhds h (h'.comp hg)).elim ** case mpr.inr.intro α✝ : Type u_1 β : Type u_2 ι₁ : Type u_3 ι₂ : Type u_4 α : Type u_5 inst✝⁶ : SemilatticeSup ι₁ inst✝⁵ : Preorder ι₂ inst✝⁴ : Nonempty ι₁ inst✝³ : TopologicalSpace α inst✝² : ConditionallyCompleteLinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α f : ι₂ → α φ : ι₁ → ι₂ l : α hf : Monotone f hg : Tendsto φ atTop atTop h : Tendsto (f ∘ φ) atTop (𝓝 l) l' : α hl' : Tendsto f atTop (𝓝 l') ⊢ Tendsto f atTop (𝓝 l) ** rwa [tendsto_nhds_unique h (hl'.comp hg)] ** Qed
isLUB_of_tendsto_atTop ** α : Type u_1 β : Type u_2 inst✝⁴ : TopologicalSpace α inst✝³ : Preorder α inst✝² : OrderClosedTopology α inst✝¹ : Nonempty β inst✝ : SemilatticeSup β f : β → α a : α hf : Monotone f ha : Tendsto f atTop (𝓝 a) ⊢ IsLUB (range f) a ** constructor ** case left α : Type u_1 β : Type u_2 inst✝⁴ : TopologicalSpace α inst✝³ : Preorder α inst✝² : OrderClosedTopology α inst✝¹ : Nonempty β inst✝ : SemilatticeSup β f : β → α a : α hf : Monotone f ha : Tendsto f atTop (𝓝 a) ⊢ a ∈ upperBounds (range f) ** rintro _ ⟨b, rfl⟩ ** case left.intro α : Type u_1 β : Type u_2 inst✝⁴ : TopologicalSpace α inst✝³ : Preorder α inst✝² : OrderClosedTopology α inst✝¹ : Nonempty β inst✝ : SemilatticeSup β f : β → α a : α hf : Monotone f ha : Tendsto f atTop (𝓝 a) b : β ⊢ f b ≤ a ** exact hf.ge_of_tendsto ha b ** case right α : Type u_1 β : Type u_2 inst✝⁴ : TopologicalSpace α inst✝³ : Preorder α inst✝² : OrderClosedTopology α inst✝¹ : Nonempty β inst✝ : SemilatticeSup β f : β → α a : α hf : Monotone f ha : Tendsto f atTop (𝓝 a) ⊢ a ∈ lowerBounds (upperBounds (range f)) ** exact fun _ hb => le_of_tendsto' ha fun x => hb (Set.mem_range_self x) ** Qed
ContinuousSMul.of_nhds_zero ** R : Type u_1 M : Type u_2 inst✝⁶ : Ring R inst✝⁵ : TopologicalSpace R inst✝⁴ : TopologicalSpace M inst✝³ : AddCommGroup M inst✝² : Module R M inst✝¹ : TopologicalRing R inst✝ : TopologicalAddGroup M hmul : Tendsto (fun p => p.1 • p.2) (𝓝 0 ×ˢ 𝓝 0) (𝓝 0) hmulleft : ∀ (m : M), Tendsto (fun a => a • m) (𝓝 0) (𝓝 0) hmulright : ∀ (a : R), Tendsto (fun m => a • m) (𝓝 0) (𝓝 0) ⊢ Continuous fun p => p.1 • p.2 ** refine continuous_of_continuousAt_zero₂ (AddMonoidHom.smul : R →+ M →+ M) ?_ ?_ ?_ <;> simpa [ContinuousAt, nhds_prod_eq] ** Qed
Submodule.eq_top_of_nonempty_interior' ** R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M hs : Set.Nonempty (interior ↑s) ⊢ s = ⊤ ** rcases hs with ⟨y, hy⟩ ** case intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : y ∈ interior ↑s ⊢ s = ⊤ ** refine' Submodule.eq_top_iff'.2 fun x => _ ** case intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : y ∈ interior ↑s x : M ⊢ x ∈ s ** rw [mem_interior_iff_mem_nhds] at hy ** case intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : ↑s ∈ 𝓝 y x : M ⊢ x ∈ s ** have : Tendsto (fun c : R => y + c • x) (𝓝[{ x : R | IsUnit x }] 0) (𝓝 (y + (0 : R) • x)) := tendsto_const_nhds.add ((tendsto_nhdsWithin_of_tendsto_nhds tendsto_id).smul tendsto_const_nhds) ** case intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : ↑s ∈ 𝓝 y x : M this : Tendsto (fun c => y + c • x) (𝓝[{x | IsUnit x}] 0) (𝓝 (y + 0 • x)) ⊢ x ∈ s ** rw [zero_smul, add_zero] at this ** case intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : ↑s ∈ 𝓝 y x : M this : Tendsto (fun c => y + c • x) (𝓝[{x | IsUnit x}] 0) (𝓝 y) ⊢ x ∈ s ** obtain ⟨_, hu : y + _ • _ ∈ s, u, rfl⟩ := nonempty_of_mem (inter_mem (Filter.mem_map.1 (this hy)) self_mem_nhdsWithin) ** case intro.intro.intro.intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : ↑s ∈ 𝓝 y x : M this : Tendsto (fun c => y + c • x) (𝓝[{x | IsUnit x}] 0) (𝓝 y) u : Rˣ hu : y + ↑u • x ∈ s ⊢ x ∈ s ** have hy' : y ∈ ↑s := mem_of_mem_nhds hy ** case intro.intro.intro.intro R : Type u_1 M : Type u_2 inst✝⁷ : Ring R inst✝⁶ : TopologicalSpace R inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : ContinuousAdd M inst✝² : Module R M inst✝¹ : ContinuousSMul R M inst✝ : NeBot (𝓝[{x | IsUnit x}] 0) s : Submodule R M y : M hy : ↑s ∈ 𝓝 y x : M this : Tendsto (fun c => y + c • x) (𝓝[{x | IsUnit x}] 0) (𝓝 y) u : Rˣ hu : y + ↑u • x ∈ s hy' : y ∈ ↑s ⊢ x ∈ s ** rwa [s.add_mem_iff_right hy', ← Units.smul_def, s.smul_mem_iff' u] at hu ** Qed
Module.punctured_nhds_neBot ** R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x : M ⊢ NeBot (𝓝[{x}ᶜ] x) ** rcases exists_ne (0 : M) with ⟨y, hy⟩ ** case intro R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 ⊢ NeBot (𝓝[{x}ᶜ] x) ** suffices : Tendsto (fun c : R => x + c • y) (𝓝[≠] 0) (𝓝[≠] x) ** case intro R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 this : Tendsto (fun c => x + c • y) (𝓝[{0}ᶜ] 0) (𝓝[{x}ᶜ] x) ⊢ NeBot (𝓝[{x}ᶜ] x) case this R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 ⊢ Tendsto (fun c => x + c • y) (𝓝[{0}ᶜ] 0) (𝓝[{x}ᶜ] x) ** exact this.neBot ** case this R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 ⊢ Tendsto (fun c => x + c • y) (𝓝[{0}ᶜ] 0) (𝓝[{x}ᶜ] x) ** refine' Tendsto.inf _ (tendsto_principal_principal.2 <| _) ** case this.refine'_1 R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 ⊢ Tendsto (fun c => x + c • y) (𝓝 0) (𝓝 x) ** convert tendsto_const_nhds.add ((@tendsto_id R _).smul_const y) ** case h.e'_5.h.e'_3 R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 ⊢ x = x + 0 • y ** rw [zero_smul, add_zero] ** case this.refine'_2 R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 ⊢ ∀ (a : R), a ∈ {0}ᶜ → x + a • y ∈ {x}ᶜ ** intro c hc ** case this.refine'_2 R : Type u_1 M : Type u_2 inst✝⁹ : Ring R inst✝⁸ : TopologicalSpace R inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : ContinuousAdd M inst✝⁴ : Module R M inst✝³ : ContinuousSMul R M inst✝² : Nontrivial M inst✝¹ : NeBot (𝓝[{0}ᶜ] 0) inst✝ : NoZeroSMulDivisors R M x y : M hy : y ≠ 0 c : R hc : c ∈ {0}ᶜ ⊢ x + c • y ∈ {x}ᶜ ** simpa [hy] using hc ** Qed
continuousSMul_induced ** ι : Type u_1 R : Type u_2 M₁ : Type u_3 M₂ : Type u_4 inst✝⁵ : Semiring R inst✝⁴ : AddCommMonoid M₁ inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₁ inst✝¹ : Module R M₂ u : TopologicalSpace R t : TopologicalSpace M₂ inst✝ : ContinuousSMul R M₂ f : M₁ →ₗ[R] M₂ ⊢ ContinuousSMul R M₁ ** let _ : TopologicalSpace M₁ := t.induced f ** ι : Type u_1 R : Type u_2 M₁ : Type u_3 M₂ : Type u_4 inst✝⁵ : Semiring R inst✝⁴ : AddCommMonoid M₁ inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₁ inst✝¹ : Module R M₂ u : TopologicalSpace R t : TopologicalSpace M₂ inst✝ : ContinuousSMul R M₂ f : M₁ →ₗ[R] M₂ x✝ : TopologicalSpace M₁ := TopologicalSpace.induced (↑f) t ⊢ ContinuousSMul R M₁ ** refine' ⟨continuous_induced_rng.2 _⟩ ** ι : Type u_1 R : Type u_2 M₁ : Type u_3 M₂ : Type u_4 inst✝⁵ : Semiring R inst✝⁴ : AddCommMonoid M₁ inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₁ inst✝¹ : Module R M₂ u : TopologicalSpace R t : TopologicalSpace M₂ inst✝ : ContinuousSMul R M₂ f : M₁ →ₗ[R] M₂ x✝ : TopologicalSpace M₁ := TopologicalSpace.induced (↑f) t ⊢ Continuous (↑f ∘ fun p => p.1 • p.2) ** simp_rw [Function.comp, f.map_smul] ** ι : Type u_1 R : Type u_2 M₁ : Type u_3 M₂ : Type u_4 inst✝⁵ : Semiring R inst✝⁴ : AddCommMonoid M₁ inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₁ inst✝¹ : Module R M₂ u : TopologicalSpace R t : TopologicalSpace M₂ inst✝ : ContinuousSMul R M₂ f : M₁ →ₗ[R] M₂ x✝ : TopologicalSpace M₁ := TopologicalSpace.induced (↑f) t ⊢ Continuous fun x => x.1 • ↑f x.2 ** exact continuous_fst.smul (continuous_induced_dom.comp continuous_snd) ** Qed
Submodule.closure_subset_topologicalClosure_span ** R R' : Type u M M' : Type v inst✝¹⁰ : Semiring R inst✝⁹ : Ring R' inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : TopologicalSpace M' inst✝⁵ : AddCommGroup M' inst✝⁴ : Module R M inst✝³ : ContinuousConstSMul R M inst✝² : Module R' M' inst✝¹ : ContinuousConstSMul R' M' inst✝ : ContinuousAdd M s : Set M ⊢ closure s ⊆ ↑(topologicalClosure (span R s)) ** rw [Submodule.topologicalClosure_coe] ** R R' : Type u M M' : Type v inst✝¹⁰ : Semiring R inst✝⁹ : Ring R' inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : TopologicalSpace M' inst✝⁵ : AddCommGroup M' inst✝⁴ : Module R M inst✝³ : ContinuousConstSMul R M inst✝² : Module R' M' inst✝¹ : ContinuousConstSMul R' M' inst✝ : ContinuousAdd M s : Set M ⊢ closure s ⊆ closure ↑(span R s) ** exact closure_mono subset_span ** Qed
Submodule.dense_iff_topologicalClosure_eq_top ** R R' : Type u M M' : Type v inst✝¹⁰ : Semiring R inst✝⁹ : Ring R' inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : TopologicalSpace M' inst✝⁵ : AddCommGroup M' inst✝⁴ : Module R M inst✝³ : ContinuousConstSMul R M inst✝² : Module R' M' inst✝¹ : ContinuousConstSMul R' M' inst✝ : ContinuousAdd M s : Submodule R M ⊢ Dense ↑s ↔ topologicalClosure s = ⊤ ** rw [← SetLike.coe_set_eq, dense_iff_closure_eq] ** R R' : Type u M M' : Type v inst✝¹⁰ : Semiring R inst✝⁹ : Ring R' inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : TopologicalSpace M' inst✝⁵ : AddCommGroup M' inst✝⁴ : Module R M inst✝³ : ContinuousConstSMul R M inst✝² : Module R' M' inst✝¹ : ContinuousConstSMul R' M' inst✝ : ContinuousAdd M s : Submodule R M ⊢ closure ↑s = Set.univ ↔ ↑(topologicalClosure s) = ↑⊤ ** simp ** Qed
Submodule.isClosed_or_dense_of_isCoatom ** R R' : Type u M M' : Type v inst✝¹⁰ : Semiring R inst✝⁹ : Ring R' inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : TopologicalSpace M' inst✝⁵ : AddCommGroup M' inst✝⁴ : Module R M inst✝³ : ContinuousConstSMul R M inst✝² : Module R' M' inst✝¹ : ContinuousConstSMul R' M' inst✝ : ContinuousAdd M s : Submodule R M hs : IsCoatom s ⊢ IsClosed ↑s ∨ Dense ↑s ** refine (hs.le_iff.mp s.le_topologicalClosure).symm.imp ?_ dense_iff_topologicalClosure_eq_top.mpr ** R R' : Type u M M' : Type v inst✝¹⁰ : Semiring R inst✝⁹ : Ring R' inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : TopologicalSpace M' inst✝⁵ : AddCommGroup M' inst✝⁴ : Module R M inst✝³ : ContinuousConstSMul R M inst✝² : Module R' M' inst✝¹ : ContinuousConstSMul R' M' inst✝ : ContinuousAdd M s : Submodule R M hs : IsCoatom s ⊢ topologicalClosure s = s → IsClosed ↑s ** exact fun h ↦ h ▸ isClosed_closure ** Qed
LinearMap.continuous_on_pi ** ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M ⊢ Continuous ↑f ** cases nonempty_fintype ι ** case intro ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι ⊢ Continuous ↑f ** classical have : (f : (ι → R) → M) = fun x => ∑ i : ι, x i • f fun j => if i = j then 1 else 0 := by ext x exact f.pi_apply_eq_sum_univ x rw [this] refine continuous_finset_sum _ fun i _ => ?_ exact (continuous_apply i).smul continuous_const ** case intro ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι ⊢ Continuous ↑f ** have : (f : (ι → R) → M) = fun x => ∑ i : ι, x i • f fun j => if i = j then 1 else 0 := by ext x exact f.pi_apply_eq_sum_univ x ** case intro ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι this : ↑f = fun x => ∑ i : ι, x i • ↑f fun j => if i = j then 1 else 0 ⊢ Continuous ↑f ** rw [this] ** case intro ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι this : ↑f = fun x => ∑ i : ι, x i • ↑f fun j => if i = j then 1 else 0 ⊢ Continuous fun x => ∑ i : ι, x i • ↑f fun j => if i = j then 1 else 0 ** refine continuous_finset_sum _ fun i _ => ?_ ** case intro ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι this : ↑f = fun x => ∑ i : ι, x i • ↑f fun j => if i = j then 1 else 0 i : ι x✝ : i ∈ Finset.univ ⊢ Continuous fun x => x i • ↑f fun j => if i = j then 1 else 0 ** exact (continuous_apply i).smul continuous_const ** ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι ⊢ ↑f = fun x => ∑ i : ι, x i • ↑f fun j => if i = j then 1 else 0 ** ext x ** case h ι : Type u_1 R : Type u_2 M : Type u_3 inst✝⁷ : Finite ι inst✝⁶ : Semiring R inst✝⁵ : TopologicalSpace R inst✝⁴ : AddCommMonoid M inst✝³ : Module R M inst✝² : TopologicalSpace M inst✝¹ : ContinuousAdd M inst✝ : ContinuousSMul R M f : (ι → R) →ₗ[R] M val✝ : Fintype ι x : ι → R ⊢ ↑f x = ∑ i : ι, x i • ↑f fun j => if i = j then 1 else 0 ** exact f.pi_apply_eq_sum_univ x ** Qed
ContinuousLinearMap.coe_injective ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ ⊢ Function.Injective toLinearMap ** intro f g H ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ f g : M₁ →SL[σ₁₂] M₂ H : ↑f = ↑g ⊢ f = g ** cases f ** case mk R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ g : M₁ →SL[σ₁₂] M₂ toLinearMap✝ : M₁ →ₛₗ[σ₁₂] M₂ cont✝ : Continuous toLinearMap✝.toFun H : ↑(mk toLinearMap✝) = ↑g ⊢ mk toLinearMap✝ = g ** cases g ** case mk.mk R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ toLinearMap✝¹ : M₁ →ₛₗ[σ₁₂] M₂ cont✝¹ : Continuous toLinearMap✝¹.toFun toLinearMap✝ : M₁ →ₛₗ[σ₁₂] M₂ cont✝ : Continuous toLinearMap✝.toFun H : ↑(mk toLinearMap✝¹) = ↑(mk toLinearMap✝) ⊢ mk toLinearMap✝¹ = mk toLinearMap✝ ** congr ** Qed
ContinuousLinearMap.map_smul ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : Module R₁ M₂ f : M₁ →L[R₁] M₂ c : R₁ x : M₁ ⊢ ↑f (c • x) = c • ↑f x ** simp only [RingHom.id_apply, ContinuousLinearMap.map_smulₛₗ] ** Qed
DenseRange.topologicalClosure_map_submodule ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²³ : Semiring R₁ inst✝²² : Semiring R₂ inst✝²¹ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝²⁰ : TopologicalSpace M₁ inst✝¹⁹ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁸ : TopologicalSpace M'₁ inst✝¹⁷ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁶ : TopologicalSpace M₂ inst✝¹⁵ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁴ : TopologicalSpace M₃ inst✝¹³ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹² : TopologicalSpace M₄ inst✝¹¹ : AddCommMonoid M₄ inst✝¹⁰ : Module R₁ M₁ inst✝⁹ : Module R₁ M'₁ inst✝⁸ : Module R₂ M₂ inst✝⁷ : Module R₃ M₃ inst✝⁶ : RingHomSurjective σ₁₂ inst✝⁵ : TopologicalSpace R₁ inst✝⁴ : TopologicalSpace R₂ inst✝³ : ContinuousSMul R₁ M₁ inst✝² : ContinuousAdd M₁ inst✝¹ : ContinuousSMul R₂ M₂ inst✝ : ContinuousAdd M₂ f : M₁ →SL[σ₁₂] M₂ hf' : DenseRange ↑f s : Submodule R₁ M₁ hs : Submodule.topologicalClosure s = ⊤ ⊢ Submodule.topologicalClosure (Submodule.map (↑f) s) = ⊤ ** rw [SetLike.ext'_iff] at hs ⊢ ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²³ : Semiring R₁ inst✝²² : Semiring R₂ inst✝²¹ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝²⁰ : TopologicalSpace M₁ inst✝¹⁹ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁸ : TopologicalSpace M'₁ inst✝¹⁷ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁶ : TopologicalSpace M₂ inst✝¹⁵ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁴ : TopologicalSpace M₃ inst✝¹³ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹² : TopologicalSpace M₄ inst✝¹¹ : AddCommMonoid M₄ inst✝¹⁰ : Module R₁ M₁ inst✝⁹ : Module R₁ M'₁ inst✝⁸ : Module R₂ M₂ inst✝⁷ : Module R₃ M₃ inst✝⁶ : RingHomSurjective σ₁₂ inst✝⁵ : TopologicalSpace R₁ inst✝⁴ : TopologicalSpace R₂ inst✝³ : ContinuousSMul R₁ M₁ inst✝² : ContinuousAdd M₁ inst✝¹ : ContinuousSMul R₂ M₂ inst✝ : ContinuousAdd M₂ f : M₁ →SL[σ₁₂] M₂ hf' : DenseRange ↑f s : Submodule R₁ M₁ hs✝ : Submodule.topologicalClosure s = ⊤ hs : ↑(Submodule.topologicalClosure s) = ↑⊤ ⊢ ↑(Submodule.topologicalClosure (Submodule.map (↑f) s)) = ↑⊤ ** simp only [Submodule.topologicalClosure_coe, Submodule.top_coe, ← dense_iff_closure_eq] at hs ⊢ ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²³ : Semiring R₁ inst✝²² : Semiring R₂ inst✝²¹ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝²⁰ : TopologicalSpace M₁ inst✝¹⁹ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁸ : TopologicalSpace M'₁ inst✝¹⁷ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁶ : TopologicalSpace M₂ inst✝¹⁵ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁴ : TopologicalSpace M₃ inst✝¹³ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹² : TopologicalSpace M₄ inst✝¹¹ : AddCommMonoid M₄ inst✝¹⁰ : Module R₁ M₁ inst✝⁹ : Module R₁ M'₁ inst✝⁸ : Module R₂ M₂ inst✝⁷ : Module R₃ M₃ inst✝⁶ : RingHomSurjective σ₁₂ inst✝⁵ : TopologicalSpace R₁ inst✝⁴ : TopologicalSpace R₂ inst✝³ : ContinuousSMul R₁ M₁ inst✝² : ContinuousAdd M₁ inst✝¹ : ContinuousSMul R₂ M₂ inst✝ : ContinuousAdd M₂ f : M₁ →SL[σ₁₂] M₂ hf' : DenseRange ↑f s : Submodule R₁ M₁ hs✝ : Submodule.topologicalClosure s = ⊤ hs : Dense ↑s ⊢ Dense ↑(Submodule.map (↑f) s) ** exact hf'.dense_image f.continuous hs ** Qed
ContinuousLinearMap.exists_ne_zero ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ f : M₁ →SL[σ₁₂] M₂ hf : f ≠ 0 ⊢ ∃ x, ↑f x ≠ 0 ** by_contra' h ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ f : M₁ →SL[σ₁₂] M₂ hf : f ≠ 0 h : ∀ (x : M₁), ↑f x = 0 ⊢ False ** exact hf (ContinuousLinearMap.ext h) ** Qed
ContinuousLinearMap.coe_eq_id ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁶ : Semiring R₁ inst✝¹⁵ : Semiring R₂ inst✝¹⁴ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ f : M₁ →L[R₁] M₁ ⊢ ↑f = LinearMap.id ↔ f = id R₁ M₁ ** rw [← coe_id, coe_inj] ** Qed
ContinuousLinearMap.coe_sum' ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : ContinuousAdd M₂ ι : Type u_9 t : Finset ι f : ι → M₁ →SL[σ₁₂] M₂ ⊢ ↑(∑ d in t, f d) = ∑ d in t, ↑(f d) ** simp only [← coe_coe, coe_sum, LinearMap.coeFn_sum] ** Qed
ContinuousLinearMap.sum_apply ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : ContinuousAdd M₂ ι : Type u_9 t : Finset ι f : ι → M₁ →SL[σ₁₂] M₂ b : M₁ ⊢ ↑(∑ d in t, f d) b = ∑ d in t, ↑(f d) b ** simp only [coe_sum', Finset.sum_apply] ** Qed
ContinuousLinearMap.comp_zero ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ g : M₂ →SL[σ₂₃] M₃ ⊢ comp g 0 = 0 ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ g : M₂ →SL[σ₂₃] M₃ x✝ : M₁ ⊢ ↑(comp g 0) x✝ = ↑0 x✝ ** simp ** Qed
ContinuousLinearMap.zero_comp ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ f : M₁ →SL[σ₁₂] M₂ ⊢ comp 0 f = 0 ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁷ : Semiring R₁ inst✝¹⁶ : Semiring R₂ inst✝¹⁵ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ f : M₁ →SL[σ₁₂] M₂ x✝ : M₁ ⊢ ↑(comp 0 f) x✝ = ↑0 x✝ ** simp ** Qed
ContinuousLinearMap.comp_add ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁹ : Semiring R₁ inst✝¹⁸ : Semiring R₂ inst✝¹⁷ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁶ : TopologicalSpace M₁ inst✝¹⁵ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁴ : TopologicalSpace M'₁ inst✝¹³ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹² : TopologicalSpace M₂ inst✝¹¹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁰ : TopologicalSpace M₃ inst✝⁹ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁸ : TopologicalSpace M₄ inst✝⁷ : AddCommMonoid M₄ inst✝⁶ : Module R₁ M₁ inst✝⁵ : Module R₁ M'₁ inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹ : ContinuousAdd M₂ inst✝ : ContinuousAdd M₃ g : M₂ →SL[σ₂₃] M₃ f₁ f₂ : M₁ →SL[σ₁₂] M₂ ⊢ comp g (f₁ + f₂) = comp g f₁ + comp g f₂ ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁹ : Semiring R₁ inst✝¹⁸ : Semiring R₂ inst✝¹⁷ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁶ : TopologicalSpace M₁ inst✝¹⁵ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁴ : TopologicalSpace M'₁ inst✝¹³ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹² : TopologicalSpace M₂ inst✝¹¹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁰ : TopologicalSpace M₃ inst✝⁹ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁸ : TopologicalSpace M₄ inst✝⁷ : AddCommMonoid M₄ inst✝⁶ : Module R₁ M₁ inst✝⁵ : Module R₁ M'₁ inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹ : ContinuousAdd M₂ inst✝ : ContinuousAdd M₃ g : M₂ →SL[σ₂₃] M₃ f₁ f₂ : M₁ →SL[σ₁₂] M₂ x✝ : M₁ ⊢ ↑(comp g (f₁ + f₂)) x✝ = ↑(comp g f₁ + comp g f₂) x✝ ** simp ** Qed
ContinuousLinearMap.add_comp ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁸ : Semiring R₁ inst✝¹⁷ : Semiring R₂ inst✝¹⁶ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁵ : TopologicalSpace M₁ inst✝¹⁴ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹³ : TopologicalSpace M'₁ inst✝¹² : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹¹ : TopologicalSpace M₂ inst✝¹⁰ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁹ : TopologicalSpace M₃ inst✝⁸ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁷ : TopologicalSpace M₄ inst✝⁶ : AddCommMonoid M₄ inst✝⁵ : Module R₁ M₁ inst✝⁴ : Module R₁ M'₁ inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ inst✝¹ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝ : ContinuousAdd M₃ g₁ g₂ : M₂ →SL[σ₂₃] M₃ f : M₁ →SL[σ₁₂] M₂ ⊢ comp (g₁ + g₂) f = comp g₁ f + comp g₂ f ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁸ : Semiring R₁ inst✝¹⁷ : Semiring R₂ inst✝¹⁶ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁵ : TopologicalSpace M₁ inst✝¹⁴ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹³ : TopologicalSpace M'₁ inst✝¹² : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹¹ : TopologicalSpace M₂ inst✝¹⁰ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁹ : TopologicalSpace M₃ inst✝⁸ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁷ : TopologicalSpace M₄ inst✝⁶ : AddCommMonoid M₄ inst✝⁵ : Module R₁ M₁ inst✝⁴ : Module R₁ M'₁ inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ inst✝¹ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝ : ContinuousAdd M₃ g₁ g₂ : M₂ →SL[σ₂₃] M₃ f : M₁ →SL[σ₁₂] M₂ x✝ : M₁ ⊢ ↑(comp (g₁ + g₂) f) x✝ = ↑(comp g₁ f + comp g₂ f) x✝ ** simp ** Qed
ContinuousLinearMap.coprod_inl_inr ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁹ : Semiring R₁ inst✝¹⁸ : Semiring R₂ inst✝¹⁷ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁶ : TopologicalSpace M₁ inst✝¹⁵ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁴ : TopologicalSpace M'₁ inst✝¹³ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹² : TopologicalSpace M₂ inst✝¹¹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁰ : TopologicalSpace M₃ inst✝⁹ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁸ : TopologicalSpace M₄ inst✝⁷ : AddCommMonoid M₄ inst✝⁶ : Module R₁ M₁ inst✝⁵ : Module R₁ M'₁ inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝¹ : ContinuousAdd M₁ inst✝ : ContinuousAdd M'₁ ⊢ coprod (inl R₁ M₁ M'₁) (inr R₁ M₁ M'₁) = id R₁ (M₁ × M'₁) ** apply coe_injective ** case a R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝¹⁹ : Semiring R₁ inst✝¹⁸ : Semiring R₂ inst✝¹⁷ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁶ : TopologicalSpace M₁ inst✝¹⁵ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁴ : TopologicalSpace M'₁ inst✝¹³ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹² : TopologicalSpace M₂ inst✝¹¹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁰ : TopologicalSpace M₃ inst✝⁹ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁸ : TopologicalSpace M₄ inst✝⁷ : AddCommMonoid M₄ inst✝⁶ : Module R₁ M₁ inst✝⁵ : Module R₁ M'₁ inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝¹ : ContinuousAdd M₁ inst✝ : ContinuousAdd M'₁ ⊢ ↑(coprod (inl R₁ M₁ M'₁) (inr R₁ M₁ M'₁)) = ↑(id R₁ (M₁ × M'₁)) ** apply LinearMap.coprod_inl_inr ** Qed
ContinuousLinearMap.smulRight_one_one ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁰ : Semiring R₁ inst✝¹⁹ : Semiring R₂ inst✝¹⁸ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁷ : TopologicalSpace M₁ inst✝¹⁶ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁵ : TopologicalSpace M'₁ inst✝¹⁴ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹³ : TopologicalSpace M₂ inst✝¹² : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹¹ : TopologicalSpace M₃ inst✝¹⁰ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁹ : TopologicalSpace M₄ inst✝⁸ : AddCommMonoid M₄ inst✝⁷ : Module R₁ M₁ inst✝⁶ : Module R₁ M'₁ inst✝⁵ : Module R₂ M₂ inst✝⁴ : Module R₃ M₃ inst✝³ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝² : Module R₁ M₂ inst✝¹ : TopologicalSpace R₁ inst✝ : ContinuousSMul R₁ M₂ c : R₁ →L[R₁] M₂ ⊢ smulRight 1 (↑c 1) = c ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁰ : Semiring R₁ inst✝¹⁹ : Semiring R₂ inst✝¹⁸ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁷ : TopologicalSpace M₁ inst✝¹⁶ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁵ : TopologicalSpace M'₁ inst✝¹⁴ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹³ : TopologicalSpace M₂ inst✝¹² : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹¹ : TopologicalSpace M₃ inst✝¹⁰ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁹ : TopologicalSpace M₄ inst✝⁸ : AddCommMonoid M₄ inst✝⁷ : Module R₁ M₁ inst✝⁶ : Module R₁ M'₁ inst✝⁵ : Module R₂ M₂ inst✝⁴ : Module R₃ M₃ inst✝³ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝² : Module R₁ M₂ inst✝¹ : TopologicalSpace R₁ inst✝ : ContinuousSMul R₁ M₂ c : R₁ →L[R₁] M₂ ⊢ ↑(smulRight 1 (↑c 1)) 1 = ↑c 1 ** simp [← ContinuousLinearMap.map_smul_of_tower] ** Qed
ContinuousLinearMap.smulRight_one_eq_iff ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁰ : Semiring R₁ inst✝¹⁹ : Semiring R₂ inst✝¹⁸ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁷ : TopologicalSpace M₁ inst✝¹⁶ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁵ : TopologicalSpace M'₁ inst✝¹⁴ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹³ : TopologicalSpace M₂ inst✝¹² : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹¹ : TopologicalSpace M₃ inst✝¹⁰ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁹ : TopologicalSpace M₄ inst✝⁸ : AddCommMonoid M₄ inst✝⁷ : Module R₁ M₁ inst✝⁶ : Module R₁ M'₁ inst✝⁵ : Module R₂ M₂ inst✝⁴ : Module R₃ M₃ inst✝³ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝² : Module R₁ M₂ inst✝¹ : TopologicalSpace R₁ inst✝ : ContinuousSMul R₁ M₂ f f' : M₂ ⊢ smulRight 1 f = smulRight 1 f' ↔ f = f' ** simp only [ext_ring_iff, smulRight_apply, one_apply, one_smul] ** Qed
ContinuousLinearMap.smulRight_comp ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²¹ : Semiring R₁ inst✝²⁰ : Semiring R₂ inst✝¹⁹ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁸ : TopologicalSpace M₁ inst✝¹⁷ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁶ : TopologicalSpace M'₁ inst✝¹⁵ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁴ : TopologicalSpace M₂ inst✝¹³ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹² : TopologicalSpace M₃ inst✝¹¹ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹⁰ : TopologicalSpace M₄ inst✝⁹ : AddCommMonoid M₄ inst✝⁸ : Module R₁ M₁ inst✝⁷ : Module R₁ M'₁ inst✝⁶ : Module R₂ M₂ inst✝⁵ : Module R₃ M₃ inst✝⁴ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝³ : Module R₁ M₂ inst✝² : TopologicalSpace R₁ inst✝¹ : ContinuousSMul R₁ M₂ inst✝ : ContinuousMul R₁ x : M₂ c : R₁ ⊢ comp (smulRight 1 x) (smulRight 1 c) = smulRight 1 (c • x) ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²¹ : Semiring R₁ inst✝²⁰ : Semiring R₂ inst✝¹⁹ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁸ : TopologicalSpace M₁ inst✝¹⁷ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁶ : TopologicalSpace M'₁ inst✝¹⁵ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁴ : TopologicalSpace M₂ inst✝¹³ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹² : TopologicalSpace M₃ inst✝¹¹ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹⁰ : TopologicalSpace M₄ inst✝⁹ : AddCommMonoid M₄ inst✝⁸ : Module R₁ M₁ inst✝⁷ : Module R₁ M'₁ inst✝⁶ : Module R₂ M₂ inst✝⁵ : Module R₃ M₃ inst✝⁴ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝³ : Module R₁ M₂ inst✝² : TopologicalSpace R₁ inst✝¹ : ContinuousSMul R₁ M₂ inst✝ : ContinuousMul R₁ x : M₂ c : R₁ ⊢ ↑(comp (smulRight 1 x) (smulRight 1 c)) 1 = ↑(smulRight 1 (c • x)) 1 ** simp [mul_smul] ** Qed
ContinuousLinearMap.toSpanSingleton_add ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²² : Semiring R₁ inst✝²¹ : Semiring R₂ inst✝²⁰ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁹ : TopologicalSpace M₁ inst✝¹⁸ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁷ : TopologicalSpace M'₁ inst✝¹⁶ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁵ : TopologicalSpace M₂ inst✝¹⁴ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹³ : TopologicalSpace M₃ inst✝¹² : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹¹ : TopologicalSpace M₄ inst✝¹⁰ : AddCommMonoid M₄ inst✝⁹ : Module R₁ M₁ inst✝⁸ : Module R₁ M'₁ inst✝⁷ : Module R₂ M₂ inst✝⁶ : Module R₃ M₃ inst✝⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝⁴ : Module R₁ M₂ inst✝³ : TopologicalSpace R₁ inst✝² : ContinuousSMul R₁ M₂ inst✝¹ : ContinuousSMul R₁ M₁ inst✝ : ContinuousAdd M₁ x y : M₁ ⊢ toSpanSingleton R₁ (x + y) = toSpanSingleton R₁ x + toSpanSingleton R₁ y ** ext1 ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²² : Semiring R₁ inst✝²¹ : Semiring R₂ inst✝²⁰ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝¹⁹ : TopologicalSpace M₁ inst✝¹⁸ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹⁷ : TopologicalSpace M'₁ inst✝¹⁶ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁵ : TopologicalSpace M₂ inst✝¹⁴ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹³ : TopologicalSpace M₃ inst✝¹² : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹¹ : TopologicalSpace M₄ inst✝¹⁰ : AddCommMonoid M₄ inst✝⁹ : Module R₁ M₁ inst✝⁸ : Module R₁ M'₁ inst✝⁷ : Module R₂ M₂ inst✝⁶ : Module R₃ M₃ inst✝⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝⁴ : Module R₁ M₂ inst✝³ : TopologicalSpace R₁ inst✝² : ContinuousSMul R₁ M₂ inst✝¹ : ContinuousSMul R₁ M₁ inst✝ : ContinuousAdd M₁ x y : M₁ ⊢ ↑(toSpanSingleton R₁ (x + y)) 1 = ↑(toSpanSingleton R₁ x + toSpanSingleton R₁ y) 1 ** simp [toSpanSingleton_apply] ** Qed
ContinuousLinearMap.toSpanSingleton_smul' ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁵ : Semiring R₁ inst✝²⁴ : Semiring R₂ inst✝²³ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝²² : TopologicalSpace M₁ inst✝²¹ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝²⁰ : TopologicalSpace M'₁ inst✝¹⁹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁸ : TopologicalSpace M₂ inst✝¹⁷ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁶ : TopologicalSpace M₃ inst✝¹⁵ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹⁴ : TopologicalSpace M₄ inst✝¹³ : AddCommMonoid M₄ inst✝¹² : Module R₁ M₁ inst✝¹¹ : Module R₁ M'₁ inst✝¹⁰ : Module R₂ M₂ inst✝⁹ : Module R₃ M₃ inst✝⁸ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝⁷ : Module R₁ M₂ inst✝⁶ : TopologicalSpace R₁ inst✝⁵ : ContinuousSMul R₁ M₂ inst✝⁴ : ContinuousSMul R₁ M₁ α : Type u_10 inst✝³ : Monoid α inst✝² : DistribMulAction α M₁ inst✝¹ : ContinuousConstSMul α M₁ inst✝ : SMulCommClass R₁ α M₁ c : α x : M₁ ⊢ toSpanSingleton R₁ (c • x) = c • toSpanSingleton R₁ x ** ext1 ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁵ : Semiring R₁ inst✝²⁴ : Semiring R₂ inst✝²³ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R₁ →+* R₃ M₁ : Type u_4 inst✝²² : TopologicalSpace M₁ inst✝²¹ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝²⁰ : TopologicalSpace M'₁ inst✝¹⁹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁸ : TopologicalSpace M₂ inst✝¹⁷ : AddCommMonoid M₂ M₃ : Type u_7 inst✝¹⁶ : TopologicalSpace M₃ inst✝¹⁵ : AddCommMonoid M₃ M₄ : Type u_8 inst✝¹⁴ : TopologicalSpace M₄ inst✝¹³ : AddCommMonoid M₄ inst✝¹² : Module R₁ M₁ inst✝¹¹ : Module R₁ M'₁ inst✝¹⁰ : Module R₂ M₂ inst✝⁹ : Module R₃ M₃ inst✝⁸ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ F : Type u_9 inst✝⁷ : Module R₁ M₂ inst✝⁶ : TopologicalSpace R₁ inst✝⁵ : ContinuousSMul R₁ M₂ inst✝⁴ : ContinuousSMul R₁ M₁ α : Type u_10 inst✝³ : Monoid α inst✝² : DistribMulAction α M₁ inst✝¹ : ContinuousConstSMul α M₁ inst✝ : SMulCommClass R₁ α M₁ c : α x : M₁ ⊢ ↑(toSpanSingleton R₁ (c • x)) 1 = ↑(c • toSpanSingleton R₁ x) 1 ** rw [toSpanSingleton_apply, smul_apply, toSpanSingleton_apply, smul_comm] ** Qed
ContinuousLinearMap.pi_eq_zero ** R : Type u_1 inst✝⁹ : Semiring R M : Type u_2 inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : Module R M M₂ : Type u_3 inst✝⁵ : TopologicalSpace M₂ inst✝⁴ : AddCommMonoid M₂ inst✝³ : Module R M₂ ι : Type u_4 φ : ι → Type u_5 inst✝² : (i : ι) → TopologicalSpace (φ i) inst✝¹ : (i : ι) → AddCommMonoid (φ i) inst✝ : (i : ι) → Module R (φ i) f : (i : ι) → M →L[R] φ i ⊢ pi f = 0 ↔ ∀ (i : ι), f i = 0 ** simp only [ext_iff, pi_apply, Function.funext_iff] ** R : Type u_1 inst✝⁹ : Semiring R M : Type u_2 inst✝⁸ : TopologicalSpace M inst✝⁷ : AddCommMonoid M inst✝⁶ : Module R M M₂ : Type u_3 inst✝⁵ : TopologicalSpace M₂ inst✝⁴ : AddCommMonoid M₂ inst✝³ : Module R M₂ ι : Type u_4 φ : ι → Type u_5 inst✝² : (i : ι) → TopologicalSpace (φ i) inst✝¹ : (i : ι) → AddCommMonoid (φ i) inst✝ : (i : ι) → Module R (φ i) f : (i : ι) → M →L[R] φ i ⊢ (∀ (x : M) (a : ι), ↑(f a) x = ↑0 x a) ↔ ∀ (i : ι) (x : M), ↑(f i) x = ↑0 x ** exact forall_swap ** Qed
ContinuousLinearMap.map_neg ** R : Type u_1 inst✝¹³ : Ring R R₂ : Type u_2 inst✝¹² : Ring R₂ R₃ : Type u_3 inst✝¹¹ : Ring R₃ M : Type u_4 inst✝¹⁰ : TopologicalSpace M inst✝⁹ : AddCommGroup M M₂ : Type u_5 inst✝⁸ : TopologicalSpace M₂ inst✝⁷ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁶ : TopologicalSpace M₃ inst✝⁵ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁴ : TopologicalSpace M₄ inst✝³ : AddCommGroup M₄ inst✝² : Module R M inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ f : M →SL[σ₁₂] M₂ x : M ⊢ ↑f (-x) = -↑f x ** exact map_neg f x ** Qed
ContinuousLinearMap.map_sub ** R : Type u_1 inst✝¹³ : Ring R R₂ : Type u_2 inst✝¹² : Ring R₂ R₃ : Type u_3 inst✝¹¹ : Ring R₃ M : Type u_4 inst✝¹⁰ : TopologicalSpace M inst✝⁹ : AddCommGroup M M₂ : Type u_5 inst✝⁸ : TopologicalSpace M₂ inst✝⁷ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁶ : TopologicalSpace M₃ inst✝⁵ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁴ : TopologicalSpace M₄ inst✝³ : AddCommGroup M₄ inst✝² : Module R M inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ f : M →SL[σ₁₂] M₂ x y : M ⊢ ↑f (x - y) = ↑f x - ↑f y ** exact map_sub f x y ** Qed
ContinuousLinearMap.comp_neg ** R : Type u_1 inst✝¹⁶ : Ring R R₂ : Type u_2 inst✝¹⁵ : Ring R₂ R₃ : Type u_3 inst✝¹⁴ : Ring R₃ M : Type u_4 inst✝¹³ : TopologicalSpace M inst✝¹² : AddCommGroup M M₂ : Type u_5 inst✝¹¹ : TopologicalSpace M₂ inst✝¹⁰ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁹ : TopologicalSpace M₃ inst✝⁸ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁷ : TopologicalSpace M₄ inst✝⁶ : AddCommGroup M₄ inst✝⁵ : Module R M inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹ : TopologicalAddGroup M₂ inst✝ : TopologicalAddGroup M₃ g : M₂ →SL[σ₂₃] M₃ f : M →SL[σ₁₂] M₂ ⊢ comp g (-f) = -comp g f ** ext x ** case h R : Type u_1 inst✝¹⁶ : Ring R R₂ : Type u_2 inst✝¹⁵ : Ring R₂ R₃ : Type u_3 inst✝¹⁴ : Ring R₃ M : Type u_4 inst✝¹³ : TopologicalSpace M inst✝¹² : AddCommGroup M M₂ : Type u_5 inst✝¹¹ : TopologicalSpace M₂ inst✝¹⁰ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁹ : TopologicalSpace M₃ inst✝⁸ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁷ : TopologicalSpace M₄ inst✝⁶ : AddCommGroup M₄ inst✝⁵ : Module R M inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹ : TopologicalAddGroup M₂ inst✝ : TopologicalAddGroup M₃ g : M₂ →SL[σ₂₃] M₃ f : M →SL[σ₁₂] M₂ x : M ⊢ ↑(comp g (-f)) x = ↑(-comp g f) x ** simp ** Qed
ContinuousLinearMap.neg_comp ** R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝ : TopologicalAddGroup M₃ g : M₂ →SL[σ₂₃] M₃ f : M →SL[σ₁₂] M₂ ⊢ comp (-g) f = -comp g f ** ext ** case h R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝ : TopologicalAddGroup M₃ g : M₂ →SL[σ₂₃] M₃ f : M →SL[σ₁₂] M₂ x✝ : M ⊢ ↑(comp (-g) f) x✝ = ↑(-comp g f) x✝ ** simp ** Qed
ContinuousLinearMap.comp_sub ** R : Type u_1 inst✝¹⁶ : Ring R R₂ : Type u_2 inst✝¹⁵ : Ring R₂ R₃ : Type u_3 inst✝¹⁴ : Ring R₃ M : Type u_4 inst✝¹³ : TopologicalSpace M inst✝¹² : AddCommGroup M M₂ : Type u_5 inst✝¹¹ : TopologicalSpace M₂ inst✝¹⁰ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁹ : TopologicalSpace M₃ inst✝⁸ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁷ : TopologicalSpace M₄ inst✝⁶ : AddCommGroup M₄ inst✝⁵ : Module R M inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹ : TopologicalAddGroup M₂ inst✝ : TopologicalAddGroup M₃ g : M₂ →SL[σ₂₃] M₃ f₁ f₂ : M →SL[σ₁₂] M₂ ⊢ comp g (f₁ - f₂) = comp g f₁ - comp g f₂ ** ext ** case h R : Type u_1 inst✝¹⁶ : Ring R R₂ : Type u_2 inst✝¹⁵ : Ring R₂ R₃ : Type u_3 inst✝¹⁴ : Ring R₃ M : Type u_4 inst✝¹³ : TopologicalSpace M inst✝¹² : AddCommGroup M M₂ : Type u_5 inst✝¹¹ : TopologicalSpace M₂ inst✝¹⁰ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁹ : TopologicalSpace M₃ inst✝⁸ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁷ : TopologicalSpace M₄ inst✝⁶ : AddCommGroup M₄ inst✝⁵ : Module R M inst✝⁴ : Module R₂ M₂ inst✝³ : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝² : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹ : TopologicalAddGroup M₂ inst✝ : TopologicalAddGroup M₃ g : M₂ →SL[σ₂₃] M₃ f₁ f₂ : M →SL[σ₁₂] M₂ x✝ : M ⊢ ↑(comp g (f₁ - f₂)) x✝ = ↑(comp g f₁ - comp g f₂) x✝ ** simp ** Qed
ContinuousLinearMap.sub_comp ** R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝ : TopologicalAddGroup M₃ g₁ g₂ : M₂ →SL[σ₂₃] M₃ f : M →SL[σ₁₂] M₂ ⊢ comp (g₁ - g₂) f = comp g₁ f - comp g₂ f ** ext ** case h R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝ : TopologicalAddGroup M₃ g₁ g₂ : M₂ →SL[σ₂₃] M₃ f : M →SL[σ₁₂] M₂ x✝ : M ⊢ ↑(comp (g₁ - g₂) f) x✝ = ↑(comp g₁ f - comp g₂ f) x✝ ** simp ** Qed
ContinuousLinearMap.smulRight_one_pow ** R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : TopologicalSpace R inst✝ : TopologicalRing R c : R n : ℕ ⊢ smulRight 1 c ^ n = smulRight 1 (c ^ n) ** induction' n with n ihn ** case zero R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : TopologicalSpace R inst✝ : TopologicalRing R c : R ⊢ smulRight 1 c ^ Nat.zero = smulRight 1 (c ^ Nat.zero) ** ext ** case zero.h R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : TopologicalSpace R inst✝ : TopologicalRing R c : R ⊢ ↑(smulRight 1 c ^ Nat.zero) 1 = ↑(smulRight 1 (c ^ Nat.zero)) 1 ** simp ** case succ R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹ : TopologicalSpace R inst✝ : TopologicalRing R c : R n : ℕ ihn : smulRight 1 c ^ n = smulRight 1 (c ^ n) ⊢ smulRight 1 c ^ Nat.succ n = smulRight 1 (c ^ Nat.succ n) ** rw [pow_succ, ihn, mul_def, smulRight_comp, smul_eq_mul, pow_succ'] ** Qed
ContinuousLinearMap.projKerOfRightInverse_apply_idem ** R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ σ₂₁ : R₂ →+* R inst✝¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝ : TopologicalAddGroup M f₁ : M →SL[σ₁₂] M₂ f₂ : M₂ →SL[σ₂₁] M h : Function.RightInverse ↑f₂ ↑f₁ x : { x // x ∈ LinearMap.ker f₁ } ⊢ ↑(projKerOfRightInverse f₁ f₂ h) ↑x = x ** ext1 ** case a R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ σ₂₁ : R₂ →+* R inst✝¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝ : TopologicalAddGroup M f₁ : M →SL[σ₁₂] M₂ f₂ : M₂ →SL[σ₂₁] M h : Function.RightInverse ↑f₂ ↑f₁ x : { x // x ∈ LinearMap.ker f₁ } ⊢ ↑(↑(projKerOfRightInverse f₁ f₂ h) ↑x) = ↑x ** simp ** Qed
ContinuousLinearMap.projKerOfRightInverse_comp_inv ** R : Type u_1 inst✝¹⁵ : Ring R R₂ : Type u_2 inst✝¹⁴ : Ring R₂ R₃ : Type u_3 inst✝¹³ : Ring R₃ M : Type u_4 inst✝¹² : TopologicalSpace M inst✝¹¹ : AddCommGroup M M₂ : Type u_5 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommGroup M₂ M₃ : Type u_6 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommGroup M₃ M₄ : Type u_7 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommGroup M₄ inst✝⁴ : Module R M inst✝³ : Module R₂ M₂ inst✝² : Module R₃ M₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ σ₂₁ : R₂ →+* R inst✝¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝ : TopologicalAddGroup M f₁ : M →SL[σ₁₂] M₂ f₂ : M₂ →SL[σ₂₁] M h : Function.RightInverse ↑f₂ ↑f₁ y : M₂ ⊢ ↑(↑(projKerOfRightInverse f₁ f₂ h) (↑f₂ y)) = ↑0 ** simp [h y] ** Qed
ContinuousLinearMap.isOpenMap_of_ne_zero ** R : Type u_1 M : Type u_2 inst✝⁷ : TopologicalSpace R inst✝⁶ : DivisionRing R inst✝⁵ : ContinuousSub R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalSpace M inst✝² : ContinuousAdd M inst✝¹ : Module R M inst✝ : ContinuousSMul R M f : M →L[R] R hf : f ≠ 0 x : M hx : ↑f x ≠ 0 y : M ⊢ Continuous fun a => y + (a - ↑f y) • (↑f x)⁻¹ • x ** continuity ** R : Type u_1 M : Type u_2 inst✝⁷ : TopologicalSpace R inst✝⁶ : DivisionRing R inst✝⁵ : ContinuousSub R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalSpace M inst✝² : ContinuousAdd M inst✝¹ : Module R M inst✝ : ContinuousSMul R M f : M →L[R] R hf : f ≠ 0 x : M hx : ↑f x ≠ 0 y : M ⊢ (fun a => y + (a - ↑f y) • (↑f x)⁻¹ • x) (↑f y) = y ** simp ** R : Type u_1 M : Type u_2 inst✝⁷ : TopologicalSpace R inst✝⁶ : DivisionRing R inst✝⁵ : ContinuousSub R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalSpace M inst✝² : ContinuousAdd M inst✝¹ : Module R M inst✝ : ContinuousSMul R M f : M →L[R] R hf : f ≠ 0 x : M hx : ↑f x ≠ 0 y : M a : R ⊢ ↑f ((fun a => y + (a - ↑f y) • (↑f x)⁻¹ • x) a) = a ** simp [hx] ** Qed
ContinuousLinearMap.comp_smul ** R : Type u_1 R₂ : Type u_2 R₃ : Type u_3 S : Type u_4 S₃ : Type u_5 inst✝³³ : Semiring R inst✝³² : Semiring R₂ inst✝³¹ : Semiring R₃ inst✝³⁰ : Monoid S inst✝²⁹ : Monoid S₃ M : Type u_6 inst✝²⁸ : TopologicalSpace M inst✝²⁷ : AddCommMonoid M inst✝²⁶ : Module R M M₂ : Type u_7 inst✝²⁵ : TopologicalSpace M₂ inst✝²⁴ : AddCommMonoid M₂ inst✝²³ : Module R₂ M₂ M₃ : Type u_8 inst✝²² : TopologicalSpace M₃ inst✝²¹ : AddCommMonoid M₃ inst✝²⁰ : Module R₃ M₃ N₂ : Type u_9 inst✝¹⁹ : TopologicalSpace N₂ inst✝¹⁸ : AddCommMonoid N₂ inst✝¹⁷ : Module R N₂ N₃ : Type u_10 inst✝¹⁶ : TopologicalSpace N₃ inst✝¹⁵ : AddCommMonoid N₃ inst✝¹⁴ : Module R N₃ inst✝¹³ : DistribMulAction S₃ M₃ inst✝¹² : SMulCommClass R₃ S₃ M₃ inst✝¹¹ : ContinuousConstSMul S₃ M₃ inst✝¹⁰ : DistribMulAction S N₃ inst✝⁹ : SMulCommClass R S N₃ inst✝⁸ : ContinuousConstSMul S N₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝⁷ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝⁶ : DistribMulAction S₃ M₂ inst✝⁵ : ContinuousConstSMul S₃ M₂ inst✝⁴ : SMulCommClass R₂ S₃ M₂ inst✝³ : DistribMulAction S N₂ inst✝² : ContinuousConstSMul S N₂ inst✝¹ : SMulCommClass R S N₂ inst✝ : LinearMap.CompatibleSMul N₂ N₃ S R hₗ : N₂ →L[R] N₃ c : S fₗ : M →L[R] N₂ ⊢ comp hₗ (c • fₗ) = c • comp hₗ fₗ ** ext x ** case h R : Type u_1 R₂ : Type u_2 R₃ : Type u_3 S : Type u_4 S₃ : Type u_5 inst✝³³ : Semiring R inst✝³² : Semiring R₂ inst✝³¹ : Semiring R₃ inst✝³⁰ : Monoid S inst✝²⁹ : Monoid S₃ M : Type u_6 inst✝²⁸ : TopologicalSpace M inst✝²⁷ : AddCommMonoid M inst✝²⁶ : Module R M M₂ : Type u_7 inst✝²⁵ : TopologicalSpace M₂ inst✝²⁴ : AddCommMonoid M₂ inst✝²³ : Module R₂ M₂ M₃ : Type u_8 inst✝²² : TopologicalSpace M₃ inst✝²¹ : AddCommMonoid M₃ inst✝²⁰ : Module R₃ M₃ N₂ : Type u_9 inst✝¹⁹ : TopologicalSpace N₂ inst✝¹⁸ : AddCommMonoid N₂ inst✝¹⁷ : Module R N₂ N₃ : Type u_10 inst✝¹⁶ : TopologicalSpace N₃ inst✝¹⁵ : AddCommMonoid N₃ inst✝¹⁴ : Module R N₃ inst✝¹³ : DistribMulAction S₃ M₃ inst✝¹² : SMulCommClass R₃ S₃ M₃ inst✝¹¹ : ContinuousConstSMul S₃ M₃ inst✝¹⁰ : DistribMulAction S N₃ inst✝⁹ : SMulCommClass R S N₃ inst✝⁸ : ContinuousConstSMul S N₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝⁷ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝⁶ : DistribMulAction S₃ M₂ inst✝⁵ : ContinuousConstSMul S₃ M₂ inst✝⁴ : SMulCommClass R₂ S₃ M₂ inst✝³ : DistribMulAction S N₂ inst✝² : ContinuousConstSMul S N₂ inst✝¹ : SMulCommClass R S N₂ inst✝ : LinearMap.CompatibleSMul N₂ N₃ S R hₗ : N₂ →L[R] N₃ c : S fₗ : M →L[R] N₂ x : M ⊢ ↑(comp hₗ (c • fₗ)) x = ↑(c • comp hₗ fₗ) x ** exact hₗ.map_smul_of_tower c (fₗ x) ** Qed
ContinuousLinearMap.comp_smulₛₗ ** R : Type u_1 R₂ : Type u_2 R₃ : Type u_3 S : Type u_4 S₃ : Type u_5 inst✝³⁶ : Semiring R inst✝³⁵ : Semiring R₂ inst✝³⁴ : Semiring R₃ inst✝³³ : Monoid S inst✝³² : Monoid S₃ M : Type u_6 inst✝³¹ : TopologicalSpace M inst✝³⁰ : AddCommMonoid M inst✝²⁹ : Module R M M₂ : Type u_7 inst✝²⁸ : TopologicalSpace M₂ inst✝²⁷ : AddCommMonoid M₂ inst✝²⁶ : Module R₂ M₂ M₃ : Type u_8 inst✝²⁵ : TopologicalSpace M₃ inst✝²⁴ : AddCommMonoid M₃ inst✝²³ : Module R₃ M₃ N₂ : Type u_9 inst✝²² : TopologicalSpace N₂ inst✝²¹ : AddCommMonoid N₂ inst✝²⁰ : Module R N₂ N₃ : Type u_10 inst✝¹⁹ : TopologicalSpace N₃ inst✝¹⁸ : AddCommMonoid N₃ inst✝¹⁷ : Module R N₃ inst✝¹⁶ : DistribMulAction S₃ M₃ inst✝¹⁵ : SMulCommClass R₃ S₃ M₃ inst✝¹⁴ : ContinuousConstSMul S₃ M₃ inst✝¹³ : DistribMulAction S N₃ inst✝¹² : SMulCommClass R S N₃ inst✝¹¹ : ContinuousConstSMul S N₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹⁰ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝⁹ : DistribMulAction S₃ M₂ inst✝⁸ : ContinuousConstSMul S₃ M₂ inst✝⁷ : SMulCommClass R₂ S₃ M₂ inst✝⁶ : DistribMulAction S N₂ inst✝⁵ : ContinuousConstSMul S N₂ inst✝⁴ : SMulCommClass R S N₂ inst✝³ : SMulCommClass R₂ R₂ M₂ inst✝² : SMulCommClass R₃ R₃ M₃ inst✝¹ : ContinuousConstSMul R₂ M₂ inst✝ : ContinuousConstSMul R₃ M₃ h : M₂ →SL[σ₂₃] M₃ c : R₂ f : M →SL[σ₁₂] M₂ ⊢ comp h (c • f) = ↑σ₂₃ c • comp h f ** ext x ** case h R : Type u_1 R₂ : Type u_2 R₃ : Type u_3 S : Type u_4 S₃ : Type u_5 inst✝³⁶ : Semiring R inst✝³⁵ : Semiring R₂ inst✝³⁴ : Semiring R₃ inst✝³³ : Monoid S inst✝³² : Monoid S₃ M : Type u_6 inst✝³¹ : TopologicalSpace M inst✝³⁰ : AddCommMonoid M inst✝²⁹ : Module R M M₂ : Type u_7 inst✝²⁸ : TopologicalSpace M₂ inst✝²⁷ : AddCommMonoid M₂ inst✝²⁶ : Module R₂ M₂ M₃ : Type u_8 inst✝²⁵ : TopologicalSpace M₃ inst✝²⁴ : AddCommMonoid M₃ inst✝²³ : Module R₃ M₃ N₂ : Type u_9 inst✝²² : TopologicalSpace N₂ inst✝²¹ : AddCommMonoid N₂ inst✝²⁰ : Module R N₂ N₃ : Type u_10 inst✝¹⁹ : TopologicalSpace N₃ inst✝¹⁸ : AddCommMonoid N₃ inst✝¹⁷ : Module R N₃ inst✝¹⁶ : DistribMulAction S₃ M₃ inst✝¹⁵ : SMulCommClass R₃ S₃ M₃ inst✝¹⁴ : ContinuousConstSMul S₃ M₃ inst✝¹³ : DistribMulAction S N₃ inst✝¹² : SMulCommClass R S N₃ inst✝¹¹ : ContinuousConstSMul S N₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝¹⁰ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝⁹ : DistribMulAction S₃ M₂ inst✝⁸ : ContinuousConstSMul S₃ M₂ inst✝⁷ : SMulCommClass R₂ S₃ M₂ inst✝⁶ : DistribMulAction S N₂ inst✝⁵ : ContinuousConstSMul S N₂ inst✝⁴ : SMulCommClass R S N₂ inst✝³ : SMulCommClass R₂ R₂ M₂ inst✝² : SMulCommClass R₃ R₃ M₃ inst✝¹ : ContinuousConstSMul R₂ M₂ inst✝ : ContinuousConstSMul R₃ M₃ h : M₂ →SL[σ₂₃] M₃ c : R₂ f : M →SL[σ₁₂] M₂ x : M ⊢ ↑(comp h (c • f)) x = ↑(↑σ₂₃ c • comp h f) x ** simp only [coe_smul', coe_comp', Function.comp_apply, Pi.smul_apply, ContinuousLinearMap.map_smulₛₗ] ** Qed
ContinuousLinearMap.prod_ext_iff ** R : Type u_1 R₂ : Type u_2 R₃ : Type u_3 S : Type u_4 S₃ : Type u_5 inst✝²⁹ : Semiring R inst✝²⁸ : Semiring R₂ inst✝²⁷ : Semiring R₃ inst✝²⁶ : Semiring S inst✝²⁵ : Semiring S₃ M : Type u_6 inst✝²⁴ : TopologicalSpace M inst✝²³ : AddCommMonoid M inst✝²² : Module R M M₂ : Type u_7 inst✝²¹ : TopologicalSpace M₂ inst✝²⁰ : AddCommMonoid M₂ inst✝¹⁹ : Module R₂ M₂ M₃ : Type u_8 inst✝¹⁸ : TopologicalSpace M₃ inst✝¹⁷ : AddCommMonoid M₃ inst✝¹⁶ : Module R₃ M₃ N₂ : Type u_9 inst✝¹⁵ : TopologicalSpace N₂ inst✝¹⁴ : AddCommMonoid N₂ inst✝¹³ : Module R N₂ N₃ : Type u_10 inst✝¹² : TopologicalSpace N₃ inst✝¹¹ : AddCommMonoid N₃ inst✝¹⁰ : Module R N₃ inst✝⁹ : Module S₃ M₃ inst✝⁸ : SMulCommClass R₃ S₃ M₃ inst✝⁷ : ContinuousConstSMul S₃ M₃ inst✝⁶ : Module S N₂ inst✝⁵ : ContinuousConstSMul S N₂ inst✝⁴ : SMulCommClass R S N₂ inst✝³ : Module S N₃ inst✝² : SMulCommClass R S N₃ inst✝¹ : ContinuousConstSMul S N₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ c : S h : M₂ →SL[σ₂₃] M₃ f✝ g✝ : M →SL[σ₁₂] M₂ x y z : M f g : M × N₂ →L[R] N₃ ⊢ f = g ↔ comp f (inl R M N₂) = comp g (inl R M N₂) ∧ comp f (inr R M N₂) = comp g (inr R M N₂) ** simp only [← coe_inj, LinearMap.prod_ext_iff] ** R : Type u_1 R₂ : Type u_2 R₃ : Type u_3 S : Type u_4 S₃ : Type u_5 inst✝²⁹ : Semiring R inst✝²⁸ : Semiring R₂ inst✝²⁷ : Semiring R₃ inst✝²⁶ : Semiring S inst✝²⁵ : Semiring S₃ M : Type u_6 inst✝²⁴ : TopologicalSpace M inst✝²³ : AddCommMonoid M inst✝²² : Module R M M₂ : Type u_7 inst✝²¹ : TopologicalSpace M₂ inst✝²⁰ : AddCommMonoid M₂ inst✝¹⁹ : Module R₂ M₂ M₃ : Type u_8 inst✝¹⁸ : TopologicalSpace M₃ inst✝¹⁷ : AddCommMonoid M₃ inst✝¹⁶ : Module R₃ M₃ N₂ : Type u_9 inst✝¹⁵ : TopologicalSpace N₂ inst✝¹⁴ : AddCommMonoid N₂ inst✝¹³ : Module R N₂ N₃ : Type u_10 inst✝¹² : TopologicalSpace N₃ inst✝¹¹ : AddCommMonoid N₃ inst✝¹⁰ : Module R N₃ inst✝⁹ : Module S₃ M₃ inst✝⁸ : SMulCommClass R₃ S₃ M₃ inst✝⁷ : ContinuousConstSMul S₃ M₃ inst✝⁶ : Module S N₂ inst✝⁵ : ContinuousConstSMul S N₂ inst✝⁴ : SMulCommClass R S N₂ inst✝³ : Module S N₃ inst✝² : SMulCommClass R S N₃ inst✝¹ : ContinuousConstSMul S N₃ σ₁₂ : R →+* R₂ σ₂₃ : R₂ →+* R₃ σ₁₃ : R →+* R₃ inst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ c : S h : M₂ →SL[σ₂₃] M₃ f✝ g✝ : M →SL[σ₁₂] M₂ x y z : M f g : M × N₂ →L[R] N₃ ⊢ LinearMap.comp (↑f) (LinearMap.inl R M N₂) = LinearMap.comp (↑g) (LinearMap.inl R M N₂) ∧ LinearMap.comp (↑f) (LinearMap.inr R M N₂) = LinearMap.comp (↑g) (LinearMap.inr R M N₂) ↔ ↑(comp f (inl R M N₂)) = ↑(comp g (inl R M N₂)) ∧ ↑(comp f (inr R M N₂)) = ↑(comp g (inr R M N₂)) ** rfl ** Qed
ContinuousLinearEquiv.toLinearEquiv_injective ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ ⊢ Function.Injective toLinearEquiv ** rintro ⟨e, _, _⟩ ⟨e', _, _⟩ rfl ** case mk.mk R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃ₛₗ[σ₁₂] M₂ continuous_toFun✝¹ : Continuous e.toFun continuous_invFun✝¹ : Continuous e.invFun continuous_toFun✝ : Continuous (↑(mk e).toLinearEquiv).toAddHom.toFun continuous_invFun✝ : Continuous (mk e).toLinearEquiv.invFun ⊢ mk e = mk (mk e).toLinearEquiv ** rfl ** Qed
ContinuousLinearEquiv.ext₁ ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁵ : Semiring R₁ inst✝²⁴ : Semiring R₂ inst✝²³ : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²² : RingHomInvPair σ₁₂ σ₂₁ inst✝²¹ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝²⁰ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁹ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁸ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁷ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁶ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹⁴ : TopologicalSpace M₁ inst✝¹³ : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹² : TopologicalSpace M'₁ inst✝¹¹ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝¹⁰ : TopologicalSpace M₂ inst✝⁹ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁸ : TopologicalSpace M₃ inst✝⁷ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁶ : TopologicalSpace M₄ inst✝⁵ : AddCommMonoid M₄ inst✝⁴ : Module R₁ M₁ inst✝³ : Module R₁ M'₁ inst✝² : Module R₂ M₂ inst✝¹ : Module R₃ M₃ inst✝ : TopologicalSpace R₁ f g : R₁ ≃L[R₁] M₁ h : ↑f 1 = ↑g 1 x : R₁ ⊢ ↑f (x * 1) = ↑g (x * 1) ** rw [← smul_eq_mul, map_smul, h, map_smul] ** Qed
ContinuousLinearEquiv.symm_toLinearEquiv ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ ⊢ (ContinuousLinearEquiv.symm e).toLinearEquiv = LinearEquiv.symm e.toLinearEquiv ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ x✝ : M₂ ⊢ ↑(ContinuousLinearEquiv.symm e).toLinearEquiv x✝ = ↑(LinearEquiv.symm e.toLinearEquiv) x✝ ** rfl ** Qed
ContinuousLinearEquiv.trans_toLinearEquiv ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e₁ : M₁ ≃SL[σ₁₂] M₂ e₂ : M₂ ≃SL[σ₂₃] M₃ ⊢ (ContinuousLinearEquiv.trans e₁ e₂).toLinearEquiv = LinearEquiv.trans e₁.toLinearEquiv e₂.toLinearEquiv ** ext ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e₁ : M₁ ≃SL[σ₁₂] M₂ e₂ : M₂ ≃SL[σ₂₃] M₃ x✝ : M₁ ⊢ ↑(ContinuousLinearEquiv.trans e₁ e₂).toLinearEquiv x✝ = ↑(LinearEquiv.trans e₁.toLinearEquiv e₂.toLinearEquiv) x✝ ** rfl ** Qed
ContinuousLinearEquiv.symm_comp_self ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ ⊢ ↑(ContinuousLinearEquiv.symm e) ∘ ↑e = id ** ext x ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ x : M₁ ⊢ (↑(ContinuousLinearEquiv.symm e) ∘ ↑e) x = id x ** exact symm_apply_apply e x ** Qed
ContinuousLinearEquiv.self_comp_symm ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ ⊢ ↑e ∘ ↑(ContinuousLinearEquiv.symm e) = id ** ext x ** case h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ x : M₂ ⊢ (↑e ∘ ↑(ContinuousLinearEquiv.symm e)) x = id x ** exact apply_symm_apply e x ** Qed
ContinuousLinearEquiv.symm_symm ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ ⊢ ContinuousLinearEquiv.symm (ContinuousLinearEquiv.symm e) = e ** ext x ** case h.h R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ x : M₁ ⊢ ↑(ContinuousLinearEquiv.symm (ContinuousLinearEquiv.symm e)) x = ↑e x ** rfl ** Qed
ContinuousLinearEquiv.image_symm_eq_preimage ** R₁ : Type u_1 R₂ : Type u_2 R₃ : Type u_3 inst✝²⁴ : Semiring R₁ inst✝²³ : Semiring R₂ inst✝²² : Semiring R₃ σ₁₂ : R₁ →+* R₂ σ₂₁ : R₂ →+* R₁ inst✝²¹ : RingHomInvPair σ₁₂ σ₂₁ inst✝²⁰ : RingHomInvPair σ₂₁ σ₁₂ σ₂₃ : R₂ →+* R₃ σ₃₂ : R₃ →+* R₂ inst✝¹⁹ : RingHomInvPair σ₂₃ σ₃₂ inst✝¹⁸ : RingHomInvPair σ₃₂ σ₂₃ σ₁₃ : R₁ →+* R₃ σ₃₁ : R₃ →+* R₁ inst✝¹⁷ : RingHomInvPair σ₁₃ σ₃₁ inst✝¹⁶ : RingHomInvPair σ₃₁ σ₁₃ inst✝¹⁵ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃ inst✝¹⁴ : RingHomCompTriple σ₃₂ σ₂₁ σ₃₁ M₁ : Type u_4 inst✝¹³ : TopologicalSpace M₁ inst✝¹² : AddCommMonoid M₁ M'₁ : Type u_5 inst✝¹¹ : TopologicalSpace M'₁ inst✝¹⁰ : AddCommMonoid M'₁ M₂ : Type u_6 inst✝⁹ : TopologicalSpace M₂ inst✝⁸ : AddCommMonoid M₂ M₃ : Type u_7 inst✝⁷ : TopologicalSpace M₃ inst✝⁶ : AddCommMonoid M₃ M₄ : Type u_8 inst✝⁵ : TopologicalSpace M₄ inst✝⁴ : AddCommMonoid M₄ inst✝³ : Module R₁ M₁ inst✝² : Module R₁ M'₁ inst✝¹ : Module R₂ M₂ inst✝ : Module R₃ M₃ e : M₁ ≃SL[σ₁₂] M₂ s : Set M₂ ⊢ ↑(ContinuousLinearEquiv.symm e) '' s = ↑e ⁻¹' s ** rw [e.symm.image_eq_preimage, e.symm_symm] ** Qed
ContinuousLinearMap.inverse_equiv ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁶ : TopologicalSpace M inst✝⁵ : TopologicalSpace M₂ inst✝⁴ : Semiring R inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₂ inst✝¹ : AddCommMonoid M inst✝ : Module R M e : M ≃L[R] M₂ ⊢ inverse ↑e = ↑(ContinuousLinearEquiv.symm e) ** have h : ∃ e' : M ≃L[R] M₂, (e' : M →L[R] M₂) = ↑e := ⟨e, rfl⟩ ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁶ : TopologicalSpace M inst✝⁵ : TopologicalSpace M₂ inst✝⁴ : Semiring R inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₂ inst✝¹ : AddCommMonoid M inst✝ : Module R M e : M ≃L[R] M₂ h : ∃ e', ↑e' = ↑e ⊢ inverse ↑e = ↑(ContinuousLinearEquiv.symm e) ** simp only [inverse, dif_pos h] ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁶ : TopologicalSpace M inst✝⁵ : TopologicalSpace M₂ inst✝⁴ : Semiring R inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₂ inst✝¹ : AddCommMonoid M inst✝ : Module R M e : M ≃L[R] M₂ h : ∃ e', ↑e' = ↑e ⊢ ↑(ContinuousLinearEquiv.symm (choose h)) = ↑(ContinuousLinearEquiv.symm e) ** congr ** case e_e.e_e R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁶ : TopologicalSpace M inst✝⁵ : TopologicalSpace M₂ inst✝⁴ : Semiring R inst✝³ : AddCommMonoid M₂ inst✝² : Module R M₂ inst✝¹ : AddCommMonoid M inst✝ : Module R M e : M ≃L[R] M₂ h : ∃ e', ↑e' = ↑e ⊢ choose h = e ** exact_mod_cast Classical.choose_spec h ** Qed
ContinuousLinearMap.ring_inverse_equiv ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M ⊢ Ring.inverse ↑e = inverse ↑e ** suffices Ring.inverse ((ContinuousLinearEquiv.unitsEquiv _ _).symm e : M →L[R] M) = inverse ↑e by convert this ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M ⊢ Ring.inverse ↑(↑(MulEquiv.symm (ContinuousLinearEquiv.unitsEquiv R M)) e) = inverse ↑e ** simp ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M ⊢ ↑(↑(MulEquiv.symm (ContinuousLinearEquiv.unitsEquiv R M)) e)⁻¹ = ↑(ContinuousLinearEquiv.symm e) ** rfl ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M this : Ring.inverse ↑(↑(MulEquiv.symm (ContinuousLinearEquiv.unitsEquiv R M)) e) = inverse ↑e ⊢ Ring.inverse ↑e = inverse ↑e ** convert this ** Qed
ContinuousLinearMap.to_ring_inverse ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ ⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e) ** by_cases h₁ : ∃ e' : M ≃L[R] M₂, e' = f ** case pos R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ h₁ : ∃ e', ↑e' = f ⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e) ** obtain ⟨e', he'⟩ := h₁ ** case pos.intro R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ e' : M ≃L[R] M₂ he' : ↑e' = f ⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e) ** rw [← he'] ** case pos.intro R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ e' : M ≃L[R] M₂ he' : ↑e' = f ⊢ inverse ↑e' = comp (Ring.inverse (comp ↑(ContinuousLinearEquiv.symm e) ↑e')) ↑(ContinuousLinearEquiv.symm e) ** change _ = Ring.inverse (e'.trans e.symm : M →L[R] M) ∘L (e.symm : M₂ →L[R] M) ** case pos.intro R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ e' : M ≃L[R] M₂ he' : ↑e' = f ⊢ inverse ↑e' = comp (Ring.inverse ↑(ContinuousLinearEquiv.trans e' (ContinuousLinearEquiv.symm e))) ↑(ContinuousLinearEquiv.symm e) ** ext ** case pos.intro.h R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ e' : M ≃L[R] M₂ he' : ↑e' = f x✝ : M₂ ⊢ ↑(inverse ↑e') x✝ = ↑(comp (Ring.inverse ↑(ContinuousLinearEquiv.trans e' (ContinuousLinearEquiv.symm e))) ↑(ContinuousLinearEquiv.symm e)) x✝ ** simp ** case neg R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ h₁ : ¬∃ e', ↑e' = f ⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e) ** suffices ¬IsUnit ((e.symm : M₂ →L[R] M).comp f) by simp [this, h₁] ** case neg R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ h₁ : ¬∃ e', ↑e' = f ⊢ ¬IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f) ** contrapose! h₁ ** case neg R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ h₁ : IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f) ⊢ ∃ e', ↑e' = f ** rcases h₁ with ⟨F, hF⟩ ** case neg.intro R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ F : (M →L[R] M)ˣ hF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f ⊢ ∃ e', ↑e' = f ** use (ContinuousLinearEquiv.unitsEquiv _ _ F).trans e ** case h R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ F : (M →L[R] M)ˣ hF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f ⊢ ↑(ContinuousLinearEquiv.trans (↑(ContinuousLinearEquiv.unitsEquiv R M) F) e) = f ** ext ** case h.h R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ F : (M →L[R] M)ˣ hF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f x✝ : M ⊢ ↑↑(ContinuousLinearEquiv.trans (↑(ContinuousLinearEquiv.unitsEquiv R M) F) e) x✝ = ↑f x✝ ** dsimp ** case h.h R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ F : (M →L[R] M)ˣ hF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f x✝ : M ⊢ ↑e (↑↑F x✝) = ↑f x✝ ** rw [hF] ** case h.h R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ F : (M →L[R] M)ˣ hF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f x✝ : M ⊢ ↑e (↑(comp (↑(ContinuousLinearEquiv.symm e)) f) x✝) = ↑f x✝ ** simp ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ e : M ≃L[R] M₂ f : M →L[R] M₂ h₁ : ¬∃ e', ↑e' = f this : ¬IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f) ⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e) ** simp [this, h₁] ** Qed
ContinuousLinearMap.ring_inverse_eq_map_inverse ** R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ ⊢ Ring.inverse = inverse ** ext ** case h.h R : Type u_1 M : Type u_2 M₂ : Type u_3 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace M₂ inst✝⁵ : Ring R inst✝⁴ : AddCommGroup M inst✝³ : TopologicalAddGroup M inst✝² : Module R M inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ x✝¹ : M →L[R] M x✝ : M ⊢ ↑(Ring.inverse x✝¹) x✝ = ↑(inverse x✝¹) x✝ ** simp [to_ring_inverse (ContinuousLinearEquiv.refl R M)] ** Qed
Submodule.ClosedComplemented.isClosed ** R : Type u_1 inst✝⁸ : Ring R M : Type u_2 inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : Module R M M₂ : Type u_3 inst✝⁴ : TopologicalSpace M₂ inst✝³ : AddCommGroup M₂ inst✝² : Module R M₂ inst✝¹ : TopologicalAddGroup M inst✝ : T1Space M p : Submodule R M h : ClosedComplemented p ⊢ IsClosed ↑p ** rcases h with ⟨f, hf⟩ ** case intro R : Type u_1 inst✝⁸ : Ring R M : Type u_2 inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : Module R M M₂ : Type u_3 inst✝⁴ : TopologicalSpace M₂ inst✝³ : AddCommGroup M₂ inst✝² : Module R M₂ inst✝¹ : TopologicalAddGroup M inst✝ : T1Space M p : Submodule R M f : M →L[R] { x // x ∈ p } hf : ∀ (x : { x // x ∈ p }), ↑f ↑x = x ⊢ IsClosed ↑p ** have : ker (id R M - p.subtypeL.comp f) = p := LinearMap.ker_id_sub_eq_of_proj hf ** case intro R : Type u_1 inst✝⁸ : Ring R M : Type u_2 inst✝⁷ : TopologicalSpace M inst✝⁶ : AddCommGroup M inst✝⁵ : Module R M M₂ : Type u_3 inst✝⁴ : TopologicalSpace M₂ inst✝³ : AddCommGroup M₂ inst✝² : Module R M₂ inst✝¹ : TopologicalAddGroup M inst✝ : T1Space M p : Submodule R M f : M →L[R] { x // x ∈ p } hf : ∀ (x : { x // x ∈ p }), ↑f ↑x = x this : LinearMap.ker (ContinuousLinearMap.id R M - comp (subtypeL p) f) = p ⊢ IsClosed ↑p ** exact this ▸ isClosed_ker _ ** Qed
Submodule.closedComplemented_bot ** R : Type u_1 inst✝⁶ : Ring R M : Type u_2 inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : Module R M M₂ : Type u_3 inst✝² : TopologicalSpace M₂ inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ x : { x // x ∈ ⊥ } ⊢ ↑0 ↑x = x ** simp only [zero_apply, eq_zero_of_bot_submodule x] ** Qed
Submodule.closedComplemented_top ** R : Type u_1 inst✝⁶ : Ring R M : Type u_2 inst✝⁵ : TopologicalSpace M inst✝⁴ : AddCommGroup M inst✝³ : Module R M M₂ : Type u_3 inst✝² : TopologicalSpace M₂ inst✝¹ : AddCommGroup M₂ inst✝ : Module R M₂ x : { x // x ∈ ⊤ } ⊢ ↑(↑(codRestrict (ContinuousLinearMap.id R M) ⊤ (_ : M → True)) ↑x) = ↑x ** simp ** Qed
UniformSpace.Completion.dist_self ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x : Completion α ⊢ dist x x = 0 ** refine' induction_on x _ _ ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α x : Completion α ⊢ IsClosed {a | dist a a = 0} ** refine' isClosed_eq _ continuous_const ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α x : Completion α ⊢ Continuous fun a => dist a a ** exact Completion.continuous_dist continuous_id continuous_id ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x : Completion α ⊢ ∀ (a : α), dist (↑α a) (↑α a) = 0 ** intro a ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x : Completion α a : α ⊢ dist (↑α a) (↑α a) = 0 ** rw [Completion.dist_eq, dist_self] ** Qed
UniformSpace.Completion.dist_comm ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α ⊢ dist x y = dist y x ** refine' induction_on₂ x y _ _ ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α ⊢ IsClosed {x | dist x.1 x.2 = dist x.2 x.1} ** exact isClosed_eq (Completion.continuous_dist continuous_fst continuous_snd) (Completion.continuous_dist continuous_snd continuous_fst) ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α ⊢ ∀ (a b : α), dist (↑α a) (↑α b) = dist (↑α b) (↑α a) ** intro a b ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α a b : α ⊢ dist (↑α a) (↑α b) = dist (↑α b) (↑α a) ** rw [Completion.dist_eq, Completion.dist_eq, dist_comm] ** Qed
UniformSpace.Completion.dist_triangle ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x y z : Completion α ⊢ dist x z ≤ dist x y + dist y z ** refine' induction_on₃ x y z _ _ ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y z : Completion α ⊢ IsClosed {x | dist x.1 x.2.2 ≤ dist x.1 x.2.1 + dist x.2.1 x.2.2} ** refine' isClosed_le _ (Continuous.add _ _) <;> apply_rules [Completion.continuous_dist, Continuous.fst, Continuous.snd, continuous_id] ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y z : Completion α ⊢ ∀ (a b c : α), dist (↑α a) (↑α c) ≤ dist (↑α a) (↑α b) + dist (↑α b) (↑α c) ** intro a b c ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y z : Completion α a b c : α ⊢ dist (↑α a) (↑α c) ≤ dist (↑α a) (↑α b) + dist (↑α b) (↑α c) ** rw [Completion.dist_eq, Completion.dist_eq, Completion.dist_eq] ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α x y z : Completion α a b c : α ⊢ dist a c ≤ dist a b + dist b c ** exact dist_triangle a b c ** Qed
UniformSpace.Completion.mem_uniformity_dist ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ⊢ s ∈ 𝓤 (Completion α) ↔ ∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ** constructor ** case mp α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ⊢ s ∈ 𝓤 (Completion α) → ∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ** intro hs ** case mp α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) ⊢ ∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ** rcases mem_uniformity_isClosed hs with ⟨t, ht, ⟨tclosed, ts⟩⟩ ** case mp.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s ⊢ ∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ** have A : { x : α × α | (↑x.1, ↑x.2) ∈ t } ∈ uniformity α := uniformContinuous_def.1 (uniformContinuous_coe α) t ht ** case mp.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ⊢ ∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ** rcases mem_uniformity_dist.1 A with ⟨ε, εpos, hε⟩ ** case mp.intro.intro.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} ⊢ ∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ** refine' ⟨ε, εpos, @fun x y hxy ↦ _⟩ ** case mp.intro.intro.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε this : ε ≤ dist x y ∨ (x, y) ∈ t ⊢ (x, y) ∈ s ** simp only [not_le.mpr hxy, false_or_iff, not_le] at this ** case mp.intro.intro.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε this : (x, y) ∈ t ⊢ (x, y) ∈ s ** exact ts this ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε ⊢ ε ≤ dist x y ∨ (x, y) ∈ t ** refine' induction_on₂ x y _ _ ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε ⊢ IsClosed {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} ** have : { x : Completion α × Completion α | ε ≤ dist x.fst x.snd ∨ (x.fst, x.snd) ∈ t } = { p : Completion α × Completion α | ε ≤ dist p.1 p.2 } ∪ t := by ext; simp ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε this : {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} = {p | ε ≤ dist p.1 p.2} ∪ t ⊢ IsClosed {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} ** rw [this] ** case refine'_1 α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε this : {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} = {p | ε ≤ dist p.1 p.2} ∪ t ⊢ IsClosed ({p | ε ≤ dist p.1 p.2} ∪ t) ** apply IsClosed.union _ tclosed ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε this : {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} = {p | ε ≤ dist p.1 p.2} ∪ t ⊢ IsClosed {p | ε ≤ dist p.1 p.2} ** exact isClosed_le continuous_const Completion.uniformContinuous_dist.continuous ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε ⊢ {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} = {p | ε ≤ dist p.1 p.2} ∪ t ** ext ** case h α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε x✝ : Completion α × Completion α ⊢ x✝ ∈ {x | ε ≤ dist x.1 x.2 ∨ (x.1, x.2) ∈ t} ↔ x✝ ∈ {p | ε ≤ dist p.1 p.2} ∪ t ** simp ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x y : Completion α hxy : dist x y < ε ⊢ ∀ (a b : α), ε ≤ dist (↑α a) (↑α b) ∨ (↑α a, ↑α b) ∈ t ** intro x y ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x✝ y✝ : Completion α hxy : dist x✝ y✝ < ε x y : α ⊢ ε ≤ dist (↑α x) (↑α y) ∨ (↑α x, ↑α y) ∈ t ** rw [Completion.dist_eq] ** case refine'_2 α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x✝ y✝ : Completion α hxy : dist x✝ y✝ < ε x y : α ⊢ ε ≤ dist x y ∨ (↑α x, ↑α y) ∈ t ** by_cases h : ε ≤ dist x y ** case pos α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x✝ y✝ : Completion α hxy : dist x✝ y✝ < ε x y : α h : ε ≤ dist x y ⊢ ε ≤ dist x y ∨ (↑α x, ↑α y) ∈ t ** exact Or.inl h ** case neg α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x✝ y✝ : Completion α hxy : dist x✝ y✝ < ε x y : α h : ¬ε ≤ dist x y ⊢ ε ≤ dist x y ∨ (↑α x, ↑α y) ∈ t ** have Z := hε (not_le.1 h) ** case neg α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x✝ y✝ : Completion α hxy : dist x✝ y✝ < ε x y : α h : ¬ε ≤ dist x y Z : (x, y) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} ⊢ ε ≤ dist x y ∨ (↑α x, ↑α y) ∈ t ** simp only [Set.mem_setOf_eq] at Z ** case neg α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) t : Set (Completion α × Completion α) ht : t ∈ 𝓤 (Completion α) tclosed : IsClosed t ts : t ⊆ s A : {x | (↑α x.1, ↑α x.2) ∈ t} ∈ 𝓤 α ε : ℝ εpos : ε > 0 hε : ∀ {a b : α}, dist a b < ε → (a, b) ∈ {x | (↑α x.1, ↑α x.2) ∈ t} x✝ y✝ : Completion α hxy : dist x✝ y✝ < ε x y : α h : ¬ε ≤ dist x y Z : (↑α x, ↑α y) ∈ t ⊢ ε ≤ dist x y ∨ (↑α x, ↑α y) ∈ t ** exact Or.inr Z ** case mpr α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ⊢ (∃ ε, ε > 0 ∧ ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s) → s ∈ 𝓤 (Completion α) ** rintro ⟨ε, εpos, hε⟩ ** case mpr.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ⊢ s ∈ 𝓤 (Completion α) ** let r : Set (ℝ × ℝ) := { p | dist p.1 p.2 < ε } ** case mpr.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} ⊢ s ∈ 𝓤 (Completion α) ** have : r ∈ uniformity ℝ := Metric.dist_mem_uniformity εpos ** case mpr.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ ⊢ s ∈ 𝓤 (Completion α) ** have T := uniformContinuous_def.1 (@Completion.uniformContinuous_dist α _) r this ** case mpr.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ T : {x | (dist x.1.1 x.1.2, dist x.2.1 x.2.2) ∈ r} ∈ 𝓤 (Completion α × Completion α) ⊢ s ∈ 𝓤 (Completion α) ** simp only [uniformity_prod_eq_prod, mem_prod_iff, exists_prop, Filter.mem_map, Set.mem_setOf_eq] at T ** case mpr.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ T : ∃ t₁, t₁ ∈ 𝓤 (Completion α) ∧ ∃ t₂, t₂ ∈ 𝓤 (Completion α) ∧ t₁ ×ˢ t₂ ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} ⊢ s ∈ 𝓤 (Completion α) ** rcases T with ⟨t1, ht1, t2, ht2, ht⟩ ** case mpr.intro.intro.intro.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} ⊢ s ∈ 𝓤 (Completion α) ** refine' mem_of_superset ht1 _ ** case mpr.intro.intro.intro.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} ⊢ t1 ⊆ s ** have A : ∀ a b : Completion α, (a, b) ∈ t1 → dist a b < ε := by intro a b hab have : ((a, b), (a, a)) ∈ t1 ×ˢ t2 := ⟨hab, refl_mem_uniformity ht2⟩ have I := ht this simp [Completion.dist_self, Real.dist_eq, Completion.dist_comm] at I exact lt_of_le_of_lt (le_abs_self _) I ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} ⊢ ∀ (a b : Completion α), (a, b) ∈ t1 → dist a b < ε ** intro a b hab ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} a b : Completion α hab : (a, b) ∈ t1 ⊢ dist a b < ε ** have : ((a, b), (a, a)) ∈ t1 ×ˢ t2 := ⟨hab, refl_mem_uniformity ht2⟩ ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this✝ : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} a b : Completion α hab : (a, b) ∈ t1 this : ((a, b), a, a) ∈ t1 ×ˢ t2 ⊢ dist a b < ε ** have I := ht this ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this✝ : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} a b : Completion α hab : (a, b) ∈ t1 this : ((a, b), a, a) ∈ t1 ×ˢ t2 I : ((a, b), a, a) ∈ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} ⊢ dist a b < ε ** simp [Completion.dist_self, Real.dist_eq, Completion.dist_comm] at I ** α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this✝ : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} a b : Completion α hab : (a, b) ∈ t1 this : ((a, b), a, a) ∈ t1 ×ˢ t2 I : |dist a b| < ε ⊢ dist a b < ε ** exact lt_of_le_of_lt (le_abs_self _) I ** case mpr.intro.intro.intro.intro.intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} A : ∀ (a b : Completion α), (a, b) ∈ t1 → dist a b < ε ⊢ t1 ⊆ s ** rintro ⟨a, b⟩ hp ** case mpr.intro.intro.intro.intro.intro.intro.mk α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} A : ∀ (a b : Completion α), (a, b) ∈ t1 → dist a b < ε a b : Completion α hp : (a, b) ∈ t1 ⊢ (a, b) ∈ s ** have : dist a b < ε := A a b hp ** case mpr.intro.intro.intro.intro.intro.intro.mk α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s r : Set (ℝ × ℝ) := {p | dist p.1 p.2 < ε} this✝ : r ∈ 𝓤 ℝ t1 : Set (Completion α × Completion α) ht1 : t1 ∈ 𝓤 (Completion α) t2 : Set (Completion α × Completion α) ht2 : t2 ∈ 𝓤 (Completion α) ht : t1 ×ˢ t2 ⊆ (fun p => ((p.1.1, p.2.1), p.1.2, p.2.2)) ⁻¹' {x | dist (dist x.1.1 x.1.2) (dist x.2.1 x.2.2) < ε} A : ∀ (a b : Completion α), (a, b) ∈ t1 → dist a b < ε a b : Completion α hp : (a, b) ∈ t1 this : dist a b < ε ⊢ (a, b) ∈ s ** exact hε this ** Qed
UniformSpace.Completion.eq_of_dist_eq_zero ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α h : dist x y = 0 ⊢ x = y ** have : SeparatedSpace (Completion α) := by infer_instance ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α h : dist x y = 0 this : SeparatedSpace (Completion α) ⊢ x = y ** refine' separated_def.1 this x y fun s hs ↦ _ ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α h : dist x y = 0 this : SeparatedSpace (Completion α) s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) ⊢ (x, y) ∈ s ** rcases (Completion.mem_uniformity_dist s).1 hs with ⟨ε, εpos, hε⟩ ** case intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α h : dist x y = 0 this : SeparatedSpace (Completion α) s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) ε : ℝ εpos : ε > 0 hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ⊢ (x, y) ∈ s ** rw [← h] at εpos ** case intro.intro α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α h : dist x y = 0 this : SeparatedSpace (Completion α) s : Set (Completion α × Completion α) hs : s ∈ 𝓤 (Completion α) ε : ℝ εpos : ε > dist x y hε : ∀ {a b : Completion α}, dist a b < ε → (a, b) ∈ s ⊢ (x, y) ∈ s ** exact hε εpos ** α : Type u β : Type v inst✝ : PseudoMetricSpace α x y : Completion α h : dist x y = 0 ⊢ SeparatedSpace (Completion α) ** infer_instance ** Qed
UniformSpace.Completion.uniformity_dist' ** α : Type u β : Type v inst✝ : PseudoMetricSpace α ⊢ 𝓤 (Completion α) = ⨅ ε, 𝓟 {p | dist p.1 p.2 < ↑ε} ** ext s ** case a α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ⊢ s ∈ 𝓤 (Completion α) ↔ s ∈ ⨅ ε, 𝓟 {p | dist p.1 p.2 < ↑ε} ** rw [mem_iInf_of_directed] ** case a α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ⊢ s ∈ 𝓤 (Completion α) ↔ ∃ i, s ∈ 𝓟 {p | dist p.1 p.2 < ↑i} ** simp [Completion.mem_uniformity_dist, subset_def] ** case a.h α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) ⊢ Directed (fun x x_1 => x ≥ x_1) fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε} ** rintro ⟨r, hr⟩ ⟨p, hp⟩ ** case a.h.mk.mk α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) r : ℝ hr : 0 < r p : ℝ hp : 0 < p ⊢ ∃ z, (fun x x_1 => x ≥ x_1) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) { val := r, property := hr }) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) z) ∧ (fun x x_1 => x ≥ x_1) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) { val := p, property := hp }) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) z) ** use ⟨min r p, lt_min hr hp⟩ ** case h α : Type u β : Type v inst✝ : PseudoMetricSpace α s : Set (Completion α × Completion α) r : ℝ hr : 0 < r p : ℝ hp : 0 < p ⊢ (fun x x_1 => x ≥ x_1) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) { val := r, property := hr }) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) { val := min r p, property := (_ : 0 < min r p) }) ∧ (fun x x_1 => x ≥ x_1) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) { val := p, property := hp }) ((fun ε => 𝓟 {p | dist p.1 p.2 < ↑ε}) { val := min r p, property := (_ : 0 < min r p) }) ** simp (config := { contextual := true }) [lt_min_iff] ** Qed
UniformSpace.Completion.uniformity_dist ** α : Type u β : Type v inst✝ : PseudoMetricSpace α ⊢ 𝓤 (Completion α) = ⨅ ε, ⨅ (_ : ε > 0), 𝓟 {p | dist p.1 p.2 < ε} ** simpa [iInf_subtype] using @Completion.uniformity_dist' α _ ** Qed
LipschitzWith.completion_extension ** α : Type u β : Type v inst✝² : PseudoMetricSpace α inst✝¹ : MetricSpace β inst✝ : CompleteSpace β f : α → β K : ℝ≥0 h : LipschitzWith K f x y : Completion α ⊢ Continuous fun x => dist (Completion.extension f x.1) (Completion.extension f x.2) ** continuity ** α : Type u β : Type v inst✝² : PseudoMetricSpace α inst✝¹ : MetricSpace β inst✝ : CompleteSpace β f : α → β K : ℝ≥0 h : LipschitzWith K f x y : Completion α ⊢ Continuous fun x => ↑K * dist x.1 x.2 ** continuity ** α : Type u β : Type v inst✝² : PseudoMetricSpace α inst✝¹ : MetricSpace β inst✝ : CompleteSpace β f : α → β K : ℝ≥0 h : LipschitzWith K f x y : Completion α ⊢ ∀ (a b : α), dist (Completion.extension f (↑α a)) (Completion.extension f (↑α b)) ≤ ↑K * dist (↑α a) (↑α b) ** simpa only [extension_coe h.uniformContinuous, Completion.dist_eq] using h.dist_le_mul ** Qed
Isometry.completion_extension ** α : Type u β : Type v inst✝² : PseudoMetricSpace α inst✝¹ : MetricSpace β inst✝ : CompleteSpace β f : α → β h : Isometry f x y : Completion α ⊢ Continuous fun x => dist (Completion.extension f x.1) (Completion.extension f x.2) ** continuity ** α : Type u β : Type v inst✝² : PseudoMetricSpace α inst✝¹ : MetricSpace β inst✝ : CompleteSpace β f : α → β h : Isometry f x y : Completion α ⊢ Continuous fun x => dist x.1 x.2 ** continuity ** α : Type u β : Type v inst✝² : PseudoMetricSpace α inst✝¹ : MetricSpace β inst✝ : CompleteSpace β f : α → β h : Isometry f x y : Completion α x✝¹ x✝ : α ⊢ dist (Completion.extension f (↑α x✝¹)) (Completion.extension f (↑α x✝)) = dist (↑α x✝¹) (↑α x✝) ** simp only [extension_coe h.uniformContinuous, Completion.dist_eq, h.dist_eq] ** Qed
MulAction.continuousSMul_compHom ** M : Type u_1 X : Type u_2 Y : Type u_3 α : Type u_4 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace X inst✝⁵ : TopologicalSpace Y inst✝⁴ : Monoid M inst✝³ : MulAction M X inst✝² : ContinuousSMul M X N : Type u_5 inst✝¹ : TopologicalSpace N inst✝ : Monoid N f : N →* M hf : Continuous ↑f ⊢ ContinuousSMul N X ** let _ : MulAction N X := MulAction.compHom _ f ** M : Type u_1 X : Type u_2 Y : Type u_3 α : Type u_4 inst✝⁷ : TopologicalSpace M inst✝⁶ : TopologicalSpace X inst✝⁵ : TopologicalSpace Y inst✝⁴ : Monoid M inst✝³ : MulAction M X inst✝² : ContinuousSMul M X N : Type u_5 inst✝¹ : TopologicalSpace N inst✝ : Monoid N f : N →* M hf : Continuous ↑f x✝ : MulAction N X := compHom X f ⊢ ContinuousSMul N X ** exact ⟨(hf.comp continuous_fst).smul continuous_snd⟩ ** Qed
continuousSMul_sInf ** ι : Sort u_1 M : Type u_2 X : Type u_3 inst✝¹ : TopologicalSpace M inst✝ : SMul M X ts : Set (TopologicalSpace X) h : ∀ (t : TopologicalSpace X), t ∈ ts → ContinuousSMul M X ⊢ Continuous fun p => p.1 • p.2 ** exact continuous_sInf_rng.2 fun t ht => continuous_sInf_dom₂ (Eq.refl _) ht (@ContinuousSMul.continuous_smul _ _ _ _ t (h t ht)) ** Qed
continuousSMul_inf ** ι : Sort u_1 M : Type u_2 X : Type u_3 inst✝³ : TopologicalSpace M inst✝² : SMul M X t₁ t₂ : TopologicalSpace X inst✝¹ : ContinuousSMul M X inst✝ : ContinuousSMul M X ⊢ ContinuousSMul M X ** refine' continuousSMul_iInf fun b => _ ** ι : Sort u_1 M : Type u_2 X : Type u_3 inst✝³ : TopologicalSpace M inst✝² : SMul M X t₁ t₂ : TopologicalSpace X inst✝¹ : ContinuousSMul M X inst✝ : ContinuousSMul M X b : Bool ⊢ ContinuousSMul M X ** cases b <;> assumption ** Qed
AddTorsor.connectedSpace ** G : Type u_1 P : Type u_2 inst✝⁵ : AddGroup G inst✝⁴ : AddTorsor G P inst✝³ : TopologicalSpace G inst✝² : PreconnectedSpace G inst✝¹ : TopologicalSpace P inst✝ : ContinuousVAdd G P ⊢ IsPreconnected Set.univ ** convert isPreconnected_univ.image (Equiv.vaddConst (Classical.arbitrary P) : G → P) (continuous_id.vadd continuous_const).continuousOn ** case h.e'_3 G : Type u_1 P : Type u_2 inst✝⁵ : AddGroup G inst✝⁴ : AddTorsor G P inst✝³ : TopologicalSpace G inst✝² : PreconnectedSpace G inst✝¹ : TopologicalSpace P inst✝ : ContinuousVAdd G P ⊢ Set.univ = ↑(Equiv.vaddConst (Classical.arbitrary P)) '' Set.univ ** rw [Set.image_univ, Equiv.range_eq_univ] ** Qed
tendsto_zero_iff_abs_tendsto_zero ** α : Type u_1 G : Type u_2 inst✝² : TopologicalSpace G inst✝¹ : LinearOrderedAddCommGroup G inst✝ : OrderTopology G l : Filter α f✝ g f : α → G ⊢ Tendsto f l (𝓝 0) ↔ Tendsto (abs ∘ f) l (𝓝 0) ** refine' ⟨fun h => (abs_zero : |(0 : G)| = 0) ▸ h.abs, fun h => _⟩ ** α : Type u_1 G : Type u_2 inst✝² : TopologicalSpace G inst✝¹ : LinearOrderedAddCommGroup G inst✝ : OrderTopology G l : Filter α f✝ g f : α → G h : Tendsto (abs ∘ f) l (𝓝 0) ⊢ Tendsto f l (𝓝 0) ** have : Tendsto (fun a => -|f a|) l (𝓝 0) := (neg_zero : -(0 : G) = 0) ▸ h.neg ** α : Type u_1 G : Type u_2 inst✝² : TopologicalSpace G inst✝¹ : LinearOrderedAddCommGroup G inst✝ : OrderTopology G l : Filter α f✝ g f : α → G h : Tendsto (abs ∘ f) l (𝓝 0) this : Tendsto (fun a => -|f a|) l (𝓝 0) ⊢ Tendsto f l (𝓝 0) ** exact tendsto_of_tendsto_of_tendsto_of_le_of_le this h (fun x => neg_abs_le_self <| f x) fun x => le_abs_self <| f x ** Qed