text
stringlengths 0
3.06M
| meta
stringlengths 57
121
|
---|---|
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ b : Basis ι R M
N : Submodule R M
ϕ : M →ₗ[R] R
hϕ : ∀ (ψ : M →ₗ[R] R), ¬map ϕ N < map ψ N
inst✝ : IsPrincipal (map ϕ N)
hgen : generator (map ϕ N) = 0
⊢ N = ⊥
[PROOFSTEP]
rw [Submodule.eq_bot_iff]
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ b : Basis ι R M
N : Submodule R M
ϕ : M →ₗ[R] R
hϕ : ∀ (ψ : M →ₗ[R] R), ¬map ϕ N < map ψ N
inst✝ : IsPrincipal (map ϕ N)
hgen : generator (map ϕ N) = 0
⊢ ∀ (x : M), x ∈ N → x = 0
[PROOFSTEP]
intro x hx
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ b : Basis ι R M
N : Submodule R M
ϕ : M →ₗ[R] R
hϕ : ∀ (ψ : M →ₗ[R] R), ¬map ϕ N < map ψ N
inst✝ : IsPrincipal (map ϕ N)
hgen : generator (map ϕ N) = 0
x : M
hx : x ∈ N
⊢ x = 0
[PROOFSTEP]
refine' b.ext_elem fun i ↦ _
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ b : Basis ι R M
N : Submodule R M
ϕ : M →ₗ[R] R
hϕ : ∀ (ψ : M →ₗ[R] R), ¬map ϕ N < map ψ N
inst✝ : IsPrincipal (map ϕ N)
hgen : generator (map ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr x) i = ↑(↑b.repr 0) i
[PROOFSTEP]
rw [(eq_bot_iff_generator_eq_zero _).mpr hgen] at hϕ
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ b : Basis ι R M
N : Submodule R M
ϕ : M →ₗ[R] R
hϕ : ∀ (ψ : M →ₗ[R] R), ¬⊥ < map ψ N
inst✝ : IsPrincipal (map ϕ N)
hgen : generator (map ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr x) i = ↑(↑b.repr 0) i
[PROOFSTEP]
rw [LinearEquiv.map_zero, Finsupp.zero_apply]
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ b : Basis ι R M
N : Submodule R M
ϕ : M →ₗ[R] R
hϕ : ∀ (ψ : M →ₗ[R] R), ¬⊥ < map ψ N
inst✝ : IsPrincipal (map ϕ N)
hgen : generator (map ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr x) i = 0
[PROOFSTEP]
exact (Submodule.eq_bot_iff _).mp (not_bot_lt_iff.1 <| hϕ (Finsupp.lapply i ∘ₗ ↑b.repr)) _ ⟨x, hx, rfl⟩
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
⊢ N = ⊥
[PROOFSTEP]
rw [Submodule.eq_bot_iff]
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
⊢ ∀ (x : M), x ∈ N → x = 0
[PROOFSTEP]
intro x hx
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
x : M
hx : x ∈ N
⊢ x = 0
[PROOFSTEP]
refine (mk_eq_zero _ _).mp (show (⟨x, hNO hx⟩ : O) = 0 from b.ext_elem fun i ↦ ?_)
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr { val := x, property := (_ : x ∈ O) }) i = ↑(↑b.repr 0) i
[PROOFSTEP]
rw [(eq_bot_iff_generator_eq_zero _).mpr hgen] at hϕ
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬⊥ < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr { val := x, property := (_ : x ∈ O) }) i = ↑(↑b.repr 0) i
[PROOFSTEP]
rw [LinearEquiv.map_zero, Finsupp.zero_apply]
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬⊥ < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr { val := x, property := (_ : x ∈ O) }) i = 0
[PROOFSTEP]
refine (Submodule.eq_bot_iff _).mp (not_bot_lt_iff.1 <| hϕ (Finsupp.lapply i ∘ₗ ↑b.repr)) _ ?_
[GOAL]
R : Type u
M : Type v
inst✝³ : Ring R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
ι : Type u_1
b✝ : Basis ι R M
N O : Submodule R M
b : Basis ι R { x // x ∈ O }
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬⊥ < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
hgen : generator (LinearMap.submoduleImage ϕ N) = 0
x : M
hx : x ∈ N
i : ι
⊢ ↑(↑b.repr { val := x, property := (_ : x ∈ O) }) i ∈
LinearMap.submoduleImage (LinearMap.comp (Finsupp.lapply i) ↑b.repr) N
[PROOFSTEP]
exact (LinearMap.mem_submoduleImage_of_le hNO).mpr ⟨x, hx, rfl⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁴ : CommRing R
inst✝³ : IsDomain R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
I : Ideal R
inst✝ : IsPrincipal I
x : R
hx : x ∈ I
⊢ x ∣ generator I ↔ I = Ideal.span {x}
[PROOFSTEP]
conv_rhs => rw [← span_singleton_generator I]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁴ : CommRing R
inst✝³ : IsDomain R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
I : Ideal R
inst✝ : IsPrincipal I
x : R
hx : x ∈ I
| I = Ideal.span {x}
[PROOFSTEP]
rw [← span_singleton_generator I]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁴ : CommRing R
inst✝³ : IsDomain R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
I : Ideal R
inst✝ : IsPrincipal I
x : R
hx : x ∈ I
| I = Ideal.span {x}
[PROOFSTEP]
rw [← span_singleton_generator I]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁴ : CommRing R
inst✝³ : IsDomain R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
I : Ideal R
inst✝ : IsPrincipal I
x : R
hx : x ∈ I
| I = Ideal.span {x}
[PROOFSTEP]
rw [← span_singleton_generator I]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁴ : CommRing R
inst✝³ : IsDomain R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
I : Ideal R
inst✝ : IsPrincipal I
x : R
hx : x ∈ I
⊢ x ∣ generator I ↔ span R {generator I} = Ideal.span {x}
[PROOFSTEP]
rw [Ideal.submodule_span_eq, Ideal.span_singleton_eq_span_singleton, ← dvd_dvd_iff_associated, ← mem_iff_generator_dvd]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁴ : CommRing R
inst✝³ : IsDomain R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
I : Ideal R
inst✝ : IsPrincipal I
x : R
hx : x ∈ I
⊢ x ∣ generator I ↔ x ∈ I ∧ x ∣ generator I
[PROOFSTEP]
exact ⟨fun h ↦ ⟨hx, h⟩, fun h ↦ h.2⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
⊢ generator (LinearMap.submoduleImage ϕ N) ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
let a : R := generator (ϕ.submoduleImage N)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
⊢ generator (LinearMap.submoduleImage ϕ N) ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
let d : R := IsPrincipal.generator (Submodule.span R {a, ψ ⟨y, hNO yN⟩})
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
⊢ generator (LinearMap.submoduleImage ϕ N) ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
have d_dvd_left : d ∣ a := (mem_iff_generator_dvd _).mp (subset_span (mem_insert _ _))
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
⊢ generator (LinearMap.submoduleImage ϕ N) ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
have d_dvd_right : d ∣ ψ ⟨y, hNO yN⟩ :=
(mem_iff_generator_dvd _).mp (subset_span (mem_insert_of_mem _ (mem_singleton _)))
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
refine' dvd_trans _ d_dvd_right
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∣ d
[PROOFSTEP]
rw [dvd_generator_iff, Ideal.span, ← span_singleton_generator (Submodule.span R {a, ψ ⟨y, hNO yN⟩})]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ span R {generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})} =
span R {generator (LinearMap.submoduleImage ϕ N)}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
obtain ⟨r₁, r₂, d_eq⟩ : ∃ r₁ r₂ : R, d = r₁ * a + r₂ * ψ ⟨y, hNO yN⟩ :=
by
obtain ⟨r₁, r₂', hr₂', hr₁⟩ := mem_span_insert.mp (IsPrincipal.generator_mem (Submodule.span R {a, ψ ⟨y, hNO yN⟩}))
obtain ⟨r₂, rfl⟩ := mem_span_singleton.mp hr₂'
exact ⟨r₁, r₂, hr₁⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ ∃ r₁ r₂, d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
obtain ⟨r₁, r₂', hr₂', hr₁⟩ := mem_span_insert.mp (IsPrincipal.generator_mem (Submodule.span R {a, ψ ⟨y, hNO yN⟩}))
[GOAL]
case intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂' : R
hr₂' : r₂' ∈ span R {↑ψ { val := y, property := (_ : y ∈ O) }}
hr₁ : generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}) = r₁ • a + r₂'
⊢ ∃ r₁ r₂, d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
obtain ⟨r₂, rfl⟩ := mem_span_singleton.mp hr₂'
[GOAL]
case intro.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
hr₂' : r₂ • ↑ψ { val := y, property := (_ : y ∈ O) } ∈ span R {↑ψ { val := y, property := (_ : y ∈ O) }}
hr₁ :
generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}) =
r₁ • a + r₂ • ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ ∃ r₁ r₂, d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
[PROOFSTEP]
exact ⟨r₁, r₂, hr₁⟩
[GOAL]
case intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ span R {generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})} =
span R {generator (LinearMap.submoduleImage ϕ N)}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
let ψ' : O →ₗ[R] R := r₁ • ϕ + r₂ • ψ
[GOAL]
case intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
⊢ span R {generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})} =
span R {generator (LinearMap.submoduleImage ϕ N)}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
have : span R { d } ≤ ψ'.submoduleImage N :=
by
rw [span_le, singleton_subset_iff, SetLike.mem_coe, LinearMap.mem_submoduleImage_of_le hNO]
refine' ⟨y, yN, _⟩
change r₁ * ϕ ⟨y, hNO yN⟩ + r₂ * ψ ⟨y, hNO yN⟩ = d
rw [d_eq, ϕy_eq]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
⊢ span R {d} ≤ LinearMap.submoduleImage ψ' N
[PROOFSTEP]
rw [span_le, singleton_subset_iff, SetLike.mem_coe, LinearMap.mem_submoduleImage_of_le hNO]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
⊢ ∃ y yN, ↑ψ' { val := y, property := (_ : y ∈ O) } = d
[PROOFSTEP]
refine' ⟨y, yN, _⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
⊢ ↑ψ' { val := y, property := (_ : y ∈ O) } = d
[PROOFSTEP]
change r₁ * ϕ ⟨y, hNO yN⟩ + r₂ * ψ ⟨y, hNO yN⟩ = d
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
⊢ r₁ * ↑ϕ { val := y, property := (_ : y ∈ O) } + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) } = d
[PROOFSTEP]
rw [d_eq, ϕy_eq]
[GOAL]
case intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
this : span R {d} ≤ LinearMap.submoduleImage ψ' N
⊢ span R {generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})} =
span R {generator (LinearMap.submoduleImage ϕ N)}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
refine' le_antisymm (this.trans (le_of_eq _)) (Ideal.span_singleton_le_span_singleton.mpr d_dvd_left)
[GOAL]
case intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
this : span R {d} ≤ LinearMap.submoduleImage ψ' N
⊢ LinearMap.submoduleImage ψ' N = span R {generator (LinearMap.submoduleImage ϕ N)}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
rw [span_singleton_generator]
[GOAL]
case intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
this : span R {d} ≤ LinearMap.submoduleImage ψ' N
⊢ LinearMap.submoduleImage ψ' N = LinearMap.submoduleImage ϕ N
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
apply (le_trans _ this).eq_of_not_gt (hϕ ψ')
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
this : span R {d} ≤ LinearMap.submoduleImage ψ' N
⊢ LinearMap.submoduleImage ϕ N ≤ span R {d}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
rw [← span_singleton_generator (ϕ.submoduleImage N)]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
r₁ r₂ : R
d_eq : d = r₁ * a + r₂ * ↑ψ { val := y, property := (_ : y ∈ O) }
ψ' : { x // x ∈ O } →ₗ[R] R := r₁ • ϕ + r₂ • ψ
this : span R {d} ≤ LinearMap.submoduleImage ψ' N
⊢ span R {generator (LinearMap.submoduleImage ϕ N)} ≤ span R {d}
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
exact Ideal.span_singleton_le_span_singleton.mpr d_dvd_left
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : ι → M
N O : Submodule R M
hNO : N ≤ O
ϕ : { x // x ∈ O } →ₗ[R] R
hϕ : ∀ (ψ : { x // x ∈ O } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
inst✝ : IsPrincipal (LinearMap.submoduleImage ϕ N)
y : M
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ O) } = generator (LinearMap.submoduleImage ϕ N)
ψ : { x // x ∈ O } →ₗ[R] R
a : R := generator (LinearMap.submoduleImage ϕ N)
d : R := generator (span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }})
d_dvd_left : d ∣ a
d_dvd_right : d ∣ ↑ψ { val := y, property := (_ : y ∈ O) }
⊢ generator (LinearMap.submoduleImage ϕ N) ∈ span R {a, ↑ψ { val := y, property := (_ : y ∈ O) }}
[PROOFSTEP]
exact subset_span (mem_insert _ _)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have : ∃ ϕ : M →ₗ[R] R, ∀ ψ : M →ₗ[R] R, ¬ϕ.submoduleImage N < ψ.submoduleImage N :=
by
obtain ⟨P, P_eq, P_max⟩ :=
set_has_maximal_iff_noetherian.mpr (inferInstance : IsNoetherian R R) _
(show (Set.range fun ψ : M →ₗ[R] R ↦ ψ.submoduleImage N).Nonempty from ⟨_, Set.mem_range.mpr ⟨0, rfl⟩⟩)
obtain ⟨ϕ, rfl⟩ := Set.mem_range.mp P_eq
exact ⟨ϕ, fun ψ hψ ↦ P_max _ ⟨_, rfl⟩ hψ⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
⊢ ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
[PROOFSTEP]
obtain ⟨P, P_eq, P_max⟩ :=
set_has_maximal_iff_noetherian.mpr (inferInstance : IsNoetherian R R) _
(show (Set.range fun ψ : M →ₗ[R] R ↦ ψ.submoduleImage N).Nonempty from ⟨_, Set.mem_range.mpr ⟨0, rfl⟩⟩)
[GOAL]
case intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
P : Submodule R R
P_eq : P ∈ range fun ψ => LinearMap.submoduleImage ψ N
P_max : ∀ (I : Submodule R R), (I ∈ range fun ψ => LinearMap.submoduleImage ψ N) → ¬P < I
⊢ ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
[PROOFSTEP]
obtain ⟨ϕ, rfl⟩ := Set.mem_range.mp P_eq
[GOAL]
case intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
ϕ : { x // x ∈ M } →ₗ[R] R
P_eq : LinearMap.submoduleImage ϕ N ∈ range fun ψ => LinearMap.submoduleImage ψ N
P_max : ∀ (I : Submodule R R), (I ∈ range fun ψ => LinearMap.submoduleImage ψ N) → ¬LinearMap.submoduleImage ϕ N < I
⊢ ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
[PROOFSTEP]
exact ⟨ϕ, fun ψ hψ ↦ P_max _ ⟨_, rfl⟩ hψ⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
let ϕ := this.choose
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have ϕ_max := this.choose_spec
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
let a := generator (ϕ.submoduleImage N)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have a_mem : a ∈ ϕ.submoduleImage N :=
generator_mem
_
-- If `a` is zero, then the submodule is trivial. So let's assume `a ≠ 0`, `N ≠ ⊥`.
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
by_cases a_zero : a = 0
[GOAL]
case pos
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : a = 0
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have := eq_bot_of_generator_maximal_submoduleImage_eq_zero b'M N_le_M ϕ_max a_zero
[GOAL]
case pos
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this✝ : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this✝
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this✝) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : a = 0
this : N = ⊥
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
contradiction
-- We claim that `ϕ⁻¹ a = y` can be taken as basis element of `N`.
[GOAL]
case neg
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
obtain ⟨y, yN, ϕy_eq⟩ := (LinearMap.mem_submoduleImage_of_le N_le_M).mp a_mem
[GOAL]
case neg.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have _ϕy_ne_zero : ϕ ⟨y, N_le_M yN⟩ ≠ 0 := fun h ↦
a_zero
(ϕy_eq.symm.trans h)
-- Write `y` as `a • y'` for some `y'`.
[GOAL]
case neg.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have hdvd : ∀ i, a ∣ b'M.coord i ⟨y, N_le_M yN⟩ := fun i ↦
generator_maximal_submoduleImage_dvd N_le_M ϕ_max y yN ϕy_eq (b'M.coord i)
[GOAL]
case neg.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
hdvd : ∀ (i : ι), a ∣ ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) }
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
choose c hc using hdvd
[GOAL]
case neg.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
let y' : O := ∑ i, c i • b'M i
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have y'M : y' ∈ M := M.sum_mem fun i _ ↦ M.smul_mem (c i) (b'M i).2
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have mk_y' : (⟨y', y'M⟩ : M) = ∑ i, c i • b'M i :=
Subtype.ext
(show y' = M.subtype _ by
simp only [LinearMap.map_sum, LinearMap.map_smul]
rfl)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
⊢ y' = ↑(Submodule.subtype M) (∑ i : ι, c i • ↑b'M i)
[PROOFSTEP]
simp only [LinearMap.map_sum, LinearMap.map_smul]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
⊢ ∑ x : ι, ↑(c x • ↑b'M x) = ∑ x : ι, c x • ↑(Submodule.subtype M) (↑b'M x)
[PROOFSTEP]
rfl
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have a_smul_y' : a • y' = y :=
by
refine Subtype.mk_eq_mk.mp (show (a • ⟨y', y'M⟩ : M) = ⟨y, N_le_M yN⟩ from ?_)
rw [← b'M.sum_repr ⟨y, N_le_M yN⟩, mk_y', Finset.smul_sum]
refine' Finset.sum_congr rfl fun i _ ↦ _
rw [← mul_smul, ← hc]
rfl
-- We found a `y` and an `a`!
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
⊢ a • y' = y
[PROOFSTEP]
refine Subtype.mk_eq_mk.mp (show (a • ⟨y', y'M⟩ : M) = ⟨y, N_le_M yN⟩ from ?_)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
⊢ a • { val := y', property := y'M } = { val := y, property := (_ : y ∈ M) }
[PROOFSTEP]
rw [← b'M.sum_repr ⟨y, N_le_M yN⟩, mk_y', Finset.smul_sum]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
⊢ ∑ x : ι, a • c x • ↑b'M x = ∑ i : ι, ↑(↑b'M.repr { val := y, property := (_ : y ∈ M) }) i • ↑b'M i
[PROOFSTEP]
refine' Finset.sum_congr rfl fun i _ ↦ _
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
i : ι
x✝ : i ∈ Finset.univ
⊢ a • c i • ↑b'M i = ↑(↑b'M.repr { val := y, property := (_ : y ∈ M) }) i • ↑b'M i
[PROOFSTEP]
rw [← mul_smul, ← hc]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
i : ι
x✝ : i ∈ Finset.univ
⊢ ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } • ↑b'M i =
↑(↑b'M.repr { val := y, property := (_ : y ∈ M) }) i • ↑b'M i
[PROOFSTEP]
rfl
-- We found a `y` and an `a`!
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
⊢ ∃ y,
y ∈ M ∧
∃ a x M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
refine' ⟨y', y'M, a, a_smul_y'.symm ▸ yN, _⟩
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have ϕy'_eq : ϕ ⟨y', y'M⟩ = 1 :=
mul_left_cancel₀ a_zero
(calc
a • ϕ ⟨y', y'M⟩ = ϕ ⟨a • y', _⟩ := (ϕ.map_smul a ⟨y', y'M⟩).symm
_ = ϕ ⟨y, N_le_M yN⟩ := by simp only [a_smul_y']
_ = a := ϕy_eq
_ = a * 1 := (mul_one a).symm)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
⊢ ↑ϕ { val := a • y', property := (_ : a • ↑{ val := y', property := y'M } ∈ M) } =
↑ϕ { val := y, property := (_ : y ∈ M) }
[PROOFSTEP]
simp only [a_smul_y']
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have ϕy'_ne_zero : ϕ ⟨y', y'M⟩ ≠ 0 := by simpa only [ϕy'_eq] using one_ne_zero
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
⊢ ↑ϕ { val := y', property := y'M } ≠ 0
[PROOFSTEP]
simpa only [ϕy'_eq] using one_ne_zero
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
let M' : Submodule R O := ϕ.ker.map M.subtype
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
let N' : Submodule R O := (ϕ.comp (ofLe N_le_M)).ker.map N.subtype
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have M'_le_M : M' ≤ M := M.map_subtype_le (LinearMap.ker ϕ)
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have N'_le_M' : N' ≤ M' := by
intro x hx
simp only [mem_map, LinearMap.mem_ker] at hx ⊢
obtain ⟨⟨x, xN⟩, hx, rfl⟩ := hx
exact ⟨⟨x, N_le_M xN⟩, hx, rfl⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
⊢ N' ≤ M'
[PROOFSTEP]
intro x hx
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
x : O
hx : x ∈ N'
⊢ x ∈ M'
[PROOFSTEP]
simp only [mem_map, LinearMap.mem_ker] at hx ⊢
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
x : O
hx : ∃ y, ↑(LinearMap.comp (Exists.choose this) (ofLe N_le_M)) y = 0 ∧ ↑(Submodule.subtype N) y = x
⊢ ∃ y, ↑(Exists.choose this) y = 0 ∧ ↑(Submodule.subtype M) y = x
[PROOFSTEP]
obtain ⟨⟨x, xN⟩, hx, rfl⟩ := hx
[GOAL]
case intro.mk.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
x : O
xN : x ∈ N
hx : ↑(LinearMap.comp (Exists.choose this) (ofLe N_le_M)) { val := x, property := xN } = 0
⊢ ∃ y, ↑(Exists.choose this) y = 0 ∧ ↑(Submodule.subtype M) y = ↑(Submodule.subtype N) { val := x, property := xN }
[PROOFSTEP]
exact ⟨⟨x, N_le_M xN⟩, hx, rfl⟩
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have N'_le_N : N' ≤ N :=
N.map_subtype_le
(LinearMap.ker (ϕ.comp (ofLe N_le_M)))
-- So fill in those results as well.
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
⊢ ∃ M',
M' ≤ M ∧
∃ N',
N' ≤ N ∧
∃ _N'_le_M' _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
refine'
⟨M', M'_le_M, N', N'_le_N, N'_le_M', _⟩
-- Note that `y'` is orthogonal to `M'`.
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
⊢ ∃ _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have y'_ortho_M' : ∀ (c : R), ∀ z ∈ M', c • y' + z = 0 → c = 0 :=
by
intro c x xM' hc
obtain ⟨⟨x, xM⟩, hx', rfl⟩ := Submodule.mem_map.mp xM'
rw [LinearMap.mem_ker] at hx'
have hc' : (c • ⟨y', y'M⟩ + ⟨x, xM⟩ : M) = 0 := by exact @Subtype.coe_injective O (· ∈ M) _ _ hc
simpa only [LinearMap.map_add, LinearMap.map_zero, LinearMap.map_smul, smul_eq_mul, add_zero, mul_eq_zero,
ϕy'_ne_zero, hx', or_false_iff] using congr_arg ϕ hc'
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
⊢ ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
[PROOFSTEP]
intro c x xM' hc
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
c : R
x : O
xM' : x ∈ M'
hc : c • y' + x = 0
⊢ c = 0
[PROOFSTEP]
obtain ⟨⟨x, xM⟩, hx', rfl⟩ := Submodule.mem_map.mp xM'
[GOAL]
case intro.mk.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
c : R
x : O
xM : x ∈ M
hx' : { val := x, property := xM } ∈ LinearMap.ker ϕ
xM' : ↑(Submodule.subtype M) { val := x, property := xM } ∈ M'
hc : c • y' + ↑(Submodule.subtype M) { val := x, property := xM } = 0
⊢ c = 0
[PROOFSTEP]
rw [LinearMap.mem_ker] at hx'
[GOAL]
case intro.mk.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
c : R
x : O
xM : x ∈ M
hx' : ↑ϕ { val := x, property := xM } = 0
xM' : ↑(Submodule.subtype M) { val := x, property := xM } ∈ M'
hc : c • y' + ↑(Submodule.subtype M) { val := x, property := xM } = 0
⊢ c = 0
[PROOFSTEP]
have hc' : (c • ⟨y', y'M⟩ + ⟨x, xM⟩ : M) = 0 := by exact @Subtype.coe_injective O (· ∈ M) _ _ hc
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
c : R
x : O
xM : x ∈ M
hx' : ↑ϕ { val := x, property := xM } = 0
xM' : ↑(Submodule.subtype M) { val := x, property := xM } ∈ M'
hc : c • y' + ↑(Submodule.subtype M) { val := x, property := xM } = 0
⊢ c • { val := y', property := y'M } + { val := x, property := xM } = 0
[PROOFSTEP]
exact @Subtype.coe_injective O (· ∈ M) _ _ hc
[GOAL]
case intro.mk.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
c : R
x : O
xM : x ∈ M
hx' : ↑ϕ { val := x, property := xM } = 0
xM' : ↑(Submodule.subtype M) { val := x, property := xM } ∈ M'
hc : c • y' + ↑(Submodule.subtype M) { val := x, property := xM } = 0
hc' : c • { val := y', property := y'M } + { val := x, property := xM } = 0
⊢ c = 0
[PROOFSTEP]
simpa only [LinearMap.map_add, LinearMap.map_zero, LinearMap.map_smul, smul_eq_mul, add_zero, mul_eq_zero, ϕy'_ne_zero,
hx', or_false_iff] using congr_arg ϕ hc'
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
⊢ ∃ _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
have ay'_ortho_N' : ∀ (c : R), ∀ z ∈ N', c • a • y' + z = 0 → c = 0 :=
by
intro c z zN' hc
refine' (mul_eq_zero.mp (y'_ortho_M' (a * c) z (N'_le_M' zN') _)).resolve_left a_zero
rw [mul_comm, mul_smul, hc]
-- So we can extend a basis for `N'` with `y`
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
⊢ ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
[PROOFSTEP]
intro c z zN' hc
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
c : R
z : O
zN' : z ∈ N'
hc : c • a • y' + z = 0
⊢ c = 0
[PROOFSTEP]
refine' (mul_eq_zero.mp (y'_ortho_M' (a * c) z (N'_le_M' zN') _)).resolve_left a_zero
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
c : R
z : O
zN' : z ∈ N'
hc : c • a • y' + z = 0
⊢ (a * c) • y' + z = 0
[PROOFSTEP]
rw [mul_comm, mul_smul, hc]
-- So we can extend a basis for `N'` with `y`
[GOAL]
case neg.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
⊢ ∃ _y_ortho_M' _ay_ortho_N',
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
refine' ⟨y'_ortho_M', ay'_ortho_N', fun n' bN' ↦ ⟨_, _⟩⟩
[GOAL]
case neg.intro.intro.intro.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
⊢ Basis (Fin (n' + 1)) R { x // x ∈ N }
[PROOFSTEP]
refine' Basis.mkFinConsOfLE y yN bN' N'_le_N _ _
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
⊢ ∀ (c : R) (x : O), x ∈ N' → c • y + x = 0 → c = 0
[PROOFSTEP]
intro c z zN' hc
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
c : R
z : O
zN' : z ∈ N'
hc : c • y + z = 0
⊢ c = 0
[PROOFSTEP]
refine' ay'_ortho_N' c z zN' _
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c✝ : ι → R
hc✝ : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c✝ i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c✝ i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c✝ i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
c : R
z : O
zN' : z ∈ N'
hc : c • y + z = 0
⊢ c • a • y' + z = 0
[PROOFSTEP]
rwa [← a_smul_y'] at hc
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
⊢ ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'
[PROOFSTEP]
intro z zN
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
z : O
zN : z ∈ N
⊢ ∃ c, z + c • y ∈ N'
[PROOFSTEP]
obtain ⟨b, hb⟩ : _ ∣ ϕ ⟨z, N_le_M zN⟩ := generator_submoduleImage_dvd_of_mem N_le_M ϕ zN
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_2.intro
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b✝ : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
z : O
zN : z ∈ N
b : R
hb : ↑ϕ { val := z, property := (_ : z ∈ M) } = generator (LinearMap.submoduleImage ϕ N) * b
⊢ ∃ c, z + c • y ∈ N'
[PROOFSTEP]
refine' ⟨-b, Submodule.mem_map.mpr ⟨⟨_, N.sub_mem zN (N.smul_mem b yN)⟩, _, _⟩⟩
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_2.intro.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b✝ : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
z : O
zN : z ∈ N
b : R
hb : ↑ϕ { val := z, property := (_ : z ∈ M) } = generator (LinearMap.submoduleImage ϕ N) * b
⊢ { val := z - b • y, property := (_ : z - b • y ∈ N) } ∈ LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M))
[PROOFSTEP]
refine' LinearMap.mem_ker.mpr (show ϕ (⟨z, N_le_M zN⟩ - b • ⟨y, N_le_M yN⟩) = 0 from _)
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_2.intro.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b✝ : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
z : O
zN : z ∈ N
b : R
hb : ↑ϕ { val := z, property := (_ : z ∈ M) } = generator (LinearMap.submoduleImage ϕ N) * b
⊢ ↑ϕ ({ val := z, property := (_ : z ∈ M) } - b • { val := y, property := (_ : y ∈ M) }) = 0
[PROOFSTEP]
rw [LinearMap.map_sub, LinearMap.map_smul, hb, ϕy_eq, smul_eq_mul, mul_comm, sub_self]
[GOAL]
case neg.intro.intro.intro.refine'_1.refine'_2.intro.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b✝ : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
z : O
zN : z ∈ N
b : R
hb : ↑ϕ { val := z, property := (_ : z ∈ M) } = generator (LinearMap.submoduleImage ϕ N) * b
⊢ ↑(Submodule.subtype N) { val := z - b • y, property := (_ : z - b • y ∈ N) } = z + -b • y
[PROOFSTEP]
simp only [sub_eq_add_neg, neg_smul, coeSubtype]
-- And extend a basis for `M'` with `y'`
[GOAL]
case neg.intro.intro.intro.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
⊢ ∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as',
∀ (i : Fin (n' + 1)),
↑(↑(Basis.mkFinConsOfLE y yN bN' N'_le_N (_ : ∀ (c : R) (z : O), z ∈ N' → c • y + z = 0 → c = 0)
(_ : ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'))
i) =
as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
intro m' hn'm' bM'
[GOAL]
case neg.intro.intro.intro.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
⊢ ∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as',
∀ (i : Fin (n' + 1)),
↑(↑(Basis.mkFinConsOfLE y yN bN' N'_le_N (_ : ∀ (c : R) (z : O), z ∈ N' → c • y + z = 0 → c = 0)
(_ : ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'))
i) =
as' i • ↑(↑bM (Fin.castLE hnm i))
[PROOFSTEP]
refine' ⟨Nat.succ_le_succ hn'm', _, _⟩
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
⊢ Basis (Fin (m' + 1)) R { x // x ∈ M }
[PROOFSTEP]
refine' Basis.mkFinConsOfLE y' y'M bM' M'_le_M y'_ortho_M' _
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
⊢ ∀ (z : O), z ∈ M → ∃ c, z + c • y' ∈ M'
[PROOFSTEP]
intro z zM
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
z : O
zM : z ∈ M
⊢ ∃ c, z + c • y' ∈ M'
[PROOFSTEP]
refine' ⟨-ϕ ⟨z, zM⟩, ⟨⟨z, zM⟩ - ϕ ⟨z, zM⟩ • ⟨y', y'M⟩, LinearMap.mem_ker.mpr _, _⟩⟩
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_1.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
z : O
zM : z ∈ M
⊢ ↑ϕ ({ val := z, property := zM } - ↑ϕ { val := z, property := zM } • { val := y', property := y'M }) = 0
[PROOFSTEP]
rw [LinearMap.map_sub, LinearMap.map_smul, ϕy'_eq, smul_eq_mul, mul_one, sub_self]
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_1.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
z : O
zM : z ∈ M
⊢ ↑(Submodule.subtype M)
({ val := z, property := zM } - ↑ϕ { val := z, property := zM } • { val := y', property := y'M }) =
z + -↑ϕ { val := z, property := zM } • y'
[PROOFSTEP]
rw [LinearMap.map_sub, LinearMap.map_smul, sub_eq_add_neg, neg_smul]
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_1.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
z : O
zM : z ∈ M
⊢ ↑(Submodule.subtype M) { val := z, property := zM } +
-(↑ϕ { val := z, property := zM } • ↑(Submodule.subtype M) { val := y', property := y'M }) =
z + -(↑ϕ { val := z, property := zM } • y')
[PROOFSTEP]
rfl
-- It remains to show the extended bases are compatible with each other.
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
⊢ ∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as',
∀ (i : Fin (n' + 1)),
↑(↑(Basis.mkFinConsOfLE y yN bN' N'_le_N (_ : ∀ (c : R) (z : O), z ∈ N' → c • y + z = 0 → c = 0)
(_ : ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'))
i) =
as' i •
↑(↑(Basis.mkFinConsOfLE y' y'M bM' M'_le_M y'_ortho_M' (_ : ∀ (z : O), z ∈ M → ∃ c, z + c • y' ∈ M'))
(Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') i))
[PROOFSTEP]
intro as h
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
⊢ ∃ as',
∀ (i : Fin (n' + 1)),
↑(↑(Basis.mkFinConsOfLE y yN bN' N'_le_N (_ : ∀ (c : R) (z : O), z ∈ N' → c • y + z = 0 → c = 0)
(_ : ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'))
i) =
as' i •
↑(↑(Basis.mkFinConsOfLE y' y'M bM' M'_le_M y'_ortho_M' (_ : ∀ (z : O), z ∈ M → ∃ c, z + c • y' ∈ M'))
(Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') i))
[PROOFSTEP]
refine' ⟨Fin.cons a as, _⟩
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
⊢ ∀ (i : Fin (n' + 1)),
↑(↑(Basis.mkFinConsOfLE y yN bN' N'_le_N (_ : ∀ (c : R) (z : O), z ∈ N' → c • y + z = 0 → c = 0)
(_ : ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'))
i) =
Fin.cons a as i •
↑(↑(Basis.mkFinConsOfLE y' y'M bM' M'_le_M y'_ortho_M' (_ : ∀ (z : O), z ∈ M → ∃ c, z + c • y' ∈ M'))
(Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') i))
[PROOFSTEP]
intro i
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
i : Fin (n' + 1)
⊢ ↑(↑(Basis.mkFinConsOfLE y yN bN' N'_le_N (_ : ∀ (c : R) (z : O), z ∈ N' → c • y + z = 0 → c = 0)
(_ : ∀ (z : O), z ∈ N → ∃ c, z + c • y ∈ N'))
i) =
Fin.cons a as i •
↑(↑(Basis.mkFinConsOfLE y' y'M bM' M'_le_M y'_ortho_M' (_ : ∀ (z : O), z ∈ M → ∃ c, z + c • y' ∈ M'))
(Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') i))
[PROOFSTEP]
rw [Basis.coe_mkFinConsOfLE, Basis.coe_mkFinConsOfLE]
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
i : Fin (n' + 1)
⊢ ↑(Fin.cons { val := y, property := yN } (↑(ofLe N'_le_N) ∘ ↑bN') i) =
Fin.cons a as i •
↑(Fin.cons { val := y', property := y'M } (↑(ofLe M'_le_M) ∘ ↑bM') (Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') i))
[PROOFSTEP]
refine' Fin.cases _ (fun i ↦ _) i
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
i : Fin (n' + 1)
⊢ ↑(Fin.cons { val := y, property := yN } (↑(ofLe N'_le_N) ∘ ↑bN') 0) =
Fin.cons a as 0 •
↑(Fin.cons { val := y', property := y'M } (↑(ofLe M'_le_M) ∘ ↑bM') (Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') 0))
[PROOFSTEP]
simp only [Fin.cons_zero, Fin.castLE_zero]
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2.refine'_1
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
i : Fin (n' + 1)
⊢ y = generator (LinearMap.submoduleImage (Exists.choose this) N) • ∑ x : ι, ↑(c x • ↑b'M x)
[PROOFSTEP]
exact a_smul_y'.symm
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
i✝ : Fin (n' + 1)
i : Fin n'
⊢ ↑(Fin.cons { val := y, property := yN } (↑(ofLe N'_le_N) ∘ ↑bN') (Fin.succ i)) =
Fin.cons a as (Fin.succ i) •
↑(Fin.cons { val := y', property := y'M } (↑(ofLe M'_le_M) ∘ ↑bM')
(Fin.castLE (_ : Nat.succ n' ≤ Nat.succ m') (Fin.succ i)))
[PROOFSTEP]
rw [Fin.castLE_succ]
[GOAL]
case neg.intro.intro.intro.refine'_2.refine'_2.refine'_2
ι : Type u_1
R : Type u_2
inst✝⁷ : CommRing R
inst✝⁶ : IsDomain R
inst✝⁵ : IsPrincipalIdealRing R
M✝ : Type u_3
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
b : ι → M✝
inst✝² : Finite ι
O : Type u_4
inst✝¹ : AddCommGroup O
inst✝ : Module R O
M N : Submodule R O
b'M : Basis ι R { x // x ∈ M }
N_bot : N ≠ ⊥
N_le_M : N ≤ M
this : ∃ ϕ, ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage ϕ N < LinearMap.submoduleImage ψ N
ϕ : { x // x ∈ M } →ₗ[R] R := Exists.choose this
ϕ_max : ∀ (ψ : { x // x ∈ M } →ₗ[R] R), ¬LinearMap.submoduleImage (Exists.choose this) N < LinearMap.submoduleImage ψ N
a : R := generator (LinearMap.submoduleImage ϕ N)
a_mem : a ∈ LinearMap.submoduleImage ϕ N
a_zero : ¬a = 0
y : O
yN : y ∈ N
ϕy_eq : ↑ϕ { val := y, property := (_ : y ∈ M) } = a
_ϕy_ne_zero : ↑ϕ { val := y, property := (_ : y ∈ M) } ≠ 0
c : ι → R
hc : ∀ (i : ι), ↑(Basis.coord b'M i) { val := y, property := (_ : y ∈ M) } = a * c i
val✝ : Fintype ι
y' : O := ∑ i : ι, ↑(c i • ↑b'M i)
y'M : y' ∈ M
mk_y' : { val := y', property := y'M } = ∑ i : ι, c i • ↑b'M i
a_smul_y' : a • y' = y
ϕy'_eq : ↑ϕ { val := y', property := y'M } = 1
ϕy'_ne_zero : ↑ϕ { val := y', property := y'M } ≠ 0
M' : Submodule R O := map (Submodule.subtype M) (LinearMap.ker ϕ)
N' : Submodule R O := map (Submodule.subtype N) (LinearMap.ker (LinearMap.comp ϕ (ofLe N_le_M)))
M'_le_M : M' ≤ M
N'_le_M' : N' ≤ M'
N'_le_N : N' ≤ N
y'_ortho_M' : ∀ (c : R) (z : O), z ∈ M' → c • y' + z = 0 → c = 0
ay'_ortho_N' : ∀ (c : R) (z : O), z ∈ N' → c • a • y' + z = 0 → c = 0
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
as : Fin n' → R
h : ∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))
i✝ : Fin (n' + 1)
i : Fin n'
⊢ ↑(Fin.cons { val := y, property := yN } (↑(ofLe N'_le_N) ∘ ↑bN') (Fin.succ i)) =
Fin.cons a as (Fin.succ i) •
↑(Fin.cons { val := y', property := y'M } (↑(ofLe M'_le_M) ∘ ↑bM') (Fin.succ (Fin.castLE (_ : n' ≤ m') i)))
[PROOFSTEP]
simp only [Fin.cons_succ, Function.comp_apply, coe_ofLe, map_coe, coeSubtype, h i]
[GOAL]
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
[PROOFSTEP]
haveI := Classical.decEq M
[GOAL]
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
[PROOFSTEP]
induction' N using inductionOnRank with N ih
[GOAL]
case intro.b
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Basis ?m.114794 R M
[PROOFSTEP]
exact b
[GOAL]
case intro.ih
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
let b' := (b.reindex (Fintype.equivFin ι)).map (LinearEquiv.ofTop _ rfl).symm
[GOAL]
case intro.ih
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
by_cases N_bot : N = ⊥
[GOAL]
case pos
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
N_bot : N = ⊥
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
[PROOFSTEP]
subst N_bot
[GOAL]
case pos
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
ih :
∀ (N' : Submodule R M),
N' ≤ ⊥ →
∀ (x : M),
x ∈ ⊥ → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ ⊥ })
[PROOFSTEP]
exact ⟨0, ⟨Basis.empty _⟩⟩
[GOAL]
case neg
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
N_bot : ¬N = ⊥
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨y, -, a, hay, M', -, N', N'_le_N, -, -, ay_ortho, h'⟩ := Submodule.basis_of_pid_aux ⊤ N b' N_bot le_top
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
N_bot : ¬N = ⊥
y : M
a : R
hay : a • y ∈ N
M' N' : Submodule R M
N'_le_N : N' ≤ N
ay_ortho : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h' :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨n', ⟨bN'⟩⟩ := ih N' N'_le_N _ hay ay_ortho
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
N_bot : ¬N = ⊥
y : M
a : R
hay : a • y ∈ N
M' N' : Submodule R M
N'_le_N : N' ≤ N
ay_ortho : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h' :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨bN, _hbN⟩ := h' n' bN'
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
this : DecidableEq M
val✝ : Fintype ι
N : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ N →
∀ (x : M),
x ∈ N → (∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) → ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N' })
b' : Basis (Fin (Fintype.card ι)) R { x // x ∈ ⊤ } :=
Basis.map (Basis.reindex b (Fintype.equivFin ι)) (LinearEquiv.symm (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤)))
N_bot : ¬N = ⊥
y : M
a : R
hay : a • y ∈ N
M' N' : Submodule R M
N'_le_N : N' ≤ N
ay_ortho : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h' :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
n' : ℕ
bN' : Basis (Fin n') R { x // x ∈ N' }
bN : Basis (Fin (n' + 1)) R { x // x ∈ N }
_hbN :
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
⊢ ∃ n, Nonempty (Basis (Fin n) R { x // x ∈ N })
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
exact ⟨n' + 1, ⟨bN⟩⟩
[GOAL]
case intro.inst
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
this : DecidableEq M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
infer_instance
[GOAL]
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
⊢ basisOfPid b ⊥ = { fst := 0, snd := Basis.empty { x // x ∈ ⊥ } }
[PROOFSTEP]
obtain ⟨n, b'⟩ := Submodule.basisOfPid b ⊥
[GOAL]
case mk
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
n : ℕ
b' : Basis (Fin n) R { x // x ∈ ⊥ }
⊢ { fst := n, snd := b' } = { fst := 0, snd := Basis.empty { x // x ∈ ⊥ } }
[PROOFSTEP]
let e : Fin n ≃ Fin 0 := b'.indexEquiv (Basis.empty _ : Basis (Fin 0) R (⊥ : Submodule R M))
[GOAL]
case mk
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
n : ℕ
b' : Basis (Fin n) R { x // x ∈ ⊥ }
e : Fin n ≃ Fin 0 := Basis.indexEquiv b' (Basis.empty { x // x ∈ ⊥ })
⊢ { fst := n, snd := b' } = { fst := 0, snd := Basis.empty { x // x ∈ ⊥ } }
[PROOFSTEP]
obtain rfl : n = 0 := by simpa using Fintype.card_eq.mpr ⟨e⟩
[GOAL]
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
n : ℕ
b' : Basis (Fin n) R { x // x ∈ ⊥ }
e : Fin n ≃ Fin 0 := Basis.indexEquiv b' (Basis.empty { x // x ∈ ⊥ })
⊢ n = 0
[PROOFSTEP]
simpa using Fintype.card_eq.mpr ⟨e⟩
[GOAL]
case mk
ι✝ : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι✝ → M
ι : Type u_4
inst✝ : Finite ι
b : Basis ι R M
b' : Basis (Fin 0) R { x // x ∈ ⊥ }
e : Fin 0 ≃ Fin 0 := Basis.indexEquiv b' (Basis.empty { x // x ∈ ⊥ })
⊢ { fst := 0, snd := b' } = { fst := 0, snd := Basis.empty { x // x ∈ ⊥ } }
[PROOFSTEP]
exact Sigma.eq rfl (Basis.eq_of_apply_eq <| finZeroElim)
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
classical
-- We define `N` as the submodule spanned by a maximal linear independent subfamily of `s`
have := exists_maximal_independent R s
let I : Set ι := this.choose
obtain
⟨indepI : LinearIndependent R (s ∘ (fun x => x) : I → M), hI :
∀ (i) (_ : i ∉ I), ∃ a : R, a ≠ 0 ∧ a • s i ∈ span R (s '' I)⟩ :=
this.choose_spec
let N :=
span R
(range <| (s ∘ (fun x => x) : I → M))
-- same as `span R (s '' I)` but more convenient
let _sI : I → N := fun i ↦
⟨s i.1, subset_span (mem_range_self i)⟩
-- `s` restricted to `I` is a basis of `N`
let sI_basis : Basis I R N := Basis.span indepI
have exists_a : ∀ i : ι, ∃ a : R, a ≠ 0 ∧ a • s i ∈ N :=
by
intro i
by_cases hi : i ∈ I
· use 1, zero_ne_one.symm
rw [one_smul]
exact subset_span (mem_range_self (⟨i, hi⟩ : I))
· simpa [image_eq_range s I] using hI i hi
choose a ha ha' using exists_a
let A := ∏ i, a i
have hA : A ≠ 0 := by
rw [Finset.prod_ne_zero_iff]
simpa using ha
let φ : M →ₗ[R] M := LinearMap.lsmul R M A
have : LinearMap.ker φ = ⊥ := @LinearMap.ker_lsmul R M _ _ _ _ _ hA
let ψ := LinearEquiv.ofInjective φ (LinearMap.ker_eq_bot.mp this)
have : LinearMap.range φ ≤ N := by
-- as announced, `A • M ⊆ N`
suffices ∀ i, φ (s i) ∈ N by
rw [LinearMap.range_eq_map, ← hs, map_span_le]
rintro _ ⟨i, rfl⟩
apply this
intro i
calc
(∏ j, a j) • s i = (∏ j in { i }ᶜ, a j) • a i • s i := by rw [Fintype.prod_eq_prod_compl_mul i, mul_smul]
_ ∈ N :=
N.smul_mem _
(ha' i)
-- Since a submodule of a free `R`-module is free, we get that `A • M` is free
obtain ⟨n, b : Basis (Fin n) R (LinearMap.range φ)⟩ := Submodule.basisOfPidOfLE this sI_basis
exact ⟨n, b.map ψ.symm⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
have := exists_maximal_independent R s
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let I : Set ι := this.choose
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
obtain
⟨indepI : LinearIndependent R (s ∘ (fun x => x) : I → M), hI :
∀ (i) (_ : i ∉ I), ∃ a : R, a ≠ 0 ∧ a • s i ∈ span R (s '' I)⟩ :=
this.choose_spec
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let N :=
span R
(range <| (s ∘ (fun x => x) : I → M))
-- same as `span R (s '' I)` but more convenient
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let _sI : I → N := fun i ↦
⟨s i.1, subset_span (mem_range_self i)⟩
-- `s` restricted to `I` is a basis of `N`
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let sI_basis : Basis I R N := Basis.span indepI
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
have exists_a : ∀ i : ι, ∃ a : R, a ≠ 0 ∧ a • s i ∈ N :=
by
intro i
by_cases hi : i ∈ I
· use 1, zero_ne_one.symm
rw [one_smul]
exact subset_span (mem_range_self (⟨i, hi⟩ : I))
· simpa [image_eq_range s I] using hI i hi
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
⊢ ∀ (i : ι), ∃ a, a ≠ 0 ∧ a • s i ∈ N
[PROOFSTEP]
intro i
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
i : ι
⊢ ∃ a, a ≠ 0 ∧ a • s i ∈ N
[PROOFSTEP]
by_cases hi : i ∈ I
[GOAL]
case pos
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
i : ι
hi : i ∈ I
⊢ ∃ a, a ≠ 0 ∧ a • s i ∈ N
[PROOFSTEP]
use 1, zero_ne_one.symm
[GOAL]
case right
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
i : ι
hi : i ∈ I
⊢ 1 • s i ∈ N
[PROOFSTEP]
rw [one_smul]
[GOAL]
case right
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
i : ι
hi : i ∈ I
⊢ s i ∈ N
[PROOFSTEP]
exact subset_span (mem_range_self (⟨i, hi⟩ : I))
[GOAL]
case neg
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
i : ι
hi : ¬i ∈ I
⊢ ∃ a, a ≠ 0 ∧ a • s i ∈ N
[PROOFSTEP]
simpa [image_eq_range s I] using hI i hi
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
exists_a : ∀ (i : ι), ∃ a, a ≠ 0 ∧ a • s i ∈ N
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
choose a ha ha' using exists_a
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let A := ∏ i, a i
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
have hA : A ≠ 0 := by
rw [Finset.prod_ne_zero_iff]
simpa using ha
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
⊢ A ≠ 0
[PROOFSTEP]
rw [Finset.prod_ne_zero_iff]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
⊢ ∀ (a_1 : ι), a_1 ∈ Finset.univ → a a_1 ≠ 0
[PROOFSTEP]
simpa using ha
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let φ : M →ₗ[R] M := LinearMap.lsmul R M A
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
have : LinearMap.ker φ = ⊥ := @LinearMap.ker_lsmul R M _ _ _ _ _ hA
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this : LinearMap.ker φ = ⊥
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
let ψ := LinearEquiv.ofInjective φ (LinearMap.ker_eq_bot.mp this)
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
have : LinearMap.range φ ≤ N := by
-- as announced, `A • M ⊆ N`
suffices ∀ i, φ (s i) ∈ N by
rw [LinearMap.range_eq_map, ← hs, map_span_le]
rintro _ ⟨i, rfl⟩
apply this
intro i
calc
(∏ j, a j) • s i = (∏ j in { i }ᶜ, a j) • a i • s i := by rw [Fintype.prod_eq_prod_compl_mul i, mul_smul]
_ ∈ N :=
N.smul_mem _
(ha' i)
-- Since a submodule of a free `R`-module is free, we get that `A • M` is free
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
⊢ LinearMap.range φ ≤ N
[PROOFSTEP]
suffices ∀ i, φ (s i) ∈ N by
rw [LinearMap.range_eq_map, ← hs, map_span_le]
rintro _ ⟨i, rfl⟩
apply this
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝¹ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝¹
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this✝ : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
this : ∀ (i : ι), ↑φ (s i) ∈ N
⊢ LinearMap.range φ ≤ N
[PROOFSTEP]
rw [LinearMap.range_eq_map, ← hs, map_span_le]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝¹ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝¹
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this✝ : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
this : ∀ (i : ι), ↑φ (s i) ∈ N
⊢ ∀ (m : M), m ∈ range s → ↑φ m ∈ N
[PROOFSTEP]
rintro _ ⟨i, rfl⟩
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝¹ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝¹
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this✝ : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
this : ∀ (i : ι), ↑φ (s i) ∈ N
i : ι
⊢ ↑φ (s i) ∈ N
[PROOFSTEP]
apply this
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
⊢ ∀ (i : ι), ↑φ (s i) ∈ N
[PROOFSTEP]
intro i
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
i : ι
⊢ ↑φ (s i) ∈ N
[PROOFSTEP]
calc
(∏ j, a j) • s i = (∏ j in { i }ᶜ, a j) • a i • s i := by rw [Fintype.prod_eq_prod_compl_mul i, mul_smul]
_ ∈ N :=
N.smul_mem _
(ha' i)
-- Since a submodule of a free `R`-module is free, we get that `A • M` is free
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
i : ι
⊢ (∏ j : ι, a j) • s i = (∏ j in {i}ᶜ, a j) • a i • s i
[PROOFSTEP]
rw [Fintype.prod_eq_prod_compl_mul i, mul_smul]
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝¹ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝¹
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this✝ : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
this : LinearMap.range φ ≤ N
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
obtain ⟨n, b : Basis (Fin n) R (LinearMap.range φ)⟩ := Submodule.basisOfPidOfLE this sI_basis
[GOAL]
case intro.mk
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b✝ : ι → M
inst✝¹ : Fintype ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
this✝¹ : ∃ I, (LinearIndependent R fun x => s ↑x) ∧ ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
I : Set ι := Exists.choose this✝¹
indepI : LinearIndependent R (s ∘ fun x => ↑x)
hI : ∀ (i : ι), ¬i ∈ I → ∃ a, a ≠ 0 ∧ a • s i ∈ span R (s '' I)
N : Submodule R M := span R (range (s ∘ fun x => ↑x))
_sI : ↑I → { x // x ∈ N } := fun i => { val := s ↑i, property := (_ : s ↑i ∈ ↑(span R (range (s ∘ fun x => ↑x)))) }
sI_basis : Basis (↑I) R { x // x ∈ N } := Basis.span indepI
a : ι → R
ha : ∀ (i : ι), a i ≠ 0
ha' : ∀ (i : ι), a i • s i ∈ N
A : R := ∏ i : ι, a i
hA : A ≠ 0
φ : M →ₗ[R] M := ↑(LinearMap.lsmul R M) A
this✝ : LinearMap.ker φ = ⊥
ψ : M ≃ₗ[R] { x // x ∈ LinearMap.range φ } := LinearEquiv.ofInjective φ (_ : Function.Injective ↑φ)
this : LinearMap.range φ ≤ N
n : ℕ
b : Basis (Fin n) R { x // x ∈ LinearMap.range φ }
⊢ (n : ℕ) × Basis (Fin n) R M
[PROOFSTEP]
exact ⟨n, b.map ψ.symm⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : _root_.Finite ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
⊢ Free R M
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : _root_.Finite ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
val✝ : Fintype ι
⊢ Free R M
[PROOFSTEP]
obtain ⟨n, b⟩ : Σ n, Basis (Fin n) R M := Module.basisOfFiniteTypeTorsionFree hs
[GOAL]
case intro.mk
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b✝ : ι → M
inst✝¹ : _root_.Finite ι
s : ι → M
hs : span R (range s) = ⊤
inst✝ : NoZeroSMulDivisors R M
val✝ : Fintype ι
n : ℕ
b : Basis (Fin n) R M
⊢ Free R M
[PROOFSTEP]
exact Module.Free.of_basis b
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b : ι → M
inst✝¹ : Finite R M
inst✝ : NoZeroSMulDivisors R M
⊢ Free R M
[PROOFSTEP]
obtain ⟨n, b⟩ : Σ n, Basis (Fin n) R M := Module.basisOfFiniteTypeTorsionFree'
[GOAL]
case mk
ι : Type u_1
R : Type u_2
inst✝⁶ : CommRing R
inst✝⁵ : IsDomain R
inst✝⁴ : IsPrincipalIdealRing R
M : Type u_3
inst✝³ : AddCommGroup M
inst✝² : Module R M
b✝ : ι → M
inst✝¹ : Finite R M
inst✝ : NoZeroSMulDivisors R M
n : ℕ
b : Basis (Fin n) R M
⊢ Free R M
[PROOFSTEP]
exact Module.Free.of_basis b
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N O : Submodule R M
N_le_O : N ≤ O
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N O : Submodule R M
N_le_O : N ≤ O
val✝ : Fintype ι
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
[PROOFSTEP]
revert N
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ ∀ (N : Submodule R M), N ≤ O → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
[PROOFSTEP]
induction' O using inductionOnRank with M0 ih
[GOAL]
case intro.b
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Basis ?m.235193 R M
[PROOFSTEP]
exact b
[GOAL]
case intro.ih
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
⊢ ∀ (N : Submodule R M), N ≤ M0 → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
intro N N_le_M0
[GOAL]
case intro.ih
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨m, b'M⟩ := M0.basisOfPid b
[GOAL]
case intro.ih.mk
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
by_cases N_bot : N = ⊥
[GOAL]
case pos
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : N = ⊥
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
[PROOFSTEP]
subst N_bot
[GOAL]
case pos
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_le_M0 : ⊥ ≤ M0
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
[PROOFSTEP]
exact ⟨0, m, Nat.zero_le _, b'M, Basis.empty _, finZeroElim, finZeroElim⟩
[GOAL]
case neg
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : ¬N = ⊥
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨y, hy, a, _, M', M'_le_M, N', _, N'_le_M', y_ortho, _, h⟩ := Submodule.basis_of_pid_aux M0 N b'M N_bot N_le_M0
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : ¬N = ⊥
y : M
hy : y ∈ M0
a : R
w✝¹ : a • y ∈ N
M' : Submodule R M
M'_le_M : M' ≤ M0
N' : Submodule R M
left✝ : N' ≤ N
N'_le_M' : N' ≤ M'
y_ortho : ∀ (c : R) (z : M), z ∈ M' → c • y + z = 0 → c = 0
w✝ : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨n', m', hn'm', bM', bN', as', has'⟩ := ih M' M'_le_M y hy y_ortho N' N'_le_M'
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : ¬N = ⊥
y : M
hy : y ∈ M0
a : R
w✝¹ : a • y ∈ N
M' : Submodule R M
M'_le_M : M' ≤ M0
N' : Submodule R M
left✝ : N' ≤ N
N'_le_M' : N' ≤ M'
y_ortho : ∀ (c : R) (z : M), z ∈ M' → c • y + z = 0 → c = 0
w✝ : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
n' m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
bN' : Basis (Fin n') R { x // x ∈ N' }
as' : Fin n' → R
has' : ∀ (i : Fin n'), ↑(↑bN' i) = ↑(as' i • ↑bM' (Fin.castLE hn'm' i))
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨bN, h'⟩ := h n' bN'
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : ¬N = ⊥
y : M
hy : y ∈ M0
a : R
w✝¹ : a • y ∈ N
M' : Submodule R M
M'_le_M : M' ≤ M0
N' : Submodule R M
left✝ : N' ≤ N
N'_le_M' : N' ≤ M'
y_ortho : ∀ (c : R) (z : M), z ∈ M' → c • y + z = 0 → c = 0
w✝ : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
n' m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
bN' : Basis (Fin n') R { x // x ∈ N' }
as' : Fin n' → R
has' : ∀ (i : Fin n'), ↑(↑bN' i) = ↑(as' i • ↑bM' (Fin.castLE hn'm' i))
bN : Basis (Fin (n' + 1)) R { x // x ∈ N }
h' :
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨hmn, bM, h''⟩ := h' m' hn'm' bM'
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : ¬N = ⊥
y : M
hy : y ∈ M0
a : R
w✝¹ : a • y ∈ N
M' : Submodule R M
M'_le_M : M' ≤ M0
N' : Submodule R M
left✝ : N' ≤ N
N'_le_M' : N' ≤ M'
y_ortho : ∀ (c : R) (z : M), z ∈ M' → c • y + z = 0 → c = 0
w✝ : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
n' m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
bN' : Basis (Fin n') R { x // x ∈ N' }
as' : Fin n' → R
has' : ∀ (i : Fin n'), ↑(↑bN' i) = ↑(as' i • ↑bM' (Fin.castLE hn'm' i))
bN : Basis (Fin (n' + 1)) R { x // x ∈ N }
h' :
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
hmn : n' + 1 ≤ m' + 1
bM : Basis (Fin (m' + 1)) R { x // x ∈ M0 }
h'' :
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hmn i))
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
obtain ⟨as, has⟩ := h'' as' has'
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
val✝ : Fintype ι
M0 : Submodule R M
ih :
∀ (N' : Submodule R M),
N' ≤ M0 →
∀ (x : M),
x ∈ M0 →
(∀ (c : R) (y : M), y ∈ N' → c • x + y = 0 → c = 0) →
∀ (N : Submodule R M), N ≤ N' → ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
N : Submodule R M
N_le_M0 : N ≤ M0
m : ℕ
b'M : Basis (Fin m) R { x // x ∈ M0 }
N_bot : ¬N = ⊥
y : M
hy : y ∈ M0
a : R
w✝¹ : a • y ∈ N
M' : Submodule R M
M'_le_M : M' ≤ M0
N' : Submodule R M
left✝ : N' ≤ N
N'_le_M' : N' ≤ M'
y_ortho : ∀ (c : R) (z : M), z ∈ M' → c • y + z = 0 → c = 0
w✝ : ∀ (c : R) (z : M), z ∈ N' → c • a • y + z = 0 → c = 0
h :
∀ (n' : ℕ) (bN' : Basis (Fin n') R { x // x ∈ N' }),
∃ bN,
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
n' m' : ℕ
hn'm' : n' ≤ m'
bM' : Basis (Fin m') R { x // x ∈ M' }
bN' : Basis (Fin n') R { x // x ∈ N' }
as' : Fin n' → R
has' : ∀ (i : Fin n'), ↑(↑bN' i) = ↑(as' i • ↑bM' (Fin.castLE hn'm' i))
bN : Basis (Fin (n' + 1)) R { x // x ∈ N }
h' :
∀ (m' : ℕ) (hn'm' : n' ≤ m') (bM' : Basis (Fin m') R { x // x ∈ M' }),
∃ hnm bM,
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hnm i))
hmn : n' + 1 ≤ m' + 1
bM : Basis (Fin (m' + 1)) R { x // x ∈ M0 }
h'' :
∀ (as : Fin n' → R),
(∀ (i : Fin n'), ↑(↑bN' i) = as i • ↑(↑bM' (Fin.castLE hn'm' i))) →
∃ as', ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as' i • ↑(↑bM (Fin.castLE hmn i))
as : Fin (n' + 1) → R
has : ∀ (i : Fin (n' + 1)), ↑(↑bN i) = as i • ↑(↑bM (Fin.castLE hmn i))
⊢ ∃ n o hno bO bN a, ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
exact
⟨_, _, hmn, bM, bN, as, has⟩
-- Porting note: Lean generates a goal Fintype ι for some reason
[GOAL]
case intro.inst
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
O : Submodule R M
val✝ : Fintype ι
⊢ Fintype ι
[PROOFSTEP]
infer_instance
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N O : Submodule R M
N_le_O : N ≤ O
⊢ (o : ℕ) × (n : ℕ) × Basis.SmithNormalForm (comap (Submodule.subtype O) N) (Fin o) n
[PROOFSTEP]
choose n o hno bO bN a snf using N.exists_smith_normal_form_of_le b O N_le_O
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N O : Submodule R M
N_le_O : N ≤ O
n o : ℕ
hno : n ≤ o
bO : Basis (Fin o) R { x // x ∈ O }
bN : Basis (Fin n) R { x // x ∈ N }
a : Fin n → R
snf : ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
⊢ (o : ℕ) × (n : ℕ) × Basis.SmithNormalForm (comap (Submodule.subtype O) N) (Fin o) n
[PROOFSTEP]
refine' ⟨o, n, bO, bN.map (comapSubtypeEquivOfLe N_le_O).symm, (Fin.castLEEmb hno).toEmbedding, a, fun i ↦ _⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N O : Submodule R M
N_le_O : N ≤ O
n o : ℕ
hno : n ≤ o
bO : Basis (Fin o) R { x // x ∈ O }
bN : Basis (Fin n) R { x // x ∈ N }
a : Fin n → R
snf : ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
i : Fin n
⊢ ↑(↑(Basis.map bN (LinearEquiv.symm (comapSubtypeEquivOfLe N_le_O))) i) =
a i • ↑bO (↑(Fin.castLEEmb hno).toEmbedding i)
[PROOFSTEP]
ext
[GOAL]
case a
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N O : Submodule R M
N_le_O : N ≤ O
n o : ℕ
hno : n ≤ o
bO : Basis (Fin o) R { x // x ∈ O }
bN : Basis (Fin n) R { x // x ∈ N }
a : Fin n → R
snf : ∀ (i : Fin n), ↑(↑bN i) = ↑(a i • ↑bO (Fin.castLE hno i))
i : Fin n
⊢ ↑↑(↑(Basis.map bN (LinearEquiv.symm (comapSubtypeEquivOfLe N_le_O))) i) =
↑(a i • ↑bO (↑(Fin.castLEEmb hno).toEmbedding i))
[PROOFSTEP]
simp only [snf, Basis.map_apply, Submodule.comapSubtypeEquivOfLe_symm_apply, Submodule.coe_smul_of_tower,
RelEmbedding.coe_toEmbedding, Fin.castLEEmb_apply]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁵ : CommRing R
inst✝⁴ : IsDomain R
inst✝³ : IsPrincipalIdealRing R
M : Type u_3
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b✝ : ι → M
inst✝ : Finite ι
b : Basis ι R M
N : Submodule R M
m n : ℕ
bM : Basis (Fin m) R { x // x ∈ ⊤ }
bN : Basis (Fin n) R { x // x ∈ comap (Submodule.subtype ⊤) N }
f : Fin n ↪ Fin m
a : Fin n → R
snf : ∀ (i : Fin n), ↑(↑bN i) = a i • ↑bM (↑f i)
bM' : Basis (Fin m) R M := Basis.map bM (LinearEquiv.ofTop ⊤ (_ : ⊤ = ⊤))
e : Fin m ≃ ι := Basis.indexEquiv bM' b
i : Fin n
⊢ ↑(↑(Basis.map bN (comapSubtypeEquivOfLe (_ : N ≤ ⊤))) i) =
a i • ↑(Basis.reindex bM' e) (↑(Function.Embedding.trans f (Equiv.toEmbedding e)) i)
[PROOFSTEP]
simp only [snf, Basis.map_apply, LinearEquiv.ofTop_apply, Submodule.coe_smul_of_tower,
Submodule.comapSubtypeEquivOfLe_apply_coe, Basis.reindex_apply, Equiv.toEmbedding_apply,
Function.Embedding.trans_apply, Equiv.symm_apply_apply]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Fintype ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
n : ℕ
bS : Basis ι R S
bI : Basis (Fin n) R { x // x ∈ restrictScalars R I }
f : Fin n ↪ ι
a : Fin n → R
snf : ∀ (i : Fin n), ↑(↑bI i) = a i • ↑bS (↑f i)
eq : Fintype.card (Fin n) = Fintype.card ι
⊢ Fintype.card (Fin n) = Fintype.card (Fin (Fintype.card ι))
[PROOFSTEP]
rw [eq, Fintype.card_fin]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Fintype ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
n : ℕ
bS : Basis ι R S
bI : Basis (Fin n) R { x // x ∈ restrictScalars R I }
f : Fin n ↪ ι
a : Fin n → R
snf : ∀ (i : Fin n), ↑(↑bI i) = a i • ↑bS (↑f i)
eq : Fintype.card (Fin n) = Fintype.card ι
e : Fin n ≃ Fin (Fintype.card ι) :=
Fintype.equivOfCardEq (_ : Fintype.card (Fin n) = Fintype.card (Fin (Fintype.card ι)))
i : Fin (Fintype.card ι)
⊢ ↑(↑(Basis.reindex bI e) i) = (a ∘ ↑e.symm) i • ↑bS (↑(Function.Embedding.trans (Equiv.toEmbedding e.symm) f) i)
[PROOFSTEP]
simp only [snf, Basis.coe_reindex, Function.Embedding.trans_apply, Equiv.toEmbedding_apply, (· ∘ ·)]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
⊢ ∃ b' a ab', ∀ (i : ι), ↑(↑ab' i) = a i • ↑b' i
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
val✝ : Fintype ι
⊢ ∃ b' a ab', ∀ (i : ι), ↑(↑ab' i) = a i • ↑b' i
[PROOFSTEP]
let ⟨bS, bI, f, a, snf⟩ := I.smithNormalForm b hI
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
val✝ : Fintype ι
bS : Basis ι R S
bI : Basis (Fin (Fintype.card ι)) R { x // x ∈ restrictScalars R I }
f : Fin (Fintype.card ι) ↪ ι
a : Fin (Fintype.card ι) → R
snf : ∀ (i : Fin (Fintype.card ι)), ↑(↑bI i) = a i • ↑bS (↑f i)
⊢ ∃ b' a ab', ∀ (i : ι), ↑(↑ab' i) = a i • ↑b' i
[PROOFSTEP]
let e : Fin (Fintype.card ι) ≃ ι :=
Equiv.ofBijective f ((Fintype.bijective_iff_injective_and_card f).mpr ⟨f.injective, Fintype.card_fin _⟩)
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
val✝ : Fintype ι
bS : Basis ι R S
bI : Basis (Fin (Fintype.card ι)) R { x // x ∈ restrictScalars R I }
f : Fin (Fintype.card ι) ↪ ι
a : Fin (Fintype.card ι) → R
snf : ∀ (i : Fin (Fintype.card ι)), ↑(↑bI i) = a i • ↑bS (↑f i)
e : Fin (Fintype.card ι) ≃ ι := Equiv.ofBijective ↑f (_ : Function.Bijective ↑f)
⊢ ∃ b' a ab', ∀ (i : ι), ↑(↑ab' i) = a i • ↑b' i
[PROOFSTEP]
have fe : ∀ i, f (e.symm i) = i := e.apply_symm_apply
[GOAL]
case intro
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
val✝ : Fintype ι
bS : Basis ι R S
bI : Basis (Fin (Fintype.card ι)) R { x // x ∈ restrictScalars R I }
f : Fin (Fintype.card ι) ↪ ι
a : Fin (Fintype.card ι) → R
snf : ∀ (i : Fin (Fintype.card ι)), ↑(↑bI i) = a i • ↑bS (↑f i)
e : Fin (Fintype.card ι) ≃ ι := Equiv.ofBijective ↑f (_ : Function.Bijective ↑f)
fe : ∀ (i : ι), ↑f (↑e.symm i) = i
⊢ ∃ b' a ab', ∀ (i : ι), ↑(↑ab' i) = a i • ↑b' i
[PROOFSTEP]
exact
⟨bS, a ∘ e.symm, (bI.reindex e).map ((restrictScalarsEquiv R S _ _).restrictScalars R), fun i ↦ by
simp only [snf, fe, Basis.map_apply, LinearEquiv.restrictScalars_apply R, Submodule.restrictScalarsEquiv_apply,
Basis.coe_reindex, (· ∘ ·)]⟩
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
val✝ : Fintype ι
bS : Basis ι R S
bI : Basis (Fin (Fintype.card ι)) R { x // x ∈ restrictScalars R I }
f : Fin (Fintype.card ι) ↪ ι
a : Fin (Fintype.card ι) → R
snf : ∀ (i : Fin (Fintype.card ι)), ↑(↑bI i) = a i • ↑bS (↑f i)
e : Fin (Fintype.card ι) ≃ ι := Equiv.ofBijective ↑f (_ : Function.Bijective ↑f)
fe : ∀ (i : ι), ↑f (↑e.symm i) = i
i : ι
⊢ ↑(↑(Basis.map (Basis.reindex bI e) (LinearEquiv.restrictScalars R (restrictScalarsEquiv R S S I))) i) =
(a ∘ ↑e.symm) i • ↑bS i
[PROOFSTEP]
simp only [snf, fe, Basis.map_apply, LinearEquiv.restrictScalars_apply R, Submodule.restrictScalarsEquiv_apply,
Basis.coe_reindex, (· ∘ ·)]
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
i : ι
⊢ smithCoeffs b I hI i ≠ 0
[PROOFSTEP]
intro hi
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
i : ι
hi : smithCoeffs b I hI i = 0
⊢ False
[PROOFSTEP]
apply Basis.ne_zero (Ideal.selfBasis b I hI) i
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
i : ι
hi : smithCoeffs b I hI i = 0
⊢ ↑(selfBasis b I hI) i = 0
[PROOFSTEP]
refine' Subtype.coe_injective _
[GOAL]
ι : Type u_1
R : Type u_2
inst✝⁸ : CommRing R
inst✝⁷ : IsDomain R
inst✝⁶ : IsPrincipalIdealRing R
M : Type u_3
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
b✝ : ι → M
S : Type u_4
inst✝³ : CommRing S
inst✝² : IsDomain S
inst✝¹ : Algebra R S
inst✝ : Finite ι
b : Basis ι R S
I : Ideal S
hI : I ≠ ⊥
i : ι
hi : smithCoeffs b I hI i = 0
⊢ (fun a => ↑a) (↑(selfBasis b I hI) i) = (fun a => ↑a) 0
[PROOFSTEP]
simp [hi]
[GOAL]
R : Type u_1
S : Type u_2
M : Type u_3
ι : Type u_4
inst✝⁶ : CommSemiring R
inst✝⁵ : Semiring S
inst✝⁴ : AddCommMonoid M
inst✝³ : Algebra R S
inst✝² : Module R M
inst✝¹ : Module S M
inst✝ : IsScalarTower R S M
hinj : Function.Injective ↑(algebraMap R S)
v : ι → M
li : LinearIndependent S v
⊢ Function.Injective fun r => r • 1
[PROOFSTEP]
rwa [Algebra.algebraMap_eq_smul_one'] at hinj
| {"mathlib_filename": "Mathlib.LinearAlgebra.FreeModule.PID", "llama_tokens": 126757} |
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
⊢ vectorSpan k ∅ = ⊥
[PROOFSTEP]
rw [vectorSpan_def, vsub_empty, Submodule.span_empty]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
⊢ vectorSpan k {p} = ⊥
[PROOFSTEP]
simp [vectorSpan_def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ Set.Nonempty (spanPoints k s) ↔ Set.Nonempty s
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ Set.Nonempty (spanPoints k s) → Set.Nonempty s
[PROOFSTEP]
contrapose
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ ¬Set.Nonempty s → ¬Set.Nonempty (spanPoints k s)
[PROOFSTEP]
rw [Set.not_nonempty_iff_eq_empty, Set.not_nonempty_iff_eq_empty]
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ s = ∅ → spanPoints k s = ∅
[PROOFSTEP]
intro h
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
h : s = ∅
⊢ spanPoints k s = ∅
[PROOFSTEP]
simp [h, spanPoints]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ Set.Nonempty s → Set.Nonempty (spanPoints k s)
[PROOFSTEP]
exact fun h => h.mono (subset_spanPoints _ _)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p : P
v : V
hp : p ∈ spanPoints k s
hv : v ∈ vectorSpan k s
⊢ v +ᵥ p ∈ spanPoints k s
[PROOFSTEP]
rcases hp with ⟨p2, ⟨hp2, ⟨v2, ⟨hv2, hv2p⟩⟩⟩⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p : P
v : V
hv : v ∈ vectorSpan k s
p2 : P
hp2 : p2 ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p = v2 +ᵥ p2
⊢ v +ᵥ p ∈ spanPoints k s
[PROOFSTEP]
rw [hv2p, vadd_vadd]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p : P
v : V
hv : v ∈ vectorSpan k s
p2 : P
hp2 : p2 ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p = v2 +ᵥ p2
⊢ v + v2 +ᵥ p2 ∈ spanPoints k s
[PROOFSTEP]
exact ⟨p2, hp2, v + v2, (vectorSpan k s).add_mem hv hv2, rfl⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 : P
hp1 : p1 ∈ spanPoints k s
hp2 : p2 ∈ spanPoints k s
⊢ p1 -ᵥ p2 ∈ vectorSpan k s
[PROOFSTEP]
rcases hp1 with ⟨p1a, ⟨hp1a, ⟨v1, ⟨hv1, hv1p⟩⟩⟩⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 : P
hp2 : p2 ∈ spanPoints k s
p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
⊢ p1 -ᵥ p2 ∈ vectorSpan k s
[PROOFSTEP]
rcases hp2 with ⟨p2a, ⟨hp2a, ⟨v2, ⟨hv2, hv2p⟩⟩⟩⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
⊢ p1 -ᵥ p2 ∈ vectorSpan k s
[PROOFSTEP]
rw [hv1p, hv2p, vsub_vadd_eq_vsub_sub (v1 +ᵥ p1a), vadd_vsub_assoc, add_comm, add_sub_assoc]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
⊢ p1a -ᵥ p2a + (v1 - v2) ∈ vectorSpan k s
[PROOFSTEP]
have hv1v2 : v1 - v2 ∈ vectorSpan k s := by
rw [sub_eq_add_neg]
apply (vectorSpan k s).add_mem hv1
rw [← neg_one_smul k v2]
exact (vectorSpan k s).smul_mem (-1 : k) hv2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
⊢ v1 - v2 ∈ vectorSpan k s
[PROOFSTEP]
rw [sub_eq_add_neg]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
⊢ v1 + -v2 ∈ vectorSpan k s
[PROOFSTEP]
apply (vectorSpan k s).add_mem hv1
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
⊢ -v2 ∈ vectorSpan k s
[PROOFSTEP]
rw [← neg_one_smul k v2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
⊢ -1 • v2 ∈ vectorSpan k s
[PROOFSTEP]
exact (vectorSpan k s).smul_mem (-1 : k) hv2
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
hv1v2 : v1 - v2 ∈ vectorSpan k s
⊢ p1a -ᵥ p2a + (v1 - v2) ∈ vectorSpan k s
[PROOFSTEP]
refine' (vectorSpan k s).add_mem _ hv1v2
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p2 p1a : P
hp1a : p1a ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hv1p : p1 = v1 +ᵥ p1a
p2a : P
hp2a : p2a ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hv2p : p2 = v2 +ᵥ p2a
hv1v2 : v1 - v2 ∈ vectorSpan k s
⊢ p1a -ᵥ p2a ∈ vectorSpan k s
[PROOFSTEP]
exact vsub_mem_vectorSpan k hp1a hp2a
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p q : AffineSubspace k P
x✝ : p.carrier = q.carrier
⊢ p = q
[PROOFSTEP]
cases p
[GOAL]
case mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
q : AffineSubspace k P
carrier✝ : Set P
smul_vsub_vadd_mem✝ :
∀ (c : k) {p1 p2 p3 : P}, p1 ∈ carrier✝ → p2 ∈ carrier✝ → p3 ∈ carrier✝ → c • (p1 -ᵥ p2) +ᵥ p3 ∈ carrier✝
x✝ : { carrier := carrier✝, smul_vsub_vadd_mem := smul_vsub_vadd_mem✝ }.carrier = q.carrier
⊢ { carrier := carrier✝, smul_vsub_vadd_mem := smul_vsub_vadd_mem✝ } = q
[PROOFSTEP]
cases q
[GOAL]
case mk.mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
carrier✝¹ : Set P
smul_vsub_vadd_mem✝¹ :
∀ (c : k) {p1 p2 p3 : P}, p1 ∈ carrier✝¹ → p2 ∈ carrier✝¹ → p3 ∈ carrier✝¹ → c • (p1 -ᵥ p2) +ᵥ p3 ∈ carrier✝¹
carrier✝ : Set P
smul_vsub_vadd_mem✝ :
∀ (c : k) {p1 p2 p3 : P}, p1 ∈ carrier✝ → p2 ∈ carrier✝ → p3 ∈ carrier✝ → c • (p1 -ᵥ p2) +ᵥ p3 ∈ carrier✝
x✝ :
{ carrier := carrier✝¹, smul_vsub_vadd_mem := smul_vsub_vadd_mem✝¹ }.carrier =
{ carrier := carrier✝, smul_vsub_vadd_mem := smul_vsub_vadd_mem✝ }.carrier
⊢ { carrier := carrier✝¹, smul_vsub_vadd_mem := smul_vsub_vadd_mem✝¹ } =
{ carrier := carrier✝, smul_vsub_vadd_mem := smul_vsub_vadd_mem✝ }
[PROOFSTEP]
congr
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s
[PROOFSTEP]
intro a b ha hb
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
a b : V
ha : a ∈ ↑s -ᵥ ↑s
hb : b ∈ ↑s -ᵥ ↑s
⊢ a + b ∈ ↑s -ᵥ ↑s
[PROOFSTEP]
rcases ha with ⟨p1, p2, hp1, hp2, rfl⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
b : V
hb : b ∈ ↑s -ᵥ ↑s
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
⊢ (fun x x_1 => x -ᵥ x_1) p1 p2 + b ∈ ↑s -ᵥ ↑s
[PROOFSTEP]
rcases hb with ⟨p3, p4, hp3, hp4, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
p3 p4 : P
hp3 : p3 ∈ ↑s
hp4 : p4 ∈ ↑s
⊢ (fun x x_1 => x -ᵥ x_1) p1 p2 + (fun x x_1 => x -ᵥ x_1) p3 p4 ∈ ↑s -ᵥ ↑s
[PROOFSTEP]
rw [← vadd_vsub_assoc]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
p3 p4 : P
hp3 : p3 ∈ ↑s
hp4 : p4 ∈ ↑s
⊢ (fun x x_1 => x -ᵥ x_1) p1 p2 +ᵥ p3 -ᵥ p4 ∈ ↑s -ᵥ ↑s
[PROOFSTEP]
refine' vsub_mem_vsub _ hp4
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
p3 p4 : P
hp3 : p3 ∈ ↑s
hp4 : p4 ∈ ↑s
⊢ (fun x x_1 => x -ᵥ x_1) p1 p2 +ᵥ p3 ∈ ↑s
[PROOFSTEP]
convert s.smul_vsub_vadd_mem 1 hp1 hp2 hp3
[GOAL]
case h.e'_4.h.e'_5
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
p3 p4 : P
hp3 : p3 ∈ ↑s
hp4 : p4 ∈ ↑s
⊢ (fun x x_1 => x -ᵥ x_1) p1 p2 = 1 • (p1 -ᵥ p2)
[PROOFSTEP]
rw [one_smul]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ 0 ∈ { carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier
[PROOFSTEP]
cases' h with p hp
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ ↑s
⊢ 0 ∈ { carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier
[PROOFSTEP]
exact vsub_self p ▸ vsub_mem_vsub hp hp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ ∀ (c : k) {x : V},
x ∈
{
toAddSubsemigroup :=
{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) },
zero_mem' :=
(_ :
0 ∈
{ carrier := ↑s -ᵥ ↑s,
add_mem' :=
(_ :
∀ {a b : V},
a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier) }.toAddSubsemigroup.carrier →
c • x ∈
{
toAddSubsemigroup :=
{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) },
zero_mem' :=
(_ :
0 ∈
{ carrier := ↑s -ᵥ ↑s,
add_mem' :=
(_ :
∀ {a b : V},
a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier) }.toAddSubsemigroup.carrier
[PROOFSTEP]
intro c v hv
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
c : k
v : V
hv :
v ∈
{
toAddSubsemigroup :=
{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) },
zero_mem' :=
(_ :
0 ∈
{ carrier := ↑s -ᵥ ↑s,
add_mem' :=
(_ :
∀ {a b : V},
a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier) }.toAddSubsemigroup.carrier
⊢ c • v ∈
{
toAddSubsemigroup :=
{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) },
zero_mem' :=
(_ :
0 ∈
{ carrier := ↑s -ᵥ ↑s,
add_mem' :=
(_ :
∀ {a b : V},
a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier) }.toAddSubsemigroup.carrier
[PROOFSTEP]
rcases hv with ⟨p1, p2, hp1, hp2, rfl⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
c : k
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
⊢ c • (fun x x_1 => x -ᵥ x_1) p1 p2 ∈
{
toAddSubsemigroup :=
{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) },
zero_mem' :=
(_ :
0 ∈
{ carrier := ↑s -ᵥ ↑s,
add_mem' :=
(_ :
∀ {a b : V},
a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier) }.toAddSubsemigroup.carrier
[PROOFSTEP]
rw [← vadd_vsub (c • (p1 -ᵥ p2)) p2]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
c : k
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
⊢ c • (p1 -ᵥ p2) +ᵥ p2 -ᵥ p2 ∈
{
toAddSubsemigroup :=
{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) },
zero_mem' :=
(_ :
0 ∈
{ carrier := ↑s -ᵥ ↑s,
add_mem' :=
(_ :
∀ {a b : V},
a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) }.carrier) }.toAddSubsemigroup.carrier
[PROOFSTEP]
refine' vsub_mem_vsub _ hp2
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
c : k
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
⊢ c • (p1 -ᵥ p2) +ᵥ p2 ∈ ↑s
[PROOFSTEP]
exact s.smul_vsub_vadd_mem c hp1 hp2 hp2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ directionOfNonempty h = direction s
[PROOFSTEP]
refine le_antisymm ?_ (Submodule.span_le.2 Set.Subset.rfl)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ directionOfNonempty h ≤ direction s
[PROOFSTEP]
rw [← SetLike.coe_subset_coe, directionOfNonempty, direction, Submodule.coe_set_mk, AddSubmonoid.coe_set_mk]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ ↑{ carrier := ↑s -ᵥ ↑s, add_mem' := (_ : ∀ {a b : V}, a ∈ ↑s -ᵥ ↑s → b ∈ ↑s -ᵥ ↑s → a + b ∈ ↑s -ᵥ ↑s) } ⊆
↑(vectorSpan k ↑s)
[PROOFSTEP]
exact (vsub_set_subset_vectorSpan k _)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
v : V
⊢ v ∈ direction s ↔ ∃ p1, p1 ∈ s ∧ ∃ p2, p2 ∈ s ∧ v = p1 -ᵥ p2
[PROOFSTEP]
rw [← SetLike.mem_coe, coe_direction_eq_vsub_set h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : Set.Nonempty ↑s
v : V
⊢ v ∈ ↑s -ᵥ ↑s ↔ ∃ p1, p1 ∈ s ∧ ∃ p2, p2 ∈ s ∧ v = p1 -ᵥ p2
[PROOFSTEP]
exact
⟨fun ⟨p1, p2, hp1, hp2, hv⟩ => ⟨p1, hp1, p2, hp2, hv.symm⟩, fun ⟨p1, hp1, p2, hp2, hv⟩ => ⟨p1, p2, hp1, hp2, hv.symm⟩⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
hv : v ∈ direction s
p : P
hp : p ∈ s
⊢ v +ᵥ p ∈ s
[PROOFSTEP]
rw [mem_direction_iff_eq_vsub ⟨p, hp⟩] at hv
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
hv : ∃ p1, p1 ∈ s ∧ ∃ p2, p2 ∈ s ∧ v = p1 -ᵥ p2
p : P
hp : p ∈ s
⊢ v +ᵥ p ∈ s
[PROOFSTEP]
rcases hv with ⟨p1, hp1, p2, hp2, hv⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
p : P
hp : p ∈ s
p1 : P
hp1 : p1 ∈ s
p2 : P
hp2 : p2 ∈ s
hv : v = p1 -ᵥ p2
⊢ v +ᵥ p ∈ s
[PROOFSTEP]
rw [hv]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
p : P
hp : p ∈ s
p1 : P
hp1 : p1 ∈ s
p2 : P
hp2 : p2 ∈ s
hv : v = p1 -ᵥ p2
⊢ p1 -ᵥ p2 +ᵥ p ∈ s
[PROOFSTEP]
convert s.smul_vsub_vadd_mem 1 hp1 hp2 hp
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
p : P
hp : p ∈ s
p1 : P
hp1 : p1 ∈ s
p2 : P
hp2 : p2 ∈ s
hv : v = p1 -ᵥ p2
⊢ p1 -ᵥ p2 +ᵥ p ∈ s ↔ 1 • (p1 -ᵥ p2) +ᵥ p ∈ s.carrier
[PROOFSTEP]
rw [one_smul]
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
p : P
hp : p ∈ s
p1 : P
hp1 : p1 ∈ s
p2 : P
hp2 : p2 ∈ s
hv : v = p1 -ᵥ p2
⊢ p1 -ᵥ p2 +ᵥ p ∈ s ↔ p1 -ᵥ p2 +ᵥ p ∈ s.carrier
[PROOFSTEP]
exact s.mem_coe k P _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
p : P
hp : p ∈ s
h : v +ᵥ p ∈ s
⊢ v ∈ direction s
[PROOFSTEP]
simpa using vsub_mem_direction h hp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
hv : v ∈ direction s
p : P
⊢ v +ᵥ p ∈ s ↔ p ∈ s
[PROOFSTEP]
refine' ⟨fun h => _, fun h => vadd_mem_of_mem_direction hv h⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
hv : v ∈ direction s
p : P
h : v +ᵥ p ∈ s
⊢ p ∈ s
[PROOFSTEP]
convert vadd_mem_of_mem_direction (Submodule.neg_mem _ hv) h
[GOAL]
case h.e'_4
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
hv : v ∈ direction s
p : P
h : v +ᵥ p ∈ s
⊢ p = -v +ᵥ (v +ᵥ p)
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
⊢ ↑(direction s) = (fun x => x -ᵥ p) '' ↑s
[PROOFSTEP]
rw [coe_direction_eq_vsub_set ⟨p, hp⟩]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
⊢ ↑s -ᵥ ↑s = (fun x => x -ᵥ p) '' ↑s
[PROOFSTEP]
refine' le_antisymm _ _
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
⊢ ↑s -ᵥ ↑s ≤ (fun x => x -ᵥ p) '' ↑s
[PROOFSTEP]
rintro v ⟨p1, p2, hp1, hp2, rfl⟩
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
p1 p2 : P
hp1 : p1 ∈ ↑s
hp2 : p2 ∈ ↑s
⊢ (fun x x_1 => x -ᵥ x_1) p1 p2 ∈ (fun x => x -ᵥ p) '' ↑s
[PROOFSTEP]
exact ⟨p1 -ᵥ p2 +ᵥ p, vadd_mem_of_mem_direction (vsub_mem_direction hp1 hp2) hp, vadd_vsub _ _⟩
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
⊢ (fun x => x -ᵥ p) '' ↑s ≤ ↑s -ᵥ ↑s
[PROOFSTEP]
rintro v ⟨p2, hp2, rfl⟩
[GOAL]
case refine'_2.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
p2 : P
hp2 : p2 ∈ ↑s
⊢ (fun x => x -ᵥ p) p2 ∈ ↑s -ᵥ ↑s
[PROOFSTEP]
exact ⟨p2, p, hp2, hp, rfl⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
⊢ ↑(direction s) = (fun x x_1 => x -ᵥ x_1) p '' ↑s
[PROOFSTEP]
ext v
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
⊢ v ∈ ↑(direction s) ↔ v ∈ (fun x x_1 => x -ᵥ x_1) p '' ↑s
[PROOFSTEP]
rw [SetLike.mem_coe, ← Submodule.neg_mem_iff, ← SetLike.mem_coe, coe_direction_eq_vsub_set_right hp,
Set.mem_image_iff_bex, Set.mem_image_iff_bex]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
⊢ (∃ x x_1, x -ᵥ p = -v) ↔ ∃ x x_1, (fun x x_2 => x -ᵥ x_2) p x = v
[PROOFSTEP]
conv_lhs =>
congr
ext
rw [← neg_vsub_eq_vsub_rev, neg_inj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
| ∃ x x_1, x -ᵥ p = -v
[PROOFSTEP]
congr
ext
rw [← neg_vsub_eq_vsub_rev, neg_inj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
| ∃ x x_1, x -ᵥ p = -v
[PROOFSTEP]
congr
ext
rw [← neg_vsub_eq_vsub_rev, neg_inj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
| ∃ x x_1, x -ᵥ p = -v
[PROOFSTEP]
congr
[GOAL]
case p
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
| fun x => ∃ x_1, x -ᵥ p = -v
[PROOFSTEP]
ext
[GOAL]
case p.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
x✝ : P
| ∃ x, x✝ -ᵥ p = -v
[PROOFSTEP]
rw [← neg_vsub_eq_vsub_rev, neg_inj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
⊢ v ∈ direction s ↔ ∃ p2, p2 ∈ s ∧ v = p2 -ᵥ p
[PROOFSTEP]
rw [← SetLike.mem_coe, coe_direction_eq_vsub_set_right hp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
⊢ v ∈ (fun x => x -ᵥ p) '' ↑s ↔ ∃ p2, p2 ∈ s ∧ v = p2 -ᵥ p
[PROOFSTEP]
exact ⟨fun ⟨p2, hp2, hv⟩ => ⟨p2, hp2, hv.symm⟩, fun ⟨p2, hp2, hv⟩ => ⟨p2, hp2, hv.symm⟩⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
⊢ v ∈ direction s ↔ ∃ p2, p2 ∈ s ∧ v = p -ᵥ p2
[PROOFSTEP]
rw [← SetLike.mem_coe, coe_direction_eq_vsub_set_left hp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
v : V
⊢ v ∈ (fun x x_1 => x -ᵥ x_1) p '' ↑s ↔ ∃ p2, p2 ∈ s ∧ v = p -ᵥ p2
[PROOFSTEP]
exact ⟨fun ⟨p2, hp2, hv⟩ => ⟨p2, hp2, hv.symm⟩, fun ⟨p2, hp2, hv⟩ => ⟨p2, hp2, hv.symm⟩⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
p2 : P
⊢ p2 -ᵥ p ∈ direction s ↔ p2 ∈ s
[PROOFSTEP]
rw [mem_direction_iff_eq_vsub_right hp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
p2 : P
⊢ (∃ p2_1, p2_1 ∈ s ∧ p2 -ᵥ p = p2_1 -ᵥ p) ↔ p2 ∈ s
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
p2 : P
⊢ p -ᵥ p2 ∈ direction s ↔ p2 ∈ s
[PROOFSTEP]
rw [mem_direction_iff_eq_vsub_left hp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p : P
hp : p ∈ s
p2 : P
⊢ (∃ p2_1, p2_1 ∈ s ∧ p -ᵥ p2 = p -ᵥ p2_1) ↔ p2 ∈ s
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
⊢ s1 = s2
[PROOFSTEP]
ext p
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
⊢ p ∈ s1 ↔ p ∈ s2
[PROOFSTEP]
have hq1 := Set.mem_of_mem_inter_left hn.some_mem
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
⊢ p ∈ s1 ↔ p ∈ s2
[PROOFSTEP]
have hq2 := Set.mem_of_mem_inter_right hn.some_mem
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
⊢ p ∈ s1 ↔ p ∈ s2
[PROOFSTEP]
constructor
[GOAL]
case h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
⊢ p ∈ s1 → p ∈ s2
[PROOFSTEP]
intro hp
[GOAL]
case h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s1
⊢ p ∈ s2
[PROOFSTEP]
rw [← vsub_vadd p hn.some]
[GOAL]
case h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s1
⊢ p -ᵥ Set.Nonempty.some hn +ᵥ Set.Nonempty.some hn ∈ s2
[PROOFSTEP]
refine' vadd_mem_of_mem_direction _ hq2
[GOAL]
case h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s1
⊢ p -ᵥ Set.Nonempty.some hn ∈ direction s2
[PROOFSTEP]
rw [← hd]
[GOAL]
case h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s1
⊢ p -ᵥ Set.Nonempty.some hn ∈ direction s1
[PROOFSTEP]
exact vsub_mem_direction hp hq1
[GOAL]
case h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
⊢ p ∈ s2 → p ∈ s1
[PROOFSTEP]
intro hp
[GOAL]
case h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s2
⊢ p ∈ s1
[PROOFSTEP]
rw [← vsub_vadd p hn.some]
[GOAL]
case h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s2
⊢ p -ᵥ Set.Nonempty.some hn +ᵥ Set.Nonempty.some hn ∈ s1
[PROOFSTEP]
refine' vadd_mem_of_mem_direction _ hq1
[GOAL]
case h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s2
⊢ p -ᵥ Set.Nonempty.some hn ∈ direction s1
[PROOFSTEP]
rw [hd]
[GOAL]
case h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
hd : direction s1 = direction s2
hn : Set.Nonempty (↑s1 ∩ ↑s2)
p : P
hq1 : Set.Nonempty.some hn ∈ ↑s1
hq2 : Set.Nonempty.some hn ∈ ↑s2
hp : p ∈ s2
⊢ p -ᵥ Set.Nonempty.some hn ∈ direction s2
[PROOFSTEP]
exact vsub_mem_direction hp hq2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a : { x // x ∈ s }
⊢ 0 +ᵥ a = a
[PROOFSTEP]
ext
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a : { x // x ∈ s }
⊢ ↑(0 +ᵥ a) = ↑a
[PROOFSTEP]
exact zero_vadd _ _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a b : { x // x ∈ direction s }
c : { x // x ∈ s }
⊢ a + b +ᵥ c = a +ᵥ (b +ᵥ c)
[PROOFSTEP]
ext
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a b : { x // x ∈ direction s }
c : { x // x ∈ s }
⊢ ↑(a + b +ᵥ c) = ↑(a +ᵥ (b +ᵥ c))
[PROOFSTEP]
apply add_vadd
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
⊢ Nonempty { x // x ∈ s }
[PROOFSTEP]
infer_instance
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a b : { x // x ∈ s }
⊢ a -ᵥ b +ᵥ b = a
[PROOFSTEP]
ext
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a b : { x // x ∈ s }
⊢ ↑(a -ᵥ b +ᵥ b) = ↑a
[PROOFSTEP]
apply AddTorsor.vsub_vadd'
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a : { x // x ∈ direction s }
b : { x // x ∈ s }
⊢ a +ᵥ b -ᵥ b = a
[PROOFSTEP]
ext
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
s : AffineSubspace k P
inst✝ : Nonempty { x // x ∈ s }
a : { x // x ∈ direction s }
b : { x // x ∈ s }
⊢ ↑(a +ᵥ b -ᵥ b) = ↑a
[PROOFSTEP]
apply AddTorsor.vadd_vsub'
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
c : k
p1 p2 p3 : P
hp1 : p1 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
hp2 : p2 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
hp3 : p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
⊢ c • (p1 -ᵥ p2) +ᵥ p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
[PROOFSTEP]
rcases hp1 with ⟨v1, hv1, hp1⟩
[GOAL]
case intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
c : k
p1 p2 p3 : P
hp2 : p2 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
hp3 : p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
v1 : V
hv1 : v1 ∈ direction
hp1 : p1 = v1 +ᵥ p
⊢ c • (p1 -ᵥ p2) +ᵥ p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
[PROOFSTEP]
rcases hp2 with ⟨v2, hv2, hp2⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
c : k
p1 p2 p3 : P
hp3 : p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
v1 : V
hv1 : v1 ∈ direction
hp1 : p1 = v1 +ᵥ p
v2 : V
hv2 : v2 ∈ direction
hp2 : p2 = v2 +ᵥ p
⊢ c • (p1 -ᵥ p2) +ᵥ p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
[PROOFSTEP]
rcases hp3 with ⟨v3, hv3, hp3⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
c : k
p1 p2 p3 : P
v1 : V
hv1 : v1 ∈ direction
hp1 : p1 = v1 +ᵥ p
v2 : V
hv2 : v2 ∈ direction
hp2 : p2 = v2 +ᵥ p
v3 : V
hv3 : v3 ∈ direction
hp3 : p3 = v3 +ᵥ p
⊢ c • (p1 -ᵥ p2) +ᵥ p3 ∈ {q | ∃ v, v ∈ direction ∧ q = v +ᵥ p}
[PROOFSTEP]
use c • (v1 - v2) + v3, direction.add_mem (direction.smul_mem c (direction.sub_mem hv1 hv2)) hv3
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
c : k
p1 p2 p3 : P
v1 : V
hv1 : v1 ∈ direction
hp1 : p1 = v1 +ᵥ p
v2 : V
hv2 : v2 ∈ direction
hp2 : p2 = v2 +ᵥ p
v3 : V
hv3 : v3 ∈ direction
hp3 : p3 = v3 +ᵥ p
⊢ c • (p1 -ᵥ p2) +ᵥ p3 = c • (v1 - v2) + v3 +ᵥ p
[PROOFSTEP]
simp [hp1, hp2, hp3, vadd_vadd]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
⊢ AffineSubspace.direction (mk' p direction) = direction
[PROOFSTEP]
ext v
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
v : V
⊢ v ∈ AffineSubspace.direction (mk' p direction) ↔ v ∈ direction
[PROOFSTEP]
rw [mem_direction_iff_eq_vsub (mk'_nonempty _ _)]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
v : V
⊢ (∃ p1, p1 ∈ mk' p direction ∧ ∃ p2, p2 ∈ mk' p direction ∧ v = p1 -ᵥ p2) ↔ v ∈ direction
[PROOFSTEP]
constructor
[GOAL]
case h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
v : V
⊢ (∃ p1, p1 ∈ mk' p direction ∧ ∃ p2, p2 ∈ mk' p direction ∧ v = p1 -ᵥ p2) → v ∈ direction
[PROOFSTEP]
rintro ⟨p1, ⟨v1, hv1, hp1⟩, p2, ⟨v2, hv2, hp2⟩, hv⟩
[GOAL]
case h.mp.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
v : V
p1 : P
v1 : V
hv1 : v1 ∈ direction
hp1 : p1 = v1 +ᵥ p
p2 : P
hv : v = p1 -ᵥ p2
v2 : V
hv2 : v2 ∈ direction
hp2 : p2 = v2 +ᵥ p
⊢ v ∈ direction
[PROOFSTEP]
rw [hv, hp1, hp2, vadd_vsub_vadd_cancel_right]
[GOAL]
case h.mp.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
v : V
p1 : P
v1 : V
hv1 : v1 ∈ direction
hp1 : p1 = v1 +ᵥ p
p2 : P
hv : v = p1 -ᵥ p2
v2 : V
hv2 : v2 ∈ direction
hp2 : p2 = v2 +ᵥ p
⊢ v1 - v2 ∈ direction
[PROOFSTEP]
exact direction.sub_mem hv1 hv2
[GOAL]
case h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
direction : Submodule k V
v : V
⊢ v ∈ direction → ∃ p1, p1 ∈ mk' p direction ∧ ∃ p2, p2 ∈ mk' p direction ∧ v = p1 -ᵥ p2
[PROOFSTEP]
exact fun hv => ⟨v +ᵥ p, vadd_mem_mk' _ hv, p, self_mem_mk' _ _, (vadd_vsub _ _).symm⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p₁ p₂ : P
direction : Submodule k V
⊢ p₂ ∈ mk' p₁ direction ↔ p₂ -ᵥ p₁ ∈ direction
[PROOFSTEP]
refine' ⟨fun h => _, fun h => _⟩
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p₁ p₂ : P
direction : Submodule k V
h : p₂ ∈ mk' p₁ direction
⊢ p₂ -ᵥ p₁ ∈ direction
[PROOFSTEP]
rw [← direction_mk' p₁ direction]
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p₁ p₂ : P
direction : Submodule k V
h : p₂ ∈ mk' p₁ direction
⊢ p₂ -ᵥ p₁ ∈ AffineSubspace.direction (mk' p₁ direction)
[PROOFSTEP]
exact vsub_mem_direction h (self_mem_mk' _ _)
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p₁ p₂ : P
direction : Submodule k V
h : p₂ -ᵥ p₁ ∈ direction
⊢ p₂ ∈ mk' p₁ direction
[PROOFSTEP]
rw [← vsub_vadd p₂ p₁]
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p₁ p₂ : P
direction : Submodule k V
h : p₂ -ᵥ p₁ ∈ direction
⊢ p₂ -ᵥ p₁ +ᵥ p₁ ∈ mk' p₁ direction
[PROOFSTEP]
exact vadd_mem_mk' p₁ h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
⊢ spanPoints k s ⊆ ↑s1
[PROOFSTEP]
rintro p ⟨p1, hp1, v, hv, hp⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
⊢ p ∈ ↑s1
[PROOFSTEP]
rw [hp]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
⊢ v +ᵥ p1 ∈ ↑s1
[PROOFSTEP]
have hp1s1 : p1 ∈ (s1 : Set P) := Set.mem_of_mem_of_subset hp1 h
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
hp1s1 : p1 ∈ ↑s1
⊢ v +ᵥ p1 ∈ ↑s1
[PROOFSTEP]
refine' vadd_mem_of_mem_direction _ hp1s1
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
hp1s1 : p1 ∈ ↑s1
⊢ v ∈ direction s1
[PROOFSTEP]
have hs : vectorSpan k s ≤ s1.direction := vectorSpan_mono k h
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
hp1s1 : p1 ∈ ↑s1
hs : vectorSpan k s ≤ direction s1
⊢ v ∈ direction s1
[PROOFSTEP]
rw [SetLike.le_def] at hs
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
hp1s1 : p1 ∈ ↑s1
hs : ∀ ⦃x : V⦄, x ∈ vectorSpan k s → x ∈ direction s1
⊢ v ∈ direction s1
[PROOFSTEP]
rw [← SetLike.mem_coe]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
s1 : AffineSubspace k P
h : s ⊆ ↑s1
p p1 : P
hp1 : p1 ∈ s
v : V
hv : v ∈ vectorSpan k s
hp : p = v +ᵥ p1
hp1s1 : p1 ∈ ↑s1
hs : ∀ ⦃x : V⦄, x ∈ vectorSpan k s → x ∈ direction s1
⊢ v ∈ ↑(direction s1)
[PROOFSTEP]
exact Set.mem_of_mem_of_subset hv hs
[GOAL]
k : Type u_1
V : Type u_2
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
s : Submodule k V
⊢ AffineSubspace.direction (toAffineSubspace s) = s
[PROOFSTEP]
ext x
[GOAL]
case h
k : Type u_1
V : Type u_2
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
s : Submodule k V
x : V
⊢ x ∈ AffineSubspace.direction (toAffineSubspace s) ↔ x ∈ s
[PROOFSTEP]
simp [← s.toAffineSubspace.vadd_mem_iff_mem_direction _ s.zero_mem]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
Q : AffineSubspace k P
p₀ p₁ : P
c : k
h₀ : p₀ ∈ Q
h₁ : p₁ ∈ Q
⊢ ↑(lineMap p₀ p₁) c ∈ Q
[PROOFSTEP]
rw [AffineMap.lineMap_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
Q : AffineSubspace k P
p₀ p₁ : P
c : k
h₀ : p₀ ∈ Q
h₁ : p₁ ∈ Q
⊢ c • (p₁ -ᵥ p₀) +ᵥ p₀ ∈ Q
[PROOFSTEP]
exact Q.smul_vsub_vadd_mem c h₁ h₀ h₀
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ AffineSubspace.direction (affineSpan k s) = vectorSpan k s
[PROOFSTEP]
apply le_antisymm
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ AffineSubspace.direction (affineSpan k s) ≤ vectorSpan k s
[PROOFSTEP]
refine' Submodule.span_le.2 _
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ ↑(affineSpan k s) -ᵥ ↑(affineSpan k s) ⊆ ↑(vectorSpan k s)
[PROOFSTEP]
rintro v ⟨p1, p3, ⟨p2, hp2, v1, hv1, hp1⟩, ⟨p4, hp4, v2, hv2, hp3⟩, rfl⟩
[GOAL]
case a.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p3 p2 : P
hp2 : p2 ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hp1 : p1 = v1 +ᵥ p2
p4 : P
hp4 : p4 ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hp3 : p3 = v2 +ᵥ p4
⊢ (fun x x_1 => x -ᵥ x_1) p1 p3 ∈ ↑(vectorSpan k s)
[PROOFSTEP]
simp only [SetLike.mem_coe]
[GOAL]
case a.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p3 p2 : P
hp2 : p2 ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hp1 : p1 = v1 +ᵥ p2
p4 : P
hp4 : p4 ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hp3 : p3 = v2 +ᵥ p4
⊢ p1 -ᵥ p3 ∈ vectorSpan k s
[PROOFSTEP]
rw [hp1, hp3, vsub_vadd_eq_vsub_sub, vadd_vsub_assoc]
[GOAL]
case a.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
p1 p3 p2 : P
hp2 : p2 ∈ s
v1 : V
hv1 : v1 ∈ vectorSpan k s
hp1 : p1 = v1 +ᵥ p2
p4 : P
hp4 : p4 ∈ s
v2 : V
hv2 : v2 ∈ vectorSpan k s
hp3 : p3 = v2 +ᵥ p4
⊢ v1 + (p2 -ᵥ p4) - v2 ∈ vectorSpan k s
[PROOFSTEP]
exact (vectorSpan k s).sub_mem ((vectorSpan k s).add_mem hv1 (vsub_mem_vectorSpan k hp2 hp4)) hv2
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : Set P
⊢ vectorSpan k s ≤ AffineSubspace.direction (affineSpan k s)
[PROOFSTEP]
exact vectorSpan_mono k (subset_spanPoints k s)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
src✝ : PartialOrder (AffineSubspace k P) := PartialOrder.lift SetLike.coe (_ : Function.Injective SetLike.coe)
s : Set (AffineSubspace k P)
c : k
p1 p2 p3 : P
hp1 : p1 ∈ ⋂ (s' : AffineSubspace k P) (_ : s' ∈ s), ↑s'
hp2 : p2 ∈ ⋂ (s' : AffineSubspace k P) (_ : s' ∈ s), ↑s'
hp3 : p3 ∈ ⋂ (s' : AffineSubspace k P) (_ : s' ∈ s), ↑s'
s2 : AffineSubspace k P
hs2 : s2 ∈ s
⊢ c • (p1 -ᵥ p2) +ᵥ p3 ∈ ↑s2
[PROOFSTEP]
rw [Set.mem_iInter₂] at *
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
src✝ : PartialOrder (AffineSubspace k P) := PartialOrder.lift SetLike.coe (_ : Function.Injective SetLike.coe)
s : Set (AffineSubspace k P)
c : k
p1 p2 p3 : P
hp1 : ∀ (i : AffineSubspace k P), i ∈ s → p1 ∈ ↑i
hp2 : ∀ (i : AffineSubspace k P), i ∈ s → p2 ∈ ↑i
hp3 : ∀ (i : AffineSubspace k P), i ∈ s → p3 ∈ ↑i
s2 : AffineSubspace k P
hs2 : s2 ∈ s
⊢ c • (p1 -ᵥ p2) +ᵥ p3 ∈ ↑s2
[PROOFSTEP]
exact s2.smul_vsub_vadd_mem c (hp1 s2 hs2) (hp2 s2 hs2) (hp3 s2 hs2)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S✝ : AffineSpace V P
src✝ : PartialOrder (AffineSubspace k P) := PartialOrder.lift SetLike.coe (_ : Function.Injective SetLike.coe)
S : Set (AffineSubspace k P)
s1 : AffineSubspace k P
hs1 : ∀ (b : AffineSubspace k P), b ∈ S → s1 ≤ b
⊢ s1 ≤ sInf S
[PROOFSTEP]
refine' Set.subset_sInter (t := (s1 : Set P)) _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S✝ : AffineSpace V P
src✝ : PartialOrder (AffineSubspace k P) := PartialOrder.lift SetLike.coe (_ : Function.Injective SetLike.coe)
S : Set (AffineSubspace k P)
s1 : AffineSubspace k P
hs1 : ∀ (b : AffineSubspace k P), b ∈ S → s1 ≤ b
⊢ ∀ (t' : Set P), (t' ∈ range fun s' => ⋂ (_ : s' ∈ S), ↑s') → ↑s1 ⊆ t'
[PROOFSTEP]
rintro t ⟨s, _hs, rfl⟩
[GOAL]
case intro.refl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S✝ : AffineSpace V P
src✝ : PartialOrder (AffineSubspace k P) := PartialOrder.lift SetLike.coe (_ : Function.Injective SetLike.coe)
S : Set (AffineSubspace k P)
s1 : AffineSubspace k P
hs1 : ∀ (b : AffineSubspace k P), b ∈ S → s1 ≤ b
s : AffineSubspace k P
⊢ ↑s1 ⊆ (fun s' => ⋂ (_ : s' ∈ S), ↑s') s
[PROOFSTEP]
exact Set.subset_iInter (hs1 s)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
s1 s2 : AffineSubspace k P
⊢ s1 < s2 ↔ s1 ≤ s2 ∧ ∃ p, p ∈ s2 ∧ ¬p ∈ s1
[PROOFSTEP]
rw [lt_iff_le_not_le, not_le_iff_exists]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p : P
⊢ ↑(affineSpan k {p}) = {p}
[PROOFSTEP]
ext x
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p x : P
⊢ x ∈ ↑(affineSpan k {p}) ↔ x ∈ {p}
[PROOFSTEP]
rw [mem_coe, ← vsub_right_mem_direction_iff_mem (mem_affineSpan k (Set.mem_singleton p)) _, direction_affineSpan]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p x : P
⊢ x -ᵥ p ∈ vectorSpan k {p} ↔ x ∈ {p}
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
⊢ p₁ ∈ affineSpan k {p₂} ↔ p₁ = p₂
[PROOFSTEP]
simp [← mem_coe]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
⊢ direction ⊤ = ⊤
[PROOFSTEP]
cases' S.Nonempty with p
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p : P
⊢ direction ⊤ = ⊤
[PROOFSTEP]
ext v
[GOAL]
case intro.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p : P
v : V
⊢ v ∈ direction ⊤ ↔ v ∈ ⊤
[PROOFSTEP]
refine' ⟨imp_intro Submodule.mem_top, fun _hv => _⟩
[GOAL]
case intro.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p : P
v : V
_hv : v ∈ ⊤
⊢ v ∈ direction ⊤
[PROOFSTEP]
have hpv : (v +ᵥ p -ᵥ p : V) ∈ (⊤ : AffineSubspace k P).direction := vsub_mem_direction (mem_top k V _) (mem_top k V _)
[GOAL]
case intro.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ p : P
v : V
_hv : v ∈ ⊤
hpv : v +ᵥ p -ᵥ p ∈ direction ⊤
⊢ v ∈ direction ⊤
[PROOFSTEP]
rwa [vadd_vsub] at hpv
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
⊢ ⊥ ≠ ⊤
[PROOFSTEP]
intro contra
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
contra : ⊥ = ⊤
⊢ False
[PROOFSTEP]
rw [← ext_iff, bot_coe, top_coe] at contra
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
contra : ∅ = univ
⊢ False
[PROOFSTEP]
exact Set.empty_ne_univ contra
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h : affineSpan k s = ⊤
⊢ Set.Nonempty s
[PROOFSTEP]
rw [Set.nonempty_iff_ne_empty]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h : affineSpan k s = ⊤
⊢ s ≠ ∅
[PROOFSTEP]
rintro rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
h : affineSpan k ∅ = ⊤
⊢ False
[PROOFSTEP]
rw [AffineSubspace.span_empty] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
h : ⊥ = ⊤
⊢ False
[PROOFSTEP]
exact bot_ne_top k V P h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h : affineSpan k s = ⊤
⊢ vectorSpan k s = ⊤
[PROOFSTEP]
rw [← direction_affineSpan, h, direction_top]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
hs : Set.Nonempty s
⊢ affineSpan k s = ⊤ ↔ vectorSpan k s = ⊤
[PROOFSTEP]
refine' ⟨vectorSpan_eq_top_of_affineSpan_eq_top k V P, _⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
hs : Set.Nonempty s
⊢ vectorSpan k s = ⊤ → affineSpan k s = ⊤
[PROOFSTEP]
intro h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
hs : Set.Nonempty s
h : vectorSpan k s = ⊤
⊢ affineSpan k s = ⊤
[PROOFSTEP]
suffices Nonempty (affineSpan k s) by
obtain ⟨p, hp : p ∈ affineSpan k s⟩ := this
rw [eq_iff_direction_eq_of_mem hp (mem_top k V p), direction_affineSpan, h, direction_top]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
hs : Set.Nonempty s
h : vectorSpan k s = ⊤
this : Nonempty { x // x ∈ affineSpan k s }
⊢ affineSpan k s = ⊤
[PROOFSTEP]
obtain ⟨p, hp : p ∈ affineSpan k s⟩ := this
[GOAL]
case intro.mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
hs : Set.Nonempty s
h : vectorSpan k s = ⊤
p : P
hp : p ∈ affineSpan k s
⊢ affineSpan k s = ⊤
[PROOFSTEP]
rw [eq_iff_direction_eq_of_mem hp (mem_top k V p), direction_affineSpan, h, direction_top]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
hs : Set.Nonempty s
h : vectorSpan k s = ⊤
⊢ Nonempty { x // x ∈ affineSpan k s }
[PROOFSTEP]
obtain ⟨x, hx⟩ := hs
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h : vectorSpan k s = ⊤
x : P
hx : x ∈ s
⊢ Nonempty { x // x ∈ affineSpan k s }
[PROOFSTEP]
exact ⟨⟨x, mem_affineSpan k hx⟩⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
inst✝ : Nontrivial P
⊢ affineSpan k s = ⊤ ↔ vectorSpan k s = ⊤
[PROOFSTEP]
cases' s.eq_empty_or_nonempty with hs hs
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
inst✝ : Nontrivial P
hs : s = ∅
⊢ affineSpan k s = ⊤ ↔ vectorSpan k s = ⊤
[PROOFSTEP]
simp [hs, subsingleton_iff_bot_eq_top, AddTorsor.subsingleton_iff V P, not_subsingleton]
[GOAL]
case inr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
inst✝ : Nontrivial P
hs : Set.Nonempty s
⊢ affineSpan k s = ⊤ ↔ vectorSpan k s = ⊤
[PROOFSTEP]
rw [affineSpan_eq_top_iff_vectorSpan_eq_top_of_nonempty k V P hs]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
p₁ p₂ : P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h : affineSpan k (range p) = ⊤
⊢ 0 < Fintype.card ι
[PROOFSTEP]
obtain ⟨-, ⟨i, -⟩⟩ := nonempty_of_affineSpan_eq_top k V P h
[GOAL]
case intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
p₁ p₂ : P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h : affineSpan k (range p) = ⊤
i : ι
⊢ 0 < Fintype.card ι
[PROOFSTEP]
exact Fintype.card_pos_iff.mpr ⟨i⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
⊢ direction ⊥ = ⊥
[PROOFSTEP]
rw [direction_eq_vectorSpan, bot_coe, vectorSpan_def, vsub_empty, Submodule.span_empty]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
Q : AffineSubspace k P
⊢ Set.Nonempty ↑Q ↔ Q ≠ ⊥
[PROOFSTEP]
rw [nonempty_iff_ne_empty]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
Q : AffineSubspace k P
⊢ ↑Q ≠ ∅ ↔ Q ≠ ⊥
[PROOFSTEP]
exact not_congr Q.coe_eq_bot_iff
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
Q : AffineSubspace k P
⊢ Q = ⊥ ∨ Set.Nonempty ↑Q
[PROOFSTEP]
rw [nonempty_iff_ne_bot]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
Q : AffineSubspace k P
⊢ Q = ⊥ ∨ Q ≠ ⊥
[PROOFSTEP]
apply eq_or_ne
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
⊢ Subsingleton P
[PROOFSTEP]
obtain ⟨p, hp⟩ := AffineSubspace.nonempty_of_affineSpan_eq_top k V P h₂
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
⊢ Subsingleton P
[PROOFSTEP]
have : s = { p } := Subset.antisymm (fun q hq => h₁ hq hp) (by simp [hp])
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
⊢ {p} ⊆ s
[PROOFSTEP]
simp [hp]
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
this : s = {p}
⊢ Subsingleton P
[PROOFSTEP]
rw [this, ← AffineSubspace.ext_iff, AffineSubspace.coe_affineSpan_singleton, AffineSubspace.top_coe, eq_comm, ←
subsingleton_iff_singleton (mem_univ _)] at h₂
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
p : P
h₂ : Set.Subsingleton univ
hp : p ∈ s
this : s = {p}
⊢ Subsingleton P
[PROOFSTEP]
exact subsingleton_of_univ_subsingleton h₂
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
⊢ s = univ
[PROOFSTEP]
obtain ⟨p, hp⟩ := AffineSubspace.nonempty_of_affineSpan_eq_top k V P h₂
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
⊢ s = univ
[PROOFSTEP]
have : s = { p } := Subset.antisymm (fun q hq => h₁ hq hp) (by simp [hp])
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
⊢ {p} ⊆ s
[PROOFSTEP]
simp [hp]
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
this : s = {p}
⊢ s = univ
[PROOFSTEP]
rw [this, eq_comm, ← subsingleton_iff_singleton (mem_univ p), subsingleton_univ_iff]
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : Set P
h₁ : Set.Subsingleton s
h₂ : affineSpan k s = ⊤
p : P
hp : p ∈ s
this : s = {p}
⊢ Subsingleton P
[PROOFSTEP]
exact subsingleton_of_subsingleton_span_eq_top h₁ h₂
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ direction s = ⊤ ↔ s = ⊤
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ direction s = ⊤ → s = ⊤
[PROOFSTEP]
intro hd
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
h : Set.Nonempty ↑s
hd : direction s = ⊤
⊢ s = ⊤
[PROOFSTEP]
rw [← direction_top k V P] at hd
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
h : Set.Nonempty ↑s
hd : direction s = direction ⊤
⊢ s = ⊤
[PROOFSTEP]
refine' ext_of_direction_eq hd _
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
h : Set.Nonempty ↑s
hd : direction s = direction ⊤
⊢ Set.Nonempty (↑s ∩ ↑⊤)
[PROOFSTEP]
simp [h]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
h : Set.Nonempty ↑s
⊢ s = ⊤ → direction s = ⊤
[PROOFSTEP]
rintro rfl
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
h : Set.Nonempty ↑⊤
⊢ direction ⊤ = ⊤
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
⊢ direction (s1 ⊓ s2) ≤ direction s1 ⊓ direction s2
[PROOFSTEP]
simp only [direction_eq_vectorSpan, vectorSpan_def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
⊢ Submodule.span k (↑(s1 ⊓ s2) -ᵥ ↑(s1 ⊓ s2)) ≤ Submodule.span k (↑s1 -ᵥ ↑s1) ⊓ Submodule.span k (↑s2 -ᵥ ↑s2)
[PROOFSTEP]
exact
le_inf (sInf_le_sInf fun p hp => trans (vsub_self_mono (inter_subset_left _ _)) hp)
(sInf_le_sInf fun p hp => trans (vsub_self_mono (inter_subset_right _ _)) hp)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s₁ s₂ : AffineSubspace k P
p : P
h₁ : p ∈ s₁
h₂ : p ∈ s₂
⊢ direction (s₁ ⊓ s₂) = direction s₁ ⊓ direction s₂
[PROOFSTEP]
ext v
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s₁ s₂ : AffineSubspace k P
p : P
h₁ : p ∈ s₁
h₂ : p ∈ s₂
v : V
⊢ v ∈ direction (s₁ ⊓ s₂) ↔ v ∈ direction s₁ ⊓ direction s₂
[PROOFSTEP]
rw [Submodule.mem_inf, ← vadd_mem_iff_mem_direction v h₁, ← vadd_mem_iff_mem_direction v h₂, ←
vadd_mem_iff_mem_direction v ((mem_inf_iff p s₁ s₂).2 ⟨h₁, h₂⟩), mem_inf_iff]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h : s1 ≤ s2
⊢ direction s1 ≤ direction s2
[PROOFSTEP]
simp only [direction_eq_vectorSpan, vectorSpan_def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h : s1 ≤ s2
⊢ Submodule.span k (↑s1 -ᵥ ↑s1) ≤ Submodule.span k (↑s2 -ᵥ ↑s2)
[PROOFSTEP]
exact vectorSpan_mono k h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h : s1 < s2
hn : Set.Nonempty ↑s1
⊢ direction s1 < direction s2
[PROOFSTEP]
cases' hn with p hp
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h : s1 < s2
p : P
hp : p ∈ ↑s1
⊢ direction s1 < direction s2
[PROOFSTEP]
rw [lt_iff_le_and_exists] at h
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h : s1 ≤ s2 ∧ ∃ p, p ∈ s2 ∧ ¬p ∈ s1
p : P
hp : p ∈ ↑s1
⊢ direction s1 < direction s2
[PROOFSTEP]
rcases h with ⟨hle, p2, hp2, hp2s1⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
p : P
hp : p ∈ ↑s1
hle : s1 ≤ s2
p2 : P
hp2 : p2 ∈ s2
hp2s1 : ¬p2 ∈ s1
⊢ direction s1 < direction s2
[PROOFSTEP]
rw [SetLike.lt_iff_le_and_exists]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
p : P
hp : p ∈ ↑s1
hle : s1 ≤ s2
p2 : P
hp2 : p2 ∈ s2
hp2s1 : ¬p2 ∈ s1
⊢ direction s1 ≤ direction s2 ∧ ∃ x, x ∈ direction s2 ∧ ¬x ∈ direction s1
[PROOFSTEP]
use direction_le hle, p2 -ᵥ p, vsub_mem_direction hp2 (hle hp)
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
p : P
hp : p ∈ ↑s1
hle : s1 ≤ s2
p2 : P
hp2 : p2 ∈ s2
hp2s1 : ¬p2 ∈ s1
⊢ ¬p2 -ᵥ p ∈ direction s1
[PROOFSTEP]
intro hm
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
p : P
hp : p ∈ ↑s1
hle : s1 ≤ s2
p2 : P
hp2 : p2 ∈ s2
hp2s1 : ¬p2 ∈ s1
hm : p2 -ᵥ p ∈ direction s1
⊢ False
[PROOFSTEP]
rw [vsub_right_mem_direction_iff_mem hp p2] at hm
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
p : P
hp : p ∈ ↑s1
hle : s1 ≤ s2
p2 : P
hp2 : p2 ∈ s2
hp2s1 : ¬p2 ∈ s1
hm : p2 ∈ s1
⊢ False
[PROOFSTEP]
exact hp2s1 hm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
⊢ direction s1 ⊔ direction s2 ≤ direction (s1 ⊔ s2)
[PROOFSTEP]
simp only [direction_eq_vectorSpan, vectorSpan_def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
⊢ Submodule.span k (↑s1 -ᵥ ↑s1) ⊔ Submodule.span k (↑s2 -ᵥ ↑s2) ≤ Submodule.span k (↑(s1 ⊔ s2) -ᵥ ↑(s1 ⊔ s2))
[PROOFSTEP]
exact
sup_le (sInf_le_sInf fun p hp => Set.Subset.trans (vsub_self_mono (le_sup_left : s1 ≤ s1 ⊔ s2)) hp)
(sInf_le_sInf fun p hp => Set.Subset.trans (vsub_self_mono (le_sup_right : s2 ≤ s1 ⊔ s2)) hp)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
he : ↑s1 ∩ ↑s2 = ∅
⊢ direction s1 ⊔ direction s2 < direction (s1 ⊔ s2)
[PROOFSTEP]
cases' h1 with p1 hp1
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h2 : Set.Nonempty ↑s2
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
⊢ direction s1 ⊔ direction s2 < direction (s1 ⊔ s2)
[PROOFSTEP]
cases' h2 with p2 hp2
[GOAL]
case intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
⊢ direction s1 ⊔ direction s2 < direction (s1 ⊔ s2)
[PROOFSTEP]
rw [SetLike.lt_iff_le_and_exists]
[GOAL]
case intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
⊢ direction s1 ⊔ direction s2 ≤ direction (s1 ⊔ s2) ∧ ∃ x, x ∈ direction (s1 ⊔ s2) ∧ ¬x ∈ direction s1 ⊔ direction s2
[PROOFSTEP]
use sup_direction_le s1 s2, p2 -ᵥ p1,
vsub_mem_direction ((le_sup_right : s2 ≤ s1 ⊔ s2) hp2) ((le_sup_left : s1 ≤ s1 ⊔ s2) hp1)
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
⊢ ¬p2 -ᵥ p1 ∈ direction s1 ⊔ direction s2
[PROOFSTEP]
intro h
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
h : p2 -ᵥ p1 ∈ direction s1 ⊔ direction s2
⊢ False
[PROOFSTEP]
rw [Submodule.mem_sup] at h
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
h : ∃ y, y ∈ direction s1 ∧ ∃ z, z ∈ direction s2 ∧ y + z = p2 -ᵥ p1
⊢ False
[PROOFSTEP]
rcases h with ⟨v1, hv1, v2, hv2, hv1v2⟩
[GOAL]
case right.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
v1 : V
hv1 : v1 ∈ direction s1
v2 : V
hv2 : v2 ∈ direction s2
hv1v2 : v1 + v2 = p2 -ᵥ p1
⊢ False
[PROOFSTEP]
rw [← sub_eq_zero, sub_eq_add_neg, neg_vsub_eq_vsub_rev, add_comm v1, add_assoc, ← vadd_vsub_assoc, ← neg_neg v2,
add_comm, ← sub_eq_add_neg, ← vsub_vadd_eq_vsub_sub, vsub_eq_zero_iff_eq] at hv1v2
[GOAL]
case right.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
v1 : V
hv1 : v1 ∈ direction s1
v2 : V
hv2 : v2 ∈ direction s2
hv1v2✝ : v1 + v2 = p2 -ᵥ p1
hv1v2 : v1 +ᵥ p1 = -v2 +ᵥ p2
⊢ False
[PROOFSTEP]
refine' Set.Nonempty.ne_empty _ he
[GOAL]
case right.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
v1 : V
hv1 : v1 ∈ direction s1
v2 : V
hv2 : v2 ∈ direction s2
hv1v2✝ : v1 + v2 = p2 -ᵥ p1
hv1v2 : v1 +ᵥ p1 = -v2 +ᵥ p2
⊢ Set.Nonempty (↑s1 ∩ ↑s2)
[PROOFSTEP]
use v1 +ᵥ p1, vadd_mem_of_mem_direction hv1 hp1
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
v1 : V
hv1 : v1 ∈ direction s1
v2 : V
hv2 : v2 ∈ direction s2
hv1v2✝ : v1 + v2 = p2 -ᵥ p1
hv1v2 : v1 +ᵥ p1 = -v2 +ᵥ p2
⊢ v1 +ᵥ p1 ∈ ↑s2
[PROOFSTEP]
rw [hv1v2]
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
he : ↑s1 ∩ ↑s2 = ∅
p1 : P
hp1 : p1 ∈ ↑s1
p2 : P
hp2 : p2 ∈ ↑s2
v1 : V
hv1 : v1 ∈ direction s1
v2 : V
hv2 : v2 ∈ direction s2
hv1v2✝ : v1 + v2 = p2 -ᵥ p1
hv1v2 : v1 +ᵥ p1 = -v2 +ᵥ p2
⊢ -v2 +ᵥ p2 ∈ ↑s2
[PROOFSTEP]
exact vadd_mem_of_mem_direction (Submodule.neg_mem _ hv2) hp2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : direction s1 ⊔ direction s2 = ⊤
⊢ Set.Nonempty (↑s1 ∩ ↑s2)
[PROOFSTEP]
by_contra h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : direction s1 ⊔ direction s2 = ⊤
h : ¬Set.Nonempty (↑s1 ∩ ↑s2)
⊢ False
[PROOFSTEP]
rw [Set.not_nonempty_iff_eq_empty] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : direction s1 ⊔ direction s2 = ⊤
h : ↑s1 ∩ ↑s2 = ∅
⊢ False
[PROOFSTEP]
have hlt := sup_direction_lt_of_nonempty_of_inter_empty h1 h2 h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : direction s1 ⊔ direction s2 = ⊤
h : ↑s1 ∩ ↑s2 = ∅
hlt : direction s1 ⊔ direction s2 < direction (s1 ⊔ s2)
⊢ False
[PROOFSTEP]
rw [hd] at hlt
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : direction s1 ⊔ direction s2 = ⊤
h : ↑s1 ∩ ↑s2 = ∅
hlt : ⊤ < direction (s1 ⊔ s2)
⊢ False
[PROOFSTEP]
exact not_top_lt hlt
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
⊢ ∃ p, ↑s1 ∩ ↑s2 = {p}
[PROOFSTEP]
cases' inter_nonempty_of_nonempty_of_sup_direction_eq_top h1 h2 hd.sup_eq_top with p hp
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
⊢ ∃ p, ↑s1 ∩ ↑s2 = {p}
[PROOFSTEP]
use p
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
⊢ ↑s1 ∩ ↑s2 = {p}
[PROOFSTEP]
ext q
[GOAL]
case h.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
q : P
⊢ q ∈ ↑s1 ∩ ↑s2 ↔ q ∈ {p}
[PROOFSTEP]
rw [Set.mem_singleton_iff]
[GOAL]
case h.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
q : P
⊢ q ∈ ↑s1 ∩ ↑s2 ↔ q = p
[PROOFSTEP]
constructor
[GOAL]
case h.h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
q : P
⊢ q ∈ ↑s1 ∩ ↑s2 → q = p
[PROOFSTEP]
rintro ⟨hq1, hq2⟩
[GOAL]
case h.h.mp.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
q : P
hq1 : q ∈ ↑s1
hq2 : q ∈ ↑s2
⊢ q = p
[PROOFSTEP]
have hqp : q -ᵥ p ∈ s1.direction ⊓ s2.direction := ⟨vsub_mem_direction hq1 hp.1, vsub_mem_direction hq2 hp.2⟩
[GOAL]
case h.h.mp.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
q : P
hq1 : q ∈ ↑s1
hq2 : q ∈ ↑s2
hqp : q -ᵥ p ∈ direction s1 ⊓ direction s2
⊢ q = p
[PROOFSTEP]
rwa [hd.inf_eq_bot, Submodule.mem_bot, vsub_eq_zero_iff_eq] at hqp
[GOAL]
case h.h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s1 s2 : AffineSubspace k P
h1 : Set.Nonempty ↑s1
h2 : Set.Nonempty ↑s2
hd : IsCompl (direction s1) (direction s2)
p : P
hp : p ∈ ↑s1 ∩ ↑s2
q : P
⊢ q = p → q ∈ ↑s1 ∩ ↑s2
[PROOFSTEP]
exact fun h => h.symm ▸ hp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
⊢ affineSpan k ↑s = s
[PROOFSTEP]
refine' le_antisymm _ (subset_spanPoints _ _)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
⊢ affineSpan k ↑s ≤ s
[PROOFSTEP]
rintro p ⟨p1, hp1, v, hv, rfl⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
p₁ p₂ : P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
v : V
hv : v ∈ vectorSpan k ↑s
⊢ v +ᵥ p1 ∈ ↑s
[PROOFSTEP]
exact vadd_mem_of_mem_direction hv hp1
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ vectorSpan k s = Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' s)
[PROOFSTEP]
rw [vectorSpan_def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ Submodule.span k (s -ᵥ s) = Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' s)
[PROOFSTEP]
refine' le_antisymm _ (Submodule.span_mono _)
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ Submodule.span k (s -ᵥ s) ≤ Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' s)
[PROOFSTEP]
rw [Submodule.span_le]
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ s -ᵥ s ⊆ ↑(Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' s))
[PROOFSTEP]
rintro v ⟨p1, p2, hp1, hp2, hv⟩
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p1 p2 : P
hp1 : p1 ∈ s
hp2 : p2 ∈ s
hv : (fun x x_1 => x -ᵥ x_1) p1 p2 = v
⊢ v ∈ ↑(Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' s))
[PROOFSTEP]
simp_rw [← vsub_sub_vsub_cancel_left p1 p2 p] at hv
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p1 p2 : P
hp1 : p1 ∈ s
hp2 : p2 ∈ s
hv : p -ᵥ p2 - (p -ᵥ p1) = v
⊢ v ∈ ↑(Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' s))
[PROOFSTEP]
rw [← hv, SetLike.mem_coe, Submodule.mem_span]
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p1 p2 : P
hp1 : p1 ∈ s
hp2 : p2 ∈ s
hv : p -ᵥ p2 - (p -ᵥ p1) = v
⊢ ∀ (p_1 : Submodule k V), (fun x x_1 => x -ᵥ x_1) p '' s ⊆ ↑p_1 → p -ᵥ p2 - (p -ᵥ p1) ∈ p_1
[PROOFSTEP]
exact fun m hm => Submodule.sub_mem _ (hm ⟨p2, hp2, rfl⟩) (hm ⟨p1, hp1, rfl⟩)
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ (fun x x_1 => x -ᵥ x_1) p '' s ⊆ s -ᵥ s
[PROOFSTEP]
rintro v ⟨p2, hp2, hv⟩
[GOAL]
case refine'_2.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p2 : P
hp2 : p2 ∈ s
hv : (fun x x_1 => x -ᵥ x_1) p p2 = v
⊢ v ∈ s -ᵥ s
[PROOFSTEP]
exact ⟨p, p2, hp, hp2, hv⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ vectorSpan k s = Submodule.span k ((fun x => x -ᵥ p) '' s)
[PROOFSTEP]
rw [vectorSpan_def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ Submodule.span k (s -ᵥ s) = Submodule.span k ((fun x => x -ᵥ p) '' s)
[PROOFSTEP]
refine' le_antisymm _ (Submodule.span_mono _)
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ Submodule.span k (s -ᵥ s) ≤ Submodule.span k ((fun x => x -ᵥ p) '' s)
[PROOFSTEP]
rw [Submodule.span_le]
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ s -ᵥ s ⊆ ↑(Submodule.span k ((fun x => x -ᵥ p) '' s))
[PROOFSTEP]
rintro v ⟨p1, p2, hp1, hp2, hv⟩
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p1 p2 : P
hp1 : p1 ∈ s
hp2 : p2 ∈ s
hv : (fun x x_1 => x -ᵥ x_1) p1 p2 = v
⊢ v ∈ ↑(Submodule.span k ((fun x => x -ᵥ p) '' s))
[PROOFSTEP]
simp_rw [← vsub_sub_vsub_cancel_right p1 p2 p] at hv
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p1 p2 : P
hp1 : p1 ∈ s
hp2 : p2 ∈ s
hv : p1 -ᵥ p - (p2 -ᵥ p) = v
⊢ v ∈ ↑(Submodule.span k ((fun x => x -ᵥ p) '' s))
[PROOFSTEP]
rw [← hv, SetLike.mem_coe, Submodule.mem_span]
[GOAL]
case refine'_1.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p1 p2 : P
hp1 : p1 ∈ s
hp2 : p2 ∈ s
hv : p1 -ᵥ p - (p2 -ᵥ p) = v
⊢ ∀ (p_1 : Submodule k V), (fun x => x -ᵥ p) '' s ⊆ ↑p_1 → p1 -ᵥ p - (p2 -ᵥ p) ∈ p_1
[PROOFSTEP]
exact fun m hm => Submodule.sub_mem _ (hm ⟨p1, hp1, rfl⟩) (hm ⟨p2, hp2, rfl⟩)
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ (fun x => x -ᵥ p) '' s ⊆ s -ᵥ s
[PROOFSTEP]
rintro v ⟨p2, hp2, hv⟩
[GOAL]
case refine'_2.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
v : V
p2 : P
hp2 : p2 ∈ s
hv : (fun x => x -ᵥ p) p2 = v
⊢ v ∈ s -ᵥ s
[PROOFSTEP]
exact ⟨p2, p, hp2, hp, hv⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ vectorSpan k s = Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' (s \ {p}))
[PROOFSTEP]
conv_lhs =>
rw [vectorSpan_eq_span_vsub_set_left k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton,
Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
| vectorSpan k s
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
| vectorSpan k s
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
| vectorSpan k s
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ Submodule.span k (insert ((fun x x_1 => x -ᵥ x_1) p p) ((fun x x_1 => x -ᵥ x_1) p '' (s \ {p}))) =
Submodule.span k ((fun x x_1 => x -ᵥ x_1) p '' (s \ {p}))
[PROOFSTEP]
simp [Submodule.span_insert_eq_span]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ vectorSpan k s = Submodule.span k ((fun x => x -ᵥ p) '' (s \ {p}))
[PROOFSTEP]
conv_lhs =>
rw [vectorSpan_eq_span_vsub_set_right k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton,
Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
| vectorSpan k s
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
| vectorSpan k s
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
| vectorSpan k s
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k hp, ← Set.insert_eq_of_mem hp, ← Set.insert_diff_singleton, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ Submodule.span k (insert (p -ᵥ p) ((fun x => x -ᵥ p) '' (s \ {p}))) =
Submodule.span k ((fun x => x -ᵥ p) '' (s \ {p}))
[PROOFSTEP]
simp [Submodule.span_insert_eq_span]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : Ring k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
inst✝¹ : DecidableEq P
inst✝ : DecidableEq V
s : Finset P
p : P
hp : p ∈ s
⊢ vectorSpan k ↑s = Submodule.span k ↑(Finset.image (fun x => x -ᵥ p) (Finset.erase s p))
[PROOFSTEP]
simp [vectorSpan_eq_span_vsub_set_right_ne _ (Finset.mem_coe.mpr hp)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
⊢ vectorSpan k (p '' s) = Submodule.span k ((fun x x_1 => x -ᵥ x_1) (p i) '' (p '' (s \ {i})))
[PROOFSTEP]
conv_lhs =>
rw [vectorSpan_eq_span_vsub_set_left k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
| vectorSpan k (p '' s)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
| vectorSpan k (p '' s)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
| vectorSpan k (p '' s)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
⊢ Submodule.span k (insert ((fun x x_1 => x -ᵥ x_1) (p i) (p i)) ((fun x x_1 => x -ᵥ x_1) (p i) '' (p '' (s \ {i})))) =
Submodule.span k ((fun x x_1 => x -ᵥ x_1) (p i) '' (p '' (s \ {i})))
[PROOFSTEP]
simp [Submodule.span_insert_eq_span]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
⊢ vectorSpan k (p '' s) = Submodule.span k ((fun x => x -ᵥ p i) '' (p '' (s \ {i})))
[PROOFSTEP]
conv_lhs =>
rw [vectorSpan_eq_span_vsub_set_right k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
| vectorSpan k (p '' s)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
| vectorSpan k (p '' s)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
| vectorSpan k (p '' s)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k (Set.mem_image_of_mem p hi), ← Set.insert_eq_of_mem hi, ←
Set.insert_diff_singleton, Set.image_insert_eq, Set.image_insert_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Set ι
i : ι
hi : i ∈ s
⊢ Submodule.span k (insert (p i -ᵥ p i) ((fun x => x -ᵥ p i) '' (p '' (s \ {i})))) =
Submodule.span k ((fun x => x -ᵥ p i) '' (p '' (s \ {i})))
[PROOFSTEP]
simp [Submodule.span_insert_eq_span]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i0 : ι
⊢ vectorSpan k (range p) = Submodule.span k (range fun i => p i0 -ᵥ p i)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_left k (Set.mem_range_self i0), ← Set.range_comp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i0 : ι
⊢ Submodule.span k (range ((fun x x_1 => x -ᵥ x_1) (p i0) ∘ p)) = Submodule.span k (range fun i => p i0 -ᵥ p i)
[PROOFSTEP]
congr
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i0 : ι
⊢ vectorSpan k (range p) = Submodule.span k (range fun i => p i -ᵥ p i0)
[PROOFSTEP]
rw [vectorSpan_eq_span_vsub_set_right k (Set.mem_range_self i0), ← Set.range_comp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i0 : ι
⊢ Submodule.span k (range ((fun x => x -ᵥ p i0) ∘ p)) = Submodule.span k (range fun i => p i -ᵥ p i0)
[PROOFSTEP]
congr
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
⊢ vectorSpan k (range p) = Submodule.span k (range fun i => p i₀ -ᵥ p ↑i)
[PROOFSTEP]
rw [← Set.image_univ, vectorSpan_image_eq_span_vsub_set_left_ne k _ (Set.mem_univ i₀)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
⊢ Submodule.span k ((fun x x_1 => x -ᵥ x_1) (p i₀) '' (p '' (univ \ {i₀}))) =
Submodule.span k (range fun i => p i₀ -ᵥ p ↑i)
[PROOFSTEP]
congr with v
[GOAL]
case e_s.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ v ∈ (fun x x_1 => x -ᵥ x_1) (p i₀) '' (p '' (univ \ {i₀})) ↔ v ∈ range fun i => p i₀ -ᵥ p ↑i
[PROOFSTEP]
simp only [Set.mem_range, Set.mem_image, Set.mem_diff, Set.mem_singleton_iff, Subtype.exists, Subtype.coe_mk]
[GOAL]
case e_s.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ (∃ x, (∃ x_1, (x_1 ∈ univ ∧ ¬x_1 = i₀) ∧ p x_1 = x) ∧ p i₀ -ᵥ x = v) ↔ ∃ a h, p i₀ -ᵥ p a = v
[PROOFSTEP]
constructor
[GOAL]
case e_s.h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ (∃ x, (∃ x_1, (x_1 ∈ univ ∧ ¬x_1 = i₀) ∧ p x_1 = x) ∧ p i₀ -ᵥ x = v) → ∃ a h, p i₀ -ᵥ p a = v
[PROOFSTEP]
rintro ⟨x, ⟨i₁, ⟨⟨_, hi₁⟩, rfl⟩⟩, hv⟩
[GOAL]
case e_s.h.mp.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
i₁ : ι
left✝ : i₁ ∈ univ
hi₁ : ¬i₁ = i₀
hv : p i₀ -ᵥ p i₁ = v
⊢ ∃ a h, p i₀ -ᵥ p a = v
[PROOFSTEP]
exact ⟨i₁, hi₁, hv⟩
[GOAL]
case e_s.h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ (∃ a h, p i₀ -ᵥ p a = v) → ∃ x, (∃ x_1, (x_1 ∈ univ ∧ ¬x_1 = i₀) ∧ p x_1 = x) ∧ p i₀ -ᵥ x = v
[PROOFSTEP]
exact fun ⟨i₁, hi₁, hv⟩ => ⟨p i₁, ⟨i₁, ⟨Set.mem_univ _, hi₁⟩, rfl⟩, hv⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
⊢ vectorSpan k (range p) = Submodule.span k (range fun i => p ↑i -ᵥ p i₀)
[PROOFSTEP]
rw [← Set.image_univ, vectorSpan_image_eq_span_vsub_set_right_ne k _ (Set.mem_univ i₀)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
⊢ Submodule.span k ((fun x => x -ᵥ p i₀) '' (p '' (univ \ {i₀}))) = Submodule.span k (range fun i => p ↑i -ᵥ p i₀)
[PROOFSTEP]
congr with v
[GOAL]
case e_s.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ v ∈ (fun x => x -ᵥ p i₀) '' (p '' (univ \ {i₀})) ↔ v ∈ range fun i => p ↑i -ᵥ p i₀
[PROOFSTEP]
simp only [Set.mem_range, Set.mem_image, Set.mem_diff, Set.mem_singleton_iff, Subtype.exists, Subtype.coe_mk]
[GOAL]
case e_s.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ (∃ x, (∃ x_1, (x_1 ∈ univ ∧ ¬x_1 = i₀) ∧ p x_1 = x) ∧ x -ᵥ p i₀ = v) ↔ ∃ a h, p a -ᵥ p i₀ = v
[PROOFSTEP]
constructor
[GOAL]
case e_s.h.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ (∃ x, (∃ x_1, (x_1 ∈ univ ∧ ¬x_1 = i₀) ∧ p x_1 = x) ∧ x -ᵥ p i₀ = v) → ∃ a h, p a -ᵥ p i₀ = v
[PROOFSTEP]
rintro ⟨x, ⟨i₁, ⟨⟨_, hi₁⟩, rfl⟩⟩, hv⟩
[GOAL]
case e_s.h.mp.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
i₁ : ι
left✝ : i₁ ∈ univ
hi₁ : ¬i₁ = i₀
hv : p i₁ -ᵥ p i₀ = v
⊢ ∃ a h, p a -ᵥ p i₀ = v
[PROOFSTEP]
exact ⟨i₁, hi₁, hv⟩
[GOAL]
case e_s.h.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i₀ : ι
v : V
⊢ (∃ a h, p a -ᵥ p i₀ = v) → ∃ x, (∃ x_1, (x_1 ∈ univ ∧ ¬x_1 = i₀) ∧ p x_1 = x) ∧ x -ᵥ p i₀ = v
[PROOFSTEP]
exact fun ⟨i₁, hi₁, hv⟩ => ⟨p i₁, ⟨i₁, ⟨Set.mem_univ _, hi₁⟩, rfl⟩, hv⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
⊢ affineSpan k s = ⊥ ↔ s = ∅
[PROOFSTEP]
rw [← not_iff_not, ← Ne.def, ← Ne.def, ← nonempty_iff_ne_bot, affineSpan_nonempty, nonempty_iff_ne_empty]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
⊢ ⊥ < affineSpan k s ↔ Set.Nonempty s
[PROOFSTEP]
rw [bot_lt_iff_ne_bot, nonempty_iff_ne_empty]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
⊢ affineSpan k s ≠ ⊥ ↔ s ≠ ∅
[PROOFSTEP]
exact (affineSpan_eq_bot _).not
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : (x : P) → x ∈ affineSpan k s → Prop
Hs : ∀ (y : P) (hys : y ∈ s), p y (_ : y ∈ ↑(affineSpan k s))
Hc :
∀ (c : k) (u : P) (hu : u ∈ affineSpan k s) (v : P) (hv : v ∈ affineSpan k s) (w : P) (hw : w ∈ affineSpan k s),
p u hu → p v hv → p w hw → p (c • (u -ᵥ v) +ᵥ w) (_ : c • (u -ᵥ v) +ᵥ w ∈ (affineSpan k s).carrier)
x : P
h : x ∈ affineSpan k s
⊢ p x h
[PROOFSTEP]
refine' Exists.elim _ fun (hx : x ∈ affineSpan k s) (hc : p x hx) => hc
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : (x : P) → x ∈ affineSpan k s → Prop
Hs : ∀ (y : P) (hys : y ∈ s), p y (_ : y ∈ ↑(affineSpan k s))
Hc :
∀ (c : k) (u : P) (hu : u ∈ affineSpan k s) (v : P) (hv : v ∈ affineSpan k s) (w : P) (hw : w ∈ affineSpan k s),
p u hu → p v hv → p w hw → p (c • (u -ᵥ v) +ᵥ w) (_ : c • (u -ᵥ v) +ᵥ w ∈ (affineSpan k s).carrier)
x : P
h : x ∈ affineSpan k s
⊢ ∃ x_1, p x x_1
[PROOFSTEP]
refine' @affineSpan_induction k V P _ _ _ _ _ _ (fun y => ∃ z, p y z) h _ _
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : (x : P) → x ∈ affineSpan k s → Prop
Hs : ∀ (y : P) (hys : y ∈ s), p y (_ : y ∈ ↑(affineSpan k s))
Hc :
∀ (c : k) (u : P) (hu : u ∈ affineSpan k s) (v : P) (hv : v ∈ affineSpan k s) (w : P) (hw : w ∈ affineSpan k s),
p u hu → p v hv → p w hw → p (c • (u -ᵥ v) +ᵥ w) (_ : c • (u -ᵥ v) +ᵥ w ∈ (affineSpan k s).carrier)
x : P
h : x ∈ affineSpan k s
⊢ ∀ (x : P), x ∈ s → (fun y => ∃ z, p y z) x
[PROOFSTEP]
exact fun y hy => ⟨subset_affineSpan _ _ hy, Hs y hy⟩
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : (x : P) → x ∈ affineSpan k s → Prop
Hs : ∀ (y : P) (hys : y ∈ s), p y (_ : y ∈ ↑(affineSpan k s))
Hc :
∀ (c : k) (u : P) (hu : u ∈ affineSpan k s) (v : P) (hv : v ∈ affineSpan k s) (w : P) (hw : w ∈ affineSpan k s),
p u hu → p v hv → p w hw → p (c • (u -ᵥ v) +ᵥ w) (_ : c • (u -ᵥ v) +ᵥ w ∈ (affineSpan k s).carrier)
x : P
h : x ∈ affineSpan k s
⊢ ∀ (c : k) (u v w : P),
(fun y => ∃ z, p y z) u →
(fun y => ∃ z, p y z) v → (fun y => ∃ z, p y z) w → (fun y => ∃ z, p y z) (c • (u -ᵥ v) +ᵥ w)
[PROOFSTEP]
exact fun c u v w hu hv hw =>
Exists.elim hu fun hu' hu =>
Exists.elim hv fun hv' hv =>
Exists.elim hw fun hw' hw => ⟨AffineSubspace.smul_vsub_vadd_mem _ _ hu' hv' hw', Hc _ _ _ _ _ _ _ hu hv hw⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
A : Set P
inst✝ : Nonempty ↑A
⊢ affineSpan k (Subtype.val ⁻¹' A) = ⊤
[PROOFSTEP]
rw [eq_top_iff]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
A : Set P
inst✝ : Nonempty ↑A
⊢ ⊤ ≤ affineSpan k (Subtype.val ⁻¹' A)
[PROOFSTEP]
rintro ⟨x, hx⟩ -
[GOAL]
case mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
A : Set P
inst✝ : Nonempty ↑A
x : P
hx : x ∈ ↑(affineSpan k A)
⊢ { val := x, property := hx } ∈ ↑(affineSpan k (Subtype.val ⁻¹' A))
[PROOFSTEP]
refine'
affineSpan_induction' (fun y hy => _) (fun c u hu v hv w hw => _) hx (p := fun y hy =>
⟨y, hy⟩ ∈ (affineSpan k (((↑) : { z // z ∈ affineSpan k A } → P) ⁻¹' A)))
-- porting note: Lean couldn't infer the motive
[GOAL]
case mk.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
A : Set P
inst✝ : Nonempty ↑A
x : P
hx : x ∈ ↑(affineSpan k A)
y : P
hy : y ∈ A
⊢ (fun y hy => { val := y, property := hy } ∈ affineSpan k (Subtype.val ⁻¹' A)) y (_ : y ∈ ↑(affineSpan k A))
[PROOFSTEP]
exact subset_affineSpan _ _ hy
[GOAL]
case mk.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
A : Set P
inst✝ : Nonempty ↑A
x : P
hx : x ∈ ↑(affineSpan k A)
c : k
u : P
hu : u ∈ affineSpan k A
v : P
hv : v ∈ affineSpan k A
w : P
hw : w ∈ affineSpan k A
⊢ (fun y hy => { val := y, property := hy } ∈ affineSpan k (Subtype.val ⁻¹' A)) u hu →
(fun y hy => { val := y, property := hy } ∈ affineSpan k (Subtype.val ⁻¹' A)) v hv →
(fun y hy => { val := y, property := hy } ∈ affineSpan k (Subtype.val ⁻¹' A)) w hw →
(fun y hy => { val := y, property := hy } ∈ affineSpan k (Subtype.val ⁻¹' A)) (c • (u -ᵥ v) +ᵥ w)
(_ : c • (u -ᵥ v) +ᵥ w ∈ (affineSpan k A).carrier)
[PROOFSTEP]
exact AffineSubspace.smul_vsub_vadd_mem _ _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
p : P
h : Submodule.span k (range Subtype.val) = ⊤
⊢ affineSpan k ({p} ∪ (fun v => v +ᵥ p) '' s) = ⊤
[PROOFSTEP]
convert ext_of_direction_eq _ ⟨p, mem_affineSpan k (Set.mem_union_left _ (Set.mem_singleton _)), mem_top k V p⟩
[GOAL]
case convert_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
p : P
h : Submodule.span k (range Subtype.val) = ⊤
⊢ direction (affineSpan k ({p} ∪ (fun v => v +ᵥ p) '' s)) = direction ⊤
[PROOFSTEP]
rw [direction_affineSpan, direction_top,
vectorSpan_eq_span_vsub_set_right k (Set.mem_union_left _ (Set.mem_singleton _) : p ∈ _), eq_top_iff, ← h]
[GOAL]
case convert_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
p : P
h : Submodule.span k (range Subtype.val) = ⊤
⊢ Submodule.span k (range Subtype.val) ≤ Submodule.span k ((fun x => x -ᵥ p) '' ({p} ∪ (fun v => v +ᵥ p) '' s))
[PROOFSTEP]
apply Submodule.span_mono
[GOAL]
case convert_1.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
p : P
h : Submodule.span k (range Subtype.val) = ⊤
⊢ range Subtype.val ⊆ (fun x => x -ᵥ p) '' ({p} ∪ (fun v => v +ᵥ p) '' s)
[PROOFSTEP]
rintro v ⟨v', rfl⟩
[GOAL]
case convert_1.h.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
p : P
h : Submodule.span k (range Subtype.val) = ⊤
v' : { x // x ∈ s }
⊢ ↑v' ∈ (fun x => x -ᵥ p) '' ({p} ∪ (fun v => v +ᵥ p) '' s)
[PROOFSTEP]
use(v' : V) +ᵥ p
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
p : P
h : Submodule.span k (range Subtype.val) = ⊤
v' : { x // x ∈ s }
⊢ ↑v' +ᵥ p ∈ {p} ∪ (fun v => v +ᵥ p) '' s ∧ (fun x => x -ᵥ p) (↑v' +ᵥ p) = ↑v'
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
⊢ vectorSpan k {p₁, p₂} = Submodule.span k {p₁ -ᵥ p₂}
[PROOFSTEP]
simp_rw [vectorSpan_eq_span_vsub_set_left k (mem_insert p₁ _), image_pair, vsub_self, Submodule.span_insert_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
⊢ vectorSpan k {p₁, p₂} = Submodule.span k {p₂ -ᵥ p₁}
[PROOFSTEP]
rw [pair_comm, vectorSpan_pair]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
v : V
⊢ v ∈ vectorSpan k {p₁, p₂} ↔ ∃ r, r • (p₁ -ᵥ p₂) = v
[PROOFSTEP]
rw [vectorSpan_pair, Submodule.mem_span_singleton]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
v : V
⊢ v ∈ vectorSpan k {p₁, p₂} ↔ ∃ r, r • (p₂ -ᵥ p₁) = v
[PROOFSTEP]
rw [vectorSpan_pair_rev, Submodule.mem_span_singleton]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
v : V
⊢ v +ᵥ p₁ ∈ affineSpan k {p₁, p₂} ↔ ∃ r, r • (p₂ -ᵥ p₁) = v
[PROOFSTEP]
rw [vadd_mem_iff_mem_direction _ (left_mem_affineSpan_pair _ _ _), direction_affineSpan, mem_vectorSpan_pair_rev]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
v : V
⊢ v +ᵥ p₂ ∈ affineSpan k {p₁, p₂} ↔ ∃ r, r • (p₁ -ᵥ p₂) = v
[PROOFSTEP]
rw [vadd_mem_iff_mem_direction _ (right_mem_affineSpan_pair _ _ _), direction_affineSpan, mem_vectorSpan_pair]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
s : AffineSubspace k P
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
⊢ affineSpan k {p₁, p₂} ≤ s
[PROOFSTEP]
rw [affineSpan_le, Set.insert_subset_iff, Set.singleton_subset_iff]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
s : AffineSubspace k P
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
⊢ p₁ ∈ ↑s ∧ p₂ ∈ ↑s
[PROOFSTEP]
exact ⟨hp₁, hp₂⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : P
ps : Set P
⊢ affineSpan k (insert p ↑(affineSpan k ps)) = affineSpan k (insert p ps)
[PROOFSTEP]
rw [Set.insert_eq, Set.insert_eq, span_union, span_union, affineSpan_coe]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : P
ps : Set P
h : p ∈ affineSpan k ps
⊢ affineSpan k (insert p ps) = affineSpan k ps
[PROOFSTEP]
rw [← mem_coe] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : P
ps : Set P
h : p ∈ ↑(affineSpan k ps)
⊢ affineSpan k (insert p ps) = affineSpan k ps
[PROOFSTEP]
rw [← affineSpan_insert_affineSpan, Set.insert_eq_of_mem h, affineSpan_coe]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : P
ps : Set P
h : p ∈ affineSpan k ps
⊢ vectorSpan k (insert p ps) = vectorSpan k ps
[PROOFSTEP]
simp_rw [← direction_affineSpan, affineSpan_insert_eq_affineSpan _ h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s1
hp2 : p2 ∈ s2
⊢ direction (s1 ⊔ s2) = direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
refine' le_antisymm _ _
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s1
hp2 : p2 ∈ s2
⊢ direction (s1 ⊔ s2) ≤ direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
change (affineSpan k ((s1 : Set P) ∪ s2)).direction ≤ _
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s1
hp2 : p2 ∈ s2
⊢ direction (affineSpan k (↑s1 ∪ ↑s2)) ≤ direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
rw [← mem_coe] at hp1
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
⊢ direction (affineSpan k (↑s1 ∪ ↑s2)) ≤ direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
rw [direction_affineSpan, vectorSpan_eq_span_vsub_set_right k (Set.mem_union_left _ hp1), Submodule.span_le]
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
⊢ (fun x => x -ᵥ p1) '' (↑s1 ∪ ↑s2) ⊆ ↑(direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1})
[PROOFSTEP]
rintro v ⟨p3, hp3, rfl⟩
[GOAL]
case refine'_1.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s1 ∪ ↑s2
⊢ (fun x => x -ᵥ p1) p3 ∈ ↑(direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1})
[PROOFSTEP]
cases' hp3 with hp3 hp3
[GOAL]
case refine'_1.intro.intro.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s1
⊢ (fun x => x -ᵥ p1) p3 ∈ ↑(direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1})
[PROOFSTEP]
rw [sup_assoc, sup_comm, SetLike.mem_coe, Submodule.mem_sup]
[GOAL]
case refine'_1.intro.intro.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s1
⊢ ∃ y, y ∈ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1} ∧ ∃ z, z ∈ direction s1 ∧ y + z = (fun x => x -ᵥ p1) p3
[PROOFSTEP]
use 0, Submodule.zero_mem _, p3 -ᵥ p1, vsub_mem_direction hp3 hp1
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s1
⊢ 0 + (p3 -ᵥ p1) = (fun x => x -ᵥ p1) p3
[PROOFSTEP]
rw [zero_add]
[GOAL]
case refine'_1.intro.intro.inr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s2
⊢ (fun x => x -ᵥ p1) p3 ∈ ↑(direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1})
[PROOFSTEP]
rw [sup_assoc, SetLike.mem_coe, Submodule.mem_sup]
[GOAL]
case refine'_1.intro.intro.inr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s2
⊢ ∃ y, y ∈ direction s1 ∧ ∃ z, z ∈ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1} ∧ y + z = (fun x => x -ᵥ p1) p3
[PROOFSTEP]
use 0, Submodule.zero_mem _, p3 -ᵥ p1
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s2
⊢ p3 -ᵥ p1 ∈ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1} ∧ 0 + (p3 -ᵥ p1) = (fun x => x -ᵥ p1) p3
[PROOFSTEP]
rw [and_comm, zero_add]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s2
⊢ p3 -ᵥ p1 = (fun x => x -ᵥ p1) p3 ∧ p3 -ᵥ p1 ∈ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
use rfl
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s2
⊢ p3 -ᵥ p1 ∈ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
rw [← vsub_add_vsub_cancel p3 p2 p1, Submodule.mem_sup]
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ ↑s1
hp2 : p2 ∈ s2
p3 : P
hp3 : p3 ∈ ↑s2
⊢ ∃ y, y ∈ direction s2 ∧ ∃ z, z ∈ Submodule.span k {p2 -ᵥ p1} ∧ y + z = p3 -ᵥ p2 + (p2 -ᵥ p1)
[PROOFSTEP]
use p3 -ᵥ p2, vsub_mem_direction hp3 hp2, p2 -ᵥ p1, Submodule.mem_span_singleton_self _
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s1
hp2 : p2 ∈ s2
⊢ direction s1 ⊔ direction s2 ⊔ Submodule.span k {p2 -ᵥ p1} ≤ direction (s1 ⊔ s2)
[PROOFSTEP]
refine' sup_le (sup_direction_le _ _) _
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s1
hp2 : p2 ∈ s2
⊢ Submodule.span k {p2 -ᵥ p1} ≤ direction (s1 ⊔ s2)
[PROOFSTEP]
rw [direction_eq_vectorSpan, vectorSpan_def]
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s1 s2 : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s1
hp2 : p2 ∈ s2
⊢ Submodule.span k {p2 -ᵥ p1} ≤ Submodule.span k (↑(s1 ⊔ s2) -ᵥ ↑(s1 ⊔ s2))
[PROOFSTEP]
exact
sInf_le_sInf fun p hp =>
Set.Subset.trans
(Set.singleton_subset_iff.2
(vsub_mem_vsub (mem_spanPoints k p2 _ (Set.mem_union_right _ hp2))
(mem_spanPoints k p1 _ (Set.mem_union_left _ hp1))))
hp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s
⊢ direction (affineSpan k (insert p2 ↑s)) = Submodule.span k {p2 -ᵥ p1} ⊔ direction s
[PROOFSTEP]
rw [sup_comm, ← Set.union_singleton, ← coe_affineSpan_singleton k V p2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s
⊢ direction (affineSpan k (↑s ∪ ↑(affineSpan k {p2}))) = direction s ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
change (s ⊔ affineSpan k { p2 }).direction = _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s
⊢ direction (s ⊔ affineSpan k {p2}) = direction s ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
rw [direction_sup hp1 (mem_affineSpan k (Set.mem_singleton _)), direction_affineSpan]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 p2 : P
hp1 : p1 ∈ s
⊢ direction s ⊔ vectorSpan k {p2} ⊔ Submodule.span k {p2 -ᵥ p1} = direction s ⊔ Submodule.span k {p2 -ᵥ p1}
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ s
p2 p : P
⊢ p ∈ affineSpan k (insert p2 ↑s) ↔ ∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
rw [← mem_coe] at hp1
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
⊢ p ∈ affineSpan k (insert p2 ↑s) ↔ ∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
rw [← vsub_right_mem_direction_iff_mem (mem_affineSpan k (Set.mem_insert_of_mem _ hp1)),
direction_affineSpan_insert hp1, Submodule.mem_sup]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
⊢ (∃ y, y ∈ Submodule.span k {p2 -ᵥ p1} ∧ ∃ z, z ∈ direction s ∧ y + z = p -ᵥ p1) ↔
∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
⊢ (∃ y, y ∈ Submodule.span k {p2 -ᵥ p1} ∧ ∃ z, z ∈ direction s ∧ y + z = p -ᵥ p1) →
∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
rintro ⟨v1, hv1, v2, hv2, hp⟩
[GOAL]
case mp.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
v1 : V
hv1 : v1 ∈ Submodule.span k {p2 -ᵥ p1}
v2 : V
hv2 : v2 ∈ direction s
hp : v1 + v2 = p -ᵥ p1
⊢ ∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
rw [Submodule.mem_span_singleton] at hv1
[GOAL]
case mp.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
v1 : V
hv1 : ∃ a, a • (p2 -ᵥ p1) = v1
v2 : V
hv2 : v2 ∈ direction s
hp : v1 + v2 = p -ᵥ p1
⊢ ∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
rcases hv1 with ⟨r, rfl⟩
[GOAL]
case mp.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
v2 : V
hv2 : v2 ∈ direction s
r : k
hp : r • (p2 -ᵥ p1) + v2 = p -ᵥ p1
⊢ ∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0
[PROOFSTEP]
use r, v2 +ᵥ p1, vadd_mem_of_mem_direction hv2 hp1
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
v2 : V
hv2 : v2 ∈ direction s
r : k
hp : r • (p2 -ᵥ p1) + v2 = p -ᵥ p1
⊢ p = r • (p2 -ᵥ p1) +ᵥ (v2 +ᵥ p1)
[PROOFSTEP]
symm at hp
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
v2 : V
hv2 : v2 ∈ direction s
r : k
hp : p -ᵥ p1 = r • (p2 -ᵥ p1) + v2
⊢ p = r • (p2 -ᵥ p1) +ᵥ (v2 +ᵥ p1)
[PROOFSTEP]
rw [← sub_eq_zero, ← vsub_vadd_eq_vsub_sub, vsub_eq_zero_iff_eq] at hp
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
v2 : V
hv2 : v2 ∈ direction s
r : k
hp✝ : p -ᵥ p1 = r • (p2 -ᵥ p1) + v2
hp : p = r • (p2 -ᵥ p1) + v2 +ᵥ p1
⊢ p = r • (p2 -ᵥ p1) +ᵥ (v2 +ᵥ p1)
[PROOFSTEP]
rw [hp, vadd_vadd]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 p : P
⊢ (∃ r p0 _hp0, p = r • (p2 -ᵥ p1) +ᵥ p0) →
∃ y, y ∈ Submodule.span k {p2 -ᵥ p1} ∧ ∃ z, z ∈ direction s ∧ y + z = p -ᵥ p1
[PROOFSTEP]
rintro ⟨r, p3, hp3, rfl⟩
[GOAL]
case mpr.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 : P
r : k
p3 : P
hp3 : p3 ∈ s
⊢ ∃ y, y ∈ Submodule.span k {p2 -ᵥ p1} ∧ ∃ z, z ∈ direction s ∧ y + z = r • (p2 -ᵥ p1) +ᵥ p3 -ᵥ p1
[PROOFSTEP]
use r • (p2 -ᵥ p1), Submodule.mem_span_singleton.2 ⟨r, rfl⟩, p3 -ᵥ p1, vsub_mem_direction hp3 hp1
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
p1 : P
hp1 : p1 ∈ ↑s
p2 : P
r : k
p3 : P
hp3 : p3 ∈ s
⊢ r • (p2 -ᵥ p1) + (p3 -ᵥ p1) = r • (p2 -ᵥ p1) +ᵥ p3 -ᵥ p1
[PROOFSTEP]
rw [vadd_vsub_assoc, add_comm]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
⊢ Submodule.map f.linear (vectorSpan k s) = vectorSpan k (↑f '' s)
[PROOFSTEP]
rw [vectorSpan_def, vectorSpan_def, f.image_vsub_image, Submodule.span_image]
-- porting note: Lean unfolds things too far with `simp` here.
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
⊢ ∀ (c : k) {p1 p2 p3 : P₂}, p1 ∈ ↑f '' ↑s → p2 ∈ ↑f '' ↑s → p3 ∈ ↑f '' ↑s → c • (p1 -ᵥ p2) +ᵥ p3 ∈ ↑f '' ↑s
[PROOFSTEP]
rintro t - - - ⟨p₁, h₁, rfl⟩ ⟨p₂, h₂, rfl⟩ ⟨p₃, h₃, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
t : k
p₁ : P₁
h₁ : p₁ ∈ ↑s
p₂ : P₁
h₂ : p₂ ∈ ↑s
p₃ : P₁
h₃ : p₃ ∈ ↑s
⊢ t • (↑f p₁ -ᵥ ↑f p₂) +ᵥ ↑f p₃ ∈ ↑f '' ↑s
[PROOFSTEP]
use t • (p₁ -ᵥ p₂) +ᵥ p₃
[GOAL]
case h
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
t : k
p₁ : P₁
h₁ : p₁ ∈ ↑s
p₂ : P₁
h₂ : p₂ ∈ ↑s
p₃ : P₁
h₃ : p₃ ∈ ↑s
⊢ t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ ↑s ∧ ↑f (t • (p₁ -ᵥ p₂) +ᵥ p₃) = t • (↑f p₁ -ᵥ ↑f p₂) +ᵥ ↑f p₃
[PROOFSTEP]
suffices t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ s by {
simp only [SetLike.mem_coe, true_and, this]
rw [AffineMap.map_vadd, map_smul, AffineMap.linearMap_vsub]
}
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
t : k
p₁ : P₁
h₁ : p₁ ∈ ↑s
p₂ : P₁
h₂ : p₂ ∈ ↑s
p₃ : P₁
h₃ : p₃ ∈ ↑s
this : t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ s
⊢ t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ ↑s ∧ ↑f (t • (p₁ -ᵥ p₂) +ᵥ p₃) = t • (↑f p₁ -ᵥ ↑f p₂) +ᵥ ↑f p₃
[PROOFSTEP]
{ simp only [SetLike.mem_coe, true_and, this]
rw [AffineMap.map_vadd, map_smul, AffineMap.linearMap_vsub]
}
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
t : k
p₁ : P₁
h₁ : p₁ ∈ ↑s
p₂ : P₁
h₂ : p₂ ∈ ↑s
p₃ : P₁
h₃ : p₃ ∈ ↑s
this : t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ s
⊢ t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ ↑s ∧ ↑f (t • (p₁ -ᵥ p₂) +ᵥ p₃) = t • (↑f p₁ -ᵥ ↑f p₂) +ᵥ ↑f p₃
[PROOFSTEP]
simp only [SetLike.mem_coe, true_and, this]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
t : k
p₁ : P₁
h₁ : p₁ ∈ ↑s
p₂ : P₁
h₂ : p₂ ∈ ↑s
p₃ : P₁
h₃ : p₃ ∈ ↑s
this : t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ s
⊢ ↑f (t • (p₁ -ᵥ p₂) +ᵥ p₃) = t • (↑f p₁ -ᵥ ↑f p₂) +ᵥ ↑f p₃
[PROOFSTEP]
rw [AffineMap.map_vadd, map_smul, AffineMap.linearMap_vsub]
[GOAL]
case h
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
t : k
p₁ : P₁
h₁ : p₁ ∈ ↑s
p₂ : P₁
h₂ : p₂ ∈ ↑s
p₃ : P₁
h₃ : p₃ ∈ ↑s
⊢ t • (p₁ -ᵥ p₂) +ᵥ p₃ ∈ s
[PROOFSTEP]
exact s.smul_vsub_vadd_mem t h₁ h₂ h₃
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f✝ f : P₁ →ᵃ[k] P₂
x : P₂
s : AffineSubspace k P₁
⊢ x ∈ map f s ↔ ∃ y, y ∈ s ∧ ↑f y = x
[PROOFSTEP]
simpa only [bex_def] using mem_image_iff_bex
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
⊢ map f s = ⊥ ↔ s = ⊥
[PROOFSTEP]
refine' ⟨fun h => _, fun h => _⟩
[GOAL]
case refine'_1
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
h : map f s = ⊥
⊢ s = ⊥
[PROOFSTEP]
rwa [← coe_eq_bot_iff, coe_map, image_eq_empty, coe_eq_bot_iff] at h
[GOAL]
case refine'_2
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
h : s = ⊥
⊢ map f s = ⊥
[PROOFSTEP]
rw [h, map_bot]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₁
⊢ direction (map f s) = Submodule.map f.linear (direction s)
[PROOFSTEP]
rw [direction_eq_vectorSpan, direction_eq_vectorSpan, coe_map, AffineMap.vectorSpan_image_eq_submodule_map]
-- porting note: again, Lean unfolds too aggressively with `simp`
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
⊢ map f (affineSpan k s) = affineSpan k (↑f '' s)
[PROOFSTEP]
rcases s.eq_empty_or_nonempty with (rfl | ⟨p, hp⟩)
[GOAL]
case inl
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
⊢ map f (affineSpan k ∅) = affineSpan k (↑f '' ∅)
[PROOFSTEP]
rw [image_empty, span_empty, span_empty, map_bot]
-- porting note: I don't know exactly why this `simp` was broken.
[GOAL]
case inr.intro
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
p : P₁
hp : p ∈ s
⊢ map f (affineSpan k s) = affineSpan k (↑f '' s)
[PROOFSTEP]
apply ext_of_direction_eq
[GOAL]
case inr.intro.hd
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
p : P₁
hp : p ∈ s
⊢ direction (map f (affineSpan k s)) = direction (affineSpan k (↑f '' s))
[PROOFSTEP]
simp [direction_affineSpan]
[GOAL]
case inr.intro.hn
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
p : P₁
hp : p ∈ s
⊢ Set.Nonempty (↑(map f (affineSpan k s)) ∩ ↑(affineSpan k (↑f '' s)))
[PROOFSTEP]
exact ⟨f p, mem_image_of_mem f (subset_affineSpan k _ hp), subset_affineSpan k _ (mem_image_of_mem f hp)⟩
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
hf : Function.Surjective ↑f
⊢ AffineSubspace.map f ⊤ = ⊤
[PROOFSTEP]
rw [← AffineSubspace.ext_iff]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
hf : Function.Surjective ↑f
⊢ ↑(AffineSubspace.map f ⊤) = ↑⊤
[PROOFSTEP]
exact image_univ_of_surjective hf
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
hf : Function.Surjective ↑f
h : affineSpan k s = ⊤
⊢ affineSpan k (↑f '' s) = ⊤
[PROOFSTEP]
rw [← AffineSubspace.map_span, h, map_top_of_surjective f hf]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
⊢ affineSpan k s = ⊤ ↔ affineSpan k (↑e '' s) = ⊤
[PROOFSTEP]
refine' ⟨(e : P₁ →ᵃ[k] P₂).span_eq_top_of_surjective e.surjective, _⟩
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
⊢ affineSpan k (↑e '' s) = ⊤ → affineSpan k s = ⊤
[PROOFSTEP]
intro h
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
h : affineSpan k (↑e '' s) = ⊤
⊢ affineSpan k s = ⊤
[PROOFSTEP]
have : s = e.symm '' (e '' s) := by rw [← image_comp]; simp
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
h : affineSpan k (↑e '' s) = ⊤
⊢ s = ↑(symm e) '' (↑e '' s)
[PROOFSTEP]
rw [← image_comp]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
h : affineSpan k (↑e '' s) = ⊤
⊢ s = ↑(symm e) ∘ ↑e '' s
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
h : affineSpan k (↑e '' s) = ⊤
this : s = ↑(symm e) '' (↑e '' s)
⊢ affineSpan k s = ⊤
[PROOFSTEP]
rw [this]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : Set P₁
e : P₁ ≃ᵃ[k] P₂
h : affineSpan k (↑e '' s) = ⊤
this : s = ↑(symm e) '' (↑e '' s)
⊢ affineSpan k (↑(symm e) '' (↑e '' s)) = ⊤
[PROOFSTEP]
exact (e.symm : P₂ →ᵃ[k] P₁).span_eq_top_of_surjective e.symm.surjective h
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₂
t : k
p₁ p₂ p₃ : P₁
hp₁ : ↑f p₁ ∈ s
hp₂ : ↑f p₂ ∈ s
hp₃ : ↑f p₃ ∈ s
⊢ ↑f (t • (p₁ -ᵥ p₂) +ᵥ p₃) ∈ s
[PROOFSTEP]
rw [AffineMap.map_vadd, LinearMap.map_smul, AffineMap.linearMap_vsub]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
s : AffineSubspace k P₂
t : k
p₁ p₂ p₃ : P₁
hp₁ : ↑f p₁ ∈ s
hp₂ : ↑f p₂ ∈ s
hp₃ : ↑f p₃ ∈ s
⊢ t • (↑f p₁ -ᵥ ↑f p₂) +ᵥ ↑f p₃ ∈ s
[PROOFSTEP]
apply s.smul_vsub_vadd_mem _ hp₁ hp₂ hp₃
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
⊢ comap f ⊤ = ⊤
[PROOFSTEP]
rw [← ext_iff]
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ →ᵃ[k] P₂
⊢ ↑(comap f ⊤) = ↑⊤
[PROOFSTEP]
exact preimage_univ (f := f)
[GOAL]
k : Type u_1
V₁ : Type u_2
P₁ : Type u_3
V₂ : Type u_4
P₂ : Type u_5
V₃ : Type u_6
P₃ : Type u_7
inst✝⁹ : Ring k
inst✝⁸ : AddCommGroup V₁
inst✝⁷ : Module k V₁
inst✝⁶ : AffineSpace V₁ P₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module k V₂
inst✝³ : AffineSpace V₂ P₂
inst✝² : AddCommGroup V₃
inst✝¹ : Module k V₃
inst✝ : AffineSpace V₃ P₃
f : P₁ ≃ᵃ[k] P₂
s : Set P₂
⊢ comap (↑f) (affineSpan k s) = affineSpan k (↑f ⁻¹' s)
[PROOFSTEP]
rw [← map_symm, map_span, AffineEquiv.coe_coe, f.image_symm]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
h : s₁ ∥ s₂
⊢ s₂ ∥ s₁
[PROOFSTEP]
rcases h with ⟨v, rfl⟩
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ : AffineSubspace k P
v : V
⊢ map (↑(constVAdd k P v)) s₁ ∥ s₁
[PROOFSTEP]
refine' ⟨-v, _⟩
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ : AffineSubspace k P
v : V
⊢ s₁ = map (↑(constVAdd k P (-v))) (map (↑(constVAdd k P v)) s₁)
[PROOFSTEP]
rw [map_map, ← coe_trans_to_affineMap, ← constVAdd_add, neg_add_self, constVAdd_zero, coe_refl_to_affineMap, map_id]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
⊢ s = map (↑(constVAdd k P 0)) s
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ s₃ : AffineSubspace k P
h₁₂ : s₁ ∥ s₂
h₂₃ : s₂ ∥ s₃
⊢ s₁ ∥ s₃
[PROOFSTEP]
rcases h₁₂ with ⟨v₁₂, rfl⟩
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₃ : AffineSubspace k P
v₁₂ : V
h₂₃ : map (↑(constVAdd k P v₁₂)) s₁ ∥ s₃
⊢ s₁ ∥ s₃
[PROOFSTEP]
rcases h₂₃ with ⟨v₂₃, rfl⟩
[GOAL]
case intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ : AffineSubspace k P
v₁₂ v₂₃ : V
⊢ s₁ ∥ map (↑(constVAdd k P v₂₃)) (map (↑(constVAdd k P v₁₂)) s₁)
[PROOFSTEP]
refine' ⟨v₂₃ + v₁₂, _⟩
[GOAL]
case intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ : AffineSubspace k P
v₁₂ v₂₃ : V
⊢ map (↑(constVAdd k P v₂₃)) (map (↑(constVAdd k P v₁₂)) s₁) = map (↑(constVAdd k P (v₂₃ + v₁₂))) s₁
[PROOFSTEP]
rw [map_map, ← coe_trans_to_affineMap, ← constVAdd_add]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
h : s₁ ∥ s₂
⊢ direction s₁ = direction s₂
[PROOFSTEP]
rcases h with ⟨v, rfl⟩
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ : AffineSubspace k P
v : V
⊢ direction s₁ = direction (map (↑(constVAdd k P v)) s₁)
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
⊢ s ∥ ⊥ ↔ s = ⊥
[PROOFSTEP]
refine' ⟨fun h => _, fun h => h ▸ Parallel.refl _⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
h : s ∥ ⊥
⊢ s = ⊥
[PROOFSTEP]
rcases h with ⟨v, h⟩
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
v : V
h : ⊥ = map (↑(constVAdd k P v)) s
⊢ s = ⊥
[PROOFSTEP]
rwa [eq_comm, map_eq_bot_iff] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s : AffineSubspace k P
⊢ ⊥ ∥ s ↔ s = ⊥
[PROOFSTEP]
rw [parallel_comm, parallel_bot_iff_eq_bot]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
⊢ s₁ ∥ s₂ ↔ direction s₁ = direction s₂ ∧ (s₁ = ⊥ ↔ s₂ = ⊥)
[PROOFSTEP]
refine' ⟨fun h => ⟨h.direction_eq, _, _⟩, fun h => _⟩
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
h : s₁ ∥ s₂
⊢ s₁ = ⊥ → s₂ = ⊥
[PROOFSTEP]
rintro rfl
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₂ : AffineSubspace k P
h : ⊥ ∥ s₂
⊢ s₂ = ⊥
[PROOFSTEP]
exact bot_parallel_iff_eq_bot.1 h
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
h : s₁ ∥ s₂
⊢ s₂ = ⊥ → s₁ = ⊥
[PROOFSTEP]
rintro rfl
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ : AffineSubspace k P
h : s₁ ∥ ⊥
⊢ s₁ = ⊥
[PROOFSTEP]
exact parallel_bot_iff_eq_bot.1 h
[GOAL]
case refine'_3
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
h : direction s₁ = direction s₂ ∧ (s₁ = ⊥ ↔ s₂ = ⊥)
⊢ s₁ ∥ s₂
[PROOFSTEP]
rcases h with ⟨hd, hb⟩
[GOAL]
case refine'_3.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
⊢ s₁ ∥ s₂
[PROOFSTEP]
by_cases hs₁ : s₁ = ⊥
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : s₁ = ⊥
⊢ s₁ ∥ s₂
[PROOFSTEP]
rw [hs₁, bot_parallel_iff_eq_bot]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : s₁ = ⊥
⊢ s₂ = ⊥
[PROOFSTEP]
exact hb.1 hs₁
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
⊢ s₁ ∥ s₂
[PROOFSTEP]
have hs₂ : s₂ ≠ ⊥ := hb.not.1 hs₁
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
⊢ s₁ ∥ s₂
[PROOFSTEP]
rcases(nonempty_iff_ne_bot s₁).2 hs₁ with ⟨p₁, hp₁⟩
[GOAL]
case neg.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
p₁ : P
hp₁ : p₁ ∈ ↑s₁
⊢ s₁ ∥ s₂
[PROOFSTEP]
rcases(nonempty_iff_ne_bot s₂).2 hs₂ with ⟨p₂, hp₂⟩
[GOAL]
case neg.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
p₁ : P
hp₁ : p₁ ∈ ↑s₁
p₂ : P
hp₂ : p₂ ∈ ↑s₂
⊢ s₁ ∥ s₂
[PROOFSTEP]
refine' ⟨p₂ -ᵥ p₁, (eq_iff_direction_eq_of_mem hp₂ _).2 _⟩
[GOAL]
case neg.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
p₁ : P
hp₁ : p₁ ∈ ↑s₁
p₂ : P
hp₂ : p₂ ∈ ↑s₂
⊢ p₂ ∈ map (↑(constVAdd k P (p₂ -ᵥ p₁))) s₁
[PROOFSTEP]
rw [mem_map]
[GOAL]
case neg.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
p₁ : P
hp₁ : p₁ ∈ ↑s₁
p₂ : P
hp₂ : p₂ ∈ ↑s₂
⊢ ∃ y, y ∈ s₁ ∧ ↑↑(constVAdd k P (p₂ -ᵥ p₁)) y = p₂
[PROOFSTEP]
refine' ⟨p₁, hp₁, _⟩
[GOAL]
case neg.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
p₁ : P
hp₁ : p₁ ∈ ↑s₁
p₂ : P
hp₂ : p₂ ∈ ↑s₂
⊢ ↑↑(constVAdd k P (p₂ -ᵥ p₁)) p₁ = p₂
[PROOFSTEP]
simp
[GOAL]
case neg.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : AffineSubspace k P
hd : direction s₁ = direction s₂
hb : s₁ = ⊥ ↔ s₂ = ⊥
hs₁ : ¬s₁ = ⊥
hs₂ : s₂ ≠ ⊥
p₁ : P
hp₁ : p₁ ∈ ↑s₁
p₂ : P
hp₂ : p₂ ∈ ↑s₂
⊢ direction s₂ = direction (map (↑(constVAdd k P (p₂ -ᵥ p₁))) s₁)
[PROOFSTEP]
simpa using hd.symm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
h : affineSpan k s₁ ∥ affineSpan k s₂
⊢ vectorSpan k s₁ = vectorSpan k s₂
[PROOFSTEP]
simp_rw [← direction_affineSpan]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
h : affineSpan k s₁ ∥ affineSpan k s₂
⊢ direction (affineSpan k s₁) = direction (affineSpan k s₂)
[PROOFSTEP]
exact h.direction_eq
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
⊢ affineSpan k s₁ ∥ affineSpan k s₂ ↔ vectorSpan k s₁ = vectorSpan k s₂ ∧ (s₁ = ∅ ↔ s₂ = ∅)
[PROOFSTEP]
repeat
rw [← direction_affineSpan, ← affineSpan_eq_bot k]
-- porting note: more issues with `simp`
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
⊢ affineSpan k s₁ ∥ affineSpan k s₂ ↔ vectorSpan k s₁ = vectorSpan k s₂ ∧ (s₁ = ∅ ↔ s₂ = ∅)
[PROOFSTEP]
rw [← direction_affineSpan, ← affineSpan_eq_bot k]
-- porting note: more issues with `simp`
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
⊢ affineSpan k s₁ ∥ affineSpan k s₂ ↔ direction (affineSpan k s₁) = vectorSpan k s₂ ∧ (affineSpan k s₁ = ⊥ ↔ s₂ = ∅)
[PROOFSTEP]
rw [← direction_affineSpan, ← affineSpan_eq_bot k]
-- porting note: more issues with `simp`
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
⊢ affineSpan k s₁ ∥ affineSpan k s₂ ↔
direction (affineSpan k s₁) = direction (affineSpan k s₂) ∧ (affineSpan k s₁ = ⊥ ↔ affineSpan k s₂ = ⊥)
[PROOFSTEP]
rw [← direction_affineSpan, ← affineSpan_eq_bot k]
-- porting note: more issues with `simp`
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
s₁ s₂ : Set P
⊢ affineSpan k s₁ ∥ affineSpan k s₂ ↔
direction (affineSpan k s₁) = direction (affineSpan k s₂) ∧ (affineSpan k s₁ = ⊥ ↔ affineSpan k s₂ = ⊥)
[PROOFSTEP]
exact parallel_iff_direction_eq_and_eq_bot_iff_eq_bot
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p₁ p₂ p₃ p₄ : P
⊢ affineSpan k {p₁, p₂} ∥ affineSpan k {p₃, p₄} ↔ vectorSpan k {p₁, p₂} = vectorSpan k {p₃, p₄}
[PROOFSTEP]
simp [affineSpan_parallel_iff_vectorSpan_eq_and_eq_empty_iff_eq_empty, ← not_nonempty_iff_eq_empty]
| {"mathlib_filename": "Mathlib.LinearAlgebra.AffineSpace.AffineSubspace", "llama_tokens": 80150} |
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
⊢ Injective toAffineMap
[PROOFSTEP]
rintro ⟨e, el, h⟩ ⟨e', el', h'⟩ H
[GOAL]
case mk.mk
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ ≃ P₂
el : V₁ ≃ₗ[k] V₂
h : ∀ (p : P₁) (v : V₁), ↑e (v +ᵥ p) = ↑el v +ᵥ ↑e p
e' : P₁ ≃ P₂
el' : V₁ ≃ₗ[k] V₂
h' : ∀ (p : P₁) (v : V₁), ↑e' (v +ᵥ p) = ↑el' v +ᵥ ↑e' p
H : ↑{ toEquiv := e, linear := el, map_vadd' := h } = ↑{ toEquiv := e', linear := el', map_vadd' := h' }
⊢ { toEquiv := e, linear := el, map_vadd' := h } = { toEquiv := e', linear := el', map_vadd' := h' }
[PROOFSTEP]
simp only [(toAffineMap_mk), (AffineMap.mk.injEq), Equiv.coe_inj, LinearEquiv.toLinearMap_inj] at H
[GOAL]
case mk.mk
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ ≃ P₂
el : V₁ ≃ₗ[k] V₂
h : ∀ (p : P₁) (v : V₁), ↑e (v +ᵥ p) = ↑el v +ᵥ ↑e p
e' : P₁ ≃ P₂
el' : V₁ ≃ₗ[k] V₂
h' : ∀ (p : P₁) (v : V₁), ↑e' (v +ᵥ p) = ↑el' v +ᵥ ↑e' p
H : e = e' ∧ el = el'
⊢ { toEquiv := e, linear := el, map_vadd' := h } = { toEquiv := e', linear := el', map_vadd' := h' }
[PROOFSTEP]
congr
[GOAL]
case mk.mk.e_toEquiv
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ ≃ P₂
el : V₁ ≃ₗ[k] V₂
h : ∀ (p : P₁) (v : V₁), ↑e (v +ᵥ p) = ↑el v +ᵥ ↑e p
e' : P₁ ≃ P₂
el' : V₁ ≃ₗ[k] V₂
h' : ∀ (p : P₁) (v : V₁), ↑e' (v +ᵥ p) = ↑el' v +ᵥ ↑e' p
H : e = e' ∧ el = el'
⊢ e = e'
case mk.mk.e_linear
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ ≃ P₂
el : V₁ ≃ₗ[k] V₂
h : ∀ (p : P₁) (v : V₁), ↑e (v +ᵥ p) = ↑el v +ᵥ ↑e p
e' : P₁ ≃ P₂
el' : V₁ ≃ₗ[k] V₂
h' : ∀ (p : P₁) (v : V₁), ↑e' (v +ᵥ p) = ↑el' v +ᵥ ↑e' p
H : e = e' ∧ el = el'
⊢ el = el'
[PROOFSTEP]
exacts [H.1, H.2]
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ → P₂
e' : V₁ ≃ₗ[k] V₂
p : P₁
h : ∀ (p' : P₁), e p' = ↑e' (p' -ᵥ p) +ᵥ e p
p' : P₁
⊢ (fun q' => ↑(LinearEquiv.symm e') (q' -ᵥ e p) +ᵥ p) (e p') = p'
[PROOFSTEP]
simp [h p', (vadd_vsub), (vsub_vadd)]
-- Porting note: `simp` needs `()`
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ → P₂
e' : V₁ ≃ₗ[k] V₂
p : P₁
h : ∀ (p' : P₁), e p' = ↑e' (p' -ᵥ p) +ᵥ e p
q' : P₂
⊢ e ((fun q' => ↑(LinearEquiv.symm e') (q' -ᵥ e p) +ᵥ p) q') = q'
[PROOFSTEP]
simp [h (e'.symm (q' -ᵥ e p) +ᵥ p), (vadd_vsub), (vsub_vadd)]
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ → P₂
e' : V₁ ≃ₗ[k] V₂
p : P₁
h : ∀ (p' : P₁), e p' = ↑e' (p' -ᵥ p) +ᵥ e p
p' : P₁
v : V₁
⊢ ↑{ toFun := e, invFun := fun q' => ↑(LinearEquiv.symm e') (q' -ᵥ e p) +ᵥ p,
left_inv := (_ : ∀ (p' : P₁), ↑(LinearEquiv.symm e') (e p' -ᵥ e p) +ᵥ p = p'),
right_inv := (_ : ∀ (q' : P₂), e (↑(LinearEquiv.symm e') (q' -ᵥ e p) +ᵥ p) = q') }
(v +ᵥ p') =
↑e' v +ᵥ
↑{ toFun := e, invFun := fun q' => ↑(LinearEquiv.symm e') (q' -ᵥ e p) +ᵥ p,
left_inv := (_ : ∀ (p' : P₁), ↑(LinearEquiv.symm e') (e p' -ᵥ e p) +ᵥ p = p'),
right_inv := (_ : ∀ (q' : P₂), e (↑(LinearEquiv.symm e') (q' -ᵥ e p) +ᵥ p) = q') }
p'
[PROOFSTEP]
simp [h p', h (v +ᵥ p'), (vadd_vsub_assoc), (vadd_vadd)]
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ ≃ᵃ[k] P₂
p : P₂
v : V₂
⊢ v +ᵥ p = ↑e.symm.symm (↑(LinearEquiv.symm e.linear) v +ᵥ ↑e.symm p)
[PROOFSTEP]
rw [Equiv.symm_symm, e.map_vadd' ((Equiv.symm e.toEquiv) p) ((LinearEquiv.symm e.linear) v),
LinearEquiv.apply_symm_apply, Equiv.apply_symm_apply]
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
e : P₁ ≃ᵃ[k] P₂
e' : P₂ ≃ᵃ[k] P₃
p : P₁
v : V₁
⊢ ↑(e.trans e'.toEquiv) (v +ᵥ p) = ↑(LinearEquiv.trans e.linear e'.linear) v +ᵥ ↑(e.trans e'.toEquiv) p
[PROOFSTEP]
simp only [LinearEquiv.trans_apply, (coe_toEquiv), (· ∘ ·), Equiv.coe_trans, (map_vadd)]
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V₁
inst✝¹⁰ : Module k V₁
inst✝⁹ : AffineSpace V₁ P₁
inst✝⁸ : AddCommGroup V₂
inst✝⁷ : Module k V₂
inst✝⁶ : AffineSpace V₂ P₂
inst✝⁵ : AddCommGroup V₃
inst✝⁴ : Module k V₃
inst✝³ : AffineSpace V₃ P₃
inst✝² : AddCommGroup V₄
inst✝¹ : Module k V₄
inst✝ : AffineSpace V₄ P₄
p p' : P₁
v : V₁
⊢ ↑(Equiv.constVSub p) (v +ᵥ p') = ↑(LinearEquiv.neg k) v +ᵥ ↑(Equiv.constVSub p) p'
[PROOFSTEP]
simp [(Equiv.coe_constVSub), (vsub_vadd_eq_vsub_sub), neg_add_eq_sub]
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹³ : Ring k
inst✝¹² : AddCommGroup V₁
inst✝¹¹ : Module k V₁
inst✝¹⁰ : AffineSpace V₁ P₁
inst✝⁹ : AddCommGroup V₂
inst✝⁸ : Module k V₂
inst✝⁷ : AffineSpace V₂ P₂
inst✝⁶ : AddCommGroup V₃
inst✝⁵ : Module k V₃
inst✝⁴ : AffineSpace V₃ P₃
inst✝³ : AddCommGroup V₄
inst✝² : Module k V₄
inst✝¹ : AffineSpace V₄ P₄
inst✝ : Invertible 2
x y : V₁
h : bit0 x = bit0 y
⊢ x = y
[PROOFSTEP]
rwa [bit0, bit0, ← two_smul k x, ← two_smul k y, (isUnit_of_invertible (2 : k)).smul_left_cancel] at h
[GOAL]
k : Type u_1
P₁ : Type u_2
P₂ : Type u_3
P₃ : Type u_4
P₄ : Type u_5
V₁ : Type u_6
V₂ : Type u_7
V₃ : Type u_8
V₄ : Type u_9
inst✝¹⁴ : Ring k
inst✝¹³ : AddCommGroup V₁
inst✝¹² : Module k V₁
inst✝¹¹ : AffineSpace V₁ P₁
inst✝¹⁰ : AddCommGroup V₂
inst✝⁹ : Module k V₂
inst✝⁸ : AffineSpace V₂ P₂
inst✝⁷ : AddCommGroup V₃
inst✝⁶ : Module k V₃
inst✝⁵ : AffineSpace V₃ P₃
inst✝⁴ : AddCommGroup V₄
inst✝³ : Module k V₄
inst✝² : AffineSpace V₄ P₄
R' : Type u_10
inst✝¹ : CommRing R'
inst✝ : Module R' V₁
c p : P₁
⊢ ↑(homothety c (-1)) p = ↑(pointReflection R' c) p
[PROOFSTEP]
simp [(homothety_apply), pointReflection_apply _, (neg_vsub_eq_vsub_rev)]
| {"mathlib_filename": "Mathlib.LinearAlgebra.AffineSpace.AffineEquiv", "llama_tokens": 5213} |
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ AffineIndependent k p ↔
∀ (w : ι → k), ∑ i : ι, w i = 0 → ↑(Finset.weightedVSub Finset.univ p) w = 0 → ∀ (i : ι), w i = 0
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ AffineIndependent k p →
∀ (w : ι → k), ∑ i : ι, w i = 0 → ↑(Finset.weightedVSub Finset.univ p) w = 0 → ∀ (i : ι), w i = 0
[PROOFSTEP]
exact fun h w hw hs i => h Finset.univ w hw hs i (Finset.mem_univ _)
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ (∀ (w : ι → k), ∑ i : ι, w i = 0 → ↑(Finset.weightedVSub Finset.univ p) w = 0 → ∀ (i : ι), w i = 0) →
AffineIndependent k p
[PROOFSTEP]
intro h s w hw hs i hi
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h : ∀ (w : ι → k), ∑ i : ι, w i = 0 → ↑(Finset.weightedVSub Finset.univ p) w = 0 → ∀ (i : ι), w i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i : ι
hi : i ∈ s
⊢ w i = 0
[PROOFSTEP]
rw [Finset.weightedVSub_indicator_subset _ _ (Finset.subset_univ s)] at hs
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h : ∀ (w : ι → k), ∑ i : ι, w i = 0 → ↑(Finset.weightedVSub Finset.univ p) w = 0 → ∀ (i : ι), w i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub Finset.univ p) (Set.indicator (↑s) w) = 0
i : ι
hi : i ∈ s
⊢ w i = 0
[PROOFSTEP]
rw [Set.sum_indicator_subset _ (Finset.subset_univ s)] at hw
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h : ∀ (w : ι → k), ∑ i : ι, w i = 0 → ↑(Finset.weightedVSub Finset.univ p) w = 0 → ∀ (i : ι), w i = 0
s : Finset ι
w : ι → k
hw : ∑ i : ι, Set.indicator (↑s) (fun i => w i) i = 0
hs : ↑(Finset.weightedVSub Finset.univ p) (Set.indicator (↑s) w) = 0
i : ι
hi : i ∈ s
⊢ w i = 0
[PROOFSTEP]
replace h := h ((↑s : Set ι).indicator w) hw hs i
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i : ι, Set.indicator (↑s) (fun i => w i) i = 0
hs : ↑(Finset.weightedVSub Finset.univ p) (Set.indicator (↑s) w) = 0
i : ι
hi : i ∈ s
h : Set.indicator (↑s) w i = 0
⊢ w i = 0
[PROOFSTEP]
simpa [hi] using h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
⊢ AffineIndependent k p ↔ LinearIndependent k fun i => p ↑i -ᵥ p i1
[PROOFSTEP]
classical
constructor
· intro h
rw [linearIndependent_iff']
intro s g hg i hi
set f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g ⟨x, hx⟩ with hfdef
let s2 : Finset ι := insert i1 (s.map (Embedding.subtype _))
have hfg : ∀ x : { x // x ≠ i1 }, g x = f x := by
intro x
rw [hfdef]
dsimp only
erw [dif_neg x.property, Subtype.coe_eta]
rw [hfg]
have hf : ∑ ι in s2, f ι = 0 :=
by
rw [Finset.sum_insert (Finset.not_mem_map_subtype_of_not_property s (Classical.not_not.2 rfl)),
Finset.sum_subtype_map_embedding fun x _ => (hfg x).symm]
rw [hfdef]
dsimp only
rw [dif_pos rfl]
exact neg_add_self _
have hs2 : s2.weightedVSub p f = (0 : V) :=
by
set f2 : ι → V := fun x => f x • (p x -ᵥ p i1) with hf2def
set g2 : { x // x ≠ i1 } → V := fun x => g x • (p x -ᵥ p i1)
have hf2g2 : ∀ x : { x // x ≠ i1 }, f2 x = g2 x :=
by
simp only [hf2def]
refine' fun x => _
rw [hfg]
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s2 f p hf (p i1), Finset.weightedVSubOfPoint_insert,
Finset.weightedVSubOfPoint_apply, Finset.sum_subtype_map_embedding fun x _ => hf2g2 x]
exact hg
exact h s2 f hf hs2 i (Finset.mem_insert_of_mem (Finset.mem_map.2 ⟨i, hi, rfl⟩))
· intro h
rw [linearIndependent_iff'] at h
intro s w hw hs i hi
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s w p hw (p i1), ← s.weightedVSubOfPoint_erase w p i1,
Finset.weightedVSubOfPoint_apply] at hs
let f : ι → V := fun i => w i • (p i -ᵥ p i1)
have hs2 : (∑ i in (s.erase i1).subtype fun i => i ≠ i1, f i) = 0 :=
by
rw [← hs]
convert Finset.sum_subtype_of_mem f fun x => Finset.ne_of_mem_erase
have h2 := h ((s.erase i1).subtype fun i => i ≠ i1) (fun x => w x) hs2
simp_rw [Finset.mem_subtype] at h2
have h2b : ∀ i ∈ s, i ≠ i1 → w i = 0 := fun i his hi => h2 ⟨i, hi⟩ (Finset.mem_erase_of_ne_of_mem hi his)
exact Finset.eq_zero_of_sum_eq_zero hw h2b i hi
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
⊢ AffineIndependent k p ↔ LinearIndependent k fun i => p ↑i -ᵥ p i1
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
⊢ AffineIndependent k p → LinearIndependent k fun i => p ↑i -ᵥ p i1
[PROOFSTEP]
intro h
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
⊢ LinearIndependent k fun i => p ↑i -ᵥ p i1
[PROOFSTEP]
rw [linearIndependent_iff']
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
⊢ ∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
[PROOFSTEP]
intro s g hg i hi
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
⊢ g i = 0
[PROOFSTEP]
set f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g ⟨x, hx⟩ with hfdef
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
⊢ g i = 0
[PROOFSTEP]
let s2 : Finset ι := insert i1 (s.map (Embedding.subtype _))
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
⊢ g i = 0
[PROOFSTEP]
have hfg : ∀ x : { x // x ≠ i1 }, g x = f x := by
intro x
rw [hfdef]
dsimp only
erw [dif_neg x.property, Subtype.coe_eta]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
⊢ ∀ (x : { x // x ≠ i1 }), g x = f ↑x
[PROOFSTEP]
intro x
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
x : { x // x ≠ i1 }
⊢ g x = f ↑x
[PROOFSTEP]
rw [hfdef]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
x : { x // x ≠ i1 }
⊢ g x = (fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }) ↑x
[PROOFSTEP]
dsimp only
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
x : { x // x ≠ i1 }
⊢ g x = if hx : ↑x = i1 then -∑ y in s, g y else g { val := ↑x, property := hx }
[PROOFSTEP]
erw [dif_neg x.property, Subtype.coe_eta]
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ g i = 0
[PROOFSTEP]
rw [hfg]
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ f ↑i = 0
[PROOFSTEP]
have hf : ∑ ι in s2, f ι = 0 :=
by
rw [Finset.sum_insert (Finset.not_mem_map_subtype_of_not_property s (Classical.not_not.2 rfl)),
Finset.sum_subtype_map_embedding fun x _ => (hfg x).symm]
rw [hfdef]
dsimp only
rw [dif_pos rfl]
exact neg_add_self _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ ∑ ι in s2, f ι = 0
[PROOFSTEP]
rw [Finset.sum_insert (Finset.not_mem_map_subtype_of_not_property s (Classical.not_not.2 rfl)),
Finset.sum_subtype_map_embedding fun x _ => (hfg x).symm]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ f i1 + ∑ x in s, g x = 0
[PROOFSTEP]
rw [hfdef]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ (fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }) i1 + ∑ x in s, g x = 0
[PROOFSTEP]
dsimp only
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ (if hx : i1 = i1 then -∑ y in s, g y else g { val := i1, property := hx }) + ∑ x in s, g x = 0
[PROOFSTEP]
rw [dif_pos rfl]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
⊢ -∑ y in s, g y + ∑ x in s, g x = 0
[PROOFSTEP]
exact neg_add_self _
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
⊢ f ↑i = 0
[PROOFSTEP]
have hs2 : s2.weightedVSub p f = (0 : V) :=
by
set f2 : ι → V := fun x => f x • (p x -ᵥ p i1) with hf2def
set g2 : { x // x ≠ i1 } → V := fun x => g x • (p x -ᵥ p i1)
have hf2g2 : ∀ x : { x // x ≠ i1 }, f2 x = g2 x :=
by
simp only [hf2def]
refine' fun x => _
rw [hfg]
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s2 f p hf (p i1), Finset.weightedVSubOfPoint_insert,
Finset.weightedVSubOfPoint_apply, Finset.sum_subtype_map_embedding fun x _ => hf2g2 x]
exact hg
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
⊢ ↑(Finset.weightedVSub s2 p) f = 0
[PROOFSTEP]
set f2 : ι → V := fun x => f x • (p x -ᵥ p i1) with hf2def
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
⊢ ↑(Finset.weightedVSub s2 p) f = 0
[PROOFSTEP]
set g2 : { x // x ≠ i1 } → V := fun x => g x • (p x -ᵥ p i1)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
g2 : { x // x ≠ i1 } → V := fun x => g x • (p ↑x -ᵥ p i1)
hg : Finset.sum s g2 = 0
⊢ ↑(Finset.weightedVSub s2 p) f = 0
[PROOFSTEP]
have hf2g2 : ∀ x : { x // x ≠ i1 }, f2 x = g2 x :=
by
simp only [hf2def]
refine' fun x => _
rw [hfg]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
g2 : { x // x ≠ i1 } → V := fun x => g x • (p ↑x -ᵥ p i1)
hg : Finset.sum s g2 = 0
⊢ ∀ (x : { x // x ≠ i1 }), f2 ↑x = g2 x
[PROOFSTEP]
simp only [hf2def]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
g2 : { x // x ≠ i1 } → V := fun x => g x • (p ↑x -ᵥ p i1)
hg : Finset.sum s g2 = 0
⊢ ∀ (x : { x // x ≠ i1 }),
(if hx : ↑x = i1 then -∑ y in s, g y else g { val := ↑x, property := hx }) • (p ↑x -ᵥ p i1) = g x • (p ↑x -ᵥ p i1)
[PROOFSTEP]
refine' fun x => _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
g2 : { x // x ≠ i1 } → V := fun x => g x • (p ↑x -ᵥ p i1)
hg : Finset.sum s g2 = 0
x : { x // x ≠ i1 }
⊢ (if hx : ↑x = i1 then -∑ y in s, g y else g { val := ↑x, property := hx }) • (p ↑x -ᵥ p i1) = g x • (p ↑x -ᵥ p i1)
[PROOFSTEP]
rw [hfg]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
g2 : { x // x ≠ i1 } → V := fun x => g x • (p ↑x -ᵥ p i1)
hg : Finset.sum s g2 = 0
hf2g2 : ∀ (x : { x // x ≠ i1 }), f2 ↑x = g2 x
⊢ ↑(Finset.weightedVSub s2 p) f = 0
[PROOFSTEP]
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s2 f p hf (p i1), Finset.weightedVSubOfPoint_insert,
Finset.weightedVSubOfPoint_apply, Finset.sum_subtype_map_embedding fun x _ => hf2g2 x]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
f2 : ι → V := fun x => f x • (p x -ᵥ p i1)
hf2def : f2 = fun x => f x • (p x -ᵥ p i1)
g2 : { x // x ≠ i1 } → V := fun x => g x • (p ↑x -ᵥ p i1)
hg : Finset.sum s g2 = 0
hf2g2 : ∀ (x : { x // x ≠ i1 }), f2 ↑x = g2 x
⊢ ∑ x in s, g2 x = 0
[PROOFSTEP]
exact hg
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : AffineIndependent k p
s : Finset { x // x ≠ i1 }
g : { x // x ≠ i1 } → k
hg : ∑ i in s, g i • (p ↑i -ᵥ p i1) = 0
i : { x // x ≠ i1 }
hi : i ∈ s
f : ι → k := fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
hfdef : f = fun x => if hx : x = i1 then -∑ y in s, g y else g { val := x, property := hx }
s2 : Finset ι := insert i1 (Finset.map (Embedding.subtype fun x => x ≠ i1) s)
hfg : ∀ (x : { x // x ≠ i1 }), g x = f ↑x
hf : ∑ ι in s2, f ι = 0
hs2 : ↑(Finset.weightedVSub s2 p) f = 0
⊢ f ↑i = 0
[PROOFSTEP]
exact h s2 f hf hs2 i (Finset.mem_insert_of_mem (Finset.mem_map.2 ⟨i, hi, rfl⟩))
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
⊢ (LinearIndependent k fun i => p ↑i -ᵥ p i1) → AffineIndependent k p
[PROOFSTEP]
intro h
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h : LinearIndependent k fun i => p ↑i -ᵥ p i1
⊢ AffineIndependent k p
[PROOFSTEP]
rw [linearIndependent_iff'] at h
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
⊢ AffineIndependent k p
[PROOFSTEP]
intro s w hw hs i hi
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i : ι
hi : i ∈ s
⊢ w i = 0
[PROOFSTEP]
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s w p hw (p i1), ← s.weightedVSubOfPoint_erase w p i1,
Finset.weightedVSubOfPoint_apply] at hs
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
⊢ w i = 0
[PROOFSTEP]
let f : ι → V := fun i => w i • (p i -ᵥ p i1)
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
⊢ w i = 0
[PROOFSTEP]
have hs2 : (∑ i in (s.erase i1).subtype fun i => i ≠ i1, f i) = 0 :=
by
rw [← hs]
convert Finset.sum_subtype_of_mem f fun x => Finset.ne_of_mem_erase
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
⊢ ∑ i in Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1), f ↑i = 0
[PROOFSTEP]
rw [← hs]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
⊢ ∑ i in Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1), f ↑i = ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1)
[PROOFSTEP]
convert Finset.sum_subtype_of_mem f fun x => Finset.ne_of_mem_erase
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
hs2 : ∑ i in Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1), f ↑i = 0
⊢ w i = 0
[PROOFSTEP]
have h2 := h ((s.erase i1).subtype fun i => i ≠ i1) (fun x => w x) hs2
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
hs2 : ∑ i in Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1), f ↑i = 0
h2 : ∀ (i : { x // x ≠ i1 }), i ∈ Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1) → (fun x => w ↑x) i = 0
⊢ w i = 0
[PROOFSTEP]
simp_rw [Finset.mem_subtype] at h2
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
hs2 : ∑ i in Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1), f ↑i = 0
h2 : ∀ (i : { x // x ≠ i1 }), ↑i ∈ Finset.erase s i1 → w ↑i = 0
⊢ w i = 0
[PROOFSTEP]
have h2b : ∀ i ∈ s, i ≠ i1 → w i = 0 := fun i his hi => h2 ⟨i, hi⟩ (Finset.mem_erase_of_ne_of_mem hi his)
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i1 : ι
h :
∀ (s : Finset { x // x ≠ i1 }) (g : { x // x ≠ i1 } → k),
∑ i in s, g i • (p ↑i -ᵥ p i1) = 0 → ∀ (i : { x // x ≠ i1 }), i ∈ s → g i = 0
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ∑ i in Finset.erase s i1, w i • (p i -ᵥ p i1) = 0
i : ι
hi : i ∈ s
f : ι → V := fun i => w i • (p i -ᵥ p i1)
hs2 : ∑ i in Finset.subtype (fun i => i ≠ i1) (Finset.erase s i1), f ↑i = 0
h2 : ∀ (i : { x // x ≠ i1 }), ↑i ∈ Finset.erase s i1 → w ↑i = 0
h2b : ∀ (i : ι), i ∈ s → i ≠ i1 → w i = 0
⊢ w i = 0
[PROOFSTEP]
exact Finset.eq_zero_of_sum_eq_zero hw h2b i hi
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
⊢ (AffineIndependent k fun p => ↑p) ↔ LinearIndependent k fun v => ↑v
[PROOFSTEP]
rw [affineIndependent_iff_linearIndependent_vsub k (fun p => p : s → P) ⟨p₁, hp₁⟩]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
⊢ (LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }) ↔ LinearIndependent k fun v => ↑v
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
⊢ (LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }) → LinearIndependent k fun v => ↑v
[PROOFSTEP]
intro h
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
⊢ LinearIndependent k fun v => ↑v
[PROOFSTEP]
have hv : ∀ v : (fun p => (p -ᵥ p₁ : V)) '' (s \ { p₁ }), (v : V) +ᵥ p₁ ∈ s \ { p₁ } := fun v =>
(vsub_left_injective p₁).mem_set_image.1 ((vadd_vsub (v : V) p₁).symm ▸ v.property)
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
hv : ∀ (v : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁}))), ↑v +ᵥ p₁ ∈ s \ {p₁}
⊢ LinearIndependent k fun v => ↑v
[PROOFSTEP]
let f : (fun p : P => (p -ᵥ p₁ : V)) '' (s \ { p₁ }) → { x : s // x ≠ ⟨p₁, hp₁⟩ } := fun x =>
⟨⟨(x : V) +ᵥ p₁, Set.mem_of_mem_diff (hv x)⟩, fun hx => Set.not_mem_of_mem_diff (hv x) (Subtype.ext_iff.1 hx)⟩
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
hv : ∀ (v : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁}))), ↑v +ᵥ p₁ ∈ s \ {p₁}
f : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁})) → { x // x ≠ { val := p₁, property := hp₁ } } :=
fun x =>
{ val := { val := ↑x +ᵥ p₁, property := (_ : ↑x +ᵥ p₁ ∈ s) },
property := (_ : { val := ↑x +ᵥ p₁, property := (_ : ↑x +ᵥ p₁ ∈ s) } = { val := p₁, property := hp₁ } → False) }
⊢ LinearIndependent k fun v => ↑v
[PROOFSTEP]
convert h.comp f fun x1 x2 hx => Subtype.ext (vadd_right_cancel p₁ (Subtype.ext_iff.1 (Subtype.ext_iff.1 hx)))
[GOAL]
case h.e'_4.h.h.e
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
hv : ∀ (v : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁}))), ↑v +ᵥ p₁ ∈ s \ {p₁}
f : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁})) → { x // x ≠ { val := p₁, property := hp₁ } } :=
fun x =>
{ val := { val := ↑x +ᵥ p₁, property := (_ : ↑x +ᵥ p₁ ∈ s) },
property := (_ : { val := ↑x +ᵥ p₁, property := (_ : ↑x +ᵥ p₁ ∈ s) } = { val := p₁, property := hp₁ } → False) }
x✝ : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁}))
⊢ Subtype.val = (fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }) ∘ f
[PROOFSTEP]
ext v
[GOAL]
case h.e'_4.h.h.e.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
hv : ∀ (v : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁}))), ↑v +ᵥ p₁ ∈ s \ {p₁}
f : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁})) → { x // x ≠ { val := p₁, property := hp₁ } } :=
fun x =>
{ val := { val := ↑x +ᵥ p₁, property := (_ : ↑x +ᵥ p₁ ∈ s) },
property := (_ : { val := ↑x +ᵥ p₁, property := (_ : ↑x +ᵥ p₁ ∈ s) } = { val := p₁, property := hp₁ } → False) }
x✝ : ↑((fun p => p -ᵥ p₁) '' (s \ {p₁}))
v : { x // x ∈ (fun p => p -ᵥ p₁) '' (s \ {p₁}) }
⊢ ↑v = ((fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }) ∘ f) v
[PROOFSTEP]
exact (vadd_vsub (v : V) p₁).symm
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
⊢ (LinearIndependent k fun v => ↑v) → LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
[PROOFSTEP]
intro h
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun v => ↑v
⊢ LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
[PROOFSTEP]
let f : { x : s // x ≠ ⟨p₁, hp₁⟩ } → (fun p : P => (p -ᵥ p₁ : V)) '' (s \ { p₁ }) := fun x =>
⟨((x : s) : P) -ᵥ p₁, ⟨x, ⟨⟨(x : s).property, fun hx => x.property (Subtype.ext hx)⟩, rfl⟩⟩⟩
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
hp₁ : p₁ ∈ s
h : LinearIndependent k fun v => ↑v
f : { x // x ≠ { val := p₁, property := hp₁ } } → ↑((fun p => p -ᵥ p₁) '' (s \ {p₁})) :=
fun x => { val := ↑↑x -ᵥ p₁, property := (_ : ∃ a, a ∈ s \ {p₁} ∧ (fun p => p -ᵥ p₁) a = ↑↑x -ᵥ p₁) }
⊢ LinearIndependent k fun i => ↑↑i -ᵥ ↑{ val := p₁, property := hp₁ }
[PROOFSTEP]
convert h.comp f fun x1 x2 hx => Subtype.ext (Subtype.ext (vsub_left_cancel (Subtype.ext_iff.1 hx)))
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
hs : ∀ (v : V), v ∈ s → v ≠ 0
p₁ : P
⊢ (LinearIndependent k fun v => ↑v) ↔ AffineIndependent k fun p => ↑p
[PROOFSTEP]
rw [affineIndependent_set_iff_linearIndependent_vsub k (Set.mem_union_left _ (Set.mem_singleton p₁))]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
hs : ∀ (v : V), v ∈ s → v ≠ 0
p₁ : P
⊢ (LinearIndependent k fun v => ↑v) ↔ LinearIndependent k fun v => ↑v
[PROOFSTEP]
have h : (fun p => (p -ᵥ p₁ : V)) '' (({ p₁ } ∪ (fun v => v +ᵥ p₁) '' s) \ { p₁ }) = s :=
by
simp_rw [Set.union_diff_left, Set.image_diff (vsub_left_injective p₁), Set.image_image, Set.image_singleton,
vsub_self, vadd_vsub, Set.image_id']
exact Set.diff_singleton_eq_self fun h => hs 0 h rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
hs : ∀ (v : V), v ∈ s → v ≠ 0
p₁ : P
⊢ (fun p => p -ᵥ p₁) '' (({p₁} ∪ (fun v => v +ᵥ p₁) '' s) \ {p₁}) = s
[PROOFSTEP]
simp_rw [Set.union_diff_left, Set.image_diff (vsub_left_injective p₁), Set.image_image, Set.image_singleton, vsub_self,
vadd_vsub, Set.image_id']
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
hs : ∀ (v : V), v ∈ s → v ≠ 0
p₁ : P
⊢ s \ {0} = s
[PROOFSTEP]
exact Set.diff_singleton_eq_self fun h => hs 0 h rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set V
hs : ∀ (v : V), v ∈ s → v ≠ 0
p₁ : P
h : (fun p => p -ᵥ p₁) '' (({p₁} ∪ (fun v => v +ᵥ p₁) '' s) \ {p₁}) = s
⊢ (LinearIndependent k fun v => ↑v) ↔ LinearIndependent k fun v => ↑v
[PROOFSTEP]
rw [h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
⊢ AffineIndependent k p ↔
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
classical
constructor
· intro ha s1 s2 w1 w2 hw1 hw2 heq
ext i
by_cases hi : i ∈ s1 ∪ s2
· rw [← sub_eq_zero]
rw [Set.sum_indicator_subset _ (Finset.subset_union_left s1 s2)] at hw1
rw [Set.sum_indicator_subset _ (Finset.subset_union_right s1 s2)] at hw2
have hws : (∑ i in s1 ∪ s2, (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) i) = 0 := by simp [hw1, hw2]
rw [Finset.affineCombination_indicator_subset _ _ (Finset.subset_union_left s1 s2),
Finset.affineCombination_indicator_subset _ _ (Finset.subset_union_right s1 s2), ← @vsub_eq_zero_iff_eq V,
Finset.affineCombination_vsub] at heq
exact ha (s1 ∪ s2) (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) hws heq i hi
· rw [← Finset.mem_coe, Finset.coe_union] at hi
have h₁ : Set.indicator (↑s1) w1 i = 0 :=
by
simp only [Set.indicator, Finset.mem_coe, ite_eq_right_iff]
intro h
by_contra
exact (mt (@Set.mem_union_left _ i ↑s1 ↑s2) hi) h
have h₂ : Set.indicator (↑s2) w2 i = 0 :=
by
simp only [Set.indicator, Finset.mem_coe, ite_eq_right_iff]
intro h
by_contra
exact (mt (@Set.mem_union_right _ i ↑s2 ↑s1) hi) h
simp [h₁, h₂]
· intro ha s w hw hs i0 hi0
let w1 : ι → k := Function.update (Function.const ι 0) i0 1
have hw1 : ∑ i in s, w1 i = 1 := by
rw [Finset.sum_update_of_mem hi0]
simp only [Finset.sum_const_zero, add_zero, const_apply]
have hw1s : s.affineCombination k p w1 = p i0 :=
s.affineCombination_of_eq_one_of_eq_zero w1 p hi0 (Function.update_same _ _ _) fun _ _ hne =>
Function.update_noteq hne _ _
let w2 := w + w1
have hw2 : ∑ i in s, w2 i = 1 := by simp_all only [Pi.add_apply, Finset.sum_add_distrib, zero_add]
have hw2s : s.affineCombination k p w2 = p i0 := by
simp_all only [← Finset.weightedVSub_vadd_affineCombination, zero_vadd]
replace ha := ha s s w2 w1 hw2 hw1 (hw1s.symm ▸ hw2s)
have hws : w2 i0 - w1 i0 = 0 := by
rw [← Finset.mem_coe] at hi0
rw [← Set.indicator_of_mem hi0 w2, ← Set.indicator_of_mem hi0 w1, ha, sub_self]
simpa using hws
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
⊢ AffineIndependent k p ↔
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
⊢ AffineIndependent k p →
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
intro ha s1 s2 w1 w2 hw1 hw2 heq
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
⊢ Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
ext i
[GOAL]
case mp.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
⊢ Set.indicator (↑s1) w1 i = Set.indicator (↑s2) w2 i
[PROOFSTEP]
by_cases hi : i ∈ s1 ∪ s2
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : i ∈ s1 ∪ s2
⊢ Set.indicator (↑s1) w1 i = Set.indicator (↑s2) w2 i
[PROOFSTEP]
rw [← sub_eq_zero]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : i ∈ s1 ∪ s2
⊢ Set.indicator (↑s1) w1 i - Set.indicator (↑s2) w2 i = 0
[PROOFSTEP]
rw [Set.sum_indicator_subset _ (Finset.subset_union_left s1 s2)] at hw1
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1 ∪ s2, Set.indicator (↑s1) (fun i => w1 i) i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : i ∈ s1 ∪ s2
⊢ Set.indicator (↑s1) w1 i - Set.indicator (↑s2) w2 i = 0
[PROOFSTEP]
rw [Set.sum_indicator_subset _ (Finset.subset_union_right s1 s2)] at hw2
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1 ∪ s2, Set.indicator (↑s1) (fun i => w1 i) i = 1
hw2 : ∑ i in s1 ∪ s2, Set.indicator (↑s2) (fun i => w2 i) i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : i ∈ s1 ∪ s2
⊢ Set.indicator (↑s1) w1 i - Set.indicator (↑s2) w2 i = 0
[PROOFSTEP]
have hws : (∑ i in s1 ∪ s2, (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) i) = 0 := by simp [hw1, hw2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1 ∪ s2, Set.indicator (↑s1) (fun i => w1 i) i = 1
hw2 : ∑ i in s1 ∪ s2, Set.indicator (↑s2) (fun i => w2 i) i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : i ∈ s1 ∪ s2
⊢ ∑ i in s1 ∪ s2, (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) i = 0
[PROOFSTEP]
simp [hw1, hw2]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1 ∪ s2, Set.indicator (↑s1) (fun i => w1 i) i = 1
hw2 : ∑ i in s1 ∪ s2, Set.indicator (↑s2) (fun i => w2 i) i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : i ∈ s1 ∪ s2
hws : ∑ i in s1 ∪ s2, (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) i = 0
⊢ Set.indicator (↑s1) w1 i - Set.indicator (↑s2) w2 i = 0
[PROOFSTEP]
rw [Finset.affineCombination_indicator_subset _ _ (Finset.subset_union_left s1 s2),
Finset.affineCombination_indicator_subset _ _ (Finset.subset_union_right s1 s2), ← @vsub_eq_zero_iff_eq V,
Finset.affineCombination_vsub] at heq
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1 ∪ s2, Set.indicator (↑s1) (fun i => w1 i) i = 1
hw2 : ∑ i in s1 ∪ s2, Set.indicator (↑s2) (fun i => w2 i) i = 1
heq : ↑(Finset.weightedVSub (s1 ∪ s2) p) (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) = 0
i : ι
hi : i ∈ s1 ∪ s2
hws : ∑ i in s1 ∪ s2, (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) i = 0
⊢ Set.indicator (↑s1) w1 i - Set.indicator (↑s2) w2 i = 0
[PROOFSTEP]
exact ha (s1 ∪ s2) (Set.indicator (↑s1) w1 - Set.indicator (↑s2) w2) hws heq i hi
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ s1 ∪ s2
⊢ Set.indicator (↑s1) w1 i = Set.indicator (↑s2) w2 i
[PROOFSTEP]
rw [← Finset.mem_coe, Finset.coe_union] at hi
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
⊢ Set.indicator (↑s1) w1 i = Set.indicator (↑s2) w2 i
[PROOFSTEP]
have h₁ : Set.indicator (↑s1) w1 i = 0 :=
by
simp only [Set.indicator, Finset.mem_coe, ite_eq_right_iff]
intro h
by_contra
exact (mt (@Set.mem_union_left _ i ↑s1 ↑s2) hi) h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
⊢ Set.indicator (↑s1) w1 i = 0
[PROOFSTEP]
simp only [Set.indicator, Finset.mem_coe, ite_eq_right_iff]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
⊢ i ∈ s1 → w1 i = 0
[PROOFSTEP]
intro h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h : i ∈ s1
⊢ w1 i = 0
[PROOFSTEP]
by_contra
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h : i ∈ s1
x✝ : ¬w1 i = 0
⊢ False
[PROOFSTEP]
exact (mt (@Set.mem_union_left _ i ↑s1 ↑s2) hi) h
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h₁ : Set.indicator (↑s1) w1 i = 0
⊢ Set.indicator (↑s1) w1 i = Set.indicator (↑s2) w2 i
[PROOFSTEP]
have h₂ : Set.indicator (↑s2) w2 i = 0 :=
by
simp only [Set.indicator, Finset.mem_coe, ite_eq_right_iff]
intro h
by_contra
exact (mt (@Set.mem_union_right _ i ↑s2 ↑s1) hi) h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h₁ : Set.indicator (↑s1) w1 i = 0
⊢ Set.indicator (↑s2) w2 i = 0
[PROOFSTEP]
simp only [Set.indicator, Finset.mem_coe, ite_eq_right_iff]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h₁ : Set.indicator (↑s1) w1 i = 0
⊢ i ∈ s2 → w2 i = 0
[PROOFSTEP]
intro h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h₁ : Set.indicator (↑s1) w1 i = 0
h : i ∈ s2
⊢ w2 i = 0
[PROOFSTEP]
by_contra
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h₁ : Set.indicator (↑s1) w1 i = 0
h : i ∈ s2
x✝ : ¬w2 i = 0
⊢ False
[PROOFSTEP]
exact (mt (@Set.mem_union_right _ i ↑s2 ↑s1) hi) h
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
heq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
i : ι
hi : ¬i ∈ ↑s1 ∪ ↑s2
h₁ : Set.indicator (↑s1) w1 i = 0
h₂ : Set.indicator (↑s2) w2 i = 0
⊢ Set.indicator (↑s1) w1 i = Set.indicator (↑s2) w2 i
[PROOFSTEP]
simp [h₁, h₂]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
⊢ (∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2) →
AffineIndependent k p
[PROOFSTEP]
intro ha s w hw hs i0 hi0
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
⊢ w i0 = 0
[PROOFSTEP]
let w1 : ι → k := Function.update (Function.const ι 0) i0 1
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
⊢ w i0 = 0
[PROOFSTEP]
have hw1 : ∑ i in s, w1 i = 1 := by
rw [Finset.sum_update_of_mem hi0]
simp only [Finset.sum_const_zero, add_zero, const_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
⊢ ∑ i in s, w1 i = 1
[PROOFSTEP]
rw [Finset.sum_update_of_mem hi0]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
⊢ 1 + ∑ x in s \ {i0}, const ι 0 x = 1
[PROOFSTEP]
simp only [Finset.sum_const_zero, add_zero, const_apply]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
⊢ w i0 = 0
[PROOFSTEP]
have hw1s : s.affineCombination k p w1 = p i0 :=
s.affineCombination_of_eq_one_of_eq_zero w1 p hi0 (Function.update_same _ _ _) fun _ _ hne =>
Function.update_noteq hne _ _
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
⊢ w i0 = 0
[PROOFSTEP]
let w2 := w + w1
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
⊢ w i0 = 0
[PROOFSTEP]
have hw2 : ∑ i in s, w2 i = 1 := by simp_all only [Pi.add_apply, Finset.sum_add_distrib, zero_add]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
⊢ ∑ i in s, w2 i = 1
[PROOFSTEP]
simp_all only [Pi.add_apply, Finset.sum_add_distrib, zero_add]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
⊢ w i0 = 0
[PROOFSTEP]
have hw2s : s.affineCombination k p w2 = p i0 := by
simp_all only [← Finset.weightedVSub_vadd_affineCombination, zero_vadd]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
⊢ ↑(Finset.affineCombination k s p) w2 = p i0
[PROOFSTEP]
simp_all only [← Finset.weightedVSub_vadd_affineCombination, zero_vadd]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
hw2s : ↑(Finset.affineCombination k s p) w2 = p i0
⊢ w i0 = 0
[PROOFSTEP]
replace ha := ha s s w2 w1 hw2 hw1 (hw1s.symm ▸ hw2s)
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
hw2s : ↑(Finset.affineCombination k s p) w2 = p i0
ha : Set.indicator (↑s) w2 = Set.indicator (↑s) w1
⊢ w i0 = 0
[PROOFSTEP]
have hws : w2 i0 - w1 i0 = 0 := by
rw [← Finset.mem_coe] at hi0
rw [← Set.indicator_of_mem hi0 w2, ← Set.indicator_of_mem hi0 w1, ha, sub_self]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
hw2s : ↑(Finset.affineCombination k s p) w2 = p i0
ha : Set.indicator (↑s) w2 = Set.indicator (↑s) w1
⊢ w2 i0 - w1 i0 = 0
[PROOFSTEP]
rw [← Finset.mem_coe] at hi0
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ ↑s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
hw2s : ↑(Finset.affineCombination k s p) w2 = p i0
ha : Set.indicator (↑s) w2 = Set.indicator (↑s) w1
⊢ w2 i0 - w1 i0 = 0
[PROOFSTEP]
rw [← Set.indicator_of_mem hi0 w2, ← Set.indicator_of_mem hi0 w1, ha, sub_self]
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
i0 : ι
hi0 : i0 ∈ s
w1 : ι → k := update (const ι 0) i0 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i0
w2 : ι → k := w + w1
hw2 : ∑ i in s, w2 i = 1
hw2s : ↑(Finset.affineCombination k s p) w2 = p i0
ha : Set.indicator (↑s) w2 = Set.indicator (↑s) w1
hws : w2 i0 - w1 i0 = 0
⊢ w i0 = 0
[PROOFSTEP]
simpa using hws
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ AffineIndependent k p ↔
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
[PROOFSTEP]
rw [affineIndependent_iff_indicator_eq_of_affineCombination_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ (∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2) ↔
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ (∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2) →
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
[PROOFSTEP]
intro h w1 w2 hw1 hw2 hweq
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
w1 w2 : ι → k
hw1 : ∑ i : ι, w1 i = 1
hw2 : ∑ i : ι, w2 i = 1
hweq : ↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2
⊢ w1 = w2
[PROOFSTEP]
simpa only [Set.indicator_univ, Finset.coe_univ] using h _ _ w1 w2 hw1 hw2 hweq
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
⊢ (∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2) →
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
intro h s1 s2 w1 w2 hw1 hw2 hweq
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
hweq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
⊢ Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
have hw1' : (∑ i, (s1 : Set ι).indicator w1 i) = 1 := by
rwa [Set.sum_indicator_subset _ (Finset.subset_univ s1)] at hw1
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
hweq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
⊢ ∑ i : ι, Set.indicator (↑s1) w1 i = 1
[PROOFSTEP]
rwa [Set.sum_indicator_subset _ (Finset.subset_univ s1)] at hw1
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
hweq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
hw1' : ∑ i : ι, Set.indicator (↑s1) w1 i = 1
⊢ Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
have hw2' : (∑ i, (s2 : Set ι).indicator w2 i) = 1 := by
rwa [Set.sum_indicator_subset _ (Finset.subset_univ s2)] at hw2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
hweq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
hw1' : ∑ i : ι, Set.indicator (↑s1) w1 i = 1
⊢ ∑ i : ι, Set.indicator (↑s2) w2 i = 1
[PROOFSTEP]
rwa [Set.sum_indicator_subset _ (Finset.subset_univ s2)] at hw2
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
hweq : ↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2
hw1' : ∑ i : ι, Set.indicator (↑s1) w1 i = 1
hw2' : ∑ i : ι, Set.indicator (↑s2) w2 i = 1
⊢ Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
rw [Finset.affineCombination_indicator_subset w1 p (Finset.subset_univ s1),
Finset.affineCombination_indicator_subset w2 p (Finset.subset_univ s2)] at hweq
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
h :
∀ (w1 w2 : ι → k),
∑ i : ι, w1 i = 1 →
∑ i : ι, w2 i = 1 →
↑(Finset.affineCombination k Finset.univ p) w1 = ↑(Finset.affineCombination k Finset.univ p) w2 → w1 = w2
s1 s2 : Finset ι
w1 w2 : ι → k
hw1 : ∑ i in s1, w1 i = 1
hw2 : ∑ i in s2, w2 i = 1
hweq :
↑(Finset.affineCombination k Finset.univ p) (Set.indicator (↑s1) w1) =
↑(Finset.affineCombination k Finset.univ p) (Set.indicator (↑s2) w2)
hw1' : ∑ i : ι, Set.indicator (↑s1) w1 i = 1
hw2' : ∑ i : ι, Set.indicator (↑s2) w2 i = 1
⊢ Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
[PROOFSTEP]
exact h _ _ hw1' hw2' hweq
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
hp : AffineIndependent k p
j : ι
w : ι → kˣ
⊢ AffineIndependent k fun i => ↑(AffineMap.lineMap (p j) (p i)) ↑(w i)
[PROOFSTEP]
rw [affineIndependent_iff_linearIndependent_vsub k _ j] at hp ⊢
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
j : ι
hp : LinearIndependent k fun i => p ↑i -ᵥ p j
w : ι → kˣ
⊢ LinearIndependent k fun i => ↑(AffineMap.lineMap (p j) (p ↑i)) ↑(w ↑i) -ᵥ ↑(AffineMap.lineMap (p j) (p j)) ↑(w j)
[PROOFSTEP]
simp only [AffineMap.lineMap_vsub_left, AffineMap.coe_const, AffineMap.lineMap_same, const_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
j : ι
hp : LinearIndependent k fun i => p ↑i -ᵥ p j
w : ι → kˣ
⊢ LinearIndependent k fun i => ↑(w ↑i) • (p ↑i -ᵥ p j)
[PROOFSTEP]
exact hp.units_smul fun i => w i
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
⊢ Injective p
[PROOFSTEP]
intro i j hij
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i j : ι
hij : p i = p j
⊢ i = j
[PROOFSTEP]
rw [affineIndependent_iff_linearIndependent_vsub _ _ j] at ha
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
i j : ι
ha : LinearIndependent k fun i => p ↑i -ᵥ p j
hij : p i = p j
⊢ i = j
[PROOFSTEP]
by_contra hij'
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
i j : ι
ha : LinearIndependent k fun i => p ↑i -ᵥ p j
hij : p i = p j
hij' : ¬i = j
⊢ False
[PROOFSTEP]
refine' ha.ne_zero ⟨i, hij'⟩ (vsub_eq_zero_iff_eq.mpr _)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
i j : ι
ha : LinearIndependent k fun i => p ↑i -ᵥ p j
hij : p i = p j
hij' : ¬i = j
⊢ p ↑{ val := i, property := hij' } = p j
[PROOFSTEP]
simp_all only [ne_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
⊢ AffineIndependent k (p ∘ ↑f)
[PROOFSTEP]
classical
intro fs w hw hs i0 hi0
let fs' := fs.map f
let w' i := if h : ∃ i2, f i2 = i then w h.choose else 0
have hw' : ∀ i2 : ι2, w' (f i2) = w i2 := by
intro i2
have h : ∃ i : ι2, f i = f i2 := ⟨i2, rfl⟩
have hs : h.choose = i2 := f.injective h.choose_spec
simp_rw [dif_pos h, hs]
have hw's : ∑ i in fs', w' i = 0 := by
rw [← hw, Finset.sum_map]
simp [hw']
have hs' : fs'.weightedVSub p w' = (0 : V) :=
by
rw [← hs, Finset.weightedVSub_map]
congr with i
simp_all only [comp_apply, EmbeddingLike.apply_eq_iff_eq, exists_eq, dite_true]
rw [← ha fs' w' hw's hs' (f i0) ((Finset.mem_map' _).2 hi0), hw']
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
⊢ AffineIndependent k (p ∘ ↑f)
[PROOFSTEP]
intro fs w hw hs i0 hi0
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
⊢ w i0 = 0
[PROOFSTEP]
let fs' := fs.map f
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
⊢ w i0 = 0
[PROOFSTEP]
let w' i := if h : ∃ i2, f i2 = i then w h.choose else 0
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
⊢ w i0 = 0
[PROOFSTEP]
have hw' : ∀ i2 : ι2, w' (f i2) = w i2 := by
intro i2
have h : ∃ i : ι2, f i = f i2 := ⟨i2, rfl⟩
have hs : h.choose = i2 := f.injective h.choose_spec
simp_rw [dif_pos h, hs]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
⊢ ∀ (i2 : ι2), w' (↑f i2) = w i2
[PROOFSTEP]
intro i2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
i2 : ι2
⊢ w' (↑f i2) = w i2
[PROOFSTEP]
have h : ∃ i : ι2, f i = f i2 := ⟨i2, rfl⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
i2 : ι2
h : ∃ i, ↑f i = ↑f i2
⊢ w' (↑f i2) = w i2
[PROOFSTEP]
have hs : h.choose = i2 := f.injective h.choose_spec
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs✝ : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
i2 : ι2
h : ∃ i, ↑f i = ↑f i2
hs : Exists.choose h = i2
⊢ w' (↑f i2) = w i2
[PROOFSTEP]
simp_rw [dif_pos h, hs]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
⊢ w i0 = 0
[PROOFSTEP]
have hw's : ∑ i in fs', w' i = 0 := by
rw [← hw, Finset.sum_map]
simp [hw']
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
⊢ ∑ i in fs', w' i = 0
[PROOFSTEP]
rw [← hw, Finset.sum_map]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
⊢ ∑ x in fs, w' (↑f x) = ∑ i in fs, w i
[PROOFSTEP]
simp [hw']
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
hw's : ∑ i in fs', w' i = 0
⊢ w i0 = 0
[PROOFSTEP]
have hs' : fs'.weightedVSub p w' = (0 : V) :=
by
rw [← hs, Finset.weightedVSub_map]
congr with i
simp_all only [comp_apply, EmbeddingLike.apply_eq_iff_eq, exists_eq, dite_true]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
hw's : ∑ i in fs', w' i = 0
⊢ ↑(Finset.weightedVSub fs' p) w' = 0
[PROOFSTEP]
rw [← hs, Finset.weightedVSub_map]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
hw's : ∑ i in fs', w' i = 0
⊢ ↑(Finset.weightedVSub fs (p ∘ ↑f)) (w' ∘ ↑f) = ↑(Finset.weightedVSub fs (p ∘ ↑f)) w
[PROOFSTEP]
congr with i
[GOAL]
case h.e_6.h.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
hw's : ∑ i in fs', w' i = 0
i : ι2
⊢ (w' ∘ ↑f) i = w i
[PROOFSTEP]
simp_all only [comp_apply, EmbeddingLike.apply_eq_iff_eq, exists_eq, dite_true]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι2 : Type u_5
f : ι2 ↪ ι
p : ι → P
ha : AffineIndependent k p
fs : Finset ι2
w : ι2 → k
hw : ∑ i in fs, w i = 0
hs : ↑(Finset.weightedVSub fs (p ∘ ↑f)) w = 0
i0 : ι2
hi0 : i0 ∈ fs
fs' : Finset ι := Finset.map f fs
w' : ι → k := fun i => if h : ∃ i2, ↑f i2 = i then w (Exists.choose h) else 0
hw' : ∀ (i2 : ι2), w' (↑f i2) = w i2
hw's : ∑ i in fs', w' i = 0
hs' : ↑(Finset.weightedVSub fs' p) w' = 0
⊢ w i0 = 0
[PROOFSTEP]
rw [← ha fs' w' hw's hs' (f i0) ((Finset.mem_map' _).2 hi0), hw']
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
⊢ AffineIndependent k fun x => ↑x
[PROOFSTEP]
let f : Set.range p → ι := fun x => x.property.choose
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
f : ↑(Set.range p) → ι := fun x => Exists.choose (_ : ↑x ∈ Set.range p)
⊢ AffineIndependent k fun x => ↑x
[PROOFSTEP]
have hf : ∀ x, p (f x) = x := fun x => x.property.choose_spec
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
f : ↑(Set.range p) → ι := fun x => Exists.choose (_ : ↑x ∈ Set.range p)
hf : ∀ (x : ↑(Set.range p)), p (f x) = ↑x
⊢ AffineIndependent k fun x => ↑x
[PROOFSTEP]
let fe : Set.range p ↪ ι := ⟨f, fun x₁ x₂ he => Subtype.ext (hf x₁ ▸ hf x₂ ▸ he ▸ rfl)⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
f : ↑(Set.range p) → ι := fun x => Exists.choose (_ : ↑x ∈ Set.range p)
hf : ∀ (x : ↑(Set.range p)), p (f x) = ↑x
fe : ↑(Set.range p) ↪ ι := { toFun := f, inj' := (_ : ∀ (x₁ x₂ : ↑(Set.range p)), f x₁ = f x₂ → x₁ = x₂) }
⊢ AffineIndependent k fun x => ↑x
[PROOFSTEP]
convert ha.comp_embedding fe
[GOAL]
case h.e'_9.h.h.e
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
f : ↑(Set.range p) → ι := fun x => Exists.choose (_ : ↑x ∈ Set.range p)
hf : ∀ (x : ↑(Set.range p)), p (f x) = ↑x
fe : ↑(Set.range p) ↪ ι := { toFun := f, inj' := (_ : ∀ (x₁ x₂ : ↑(Set.range p)), f x₁ = f x₂ → x₁ = x₂) }
x✝ : ↑(Set.range p)
⊢ Subtype.val = p ∘ ↑fe
[PROOFSTEP]
ext
[GOAL]
case h.e'_9.h.h.e.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
ha : AffineIndependent k p
f : ↑(Set.range p) → ι := fun x => Exists.choose (_ : ↑x ∈ Set.range p)
hf : ∀ (x : ↑(Set.range p)), p (f x) = ↑x
fe : ↑(Set.range p) ↪ ι := { toFun := f, inj' := (_ : ∀ (x₁ x₂ : ↑(Set.range p)), f x₁ = f x₂ → x₁ = x₂) }
x✝¹ : ↑(Set.range p)
x✝ : { x // x ∈ Set.range p }
⊢ ↑x✝ = (p ∘ ↑fe) x✝
[PROOFSTEP]
simp [hf]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
⊢ AffineIndependent k (p ∘ ↑e) ↔ AffineIndependent k p
[PROOFSTEP]
refine' ⟨_, AffineIndependent.comp_embedding e.toEmbedding⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
⊢ AffineIndependent k (p ∘ ↑e) → AffineIndependent k p
[PROOFSTEP]
intro h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
h : AffineIndependent k (p ∘ ↑e)
⊢ AffineIndependent k p
[PROOFSTEP]
have : p = p ∘ e ∘ e.symm.toEmbedding := by
ext
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
h : AffineIndependent k (p ∘ ↑e)
⊢ p = p ∘ ↑e ∘ ↑(Equiv.toEmbedding e.symm)
[PROOFSTEP]
ext
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
h : AffineIndependent k (p ∘ ↑e)
x✝ : ι'
⊢ p x✝ = (p ∘ ↑e ∘ ↑(Equiv.toEmbedding e.symm)) x✝
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
h : AffineIndependent k (p ∘ ↑e)
this : p = p ∘ ↑e ∘ ↑(Equiv.toEmbedding e.symm)
⊢ AffineIndependent k p
[PROOFSTEP]
rw [this]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
ι' : Type u_5
e : ι ≃ ι'
p : ι' → P
h : AffineIndependent k (p ∘ ↑e)
this : p = p ∘ ↑e ∘ ↑(Equiv.toEmbedding e.symm)
⊢ AffineIndependent k (p ∘ ↑e ∘ ↑(Equiv.toEmbedding e.symm))
[PROOFSTEP]
exact h.comp_embedding e.symm.toEmbedding
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hai : AffineIndependent k (↑f ∘ p)
⊢ AffineIndependent k p
[PROOFSTEP]
cases' isEmpty_or_nonempty ι with h h
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hai : AffineIndependent k (↑f ∘ p)
h : IsEmpty ι
⊢ AffineIndependent k p
[PROOFSTEP]
haveI := h
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hai : AffineIndependent k (↑f ∘ p)
h this : IsEmpty ι
⊢ AffineIndependent k p
[PROOFSTEP]
apply affineIndependent_of_subsingleton
[GOAL]
case inr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hai : AffineIndependent k (↑f ∘ p)
h : Nonempty ι
⊢ AffineIndependent k p
[PROOFSTEP]
obtain ⟨i⟩ := h
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hai : AffineIndependent k (↑f ∘ p)
i : ι
⊢ AffineIndependent k p
[PROOFSTEP]
rw [affineIndependent_iff_linearIndependent_vsub k p i]
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hai : AffineIndependent k (↑f ∘ p)
i : ι
⊢ LinearIndependent k fun i_1 => p ↑i_1 -ᵥ p i
[PROOFSTEP]
simp_rw [affineIndependent_iff_linearIndependent_vsub k (f ∘ p) i, Function.comp_apply, ← f.linearMap_vsub] at hai
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
i : ι
hai : LinearIndependent k fun i_1 => ↑f.linear (p ↑i_1 -ᵥ p i)
⊢ LinearIndependent k fun i_1 => p ↑i_1 -ᵥ p i
[PROOFSTEP]
exact LinearIndependent.of_comp f.linear hai
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
hai : AffineIndependent k p
f : P →ᵃ[k] P₂
hf : Injective ↑f
⊢ AffineIndependent k (↑f ∘ p)
[PROOFSTEP]
cases' isEmpty_or_nonempty ι with h h
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
hai : AffineIndependent k p
f : P →ᵃ[k] P₂
hf : Injective ↑f
h : IsEmpty ι
⊢ AffineIndependent k (↑f ∘ p)
[PROOFSTEP]
haveI := h
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
hai : AffineIndependent k p
f : P →ᵃ[k] P₂
hf : Injective ↑f
h this : IsEmpty ι
⊢ AffineIndependent k (↑f ∘ p)
[PROOFSTEP]
apply affineIndependent_of_subsingleton
[GOAL]
case inr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
hai : AffineIndependent k p
f : P →ᵃ[k] P₂
hf : Injective ↑f
h : Nonempty ι
⊢ AffineIndependent k (↑f ∘ p)
[PROOFSTEP]
obtain ⟨i⟩ := h
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
hai : AffineIndependent k p
f : P →ᵃ[k] P₂
hf : Injective ↑f
i : ι
⊢ AffineIndependent k (↑f ∘ p)
[PROOFSTEP]
rw [affineIndependent_iff_linearIndependent_vsub k p i] at hai
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hf : Injective ↑f
i : ι
hai : LinearIndependent k fun i_1 => p ↑i_1 -ᵥ p i
⊢ AffineIndependent k (↑f ∘ p)
[PROOFSTEP]
simp_rw [affineIndependent_iff_linearIndependent_vsub k (f ∘ p) i, Function.comp_apply, ← f.linearMap_vsub]
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hf : Injective ↑f
i : ι
hai : LinearIndependent k fun i_1 => p ↑i_1 -ᵥ p i
⊢ LinearIndependent k fun i_1 => ↑f.linear (p ↑i_1 -ᵥ p i)
[PROOFSTEP]
have hf' : LinearMap.ker f.linear = ⊥ := by rwa [LinearMap.ker_eq_bot, f.linear_injective_iff]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hf : Injective ↑f
i : ι
hai : LinearIndependent k fun i_1 => p ↑i_1 -ᵥ p i
⊢ LinearMap.ker f.linear = ⊥
[PROOFSTEP]
rwa [LinearMap.ker_eq_bot, f.linear_injective_iff]
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
f : P →ᵃ[k] P₂
hf : Injective ↑f
i : ι
hai : LinearIndependent k fun i_1 => p ↑i_1 -ᵥ p i
hf' : LinearMap.ker f.linear = ⊥
⊢ LinearIndependent k fun i_1 => ↑f.linear (p ↑i_1 -ᵥ p i)
[PROOFSTEP]
exact LinearIndependent.map' hai f.linear hf'
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
s : Set P
e : P ≃ᵃ[k] P₂
⊢ AffineIndependent k Subtype.val ↔ AffineIndependent k Subtype.val
[PROOFSTEP]
have : e ∘ ((↑) : s → P) = ((↑) : e '' s → P₂) ∘ (e : P ≃ P₂).image s := rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module k V
inst✝³ : AffineSpace V P
ι : Type u_4
V₂ : Type u_5
P₂ : Type u_6
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
s : Set P
e : P ≃ᵃ[k] P₂
this : ↑e ∘ Subtype.val = Subtype.val ∘ ↑(Equiv.image (↑e) s)
⊢ AffineIndependent k Subtype.val ↔ AffineIndependent k Subtype.val
[PROOFSTEP]
rw [← e.affineIndependent_iff, this, affineIndependent_equiv]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
p0 : P
hp0s1 : p0 ∈ affineSpan k (p '' s1)
hp0s2 : p0 ∈ affineSpan k (p '' s2)
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
rw [Set.image_eq_range] at hp0s1 hp0s2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
p0 : P
hp0s1 : p0 ∈ affineSpan k (Set.range fun x => p ↑x)
hp0s2 : p0 ∈ affineSpan k (Set.range fun x => p ↑x)
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
rw [mem_affineSpan_iff_eq_affineCombination, ← Finset.eq_affineCombination_subset_iff_eq_affineCombination_subtype] at
hp0s1 hp0s2
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
p0 : P
hp0s1 : ∃ fs x w x, p0 = ↑(Finset.affineCombination k fs p) w
hp0s2 : ∃ fs x w x, p0 = ↑(Finset.affineCombination k fs p) w
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
rcases hp0s1 with ⟨fs1, hfs1, w1, hw1, hp0s1⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
p0 : P
hp0s2 : ∃ fs x w x, p0 = ↑(Finset.affineCombination k fs p) w
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
rcases hp0s2 with ⟨fs2, hfs2, w2, hw2, hp0s2⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
rw [affineIndependent_iff_indicator_eq_of_affineCombination_eq] at ha
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha :
∀ (s1 s2 : Finset ι) (w1 w2 : ι → k),
∑ i in s1, w1 i = 1 →
∑ i in s2, w2 i = 1 →
↑(Finset.affineCombination k s1 p) w1 = ↑(Finset.affineCombination k s2 p) w2 →
Set.indicator (↑s1) w1 = Set.indicator (↑s2) w2
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
replace ha := ha fs1 fs2 w1 w2 hw1 hw2 (hp0s1 ▸ hp0s2)
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
ha : Set.indicator (↑fs1) w1 = Set.indicator (↑fs2) w2
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
have hnz : ∑ i in fs1, w1 i ≠ 0 := hw1.symm ▸ one_ne_zero
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
ha : Set.indicator (↑fs1) w1 = Set.indicator (↑fs2) w2
hnz : ∑ i in fs1, w1 i ≠ 0
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
rcases Finset.exists_ne_zero_of_sum_ne_zero hnz with ⟨i, hifs1, hinz⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
ha : Set.indicator (↑fs1) w1 = Set.indicator (↑fs2) w2
hnz : ∑ i in fs1, w1 i ≠ 0
i : ι
hifs1 : i ∈ fs1
hinz : w1 i ≠ 0
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
simp_rw [← Set.indicator_of_mem (Finset.mem_coe.2 hifs1) w1, ha] at hinz
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
ha : Set.indicator (↑fs1) w1 = Set.indicator (↑fs2) w2
hnz : ∑ i in fs1, w1 i ≠ 0
i : ι
hifs1 : i ∈ fs1
hinz : Set.indicator (↑fs2) w2 i ≠ 0
⊢ ∃ i, i ∈ s1 ∩ s2
[PROOFSTEP]
use i, hfs1 hifs1
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
s1 s2 : Set ι
p0 : P
fs1 : Finset ι
hfs1 : ↑fs1 ⊆ s1
w1 : ι → k
hw1 : ∑ i in fs1, w1 i = 1
hp0s1 : p0 = ↑(Finset.affineCombination k fs1 p) w1
fs2 : Finset ι
hfs2 : ↑fs2 ⊆ s2
w2 : ι → k
hw2 : ∑ i in fs2, w2 i = 1
hp0s2 : p0 = ↑(Finset.affineCombination k fs2 p) w2
ha : Set.indicator (↑fs1) w1 = Set.indicator (↑fs2) w2
hnz : ∑ i in fs1, w1 i ≠ 0
i : ι
hifs1 : i ∈ fs1
hinz : Set.indicator (↑fs2) w2 i ≠ 0
⊢ i ∈ s2
[PROOFSTEP]
exact hfs2 (Set.mem_of_indicator_ne_zero hinz)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
hd : Disjoint s1 s2
⊢ Disjoint ↑(affineSpan k (p '' s1)) ↑(affineSpan k (p '' s2))
[PROOFSTEP]
refine' Set.disjoint_left.2 fun p0 hp0s1 hp0s2 => _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
hd : Disjoint s1 s2
p0 : P
hp0s1 : p0 ∈ ↑(affineSpan k (p '' s1))
hp0s2 : p0 ∈ ↑(affineSpan k (p '' s2))
⊢ False
[PROOFSTEP]
cases' ha.exists_mem_inter_of_exists_mem_inter_affineSpan hp0s1 hp0s2 with i hi
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
s1 s2 : Set ι
hd : Disjoint s1 s2
p0 : P
hp0s1 : p0 ∈ ↑(affineSpan k (p '' s1))
hp0s2 : p0 ∈ ↑(affineSpan k (p '' s2))
i : ι
hi : i ∈ s1 ∩ s2
⊢ False
[PROOFSTEP]
exact Set.disjoint_iff.1 hd hi
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i : ι
s : Set ι
⊢ p i ∈ affineSpan k (p '' s) ↔ i ∈ s
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i : ι
s : Set ι
⊢ p i ∈ affineSpan k (p '' s) → i ∈ s
[PROOFSTEP]
intro hs
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i : ι
s : Set ι
hs : p i ∈ affineSpan k (p '' s)
⊢ i ∈ s
[PROOFSTEP]
have h :=
AffineIndependent.exists_mem_inter_of_exists_mem_inter_affineSpan ha hs
(mem_affineSpan k (Set.mem_image_of_mem _ (Set.mem_singleton _)))
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i : ι
s : Set ι
hs : p i ∈ affineSpan k (p '' s)
h : ∃ i_1, i_1 ∈ s ∩ {i}
⊢ i ∈ s
[PROOFSTEP]
rwa [← Set.nonempty_def, Set.inter_singleton_nonempty] at h
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i : ι
s : Set ι
⊢ i ∈ s → p i ∈ affineSpan k (p '' s)
[PROOFSTEP]
exact fun h => mem_affineSpan k (Set.mem_image_of_mem p h)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
ha : AffineIndependent k p
i : ι
s : Set ι
⊢ ¬p i ∈ affineSpan k (p '' (s \ {i}))
[PROOFSTEP]
simp [ha]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
h : ¬AffineIndependent k Subtype.val
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
classical
rw [affineIndependent_iff_of_fintype] at h
simp only [exists_prop, not_forall] at h
obtain ⟨w, hw, hwt, i, hi⟩ := h
simp only [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero _ w ((↑) : t → V) hw 0, vsub_eq_sub,
Finset.weightedVSubOfPoint_apply, sub_zero] at hwt
let f : ∀ x : V, x ∈ t → k := fun x hx => w ⟨x, hx⟩
refine' ⟨fun x => if hx : x ∈ t then f x hx else (0 : k), _, _, by use i; simp [hi]⟩
suffices (∑ e : V in t, dite (e ∈ t) (fun hx => f e hx • e) fun _ => 0) = 0
by
convert this
rename V => x
by_cases hx : x ∈ t <;> simp [hx]
all_goals simp only [Finset.sum_dite_of_true fun _ h => h, Finset.mk_coe, hwt, hw]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
h : ¬AffineIndependent k Subtype.val
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
rw [affineIndependent_iff_of_fintype] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
h :
¬∀ (w : { x // x ∈ t } → k),
∑ i : { x // x ∈ t }, w i = 0 →
↑(Finset.weightedVSub Finset.univ Subtype.val) w = 0 → ∀ (i : { x // x ∈ t }), w i = 0
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
simp only [exists_prop, not_forall] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
h : ∃ x, ∑ i : { x // x ∈ t }, x i = 0 ∧ ↑(Finset.weightedVSub Finset.univ Subtype.val) x = 0 ∧ ∃ x_1, ¬x x_1 = 0
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
obtain ⟨w, hw, hwt, i, hi⟩ := h
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
hwt : ↑(Finset.weightedVSub Finset.univ Subtype.val) w = 0
i : { x // x ∈ t }
hi : ¬w i = 0
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
simp only [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero _ w ((↑) : t → V) hw 0, vsub_eq_sub,
Finset.weightedVSubOfPoint_apply, sub_zero] at hwt
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
let f : ∀ x : V, x ∈ t → k := fun x hx => w ⟨x, hx⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ∃ f, ∑ e in t, f e • e = 0 ∧ ∑ e in t, f e = 0 ∧ ∃ x, x ∈ t ∧ f x ≠ 0
[PROOFSTEP]
refine' ⟨fun x => if hx : x ∈ t then f x hx else (0 : k), _, _, by use i; simp [hi]⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ∃ x, x ∈ t ∧ (fun x => if hx : x ∈ t then f x hx else 0) x ≠ 0
[PROOFSTEP]
use i
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ↑i ∈ t ∧ (fun x => if hx : x ∈ t then f x hx else 0) ↑i ≠ 0
[PROOFSTEP]
simp [hi]
[GOAL]
case intro.intro.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ∑ e in t, (fun x => if hx : x ∈ t then f x hx else 0) e • e = 0
case intro.intro.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ∑ e in t, (fun x => if hx : x ∈ t then f x hx else 0) e = 0
[PROOFSTEP]
suffices (∑ e : V in t, dite (e ∈ t) (fun hx => f e hx • e) fun _ => 0) = 0
by
convert this
rename V => x
by_cases hx : x ∈ t <;> simp [hx]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
this : (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
⊢ ∑ e in t, (fun x => if hx : x ∈ t then f x hx else 0) e • e = 0
[PROOFSTEP]
convert this
[GOAL]
case h.e'_2.a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
this : (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
x✝ : V
a✝ : x✝ ∈ t
⊢ (fun x => if hx : x ∈ t then f x hx else 0) x✝ • x✝ = if hx : x✝ ∈ t then f x✝ hx • x✝ else 0
[PROOFSTEP]
rename V => x
[GOAL]
case h.e'_2.a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
this : (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
x : V
a✝ : x ∈ t
⊢ (fun x => if hx : x ∈ t then f x hx else 0) x • x = if hx : x ∈ t then f x hx • x else 0
[PROOFSTEP]
by_cases hx : x ∈ t
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
this : (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
x : V
a✝ hx : x ∈ t
⊢ (fun x => if hx : x ∈ t then f x hx else 0) x • x = if hx : x ∈ t then f x hx • x else 0
[PROOFSTEP]
simp [hx]
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
this : (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
x : V
a✝ : x ∈ t
hx : ¬x ∈ t
⊢ (fun x => if hx : x ∈ t then f x hx else 0) x • x = if hx : x ∈ t then f x hx • x else 0
[PROOFSTEP]
simp [hx]
[GOAL]
case intro.intro.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
case intro.intro.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ∑ e in t, (fun x => if hx : x ∈ t then f x hx else 0) e = 0
[PROOFSTEP]
all_goals simp only [Finset.sum_dite_of_true fun _ h => h, Finset.mk_coe, hwt, hw]
[GOAL]
case intro.intro.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ (∑ e in t, if hx : e ∈ t then f e hx • e else 0) = 0
[PROOFSTEP]
simp only [Finset.sum_dite_of_true fun _ h => h, Finset.mk_coe, hwt, hw]
[GOAL]
case intro.intro.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
t : Finset V
w : { x // x ∈ t } → k
hw : ∑ i : { x // x ∈ t }, w i = 0
i : { x // x ∈ t }
hi : ¬w i = 0
hwt : ∑ x : { x // x ∈ t }, w x • ↑x = 0
f : (x : V) → x ∈ t → k := fun x hx => w { val := x, property := hx }
⊢ ∑ e in t, (fun x => if hx : x ∈ t then f x hx else 0) e = 0
[PROOFSTEP]
simp only [Finset.sum_dite_of_true fun _ h => h, Finset.mk_coe, hwt, hw]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι✝ : Type u_4
ι : Type u_5
p : ι → V
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
⊢ (↑(Finset.weightedVSub s p) w = 0 → ∀ (i : ι), i ∈ s → w i = 0) ↔ ∑ e in s, w e • p e = 0 → ∀ (e : ι), e ∈ s → w e = 0
[PROOFSTEP]
simp [s.weightedVSub_eq_linear_combination hw]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
⊢ ↑(Finset.weightedVSub s p) w ∈
vectorSpan k {↑(Finset.affineCombination k s p) w₁, ↑(Finset.affineCombination k s p) w₂} ↔
∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
rw [mem_vectorSpan_pair]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
⊢ (∃ r,
r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) =
↑(Finset.weightedVSub s p) w) ↔
∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
refine' ⟨fun h => _, fun h => _⟩
[GOAL]
case refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h✝ : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
h :
∃ r, r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
⊢ ∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
rcases h with ⟨r, hr⟩
[GOAL]
case refine'_1.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr : r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
⊢ ∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
refine' ⟨r, fun i hi => _⟩
[GOAL]
case refine'_1.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr : r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
i : ι
hi : i ∈ s
⊢ w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
rw [s.affineCombination_vsub, ← s.weightedVSub_const_smul, ← sub_eq_zero, ← map_sub] at hr
[GOAL]
case refine'_1.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr✝ : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂)) = ↑(Finset.weightedVSub s p) w
hr : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂) - w) = 0
i : ι
hi : i ∈ s
⊢ w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
have hw' : (∑ j in s, (r • (w₁ - w₂) - w) j) = 0 := by
simp_rw [Pi.sub_apply, Pi.smul_apply, Pi.sub_apply, smul_sub, Finset.sum_sub_distrib, ← Finset.smul_sum, hw, hw₁, hw₂,
sub_self]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr✝ : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂)) = ↑(Finset.weightedVSub s p) w
hr : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂) - w) = 0
i : ι
hi : i ∈ s
⊢ ∑ j in s, (r • (w₁ - w₂) - w) j = 0
[PROOFSTEP]
simp_rw [Pi.sub_apply, Pi.smul_apply, Pi.sub_apply, smul_sub, Finset.sum_sub_distrib, ← Finset.smul_sum, hw, hw₁, hw₂,
sub_self]
[GOAL]
case refine'_1.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr✝ : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂)) = ↑(Finset.weightedVSub s p) w
hr : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂) - w) = 0
i : ι
hi : i ∈ s
hw' : ∑ j in s, (r • (w₁ - w₂) - w) j = 0
⊢ w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
have hr' := h s _ hw' hr i hi
[GOAL]
case refine'_1.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr✝ : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂)) = ↑(Finset.weightedVSub s p) w
hr : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂) - w) = 0
i : ι
hi : i ∈ s
hw' : ∑ j in s, (r • (w₁ - w₂) - w) j = 0
hr' : (r • (w₁ - w₂) - w) i = 0
⊢ w i = r * (w₁ i - w₂ i)
[PROOFSTEP]
rw [eq_comm, ← sub_eq_zero, ← smul_eq_mul]
[GOAL]
case refine'_1.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr✝ : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂)) = ↑(Finset.weightedVSub s p) w
hr : ↑(Finset.weightedVSub s p) (r • (w₁ - w₂) - w) = 0
i : ι
hi : i ∈ s
hw' : ∑ j in s, (r • (w₁ - w₂) - w) j = 0
hr' : (r • (w₁ - w₂) - w) i = 0
⊢ r • (w₁ i - w₂ i) - w i = 0
[PROOFSTEP]
exact hr'
[GOAL]
case refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h✝ : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
h : ∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
⊢ ∃ r, r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rcases h with ⟨r, hr⟩
[GOAL]
case refine'_2.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr : ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
⊢ ∃ r, r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
refine' ⟨r, _⟩
[GOAL]
case refine'_2.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr : ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
⊢ r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
let w' i := r * (w₁ i - w₂ i)
[GOAL]
case refine'_2.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
hr : ∀ (i : ι), i ∈ s → w i = r * (w₁ i - w₂ i)
w' : ι → k := fun i => r * (w₁ i - w₂ i)
⊢ r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
change ∀ i ∈ s, w i = w' i at hr
[GOAL]
case refine'_2.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
w' : ι → k := fun i => r * (w₁ i - w₂ i)
hr : ∀ (i : ι), i ∈ s → w i = w' i
⊢ r • (↑(Finset.affineCombination k s p) w₁ -ᵥ ↑(Finset.affineCombination k s p) w₂) = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rw [s.weightedVSub_congr hr fun _ _ => rfl, s.affineCombination_vsub, ← s.weightedVSub_const_smul]
[GOAL]
case refine'_2.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 0
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
r : k
w' : ι → k := fun i => r * (w₁ i - w₂ i)
hr : ∀ (i : ι), i ∈ s → w i = w' i
⊢ ↑(Finset.weightedVSub s p) (r • (w₁ - w₂)) = ↑(Finset.weightedVSub s fun x => p x) fun i => w' i
[PROOFSTEP]
congr
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
x✝ : ∑ i in s, w i = 1
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
⊢ ↑(Finset.affineCombination k s p) w ∈
affineSpan k {↑(Finset.affineCombination k s p) w₁, ↑(Finset.affineCombination k s p) w₂} ↔
∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₂ i - w₁ i) + w₁ i
[PROOFSTEP]
rw [← vsub_vadd (s.affineCombination k p w) (s.affineCombination k p w₁),
AffineSubspace.vadd_mem_iff_mem_direction _ (left_mem_affineSpan_pair _ _ _), direction_affineSpan,
s.affineCombination_vsub, Set.pair_comm, weightedVSub_mem_vectorSpan_pair h _ hw₂ hw₁]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
x✝ : ∑ i in s, w i = 1
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
⊢ (∃ r, ∀ (i : ι), i ∈ s → (w - w₁) i = r * (w₂ i - w₁ i)) ↔ ∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₂ i - w₁ i) + w₁ i
[PROOFSTEP]
simp only [Pi.sub_apply, sub_eq_iff_eq_add]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
x✝ : ∑ i in s, w i = 1
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
⊢ ∑ i in s, (w - w₁) i = 0
[PROOFSTEP]
simp_all only [Pi.sub_apply, Finset.sum_sub_distrib, sub_self]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
h : AffineIndependent k fun p => ↑p
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
rcases s.eq_empty_or_nonempty with (rfl | ⟨p₁, hp₁⟩)
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have p₁ : P := AddTorsor.Nonempty.some
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
let hsv := Basis.ofVectorSpace k V
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have hsvi := hsv.linearIndependent
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : LinearIndependent k ↑hsv
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have hsvt := hsv.span_eq
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : LinearIndependent k ↑hsv
hsvt : Submodule.span k (Set.range ↑hsv) = ⊤
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
rw [Basis.coe_ofVectorSpace] at hsvi hsvt
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have h0 : ∀ v : V, v ∈ Basis.ofVectorSpaceIndex _ _ → v ≠ 0 :=
by
intro v hv
simpa using hsv.ne_zero ⟨v, hv⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
⊢ ∀ (v : V), v ∈ Basis.ofVectorSpaceIndex (?m.389241 v) V → v ≠ 0
[PROOFSTEP]
intro v hv
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
v : V
hv : v ∈ Basis.ofVectorSpaceIndex (?m.389241 v) V
⊢ v ≠ 0
[PROOFSTEP]
simpa using hsv.ne_zero ⟨v, hv⟩
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
h0 : ∀ (v : V), v ∈ Basis.ofVectorSpaceIndex k V → v ≠ 0
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
rw [linearIndependent_set_iff_affineIndependent_vadd_union_singleton k h0 p₁] at hsvi
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
h : AffineIndependent k fun p => ↑p
p₁ : P
hsv : Basis (↑(Basis.ofVectorSpaceIndex k V)) k V := Basis.ofVectorSpace k V
hsvi : AffineIndependent k fun p => ↑p
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
h0 : ∀ (v : V), v ∈ Basis.ofVectorSpaceIndex k V → v ≠ 0
⊢ ∃ t, ∅ ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
exact
⟨{ p₁ } ∪ (fun v => v +ᵥ p₁) '' _, Set.empty_subset _, hsvi,
affineSpan_singleton_union_vadd_eq_top_of_span_eq_top p₁ hsvt⟩
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
h : AffineIndependent k fun p => ↑p
p₁ : P
hp₁ : p₁ ∈ s
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
rw [affineIndependent_set_iff_linearIndependent_vsub k hp₁] at h
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
let bsv := Basis.extend h
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have hsvi := bsv.linearIndependent
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k ↑bsv
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have hsvt := bsv.span_eq
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k ↑bsv
hsvt : Submodule.span k (Set.range ↑bsv) = ⊤
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
rw [Basis.coe_extend] at hsvi hsvt
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have hsv := h.subset_extend (Set.subset_univ _)
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
have h0 : ∀ v : V, v ∈ h.extend _ → v ≠ 0 := by
intro v hv
simpa using bsv.ne_zero ⟨v, hv⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
⊢ ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ ?m.393529 v) → v ≠ 0
[PROOFSTEP]
intro v hv
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
v : V
hv : v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ ?m.393529 v)
⊢ v ≠ 0
[PROOFSTEP]
simpa using bsv.ne_zero ⟨v, hv⟩
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : LinearIndependent k Subtype.val
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
h0 : ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ) → v ≠ 0
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
rw [linearIndependent_set_iff_affineIndependent_vadd_union_singleton k h0 p₁] at hsvi
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : AffineIndependent k fun p => ↑p
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
h0 : ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ) → v ≠ 0
⊢ ∃ t, s ⊆ t ∧ (AffineIndependent k fun p => ↑p) ∧ affineSpan k t = ⊤
[PROOFSTEP]
refine' ⟨{ p₁ } ∪ (fun v => v +ᵥ p₁) '' h.extend (Set.subset_univ _), _, _⟩
[GOAL]
case inr.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : AffineIndependent k fun p => ↑p
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
h0 : ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ) → v ≠ 0
⊢ s ⊆ {p₁} ∪ (fun v => v +ᵥ p₁) '' LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
[PROOFSTEP]
refine' Set.Subset.trans _ (Set.union_subset_union_right _ (Set.image_subset _ hsv))
[GOAL]
case inr.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : AffineIndependent k fun p => ↑p
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
h0 : ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ) → v ≠ 0
⊢ s ⊆ {p₁} ∪ (fun v => v +ᵥ p₁) '' ((fun p => p -ᵥ p₁) '' (s \ {p₁}))
[PROOFSTEP]
simp [Set.image_image]
[GOAL]
case inr.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : AffineIndependent k fun p => ↑p
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
h0 : ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ) → v ≠ 0
⊢ (AffineIndependent k fun p => ↑p) ∧
affineSpan k
({p₁} ∪ (fun v => v +ᵥ p₁) '' LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)) =
⊤
[PROOFSTEP]
use hsvi
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p₁ : P
h : LinearIndependent k fun v => ↑v
hp₁ : p₁ ∈ s
bsv : Basis (↑(LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ))) k V := Basis.extend h
hsvi : AffineIndependent k fun p => ↑p
hsvt : Submodule.span k (Set.range Subtype.val) = ⊤
hsv : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)
h0 : ∀ (v : V), v ∈ LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ) → v ≠ 0
⊢ affineSpan k
({p₁} ∪ (fun v => v +ᵥ p₁) '' LinearIndependent.extend h (_ : (fun p => p -ᵥ p₁) '' (s \ {p₁}) ⊆ Set.univ)) =
⊤
[PROOFSTEP]
exact affineSpan_singleton_union_vadd_eq_top_of_span_eq_top p₁ hsvt
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
⊢ ∃ t x, affineSpan k t = affineSpan k s ∧ AffineIndependent k Subtype.val
[PROOFSTEP]
rcases s.eq_empty_or_nonempty with (rfl | ⟨p, hp⟩)
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
⊢ ∃ t x, affineSpan k t = affineSpan k ∅ ∧ AffineIndependent k Subtype.val
[PROOFSTEP]
exact ⟨∅, Set.empty_subset ∅, rfl, affineIndependent_of_subsingleton k _⟩
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
⊢ ∃ t x, affineSpan k t = affineSpan k s ∧ AffineIndependent k Subtype.val
[PROOFSTEP]
obtain ⟨b, hb₁, hb₂, hb₃⟩ := exists_linearIndependent k ((Equiv.vaddConst p).symm '' s)
[GOAL]
case inr.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = Submodule.span k (↑(Equiv.vaddConst p).symm '' s)
hb₃ : LinearIndependent k Subtype.val
⊢ ∃ t x, affineSpan k t = affineSpan k s ∧ AffineIndependent k Subtype.val
[PROOFSTEP]
have hb₀ : ∀ v : V, v ∈ b → v ≠ 0 := fun v hv => hb₃.ne_zero (⟨v, hv⟩ : b)
[GOAL]
case inr.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = Submodule.span k (↑(Equiv.vaddConst p).symm '' s)
hb₃ : LinearIndependent k Subtype.val
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ ∃ t x, affineSpan k t = affineSpan k s ∧ AffineIndependent k Subtype.val
[PROOFSTEP]
rw [linearIndependent_set_iff_affineIndependent_vadd_union_singleton k hb₀ p] at hb₃
[GOAL]
case inr.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = Submodule.span k (↑(Equiv.vaddConst p).symm '' s)
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ ∃ t x, affineSpan k t = affineSpan k s ∧ AffineIndependent k Subtype.val
[PROOFSTEP]
refine' ⟨{ p } ∪ Equiv.vaddConst p '' b, _, _, hb₃⟩
[GOAL]
case inr.intro.intro.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = Submodule.span k (↑(Equiv.vaddConst p).symm '' s)
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ {p} ∪ ↑(Equiv.vaddConst p) '' b ⊆ s
[PROOFSTEP]
apply Set.union_subset (Set.singleton_subset_iff.mpr hp)
[GOAL]
case inr.intro.intro.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = Submodule.span k (↑(Equiv.vaddConst p).symm '' s)
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ ↑(Equiv.vaddConst p) '' b ⊆ s
[PROOFSTEP]
rwa [← (Equiv.vaddConst p).subset_image' b s]
[GOAL]
case inr.intro.intro.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = Submodule.span k (↑(Equiv.vaddConst p).symm '' s)
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ affineSpan k ({p} ∪ ↑(Equiv.vaddConst p) '' b) = affineSpan k s
[PROOFSTEP]
rw [Equiv.coe_vaddConst_symm, ← vectorSpan_eq_span_vsub_set_right k hp] at hb₂
[GOAL]
case inr.intro.intro.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ affineSpan k ({p} ∪ ↑(Equiv.vaddConst p) '' b) = affineSpan k s
[PROOFSTEP]
apply AffineSubspace.ext_of_direction_eq
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hd
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ AffineSubspace.direction (affineSpan k ({p} ∪ ↑(Equiv.vaddConst p) '' b)) = AffineSubspace.direction (affineSpan k s)
[PROOFSTEP]
have : Submodule.span k b = Submodule.span k (insert 0 b) := by simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ Submodule.span k b = Submodule.span k (insert 0 b)
[PROOFSTEP]
simp
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hd
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
this : Submodule.span k b = Submodule.span k (insert 0 b)
⊢ AffineSubspace.direction (affineSpan k ({p} ∪ ↑(Equiv.vaddConst p) '' b)) = AffineSubspace.direction (affineSpan k s)
[PROOFSTEP]
simp only [direction_affineSpan, ← hb₂, Equiv.coe_vaddConst, Set.singleton_union,
vectorSpan_eq_span_vsub_set_right k (Set.mem_insert p _), this]
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hd
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
this : Submodule.span k b = Submodule.span k (insert 0 b)
⊢ Submodule.span k ((fun x => x -ᵥ p) '' insert p ((fun a => a +ᵥ p) '' b)) = Submodule.span k (insert 0 b)
[PROOFSTEP]
congr
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hd.e_s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
this : Submodule.span k b = Submodule.span k (insert 0 b)
⊢ (fun x => x -ᵥ p) '' insert p ((fun a => a +ᵥ p) '' b) = insert 0 b
[PROOFSTEP]
change (Equiv.vaddConst p).symm '' insert p (Equiv.vaddConst p '' b) = _
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hd.e_s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
this : Submodule.span k b = Submodule.span k (insert 0 b)
⊢ ↑(Equiv.vaddConst p).symm '' insert p (↑(Equiv.vaddConst p) '' b) = insert 0 b
[PROOFSTEP]
rw [Set.image_insert_eq, ← Set.image_comp]
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hd.e_s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
this : Submodule.span k b = Submodule.span k (insert 0 b)
⊢ insert (↑(Equiv.vaddConst p).symm p) (↑(Equiv.vaddConst p).symm ∘ ↑(Equiv.vaddConst p) '' b) = insert 0 b
[PROOFSTEP]
simp
[GOAL]
case inr.intro.intro.intro.intro.refine'_2.hn
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ Set.Nonempty (↑(affineSpan k ({p} ∪ ↑(Equiv.vaddConst p) '' b)) ∩ ↑(affineSpan k s))
[PROOFSTEP]
use p
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ p ∈ ↑(affineSpan k ({p} ∪ ↑(Equiv.vaddConst p) '' b)) ∩ ↑(affineSpan k s)
[PROOFSTEP]
simp only [Equiv.coe_vaddConst, Set.singleton_union, Set.mem_inter_iff, coe_affineSpan]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Set P
p : P
hp : p ∈ s
b : Set V
hb₁ : b ⊆ ↑(Equiv.vaddConst p).symm '' s
hb₂ : Submodule.span k b = vectorSpan k s
hb₃ : AffineIndependent k fun p_1 => ↑p_1
hb₀ : ∀ (v : V), v ∈ b → v ≠ 0
⊢ p ∈ spanPoints k (insert p ((fun a => a +ᵥ p) '' b)) ∧ p ∈ spanPoints k s
[PROOFSTEP]
exact ⟨mem_spanPoints k _ _ (Set.mem_insert p _), mem_spanPoints k _ _ hp⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
⊢ AffineIndependent k ![p₁, p₂]
[PROOFSTEP]
rw [affineIndependent_iff_linearIndependent_vsub k ![p₁, p₂] 0]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
⊢ LinearIndependent k fun i => Matrix.vecCons p₁ ![p₂] ↑i -ᵥ Matrix.vecCons p₁ ![p₂] 0
[PROOFSTEP]
let i₁ : { x // x ≠ (0 : Fin 2) } := ⟨1, by norm_num⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
⊢ 1 ≠ 0
[PROOFSTEP]
norm_num
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
⊢ LinearIndependent k fun i => Matrix.vecCons p₁ ![p₂] ↑i -ᵥ Matrix.vecCons p₁ ![p₂] 0
[PROOFSTEP]
have he' : ∀ i, i = i₁ := by
rintro ⟨i, hi⟩
ext
fin_cases i
· simp at hi
· simp only [Fin.val_one]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
⊢ ∀ (i : { x // x ≠ 0 }), i = i₁
[PROOFSTEP]
rintro ⟨i, hi⟩
[GOAL]
case mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
i : Fin 2
hi : i ≠ 0
⊢ { val := i, property := hi } = i₁
[PROOFSTEP]
ext
[GOAL]
case mk.a.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
i : Fin 2
hi : i ≠ 0
⊢ ↑↑{ val := i, property := hi } = ↑↑i₁
[PROOFSTEP]
fin_cases i
[GOAL]
case mk.a.h.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
hi : { val := 0, isLt := (_ : 0 < 2) } ≠ 0
⊢ ↑↑{ val := { val := 0, isLt := (_ : 0 < 2) }, property := hi } = ↑↑i₁
[PROOFSTEP]
simp at hi
[GOAL]
case mk.a.h.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
hi : { val := 1, isLt := (_ : (fun a => a < 2) 1) } ≠ 0
⊢ ↑↑{ val := { val := 1, isLt := (_ : (fun a => a < 2) 1) }, property := hi } = ↑↑i₁
[PROOFSTEP]
simp only [Fin.val_one]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
he' : ∀ (i : { x // x ≠ 0 }), i = i₁
⊢ LinearIndependent k fun i => Matrix.vecCons p₁ ![p₂] ↑i -ᵥ Matrix.vecCons p₁ ![p₂] 0
[PROOFSTEP]
haveI : Unique { x // x ≠ (0 : Fin 2) } := ⟨⟨i₁⟩, he'⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
he' : ∀ (i : { x // x ≠ 0 }), i = i₁
this : Unique { x // x ≠ 0 }
⊢ LinearIndependent k fun i => Matrix.vecCons p₁ ![p₂] ↑i -ᵥ Matrix.vecCons p₁ ![p₂] 0
[PROOFSTEP]
apply linearIndependent_unique
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
he' : ∀ (i : { x // x ≠ 0 }), i = i₁
this : Unique { x // x ≠ 0 }
⊢ Matrix.vecCons p₁ ![p₂] ↑default -ᵥ Matrix.vecCons p₁ ![p₂] 0 ≠ 0
[PROOFSTEP]
rw [he' default]
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p₁ p₂ : P
h : p₁ ≠ p₂
i₁ : { x // x ≠ 0 } := { val := 1, property := (_ : 1 ≠ 0) }
he' : ∀ (i : { x // x ≠ 0 }), i = i₁
this : Unique { x // x ≠ 0 }
⊢ Matrix.vecCons p₁ ![p₂] ↑i₁ -ᵥ Matrix.vecCons p₁ ![p₂] 0 ≠ 0
[PROOFSTEP]
simpa using h.symm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
⊢ AffineIndependent k p
[PROOFSTEP]
classical
intro s w hw hs
let s' : Finset { y // y ≠ i } := s.subtype (· ≠ i)
let p' : { y // y ≠ i } → P := fun x => p x
by_cases his : i ∈ s ∧ w i ≠ 0
· refine' False.elim (hi _)
let wm : ι → k := -(w i)⁻¹ • w
have hms : s.weightedVSub p wm = (0 : V) := by simp [hs]
have hwm : ∑ i in s, wm i = 0 := by simp [← Finset.mul_sum, hw]
have hwmi : wm i = -1 := by simp [his.2]
let w' : { y // y ≠ i } → k := fun x => wm x
have hw' : ∑ x in s', w' x = 1 := by
simp_rw [Finset.sum_subtype_eq_sum_filter]
rw [← s.sum_filter_add_sum_filter_not (· ≠ i)] at hwm
simp_rw [Classical.not_not] at hwm
erw [Finset.filter_eq'] at hwm
simp_rw [if_pos his.1, Finset.sum_singleton, hwmi, ← sub_eq_add_neg, sub_eq_zero] at hwm
exact hwm
rw [← s.affineCombination_eq_of_weightedVSub_eq_zero_of_eq_neg_one hms his.1 hwmi, ←
(Subtype.range_coe : _ = {x | x ≠ i}), ← Set.range_comp, ← s.affineCombination_subtype_eq_filter]
exact affineCombination_mem_affineSpan hw' p'
· rw [not_and_or, Classical.not_not] at his
let w' : { y // y ≠ i } → k := fun x => w x
have hw' : ∑ x in s', w' x = 0 := by
simp_rw [Finset.sum_subtype_eq_sum_filter]
rw [Finset.sum_filter_of_ne, hw]
rintro x hxs hwx rfl
exact hwx (his.neg_resolve_left hxs)
have hs' : s'.weightedVSub p' w' = (0 : V) :=
by
simp_rw [Finset.weightedVSub_subtype_eq_filter]
rw [Finset.weightedVSub_filter_of_ne, hs]
rintro x hxs hwx rfl
exact hwx (his.neg_resolve_left hxs)
intro j hj
by_cases hji : j = i
· rw [hji] at hj
exact hji.symm ▸ his.neg_resolve_left hj
· exact ha s' w' hw' hs' ⟨j, hji⟩ (Finset.mem_subtype.2 hj)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
⊢ AffineIndependent k p
[PROOFSTEP]
intro s w hw hs
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
let s' : Finset { y // y ≠ i } := s.subtype (· ≠ i)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
let p' : { y // y ≠ i } → P := fun x => p x
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
by_cases his : i ∈ s ∧ w i ≠ 0
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
refine' False.elim (hi _)
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
let wm : ι → k := -(w i)⁻¹ • w
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
have hms : s.weightedVSub p wm = (0 : V) := by simp [hs]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
⊢ ↑(Finset.weightedVSub s p) wm = 0
[PROOFSTEP]
simp [hs]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
have hwm : ∑ i in s, wm i = 0 := by simp [← Finset.mul_sum, hw]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
⊢ ∑ i in s, wm i = 0
[PROOFSTEP]
simp [← Finset.mul_sum, hw]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
have hwmi : wm i = -1 := by simp [his.2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
⊢ wm i = -1
[PROOFSTEP]
simp [his.2]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
hwmi : wm i = -1
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
let w' : { y // y ≠ i } → k := fun x => wm x
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
have hw' : ∑ x in s', w' x = 1 := by
simp_rw [Finset.sum_subtype_eq_sum_filter]
rw [← s.sum_filter_add_sum_filter_not (· ≠ i)] at hwm
simp_rw [Classical.not_not] at hwm
erw [Finset.filter_eq'] at hwm
simp_rw [if_pos his.1, Finset.sum_singleton, hwmi, ← sub_eq_add_neg, sub_eq_zero] at hwm
exact hwm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
⊢ ∑ x in s', w' x = 1
[PROOFSTEP]
simp_rw [Finset.sum_subtype_eq_sum_filter]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
⊢ ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x = 1
[PROOFSTEP]
rw [← s.sum_filter_add_sum_filter_not (· ≠ i)] at hwm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ x in Finset.filter (fun x => x ≠ i) s, wm x + ∑ x in Finset.filter (fun x => ¬x ≠ i) s, wm x = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
⊢ ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x = 1
[PROOFSTEP]
simp_rw [Classical.not_not] at hwm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
hwm :
∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x +
∑ x in Finset.filter (fun x => x = i) s, (-(w i)⁻¹ • w) x =
0
⊢ ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x = 1
[PROOFSTEP]
erw [Finset.filter_eq'] at hwm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
hwm : ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x + ∑ x in if i ∈ s then {i} else ∅, (-(w i)⁻¹ • w) x = 0
⊢ ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x = 1
[PROOFSTEP]
simp_rw [if_pos his.1, Finset.sum_singleton, hwmi, ← sub_eq_add_neg, sub_eq_zero] at hwm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
hwm : ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x = 1
⊢ ∑ x in Finset.filter (fun x => x ≠ i) s, (-(w i)⁻¹ • w) x = 1
[PROOFSTEP]
exact hwm
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
hw' : ∑ x in s', w' x = 1
⊢ p i ∈ affineSpan k (p '' {x | x ≠ i})
[PROOFSTEP]
rw [← s.affineCombination_eq_of_weightedVSub_eq_zero_of_eq_neg_one hms his.1 hwmi, ←
(Subtype.range_coe : _ = {x | x ≠ i}), ← Set.range_comp, ← s.affineCombination_subtype_eq_filter]
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : i ∈ s ∧ w i ≠ 0
wm : ι → k := -(w i)⁻¹ • w
hms : ↑(Finset.weightedVSub s p) wm = 0
hwm : ∑ i in s, wm i = 0
hwmi : wm i = -1
w' : { y // y ≠ i } → k := fun x => wm ↑x
hw' : ∑ x in s', w' x = 1
⊢ (↑(Finset.affineCombination k (Finset.subtype (fun x => x ≠ i) s) fun i_1 => p ↑i_1) fun i_1 => wm ↑i_1) ∈
affineSpan k (Set.range (p ∘ Subtype.val))
[PROOFSTEP]
exact affineCombination_mem_affineSpan hw' p'
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬(i ∈ s ∧ w i ≠ 0)
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
rw [not_and_or, Classical.not_not] at his
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
let w' : { y // y ≠ i } → k := fun x => w x
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
have hw' : ∑ x in s', w' x = 0 := by
simp_rw [Finset.sum_subtype_eq_sum_filter]
rw [Finset.sum_filter_of_ne, hw]
rintro x hxs hwx rfl
exact hwx (his.neg_resolve_left hxs)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
⊢ ∑ x in s', w' x = 0
[PROOFSTEP]
simp_rw [Finset.sum_subtype_eq_sum_filter]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
⊢ ∑ x in Finset.filter (fun x => x ≠ i) s, w x = 0
[PROOFSTEP]
rw [Finset.sum_filter_of_ne, hw]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
⊢ ∀ (x : ι), x ∈ s → w x ≠ 0 → x ≠ i
[PROOFSTEP]
rintro x hxs hwx rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
x : ι
hxs : x ∈ s
hwx : w x ≠ 0
ha : AffineIndependent k fun x_1 => p ↑x_1
hi : ¬p x ∈ affineSpan k (p '' {x_1 | x_1 ≠ x})
s' : Finset { y // y ≠ x } := Finset.subtype (fun x_1 => x_1 ≠ x) s
p' : { y // y ≠ x } → P := fun x_1 => p ↑x_1
his : ¬x ∈ s ∨ w x = 0
w' : { y // y ≠ x } → k := fun x_1 => w ↑x_1
⊢ False
[PROOFSTEP]
exact hwx (his.neg_resolve_left hxs)
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
have hs' : s'.weightedVSub p' w' = (0 : V) :=
by
simp_rw [Finset.weightedVSub_subtype_eq_filter]
rw [Finset.weightedVSub_filter_of_ne, hs]
rintro x hxs hwx rfl
exact hwx (his.neg_resolve_left hxs)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
⊢ ↑(Finset.weightedVSub s' p') w' = 0
[PROOFSTEP]
simp_rw [Finset.weightedVSub_subtype_eq_filter]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
⊢ ↑(Finset.weightedVSub (Finset.filter (fun x => x ≠ i) s) p) w = 0
[PROOFSTEP]
rw [Finset.weightedVSub_filter_of_ne, hs]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
⊢ ∀ (i_1 : ι), i_1 ∈ s → w i_1 ≠ 0 → i_1 ≠ i
[PROOFSTEP]
rintro x hxs hwx rfl
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
x : ι
hxs : x ∈ s
hwx : w x ≠ 0
ha : AffineIndependent k fun x_1 => p ↑x_1
hi : ¬p x ∈ affineSpan k (p '' {x_1 | x_1 ≠ x})
s' : Finset { y // y ≠ x } := Finset.subtype (fun x_1 => x_1 ≠ x) s
p' : { y // y ≠ x } → P := fun x_1 => p ↑x_1
his : ¬x ∈ s ∨ w x = 0
w' : { y // y ≠ x } → k := fun x_1 => w ↑x_1
hw' : ∑ x in s', w' x = 0
⊢ False
[PROOFSTEP]
exact hwx (his.neg_resolve_left hxs)
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
hs' : ↑(Finset.weightedVSub s' p') w' = 0
⊢ ∀ (i : ι), i ∈ s → w i = 0
[PROOFSTEP]
intro j hj
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
hs' : ↑(Finset.weightedVSub s' p') w' = 0
j : ι
hj : j ∈ s
⊢ w j = 0
[PROOFSTEP]
by_cases hji : j = i
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
hs' : ↑(Finset.weightedVSub s' p') w' = 0
j : ι
hj : j ∈ s
hji : j = i
⊢ w j = 0
[PROOFSTEP]
rw [hji] at hj
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
hs' : ↑(Finset.weightedVSub s' p') w' = 0
j : ι
hj : i ∈ s
hji : j = i
⊢ w j = 0
[PROOFSTEP]
exact hji.symm ▸ his.neg_resolve_left hj
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
i : ι
ha : AffineIndependent k fun x => p ↑x
hi : ¬p i ∈ affineSpan k (p '' {x | x ≠ i})
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
hs : ↑(Finset.weightedVSub s p) w = 0
s' : Finset { y // y ≠ i } := Finset.subtype (fun x => x ≠ i) s
p' : { y // y ≠ i } → P := fun x => p ↑x
his : ¬i ∈ s ∨ w i = 0
w' : { y // y ≠ i } → k := fun x => w ↑x
hw' : ∑ x in s', w' x = 0
hs' : ↑(Finset.weightedVSub s' p') w' = 0
j : ι
hj : j ∈ s
hji : ¬j = i
⊢ w j = 0
[PROOFSTEP]
exact ha s' w' hw' hs' ⟨j, hji⟩ (Finset.mem_subtype.2 hj)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
⊢ AffineIndependent k ![p₁, p₂, p₃]
[PROOFSTEP]
have ha : AffineIndependent k fun x : { x : Fin 3 // x ≠ 2 } => ![p₁, p₂, p₃] x :=
by
rw [← affineIndependent_equiv (finSuccAboveEquiv (2 : Fin 3)).toEquiv]
convert affineIndependent_of_ne k hp₁p₂
ext x
fin_cases x <;> rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
⊢ AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
[PROOFSTEP]
rw [← affineIndependent_equiv (finSuccAboveEquiv (2 : Fin 3)).toEquiv]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
⊢ AffineIndependent k ((fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x) ∘ ↑(finSuccAboveEquiv 2).toEquiv)
[PROOFSTEP]
convert affineIndependent_of_ne k hp₁p₂
[GOAL]
case h.e'_9
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
⊢ (fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x) ∘ ↑(finSuccAboveEquiv 2).toEquiv = ![p₁, p₂]
[PROOFSTEP]
ext x
[GOAL]
case h.e'_9.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
x : Fin 2
⊢ ((fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x) ∘ ↑(finSuccAboveEquiv 2).toEquiv) x = Matrix.vecCons p₁ ![p₂] x
[PROOFSTEP]
fin_cases x
[GOAL]
case h.e'_9.h.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
⊢ ((fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x) ∘ ↑(finSuccAboveEquiv 2).toEquiv) { val := 0, isLt := (_ : 0 < 2) } =
Matrix.vecCons p₁ ![p₂] { val := 0, isLt := (_ : 0 < 2) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_9.h.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
⊢ ((fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x) ∘ ↑(finSuccAboveEquiv 2).toEquiv)
{ val := 1, isLt := (_ : (fun a => a < 2) 1) } =
Matrix.vecCons p₁ ![p₂] { val := 1, isLt := (_ : (fun a => a < 2) 1) }
[PROOFSTEP]
rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
⊢ AffineIndependent k ![p₁, p₂, p₃]
[PROOFSTEP]
refine' ha.affineIndependent_of_not_mem_span _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
⊢ ¬Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
[PROOFSTEP]
intro h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
⊢ False
[PROOFSTEP]
refine' hp₃ ((AffineSubspace.le_def' _ s).1 _ p₃ h)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
⊢ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2}) ≤ s
[PROOFSTEP]
simp_rw [affineSpan_le, Set.image_subset_iff, Set.subset_def, Set.mem_preimage]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
⊢ ∀ (x : Fin 3), x ∈ {x | x ≠ 2} → Matrix.vecCons p₁ ![p₂, p₃] x ∈ ↑s
[PROOFSTEP]
intro x
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
x : Fin 3
⊢ x ∈ {x | x ≠ 2} → Matrix.vecCons p₁ ![p₂, p₃] x ∈ ↑s
[PROOFSTEP]
fin_cases x
[GOAL]
case head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
⊢ { val := 0, isLt := (_ : 0 < 3) } ∈ {x | x ≠ 2} → Matrix.vecCons p₁ ![p₂, p₃] { val := 0, isLt := (_ : 0 < 3) } ∈ ↑s
[PROOFSTEP]
simp [hp₁, hp₂]
[GOAL]
case tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
⊢ { val := 1, isLt := (_ : (fun a => a < 3) 1) } ∈ {x | x ≠ 2} →
Matrix.vecCons p₁ ![p₂, p₃] { val := 1, isLt := (_ : (fun a => a < 3) 1) } ∈ ↑s
[PROOFSTEP]
simp [hp₁, hp₂]
[GOAL]
case tail.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₂ : p₁ ≠ p₂
hp₁ : p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : ¬p₃ ∈ s
ha : AffineIndependent k fun x => Matrix.vecCons p₁ ![p₂, p₃] ↑x
h : Matrix.vecCons p₁ ![p₂, p₃] 2 ∈ affineSpan k (![p₁, p₂, p₃] '' {x | x ≠ 2})
⊢ { val := 2, isLt := (_ : (fun a => (fun a => a < 3) a) 2) } ∈ {x | x ≠ 2} →
Matrix.vecCons p₁ ![p₂, p₃] { val := 2, isLt := (_ : (fun a => (fun a => a < 3) a) 2) } ∈ ↑s
[PROOFSTEP]
simp [hp₁, hp₂]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ AffineIndependent k ![p₁, p₂, p₃]
[PROOFSTEP]
rw [← affineIndependent_equiv (Equiv.swap (1 : Fin 3) 2)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ AffineIndependent k (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 1 2))
[PROOFSTEP]
convert affineIndependent_of_ne_of_mem_of_mem_of_not_mem hp₁p₃ hp₁ hp₃ hp₂ using 1
[GOAL]
case h.e'_9
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ ![p₁, p₂, p₃] ∘ ↑(Equiv.swap 1 2) = ![p₁, p₃, p₂]
[PROOFSTEP]
ext x
[GOAL]
case h.e'_9.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
x : Fin 3
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 1 2)) x = Matrix.vecCons p₁ ![p₃, p₂] x
[PROOFSTEP]
fin_cases x
[GOAL]
case h.e'_9.h.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 1 2)) { val := 0, isLt := (_ : 0 < 3) } =
Matrix.vecCons p₁ ![p₃, p₂] { val := 0, isLt := (_ : 0 < 3) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_9.h.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 1 2)) { val := 1, isLt := (_ : (fun a => a < 3) 1) } =
Matrix.vecCons p₁ ![p₃, p₂] { val := 1, isLt := (_ : (fun a => a < 3) 1) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_9.h.tail.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₁p₃ : p₁ ≠ p₃
hp₁ : p₁ ∈ s
hp₂ : ¬p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 1 2)) { val := 2, isLt := (_ : (fun a => (fun a => a < 3) a) 2) } =
Matrix.vecCons p₁ ![p₃, p₂] { val := 2, isLt := (_ : (fun a => (fun a => a < 3) a) 2) }
[PROOFSTEP]
rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ AffineIndependent k ![p₁, p₂, p₃]
[PROOFSTEP]
rw [← affineIndependent_equiv (Equiv.swap (0 : Fin 3) 2)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ AffineIndependent k (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 0 2))
[PROOFSTEP]
convert affineIndependent_of_ne_of_mem_of_mem_of_not_mem hp₂p₃.symm hp₃ hp₂ hp₁ using 1
[GOAL]
case h.e'_9
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ ![p₁, p₂, p₃] ∘ ↑(Equiv.swap 0 2) = ![p₃, p₂, p₁]
[PROOFSTEP]
ext x
[GOAL]
case h.e'_9.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
x : Fin 3
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 0 2)) x = Matrix.vecCons p₃ ![p₂, p₁] x
[PROOFSTEP]
fin_cases x
[GOAL]
case h.e'_9.h.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 0 2)) { val := 0, isLt := (_ : 0 < 3) } =
Matrix.vecCons p₃ ![p₂, p₁] { val := 0, isLt := (_ : 0 < 3) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_9.h.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 0 2)) { val := 1, isLt := (_ : (fun a => a < 3) 1) } =
Matrix.vecCons p₃ ![p₂, p₁] { val := 1, isLt := (_ : (fun a => a < 3) 1) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_9.h.tail.tail.head
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : AffineSubspace k P
p₁ p₂ p₃ : P
hp₂p₃ : p₂ ≠ p₃
hp₁ : ¬p₁ ∈ s
hp₂ : p₂ ∈ s
hp₃ : p₃ ∈ s
⊢ (![p₁, p₂, p₃] ∘ ↑(Equiv.swap 0 2)) { val := 2, isLt := (_ : (fun a => (fun a => a < 3) a) 2) } =
Matrix.vecCons p₃ ![p₂, p₁] { val := 2, isLt := (_ : (fun a => (fun a => a < 3) a) 2) }
[PROOFSTEP]
rfl
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
hs :
↑(Finset.affineCombination k s p) w ∈
affineSpan k {↑(Finset.affineCombination k s p) w₁, ↑(Finset.affineCombination k s p) w₂}
i j : ι
hi : i ∈ s
hj : j ∈ s
hi0 : w₁ i = 0
hj0 : w₁ j = 0
hij : ↑SignType.sign (w₂ i) = ↑SignType.sign (w₂ j)
⊢ ↑SignType.sign (w i) = ↑SignType.sign (w j)
[PROOFSTEP]
rw [affineCombination_mem_affineSpan_pair h hw hw₁ hw₂] at hs
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
hs : ∃ r, ∀ (i : ι), i ∈ s → w i = r * (w₂ i - w₁ i) + w₁ i
i j : ι
hi : i ∈ s
hj : j ∈ s
hi0 : w₁ i = 0
hj0 : w₁ j = 0
hij : ↑SignType.sign (w₂ i) = ↑SignType.sign (w₂ j)
⊢ ↑SignType.sign (w i) = ↑SignType.sign (w j)
[PROOFSTEP]
rcases hs with ⟨r, hr⟩
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w w₁ w₂ : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
hw₁ : ∑ i in s, w₁ i = 1
hw₂ : ∑ i in s, w₂ i = 1
i j : ι
hi : i ∈ s
hj : j ∈ s
hi0 : w₁ i = 0
hj0 : w₁ j = 0
hij : ↑SignType.sign (w₂ i) = ↑SignType.sign (w₂ j)
r : k
hr : ∀ (i : ι), i ∈ s → w i = r * (w₂ i - w₁ i) + w₁ i
⊢ ↑SignType.sign (w i) = ↑SignType.sign (w j)
[PROOFSTEP]
rw [hr i hi, hr j hj, hi0, hj0, add_zero, add_zero, sub_zero, sub_zero, sign_mul, sign_mul, hij]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
i₁ i₂ i₃ : ι
h₁ : i₁ ∈ s
h₂ : i₂ ∈ s
h₃ : i₃ ∈ s
h₁₂ : i₁ ≠ i₂
h₁₃ : i₁ ≠ i₃
h₂₃ : i₂ ≠ i₃
c : k
hc0 : 0 < c
hc1 : c < 1
hs : ↑(Finset.affineCombination k s p) w ∈ affineSpan k {p i₁, ↑(AffineMap.lineMap (p i₂) (p i₃)) c}
⊢ ↑SignType.sign (w i₂) = ↑SignType.sign (w i₃)
[PROOFSTEP]
classical
rw [← s.affineCombination_affineCombinationSingleWeights k p h₁, ←
s.affineCombination_affineCombinationLineMapWeights p h₂ h₃ c] at hs
refine'
sign_eq_of_affineCombination_mem_affineSpan_pair h hw (s.sum_affineCombinationSingleWeights k h₁)
(s.sum_affineCombinationLineMapWeights h₂ h₃ c) hs h₂ h₃
(Finset.affineCombinationSingleWeights_apply_of_ne k h₁₂.symm)
(Finset.affineCombinationSingleWeights_apply_of_ne k h₁₃.symm) _
rw [Finset.affineCombinationLineMapWeights_apply_left h₂₃, Finset.affineCombinationLineMapWeights_apply_right h₂₃]
simp_all only [sub_pos, sign_pos]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
i₁ i₂ i₃ : ι
h₁ : i₁ ∈ s
h₂ : i₂ ∈ s
h₃ : i₃ ∈ s
h₁₂ : i₁ ≠ i₂
h₁₃ : i₁ ≠ i₃
h₂₃ : i₂ ≠ i₃
c : k
hc0 : 0 < c
hc1 : c < 1
hs : ↑(Finset.affineCombination k s p) w ∈ affineSpan k {p i₁, ↑(AffineMap.lineMap (p i₂) (p i₃)) c}
⊢ ↑SignType.sign (w i₂) = ↑SignType.sign (w i₃)
[PROOFSTEP]
rw [← s.affineCombination_affineCombinationSingleWeights k p h₁, ←
s.affineCombination_affineCombinationLineMapWeights p h₂ h₃ c] at hs
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
i₁ i₂ i₃ : ι
h₁ : i₁ ∈ s
h₂ : i₂ ∈ s
h₃ : i₃ ∈ s
h₁₂ : i₁ ≠ i₂
h₁₃ : i₁ ≠ i₃
h₂₃ : i₂ ≠ i₃
c : k
hc0 : 0 < c
hc1 : c < 1
hs :
↑(Finset.affineCombination k s p) w ∈
affineSpan k
{↑(Finset.affineCombination k s p) (Finset.affineCombinationSingleWeights k i₁),
↑(Finset.affineCombination k s p) (Finset.affineCombinationLineMapWeights i₂ i₃ c)}
⊢ ↑SignType.sign (w i₂) = ↑SignType.sign (w i₃)
[PROOFSTEP]
refine'
sign_eq_of_affineCombination_mem_affineSpan_pair h hw (s.sum_affineCombinationSingleWeights k h₁)
(s.sum_affineCombinationLineMapWeights h₂ h₃ c) hs h₂ h₃
(Finset.affineCombinationSingleWeights_apply_of_ne k h₁₂.symm)
(Finset.affineCombinationSingleWeights_apply_of_ne k h₁₃.symm) _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
i₁ i₂ i₃ : ι
h₁ : i₁ ∈ s
h₂ : i₂ ∈ s
h₃ : i₃ ∈ s
h₁₂ : i₁ ≠ i₂
h₁₃ : i₁ ≠ i₃
h₂₃ : i₂ ≠ i₃
c : k
hc0 : 0 < c
hc1 : c < 1
hs :
↑(Finset.affineCombination k s p) w ∈
affineSpan k
{↑(Finset.affineCombination k s p) (Finset.affineCombinationSingleWeights k i₁),
↑(Finset.affineCombination k s p) (Finset.affineCombinationLineMapWeights i₂ i₃ c)}
⊢ ↑SignType.sign (Finset.affineCombinationLineMapWeights i₂ i₃ c i₂) =
↑SignType.sign (Finset.affineCombinationLineMapWeights i₂ i₃ c i₃)
[PROOFSTEP]
rw [Finset.affineCombinationLineMapWeights_apply_left h₂₃, Finset.affineCombinationLineMapWeights_apply_right h₂₃]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : LinearOrderedRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
h : AffineIndependent k p
w : ι → k
s : Finset ι
hw : ∑ i in s, w i = 1
i₁ i₂ i₃ : ι
h₁ : i₁ ∈ s
h₂ : i₂ ∈ s
h₃ : i₃ ∈ s
h₁₂ : i₁ ≠ i₂
h₁₃ : i₁ ≠ i₃
h₂₃ : i₂ ≠ i₃
c : k
hc0 : 0 < c
hc1 : c < 1
hs :
↑(Finset.affineCombination k s p) w ∈
affineSpan k
{↑(Finset.affineCombination k s p) (Finset.affineCombinationSingleWeights k i₁),
↑(Finset.affineCombination k s p) (Finset.affineCombinationLineMapWeights i₂ i₃ c)}
⊢ ↑SignType.sign (1 - c) = ↑SignType.sign c
[PROOFSTEP]
simp_all only [sub_pos, sign_pos]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
⊢ Subsingleton (Fin (1 + 0))
[PROOFSTEP]
rw [add_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
p : P
⊢ Subsingleton (Fin 1)
[PROOFSTEP]
infer_instance
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s1 s2 : Simplex k P n
h : ∀ (i : Fin (n + 1)), points s1 i = points s2 i
⊢ s1 = s2
[PROOFSTEP]
cases s1
[GOAL]
case mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s2 : Simplex k P n
points✝ : Fin (n + 1) → P
Independent✝ : AffineIndependent k points✝
h : ∀ (i : Fin (n + 1)), points { points := points✝, Independent := Independent✝ } i = points s2 i
⊢ { points := points✝, Independent := Independent✝ } = s2
[PROOFSTEP]
cases s2
[GOAL]
case mk.mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
points✝¹ : Fin (n + 1) → P
Independent✝¹ : AffineIndependent k points✝¹
points✝ : Fin (n + 1) → P
Independent✝ : AffineIndependent k points✝
h :
∀ (i : Fin (n + 1)),
points { points := points✝¹, Independent := Independent✝¹ } i =
points { points := points✝, Independent := Independent✝ } i
⊢ { points := points✝¹, Independent := Independent✝¹ } = { points := points✝, Independent := Independent✝ }
[PROOFSTEP]
congr with i
[GOAL]
case mk.mk.e_points.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
points✝¹ : Fin (n + 1) → P
Independent✝¹ : AffineIndependent k points✝¹
points✝ : Fin (n + 1) → P
Independent✝ : AffineIndependent k points✝
h :
∀ (i : Fin (n + 1)),
points { points := points✝¹, Independent := Independent✝¹ } i =
points { points := points✝, Independent := Independent✝ } i
i : Fin (n + 1)
⊢ points✝¹ i = points✝ i
[PROOFSTEP]
exact h i
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
i : Fin (n + 1)
⊢ face s (_ : Finset.card {i} = 1) = mkOfPoint k (points s i)
[PROOFSTEP]
ext
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
i : Fin (n + 1)
i✝ : Fin (0 + 1)
⊢ points (face s (_ : Finset.card {i} = 1)) i✝ = points (mkOfPoint k (points s i)) i✝
[PROOFSTEP]
simp only [Affine.Simplex.mkOfPoint_points, Affine.Simplex.face_points]
-- Porting note: `simp` can't use the next lemma
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
i : Fin (n + 1)
i✝ : Fin (0 + 1)
⊢ points s (↑(Finset.orderEmbOfFin {i} (_ : Finset.card {i} = 1)) i✝) = points s i
[PROOFSTEP]
rw [Finset.orderEmbOfFin_singleton]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
fs : Finset (Fin (n + 1))
m : ℕ
h : Finset.card fs = m + 1
⊢ Set.range (face s h).points = s.points '' ↑fs
[PROOFSTEP]
rw [face_points', Set.range_comp, Finset.range_orderEmbOfFin]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
m n : ℕ
s : Simplex k P m
e : Fin (m + 1) ≃ Fin (n + 1)
⊢ reindex (reindex s e) e.symm = s
[PROOFSTEP]
rw [← reindex_trans, Equiv.self_trans_symm, reindex_refl]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
m n : ℕ
s : Simplex k P m
e : Fin (n + 1) ≃ Fin (m + 1)
⊢ reindex (reindex s e.symm) e = s
[PROOFSTEP]
rw [← reindex_trans, Equiv.symm_trans_self, reindex_refl]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
m n : ℕ
s : Simplex k P m
e : Fin (m + 1) ≃ Fin (n + 1)
⊢ Set.range (reindex s e).points = Set.range s.points
[PROOFSTEP]
rw [reindex, Set.range_comp, Equiv.range_eq_univ, Set.image_univ]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
fs : Finset (Fin (n + 1))
m : ℕ
h : Finset.card fs = m + 1
⊢ Finset.centroid k Finset.univ (face s h).points = Finset.centroid k fs s.points
[PROOFSTEP]
convert (Finset.univ.centroid_map k (fs.orderEmbOfFin h).toEmbedding s.points).symm
[GOAL]
case h.e'_3.h.e'_9
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
fs : Finset (Fin (n + 1))
m : ℕ
h : Finset.card fs = m + 1
⊢ fs = Finset.map (Finset.orderEmbOfFin fs h).toEmbedding Finset.univ
[PROOFSTEP]
rw [← Finset.coe_inj, Finset.coe_map, Finset.coe_univ, Set.image_univ]
[GOAL]
case h.e'_3.h.e'_9
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s : Simplex k P n
fs : Finset (Fin (n + 1))
m : ℕ
h : Finset.card fs = m + 1
⊢ ↑fs = Set.range ↑(Finset.orderEmbOfFin fs h).toEmbedding
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
⊢ Finset.centroid k fs₁ s.points = Finset.centroid k fs₂ s.points ↔ fs₁ = fs₂
[PROOFSTEP]
refine' ⟨fun h => _, @congrArg _ _ fs₁ fs₂ (fun z => Finset.centroid k z s.points)⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h : Finset.centroid k fs₁ s.points = Finset.centroid k fs₂ s.points
⊢ fs₁ = fs₂
[PROOFSTEP]
rw [Finset.centroid_eq_affineCombination_fintype, Finset.centroid_eq_affineCombination_fintype] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
⊢ fs₁ = fs₂
[PROOFSTEP]
have ha :=
(affineIndependent_iff_indicator_eq_of_affineCombination_eq k s.points).1 s.Independent _ _ _ _
(fs₁.sum_centroidWeightsIndicator_eq_one_of_card_eq_add_one k h₁)
(fs₂.sum_centroidWeightsIndicator_eq_one_of_card_eq_add_one k h₂) h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
ha :
(Set.indicator ↑Finset.univ fun i => Finset.centroidWeightsIndicator k fs₁ i) =
Set.indicator ↑Finset.univ fun i => Finset.centroidWeightsIndicator k fs₂ i
⊢ fs₁ = fs₂
[PROOFSTEP]
simp_rw [Finset.coe_univ, Set.indicator_univ, Function.funext_iff, Finset.centroidWeightsIndicator_def,
Finset.centroidWeights, h₁, h₂] at ha
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
ha :
∀ (a : Fin (n + 1)),
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) a =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) a
⊢ fs₁ = fs₂
[PROOFSTEP]
ext i
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
ha :
∀ (a : Fin (n + 1)),
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) a =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) a
i : Fin (n + 1)
⊢ i ∈ fs₁ ↔ i ∈ fs₂
[PROOFSTEP]
specialize ha i
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
⊢ i ∈ fs₁ ↔ i ∈ fs₂
[PROOFSTEP]
have key : ∀ n : ℕ, (n : k) + 1 ≠ 0 := fun n h => by norm_cast at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n✝ : ℕ
s : Simplex k P n✝
fs₁ fs₂ : Finset (Fin (n✝ + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h✝ :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n✝ + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n✝ + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n✝ + 1)) (↑(m₂ + 1))⁻¹) i
n : ℕ
h : ↑n + 1 = 0
⊢ False
[PROOFSTEP]
norm_cast at h
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
⊢ i ∈ fs₁ ↔ i ∈ fs₂
[PROOFSTEP]
constructor
[GOAL]
case a.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
⊢ i ∈ fs₁ → i ∈ fs₂
[PROOFSTEP]
intro hi
[GOAL]
case a.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
⊢ i ∈ fs₂ → i ∈ fs₁
[PROOFSTEP]
intro hi
[GOAL]
case a.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
hi : i ∈ fs₁
⊢ i ∈ fs₂
[PROOFSTEP]
by_contra hni
[GOAL]
case a.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
hi : i ∈ fs₂
⊢ i ∈ fs₁
[PROOFSTEP]
by_contra hni
[GOAL]
case a.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
hi : i ∈ fs₁
hni : ¬i ∈ fs₂
⊢ False
[PROOFSTEP]
simp [hni, hi, key] at ha
[GOAL]
case a.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
h :
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₁) =
↑(Finset.affineCombination k Finset.univ s.points) (Finset.centroidWeightsIndicator k fs₂)
i : Fin (n + 1)
ha :
Set.indicator (↑fs₁) (const (Fin (n + 1)) (↑(m₁ + 1))⁻¹) i =
Set.indicator (↑fs₂) (const (Fin (n + 1)) (↑(m₂ + 1))⁻¹) i
key : ∀ (n : ℕ), ↑n + 1 ≠ 0
hi : i ∈ fs₂
hni : ¬i ∈ fs₁
⊢ False
[PROOFSTEP]
simpa [hni, hi, key] using ha.symm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
⊢ Finset.centroid k Finset.univ (face s h₁).points = Finset.centroid k Finset.univ (face s h₂).points ↔ fs₁ = fs₂
[PROOFSTEP]
rw [face_centroid_eq_centroid, face_centroid_eq_centroid]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : CharZero k
n : ℕ
s : Simplex k P n
fs₁ fs₂ : Finset (Fin (n + 1))
m₁ m₂ : ℕ
h₁ : Finset.card fs₁ = m₁ + 1
h₂ : Finset.card fs₂ = m₂ + 1
⊢ Finset.centroid k fs₁ s.points = Finset.centroid k fs₂ s.points ↔ fs₁ = fs₂
[PROOFSTEP]
exact s.centroid_eq_iff h₁ h₂
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s₁ s₂ : Simplex k P n
h : Set.range s₁.points = Set.range s₂.points
⊢ Finset.centroid k Finset.univ s₁.points = Finset.centroid k Finset.univ s₂.points
[PROOFSTEP]
rw [← Set.image_univ, ← Set.image_univ, ← Finset.coe_univ] at h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
n : ℕ
s₁ s₂ : Simplex k P n
h✝ : s₁.points '' Set.univ = s₂.points '' Set.univ
h : s₁.points '' ↑Finset.univ = s₂.points '' ↑Finset.univ
⊢ Finset.centroid k Finset.univ s₁.points = Finset.centroid k Finset.univ s₂.points
[PROOFSTEP]
exact
Finset.univ.centroid_eq_of_inj_on_of_image_eq k _ (fun _ _ _ _ he => AffineIndependent.injective s₁.Independent he)
(fun _ _ _ _ he => AffineIndependent.injective s₂.Independent he) h
| {"mathlib_filename": "Mathlib.LinearAlgebra.AffineSpace.Independent", "llama_tokens": 115958} |
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
⊢ lowerInv hS = (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))ᵀ
[PROOFSTEP]
letI := NormedAddCommGroup.ofMatrix hS.transpose
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
this : NormedAddCommGroup (n → 𝕜) := NormedAddCommGroup.ofMatrix (_ : PosDef Sᵀ)
⊢ lowerInv hS = (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))ᵀ
[PROOFSTEP]
letI := InnerProductSpace.ofMatrix hS.transpose
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
this✝ : NormedAddCommGroup (n → 𝕜) := NormedAddCommGroup.ofMatrix (_ : PosDef Sᵀ)
this : InnerProductSpace 𝕜 (n → 𝕜) := InnerProductSpace.ofMatrix (_ : PosDef Sᵀ)
⊢ lowerInv hS = (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))ᵀ
[PROOFSTEP]
ext i j
[GOAL]
case a.h
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
this✝ : NormedAddCommGroup (n → 𝕜) := NormedAddCommGroup.ofMatrix (_ : PosDef Sᵀ)
this : InnerProductSpace 𝕜 (n → 𝕜) := InnerProductSpace.ofMatrix (_ : PosDef Sᵀ)
i j : n
⊢ lowerInv hS i j = (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))ᵀ i j
[PROOFSTEP]
rw [LDL.lowerInv, Basis.coePiBasisFun.toMatrix_eq_transpose, coe_gramSchmidtBasis]
[GOAL]
case a.h
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
this✝ : NormedAddCommGroup (n → 𝕜) := NormedAddCommGroup.ofMatrix (_ : PosDef Sᵀ)
this : InnerProductSpace 𝕜 (n → 𝕜) := InnerProductSpace.ofMatrix (_ : PosDef Sᵀ)
i j : n
⊢ gramSchmidt 𝕜 (↑(Pi.basisFun 𝕜 n)) i j = (gramSchmidt 𝕜 ↑(Pi.basisFun 𝕜 n))ᵀᵀ i j
[PROOFSTEP]
rfl
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
⊢ Invertible (lowerInv hS)
[PROOFSTEP]
rw [LDL.lowerInv_eq_gramSchmidtBasis]
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
⊢ Invertible (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))ᵀ
[PROOFSTEP]
haveI :=
Basis.invertibleToMatrix (Pi.basisFun 𝕜 n)
(@gramSchmidtBasis 𝕜 (n → 𝕜) _ (_ : _) (InnerProductSpace.ofMatrix hS.transpose) n _ _ _ (Pi.basisFun 𝕜 n))
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
this : Invertible (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))
⊢ Invertible (Basis.toMatrix (Pi.basisFun 𝕜 n) ↑(gramSchmidtBasis (Pi.basisFun 𝕜 n)))ᵀ
[PROOFSTEP]
infer_instance
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
hij : i < j
⊢ lowerInv hS i j = 0
[PROOFSTEP]
rw [←
@gramSchmidt_triangular 𝕜 (n → 𝕜) _ (_ : _) (InnerProductSpace.ofMatrix hS.transpose) n _ _ _ i j hij
(Pi.basisFun 𝕜 n),
Pi.basisFun_repr, LDL.lowerInv]
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
⊢ diag hS = lowerInv hS * S * (lowerInv hS)ᴴ
[PROOFSTEP]
ext i j
[GOAL]
case a.h
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
⊢ diag hS i j = (lowerInv hS * S * (lowerInv hS)ᴴ) i j
[PROOFSTEP]
by_cases hij : i = j
[GOAL]
case pos
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
hij : i = j
⊢ diag hS i j = (lowerInv hS * S * (lowerInv hS)ᴴ) i j
[PROOFSTEP]
simp only [diag, diagEntries, EuclideanSpace.inner_piLp_equiv_symm, star_star, hij, diagonal_apply_eq, Matrix.mul_assoc]
[GOAL]
case pos
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
hij : i = j
⊢ lowerInv hS j ⬝ᵥ mulVec S (star (lowerInv hS j)) = (lowerInv hS * (S * (lowerInv hS)ᴴ)) j j
[PROOFSTEP]
rfl
[GOAL]
case neg
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
hij : ¬i = j
⊢ diag hS i j = (lowerInv hS * S * (lowerInv hS)ᴴ) i j
[PROOFSTEP]
simp only [LDL.diag, hij, diagonal_apply_ne, Ne.def, not_false_iff, mul_mul_apply]
[GOAL]
case neg
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
hij : ¬i = j
⊢ 0 = lowerInv hS i ⬝ᵥ mulVec S ((lowerInv hS)ᴴᵀ j)
[PROOFSTEP]
rw [conjTranspose, transpose_map, transpose_transpose, dotProduct_mulVec,
(LDL.lowerInv_orthogonal hS fun h : j = i => hij h.symm).symm, ← inner_conj_symm, mulVec_transpose,
EuclideanSpace.inner_piLp_equiv_symm, ← IsROrC.star_def, ← star_dotProduct_star, dotProduct_comm, star_star]
[GOAL]
case neg
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
i j : n
hij : ¬i = j
⊢ vecMul (lowerInv hS i) S ⬝ᵥ star (lowerInv hS j) = vecMul (lowerInv hS i) S ⬝ᵥ map (lowerInv hS) star j
[PROOFSTEP]
rfl
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
⊢ lower hS * diag hS * (lower hS)ᴴ = S
[PROOFSTEP]
rw [LDL.lower, conjTranspose_nonsing_inv, Matrix.mul_assoc,
Matrix.inv_mul_eq_iff_eq_mul_of_invertible (LDL.lowerInv hS), Matrix.mul_inv_eq_iff_eq_mul_of_invertible]
[GOAL]
𝕜 : Type u_1
inst✝⁴ : IsROrC 𝕜
n : Type u_2
inst✝³ : LinearOrder n
inst✝² : IsWellOrder n fun x x_1 => x < x_1
inst✝¹ : LocallyFiniteOrderBot n
S : Matrix n n 𝕜
inst✝ : Fintype n
hS : PosDef S
⊢ diag hS = lowerInv hS * S * (lowerInv hS)ᴴ
[PROOFSTEP]
exact LDL.diag_eq_lowerInv_conj hS
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.LDL", "llama_tokens": 3555} |
[GOAL]
K : Type u_1
V₁ : Type u_2
V₂ : Type u_3
ι₁ : Type u_4
ι₂ : Type u_5
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V₁
inst✝⁶ : Module K V₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module K V₂
inst✝³ : Fintype ι₁
inst✝² : Fintype ι₂
inst✝¹ : DecidableEq ι₁
inst✝ : DecidableEq ι₂
B₁ : Basis ι₁ K V₁
B₂ : Basis ι₂ K V₂
u : V₁ →ₗ[K] V₂
⊢ ↑(toMatrix (Basis.dualBasis B₂) (Basis.dualBasis B₁)) (↑Module.Dual.transpose u) = (↑(toMatrix B₁ B₂) u)ᵀ
[PROOFSTEP]
ext i j
[GOAL]
case a.h
K : Type u_1
V₁ : Type u_2
V₂ : Type u_3
ι₁ : Type u_4
ι₂ : Type u_5
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V₁
inst✝⁶ : Module K V₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module K V₂
inst✝³ : Fintype ι₁
inst✝² : Fintype ι₂
inst✝¹ : DecidableEq ι₁
inst✝ : DecidableEq ι₂
B₁ : Basis ι₁ K V₁
B₂ : Basis ι₂ K V₂
u : V₁ →ₗ[K] V₂
i : ι₁
j : ι₂
⊢ ↑(toMatrix (Basis.dualBasis B₂) (Basis.dualBasis B₁)) (↑Module.Dual.transpose u) i j = (↑(toMatrix B₁ B₂) u)ᵀ i j
[PROOFSTEP]
simp only [LinearMap.toMatrix_apply, Module.Dual.transpose_apply, B₁.dualBasis_repr, B₂.dualBasis_apply,
Matrix.transpose_apply, LinearMap.comp_apply]
[GOAL]
K : Type u_1
V₁ : Type u_2
V₂ : Type u_3
ι₁ : Type u_4
ι₂ : Type u_5
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V₁
inst✝⁶ : Module K V₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module K V₂
inst✝³ : Fintype ι₁
inst✝² : Fintype ι₂
inst✝¹ : DecidableEq ι₁
inst✝ : DecidableEq ι₂
B₁ : Basis ι₁ K V₁
B₂ : Basis ι₂ K V₂
M : Matrix ι₁ ι₂ K
⊢ ↑(toLin (Basis.dualBasis B₁) (Basis.dualBasis B₂)) Mᵀ = ↑Module.Dual.transpose (↑(toLin B₂ B₁) M)
[PROOFSTEP]
apply (LinearMap.toMatrix B₁.dualBasis B₂.dualBasis).injective
[GOAL]
case a
K : Type u_1
V₁ : Type u_2
V₂ : Type u_3
ι₁ : Type u_4
ι₂ : Type u_5
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V₁
inst✝⁶ : Module K V₁
inst✝⁵ : AddCommGroup V₂
inst✝⁴ : Module K V₂
inst✝³ : Fintype ι₁
inst✝² : Fintype ι₂
inst✝¹ : DecidableEq ι₁
inst✝ : DecidableEq ι₂
B₁ : Basis ι₁ K V₁
B₂ : Basis ι₂ K V₂
M : Matrix ι₁ ι₂ K
⊢ ↑(LinearMap.toMatrix (Basis.dualBasis B₁) (Basis.dualBasis B₂))
(↑(toLin (Basis.dualBasis B₁) (Basis.dualBasis B₂)) Mᵀ) =
↑(LinearMap.toMatrix (Basis.dualBasis B₁) (Basis.dualBasis B₂)) (↑Module.Dual.transpose (↑(toLin B₂ B₁) M))
[PROOFSTEP]
rw [LinearMap.toMatrix_toLin, LinearMap.toMatrix_transpose, LinearMap.toMatrix_toLin]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Dual", "llama_tokens": 1206} |
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
⊢ IsSymm (Matrix.fromBlocks A B C D)
[PROOFSTEP]
have hCB : Cᵀ = B := by
rw [← hBC]
simp
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
⊢ Cᵀ = B
[PROOFSTEP]
rw [← hBC]
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
⊢ Bᵀᵀ = B
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
hCB : Cᵀ = B
⊢ IsSymm (Matrix.fromBlocks A B C D)
[PROOFSTEP]
unfold Matrix.IsSymm
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
hCB : Cᵀ = B
⊢ (Matrix.fromBlocks A B C D)ᵀ = Matrix.fromBlocks A B C D
[PROOFSTEP]
rw [fromBlocks_transpose]
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
hCB : Cᵀ = B
⊢ Matrix.fromBlocks Aᵀ Cᵀ Bᵀ Dᵀ = Matrix.fromBlocks A B C D
[PROOFSTEP]
congr
[GOAL]
α : Type u_1
β : Type u_2
n : Type u_3
m : Type u_4
R : Type u_5
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsSymm A
hBC : Bᵀ = C
hD : IsSymm D
hCB : Cᵀ = B
⊢ Matrix.fromBlocks Aᵀ Cᵀ Bᵀ Dᵀ = Matrix.fromBlocks A B C D
[PROOFSTEP]
rw [hA, hCB, hBC, hD]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Symmetric", "llama_tokens": 960} |
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² x✝¹ x✝ : M
⊢ (fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
(x✝² + x✝¹) x✝ =
(fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝² x✝ +
(fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝¹ x✝
[PROOFSTEP]
simp only [LinearMap.map_add, add_mul]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² x✝¹ x✝ : M
⊢ {
val :=
↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝ + ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝,
property :=
(_ :
(fun x => x ∈ even Q)
(↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝ +
↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝)) } =
{ val := ↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝,
property := (_ : ↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝ ∈ evenOdd Q 0) } +
{ val := ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝,
property := (_ : ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝ ∈ evenOdd Q 0) }
[PROOFSTEP]
rfl
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² : R
x✝¹ x✝ : M
⊢ (fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
(x✝² • x✝¹) x✝ =
x✝² •
(fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝¹ x✝
[PROOFSTEP]
simp only [LinearMap.map_smul, smul_mul_assoc]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² : R
x✝¹ x✝ : M
⊢ { val := x✝² • (↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝),
property := (_ : (fun x => x ∈ even Q) (x✝² • (↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝))) } =
x✝² •
{ val := ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝,
property := (_ : ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝ ∈ evenOdd Q 0) }
[PROOFSTEP]
rfl
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² x✝¹ x✝ : M
⊢ (fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝² (x✝¹ + x✝) =
(fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝² x✝¹ +
(fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝² x✝
[PROOFSTEP]
simp only [LinearMap.map_add, mul_add]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² x✝¹ x✝ : M
⊢ {
val :=
↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝¹ +
↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝,
property :=
(_ :
(fun x => x ∈ even Q)
(↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝¹ +
↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝)) } =
{ val := ↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝¹,
property := (_ : ↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝¹ ∈ evenOdd Q 0) } +
{ val := ↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝,
property := (_ : ↑(CliffordAlgebra.ι Q) x✝² * ↑(CliffordAlgebra.ι Q) x✝ ∈ evenOdd Q 0) }
[PROOFSTEP]
rfl
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² : R
x✝¹ x✝ : M
⊢ (fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝¹ (x✝² • x✝) =
x✝² •
(fun m₁ m₂ =>
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ ∈ evenOdd Q 0) })
x✝¹ x✝
[PROOFSTEP]
simp only [LinearMap.map_smul, mul_smul_comm]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
x✝² : R
x✝¹ x✝ : M
⊢ { val := x✝² • (↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝),
property := (_ : (fun x => x ∈ even Q) (x✝² • (↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝))) } =
x✝² •
{ val := ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝,
property := (_ : ↑(CliffordAlgebra.ι Q) x✝¹ * ↑(CliffordAlgebra.ι Q) x✝ ∈ evenOdd Q 0) }
[PROOFSTEP]
rfl
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
m₁ m₂ m₃ : M
⊢ ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * (↑(CliffordAlgebra.ι Q) m₂ * ↑(CliffordAlgebra.ι Q) m₃) =
↑(CliffordAlgebra.ι Q) m₁ * (↑(CliffordAlgebra.ι Q) m₂ * ↑(CliffordAlgebra.ι Q) m₂ * ↑(CliffordAlgebra.ι Q) m₃)
[PROOFSTEP]
simp only [mul_assoc]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
m₁ m₂ m₃ : M
⊢ ↑(CliffordAlgebra.ι Q) m₁ * (↑(CliffordAlgebra.ι Q) m₂ * ↑(CliffordAlgebra.ι Q) m₂ * ↑(CliffordAlgebra.ι Q) m₃) =
↑Q m₂ • (↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₃)
[PROOFSTEP]
rw [Algebra.smul_def, ι_sq_scalar, Algebra.left_comm]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : EvenHom.compr₂ (ι Q) f = EvenHom.compr₂ (ι Q) g
⊢ f = g
[PROOFSTEP]
rw [EvenHom.ext_iff] at h
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
⊢ f = g
[PROOFSTEP]
ext ⟨x, hx⟩
[GOAL]
case H.mk
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x : CliffordAlgebra Q
hx : x ∈ even Q
⊢ ↑f { val := x, property := hx } = ↑g { val := x, property := hx }
[PROOFSTEP]
refine' even_induction _ _ _ _ _ hx
[GOAL]
case H.mk.refine'_1
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x : CliffordAlgebra Q
hx : x ∈ even Q
⊢ ∀ (r : R),
↑f
{ val := ↑(algebraMap R (CliffordAlgebra ?m.107570)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra ?m.107570)) r ∈ evenOdd ?m.107570 0) } =
↑g
{ val := ↑(algebraMap R (CliffordAlgebra ?m.107570)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra ?m.107570)) r ∈ evenOdd ?m.107570 0) }
[PROOFSTEP]
intro r
[GOAL]
case H.mk.refine'_1
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x : CliffordAlgebra Q
hx : x ∈ even Q
r : R
⊢ ↑f
{ val := ↑(algebraMap R (CliffordAlgebra ?m.107570)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra ?m.107570)) r ∈ evenOdd ?m.107570 0) } =
↑g
{ val := ↑(algebraMap R (CliffordAlgebra ?m.107570)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra ?m.107570)) r ∈ evenOdd ?m.107570 0) }
[PROOFSTEP]
exact (f.commutes r).trans (g.commutes r).symm
[GOAL]
case H.mk.refine'_2
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x : CliffordAlgebra Q
hx : x ∈ even Q
⊢ ∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0} {hy : y ∈ evenOdd Q 0},
↑f { val := x, property := hx } = ↑g { val := x, property := hx } →
↑f { val := y, property := hy } = ↑g { val := y, property := hy } →
↑f { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) } =
↑g { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) }
[PROOFSTEP]
intro x y hx hy ihx ihy
[GOAL]
case H.mk.refine'_2
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ even Q
x y : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
hy : y ∈ evenOdd Q 0
ihx : ↑f { val := x, property := hx } = ↑g { val := x, property := hx }
ihy : ↑f { val := y, property := hy } = ↑g { val := y, property := hy }
⊢ ↑f { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) } =
↑g { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) }
[PROOFSTEP]
have := congr_arg₂ (· + ·) ihx ihy
[GOAL]
case H.mk.refine'_2
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ even Q
x y : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
hy : y ∈ evenOdd Q 0
ihx : ↑f { val := x, property := hx } = ↑g { val := x, property := hx }
ihy : ↑f { val := y, property := hy } = ↑g { val := y, property := hy }
this :
(fun x_1 x_2 => x_1 + x_2) (↑f { val := x, property := hx }) (↑f { val := y, property := hy }) =
(fun x_1 x_2 => x_1 + x_2) (↑g { val := x, property := hx }) (↑g { val := y, property := hy })
⊢ ↑f { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) } =
↑g { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) }
[PROOFSTEP]
exact (f.map_add _ _).trans (this.trans <| (g.map_add _ _).symm)
[GOAL]
case H.mk.refine'_3
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x : CliffordAlgebra Q
hx : x ∈ even Q
⊢ ∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0},
↑f { val := x, property := hx } = ↑g { val := x, property := hx } →
↑f
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) } =
↑g
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) }
[PROOFSTEP]
intro m₁ m₂ x hx ih
[GOAL]
case H.mk.refine'_3
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ even Q
m₁ m₂ : M
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
ih : ↑f { val := x, property := hx } = ↑g { val := x, property := hx }
⊢ ↑f
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) } =
↑g
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) }
[PROOFSTEP]
have := congr_arg₂ (· * ·) (LinearMap.congr_fun (LinearMap.congr_fun h m₁) m₂) ih
[GOAL]
case H.mk.refine'_3
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ : EvenHom Q A
f g : { x // x ∈ even Q } →ₐ[R] A
h : (EvenHom.compr₂ (ι Q) f).bilin = (EvenHom.compr₂ (ι Q) g).bilin
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ even Q
m₁ m₂ : M
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
ih : ↑f { val := x, property := hx } = ↑g { val := x, property := hx }
this :
(fun x_1 x_2 => x_1 * x_2) (↑(↑(EvenHom.compr₂ (ι Q) f).bilin m₁) m₂) (↑f { val := x, property := hx }) =
(fun x_1 x_2 => x_1 * x_2) (↑(↑(EvenHom.compr₂ (ι Q) g).bilin m₁) m₂) (↑g { val := x, property := hx })
⊢ ↑f
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) } =
↑g
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) }
[PROOFSTEP]
exact (f.map_mul _ _).trans (this.trans <| (g.map_mul _ _).symm)
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m₁ m₂ : M
a : A × { x // x ∈ CliffordAlgebra.even.lift.S f }
m₃ : M
⊢ ↑(↑f.bilin m₃) (m₁ + m₂) * a.fst = ↑(↑f.bilin m₃) m₁ * a.fst + ↑(↑f.bilin m₃) m₂ * a.fst
[PROOFSTEP]
rw [map_add, add_mul]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
c : R
m : M
a : A × { x // x ∈ CliffordAlgebra.even.lift.S f }
m₃ : M
⊢ ↑(↑f.bilin m₃) (c • m) * a.fst = c • (↑(↑f.bilin m₃) m * a.fst)
[PROOFSTEP]
rw [LinearMap.map_smul, smul_mul_assoc]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }
⊢ ↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x
[PROOFSTEP]
obtain ⟨a, ⟨g, hg⟩⟩ := x
[GOAL]
case mk.mk
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
⊢ ↑(↑(CliffordAlgebra.even.lift.fFold f) m)
(↑(↑(CliffordAlgebra.even.lift.fFold f) m) (a, { val := g, property := hg })) =
↑Q m • (a, { val := g, property := hg })
[PROOFSTEP]
ext : 2
[GOAL]
case mk.mk.h₁
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
⊢ (↑(↑(CliffordAlgebra.even.lift.fFold f) m)
(↑(↑(CliffordAlgebra.even.lift.fFold f) m) (a, { val := g, property := hg }))).fst =
(↑Q m • (a, { val := g, property := hg })).fst
[PROOFSTEP]
change f.bilin m m * a = Q m • a
[GOAL]
case mk.mk.h₁
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
⊢ ↑(↑f.bilin m) m * a = ↑Q m • a
[PROOFSTEP]
rw [Algebra.smul_def, f.contract]
[GOAL]
case mk.mk.h₂.a
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
⊢ ↑(↑(↑(CliffordAlgebra.even.lift.fFold f) m)
(↑(↑(CliffordAlgebra.even.lift.fFold f) m) (a, { val := g, property := hg }))).snd =
↑(↑Q m • (a, { val := g, property := hg })).snd
[PROOFSTEP]
ext m₁
[GOAL]
case mk.mk.h₂.a.h
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ↑↑(↑(↑(CliffordAlgebra.even.lift.fFold f) m)
(↑(↑(CliffordAlgebra.even.lift.fFold f) m) (a, { val := g, property := hg }))).snd
m₁ =
↑↑(↑Q m • (a, { val := g, property := hg })).snd m₁
[PROOFSTEP]
change f.bilin _ _ * g m = Q m • g m₁
[GOAL]
case mk.mk.h₂.a.h
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ↑(↑f.bilin m₁) m * ↑g m = ↑Q m • ↑g m₁
[PROOFSTEP]
apply Submodule.span_induction' _ _ _ _ hg
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ∀ (x : M →ₗ[R] A),
x ∈ {f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)} →
↑(↑f.bilin m₁) m * ↑x m = ↑Q m • ↑x m₁
[PROOFSTEP]
rintro _ ⟨b, m₃, rfl⟩
[GOAL]
case intro.intro
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
b : A
m₃ : M
⊢ ↑(↑f.bilin m₁) m * ↑(↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₃)) (LinearMap.mulRight R b)) m =
↑Q m • ↑(↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₃)) (LinearMap.mulRight R b)) m₁
[PROOFSTEP]
change f.bilin _ _ * (f.bilin _ _ * b) = Q m • (f.bilin _ _ * b)
[GOAL]
case intro.intro
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
b : A
m₃ : M
⊢ ↑(↑f.bilin m₁) m * (↑(↑f.bilin m) m₃ * b) = ↑Q m • (↑(↑f.bilin m₁) m₃ * b)
[PROOFSTEP]
rw [← smul_mul_assoc, ← mul_assoc, f.contract_mid]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ↑(↑f.bilin m₁) m * ↑0 m = ↑Q m • ↑0 m₁
[PROOFSTEP]
change
f.bilin m₁ m * 0 =
Q m •
(0 : A)
-- porting note: `•` now needs the type of `0`
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ↑(↑f.bilin m₁) m * 0 = ↑Q m • 0
[PROOFSTEP]
rw [mul_zero, smul_zero]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ∀ (x : M →ₗ[R] A),
x ∈
Submodule.span R
{f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)} →
∀ (y : M →ₗ[R] A),
y ∈
Submodule.span R
{f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)} →
↑(↑f.bilin m₁) m * ↑x m = ↑Q m • ↑x m₁ →
↑(↑f.bilin m₁) m * ↑y m = ↑Q m • ↑y m₁ → ↑(↑f.bilin m₁) m * ↑(x + y) m = ↑Q m • ↑(x + y) m₁
[PROOFSTEP]
rintro x hx y hy ihx ihy
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
x : M →ₗ[R] A
hx :
x ∈
Submodule.span R {f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)}
y : M →ₗ[R] A
hy :
y ∈
Submodule.span R {f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)}
ihx : ↑(↑f.bilin m₁) m * ↑x m = ↑Q m • ↑x m₁
ihy : ↑(↑f.bilin m₁) m * ↑y m = ↑Q m • ↑y m₁
⊢ ↑(↑f.bilin m₁) m * ↑(x + y) m = ↑Q m • ↑(x + y) m₁
[PROOFSTEP]
rw [LinearMap.add_apply, LinearMap.add_apply, mul_add, smul_add, ihx, ihy]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
⊢ ∀ (a : R) (x : M →ₗ[R] A),
x ∈
Submodule.span R
{f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)} →
↑(↑f.bilin m₁) m * ↑x m = ↑Q m • ↑x m₁ → ↑(↑f.bilin m₁) m * ↑(a • x) m = ↑Q m • ↑(a • x) m₁
[PROOFSTEP]
rintro x hx c ihx
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m : M
a : A
g : M →ₗ[R] A
hg : g ∈ CliffordAlgebra.even.lift.S f
m₁ : M
x : R
hx : M →ₗ[R] A
c :
hx ∈
Submodule.span R {f' | ∃ x m₂, f' = ↑(LinearMap.lcomp R A (↑(LinearMap.flip f.bilin) m₂)) (LinearMap.mulRight R x)}
ihx : ↑(↑f.bilin m₁) m * ↑hx m = ↑Q m • ↑hx m₁
⊢ ↑(↑f.bilin m₁) m * ↑(x • hx) m = ↑Q m • ↑(x • hx) m₁
[PROOFSTEP]
rw [LinearMap.smul_apply, LinearMap.smul_apply, mul_smul_comm, ihx, smul_comm]
-- Porting note: In Lean 3, `aux_apply` isn't a simp lemma. I changed `{ attrs := [] }` to
-- `{ isSimp := false }`, so that `aux_apply` isn't a simp lemma.
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ f : EvenHom Q A
⊢ { x // x ∈ even Q } →ₗ[R] A
[PROOFSTEP]
refine ?_ ∘ₗ (even Q).val.toLinearMap
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ f : EvenHom Q A
⊢ CliffordAlgebra Q →ₗ[R] A
[PROOFSTEP]
letI : AddCommGroup (S f) := AddSubgroupClass.toAddCommGroup _
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f✝ f : EvenHom Q A
this : AddCommGroup { x // x ∈ CliffordAlgebra.even.lift.S f } :=
AddSubgroupClass.toAddCommGroup (CliffordAlgebra.even.lift.S f)
⊢ CliffordAlgebra Q →ₗ[R] A
[PROOFSTEP]
exact LinearMap.fst R _ _ ∘ₗ foldr Q (fFold f) (fFold_fFold f) (1, 0)
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m₁ m₂ : M
⊢ (↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
(↑(CliffordAlgebra.ι Q) m₂)))
(↑(CliffordAlgebra.ι Q) m₁)).fst =
↑(↑f.bilin m₁) m₂
[PROOFSTEP]
rw [foldr_ι, foldr_ι]
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
m₁ m₂ : M
⊢ (↑(↑(CliffordAlgebra.even.lift.fFold f) m₁) (↑(↑(CliffordAlgebra.even.lift.fFold f) m₂) (1, 0))).fst =
↑(↑f.bilin m₁) m₂
[PROOFSTEP]
exact mul_one _
[GOAL]
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x y : { x // x ∈ even Q }
⊢ ↑(aux f) (x * y) = ↑(aux f) x * ↑(aux f) y
[PROOFSTEP]
cases' x with x x_property
[GOAL]
case mk
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
y : { x // x ∈ even Q }
x : CliffordAlgebra Q
x_property : x ∈ even Q
⊢ ↑(aux f) ({ val := x, property := x_property } * y) = ↑(aux f) { val := x, property := x_property } * ↑(aux f) y
[PROOFSTEP]
cases y
[GOAL]
case mk.mk
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
⊢ ↑(aux f) ({ val := x, property := x_property } * { val := val✝, property := property✝ }) =
↑(aux f) { val := x, property := x_property } * ↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
refine' (congr_arg Prod.fst (foldr_mul _ _ _ _ _ _)).trans _
[GOAL]
case mk.mk
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
⊢ (↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
↑{ val := val✝, property := property✝ }))
↑{ val := x, property := x_property }).fst =
↑(aux f) { val := x, property := x_property } * ↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
dsimp only
[GOAL]
case mk.mk
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
⊢ (↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := x_property } * ↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
refine' even_induction Q _ _ _ _ x_property
[GOAL]
case mk.mk.refine'_1
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
⊢ ∀ (r : R),
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
(↑(algebraMap R (CliffordAlgebra Q)) r)).fst =
↑(aux f)
{ val := ↑(algebraMap R (CliffordAlgebra Q)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ evenOdd Q 0) } *
↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
intro r
[GOAL]
case mk.mk.refine'_1
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
r : R
⊢ (↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
(↑(algebraMap R (CliffordAlgebra Q)) r)).fst =
↑(aux f)
{ val := ↑(algebraMap R (CliffordAlgebra Q)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ evenOdd Q 0) } *
↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
rw [foldr_algebraMap, aux_algebraMap]
[GOAL]
case mk.mk.refine'_1
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
r : R
⊢ (r •
↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝).fst =
↑(algebraMap R A) r * ↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
exact Algebra.smul_def r _
[GOAL]
case mk.mk.refine'_2
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
⊢ ∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0} {hy : y ∈ evenOdd Q 0},
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ } →
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m)
(↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
y).fst =
↑(aux f) { val := y, property := hy } * ↑(aux f) { val := val✝, property := property✝ } →
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m)
(↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
(x + y)).fst =
↑(aux f) { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) } *
↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
intro x y hx hy ihx ihy
[GOAL]
case mk.mk.refine'_2
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x✝ : CliffordAlgebra Q
x_property : x✝ ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
x y : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
hy : y ∈ evenOdd Q 0
ihx :
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ }
ihy :
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
y).fst =
↑(aux f) { val := y, property := hy } * ↑(aux f) { val := val✝, property := property✝ }
⊢ (↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
(x + y)).fst =
↑(aux f) { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) } * ↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
rw [LinearMap.map_add, Prod.fst_add, ihx, ihy, ← add_mul, ← LinearMap.map_add]
[GOAL]
case mk.mk.refine'_2
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x✝ : CliffordAlgebra Q
x_property : x✝ ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
x y : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
hy : y ∈ evenOdd Q 0
ihx :
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ }
ihy :
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
y).fst =
↑(aux f) { val := y, property := hy } * ↑(aux f) { val := val✝, property := property✝ }
⊢ ↑(aux f) ({ val := x, property := hx } + { val := y, property := hy }) *
↑(aux f) { val := val✝, property := property✝ } =
↑(aux f) { val := x + y, property := (_ : x + y ∈ evenOdd Q 0) } * ↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
rfl
[GOAL]
case mk.mk.refine'_3
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x : CliffordAlgebra Q
x_property : x ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
⊢ ∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0},
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ } →
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
(↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x)).fst =
↑(aux f)
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) } *
↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
rintro m₁ m₂ x (hx : x ∈ even Q) ih
[GOAL]
case mk.mk.refine'_3
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x✝ : CliffordAlgebra Q
x_property : x✝ ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
m₁ m₂ : M
x : CliffordAlgebra Q
hx : x ∈ even Q
ih :
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ }
⊢ (↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
(↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x)).fst =
↑(aux f)
{ val := ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x,
property := (_ : ↑(CliffordAlgebra.ι Q) m₁ * ↑(CliffordAlgebra.ι Q) m₂ * x ∈ evenOdd Q 0) } *
↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
rw [aux_apply, foldr_mul, foldr_mul, foldr_ι, foldr_ι, fst_fFold_fFold, ih, ← mul_assoc, Subtype.coe_mk, foldr_mul,
foldr_mul, foldr_ι, foldr_ι, fst_fFold_fFold]
[GOAL]
case mk.mk.refine'_3
R : Type uR
M : Type uM
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
A : Type uA
B : Type uB
inst✝³ : Ring A
inst✝² : Ring B
inst✝¹ : Algebra R A
inst✝ : Algebra R B
f : EvenHom Q A
x✝ : CliffordAlgebra Q
x_property : x✝ ∈ even Q
val✝ : CliffordAlgebra Q
property✝ : val✝ ∈ even Q
m₁ m₂ : M
x : CliffordAlgebra Q
hx : x ∈ even Q
ih :
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) = ↑Q m • x))
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
val✝))
x).fst =
↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ }
⊢ ↑(↑f.bilin m₁) m₂ * ↑(aux f) { val := x, property := hx } * ↑(aux f) { val := val✝, property := property✝ } =
↑(↑f.bilin m₁) m₂ *
(↑(↑(foldr Q (CliffordAlgebra.even.lift.fFold f)
(_ :
∀ (m : M) (x : A × { x // x ∈ CliffordAlgebra.even.lift.S f }),
↑(↑(CliffordAlgebra.even.lift.fFold f) m) (↑(↑(CliffordAlgebra.even.lift.fFold f) m) x) =
↑Q m • x))
(1, 0))
x).fst *
↑(aux f) { val := val✝, property := property✝ }
[PROOFSTEP]
rfl
| {"mathlib_filename": "Mathlib.LinearAlgebra.CliffordAlgebra.Even", "llama_tokens": 23761} |
{"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Orthogonal", "llama_tokens": 0} |
|
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
⊢ (∀ (i j : n), star (A j i) = A i j) → IsHermitian A
[PROOFSTEP]
intro h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
h : ∀ (i j : n), star (A j i) = A i j
⊢ IsHermitian A
[PROOFSTEP]
ext i j
[GOAL]
case a.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
h : ∀ (i j : n), star (A j i) = A i j
i j : n
⊢ Aᴴ i j = A i j
[PROOFSTEP]
exact h i j
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
h : IsHermitian A
⊢ IsHermitian Aᵀ
[PROOFSTEP]
rw [IsHermitian, conjTranspose, transpose_map]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
h : IsHermitian A
⊢ (Matrix.map Aᵀ star)ᵀ = Aᵀ
[PROOFSTEP]
exact congr_arg Matrix.transpose h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
⊢ IsHermitian Aᵀ → IsHermitian A
[PROOFSTEP]
intro h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
h : IsHermitian Aᵀ
⊢ IsHermitian A
[PROOFSTEP]
rw [← transpose_transpose A]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
h : IsHermitian Aᵀ
⊢ IsHermitian Aᵀᵀ
[PROOFSTEP]
exact IsHermitian.transpose h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : Star α
inst✝ : Star β
A : Matrix n n α
e : m ≃ n
h : IsHermitian (submatrix A ↑e ↑e)
⊢ IsHermitian A
[PROOFSTEP]
simpa using h.submatrix e.symm
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝ : InvolutiveStar α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsHermitian A
hBC : Bᴴ = C
hD : IsHermitian D
⊢ IsHermitian (Matrix.fromBlocks A B C D)
[PROOFSTEP]
have hCB : Cᴴ = B := by rw [← hBC, conjTranspose_conjTranspose]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝ : InvolutiveStar α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsHermitian A
hBC : Bᴴ = C
hD : IsHermitian D
⊢ Cᴴ = B
[PROOFSTEP]
rw [← hBC, conjTranspose_conjTranspose]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝ : InvolutiveStar α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsHermitian A
hBC : Bᴴ = C
hD : IsHermitian D
hCB : Cᴴ = B
⊢ IsHermitian (Matrix.fromBlocks A B C D)
[PROOFSTEP]
unfold Matrix.IsHermitian
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝ : InvolutiveStar α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
hA : IsHermitian A
hBC : Bᴴ = C
hD : IsHermitian D
hCB : Cᴴ = B
⊢ (Matrix.fromBlocks A B C D)ᴴ = Matrix.fromBlocks A B C D
[PROOFSTEP]
rw [fromBlocks_conjTranspose, hBC, hCB, hA, hD]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝⁴ : NonUnitalSemiring α
inst✝³ : StarRing α
inst✝² : NonUnitalSemiring β
inst✝¹ : StarRing β
inst✝ : Fintype n
A : Matrix m n α
⊢ IsHermitian (A * Aᴴ)
[PROOFSTEP]
rw [IsHermitian, conjTranspose_mul, conjTranspose_conjTranspose]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝⁴ : NonUnitalSemiring α
inst✝³ : StarRing α
inst✝² : NonUnitalSemiring β
inst✝¹ : StarRing β
inst✝ : Fintype m
A : Matrix m n α
⊢ IsHermitian (Aᴴ * A)
[PROOFSTEP]
rw [IsHermitian, conjTranspose_mul, conjTranspose_conjTranspose]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝⁴ : NonUnitalSemiring α
inst✝³ : StarRing α
inst✝² : NonUnitalSemiring β
inst✝¹ : StarRing β
inst✝ : Fintype m
A : Matrix m m α
B : Matrix m n α
hA : IsHermitian A
⊢ IsHermitian (Bᴴ * A * B)
[PROOFSTEP]
simp only [IsHermitian, conjTranspose_mul, conjTranspose_conjTranspose, hA.eq, Matrix.mul_assoc]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝⁴ : NonUnitalSemiring α
inst✝³ : StarRing α
inst✝² : NonUnitalSemiring β
inst✝¹ : StarRing β
inst✝ : Fintype m
A : Matrix m m α
B : Matrix n m α
hA : IsHermitian A
⊢ IsHermitian (B * A * Bᴴ)
[PROOFSTEP]
simp only [IsHermitian, conjTranspose_mul, conjTranspose_conjTranspose, hA.eq, Matrix.mul_assoc]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : CommRing α
inst✝² : StarRing α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
hA : IsHermitian A
⊢ IsHermitian A⁻¹
[PROOFSTEP]
simp [IsHermitian, conjTranspose_nonsing_inv, hA.eq]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝⁴ : CommRing α
inst✝³ : StarRing α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
inst✝ : Invertible A
h : IsHermitian A⁻¹
⊢ IsHermitian A
[PROOFSTEP]
rw [← inv_inv_of_invertible A]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝⁴ : CommRing α
inst✝³ : StarRing α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
inst✝ : Invertible A
h : IsHermitian A⁻¹
⊢ IsHermitian A⁻¹⁻¹
[PROOFSTEP]
exact IsHermitian.inv h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : CommRing α
inst✝² : StarRing α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
hA : IsHermitian A
⊢ IsHermitian (Matrix.adjugate A)
[PROOFSTEP]
simp [IsHermitian, adjugate_conjTranspose, hA.eq]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝¹ : IsROrC α
inst✝ : IsROrC β
A : Matrix n n α
h : IsHermitian A
i : n
⊢ ↑(↑re (A i i)) = A i i
[PROOFSTEP]
rw [← conj_eq_iff_re, ← star_def, ← conjTranspose_apply, h.eq]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
⊢ IsHermitian A ↔ LinearMap.IsSymmetric (↑toEuclideanLin A)
[PROOFSTEP]
rw [LinearMap.IsSymmetric, (PiLp.equiv 2 fun _ : n => α).symm.surjective.forall₂]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
⊢ IsHermitian A ↔
∀ (x₁ x₂ : n → α),
inner (↑(↑toEuclideanLin A) (↑(PiLp.equiv 2 fun x => α).symm x₁)) (↑(PiLp.equiv 2 fun x => α).symm x₂) =
inner (↑(PiLp.equiv 2 fun x => α).symm x₁) (↑(↑toEuclideanLin A) (↑(PiLp.equiv 2 fun x => α).symm x₂))
[PROOFSTEP]
simp only [toEuclideanLin_piLp_equiv_symm, EuclideanSpace.inner_piLp_equiv_symm, toLin'_apply, star_mulVec,
dotProduct_mulVec]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
⊢ IsHermitian A ↔ ∀ (x₁ x₂ : n → α), vecMul (star x₁) Aᴴ ⬝ᵥ x₂ = vecMul (star x₁) A ⬝ᵥ x₂
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
⊢ IsHermitian A → ∀ (x₁ x₂ : n → α), vecMul (star x₁) Aᴴ ⬝ᵥ x₂ = vecMul (star x₁) A ⬝ᵥ x₂
[PROOFSTEP]
rintro (h : Aᴴ = A) x y
[GOAL]
case mp
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
h : Aᴴ = A
x y : n → α
⊢ vecMul (star x) Aᴴ ⬝ᵥ y = vecMul (star x) A ⬝ᵥ y
[PROOFSTEP]
rw [h]
[GOAL]
case mpr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
⊢ (∀ (x₁ x₂ : n → α), vecMul (star x₁) Aᴴ ⬝ᵥ x₂ = vecMul (star x₁) A ⬝ᵥ x₂) → IsHermitian A
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
h : ∀ (x₁ x₂ : n → α), vecMul (star x₁) Aᴴ ⬝ᵥ x₂ = vecMul (star x₁) A ⬝ᵥ x₂
⊢ IsHermitian A
[PROOFSTEP]
ext i j
[GOAL]
case mpr.a.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
A✝ : Matrix n n α
inst✝³ : IsROrC α
inst✝² : IsROrC β
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n α
h : ∀ (x₁ x₂ : n → α), vecMul (star x₁) Aᴴ ⬝ᵥ x₂ = vecMul (star x₁) A ⬝ᵥ x₂
i j : n
⊢ Aᴴ i j = A i j
[PROOFSTEP]
simpa only [(Pi.single_star i 1).symm, ← star_mulVec, mul_one, dotProduct_single, single_vecMul, star_one,
one_mul] using h (Pi.single i 1) (Pi.single j 1)
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Hermitian", "llama_tokens": 4623} |
[GOAL]
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
⊢ Nondegenerate M
[PROOFSTEP]
intro v hv
[GOAL]
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
hv : ∀ (w : m → A), v ⬝ᵥ mulVec M w = 0
⊢ v = 0
[PROOFSTEP]
ext i
[GOAL]
case h
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
hv : ∀ (w : m → A), v ⬝ᵥ mulVec M w = 0
i : m
⊢ v i = OfNat.ofNat 0 i
[PROOFSTEP]
specialize hv (M.cramer (Pi.single i 1))
[GOAL]
case h
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
⊢ v i = OfNat.ofNat 0 i
[PROOFSTEP]
refine' (mul_eq_zero.mp _).resolve_right hM
[GOAL]
case h
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
⊢ v i * det M = 0
[PROOFSTEP]
convert hv
[GOAL]
case h.e'_2
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
⊢ v i * det M = v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1))
[PROOFSTEP]
simp only [mulVec_cramer M (Pi.single i 1), dotProduct, Pi.smul_apply, smul_eq_mul]
[GOAL]
case h.e'_2
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
⊢ v i * det M = Finset.sum Finset.univ fun x => v x * (det M * Pi.single i 1 x)
[PROOFSTEP]
rw [Finset.sum_eq_single i, Pi.single_eq_same, mul_one]
[GOAL]
case h.e'_2.h₀
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
⊢ ∀ (b : m), b ∈ Finset.univ → b ≠ i → v b * (det M * Pi.single i 1 b) = 0
[PROOFSTEP]
intro j _ hj
[GOAL]
case h.e'_2.h₀
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
j : m
a✝ : j ∈ Finset.univ
hj : j ≠ i
⊢ v j * (det M * Pi.single i 1 j) = 0
[PROOFSTEP]
simp [hj]
[GOAL]
case h.e'_2.h₁
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
⊢ ¬i ∈ Finset.univ → v i * (det M * Pi.single i 1 i) = 0
[PROOFSTEP]
intros
[GOAL]
case h.e'_2.h₁
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
a✝ : ¬i ∈ Finset.univ
⊢ v i * (det M * Pi.single i 1 i) = 0
[PROOFSTEP]
have := Finset.mem_univ i
[GOAL]
case h.e'_2.h₁
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
i : m
hv : v ⬝ᵥ mulVec M (↑(cramer M) (Pi.single i 1)) = 0
a✝ : ¬i ∈ Finset.univ
this : i ∈ Finset.univ
⊢ v i * (det M * Pi.single i 1 i) = 0
[PROOFSTEP]
contradiction
[GOAL]
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
hv : vecMul v M = 0
w : m → A
⊢ v ⬝ᵥ mulVec M w = 0
[PROOFSTEP]
rw [dotProduct_mulVec, hv, zero_dotProduct]
[GOAL]
m : Type u_1
R : Type u_2
A : Type u_3
inst✝⁴ : Fintype m
inst✝³ : CommRing R
inst✝² : CommRing A
inst✝¹ : IsDomain A
inst✝ : DecidableEq m
M : Matrix m m A
hM : det M ≠ 0
v : m → A
hv : mulVec M v = 0
⊢ det Mᵀ ≠ 0
[PROOFSTEP]
rwa [det_transpose]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Nondegenerate", "llama_tokens": 2556} |
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V1
inst✝⁴ : Module k V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V2
inst✝ : AffineSpace V2 P2
x✝¹ x✝ : P1 →ᵃ[k] P2
f : P1 → P2
f_linear : V1 →ₗ[k] V2
f_add : ∀ (p : P1) (v : V1), f (v +ᵥ p) = ↑f_linear v +ᵥ f p
g : P1 → P2
g_linear : V1 →ₗ[k] V2
g_add : ∀ (p : P1) (v : V1), g (v +ᵥ p) = ↑g_linear v +ᵥ g p
h : f = g
⊢ { toFun := f, linear := f_linear, map_vadd' := f_add } = { toFun := g, linear := g_linear, map_vadd' := g_add }
[PROOFSTEP]
cases' (AddTorsor.Nonempty : Nonempty P1) with p
[GOAL]
case intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V1
inst✝⁴ : Module k V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V2
inst✝ : AffineSpace V2 P2
x✝¹ x✝ : P1 →ᵃ[k] P2
f : P1 → P2
f_linear : V1 →ₗ[k] V2
f_add : ∀ (p : P1) (v : V1), f (v +ᵥ p) = ↑f_linear v +ᵥ f p
g : P1 → P2
g_linear : V1 →ₗ[k] V2
g_add : ∀ (p : P1) (v : V1), g (v +ᵥ p) = ↑g_linear v +ᵥ g p
h : f = g
p : P1
⊢ { toFun := f, linear := f_linear, map_vadd' := f_add } = { toFun := g, linear := g_linear, map_vadd' := g_add }
[PROOFSTEP]
congr with v
[GOAL]
case intro.e_linear.h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V1
inst✝⁴ : Module k V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V2
inst✝ : AffineSpace V2 P2
x✝¹ x✝ : P1 →ᵃ[k] P2
f : P1 → P2
f_linear : V1 →ₗ[k] V2
f_add : ∀ (p : P1) (v : V1), f (v +ᵥ p) = ↑f_linear v +ᵥ f p
g : P1 → P2
g_linear : V1 →ₗ[k] V2
g_add : ∀ (p : P1) (v : V1), g (v +ᵥ p) = ↑g_linear v +ᵥ g p
h : f = g
p : P1
v : V1
⊢ ↑f_linear v = ↑g_linear v
[PROOFSTEP]
apply vadd_right_cancel (f p)
[GOAL]
case intro.e_linear.h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
inst✝⁶ : Ring k
inst✝⁵ : AddCommGroup V1
inst✝⁴ : Module k V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V2
inst✝ : AffineSpace V2 P2
x✝¹ x✝ : P1 →ᵃ[k] P2
f : P1 → P2
f_linear : V1 →ₗ[k] V2
f_add : ∀ (p : P1) (v : V1), f (v +ᵥ p) = ↑f_linear v +ᵥ f p
g : P1 → P2
g_linear : V1 →ₗ[k] V2
g_add : ∀ (p : P1) (v : V1), g (v +ᵥ p) = ↑g_linear v +ᵥ g p
h : f = g
p : P1
v : V1
⊢ ↑f_linear v +ᵥ f p = ↑g_linear v +ᵥ f p
[PROOFSTEP]
erw [← f_add, h, ← g_add]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p1 p2 : P1
⊢ ↑f.linear (p1 -ᵥ p2) = ↑f p1 -ᵥ ↑f p2
[PROOFSTEP]
conv_rhs => rw [← vsub_vadd p1 p2, map_vadd, vadd_vsub]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p1 p2 : P1
| ↑f p1 -ᵥ ↑f p2
[PROOFSTEP]
rw [← vsub_vadd p1 p2, map_vadd, vadd_vsub]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p1 p2 : P1
| ↑f p1 -ᵥ ↑f p2
[PROOFSTEP]
rw [← vsub_vadd p1 p2, map_vadd, vadd_vsub]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p1 p2 : P1
| ↑f p1 -ᵥ ↑f p2
[PROOFSTEP]
rw [← vsub_vadd p1 p2, map_vadd, vadd_vsub]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p : P2
x✝¹ : P1
x✝ : V1
this : AddAction V2 P2 := inferInstance
⊢ Function.const P1 p (x✝ +ᵥ x✝¹) = ↑0 x✝ +ᵥ Function.const P1 p x✝¹
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
⊢ f.linear = 0 ↔ ∃ q, f = const k P1 q
[PROOFSTEP]
refine' ⟨fun h => _, fun h => _⟩
[GOAL]
case refine'_1
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
h : f.linear = 0
⊢ ∃ q, f = const k P1 q
[PROOFSTEP]
use f (Classical.arbitrary P1)
[GOAL]
case h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
h : f.linear = 0
⊢ f = const k P1 (↑f (Classical.arbitrary P1))
[PROOFSTEP]
ext
[GOAL]
case h.h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
h : f.linear = 0
p✝ : P1
⊢ ↑f p✝ = ↑(const k P1 (↑f (Classical.arbitrary P1))) p✝
[PROOFSTEP]
rw [coe_const, Function.const_apply, ← @vsub_eq_zero_iff_eq V2, ← f.linearMap_vsub, h, LinearMap.zero_apply]
[GOAL]
case refine'_2
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
h : ∃ q, f = const k P1 q
⊢ f.linear = 0
[PROOFSTEP]
rcases h with ⟨q, rfl⟩
[GOAL]
case refine'_2.intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
q : P2
⊢ (const k P1 q).linear = 0
[PROOFSTEP]
exact const_linear k P1 q
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 → P2
f' : V1 →ₗ[k] V2
p : P1
h : ∀ (p' : P1), f p' = ↑f' (p' -ᵥ p) +ᵥ f p
p' : P1
v : V1
⊢ f (v +ᵥ p') = ↑f' v +ᵥ f p'
[PROOFSTEP]
rw [h, h p', vadd_vsub_assoc, f'.map_add, vadd_vadd]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹⁵ : Ring k
inst✝¹⁴ : AddCommGroup V1
inst✝¹³ : Module k V1
inst✝¹² : AffineSpace V1 P1
inst✝¹¹ : AddCommGroup V2
inst✝¹⁰ : Module k V2
inst✝⁹ : AffineSpace V2 P2
inst✝⁸ : AddCommGroup V3
inst✝⁷ : Module k V3
inst✝⁶ : AffineSpace V3 P3
inst✝⁵ : AddCommGroup V4
inst✝⁴ : Module k V4
inst✝³ : AffineSpace V4 P4
R : Type u_10
inst✝² : Monoid R
inst✝¹ : DistribMulAction R V2
inst✝ : SMulCommClass k R V2
c : R
f : P1 →ᵃ[k] V2
p : P1
v : V1
⊢ (c • ↑f) (v +ᵥ p) = ↑(c • f.linear) v +ᵥ (c • ↑f) p
[PROOFSTEP]
simp [smul_add, map_vadd f]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f g : P1 →ᵃ[k] V2
p : P1
v : V1
⊢ (↑f + ↑g) (v +ᵥ p) = ↑(f.linear + g.linear) v +ᵥ (↑f + ↑g) p
[PROOFSTEP]
simp [add_add_add_comm, (map_vadd)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f g : P1 →ᵃ[k] V2
p : P1
v : V1
⊢ (↑f - ↑g) (v +ᵥ p) = ↑(f.linear - g.linear) v +ᵥ (↑f - ↑g) p
[PROOFSTEP]
simp [sub_add_sub_comm, (map_vadd)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] V2
p : P1
v : V1
⊢ (-↑f) (v +ᵥ p) = ↑(-f.linear) v +ᵥ (-↑f) p
[PROOFSTEP]
simp [add_comm, map_vadd f]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] V2
g : P1 →ᵃ[k] P2
this : AddAction V2 P2 := inferInstance
p : P1
v : V1
⊢ (fun p => ↑f p +ᵥ ↑g p) (v +ᵥ p) = ↑(f.linear + g.linear) v +ᵥ (fun p => ↑f p +ᵥ ↑g p) p
[PROOFSTEP]
simp [vadd_vadd, add_right_comm, (map_vadd)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f g : P1 →ᵃ[k] P2
p : P1
v : V1
⊢ (fun p => ↑f p -ᵥ ↑g p) (v +ᵥ p) = ↑(f.linear - g.linear) v +ᵥ (fun p => ↑f p -ᵥ ↑g p) p
[PROOFSTEP]
simp [(map_vadd), (vsub_vadd_eq_vsub_sub), (vadd_vsub_assoc), add_sub, sub_add_eq_add_sub]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P2 →ᵃ[k] P3
g : P1 →ᵃ[k] P2
⊢ ∀ (p : P1) (v : V1), (↑f ∘ ↑g) (v +ᵥ p) = ↑(LinearMap.comp f.linear g.linear) v +ᵥ (↑f ∘ ↑g) p
[PROOFSTEP]
intro p v
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P2 →ᵃ[k] P3
g : P1 →ᵃ[k] P2
p : P1
v : V1
⊢ (↑f ∘ ↑g) (v +ᵥ p) = ↑(LinearMap.comp f.linear g.linear) v +ᵥ (↑f ∘ ↑g) p
[PROOFSTEP]
rw [Function.comp_apply, g.map_vadd, f.map_vadd]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P2 →ᵃ[k] P3
g : P1 →ᵃ[k] P2
p : P1
v : V1
⊢ ↑f.linear (↑g.linear v) +ᵥ ↑f (↑g p) = ↑(LinearMap.comp f.linear g.linear) v +ᵥ (↑f ∘ ↑g) p
[PROOFSTEP]
rfl
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
⊢ Function.Injective ↑f.linear ↔ Function.Injective ↑f
[PROOFSTEP]
obtain ⟨p⟩ := (inferInstance : Nonempty P1)
[GOAL]
case intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
⊢ Function.Injective ↑f.linear ↔ Function.Injective ↑f
[PROOFSTEP]
have h : ⇑f.linear = (Equiv.vaddConst (f p)).symm ∘ f ∘ Equiv.vaddConst p :=
by
ext v
simp [f.map_vadd, vadd_vsub_assoc]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
⊢ ↑f.linear = ↑(Equiv.vaddConst (↑f p)).symm ∘ ↑f ∘ ↑(Equiv.vaddConst p)
[PROOFSTEP]
ext v
[GOAL]
case h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
v : V1
⊢ ↑f.linear v = (↑(Equiv.vaddConst (↑f p)).symm ∘ ↑f ∘ ↑(Equiv.vaddConst p)) v
[PROOFSTEP]
simp [f.map_vadd, vadd_vsub_assoc]
[GOAL]
case intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
h : ↑f.linear = ↑(Equiv.vaddConst (↑f p)).symm ∘ ↑f ∘ ↑(Equiv.vaddConst p)
⊢ Function.Injective ↑f.linear ↔ Function.Injective ↑f
[PROOFSTEP]
rw [h, Equiv.comp_injective, Equiv.injective_comp]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
⊢ Function.Surjective ↑f.linear ↔ Function.Surjective ↑f
[PROOFSTEP]
obtain ⟨p⟩ := (inferInstance : Nonempty P1)
[GOAL]
case intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
⊢ Function.Surjective ↑f.linear ↔ Function.Surjective ↑f
[PROOFSTEP]
have h : ⇑f.linear = (Equiv.vaddConst (f p)).symm ∘ f ∘ Equiv.vaddConst p :=
by
ext v
simp [f.map_vadd, vadd_vsub_assoc]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
⊢ ↑f.linear = ↑(Equiv.vaddConst (↑f p)).symm ∘ ↑f ∘ ↑(Equiv.vaddConst p)
[PROOFSTEP]
ext v
[GOAL]
case h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
v : V1
⊢ ↑f.linear v = (↑(Equiv.vaddConst (↑f p)).symm ∘ ↑f ∘ ↑(Equiv.vaddConst p)) v
[PROOFSTEP]
simp [f.map_vadd, vadd_vsub_assoc]
[GOAL]
case intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p : P1
h : ↑f.linear = ↑(Equiv.vaddConst (↑f p)).symm ∘ ↑f ∘ ↑(Equiv.vaddConst p)
⊢ Function.Surjective ↑f.linear ↔ Function.Surjective ↑f
[PROOFSTEP]
rw [h, Equiv.comp_surjective, Equiv.surjective_comp]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
⊢ ↑f '' s -ᵥ ↑f '' t = ↑f.linear '' (s -ᵥ t)
[PROOFSTEP]
ext v
[GOAL]
case h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
v : V2
⊢ v ∈ ↑f '' s -ᵥ ↑f '' t ↔ v ∈ ↑f.linear '' (s -ᵥ t)
[PROOFSTEP]
simp only [(Set.mem_vsub), Set.mem_image, exists_exists_and_eq_and, exists_and_left, ← f.linearMap_vsub]
[GOAL]
case h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
v : V2
⊢ (∃ a, a ∈ s ∧ ∃ a_1, a_1 ∈ t ∧ ↑f.linear (a -ᵥ a_1) = v) ↔
∃ x, (∃ x_1, x_1 ∈ s ∧ ∃ x_2, x_2 ∈ t ∧ x_1 -ᵥ x_2 = x) ∧ ↑f.linear x = v
[PROOFSTEP]
constructor
[GOAL]
case h.mp
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
v : V2
⊢ (∃ a, a ∈ s ∧ ∃ a_1, a_1 ∈ t ∧ ↑f.linear (a -ᵥ a_1) = v) →
∃ x, (∃ x_1, x_1 ∈ s ∧ ∃ x_2, x_2 ∈ t ∧ x_1 -ᵥ x_2 = x) ∧ ↑f.linear x = v
[PROOFSTEP]
rintro ⟨x, hx, y, hy, hv⟩
[GOAL]
case h.mp.intro.intro.intro.intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
v : V2
x : P1
hx : x ∈ s
y : P1
hy : y ∈ t
hv : ↑f.linear (x -ᵥ y) = v
⊢ ∃ x, (∃ x_1, x_1 ∈ s ∧ ∃ x_2, x_2 ∈ t ∧ x_1 -ᵥ x_2 = x) ∧ ↑f.linear x = v
[PROOFSTEP]
exact ⟨x -ᵥ y, ⟨x, hx, y, hy, rfl⟩, hv⟩
[GOAL]
case h.mpr
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
v : V2
⊢ (∃ x, (∃ x_1, x_1 ∈ s ∧ ∃ x_2, x_2 ∈ t ∧ x_1 -ᵥ x_2 = x) ∧ ↑f.linear x = v) →
∃ a, a ∈ s ∧ ∃ a_1, a_1 ∈ t ∧ ↑f.linear (a -ᵥ a_1) = v
[PROOFSTEP]
rintro ⟨-, ⟨x, hx, y, hy, rfl⟩, rfl⟩
[GOAL]
case h.mpr.intro.intro.intro.intro.intro.intro
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
s t : Set P1
f : P1 →ᵃ[k] P2
x : P1
hx : x ∈ s
y : P1
hy : y ∈ t
⊢ ∃ a, a ∈ s ∧ ∃ a_1, a_1 ∈ t ∧ ↑f.linear (a -ᵥ a_1) = ↑f.linear (x -ᵥ y)
[PROOFSTEP]
exact ⟨x, hx, y, hy, rfl⟩
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : V1
c : k
⊢ ↑(lineMap p₀ p₁) c = (1 - c) • p₀ + c • p₁
[PROOFSTEP]
simp [lineMap_apply_module', smul_sub, sub_smul]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : V1
c : k
⊢ c • p₁ - c • p₀ + p₀ = p₀ - c • p₀ + c • p₁
[PROOFSTEP]
abel
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : V1
c : k
⊢ c • p₁ - c • p₀ + p₀ = p₀ - c • p₀ + c • p₁
[PROOFSTEP]
abel
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p : P1
v : V1
c : k
⊢ ↑(lineMap p (v +ᵥ p)) c = c • v +ᵥ p
[PROOFSTEP]
rw [lineMap_apply, vadd_vsub]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p : P1
c : k
⊢ ↑(lineMap p p) c = p
[PROOFSTEP]
letI : AddAction V1 P1 := inferInstance
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p : P1
c : k
this : AddAction V1 P1 := inferInstance
⊢ ↑(lineMap p p) c = p
[PROOFSTEP]
simp [(lineMap_apply), (vsub_self)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
⊢ ↑(lineMap p₀ p₁) 0 = p₀
[PROOFSTEP]
letI : AddAction V1 P1 := inferInstance
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
this : AddAction V1 P1 := inferInstance
⊢ ↑(lineMap p₀ p₁) 0 = p₀
[PROOFSTEP]
simp [(lineMap_apply)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
⊢ ↑(lineMap p₀ p₁) 1 = p₁
[PROOFSTEP]
simp [(lineMap_apply), (vsub_vadd)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k V4
inst✝¹ : AffineSpace V4 P4
inst✝ : NoZeroSMulDivisors k V1
p₀ p₁ : P1
c₁ c₂ : k
⊢ ↑(lineMap p₀ p₁) c₁ = ↑(lineMap p₀ p₁) c₂ ↔ p₀ = p₁ ∨ c₁ = c₂
[PROOFSTEP]
rw [lineMap_apply, lineMap_apply, ← @vsub_eq_zero_iff_eq V1, vadd_vsub_vadd_cancel_right, ← sub_smul, smul_eq_zero,
sub_eq_zero, vsub_eq_zero_iff_eq, or_comm, eq_comm]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k V4
inst✝¹ : AffineSpace V4 P4
inst✝ : NoZeroSMulDivisors k V1
p₀ p₁ : P1
c : k
⊢ ↑(lineMap p₀ p₁) c = p₀ ↔ p₀ = p₁ ∨ c = 0
[PROOFSTEP]
rw [← @lineMap_eq_lineMap_iff k V1, lineMap_apply_zero]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k V4
inst✝¹ : AffineSpace V4 P4
inst✝ : NoZeroSMulDivisors k V1
p₀ p₁ : P1
c : k
⊢ ↑(lineMap p₀ p₁) c = p₁ ↔ p₀ = p₁ ∨ c = 1
[PROOFSTEP]
rw [← @lineMap_eq_lineMap_iff k V1, lineMap_apply_one]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : P1 →ᵃ[k] P2
p₀ p₁ : P1
c : k
⊢ ↑f (↑(lineMap p₀ p₁) c) = ↑(lineMap (↑f p₀) (↑f p₁)) c
[PROOFSTEP]
simp [(lineMap_apply), (map_vadd), (linearMap_vsub)]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
⊢ lineMap p₀ p₁ = comp (lineMap p₁ p₀) (lineMap 1 0)
[PROOFSTEP]
rw [comp_lineMap]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
⊢ lineMap p₀ p₁ = lineMap (↑(lineMap p₁ p₀) 1) (↑(lineMap p₁ p₀) 0)
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
c : k
⊢ ↑(lineMap p₀ p₁) (1 - c) = ↑(lineMap p₁ p₀) c
[PROOFSTEP]
rw [lineMap_symm p₀, comp_apply]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
c : k
⊢ ↑(lineMap p₁ p₀) (↑(lineMap 1 0) (1 - c)) = ↑(lineMap p₁ p₀) c
[PROOFSTEP]
congr
[GOAL]
case h.e_6.h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
c : k
⊢ ↑(lineMap 1 0) (1 - c) = c
[PROOFSTEP]
simp [lineMap_apply]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
c : k
⊢ p₀ -ᵥ ↑(lineMap p₀ p₁) c = c • (p₀ -ᵥ p₁)
[PROOFSTEP]
rw [← neg_vsub_eq_vsub_rev, lineMap_vsub_left, ← smul_neg, neg_vsub_eq_vsub_rev]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
c : k
⊢ ↑(lineMap p₀ p₁) c -ᵥ p₁ = (1 - c) • (p₀ -ᵥ p₁)
[PROOFSTEP]
rw [← lineMap_apply_one_sub, lineMap_vsub_left]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
p₀ p₁ : P1
c : k
⊢ p₁ -ᵥ ↑(lineMap p₀ p₁) c = (1 - c) • (p₁ -ᵥ p₀)
[PROOFSTEP]
rw [← lineMap_apply_one_sub, left_vsub_lineMap]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : V1 →ᵃ[k] V2
⊢ ↑f = ↑f.linear + fun x => ↑f 0
[PROOFSTEP]
ext x
[GOAL]
case h
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : V1 →ᵃ[k] V2
x : V1
⊢ ↑f x = (↑f.linear + fun x => ↑f 0) x
[PROOFSTEP]
calc
f x = f.linear x +ᵥ f 0 := by rw [← f.map_vadd, vadd_eq_add, add_zero]
_ = (f.linear + fun _ : V1 => f 0) x := rfl
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : V1 →ᵃ[k] V2
x : V1
⊢ ↑f x = ↑f.linear x +ᵥ ↑f 0
[PROOFSTEP]
rw [← f.map_vadd, vadd_eq_add, add_zero]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : V1 →ᵃ[k] V2
⊢ ↑f.linear = ↑f - fun x => ↑f 0
[PROOFSTEP]
rw [decomp]
[GOAL]
k : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹² : Ring k
inst✝¹¹ : AddCommGroup V1
inst✝¹⁰ : Module k V1
inst✝⁹ : AffineSpace V1 P1
inst✝⁸ : AddCommGroup V2
inst✝⁷ : Module k V2
inst✝⁶ : AffineSpace V2 P2
inst✝⁵ : AddCommGroup V3
inst✝⁴ : Module k V3
inst✝³ : AffineSpace V3 P3
inst✝² : AddCommGroup V4
inst✝¹ : Module k V4
inst✝ : AffineSpace V4 P4
f : V1 →ᵃ[k] V2
⊢ ↑f.linear = (↑f.linear + fun x => ↑f 0) - fun x => (↑f.linear + fun x => ↑f 0) 0
[PROOFSTEP]
simp only [LinearMap.map_zero, Pi.add_apply, add_sub_cancel, zero_add]
[GOAL]
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b : k
⊢ ↑f '' Set.uIcc a b = Set.uIcc (↑f a) (↑f b)
[PROOFSTEP]
have : ⇑f = (fun x => x + f 0) ∘ fun x => x * (f 1 - f 0) :=
by
ext x
change f x = x • (f 1 -ᵥ f 0) +ᵥ f 0
rw [← f.linearMap_vsub, ← f.linear.map_smul, ← f.map_vadd]
simp only [vsub_eq_sub, add_zero, mul_one, vadd_eq_add, sub_zero, smul_eq_mul]
[GOAL]
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b : k
⊢ ↑f = (fun x => x + ↑f 0) ∘ fun x => x * (↑f 1 - ↑f 0)
[PROOFSTEP]
ext x
[GOAL]
case h
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b x : k
⊢ ↑f x = ((fun x => x + ↑f 0) ∘ fun x => x * (↑f 1 - ↑f 0)) x
[PROOFSTEP]
change f x = x • (f 1 -ᵥ f 0) +ᵥ f 0
[GOAL]
case h
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b x : k
⊢ ↑f x = x • (↑f 1 -ᵥ ↑f 0) +ᵥ ↑f 0
[PROOFSTEP]
rw [← f.linearMap_vsub, ← f.linear.map_smul, ← f.map_vadd]
[GOAL]
case h
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b x : k
⊢ ↑f x = ↑f (x • (1 -ᵥ 0) +ᵥ 0)
[PROOFSTEP]
simp only [vsub_eq_sub, add_zero, mul_one, vadd_eq_add, sub_zero, smul_eq_mul]
[GOAL]
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b : k
this : ↑f = (fun x => x + ↑f 0) ∘ fun x => x * (↑f 1 - ↑f 0)
⊢ ↑f '' Set.uIcc a b = Set.uIcc (↑f a) (↑f b)
[PROOFSTEP]
rw [this, Set.image_comp]
[GOAL]
k✝ : Type u_1
V1 : Type u_2
P1 : Type u_3
V2 : Type u_4
P2 : Type u_5
V3 : Type u_6
P3 : Type u_7
V4 : Type u_8
P4 : Type u_9
inst✝¹³ : Ring k✝
inst✝¹² : AddCommGroup V1
inst✝¹¹ : Module k✝ V1
inst✝¹⁰ : AffineSpace V1 P1
inst✝⁹ : AddCommGroup V2
inst✝⁸ : Module k✝ V2
inst✝⁷ : AffineSpace V2 P2
inst✝⁶ : AddCommGroup V3
inst✝⁵ : Module k✝ V3
inst✝⁴ : AffineSpace V3 P3
inst✝³ : AddCommGroup V4
inst✝² : Module k✝ V4
inst✝¹ : AffineSpace V4 P4
k : Type u_10
inst✝ : LinearOrderedField k
f : k →ᵃ[k] k
a b : k
this : ↑f = (fun x => x + ↑f 0) ∘ fun x => x * (↑f 1 - ↑f 0)
⊢ (fun x => x + ↑f 0) '' ((fun x => x * (↑f 1 - ↑f 0)) '' Set.uIcc a b) =
Set.uIcc (((fun x => x + ↑f 0) ∘ fun x => x * (↑f 1 - ↑f 0)) a)
(((fun x => x + ↑f 0) ∘ fun x => x * (↑f 1 - ↑f 0)) b)
[PROOFSTEP]
simp only [Set.image_add_const_uIcc, Set.image_mul_const_uIcc, Function.comp_apply]
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
⊢ ∀ (x y : V1 →ᵃ[k] V2),
(fun f => (↑f 0, f.linear)) (x + y) = (fun f => (↑f 0, f.linear)) x + (fun f => (↑f 0, f.linear)) y
[PROOFSTEP]
simp
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
⊢ ∀ (r : R) (x : V1 →ᵃ[k] V2),
AddHom.toFun
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) }
x
[PROOFSTEP]
simp
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
f : V1 →ᵃ[k] V2
⊢ (fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst)
(AddHom.toFun
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ :
∀ (a : R) (a_1 : V1 →ᵃ[k] V2), (a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom
f) =
f
[PROOFSTEP]
ext
[GOAL]
case h
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
f : V1 →ᵃ[k] V2
p✝ : V1
⊢ ↑((fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst)
(AddHom.toFun
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ :
∀ (a : R) (a_1 : V1 →ᵃ[k] V2),
(a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom
f))
p✝ =
↑f p✝
[PROOFSTEP]
rw [f.decomp]
[GOAL]
case h
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
f : V1 →ᵃ[k] V2
p✝ : V1
⊢ ↑((fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst)
(AddHom.toFun
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ :
∀ (a : R) (a_1 : V1 →ᵃ[k] V2),
(a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom
f))
p✝ =
(↑f.linear + fun x => ↑f 0) p✝
[PROOFSTEP]
simp [const_apply _ _]
-- porting note: `simp` needs `_`s to use this lemma
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
⊢ Function.RightInverse (fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst)
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ :
∀ (a : R) (a_1 : V1 →ᵃ[k] V2),
(a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom.toFun
[PROOFSTEP]
rintro ⟨v, f⟩
[GOAL]
case mk
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
v : V2
f : V1 →ₗ[k] V2
⊢ AddHom.toFun
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ : ∀ (a : R) (a_1 : V1 →ᵃ[k] V2), (a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom
((fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst) (v, f)) =
(v, f)
[PROOFSTEP]
ext
[GOAL]
case mk.h₁
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
v : V2
f : V1 →ₗ[k] V2
⊢ (AddHom.toFun
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ :
∀ (a : R) (a_1 : V1 →ᵃ[k] V2), (a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom
((fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst) (v, f))).fst =
(v, f).fst
[PROOFSTEP]
simp [const_apply _ _, const_linear _ _]
-- porting note: `simp` needs `_`s
[GOAL]
case mk.h₂.h
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁸ : Ring k
inst✝⁷ : AddCommGroup V1
inst✝⁶ : AffineSpace V1 P1
inst✝⁵ : AddCommGroup V2
inst✝⁴ : Module k V1
inst✝³ : Module k V2
inst✝² : Semiring R
inst✝¹ : Module R V2
inst✝ : SMulCommClass k R V2
v : V2
f : V1 →ₗ[k] V2
x✝ : V1
⊢ ↑(AddHom.toFun
{
toAddHom :=
{ toFun := fun f => (↑f 0, f.linear),
map_add' :=
(_ :
∀ (a a_1 : V1 →ᵃ[k] V2),
(↑a 0 + ↑a_1 0, a.linear + a_1.linear) = (↑a 0 + ↑a_1 0, a.linear + a_1.linear)) },
map_smul' :=
(_ :
∀ (a : R) (a_1 : V1 →ᵃ[k] V2),
(a • ↑a_1 0, a • a_1.linear) = (a • ↑a_1 0, a • a_1.linear)) }.toAddHom
((fun p => LinearMap.toAffineMap p.snd + const k V1 p.fst) (v, f))).snd
x✝ =
↑(v, f).snd x✝
[PROOFSTEP]
simp [const_apply _ _, const_linear _ _]
-- porting note: `simp` needs `_`s
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁵ : CommRing k
inst✝⁴ : AddCommGroup V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V1
inst✝ : Module k V2
c : P1
⊢ homothety c 1 = id k P1
[PROOFSTEP]
ext p
[GOAL]
case h
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁵ : CommRing k
inst✝⁴ : AddCommGroup V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V1
inst✝ : Module k V2
c p : P1
⊢ ↑(homothety c 1) p = ↑(id k P1) p
[PROOFSTEP]
simp [homothety_apply]
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁵ : CommRing k
inst✝⁴ : AddCommGroup V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V1
inst✝ : Module k V2
c : P1
r₁ r₂ : k
p : P1
⊢ ↑(homothety c (r₁ * r₂)) p = ↑(homothety c r₁) (↑(homothety c r₂) p)
[PROOFSTEP]
simp only [homothety_apply, mul_smul, vadd_vsub]
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁵ : CommRing k
inst✝⁴ : AddCommGroup V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V1
inst✝ : Module k V2
c : P1
⊢ homothety c 0 = const k P1 c
[PROOFSTEP]
ext p
[GOAL]
case h
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁵ : CommRing k
inst✝⁴ : AddCommGroup V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V1
inst✝ : Module k V2
c p : P1
⊢ ↑(homothety c 0) p = ↑(const k P1 c) p
[PROOFSTEP]
simp [homothety_apply]
[GOAL]
R : Type u_1
k : Type u_2
V1 : Type u_3
P1 : Type u_4
V2 : Type u_5
inst✝⁵ : CommRing k
inst✝⁴ : AddCommGroup V1
inst✝³ : AffineSpace V1 P1
inst✝² : AddCommGroup V2
inst✝¹ : Module k V1
inst✝ : Module k V2
c : P1
r₁ r₂ : k
⊢ homothety c (r₁ + r₂) = r₁ • (id k P1 -ᵥ const k P1 c) +ᵥ homothety c r₂
[PROOFSTEP]
simp only [homothety_def, add_smul, vadd_vadd]
[GOAL]
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝⁴ : Ring 𝕜
inst✝³ : AddCommGroup E
inst✝² : AddCommGroup F
inst✝¹ : Module 𝕜 E
inst✝ : Module 𝕜 F
x y : E
a b : 𝕜
f : E →ᵃ[𝕜] F
h : a + b = 1
⊢ ↑f (a • x + b • y) = a • ↑f x + b • ↑f y
[PROOFSTEP]
simp only [Convex.combo_eq_smul_sub_add h, ← vsub_eq_sub]
[GOAL]
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝⁴ : Ring 𝕜
inst✝³ : AddCommGroup E
inst✝² : AddCommGroup F
inst✝¹ : Module 𝕜 E
inst✝ : Module 𝕜 F
x y : E
a b : 𝕜
f : E →ᵃ[𝕜] F
h : a + b = 1
⊢ ↑f (b • (y -ᵥ x) + x) = b • (↑f y -ᵥ ↑f x) + ↑f x
[PROOFSTEP]
exact f.apply_lineMap _ _ _
| {"mathlib_filename": "Mathlib.LinearAlgebra.AffineSpace.AffineMap", "llama_tokens": 29871} |
[GOAL]
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
⊢ M ≃ₗ[R] M
[PROOFSTEP]
refine'
{ toLin b b A with
toFun := toLin b b A
invFun := toLin b b A⁻¹
left_inv := fun x => _
right_inv := fun x => _ }
[GOAL]
case refine'_1
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
src✝ : (fun x => M →ₗ[R] M) A := ↑(toLin b b) A
x : M
⊢ ↑(↑(toLin b b) A⁻¹)
(AddHom.toFun
{
toAddHom :=
{ toFun := ↑(↑(toLin b b) A),
map_add' :=
(_ :
∀ (x y : M),
AddHom.toFun src✝.toAddHom (x + y) =
AddHom.toFun src✝.toAddHom x + AddHom.toFun src✝.toAddHom y) },
map_smul' :=
(_ :
∀ (r : R) (x : M),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
x) =
x
[PROOFSTEP]
simp only
[GOAL]
case refine'_2
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
src✝ : (fun x => M →ₗ[R] M) A := ↑(toLin b b) A
x : M
⊢ AddHom.toFun
{
toAddHom :=
{ toFun := ↑(↑(toLin b b) A),
map_add' :=
(_ :
∀ (x y : M),
AddHom.toFun src✝.toAddHom (x + y) = AddHom.toFun src✝.toAddHom x + AddHom.toFun src✝.toAddHom y) },
map_smul' :=
(_ :
∀ (r : R) (x : M),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
(↑(↑(toLin b b) A⁻¹) x) =
x
[PROOFSTEP]
simp only
[GOAL]
case refine'_1
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
src✝ : (fun x => M →ₗ[R] M) A := ↑(toLin b b) A
x : M
⊢ ↑(↑(toLin b b) A⁻¹) (↑(↑(toLin b b) A) x) = x
[PROOFSTEP]
rw [← LinearMap.comp_apply]
[GOAL]
case refine'_2
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
src✝ : (fun x => M →ₗ[R] M) A := ↑(toLin b b) A
x : M
⊢ ↑(↑(toLin b b) A) (↑(↑(toLin b b) A⁻¹) x) = x
[PROOFSTEP]
rw [← LinearMap.comp_apply]
[GOAL]
case refine'_1
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
src✝ : (fun x => M →ₗ[R] M) A := ↑(toLin b b) A
x : M
⊢ ↑(comp (↑(toLin b b) A⁻¹) (↑(toLin b b) A)) x = x
[PROOFSTEP]
simp only [← Matrix.toLin_mul b b b, Matrix.nonsing_inv_mul _ hA, Matrix.mul_nonsing_inv _ hA, toLin_one,
LinearMap.id_apply]
[GOAL]
case refine'_2
n : Type u_1
inst✝⁴ : Fintype n
R : Type u_2
M : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
b : Basis n R M
inst✝ : DecidableEq n
A : Matrix n n R
hA : IsUnit (det A)
src✝ : (fun x => M →ₗ[R] M) A := ↑(toLin b b) A
x : M
⊢ ↑(comp (↑(toLin b b) A) (↑(toLin b b) A⁻¹)) x = x
[PROOFSTEP]
simp only [← Matrix.toLin_mul b b b, Matrix.nonsing_inv_mul _ hA, Matrix.mul_nonsing_inv _ hA, toLin_one,
LinearMap.id_apply]
[GOAL]
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
⊢ (∃ v x, mulVec M v = 0) ↔ det M = 0
[PROOFSTEP]
constructor
[GOAL]
case mp
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
⊢ (∃ v x, mulVec M v = 0) → det M = 0
[PROOFSTEP]
rintro ⟨v, hv, mul_eq⟩
[GOAL]
case mp.intro.intro
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
v : n → K
hv : v ≠ 0
mul_eq : mulVec M v = 0
⊢ det M = 0
[PROOFSTEP]
contrapose! hv
[GOAL]
case mp.intro.intro
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
v : n → K
mul_eq : mulVec M v = 0
hv : det M ≠ 0
⊢ v = 0
[PROOFSTEP]
exact eq_zero_of_mulVec_eq_zero hv mul_eq
[GOAL]
case mpr
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
⊢ det M = 0 → ∃ v x, mulVec M v = 0
[PROOFSTEP]
contrapose!
[GOAL]
case mpr
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
⊢ (∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0) → det M ≠ 0
[PROOFSTEP]
intro h
[GOAL]
case mpr
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
⊢ det M ≠ 0
[PROOFSTEP]
have : Function.Injective (Matrix.toLin' M) := by
simpa only [← LinearMap.ker_eq_bot, ker_toLin'_eq_bot_iff, not_imp_not] using h
[GOAL]
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
⊢ Function.Injective ↑(↑toLin' M)
[PROOFSTEP]
simpa only [← LinearMap.ker_eq_bot, ker_toLin'_eq_bot_iff, not_imp_not] using h
[GOAL]
case mpr
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
this : Function.Injective ↑(↑toLin' M)
⊢ det M ≠ 0
[PROOFSTEP]
have : M * LinearMap.toMatrix' ((LinearEquiv.ofInjectiveEndo (Matrix.toLin' M) this).symm : (n → K) →ₗ[K] n → K) = 1 :=
by
refine' Matrix.toLin'.injective (LinearMap.ext fun v => _)
rw [Matrix.toLin'_mul, Matrix.toLin'_one, Matrix.toLin'_toMatrix', LinearMap.comp_apply]
exact (LinearEquiv.ofInjectiveEndo (Matrix.toLin' M) this).apply_symm_apply v
[GOAL]
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
this : Function.Injective ↑(↑toLin' M)
⊢ M * ↑toMatrix' ↑(LinearEquiv.symm (LinearEquiv.ofInjectiveEndo (↑toLin' M) this)) = 1
[PROOFSTEP]
refine' Matrix.toLin'.injective (LinearMap.ext fun v => _)
[GOAL]
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
this : Function.Injective ↑(↑toLin' M)
v : n → K
⊢ ↑(↑toLin' (M * ↑toMatrix' ↑(LinearEquiv.symm (LinearEquiv.ofInjectiveEndo (↑toLin' M) this)))) v = ↑(↑toLin' 1) v
[PROOFSTEP]
rw [Matrix.toLin'_mul, Matrix.toLin'_one, Matrix.toLin'_toMatrix', LinearMap.comp_apply]
[GOAL]
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
this : Function.Injective ↑(↑toLin' M)
v : n → K
⊢ ↑(↑toLin' M) (↑↑(LinearEquiv.symm (LinearEquiv.ofInjectiveEndo (↑toLin' M) this)) v) = ↑LinearMap.id v
[PROOFSTEP]
exact (LinearEquiv.ofInjectiveEndo (Matrix.toLin' M) this).apply_symm_apply v
[GOAL]
case mpr
n : Type u_1
inst✝⁵ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M✝
inst✝² : Module R M✝
K : Type u_4
inst✝¹ : DecidableEq n
inst✝ : Field K
M : Matrix n n K
h : ∀ (v : n → K), v ≠ 0 → mulVec M v ≠ 0
this✝ : Function.Injective ↑(↑toLin' M)
this : M * ↑toMatrix' ↑(LinearEquiv.symm (LinearEquiv.ofInjectiveEndo (↑toLin' M) this✝)) = 1
⊢ det M ≠ 0
[PROOFSTEP]
exact Matrix.det_ne_zero_of_right_inverse this
[GOAL]
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
⊢ (∃ v x, mulVec M v = 0) ↔ det M = 0
[PROOFSTEP]
have : (∃ (v : _) (_ : v ≠ 0), mulVec ((algebraMap A K).mapMatrix M) v = 0) ↔ _ := exists_mulVec_eq_zero_iff_aux
[GOAL]
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this :
(∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det (↑(RingHom.mapMatrix (algebraMap A K)) M) = 0
⊢ (∃ v x, mulVec M v = 0) ↔ det M = 0
[PROOFSTEP]
rw [← RingHom.map_det, IsFractionRing.to_map_eq_zero_iff] at this
[GOAL]
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
⊢ (∃ v x, mulVec M v = 0) ↔ det M = 0
[PROOFSTEP]
refine' Iff.trans _ this
[GOAL]
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
⊢ (∃ v x, mulVec M v = 0) ↔ ∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
[PROOFSTEP]
constructor
[GOAL]
case mp
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
⊢ (∃ v x, mulVec M v = 0) → ∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
[PROOFSTEP]
rintro ⟨v, hv, mul_eq⟩
[GOAL]
case mpr
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
⊢ (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) → ∃ v x, mulVec M v = 0
[PROOFSTEP]
rintro ⟨v, hv, mul_eq⟩
[GOAL]
case mp.intro.intro
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → A
hv : v ≠ 0
mul_eq : mulVec M v = 0
⊢ ∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
[PROOFSTEP]
refine' ⟨fun i => algebraMap _ _ (v i), mt (fun h => funext fun i => _) hv, _⟩
[GOAL]
case mp.intro.intro.refine'_1
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → A
hv : v ≠ 0
mul_eq : mulVec M v = 0
h : (fun i => ↑(algebraMap A K) (v i)) = 0
i : n
⊢ v i = OfNat.ofNat 0 i
[PROOFSTEP]
exact IsFractionRing.to_map_eq_zero_iff.mp (congr_fun h i)
[GOAL]
case mp.intro.intro.refine'_2
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → A
hv : v ≠ 0
mul_eq : mulVec M v = 0
⊢ (mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) fun i => ↑(algebraMap A K) (v i)) = 0
[PROOFSTEP]
ext i
[GOAL]
case mp.intro.intro.refine'_2.h
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → A
hv : v ≠ 0
mul_eq : mulVec M v = 0
i : n
⊢ mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) (fun i => ↑(algebraMap A K) (v i)) i = OfNat.ofNat 0 i
[PROOFSTEP]
refine' (RingHom.map_mulVec _ _ _ i).symm.trans _
[GOAL]
case mp.intro.intro.refine'_2.h
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → A
hv : v ≠ 0
mul_eq : mulVec M v = 0
i : n
⊢ ↑(algebraMap A K) (mulVec (fun i j => M i j) (fun i => v i) i) = OfNat.ofNat 0 i
[PROOFSTEP]
rw [mul_eq, Pi.zero_apply, RingHom.map_zero, Pi.zero_apply]
[GOAL]
case mpr.intro.intro
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
⊢ ∃ v x, mulVec M v = 0
[PROOFSTEP]
letI := Classical.decEq K
[GOAL]
case mpr.intro.intro
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
⊢ ∃ v x, mulVec M v = 0
[PROOFSTEP]
obtain ⟨⟨b, hb⟩, ba_eq⟩ := IsLocalization.exist_integer_multiples_of_finset (nonZeroDivisors A) (Finset.univ.image v)
[GOAL]
case mpr.intro.intro.intro.mk
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
ba_eq : ∀ (a : K), a ∈ Finset.image v Finset.univ → IsLocalization.IsInteger A (↑{ val := b, property := hb } • a)
⊢ ∃ v x, mulVec M v = 0
[PROOFSTEP]
choose f hf using ba_eq
[GOAL]
case mpr.intro.intro.intro.mk
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
⊢ ∃ v x, mulVec M v = 0
[PROOFSTEP]
refine' ⟨fun i => f _ (Finset.mem_image.mpr ⟨i, Finset.mem_univ i, rfl⟩), mt (fun h => funext fun i => _) hv, _⟩
[GOAL]
case mpr.intro.intro.intro.mk.refine'_1
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
h : (fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) = 0
i : n
⊢ v i = OfNat.ofNat 0 i
[PROOFSTEP]
have := congr_arg (algebraMap A K) (congr_fun h i)
[GOAL]
case mpr.intro.intro.intro.mk.refine'_1
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝¹ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this✝ : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
h : (fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) = 0
i : n
this : ↑(algebraMap A K) (f (v i) (_ : v i ∈ Finset.image v Finset.univ)) = ↑(algebraMap A K) (OfNat.ofNat 0 i)
⊢ v i = OfNat.ofNat 0 i
[PROOFSTEP]
rw [hf, Subtype.coe_mk, Pi.zero_apply, RingHom.map_zero, Algebra.smul_def, mul_eq_zero,
IsFractionRing.to_map_eq_zero_iff] at this
[GOAL]
case mpr.intro.intro.intro.mk.refine'_1
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝¹ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this✝ : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
h : (fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) = 0
i : n
this : b = 0 ∨ v i = 0
⊢ v i = OfNat.ofNat 0 i
[PROOFSTEP]
exact this.resolve_left (nonZeroDivisors.ne_zero hb)
[GOAL]
case mpr.intro.intro.intro.mk.refine'_2
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
⊢ (mulVec M fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) = 0
[PROOFSTEP]
ext i
[GOAL]
case mpr.intro.intro.intro.mk.refine'_2.h
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
i : n
⊢ mulVec M (fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) i = OfNat.ofNat 0 i
[PROOFSTEP]
refine' IsFractionRing.injective A K _
[GOAL]
case mpr.intro.intro.intro.mk.refine'_2.h
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
i : n
⊢ ↑(algebraMap A K) (mulVec M (fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) i) =
↑(algebraMap A K) (OfNat.ofNat 0 i)
[PROOFSTEP]
calc
algebraMap A K (M.mulVec (fun i : n => f (v i) _) i) =
((algebraMap A K).mapMatrix M).mulVec (algebraMap _ K b • v) i :=
?_
_ = 0 := ?_
_ = algebraMap A K 0 := (RingHom.map_zero _).symm
[GOAL]
case mpr.intro.intro.intro.mk.refine'_2.h.calc_1
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
i : n
⊢ ↑(algebraMap A K) (mulVec M (fun i => f (v i) (_ : v i ∈ Finset.image v Finset.univ)) i) =
mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) (↑(algebraMap A K) b • v) i
[PROOFSTEP]
simp_rw [RingHom.map_mulVec, mulVec, dotProduct, Function.comp_apply, hf, RingHom.mapMatrix_apply, Pi.smul_apply,
smul_eq_mul, Algebra.smul_def]
[GOAL]
case mpr.intro.intro.intro.mk.refine'_2.h.calc_2
n : Type u_1
inst✝⁹ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁸ : CommRing R
inst✝⁷ : AddCommGroup M✝
inst✝⁶ : Module R M✝
A : Type u_4
K : Type u_5
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing A
inst✝³ : Nontrivial A
inst✝² : Field K
inst✝¹ : Algebra A K
inst✝ : IsFractionRing A K
M : Matrix n n A
this✝ : (∃ v x, mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0) ↔ det M = 0
v : n → K
hv : v ≠ 0
mul_eq : mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) v = 0
this : DecidableEq K := Classical.decEq K
b : A
hb : b ∈ nonZeroDivisors A
f : (a : K) → a ∈ Finset.image v Finset.univ → A
hf : ∀ (a : K) (a_1 : a ∈ Finset.image v Finset.univ), ↑(algebraMap A K) (f a a_1) = ↑{ val := b, property := hb } • a
i : n
⊢ mulVec (↑(RingHom.mapMatrix (algebraMap A K)) M) (↑(algebraMap A K) b • v) i = 0
[PROOFSTEP]
rw [mulVec_smul, mul_eq, Pi.smul_apply, Pi.zero_apply, smul_zero]
[GOAL]
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
⊢ (∃ v x, vecMul v M = 0) ↔ det M = 0
[PROOFSTEP]
simpa only [← M.det_transpose, ← mulVec_transpose] using exists_mulVec_eq_zero_iff
[GOAL]
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
⊢ Nondegenerate M ↔ det M ≠ 0
[PROOFSTEP]
refine' Iff.trans _ (not_iff_not.mpr exists_vecMul_eq_zero_iff)
[GOAL]
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
⊢ Nondegenerate M ↔ ¬∃ v x, vecMul v M = 0
[PROOFSTEP]
simp only [not_exists]
[GOAL]
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
⊢ Nondegenerate M ↔ ∀ (x : n → A), x ≠ 0 → ¬vecMul x M = 0
[PROOFSTEP]
constructor
[GOAL]
case mp
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
⊢ Nondegenerate M → ∀ (x : n → A), x ≠ 0 → ¬vecMul x M = 0
[PROOFSTEP]
intro hM v hv hMv
[GOAL]
case mp
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
hM : Nondegenerate M
v : n → A
hv : v ≠ 0
hMv : vecMul v M = 0
⊢ False
[PROOFSTEP]
obtain ⟨w, hwMv⟩ := hM.exists_not_ortho_of_ne_zero hv
[GOAL]
case mp.intro
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
hM : Nondegenerate M
v : n → A
hv : v ≠ 0
hMv : vecMul v M = 0
w : n → A
hwMv : v ⬝ᵥ mulVec M w ≠ 0
⊢ False
[PROOFSTEP]
simp [dotProduct_mulVec, hMv, zero_dotProduct, ne_eq, not_true] at hwMv
[GOAL]
case mpr
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
⊢ (∀ (x : n → A), x ≠ 0 → ¬vecMul x M = 0) → Nondegenerate M
[PROOFSTEP]
intro h v hv
[GOAL]
case mpr
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
h : ∀ (x : n → A), x ≠ 0 → ¬vecMul x M = 0
v : n → A
hv : ∀ (w : n → A), v ⬝ᵥ mulVec M w = 0
⊢ v = 0
[PROOFSTEP]
refine' not_imp_not.mp (h v) (funext fun i => _)
[GOAL]
case mpr
n : Type u_1
inst✝⁶ : Fintype n
R : Type u_2
M✝ : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M✝
inst✝³ : Module R M✝
A : Type u_4
inst✝² : DecidableEq n
inst✝¹ : CommRing A
inst✝ : IsDomain A
M : Matrix n n A
h : ∀ (x : n → A), x ≠ 0 → ¬vecMul x M = 0
v : n → A
hv : ∀ (w : n → A), v ⬝ᵥ mulVec M w = 0
i : n
⊢ vecMul v M i = OfNat.ofNat 0 i
[PROOFSTEP]
simpa only [dotProduct_mulVec, dotProduct_single, mul_one] using hv (Pi.single i 1)
[GOAL]
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (j : n), 0 < ∑ i : n, A i j
⊢ det A ≠ 0
[PROOFSTEP]
cases isEmpty_or_nonempty n
[GOAL]
case inl
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (j : n), 0 < ∑ i : n, A i j
h✝ : IsEmpty n
⊢ det A ≠ 0
[PROOFSTEP]
simp
[GOAL]
case inr
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (j : n), 0 < ∑ i : n, A i j
h✝ : Nonempty n
⊢ det A ≠ 0
[PROOFSTEP]
contrapose! h2
[GOAL]
case inr
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
⊢ ∃ j, ∑ i : n, A i j ≤ 0
[PROOFSTEP]
obtain ⟨v, ⟨h_vnz, h_vA⟩⟩ := Matrix.exists_vecMul_eq_zero_iff.mpr h2
[GOAL]
case inr.intro.intro
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
⊢ ∃ j, ∑ i : n, A i j ≤ 0
[PROOFSTEP]
wlog h_sup : 0 < Finset.sup' Finset.univ Finset.univ_nonempty v
[GOAL]
case inr.intro.intro.inr
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
h_sup : ¬0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
⊢ ∃ j, ∑ i : n, A i j ≤ 0
[PROOFSTEP]
refine this h1 inferInstance h2 (-1 • v) ?_ ?_ ?_
[GOAL]
case inr.intro.intro.inr.refine_1
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
h_sup : ¬0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
⊢ -1 • v ≠ 0
[PROOFSTEP]
exact smul_ne_zero (by norm_num) h_vnz
[GOAL]
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
h_sup : ¬0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
⊢ -1 ≠ 0
[PROOFSTEP]
norm_num
[GOAL]
case inr.intro.intro.inr.refine_2
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
h_sup : ¬0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
⊢ (vecMul (-1 • v) fun i j => A i j) = 0
[PROOFSTEP]
rw [Matrix.vecMul_smul, h_vA, smul_zero]
[GOAL]
case inr.intro.intro.inr.refine_3
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
h_sup : ¬0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
⊢ 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) (-1 • v)
[PROOFSTEP]
obtain ⟨i, hi⟩ := Function.ne_iff.mp h_vnz
[GOAL]
case inr.intro.intro.inr.refine_3.intro
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
h_sup : ¬0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
i : n
hi : v i ≠ OfNat.ofNat 0 i
⊢ 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) (-1 • v)
[PROOFSTEP]
simp_rw [Finset.lt_sup'_iff, Finset.mem_univ, true_and] at h_sup ⊢
[GOAL]
case inr.intro.intro.inr.refine_3.intro
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
i : n
hi : v i ≠ OfNat.ofNat 0 i
h_sup : ¬∃ b, 0 < v b
⊢ ∃ b, 0 < (-1 • v) b
[PROOFSTEP]
simp_rw [not_exists, not_lt] at h_sup
[GOAL]
case inr.intro.intro.inr.refine_3.intro
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
i : n
hi : v i ≠ OfNat.ofNat 0 i
h_sup : ∀ (x : n), v x ≤ 0
⊢ ∃ b, 0 < (-1 • v) b
[PROOFSTEP]
refine ⟨i, ?_⟩
[GOAL]
case inr.intro.intro.inr.refine_3.intro
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
i : n
hi : v i ≠ OfNat.ofNat 0 i
h_sup : ∀ (x : n), v x ≤ 0
⊢ 0 < (-1 • v) i
[PROOFSTEP]
rw [Pi.smul_apply, neg_smul, one_smul, Left.neg_pos_iff]
[GOAL]
case inr.intro.intro.inr.refine_3.intro
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
this :
∀ {n : Type u_1} [inst : Fintype n] [inst_1 : DecidableEq n] {S : Type u_2} [inst_2 : LinearOrderedCommRing S]
{A : Matrix n n S},
(∀ (i j : n), i ≠ j → A i j < 0) →
∀ (h : Nonempty n),
det A = 0 →
∀ (v : n → S),
v ≠ 0 →
vecMul v A = 0 → 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v → ∃ j, ∑ i : n, A i j ≤ 0
i : n
hi : v i ≠ OfNat.ofNat 0 i
h_sup : ∀ (x : n), v x ≤ 0
⊢ v i < 0
[PROOFSTEP]
refine Ne.lt_of_le hi (h_sup i)
[GOAL]
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
⊢ ∃ j, ∑ i : n, A i j ≤ 0
[PROOFSTEP]
obtain ⟨j₀, -, h_j₀⟩ := Finset.exists_mem_eq_sup' Finset.univ_nonempty v
[GOAL]
case intro.intro
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
⊢ ∃ j, ∑ i : n, A i j ≤ 0
[PROOFSTEP]
refine ⟨j₀, ?_⟩
[GOAL]
case intro.intro
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
⊢ ∑ i : n, A i j₀ ≤ 0
[PROOFSTEP]
rw [← mul_le_mul_left (h_j₀ ▸ h_sup), Finset.mul_sum, mul_zero]
[GOAL]
case intro.intro
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
⊢ ∑ x : n, v j₀ * A x j₀ ≤ 0
[PROOFSTEP]
rw [show 0 = ∑ i, v i * A i j₀ from (congrFun h_vA j₀).symm]
[GOAL]
case intro.intro
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
⊢ ∑ x : n, v j₀ * A x j₀ ≤ ∑ i : n, v i * A i j₀
[PROOFSTEP]
refine Finset.sum_le_sum (fun i hi => ?_)
[GOAL]
case intro.intro
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
i : n
hi : i ∈ Finset.univ
⊢ v j₀ * A i j₀ ≤ v i * A i j₀
[PROOFSTEP]
by_cases h : i = j₀
[GOAL]
case pos
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
i : n
hi : i ∈ Finset.univ
h : i = j₀
⊢ v j₀ * A i j₀ ≤ v i * A i j₀
[PROOFSTEP]
rw [h]
[GOAL]
case neg
n✝ : Type u_1
inst✝³ : Fintype n✝
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h✝ : Nonempty n
h2 : det A = 0
v : n → S
h_vnz : v ≠ 0
h_vA : vecMul v A = 0
h_sup : 0 < Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v
j₀ : n
h_j₀ : Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) v = v j₀
i : n
hi : i ∈ Finset.univ
h : ¬i = j₀
⊢ v j₀ * A i j₀ ≤ v i * A i j₀
[PROOFSTEP]
exact (mul_le_mul_right_of_neg (h1 i j₀ h)).mpr (h_j₀ ▸ Finset.le_sup' v hi)
[GOAL]
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (i : n), 0 < ∑ j : n, A i j
⊢ det A ≠ 0
[PROOFSTEP]
rw [← Matrix.det_transpose]
[GOAL]
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (i : n), 0 < ∑ j : n, A i j
⊢ det Aᵀ ≠ 0
[PROOFSTEP]
refine det_ne_zero_of_sum_col_pos ?_ ?_
[GOAL]
case refine_1
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (i : n), 0 < ∑ j : n, A i j
⊢ ∀ (i j : n), i ≠ j → Aᵀ i j < 0
[PROOFSTEP]
simp_rw [Matrix.transpose_apply]
[GOAL]
case refine_1
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (i : n), 0 < ∑ j : n, A i j
⊢ ∀ (i j : n), i ≠ j → A j i < 0
[PROOFSTEP]
exact fun i j h => h1 j i h.symm
[GOAL]
case refine_2
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (i : n), 0 < ∑ j : n, A i j
⊢ ∀ (j : n), 0 < ∑ i : n, Aᵀ i j
[PROOFSTEP]
simp_rw [Matrix.transpose_apply]
[GOAL]
case refine_2
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
S : Type u_2
inst✝ : LinearOrderedCommRing S
A : Matrix n n S
h1 : ∀ (i j : n), i ≠ j → A i j < 0
h2 : ∀ (i : n), 0 < ∑ j : n, A i j
⊢ ∀ (j : n), 0 < ∑ x : n, A j x
[PROOFSTEP]
exact h2
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.ToLinearEquiv", "llama_tokens": 22978} |
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Zero α
inst✝ : DecidableEq n
A : Matrix n n α
h : IsDiag A
i j : n
⊢ diagonal (diag A) i j = A i j
[PROOFSTEP]
obtain rfl | hij := Decidable.eq_or_ne i j
[GOAL]
case inl
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Zero α
inst✝ : DecidableEq n
A : Matrix n n α
h : IsDiag A
i : n
⊢ diagonal (diag A) i i = A i i
[PROOFSTEP]
rw [diagonal_apply_eq, diag]
[GOAL]
case inr
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Zero α
inst✝ : DecidableEq n
A : Matrix n n α
h : IsDiag A
i j : n
hij : i ≠ j
⊢ diagonal (diag A) i j = A i j
[PROOFSTEP]
rw [diagonal_apply_ne _ hij, h hij]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Zero α
inst✝ : Zero β
A : Matrix n n α
ha : IsDiag A
f : α → β
hf : f 0 = 0
⊢ IsDiag (Matrix.map A f)
[PROOFSTEP]
intro i j h
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Zero α
inst✝ : Zero β
A : Matrix n n α
ha : IsDiag A
f : α → β
hf : f 0 = 0
i j : n
h : i ≠ j
⊢ Matrix.map A f i j = 0
[PROOFSTEP]
simp [ha h, hf]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : AddGroup α
A : Matrix n n α
ha : IsDiag A
⊢ IsDiag (-A)
[PROOFSTEP]
intro i j h
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : AddGroup α
A : Matrix n n α
ha : IsDiag A
i j : n
h : i ≠ j
⊢ (-A) i j = 0
[PROOFSTEP]
simp [ha h]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : AddZeroClass α
A B : Matrix n n α
ha : IsDiag A
hb : IsDiag B
⊢ IsDiag (A + B)
[PROOFSTEP]
intro i j h
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : AddZeroClass α
A B : Matrix n n α
ha : IsDiag A
hb : IsDiag B
i j : n
h : i ≠ j
⊢ (A + B) i j = 0
[PROOFSTEP]
simp [ha h, hb h]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : AddGroup α
A B : Matrix n n α
ha : IsDiag A
hb : IsDiag B
⊢ IsDiag (A - B)
[PROOFSTEP]
intro i j h
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : AddGroup α
A B : Matrix n n α
ha : IsDiag A
hb : IsDiag B
i j : n
h : i ≠ j
⊢ (A - B) i j = 0
[PROOFSTEP]
simp [ha h, hb h]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝² : Monoid R
inst✝¹ : AddMonoid α
inst✝ : DistribMulAction R α
k : R
A : Matrix n n α
ha : IsDiag A
⊢ IsDiag (k • A)
[PROOFSTEP]
intro i j h
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝² : Monoid R
inst✝¹ : AddMonoid α
inst✝ : DistribMulAction R α
k : R
A : Matrix n n α
ha : IsDiag A
i j : n
h : i ≠ j
⊢ (k • A) i j = 0
[PROOFSTEP]
simp [ha h]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Semiring α
inst✝ : StarRing α
A : Matrix n n α
ha : IsDiag Aᴴ
⊢ IsDiag A
[PROOFSTEP]
convert ha.conjTranspose
[GOAL]
case h.e'_4
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝¹ : Semiring α
inst✝ : StarRing α
A : Matrix n n α
ha : IsDiag Aᴴ
⊢ A = Aᴴᴴ
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : MulZeroClass α
A : Matrix m m α
B : Matrix n n α
hA : IsDiag A
hB : IsDiag B
⊢ IsDiag (kroneckerMap (fun x x_1 => x * x_1) A B)
[PROOFSTEP]
rintro ⟨a, b⟩ ⟨c, d⟩ h
[GOAL]
case mk.mk
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : MulZeroClass α
A : Matrix m m α
B : Matrix n n α
hA : IsDiag A
hB : IsDiag B
a : m
b : n
c : m
d : n
h : (a, b) ≠ (c, d)
⊢ kroneckerMap (fun x x_1 => x * x_1) A B (a, b) (c, d) = 0
[PROOFSTEP]
simp only [Prod.mk.inj_iff, Ne.def, not_and_or] at h
[GOAL]
case mk.mk
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : MulZeroClass α
A : Matrix m m α
B : Matrix n n α
hA : IsDiag A
hB : IsDiag B
a : m
b : n
c : m
d : n
h : ¬a = c ∨ ¬b = d
⊢ kroneckerMap (fun x x_1 => x * x_1) A B (a, b) (c, d) = 0
[PROOFSTEP]
cases' h with hac hbd
[GOAL]
case mk.mk.inl
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : MulZeroClass α
A : Matrix m m α
B : Matrix n n α
hA : IsDiag A
hB : IsDiag B
a : m
b : n
c : m
d : n
hac : ¬a = c
⊢ kroneckerMap (fun x x_1 => x * x_1) A B (a, b) (c, d) = 0
[PROOFSTEP]
simp [hA hac]
[GOAL]
case mk.mk.inr
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : MulZeroClass α
A : Matrix m m α
B : Matrix n n α
hA : IsDiag A
hB : IsDiag B
a : m
b : n
c : m
d : n
hbd : ¬b = d
⊢ kroneckerMap (fun x x_1 => x * x_1) A B (a, b) (c, d) = 0
[PROOFSTEP]
simp [hB hbd]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix n n α
h : IsDiag A
⊢ IsSymm A
[PROOFSTEP]
ext i j
[GOAL]
case a.h
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix n n α
h : IsDiag A
i j : n
⊢ Aᵀ i j = A i j
[PROOFSTEP]
by_cases g : i = j
[GOAL]
case pos
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix n n α
h : IsDiag A
i j : n
g : i = j
⊢ Aᵀ i j = A i j
[PROOFSTEP]
rw [g, transpose_apply]
[GOAL]
case neg
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix n n α
h : IsDiag A
i j : n
g : ¬i = j
⊢ Aᵀ i j = A i j
[PROOFSTEP]
simp [h g, h (Ne.symm g)]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
D : Matrix n n α
ha : IsDiag A
hd : IsDiag D
⊢ IsDiag (Matrix.fromBlocks A 0 0 D)
[PROOFSTEP]
rintro (i | i) (j | j) hij
[GOAL]
case inl.inl
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
D : Matrix n n α
ha : IsDiag A
hd : IsDiag D
i j : m
hij : Sum.inl i ≠ Sum.inl j
⊢ Matrix.fromBlocks A 0 0 D (Sum.inl i) (Sum.inl j) = 0
[PROOFSTEP]
exact ha (ne_of_apply_ne _ hij)
[GOAL]
case inl.inr
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
D : Matrix n n α
ha : IsDiag A
hd : IsDiag D
i : m
j : n
hij : Sum.inl i ≠ Sum.inr j
⊢ Matrix.fromBlocks A 0 0 D (Sum.inl i) (Sum.inr j) = 0
[PROOFSTEP]
rfl
[GOAL]
case inr.inl
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
D : Matrix n n α
ha : IsDiag A
hd : IsDiag D
i : n
j : m
hij : Sum.inr i ≠ Sum.inl j
⊢ Matrix.fromBlocks A 0 0 D (Sum.inr i) (Sum.inl j) = 0
[PROOFSTEP]
rfl
[GOAL]
case inr.inr
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
D : Matrix n n α
ha : IsDiag A
hd : IsDiag D
i j : n
hij : Sum.inr i ≠ Sum.inr j
⊢ Matrix.fromBlocks A 0 0 D (Sum.inr i) (Sum.inr j) = 0
[PROOFSTEP]
exact hd (ne_of_apply_ne _ hij)
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
⊢ IsDiag (fromBlocks A B C D) ↔ IsDiag A ∧ B = 0 ∧ C = 0 ∧ IsDiag D
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
⊢ IsDiag (fromBlocks A B C D) → IsDiag A ∧ B = 0 ∧ C = 0 ∧ IsDiag D
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
h : IsDiag (fromBlocks A B C D)
⊢ IsDiag A ∧ B = 0 ∧ C = 0 ∧ IsDiag D
[PROOFSTEP]
refine' ⟨fun i j hij => _, ext fun i j => _, ext fun i j => _, fun i j hij => _⟩
[GOAL]
case mp.refine'_1
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
h : IsDiag (fromBlocks A B C D)
i j : m
hij : i ≠ j
⊢ A i j = 0
[PROOFSTEP]
exact h (Sum.inl_injective.ne hij)
[GOAL]
case mp.refine'_2
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
h : IsDiag (fromBlocks A B C D)
i : m
j : n
⊢ B i j = OfNat.ofNat 0 i j
[PROOFSTEP]
exact h Sum.inl_ne_inr
[GOAL]
case mp.refine'_3
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
h : IsDiag (fromBlocks A B C D)
i : n
j : m
⊢ C i j = OfNat.ofNat 0 i j
[PROOFSTEP]
exact h Sum.inr_ne_inl
[GOAL]
case mp.refine'_4
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
h : IsDiag (fromBlocks A B C D)
i j : n
hij : i ≠ j
⊢ D i j = 0
[PROOFSTEP]
exact h (Sum.inr_injective.ne hij)
[GOAL]
case mpr
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
⊢ IsDiag A ∧ B = 0 ∧ C = 0 ∧ IsDiag D → IsDiag (fromBlocks A B C D)
[PROOFSTEP]
rintro ⟨ha, hb, hc, hd⟩
[GOAL]
case mpr.intro.intro.intro
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
B : Matrix m n α
C : Matrix n m α
D : Matrix n n α
ha : IsDiag A
hb : B = 0
hc : C = 0
hd : IsDiag D
⊢ IsDiag (fromBlocks A B C D)
[PROOFSTEP]
convert IsDiag.fromBlocks ha hd
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
C : Matrix n m α
D : Matrix n n α
h : IsSymm (Matrix.fromBlocks A 0 C D)
ha : IsDiag A
hd : IsDiag D
⊢ IsDiag (Matrix.fromBlocks A 0 C D)
[PROOFSTEP]
rw [← (isSymm_fromBlocks_iff.1 h).2.1]
[GOAL]
α : Type u_1
β : Type u_2
R : Type u_3
n : Type u_4
m : Type u_5
inst✝ : Zero α
A : Matrix m m α
C : Matrix n m α
D : Matrix n n α
h : IsSymm (Matrix.fromBlocks A 0 C D)
ha : IsDiag A
hd : IsDiag D
⊢ IsDiag (Matrix.fromBlocks A 0 0ᵀ D)
[PROOFSTEP]
exact ha.fromBlocks hd
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.IsDiag", "llama_tokens": 5123} |
[GOAL]
⊢ univ = {0, 1}
[PROOFSTEP]
ext x
[GOAL]
case a
x : Fin 2
⊢ x ∈ univ ↔ x ∈ {0, 1}
[PROOFSTEP]
fin_cases x
[GOAL]
case a.head
⊢ { val := 0, isLt := (_ : 0 < 2) } ∈ univ ↔ { val := 0, isLt := (_ : 0 < 2) } ∈ {0, 1}
[PROOFSTEP]
simp
[GOAL]
case a.tail.head
⊢ { val := 1, isLt := (_ : (fun a => a < 2) 1) } ∈ univ ↔ { val := 1, isLt := (_ : (fun a => a < 2) 1) } ∈ {0, 1}
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
⊢ ↑(weightedVSubOfPoint s p b) w = ∑ i in s, w i • (p i -ᵥ b)
[PROOFSTEP]
simp [weightedVSubOfPoint, LinearMap.sum_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p b : P
⊢ ↑(weightedVSubOfPoint s (fun x => p) b) w = (∑ i in s, w i) • (p -ᵥ b)
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, sum_smul]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ∈ s → w₁ i = w₂ i
p₁ p₂ : ι → P
hp : ∀ (i : ι), i ∈ s → p₁ i = p₂ i
b : P
⊢ ↑(weightedVSubOfPoint s p₁ b) w₁ = ↑(weightedVSubOfPoint s p₂ b) w₂
[PROOFSTEP]
simp_rw [weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ∈ s → w₁ i = w₂ i
p₁ p₂ : ι → P
hp : ∀ (i : ι), i ∈ s → p₁ i = p₂ i
b : P
⊢ ∑ i in s, w₁ i • (p₁ i -ᵥ b) = ∑ i in s, w₂ i • (p₂ i -ᵥ b)
[PROOFSTEP]
refine sum_congr rfl fun i hi => ?_
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ∈ s → w₁ i = w₂ i
p₁ p₂ : ι → P
hp : ∀ (i : ι), i ∈ s → p₁ i = p₂ i
b : P
i : ι
hi : i ∈ s
⊢ w₁ i • (p₁ i -ᵥ b) = w₂ i • (p₂ i -ᵥ b)
[PROOFSTEP]
rw [hw i hi, hp i hi]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
j : ι
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ≠ j → w₁ i = w₂ i
⊢ ↑(weightedVSubOfPoint s p (p j)) w₁ = ↑(weightedVSubOfPoint s p (p j)) w₂
[PROOFSTEP]
simp only [Finset.weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
j : ι
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ≠ j → w₁ i = w₂ i
⊢ ∑ i in s, w₁ i • (p i -ᵥ p j) = ∑ i in s, w₂ i • (p i -ᵥ p j)
[PROOFSTEP]
congr
[GOAL]
case e_f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
j : ι
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ≠ j → w₁ i = w₂ i
⊢ (fun i => w₁ i • (p i -ᵥ p j)) = fun i => w₂ i • (p i -ᵥ p j)
[PROOFSTEP]
ext i
[GOAL]
case e_f.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
j : ι
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ≠ j → w₁ i = w₂ i
i : ι
⊢ w₁ i • (p i -ᵥ p j) = w₂ i • (p i -ᵥ p j)
[PROOFSTEP]
cases' eq_or_ne i j with h h
[GOAL]
case e_f.h.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
j : ι
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ≠ j → w₁ i = w₂ i
i : ι
h : i = j
⊢ w₁ i • (p i -ᵥ p j) = w₂ i • (p i -ᵥ p j)
[PROOFSTEP]
simp [h]
[GOAL]
case e_f.h.inr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
j : ι
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ≠ j → w₁ i = w₂ i
i : ι
h : i ≠ j
⊢ w₁ i • (p i -ᵥ p j) = w₂ i • (p i -ᵥ p j)
[PROOFSTEP]
simp [hw i h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
⊢ ↑(weightedVSubOfPoint s p b₁) w = ↑(weightedVSubOfPoint s p b₂) w
[PROOFSTEP]
apply eq_of_sub_eq_zero
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
⊢ ↑(weightedVSubOfPoint s p b₁) w - ↑(weightedVSubOfPoint s p b₂) w = 0
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply, ← sum_sub_distrib]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
⊢ ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)) = 0
[PROOFSTEP]
conv_lhs =>
congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
[GOAL]
case s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| s
case f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
·skip
[GOAL]
case s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| s
[PROOFSTEP]
skip
[GOAL]
case s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| s
[PROOFSTEP]
skip
[GOAL]
case s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| s
[PROOFSTEP]
skip
[GOAL]
case f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
ext
[GOAL]
case f.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
x✝ : ι
| w x✝ • (p x✝ -ᵥ b₁) - w x✝ • (p x✝ -ᵥ b₂)
[PROOFSTEP]
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 0
b₁ b₂ : P
⊢ ∑ x in s, w x • (b₂ -ᵥ b₁) = 0
[PROOFSTEP]
rw [← sum_smul, h, zero_smul]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
⊢ ↑(weightedVSubOfPoint s p b₁) w +ᵥ b₁ = ↑(weightedVSubOfPoint s p b₂) w +ᵥ b₂
[PROOFSTEP]
erw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply, ← @vsub_eq_zero_iff_eq V, vadd_vsub_assoc,
vsub_vadd_eq_vsub_sub, ← add_sub_assoc, add_comm, add_sub_assoc, ← sum_sub_distrib]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
⊢ b₁ -ᵥ b₂ + ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)) = 0
[PROOFSTEP]
conv_lhs =>
congr
·skip
· congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂ + ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
·skip
· congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂ + ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
·skip
· congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂ + ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
·skip
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂
[PROOFSTEP]
skip
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂
[PROOFSTEP]
skip
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| b₁ -ᵥ b₂
[PROOFSTEP]
skip
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
· congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
·skip
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂))
[PROOFSTEP]
congr
[GOAL]
case a.s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| s
case a.f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
·skip
[GOAL]
case a.s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| s
[PROOFSTEP]
skip
[GOAL]
case a.s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| s
[PROOFSTEP]
skip
[GOAL]
case a.s
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| s
[PROOFSTEP]
skip
[GOAL]
case a.f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
· ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case a.f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case a.f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
ext
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
case a.f
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
| fun x => w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)
[PROOFSTEP]
ext
[GOAL]
case a.f.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
x✝ : ι
| w x✝ • (p x✝ -ᵥ b₁) - w x✝ • (p x✝ -ᵥ b₂)
[PROOFSTEP]
rw [← smul_sub, vsub_sub_vsub_cancel_left]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
h : ∑ i in s, w i = 1
b₁ b₂ : P
⊢ b₁ -ᵥ b₂ + ∑ x in s, w x • (b₂ -ᵥ b₁) = 0
[PROOFSTEP]
rw [← sum_smul, h, one_smul, vsub_add_vsub_cancel, vsub_self]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
w : ι → k
p : ι → P
i : ι
⊢ ↑(weightedVSubOfPoint (erase s i) p (p i)) w = ↑(weightedVSubOfPoint s p (p i)) w
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
w : ι → k
p : ι → P
i : ι
⊢ ∑ i_1 in erase s i, w i_1 • (p i_1 -ᵥ p i) = ∑ i_1 in s, w i_1 • (p i_1 -ᵥ p i)
[PROOFSTEP]
apply sum_erase
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
w : ι → k
p : ι → P
i : ι
⊢ w i • (p i -ᵥ p i) = 0
[PROOFSTEP]
rw [vsub_self, smul_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
w : ι → k
p : ι → P
i : ι
⊢ ↑(weightedVSubOfPoint (insert i s) p (p i)) w = ↑(weightedVSubOfPoint s p (p i)) w
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
w : ι → k
p : ι → P
i : ι
⊢ ∑ i_1 in insert i s, w i_1 • (p i_1 -ᵥ p i) = ∑ i_1 in s, w i_1 • (p i_1 -ᵥ p i)
[PROOFSTEP]
apply sum_insert_zero
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
w : ι → k
p : ι → P
i : ι
⊢ w i • (p i -ᵥ p i) = 0
[PROOFSTEP]
rw [vsub_self, smul_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
w : ι → k
p : ι → P
b : P
s₁ s₂ : Finset ι
h : s₁ ⊆ s₂
⊢ ↑(weightedVSubOfPoint s₁ p b) w = ↑(weightedVSubOfPoint s₂ p b) (Set.indicator (↑s₁) w)
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
w : ι → k
p : ι → P
b : P
s₁ s₂ : Finset ι
h : s₁ ⊆ s₂
⊢ ∑ i in s₁, w i • (p i -ᵥ b) = ∑ i in s₂, Set.indicator (↑s₁) w i • (p i -ᵥ b)
[PROOFSTEP]
exact Set.sum_indicator_subset_of_eq_zero w (fun i wi => wi • (p i -ᵥ b : V)) h fun i => zero_smul k _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
e : ι₂ ↪ ι
w : ι → k
p : ι → P
b : P
⊢ ↑(weightedVSubOfPoint (map e s₂) p b) w = ↑(weightedVSubOfPoint s₂ (p ∘ ↑e) b) (w ∘ ↑e)
[PROOFSTEP]
simp_rw [weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
e : ι₂ ↪ ι
w : ι → k
p : ι → P
b : P
⊢ ∑ i in map e s₂, w i • (p i -ᵥ b) = ∑ i in s₂, (w ∘ ↑e) i • ((p ∘ ↑e) i -ᵥ b)
[PROOFSTEP]
exact Finset.sum_map _ _ _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₁ p₂ : ι → P
b : P
⊢ ∑ i in s, w i • (p₁ i -ᵥ p₂ i) = ↑(weightedVSubOfPoint s p₁ b) w - ↑(weightedVSubOfPoint s p₂ b) w
[PROOFSTEP]
simp_rw [weightedVSubOfPoint_apply, ← sum_sub_distrib, ← smul_sub, vsub_sub_vsub_cancel_right]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₁ : ι → P
p₂ b : P
⊢ ∑ i in s, w i • (p₁ i -ᵥ p₂) = ↑(weightedVSubOfPoint s p₁ b) w - (∑ i in s, w i) • (p₂ -ᵥ b)
[PROOFSTEP]
rw [sum_smul_vsub_eq_weightedVSubOfPoint_sub, weightedVSubOfPoint_apply_const]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₂ : ι → P
p₁ b : P
⊢ ∑ i in s, w i • (p₁ -ᵥ p₂ i) = (∑ i in s, w i) • (p₁ -ᵥ b) - ↑(weightedVSubOfPoint s p₂ b) w
[PROOFSTEP]
rw [sum_smul_vsub_eq_weightedVSubOfPoint_sub, weightedVSubOfPoint_apply_const]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
inst✝ : DecidableEq ι
s₂ : Finset ι
h : s₂ ⊆ s
w : ι → k
p : ι → P
b : P
⊢ ↑(weightedVSubOfPoint (s \ s₂) p b) w + ↑(weightedVSubOfPoint s₂ p b) w = ↑(weightedVSubOfPoint s p b) w
[PROOFSTEP]
simp_rw [weightedVSubOfPoint_apply, sum_sdiff h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
inst✝ : DecidableEq ι
s₂ : Finset ι
h : s₂ ⊆ s
w : ι → k
p : ι → P
b : P
⊢ ↑(weightedVSubOfPoint (s \ s₂) p b) w - ↑(weightedVSubOfPoint s₂ p b) (-w) = ↑(weightedVSubOfPoint s p b) w
[PROOFSTEP]
rw [map_neg, sub_neg_eq_add, s.weightedVSubOfPoint_sdiff h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
pred : ι → Prop
inst✝ : DecidablePred pred
⊢ (↑(weightedVSubOfPoint (Finset.subtype pred s) (fun i => p ↑i) b) fun i => w ↑i) =
↑(weightedVSubOfPoint (filter pred s) p b) w
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply, ← sum_subtype_eq_sum_filter]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
pred : ι → Prop
inst✝ : DecidablePred pred
h : ∀ (i : ι), i ∈ s → w i ≠ 0 → pred i
⊢ ↑(weightedVSubOfPoint (filter pred s) p b) w = ↑(weightedVSubOfPoint s p b) w
[PROOFSTEP]
rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply, sum_filter_of_ne]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
pred : ι → Prop
inst✝ : DecidablePred pred
h : ∀ (i : ι), i ∈ s → w i ≠ 0 → pred i
⊢ ∀ (x : ι), x ∈ s → w x • (p x -ᵥ b) ≠ 0 → pred x
[PROOFSTEP]
intro i hi hne
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
pred : ι → Prop
inst✝ : DecidablePred pred
h : ∀ (i : ι), i ∈ s → w i ≠ 0 → pred i
i : ι
hi : i ∈ s
hne : w i • (p i -ᵥ b) ≠ 0
⊢ pred i
[PROOFSTEP]
refine' h i hi _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
pred : ι → Prop
inst✝ : DecidablePred pred
h : ∀ (i : ι), i ∈ s → w i ≠ 0 → pred i
i : ι
hi : i ∈ s
hne : w i • (p i -ᵥ b) ≠ 0
⊢ w i ≠ 0
[PROOFSTEP]
intro hw
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
pred : ι → Prop
inst✝ : DecidablePred pred
h : ∀ (i : ι), i ∈ s → w i ≠ 0 → pred i
i : ι
hi : i ∈ s
hne : w i • (p i -ᵥ b) ≠ 0
hw : w i = 0
⊢ False
[PROOFSTEP]
simp [hw] at hne
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
b : P
c : k
⊢ ↑(weightedVSubOfPoint s p b) (c • w) = c • ↑(weightedVSubOfPoint s p b) w
[PROOFSTEP]
simp_rw [weightedVSubOfPoint_apply, smul_sum, Pi.smul_apply, smul_smul, smul_eq_mul]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
⊢ ↑(weightedVSub s p) w = ∑ i in s, w i • (p i -ᵥ Classical.choice (_ : Nonempty P))
[PROOFSTEP]
simp [weightedVSub, LinearMap.sum_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : P
h : ∑ i in s, w i = 0
⊢ ↑(weightedVSub s fun x => p) w = 0
[PROOFSTEP]
rw [weightedVSub, weightedVSubOfPoint_apply_const, h, zero_smul]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
⊢ ↑(weightedVSub ∅ p) w = 0
[PROOFSTEP]
simp [weightedVSub_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₁ : ι → P
p₂ : P
h : ∑ i in s, w i = 0
⊢ ∑ i in s, w i • (p₁ i -ᵥ p₂) = ↑(weightedVSub s p₁) w
[PROOFSTEP]
rw [sum_smul_vsub_eq_weightedVSub_sub, s.weightedVSub_apply_const _ _ h, sub_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₂ : ι → P
p₁ : P
h : ∑ i in s, w i = 0
⊢ ∑ i in s, w i • (p₁ -ᵥ p₂ i) = -↑(weightedVSub s p₂) w
[PROOFSTEP]
rw [sum_smul_vsub_eq_weightedVSub_sub, s.weightedVSub_apply_const _ _ h, zero_sub]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
w₁ w₂ : ι → k
⊢ (fun w => ↑(weightedVSubOfPoint s p (Classical.choice (_ : Nonempty P))) w +ᵥ Classical.choice (_ : Nonempty P))
(w₂ +ᵥ w₁) =
↑(weightedVSub s p) w₂ +ᵥ
(fun w => ↑(weightedVSubOfPoint s p (Classical.choice (_ : Nonempty P))) w +ᵥ Classical.choice (_ : Nonempty P))
w₁
[PROOFSTEP]
simp_rw [vadd_vadd, weightedVSub, vadd_eq_add, LinearMap.map_add]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : P
h : ∑ i in s, w i = 1
⊢ ↑(affineCombination k s fun x => p) w = p
[PROOFSTEP]
rw [affineCombination_apply, s.weightedVSubOfPoint_apply_const, h, one_smul, vsub_vadd]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w₁ w₂ : ι → k
hw : ∀ (i : ι), i ∈ s → w₁ i = w₂ i
p₁ p₂ : ι → P
hp : ∀ (i : ι), i ∈ s → p₁ i = p₂ i
⊢ ↑(affineCombination k s p₁) w₁ = ↑(affineCombination k s p₂) w₂
[PROOFSTEP]
simp_rw [affineCombination_apply, s.weightedVSubOfPoint_congr hw hp]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w₁ w₂ : ι → k
p : ι → P
⊢ ↑(weightedVSub s p) w₁ +ᵥ ↑(affineCombination k s p) w₂ = ↑(affineCombination k s p) (w₁ + w₂)
[PROOFSTEP]
rw [← vadd_eq_add, AffineMap.map_vadd, affineCombination_linear]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w₁ w₂ : ι → k
p : ι → P
⊢ ↑(affineCombination k s p) w₁ -ᵥ ↑(affineCombination k s p) w₂ = ↑(weightedVSub s p) (w₁ - w₂)
[PROOFSTEP]
rw [← AffineMap.linearMap_vsub, affineCombination_linear, vsub_eq_sub]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
⊢ ↑(affineCombination k (attach s) f) (w ∘ f) = ↑(affineCombination k (image f univ) id) w
[PROOFSTEP]
simp only [affineCombination, weightedVSubOfPoint_apply, id.def, vadd_right_cancel_iff, Function.comp_apply,
AffineMap.coe_mk]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
⊢ ∑ x in attach s, w (f x) • (f x -ᵥ Classical.choice (_ : Nonempty P)) =
∑ x in image f univ, w x • (x -ᵥ Classical.choice (_ : Nonempty P))
[PROOFSTEP]
let g₁ : s → V := fun i => w (f i) • (f i -ᵥ Classical.choice S.Nonempty)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
⊢ ∑ x in attach s, w (f x) • (f x -ᵥ Classical.choice (_ : Nonempty P)) =
∑ x in image f univ, w x • (x -ᵥ Classical.choice (_ : Nonempty P))
[PROOFSTEP]
let g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice S.Nonempty)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
⊢ ∑ x in attach s, w (f x) • (f x -ᵥ Classical.choice (_ : Nonempty P)) =
∑ x in image f univ, w x • (x -ᵥ Classical.choice (_ : Nonempty P))
[PROOFSTEP]
change univ.sum g₁ = (image f univ).sum g₂
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
⊢ Finset.sum univ g₁ = Finset.sum (image f univ) g₂
[PROOFSTEP]
have hgf : g₁ = g₂ ∘ f := by
ext
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
⊢ g₁ = g₂ ∘ f
[PROOFSTEP]
ext
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
x✝ : { x // x ∈ s }
⊢ g₁ x✝ = (g₂ ∘ f) x✝
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
hgf : g₁ = g₂ ∘ f
⊢ Finset.sum univ g₁ = Finset.sum (image f univ) g₂
[PROOFSTEP]
rw [hgf, sum_image]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
hgf : g₁ = g₂ ∘ f
⊢ Finset.sum univ (g₂ ∘ f) = ∑ x : { x // x ∈ s }, w (f x) • (f x -ᵥ Classical.choice (_ : Nonempty P))
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
hgf : g₁ = g₂ ∘ f
⊢ ∀ (x : { x // x ∈ s }), x ∈ univ → ∀ (y : { x // x ∈ s }), y ∈ univ → f x = f y → x = y
[PROOFSTEP]
simp only [Function.comp_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq P
s : Finset P
w : P → k
f : { x // x ∈ s } → P
hf : Function.Injective f
g₁ : { x // x ∈ s } → V := fun i => w (f i) • (f i -ᵥ Classical.choice (_ : Nonempty P))
g₂ : P → V := fun i => w i • (i -ᵥ Classical.choice (_ : Nonempty P))
hgf : g₁ = g₂ ∘ f
⊢ ∀ (x : { x // x ∈ s }), x ∈ univ → ∀ (y : { x // x ∈ s }), y ∈ univ → f x = f y → x = y
[PROOFSTEP]
exact fun _ _ _ _ hxy => hf hxy
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset P
w : P → k
⊢ ↑(affineCombination k (attach s) Subtype.val) (w ∘ Subtype.val) = ↑(affineCombination k s id) w
[PROOFSTEP]
classical rw [attach_affineCombination_of_injective s w ((↑) : s → P) Subtype.coe_injective, univ_eq_attach,
attach_image_val]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset P
w : P → k
⊢ ↑(affineCombination k (attach s) Subtype.val) (w ∘ Subtype.val) = ↑(affineCombination k s id) w
[PROOFSTEP]
rw [attach_affineCombination_of_injective s w ((↑) : s → P) Subtype.coe_injective, univ_eq_attach, attach_image_val]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι✝ : Type u_4
s✝ : Finset ι✝
ι₂ : Type u_5
s₂ : Finset ι₂
ι : Type u_6
s : Finset ι
w : ι → k
p : ι → V
hw : Finset.sum s w = 0
⊢ ↑(weightedVSub s p) w = ∑ i in s, w i • p i
[PROOFSTEP]
simp [s.weightedVSub_apply, vsub_eq_sub, smul_sub, ← Finset.sum_smul, hw]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset ι
p : ι → V
w : ι → k
hw : ∑ i in s, w i = 1
⊢ ↑(affineCombination k s p) w = ∑ i in s, w i • p i
[PROOFSTEP]
simp [s.affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w p hw 0]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
⊢ ↑(affineCombination k s p) w = p i
[PROOFSTEP]
have h1 : ∑ i in s, w i = 1 := hwi ▸ sum_eq_single i hw0 fun h => False.elim (h his)
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
⊢ ↑(affineCombination k s p) w = p i
[PROOFSTEP]
rw [s.affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w p h1 (p i), weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
⊢ ∑ i_1 in s, w i_1 • (p i_1 -ᵥ p i) +ᵥ p i = p i
[PROOFSTEP]
convert zero_vadd V (p i)
[GOAL]
case h.e'_2.h.e'_5
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
⊢ ∑ i_1 in s, w i_1 • (p i_1 -ᵥ p i) = 0
[PROOFSTEP]
refine sum_eq_zero ?_
[GOAL]
case h.e'_2.h.e'_5
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
⊢ ∀ (x : ι), x ∈ s → w x • (p x -ᵥ p i) = 0
[PROOFSTEP]
intro i2 hi2
[GOAL]
case h.e'_2.h.e'_5
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
i2 : ι
hi2 : i2 ∈ s
⊢ w i2 • (p i2 -ᵥ p i) = 0
[PROOFSTEP]
by_cases h : i2 = i
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
i2 : ι
hi2 : i2 ∈ s
h : i2 = i
⊢ w i2 • (p i2 -ᵥ p i) = 0
[PROOFSTEP]
simp [h]
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
i : ι
his : i ∈ s
hwi : w i = 1
hw0 : ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → w i2 = 0
h1 : ∑ i in s, w i = 1
i2 : ι
hi2 : i2 ∈ s
h : ¬i2 = i
⊢ w i2 • (p i2 -ᵥ p i) = 0
[PROOFSTEP]
simp [hw0 i2 hi2 h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
w : ι → k
p : ι → P
s₁ s₂ : Finset ι
h : s₁ ⊆ s₂
⊢ ↑(affineCombination k s₁ p) w = ↑(affineCombination k s₂ p) (Set.indicator (↑s₁) w)
[PROOFSTEP]
rw [affineCombination_apply, affineCombination_apply, weightedVSubOfPoint_indicator_subset _ _ _ h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
e : ι₂ ↪ ι
w : ι → k
p : ι → P
⊢ ↑(affineCombination k (map e s₂) p) w = ↑(affineCombination k s₂ (p ∘ ↑e)) (w ∘ ↑e)
[PROOFSTEP]
simp_rw [affineCombination_apply, weightedVSubOfPoint_map]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₁ p₂ : ι → P
⊢ ∑ i in s, w i • (p₁ i -ᵥ p₂ i) = ↑(affineCombination k s p₁) w -ᵥ ↑(affineCombination k s p₂) w
[PROOFSTEP]
simp_rw [affineCombination_apply, vadd_vsub_vadd_cancel_right]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₁ p₂ : ι → P
⊢ ∑ i in s, w i • (p₁ i -ᵥ p₂ i) =
↑(weightedVSubOfPoint s p₁ (Classical.choice (_ : Nonempty P))) w -
↑(weightedVSubOfPoint s p₂ (Classical.choice (_ : Nonempty P))) w
[PROOFSTEP]
exact s.sum_smul_vsub_eq_weightedVSubOfPoint_sub _ _ _ _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₁ : ι → P
p₂ : P
h : ∑ i in s, w i = 1
⊢ ∑ i in s, w i • (p₁ i -ᵥ p₂) = ↑(affineCombination k s p₁) w -ᵥ p₂
[PROOFSTEP]
rw [sum_smul_vsub_eq_affineCombination_vsub, affineCombination_apply_const _ _ _ h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p₂ : ι → P
p₁ : P
h : ∑ i in s, w i = 1
⊢ ∑ i in s, w i • (p₁ -ᵥ p₂ i) = p₁ -ᵥ ↑(affineCombination k s p₂) w
[PROOFSTEP]
rw [sum_smul_vsub_eq_affineCombination_vsub, affineCombination_apply_const _ _ _ h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
inst✝ : DecidableEq ι
s₂ : Finset ι
h : s₂ ⊆ s
w : ι → k
p : ι → P
⊢ ↑(affineCombination k (s \ s₂) p) w -ᵥ ↑(affineCombination k s₂ p) (-w) = ↑(weightedVSub s p) w
[PROOFSTEP]
simp_rw [affineCombination_apply, vadd_vsub_vadd_cancel_right]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂✝ : Finset ι₂
inst✝ : DecidableEq ι
s₂ : Finset ι
h : s₂ ⊆ s
w : ι → k
p : ι → P
⊢ ↑(weightedVSubOfPoint (s \ s₂) p (Classical.choice (_ : Nonempty P))) w -
↑(weightedVSubOfPoint s₂ p (Classical.choice (_ : Nonempty P))) (-w) =
↑(weightedVSub s p) w
[PROOFSTEP]
exact s.weightedVSub_sdiff_sub h _ _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
hw : ↑(weightedVSub s p) w = 0
i : ι
inst✝ : DecidablePred fun x => x ≠ i
his : i ∈ s
hwi : w i = -1
⊢ ↑(affineCombination k (filter (fun x => x ≠ i) s) p) w = p i
[PROOFSTEP]
classical
rw [← @vsub_eq_zero_iff_eq V, ← hw, ← s.affineCombination_sdiff_sub (singleton_subset_iff.2 his),
sdiff_singleton_eq_erase, ← filter_ne']
congr
refine' (affineCombination_of_eq_one_of_eq_zero _ _ _ (mem_singleton_self _) _ _).symm
· simp [hwi]
· simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
hw : ↑(weightedVSub s p) w = 0
i : ι
inst✝ : DecidablePred fun x => x ≠ i
his : i ∈ s
hwi : w i = -1
⊢ ↑(affineCombination k (filter (fun x => x ≠ i) s) p) w = p i
[PROOFSTEP]
rw [← @vsub_eq_zero_iff_eq V, ← hw, ← s.affineCombination_sdiff_sub (singleton_subset_iff.2 his),
sdiff_singleton_eq_erase, ← filter_ne']
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
hw : ↑(weightedVSub s p) w = 0
i : ι
inst✝ : DecidablePred fun x => x ≠ i
his : i ∈ s
hwi : w i = -1
⊢ ↑(affineCombination k (filter (fun x => x ≠ i) s) p) w -ᵥ p i =
↑(affineCombination k (filter (fun a => a ≠ i) s) p) w -ᵥ ↑(affineCombination k {i} p) (-w)
[PROOFSTEP]
congr
[GOAL]
case e_a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
hw : ↑(weightedVSub s p) w = 0
i : ι
inst✝ : DecidablePred fun x => x ≠ i
his : i ∈ s
hwi : w i = -1
⊢ p i = ↑(affineCombination k {i} p) (-w)
[PROOFSTEP]
refine' (affineCombination_of_eq_one_of_eq_zero _ _ _ (mem_singleton_self _) _ _).symm
[GOAL]
case e_a.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
hw : ↑(weightedVSub s p) w = 0
i : ι
inst✝ : DecidablePred fun x => x ≠ i
his : i ∈ s
hwi : w i = -1
⊢ (-w) i = 1
[PROOFSTEP]
simp [hwi]
[GOAL]
case e_a.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
hw : ↑(weightedVSub s p) w = 0
i : ι
inst✝ : DecidablePred fun x => x ≠ i
his : i ∈ s
hwi : w i = -1
⊢ ∀ (i2 : ι), i2 ∈ {i} → i2 ≠ i → (-w) i2 = 0
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
pred : ι → Prop
inst✝ : DecidablePred pred
⊢ (↑(affineCombination k (Finset.subtype pred s) fun i => p ↑i) fun i => w ↑i) =
↑(affineCombination k (filter pred s) p) w
[PROOFSTEP]
rw [affineCombination_apply, affineCombination_apply, weightedVSubOfPoint_subtype_eq_filter]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
w : ι → k
p : ι → P
pred : ι → Prop
inst✝ : DecidablePred pred
h : ∀ (i : ι), i ∈ s → w i ≠ 0 → pred i
⊢ ↑(affineCombination k (filter pred s) p) w = ↑(affineCombination k s p) w
[PROOFSTEP]
rw [affineCombination_apply, affineCombination_apply, s.weightedVSubOfPoint_filter_of_ne _ _ _ h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
v : V
x : k
s : Set ι
p : ι → P
b : P
⊢ (∃ fs x_1 w x, v = ↑(weightedVSubOfPoint fs p b) w) ↔ ∃ fs w x, v = ↑(weightedVSubOfPoint fs (fun i => p ↑i) b) w
[PROOFSTEP]
classical
simp_rw [weightedVSubOfPoint_apply]
constructor
· rintro ⟨fs, hfs, w, rfl, rfl⟩
exact ⟨fs.subtype s, fun i => w i, sum_subtype_of_mem _ hfs, (sum_subtype_of_mem _ hfs).symm⟩
· rintro ⟨fs, w, rfl, rfl⟩
refine'
⟨fs.map (Function.Embedding.subtype _), map_subtype_subset _, fun i => if h : i ∈ s then w ⟨i, h⟩ else 0, _,
_⟩ <;>
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
v : V
x : k
s : Set ι
p : ι → P
b : P
⊢ (∃ fs x_1 w x, v = ↑(weightedVSubOfPoint fs p b) w) ↔ ∃ fs w x, v = ↑(weightedVSubOfPoint fs (fun i => p ↑i) b) w
[PROOFSTEP]
simp_rw [weightedVSubOfPoint_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
v : V
x : k
s : Set ι
p : ι → P
b : P
⊢ (∃ fs h w h, v = ∑ i in fs, w i • (p i -ᵥ b)) ↔ ∃ fs w h, v = ∑ i in fs, w i • (p ↑i -ᵥ b)
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
v : V
x : k
s : Set ι
p : ι → P
b : P
⊢ (∃ fs h w h, v = ∑ i in fs, w i • (p i -ᵥ b)) → ∃ fs w h, v = ∑ i in fs, w i • (p ↑i -ᵥ b)
[PROOFSTEP]
rintro ⟨fs, hfs, w, rfl, rfl⟩
[GOAL]
case mp.intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Set ι
p : ι → P
b : P
fs : Finset ι
hfs : ↑fs ⊆ s
w : ι → k
⊢ ∃ fs_1 w_1 h, ∑ i in fs, w i • (p i -ᵥ b) = ∑ i in fs_1, w_1 i • (p ↑i -ᵥ b)
[PROOFSTEP]
exact ⟨fs.subtype s, fun i => w i, sum_subtype_of_mem _ hfs, (sum_subtype_of_mem _ hfs).symm⟩
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
v : V
x : k
s : Set ι
p : ι → P
b : P
⊢ (∃ fs w h, v = ∑ i in fs, w i • (p ↑i -ᵥ b)) → ∃ fs h w h, v = ∑ i in fs, w i • (p i -ᵥ b)
[PROOFSTEP]
rintro ⟨fs, w, rfl, rfl⟩
[GOAL]
case mpr.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Set ι
p : ι → P
b : P
fs : Finset ↑s
w : ↑s → k
⊢ ∃ fs_1 h w_1 h, ∑ i in fs, w i • (p ↑i -ᵥ b) = ∑ i in fs_1, w_1 i • (p i -ᵥ b)
[PROOFSTEP]
refine' ⟨fs.map (Function.Embedding.subtype _), map_subtype_subset _, fun i => if h : i ∈ s then w ⟨i, h⟩ else 0, _, _⟩
[GOAL]
case mpr.intro.intro.intro.refine'_1
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Set ι
p : ι → P
b : P
fs : Finset ↑s
w : ↑s → k
⊢ ∑ i in map (Function.Embedding.subtype fun x => x ∈ s) fs,
(fun i => if h : i ∈ s then w { val := i, property := h } else 0) i =
∑ i in fs, w i
[PROOFSTEP]
simp
[GOAL]
case mpr.intro.intro.intro.refine'_2
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Set ι
p : ι → P
b : P
fs : Finset ↑s
w : ↑s → k
⊢ ∑ i in fs, w i • (p ↑i -ᵥ b) =
∑ i in map (Function.Embedding.subtype fun x => x ∈ s) fs,
(fun i => if h : i ∈ s then w { val := i, property := h } else 0) i • (p i -ᵥ b)
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p0 : P
s : Set ι
p : ι → P
⊢ (∃ fs x w x, p0 = ↑(affineCombination k fs p) w) ↔ ∃ fs w x, p0 = ↑(affineCombination k fs fun i => p ↑i) w
[PROOFSTEP]
simp_rw [affineCombination_apply, eq_vadd_iff_vsub_eq]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝² : Ring k
inst✝¹ : AddCommGroup V
inst✝ : Module k V
S : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p0 : P
s : Set ι
p : ι → P
⊢ (∃ fs h w h,
p0 -ᵥ Classical.choice (_ : Nonempty P) = ↑(weightedVSubOfPoint fs p (Classical.choice (_ : Nonempty P))) w) ↔
∃ fs w h,
p0 -ᵥ Classical.choice (_ : Nonempty P) =
↑(weightedVSubOfPoint fs (fun i => p ↑i) (Classical.choice (_ : Nonempty P))) w
[PROOFSTEP]
exact eq_weightedVSubOfPoint_subset_iff_eq_weightedVSubOfPoint_subtype
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : Ring k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
V₂ : Type u_6
P₂ : Type u_7
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
w : ι → k
hw : Finset.sum s w = 1
f : P →ᵃ[k] P₂
⊢ ↑f (↑(affineCombination k s p) w) = ↑(affineCombination k s (↑f ∘ p)) w
[PROOFSTEP]
have b := Classical.choice (inferInstance : AffineSpace V P).Nonempty
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : Ring k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
V₂ : Type u_6
P₂ : Type u_7
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
w : ι → k
hw : Finset.sum s w = 1
f : P →ᵃ[k] P₂
b : P
⊢ ↑f (↑(affineCombination k s p) w) = ↑(affineCombination k s (↑f ∘ p)) w
[PROOFSTEP]
have b₂ := Classical.choice (inferInstance : AffineSpace V₂ P₂).Nonempty
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : Ring k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
V₂ : Type u_6
P₂ : Type u_7
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
w : ι → k
hw : Finset.sum s w = 1
f : P →ᵃ[k] P₂
b : P
b₂ : P₂
⊢ ↑f (↑(affineCombination k s p) w) = ↑(affineCombination k s (↑f ∘ p)) w
[PROOFSTEP]
rw [s.affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w p hw b,
s.affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w (f ∘ p) hw b₂, ←
s.weightedVSubOfPoint_vadd_eq_of_sum_eq_one w (f ∘ p) hw (f b) b₂]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : Ring k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
V₂ : Type u_6
P₂ : Type u_7
inst✝² : AddCommGroup V₂
inst✝¹ : Module k V₂
inst✝ : AffineSpace V₂ P₂
p : ι → P
w : ι → k
hw : Finset.sum s w = 1
f : P →ᵃ[k] P₂
b : P
b₂ : P₂
⊢ ↑f (↑(weightedVSubOfPoint s p b) w +ᵥ b) = ↑(weightedVSubOfPoint s (↑f ∘ p) (↑f b)) w +ᵥ ↑f b
[PROOFSTEP]
simp only [weightedVSubOfPoint_apply, RingHom.id_apply, AffineMap.map_vadd, LinearMap.map_smulₛₗ,
AffineMap.linearMap_vsub, LinearMap.map_sum, Function.comp_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i : ι
⊢ affineCombinationSingleWeights k i i = 1
[PROOFSTEP]
simp [affineCombinationSingleWeights]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
h : j ≠ i
⊢ affineCombinationSingleWeights k i j = 0
[PROOFSTEP]
simp [affineCombinationSingleWeights, h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i : ι
h : i ∈ s
⊢ ∑ j in s, affineCombinationSingleWeights k i j = 1
[PROOFSTEP]
rw [← affineCombinationSingleWeights_apply_self k i]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i : ι
h : i ∈ s
⊢ ∑ j in s, affineCombinationSingleWeights k i j = affineCombinationSingleWeights k i i
[PROOFSTEP]
exact sum_eq_single_of_mem i h fun j _ hj => affineCombinationSingleWeights_apply_of_ne k hj
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i : ι
⊢ weightedVSubVSubWeights k i i = 0
[PROOFSTEP]
simp [weightedVSubVSubWeights]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
h : i ≠ j
⊢ weightedVSubVSubWeights k i j i = 1
[PROOFSTEP]
simp [weightedVSubVSubWeights, h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
h : i ≠ j
⊢ weightedVSubVSubWeights k i j j = -1
[PROOFSTEP]
simp [weightedVSubVSubWeights, h.symm]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j t : ι
hi : t ≠ i
hj : t ≠ j
⊢ weightedVSubVSubWeights k i j t = 0
[PROOFSTEP]
simp [weightedVSubVSubWeights, hi, hj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
hi : i ∈ s
hj : j ∈ s
⊢ ∑ t in s, weightedVSubVSubWeights k i j t = 0
[PROOFSTEP]
simp_rw [weightedVSubVSubWeights, Pi.sub_apply, sum_sub_distrib]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
hi : i ∈ s
hj : j ∈ s
⊢ ∑ x in s, affineCombinationSingleWeights k i x - ∑ x in s, affineCombinationSingleWeights k j x = 0
[PROOFSTEP]
simp [hi, hj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i : ι
c : k
⊢ affineCombinationLineMapWeights i i c = affineCombinationSingleWeights k i
[PROOFSTEP]
simp [affineCombinationLineMapWeights]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
h : i ≠ j
c : k
⊢ affineCombinationLineMapWeights i j c i = 1 - c
[PROOFSTEP]
simp [affineCombinationLineMapWeights, h.symm, sub_eq_neg_add]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
h : i ≠ j
c : k
⊢ affineCombinationLineMapWeights i j c j = c
[PROOFSTEP]
simp [affineCombinationLineMapWeights, h.symm]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j t : ι
hi : t ≠ i
hj : t ≠ j
c : k
⊢ affineCombinationLineMapWeights i j c t = 0
[PROOFSTEP]
simp [affineCombinationLineMapWeights, hi, hj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
hi : i ∈ s
hj : j ∈ s
c : k
⊢ ∑ t in s, affineCombinationLineMapWeights i j c t = 1
[PROOFSTEP]
simp_rw [affineCombinationLineMapWeights, Pi.add_apply, sum_add_distrib]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
i j : ι
hi : i ∈ s
hj : j ∈ s
c : k
⊢ ∑ x in s, (c • weightedVSubVSubWeights k j i) x + ∑ x in s, affineCombinationSingleWeights k i x = 1
[PROOFSTEP]
simp [hi, hj, ← mul_sum]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
p : ι → P
i : ι
hi : i ∈ s
⊢ ↑(affineCombination k s p) (affineCombinationSingleWeights k i) = p i
[PROOFSTEP]
refine' s.affineCombination_of_eq_one_of_eq_zero _ _ hi (by simp) _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
p : ι → P
i : ι
hi : i ∈ s
⊢ affineCombinationSingleWeights k i i = 1
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
p : ι → P
i : ι
hi : i ∈ s
⊢ ∀ (i2 : ι), i2 ∈ s → i2 ≠ i → affineCombinationSingleWeights k i i2 = 0
[PROOFSTEP]
rintro j - hj
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
p : ι → P
i : ι
hi : i ∈ s
j : ι
hj : j ≠ i
⊢ affineCombinationSingleWeights k i j = 0
[PROOFSTEP]
simp [hj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
p : ι → P
i j : ι
hi : i ∈ s
hj : j ∈ s
⊢ ↑(weightedVSub s p) (weightedVSubVSubWeights k i j) = p i -ᵥ p j
[PROOFSTEP]
rw [weightedVSubVSubWeights, ← affineCombination_vsub, s.affineCombination_affineCombinationSingleWeights k p hi,
s.affineCombination_affineCombinationSingleWeights k p hj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
S : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : DecidableEq ι
p : ι → P
i j : ι
hi : i ∈ s
hj : j ∈ s
c : k
⊢ ↑(affineCombination k s p) (affineCombinationLineMapWeights i j c) = ↑(AffineMap.lineMap (p i) (p j)) c
[PROOFSTEP]
rw [affineCombinationLineMapWeights, ← weightedVSub_vadd_affineCombination, weightedVSub_const_smul,
s.affineCombination_affineCombinationSingleWeights k p hi, s.weightedVSub_weightedVSubVSubWeights k p hj hi,
AffineMap.lineMap_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
h : ↑(card s) ≠ 0
⊢ ∑ i in s, centroidWeights k s i = 1
[PROOFSTEP]
simp [h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : CharZero k
h : card s ≠ 0
⊢ ∑ i in s, centroidWeights k s i = 1
[PROOFSTEP]
simp only [centroidWeights_apply, sum_const, nsmul_eq_mul, ne_eq, Nat.cast_eq_zero, card_eq_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : CharZero k
h : card s ≠ 0
⊢ ↑(card s) * (↑(card s))⁻¹ = 1
[PROOFSTEP]
refine mul_inv_cancel ?_
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : CharZero k
h : card s ≠ 0
⊢ ↑(card s) ≠ 0
[PROOFSTEP]
norm_cast
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset P
⊢ centroid k univ Subtype.val = centroid k s id
[PROOFSTEP]
rw [centroid, centroid, ← s.attach_affineCombination_coe]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset P
⊢ ↑(affineCombination k univ Subtype.val) (centroidWeights k univ) =
↑(affineCombination k (attach s) Subtype.val) (centroidWeights k s ∘ Subtype.val)
[PROOFSTEP]
congr
[GOAL]
case h.e_6.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset P
⊢ centroidWeights k univ = centroidWeights k s ∘ Subtype.val
[PROOFSTEP]
ext
[GOAL]
case h.e_6.h.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s✝ : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
s : Finset P
x✝ : { x // x ∈ s }
⊢ centroidWeights k univ x✝ = (centroidWeights k s ∘ Subtype.val) x✝
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
i : ι
⊢ centroid k {i} p = p i
[PROOFSTEP]
simp [centroid_def, affineCombination_apply]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
⊢ centroid k {i₁, i₂} p = 2⁻¹ • (p i₂ -ᵥ p i₁) +ᵥ p i₁
[PROOFSTEP]
by_cases h : i₁ = i₂
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : i₁ = i₂
⊢ centroid k {i₁, i₂} p = 2⁻¹ • (p i₂ -ᵥ p i₁) +ᵥ p i₁
[PROOFSTEP]
simp [h]
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : ¬i₁ = i₂
⊢ centroid k {i₁, i₂} p = 2⁻¹ • (p i₂ -ᵥ p i₁) +ᵥ p i₁
[PROOFSTEP]
have hc : (card ({ i₁, i₂ } : Finset ι) : k) ≠ 0 :=
by
rw [card_insert_of_not_mem (not_mem_singleton.2 h), card_singleton]
norm_num
exact nonzero_of_invertible _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : ¬i₁ = i₂
⊢ ↑(card {i₁, i₂}) ≠ 0
[PROOFSTEP]
rw [card_insert_of_not_mem (not_mem_singleton.2 h), card_singleton]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : ¬i₁ = i₂
⊢ ↑(1 + 1) ≠ 0
[PROOFSTEP]
norm_num
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : ¬i₁ = i₂
⊢ ¬2 = 0
[PROOFSTEP]
exact nonzero_of_invertible _
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : ¬i₁ = i₂
hc : ↑(card {i₁, i₂}) ≠ 0
⊢ centroid k {i₁, i₂} p = 2⁻¹ • (p i₂ -ᵥ p i₁) +ᵥ p i₁
[PROOFSTEP]
rw [centroid_def,
affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one _ _ _
(sum_centroidWeights_eq_one_of_cast_card_ne_zero _ hc) (p i₁)]
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : DecidableEq ι
inst✝ : Invertible 2
p : ι → P
i₁ i₂ : ι
h : ¬i₁ = i₂
hc : ↑(card {i₁, i₂}) ≠ 0
⊢ (↑(weightedVSubOfPoint {i₁, i₂} p (p i₁)) fun i => centroidWeights k {i₁, i₂} i) +ᵥ p i₁ =
2⁻¹ • (p i₂ -ᵥ p i₁) +ᵥ p i₁
[PROOFSTEP]
simp [h, one_add_one_eq_two]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : Invertible 2
p : Fin 2 → P
⊢ centroid k univ p = 2⁻¹ • (p 1 -ᵥ p 0) +ᵥ p 0
[PROOFSTEP]
rw [univ_fin2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝ : Invertible 2
p : Fin 2 → P
⊢ centroid k {0, 1} p = 2⁻¹ • (p 1 -ᵥ p 0) +ᵥ p 0
[PROOFSTEP]
convert centroid_pair k p 0 1
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
e : ι₂ ↪ ι
p : ι → P
⊢ centroid k (map e s₂) p = centroid k s₂ (p ∘ ↑e)
[PROOFSTEP]
simp [centroid_def, affineCombination_map, centroidWeights]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : CharZero k
inst✝ : Fintype ι
h : card s ≠ 0
⊢ ∑ i : ι, centroidWeightsIndicator k s i = 1
[PROOFSTEP]
rw [sum_centroidWeightsIndicator]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : CharZero k
inst✝ : Fintype ι
h : card s ≠ 0
⊢ ∑ i in s, centroidWeights k s i = 1
[PROOFSTEP]
exact s.sum_centroidWeights_eq_one_of_card_ne_zero k h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : CharZero k
inst✝ : Fintype ι
h : Finset.Nonempty s
⊢ ∑ i : ι, centroidWeightsIndicator k s i = 1
[PROOFSTEP]
rw [sum_centroidWeightsIndicator]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : CharZero k
inst✝ : Fintype ι
h : Finset.Nonempty s
⊢ ∑ i in s, centroidWeights k s i = 1
[PROOFSTEP]
exact s.sum_centroidWeights_eq_one_of_nonempty k h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : CharZero k
inst✝ : Fintype ι
n : ℕ
h : card s = n + 1
⊢ ∑ i : ι, centroidWeightsIndicator k s i = 1
[PROOFSTEP]
rw [sum_centroidWeightsIndicator]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁵ : DivisionRing k
inst✝⁴ : AddCommGroup V
inst✝³ : Module k V
inst✝² : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
inst✝¹ : CharZero k
inst✝ : Fintype ι
n : ℕ
h : card s = n + 1
⊢ ∑ i in s, centroidWeights k s i = 1
[PROOFSTEP]
exact s.sum_centroidWeights_eq_one_of_card_eq_add_one k h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
let f : p '' ↑s → ι := fun x => x.property.choose
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
have hf : ∀ x, f x ∈ s ∧ p (f x) = x := fun x => x.property.choose_spec
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
let f' : ps → ι := fun x => f ⟨x, hps ▸ x.property⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
have hf' : ∀ x, f' x ∈ s ∧ p (f' x) = x := fun x => hf ⟨x, hps ▸ x.property⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
have hf'i : Function.Injective f' := by
intro x y h
rw [Subtype.ext_iff, ← (hf' x).2, ← (hf' y).2, h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
⊢ Function.Injective f'
[PROOFSTEP]
intro x y h
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
x y : ↑ps
h : f' x = f' y
⊢ x = y
[PROOFSTEP]
rw [Subtype.ext_iff, ← (hf' x).2, ← (hf' y).2, h]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
let f'e : ps ↪ ι := ⟨f', hf'i⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
have hu : Finset.univ.map f'e = s := by
ext x
rw [mem_map]
constructor
· rintro ⟨i, _, rfl⟩
exact (hf' i).1
· intro hx
use⟨p x, hps.symm ▸ Set.mem_image_of_mem _ hx⟩, mem_univ _
refine' hi _ (hf' _).1 _ hx _
rw [(hf' _).2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
⊢ map f'e univ = s
[PROOFSTEP]
ext x
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
⊢ x ∈ map f'e univ ↔ x ∈ s
[PROOFSTEP]
rw [mem_map]
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
⊢ (∃ a, a ∈ univ ∧ ↑f'e a = x) ↔ x ∈ s
[PROOFSTEP]
constructor
[GOAL]
case a.mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
⊢ (∃ a, a ∈ univ ∧ ↑f'e a = x) → x ∈ s
[PROOFSTEP]
rintro ⟨i, _, rfl⟩
[GOAL]
case a.mp.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
i : ↑ps
left✝ : i ∈ univ
⊢ ↑f'e i ∈ s
[PROOFSTEP]
exact (hf' i).1
[GOAL]
case a.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
⊢ x ∈ s → ∃ a, a ∈ univ ∧ ↑f'e a = x
[PROOFSTEP]
intro hx
[GOAL]
case a.mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
hx : x ∈ s
⊢ ∃ a, a ∈ univ ∧ ↑f'e a = x
[PROOFSTEP]
use⟨p x, hps.symm ▸ Set.mem_image_of_mem _ hx⟩, mem_univ _
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
hx : x ∈ s
⊢ ↑f'e { val := p x, property := (_ : p x ∈ ps) } = x
[PROOFSTEP]
refine' hi _ (hf' _).1 _ hx _
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
x : ι
hx : x ∈ s
⊢ p (f' { val := p x, property := (_ : p x ∈ ps) }) = p x
[PROOFSTEP]
rw [(hf' _).2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
hu : map f'e univ = s
⊢ centroid k s p = centroid k univ fun x => ↑x
[PROOFSTEP]
rw [← hu, centroid_map]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
hu : map f'e univ = s
⊢ centroid k univ (p ∘ ↑f'e) = centroid k univ fun x => ↑x
[PROOFSTEP]
congr with x
[GOAL]
case e_p.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
hu : map f'e univ = s
x : ↑ps
⊢ (p ∘ ↑f'e) x = ↑x
[PROOFSTEP]
change p (f' x) = ↑x
[GOAL]
case e_p.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : DivisionRing k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
ps : Set P
inst✝ : Fintype ↑ps
hps : ps = p '' ↑s
f : ↑(p '' ↑s) → ι := fun x => Exists.choose (_ : ↑x ∈ p '' ↑s)
hf : ∀ (x : ↑(p '' ↑s)), f x ∈ s ∧ p (f x) = ↑x
f' : ↑ps → ι := fun x => f { val := ↑x, property := (_ : ↑x ∈ p '' ↑s) }
hf' : ∀ (x : ↑ps), f' x ∈ s ∧ p (f' x) = ↑x
hf'i : Function.Injective f'
f'e : ↑ps ↪ ι := { toFun := f', inj' := hf'i }
hu : map f'e univ = s
x : ↑ps
⊢ p (f' x) = ↑x
[PROOFSTEP]
rw [(hf' x).2]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
p₂ : ι₂ → P
hi₂ : ∀ (i : ι₂), i ∈ s₂ → ∀ (j : ι₂), j ∈ s₂ → p₂ i = p₂ j → i = j
he : p '' ↑s = p₂ '' ↑s₂
⊢ centroid k s p = centroid k s₂ p₂
[PROOFSTEP]
classical rw [s.centroid_eq_centroid_image_of_inj_on k hi rfl, s₂.centroid_eq_centroid_image_of_inj_on k hi₂ he]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : DivisionRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
ι₂ : Type u_5
s₂ : Finset ι₂
p : ι → P
hi : ∀ (i : ι), i ∈ s → ∀ (j : ι), j ∈ s → p i = p j → i = j
p₂ : ι₂ → P
hi₂ : ∀ (i : ι₂), i ∈ s₂ → ∀ (j : ι₂), j ∈ s₂ → p₂ i = p₂ j → i = j
he : p '' ↑s = p₂ '' ↑s₂
⊢ centroid k s p = centroid k s₂ p₂
[PROOFSTEP]
rw [s.centroid_eq_centroid_image_of_inj_on k hi rfl, s₂.centroid_eq_centroid_image_of_inj_on k hi₂ he]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
⊢ ↑(Finset.weightedVSub s p) w ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
classical
rcases isEmpty_or_nonempty ι with (hι | ⟨⟨i0⟩⟩)
· simp [Finset.eq_empty_of_isEmpty s]
· rw [vectorSpan_range_eq_span_range_vsub_right k p i0, ← Set.image_univ, Finsupp.mem_span_image_iff_total,
Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s w p h (p i0), Finset.weightedVSubOfPoint_apply]
let w' := Set.indicator (↑s) w
have hwx : ∀ i, w' i ≠ 0 → i ∈ s := fun i => Set.mem_of_indicator_ne_zero
use Finsupp.onFinset s w' hwx, Set.subset_univ _
rw [Finsupp.total_apply, Finsupp.onFinset_sum hwx]
· apply Finset.sum_congr rfl
intro i hi
simp [Set.indicator_apply, if_pos hi]
· exact fun _ => zero_smul k _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
⊢ ↑(Finset.weightedVSub s p) w ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
rcases isEmpty_or_nonempty ι with (hι | ⟨⟨i0⟩⟩)
[GOAL]
case inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
hι : IsEmpty ι
⊢ ↑(Finset.weightedVSub s p) w ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
simp [Finset.eq_empty_of_isEmpty s]
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
⊢ ↑(Finset.weightedVSub s p) w ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
rw [vectorSpan_range_eq_span_range_vsub_right k p i0, ← Set.image_univ, Finsupp.mem_span_image_iff_total,
Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero s w p h (p i0), Finset.weightedVSubOfPoint_apply]
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
⊢ ∃ l,
l ∈ Finsupp.supported k k Set.univ ∧
↑(Finsupp.total ι ((fun x => V) w) k fun i => p i -ᵥ p i0) l = ∑ i in s, w i • (p i -ᵥ p i0)
[PROOFSTEP]
let w' := Set.indicator (↑s) w
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
⊢ ∃ l,
l ∈ Finsupp.supported k k Set.univ ∧
↑(Finsupp.total ι ((fun x => V) w) k fun i => p i -ᵥ p i0) l = ∑ i in s, w i • (p i -ᵥ p i0)
[PROOFSTEP]
have hwx : ∀ i, w' i ≠ 0 → i ∈ s := fun i => Set.mem_of_indicator_ne_zero
[GOAL]
case inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
hwx : ∀ (i : ι), w' i ≠ 0 → i ∈ s
⊢ ∃ l,
l ∈ Finsupp.supported k k Set.univ ∧
↑(Finsupp.total ι ((fun x => V) w) k fun i => p i -ᵥ p i0) l = ∑ i in s, w i • (p i -ᵥ p i0)
[PROOFSTEP]
use Finsupp.onFinset s w' hwx, Set.subset_univ _
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
hwx : ∀ (i : ι), w' i ≠ 0 → i ∈ s
⊢ ↑(Finsupp.total ι ((fun x => V) w) k fun i => p i -ᵥ p i0) (Finsupp.onFinset s w' hwx) = ∑ i in s, w i • (p i -ᵥ p i0)
[PROOFSTEP]
rw [Finsupp.total_apply, Finsupp.onFinset_sum hwx]
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
hwx : ∀ (i : ι), w' i ≠ 0 → i ∈ s
⊢ ∑ a in s, w' a • (p a -ᵥ p i0) = ∑ i in s, w i • (p i -ᵥ p i0)
[PROOFSTEP]
apply Finset.sum_congr rfl
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
hwx : ∀ (i : ι), w' i ≠ 0 → i ∈ s
⊢ ∀ (x : ι), x ∈ s → w' x • (p x -ᵥ p i0) = w x • (p x -ᵥ p i0)
[PROOFSTEP]
intro i hi
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
hwx : ∀ (i : ι), w' i ≠ 0 → i ∈ s
i : ι
hi : i ∈ s
⊢ w' i • (p i -ᵥ p i0) = w i • (p i -ᵥ p i0)
[PROOFSTEP]
simp [Set.indicator_apply, if_pos hi]
[GOAL]
case right
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
p : ι → P
i0 : ι
w' : ι → k := Set.indicator (↑s) w
hwx : ∀ (i : ι), w' i ≠ 0 → i ∈ s
⊢ ∀ (a : ι), 0 • (p a -ᵥ p i0) = 0
[PROOFSTEP]
exact fun _ => zero_smul k _
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
classical
have hnz : ∑ i in s, w i ≠ 0 := h.symm ▸ one_ne_zero
have hn : s.Nonempty := Finset.nonempty_of_sum_ne_zero hnz
cases' hn with i1 hi1
let w1 : ι → k := Function.update (Function.const ι 0) i1 1
have hw1 : ∑ i in s, w1 i = 1 := by
simp only [Pi.const_zero, Finset.sum_update_of_mem hi1, Pi.zero_apply, Finset.sum_const_zero, add_zero]
have hw1s : s.affineCombination k p w1 = p i1 :=
s.affineCombination_of_eq_one_of_eq_zero w1 p hi1 (Function.update_same _ _ _) fun _ _ hne =>
Function.update_noteq hne _ _
have hv : s.affineCombination k p w -ᵥ p i1 ∈ (affineSpan k (Set.range p)).direction :=
by
rw [direction_affineSpan, ← hw1s, Finset.affineCombination_vsub]
apply weightedVSub_mem_vectorSpan
change (Finset.sum s fun i => w i - w1 i) = 0
simp only [Finset.sum_sub_distrib, h, hw1, sub_self]
rw [← vsub_vadd (s.affineCombination k p w) (p i1)]
exact AffineSubspace.vadd_mem_of_mem_direction hv (mem_affineSpan k (Set.mem_range_self _))
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have hnz : ∑ i in s, w i ≠ 0 := h.symm ▸ one_ne_zero
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have hn : s.Nonempty := Finset.nonempty_of_sum_ne_zero hnz
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
hn : Finset.Nonempty s
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
cases' hn with i1 hi1
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
let w1 : ι → k := Function.update (Function.const ι 0) i1 1
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have hw1 : ∑ i in s, w1 i = 1 := by
simp only [Pi.const_zero, Finset.sum_update_of_mem hi1, Pi.zero_apply, Finset.sum_const_zero, add_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
⊢ ∑ i in s, w1 i = 1
[PROOFSTEP]
simp only [Pi.const_zero, Finset.sum_update_of_mem hi1, Pi.zero_apply, Finset.sum_const_zero, add_zero]
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have hw1s : s.affineCombination k p w1 = p i1 :=
s.affineCombination_of_eq_one_of_eq_zero w1 p hi1 (Function.update_same _ _ _) fun _ _ hne =>
Function.update_noteq hne _ _
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have hv : s.affineCombination k p w -ᵥ p i1 ∈ (affineSpan k (Set.range p)).direction :=
by
rw [direction_affineSpan, ← hw1s, Finset.affineCombination_vsub]
apply weightedVSub_mem_vectorSpan
change (Finset.sum s fun i => w i - w1 i) = 0
simp only [Finset.sum_sub_distrib, h, hw1, sub_self]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
⊢ ↑(Finset.affineCombination k s p) w -ᵥ p i1 ∈ AffineSubspace.direction (affineSpan k (Set.range p))
[PROOFSTEP]
rw [direction_affineSpan, ← hw1s, Finset.affineCombination_vsub]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
⊢ ↑(Finset.weightedVSub s p) (w - w1) ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
apply weightedVSub_mem_vectorSpan
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
⊢ ∑ i in s, (w - w1) i = 0
[PROOFSTEP]
change (Finset.sum s fun i => w i - w1 i) = 0
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
⊢ ∑ i in s, (w i - w1 i) = 0
[PROOFSTEP]
simp only [Finset.sum_sub_distrib, h, hw1, sub_self]
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
hv : ↑(Finset.affineCombination k s p) w -ᵥ p i1 ∈ AffineSubspace.direction (affineSpan k (Set.range p))
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
rw [← vsub_vadd (s.affineCombination k p w) (p i1)]
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 1
p : ι → P
hnz : ∑ i in s, w i ≠ 0
i1 : ι
hi1 : i1 ∈ s
w1 : ι → k := Function.update (Function.const ι 0) i1 1
hw1 : ∑ i in s, w1 i = 1
hw1s : ↑(Finset.affineCombination k s p) w1 = p i1
hv : ↑(Finset.affineCombination k s p) w -ᵥ p i1 ∈ AffineSubspace.direction (affineSpan k (Set.range p))
⊢ ↑(Finset.affineCombination k s p) w -ᵥ p i1 +ᵥ p i1 ∈ affineSpan k (Set.range p)
[PROOFSTEP]
exact AffineSubspace.vadd_mem_of_mem_direction hv (mem_affineSpan k (Set.mem_range_self _))
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
⊢ v ∈ vectorSpan k (Set.range p) ↔ ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
classical
constructor
· rcases isEmpty_or_nonempty ι with (hι | ⟨⟨i0⟩⟩)
swap
· rw [vectorSpan_range_eq_span_range_vsub_right k p i0, ← Set.image_univ, Finsupp.mem_span_image_iff_total]
rintro ⟨l, _, hv⟩
use insert i0 l.support
set w := (l : ι → k) - Function.update (Function.const ι 0 : ι → k) i0 (∑ i in l.support, l i) with hwdef
use w
have hw : ∑ i in insert i0 l.support, w i = 0 := by
rw [hwdef]
simp_rw [Pi.sub_apply, Finset.sum_sub_distrib, Finset.sum_update_of_mem (Finset.mem_insert_self _ _),
Finset.sum_insert_of_eq_zero_if_not_mem Finsupp.not_mem_support_iff.1]
simp only [Finsupp.mem_support_iff, ne_eq, Finset.mem_insert, true_or, not_true, Function.const_apply,
Finset.sum_const_zero, add_zero, sub_self]
use hw
have hz : w i0 • (p i0 -ᵥ p i0 : V) = 0 := (vsub_self (p i0)).symm ▸ smul_zero _
change (fun i => w i • (p i -ᵥ p i0 : V)) i0 = 0 at hz
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero _ w p hw (p i0), Finset.weightedVSubOfPoint_apply, ←
hv, Finsupp.total_apply, @Finset.sum_insert_zero _ _ l.support i0 _ _ _ hz]
change (∑ i in l.support, l i • _) = _
congr with i
by_cases h : i = i0
· simp [h]
· simp [hwdef, h]
· rw [Set.range_eq_empty, vectorSpan_empty, Submodule.mem_bot]
rintro rfl
use∅
simp
· rintro ⟨s, w, hw, rfl⟩
exact weightedVSub_mem_vectorSpan hw p
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
⊢ v ∈ vectorSpan k (Set.range p) ↔ ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
⊢ v ∈ vectorSpan k (Set.range p) → ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rcases isEmpty_or_nonempty ι with (hι | ⟨⟨i0⟩⟩)
[GOAL]
case mp.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
hι : IsEmpty ι
⊢ v ∈ vectorSpan k (Set.range p) → ∃ s w x, v = ↑(Finset.weightedVSub s p) w
case mp.inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
⊢ v ∈ vectorSpan k (Set.range p) → ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
swap
[GOAL]
case mp.inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
⊢ v ∈ vectorSpan k (Set.range p) → ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rw [vectorSpan_range_eq_span_range_vsub_right k p i0, ← Set.image_univ, Finsupp.mem_span_image_iff_total]
[GOAL]
case mp.inr.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
⊢ (∃ l, l ∈ Finsupp.supported k k Set.univ ∧ ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v) →
∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rintro ⟨l, _, hv⟩
[GOAL]
case mp.inr.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
⊢ ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
use insert i0 l.support
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
⊢ ∃ w x, v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
set w := (l : ι → k) - Function.update (Function.const ι 0 : ι → k) i0 (∑ i in l.support, l i) with hwdef
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
⊢ ∃ w x, v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
use w
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
⊢ ∃ x, v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
have hw : ∑ i in insert i0 l.support, w i = 0 := by
rw [hwdef]
simp_rw [Pi.sub_apply, Finset.sum_sub_distrib, Finset.sum_update_of_mem (Finset.mem_insert_self _ _),
Finset.sum_insert_of_eq_zero_if_not_mem Finsupp.not_mem_support_iff.1]
simp only [Finsupp.mem_support_iff, ne_eq, Finset.mem_insert, true_or, not_true, Function.const_apply,
Finset.sum_const_zero, add_zero, sub_self]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
⊢ ∑ i in insert i0 l.support, w i = 0
[PROOFSTEP]
rw [hwdef]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
⊢ ∑ i in insert i0 l.support, (↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)) i = 0
[PROOFSTEP]
simp_rw [Pi.sub_apply, Finset.sum_sub_distrib, Finset.sum_update_of_mem (Finset.mem_insert_self _ _),
Finset.sum_insert_of_eq_zero_if_not_mem Finsupp.not_mem_support_iff.1]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
⊢ ∑ x in l.support, ↑l x - (∑ x in l.support, ↑l x + ∑ x in insert i0 l.support \ {i0}, Function.const ι 0 x) = 0
[PROOFSTEP]
simp only [Finsupp.mem_support_iff, ne_eq, Finset.mem_insert, true_or, not_true, Function.const_apply,
Finset.sum_const_zero, add_zero, sub_self]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
⊢ ∃ x, v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
use hw
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
⊢ v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
have hz : w i0 • (p i0 -ᵥ p i0 : V) = 0 := (vsub_self (p i0)).symm ▸ smul_zero _
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : w i0 • (p i0 -ᵥ p i0) = 0
⊢ v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
change (fun i => w i • (p i -ᵥ p i0 : V)) i0 = 0 at hz
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : (fun i => w i • (p i -ᵥ p i0)) i0 = 0
⊢ v = ↑(Finset.weightedVSub (insert i0 l.support) p) w
[PROOFSTEP]
rw [Finset.weightedVSub_eq_weightedVSubOfPoint_of_sum_eq_zero _ w p hw (p i0), Finset.weightedVSubOfPoint_apply, ← hv,
Finsupp.total_apply, @Finset.sum_insert_zero _ _ l.support i0 _ _ _ hz]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : (fun i => w i • (p i -ᵥ p i0)) i0 = 0
⊢ (Finsupp.sum l fun i a => a • (p i -ᵥ p i0)) = ∑ x in l.support, w x • (p x -ᵥ p i0)
[PROOFSTEP]
change (∑ i in l.support, l i • _) = _
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : (fun i => w i • (p i -ᵥ p i0)) i0 = 0
⊢ ∑ i in l.support, ↑l i • (p i -ᵥ p i0) = ∑ x in l.support, w x • (p x -ᵥ p i0)
[PROOFSTEP]
congr with i
[GOAL]
case h.e_f.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : (fun i => w i • (p i -ᵥ p i0)) i0 = 0
i : ι
⊢ ↑l i • (p i -ᵥ p i0) = w i • (p i -ᵥ p i0)
[PROOFSTEP]
by_cases h : i = i0
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : (fun i => w i • (p i -ᵥ p i0)) i0 = 0
i : ι
h : i = i0
⊢ ↑l i • (p i -ᵥ p i0) = w i • (p i -ᵥ p i0)
[PROOFSTEP]
simp [h]
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
i0 : ι
l : ι →₀ k
left✝ : l ∈ Finsupp.supported k k Set.univ
hv : ↑(Finsupp.total ι V k fun i => p i -ᵥ p i0) l = v
w : (a : ι) → (fun x => k) a := ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hwdef : w = ↑l - Function.update (Function.const ι 0) i0 (∑ i in l.support, ↑l i)
hw : ∑ i in insert i0 l.support, w i = 0
hz : (fun i => w i • (p i -ᵥ p i0)) i0 = 0
i : ι
h : ¬i = i0
⊢ ↑l i • (p i -ᵥ p i0) = w i • (p i -ᵥ p i0)
[PROOFSTEP]
simp [hwdef, h]
[GOAL]
case mp.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
hι : IsEmpty ι
⊢ v ∈ vectorSpan k (Set.range p) → ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rw [Set.range_eq_empty, vectorSpan_empty, Submodule.mem_bot]
[GOAL]
case mp.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
hι : IsEmpty ι
⊢ v = 0 → ∃ s w x, v = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
rintro rfl
[GOAL]
case mp.inl
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
hι : IsEmpty ι
⊢ ∃ s w x, 0 = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
use∅
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
hι : IsEmpty ι
⊢ ∃ w x, 0 = ↑(Finset.weightedVSub ∅ p) w
[PROOFSTEP]
simp
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
v : V
p : ι → P
⊢ (∃ s w x, v = ↑(Finset.weightedVSub s p) w) → v ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
rintro ⟨s, w, hw, rfl⟩
[GOAL]
case mpr.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 0
⊢ ↑(Finset.weightedVSub s p) w ∈ vectorSpan k (Set.range p)
[PROOFSTEP]
exact weightedVSub_mem_vectorSpan hw p
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
classical
have hn : (affineSpan k (Set.range p) : Set P).Nonempty := ⟨p1, h⟩
rw [affineSpan_nonempty, Set.range_nonempty_iff_nonempty] at hn
cases' hn with i0
have h0 : p i0 ∈ affineSpan k (Set.range p) := mem_affineSpan k (Set.mem_range_self i0)
have hd : p1 -ᵥ p i0 ∈ (affineSpan k (Set.range p)).direction := AffineSubspace.vsub_mem_direction h h0
rw [direction_affineSpan, mem_vectorSpan_iff_eq_weightedVSub] at hd
rcases hd with ⟨s, w, h, hs⟩
let s' := insert i0 s
let w' := Set.indicator (↑s) w
have h' : ∑ i in s', w' i = 0 := by rw [← h, Set.sum_indicator_subset _ (Finset.subset_insert i0 s)]
have hs' : s'.weightedVSub p w' = p1 -ᵥ p i0 := by
rw [hs]
exact (Finset.weightedVSub_indicator_subset _ _ (Finset.subset_insert i0 s)).symm
let w0 : ι → k := Function.update (Function.const ι 0) i0 1
have hw0 : ∑ i in s', w0 i = 1 :=
by
rw [Finset.sum_update_of_mem (Finset.mem_insert_self _ _)]
simp only [Finset.mem_insert, true_or, not_true, Function.const_apply, Finset.sum_const_zero, add_zero]
have hw0s : s'.affineCombination k p w0 = p i0 :=
s'.affineCombination_of_eq_one_of_eq_zero w0 p (Finset.mem_insert_self _ _) (Function.update_same _ _ _)
fun _ _ hne => Function.update_noteq hne _ _
use s', w0 + w'
constructor
· rw [add_comm, ← Finset.weightedVSub_vadd_affineCombination, hw0s, hs', vsub_vadd]
·
-- Porting note: proof was `simp [Pi.add_apply, Finset.sum_add_distrib, hw0, h']`
change (Finset.sum s' fun i => w0 i + w' i) = 1
simp only [Finset.sum_add_distrib, hw0, h', add_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have hn : (affineSpan k (Set.range p) : Set P).Nonempty := ⟨p1, h⟩
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
hn : Set.Nonempty ↑(affineSpan k (Set.range p))
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
rw [affineSpan_nonempty, Set.range_nonempty_iff_nonempty] at hn
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
hn : Nonempty ι
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
cases' hn with i0
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
i0 : ι
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have h0 : p i0 ∈ affineSpan k (Set.range p) := mem_affineSpan k (Set.mem_range_self i0)
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have hd : p1 -ᵥ p i0 ∈ (affineSpan k (Set.range p)).direction := AffineSubspace.vsub_mem_direction h h0
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
hd : p1 -ᵥ p i0 ∈ AffineSubspace.direction (affineSpan k (Set.range p))
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
rw [direction_affineSpan, mem_vectorSpan_iff_eq_weightedVSub] at hd
[GOAL]
case intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
hd : ∃ s w x, p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
rcases hd with ⟨s, w, h, hs⟩
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
let s' := insert i0 s
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
let w' := Set.indicator (↑s) w
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have h' : ∑ i in s', w' i = 0 := by rw [← h, Set.sum_indicator_subset _ (Finset.subset_insert i0 s)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
⊢ ∑ i in s', w' i = 0
[PROOFSTEP]
rw [← h, Set.sum_indicator_subset _ (Finset.subset_insert i0 s)]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have hs' : s'.weightedVSub p w' = p1 -ᵥ p i0 := by
rw [hs]
exact (Finset.weightedVSub_indicator_subset _ _ (Finset.subset_insert i0 s)).symm
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
⊢ ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
[PROOFSTEP]
rw [hs]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
⊢ ↑(Finset.weightedVSub s' p) w' = ↑(Finset.weightedVSub s p) w
[PROOFSTEP]
exact (Finset.weightedVSub_indicator_subset _ _ (Finset.subset_insert i0 s)).symm
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
let w0 : ι → k := Function.update (Function.const ι 0) i0 1
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have hw0 : ∑ i in s', w0 i = 1 :=
by
rw [Finset.sum_update_of_mem (Finset.mem_insert_self _ _)]
simp only [Finset.mem_insert, true_or, not_true, Function.const_apply, Finset.sum_const_zero, add_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
⊢ ∑ i in s', w0 i = 1
[PROOFSTEP]
rw [Finset.sum_update_of_mem (Finset.mem_insert_self _ _)]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
⊢ 1 + ∑ x in insert i0 s \ {i0}, Function.const ι 0 x = 1
[PROOFSTEP]
simp only [Finset.mem_insert, true_or, not_true, Function.const_apply, Finset.sum_const_zero, add_zero]
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
hw0 : ∑ i in s', w0 i = 1
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
have hw0s : s'.affineCombination k p w0 = p i0 :=
s'.affineCombination_of_eq_one_of_eq_zero w0 p (Finset.mem_insert_self _ _) (Function.update_same _ _ _)
fun _ _ hne => Function.update_noteq hne _ _
[GOAL]
case intro.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
hw0 : ∑ i in s', w0 i = 1
hw0s : ↑(Finset.affineCombination k s' p) w0 = p i0
⊢ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
use s', w0 + w'
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
hw0 : ∑ i in s', w0 i = 1
hw0s : ↑(Finset.affineCombination k s' p) w0 = p i0
⊢ ∃ x, p1 = ↑(Finset.affineCombination k s' p) (w0 + w')
[PROOFSTEP]
constructor
[GOAL]
case h.h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
hw0 : ∑ i in s', w0 i = 1
hw0s : ↑(Finset.affineCombination k s' p) w0 = p i0
⊢ p1 = ↑(Finset.affineCombination k s' p) (w0 + w')
[PROOFSTEP]
rw [add_comm, ← Finset.weightedVSub_vadd_affineCombination, hw0s, hs', vsub_vadd]
[GOAL]
case h.w
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
hw0 : ∑ i in s', w0 i = 1
hw0s : ↑(Finset.affineCombination k s' p) w0 = p i0
⊢ ∑ i in s', (w0 + w') i = 1
[PROOFSTEP]
change (Finset.sum s' fun i => w0 i + w' i) = 1
[GOAL]
case h.w
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : Ring k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
p1 : P
p : ι → P
h✝ : p1 ∈ affineSpan k (Set.range p)
i0 : ι
h0 : p i0 ∈ affineSpan k (Set.range p)
s : Finset ι
w : ι → k
h : ∑ i in s, w i = 0
hs : p1 -ᵥ p i0 = ↑(Finset.weightedVSub s p) w
s' : Finset ι := insert i0 s
w' : ι → k := Set.indicator (↑s) w
h' : ∑ i in s', w' i = 0
hs' : ↑(Finset.weightedVSub s' p) w' = p1 -ᵥ p i0
w0 : ι → k := Function.update (Function.const ι 0) i0 1
hw0 : ∑ i in s', w0 i = 1
hw0s : ↑(Finset.affineCombination k s' p) w0 = p i0
⊢ ∑ i in s', (w0 i + w' i) = 1
[PROOFSTEP]
simp only [Finset.sum_add_distrib, hw0, h', add_zero]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
⊢ ∃ w x, p1 = ↑(Finset.affineCombination k Finset.univ p) w
[PROOFSTEP]
classical
obtain ⟨s, w, hw, rfl⟩ := eq_affineCombination_of_mem_affineSpan h
refine' ⟨(s : Set ι).indicator w, _, Finset.affineCombination_indicator_subset w p s.subset_univ⟩
simp only [Finset.mem_coe, Set.indicator_apply, ← hw]
rw [Fintype.sum_extend_by_zero s w]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p1 : P
p : ι → P
h : p1 ∈ affineSpan k (Set.range p)
⊢ ∃ w x, p1 = ↑(Finset.affineCombination k Finset.univ p) w
[PROOFSTEP]
obtain ⟨s, w, hw, rfl⟩ := eq_affineCombination_of_mem_affineSpan h
[GOAL]
case intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 1
h : ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
⊢ ∃ w_1 x, ↑(Finset.affineCombination k s p) w = ↑(Finset.affineCombination k Finset.univ p) w_1
[PROOFSTEP]
refine' ⟨(s : Set ι).indicator w, _, Finset.affineCombination_indicator_subset w p s.subset_univ⟩
[GOAL]
case intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 1
h : ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
⊢ ∑ i : ι, Set.indicator (↑s) w i = 1
[PROOFSTEP]
simp only [Finset.mem_coe, Set.indicator_apply, ← hw]
[GOAL]
case intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Fintype ι
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 1
h : ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
⊢ (∑ x : ι, if x ∈ s then w x else 0) = ∑ i in s, w i
[PROOFSTEP]
rw [Fintype.sum_extend_by_zero s w]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p1 : P
p : ι → P
⊢ p1 ∈ affineSpan k (Set.range p) ↔ ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p1 : P
p : ι → P
⊢ p1 ∈ affineSpan k (Set.range p) → ∃ s w x, p1 = ↑(Finset.affineCombination k s p) w
[PROOFSTEP]
exact eq_affineCombination_of_mem_affineSpan
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p1 : P
p : ι → P
⊢ (∃ s w x, p1 = ↑(Finset.affineCombination k s p) w) → p1 ∈ affineSpan k (Set.range p)
[PROOFSTEP]
rintro ⟨s, w, hw, rfl⟩
[GOAL]
case mpr.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 1
⊢ ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
[PROOFSTEP]
exact affineCombination_mem_affineSpan hw p
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
q : P
⊢ q ∈ affineSpan k (Set.range p) ↔ ∃ s w, q = ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j
[PROOFSTEP]
constructor
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
q : P
⊢ q ∈ affineSpan k (Set.range p) → ∃ s w, q = ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j
[PROOFSTEP]
intro hq
[GOAL]
case mp
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
q : P
hq : q ∈ affineSpan k (Set.range p)
⊢ ∃ s w, q = ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j
[PROOFSTEP]
obtain ⟨s, w, hw, rfl⟩ := eq_affineCombination_of_mem_affineSpan hq
[GOAL]
case mp.intro.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
hw : ∑ i in s, w i = 1
hq : ↑(Finset.affineCombination k s p) w ∈ affineSpan k (Set.range p)
⊢ ∃ s_1 w_1, ↑(Finset.affineCombination k s p) w = ↑(Finset.weightedVSubOfPoint s_1 p (p j)) w_1 +ᵥ p j
[PROOFSTEP]
exact ⟨s, w, s.affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w p hw (p j)⟩
[GOAL]
case mpr
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
q : P
⊢ (∃ s w, q = ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j) → q ∈ affineSpan k (Set.range p)
[PROOFSTEP]
rintro ⟨s, w, rfl⟩
[GOAL]
case mpr.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
⊢ ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j ∈ affineSpan k (Set.range p)
[PROOFSTEP]
classical
let w' : ι → k := Function.update w j (1 - (s \ { j }).sum w)
have h₁ : (insert j s).sum w' = 1 := by
by_cases hj : j ∈ s
· simp [Finset.sum_update_of_mem hj, Finset.insert_eq_of_mem hj]
· simp [Finset.sum_insert hj, Finset.sum_update_of_not_mem hj, hj]
have hww : ∀ i, i ≠ j → w i = w' i := by
intro i hij
simp [hij]
rw [s.weightedVSubOfPoint_eq_of_weights_eq p j w w' hww, ← s.weightedVSubOfPoint_insert w' p j, ←
(insert j s).affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w' p h₁ (p j)]
exact affineCombination_mem_affineSpan h₁ p
[GOAL]
case mpr.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
⊢ ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j ∈ affineSpan k (Set.range p)
[PROOFSTEP]
let w' : ι → k := Function.update w j (1 - (s \ { j }).sum w)
[GOAL]
case mpr.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
⊢ ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have h₁ : (insert j s).sum w' = 1 := by
by_cases hj : j ∈ s
· simp [Finset.sum_update_of_mem hj, Finset.insert_eq_of_mem hj]
· simp [Finset.sum_insert hj, Finset.sum_update_of_not_mem hj, hj]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
⊢ Finset.sum (insert j s) w' = 1
[PROOFSTEP]
by_cases hj : j ∈ s
[GOAL]
case pos
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
hj : j ∈ s
⊢ Finset.sum (insert j s) w' = 1
[PROOFSTEP]
simp [Finset.sum_update_of_mem hj, Finset.insert_eq_of_mem hj]
[GOAL]
case neg
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
hj : ¬j ∈ s
⊢ Finset.sum (insert j s) w' = 1
[PROOFSTEP]
simp [Finset.sum_insert hj, Finset.sum_update_of_not_mem hj, hj]
[GOAL]
case mpr.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
h₁ : Finset.sum (insert j s) w' = 1
⊢ ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j ∈ affineSpan k (Set.range p)
[PROOFSTEP]
have hww : ∀ i, i ≠ j → w i = w' i := by
intro i hij
simp [hij]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
h₁ : Finset.sum (insert j s) w' = 1
⊢ ∀ (i : ι), i ≠ j → w i = w' i
[PROOFSTEP]
intro i hij
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
h₁ : Finset.sum (insert j s) w' = 1
i : ι
hij : i ≠ j
⊢ w i = w' i
[PROOFSTEP]
simp [hij]
[GOAL]
case mpr.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
h₁ : Finset.sum (insert j s) w' = 1
hww : ∀ (i : ι), i ≠ j → w i = w' i
⊢ ↑(Finset.weightedVSubOfPoint s p (p j)) w +ᵥ p j ∈ affineSpan k (Set.range p)
[PROOFSTEP]
rw [s.weightedVSubOfPoint_eq_of_weights_eq p j w w' hww, ← s.weightedVSubOfPoint_insert w' p j, ←
(insert j s).affineCombination_eq_weightedVSubOfPoint_vadd_of_sum_eq_one w' p h₁ (p j)]
[GOAL]
case mpr.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
ι : Type u_4
inst✝ : Nontrivial k
p : ι → P
j : ι
s : Finset ι
w : ι → k
w' : ι → k := Function.update w j (1 - Finset.sum (s \ {j}) w)
h₁ : Finset.sum (insert j s) w' = 1
hww : ∀ (i : ι), i ≠ j → w i = w' i
⊢ ↑(Finset.affineCombination k (insert j s) p) w' ∈ affineSpan k (Set.range p)
[PROOFSTEP]
exact affineCombination_mem_affineSpan h₁ p
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
⊢ affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)) = affineSpan k s
[PROOFSTEP]
have : s = Set.range ((↑) : s → P) := by simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
⊢ s = Set.range Subtype.val
[PROOFSTEP]
simp
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
⊢ affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)) = affineSpan k s
[PROOFSTEP]
conv_rhs => rw [this]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
| affineSpan k s
[PROOFSTEP]
rw [this]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
| affineSpan k s
[PROOFSTEP]
rw [this]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
| affineSpan k s
[PROOFSTEP]
rw [this]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
⊢ affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)) = affineSpan k (Set.range Subtype.val)
[PROOFSTEP]
apply le_antisymm <;> intro q hq <;>
erw [mem_affineSpan_iff_eq_weightedVSubOfPoint_vadd k V _ (⟨p, hp⟩ : s) q] at hq ⊢ <;>
obtain ⟨t, μ, rfl⟩ := hq <;>
use t <;>
[use fun x => μ x * ↑(w x); use fun x => μ x * ↑(w x)⁻¹]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
⊢ affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)) = affineSpan k (Set.range Subtype.val)
[PROOFSTEP]
apply le_antisymm
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
⊢ affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)) ≤ affineSpan k (Set.range Subtype.val)
[PROOFSTEP]
intro q hq
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
⊢ affineSpan k (Set.range Subtype.val) ≤ affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
[PROOFSTEP]
intro q hq
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
q : P
hq : q ∈ ↑(affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)))
⊢ q ∈ ↑(affineSpan k (Set.range Subtype.val))
[PROOFSTEP]
erw [mem_affineSpan_iff_eq_weightedVSubOfPoint_vadd k V _ (⟨p, hp⟩ : s) q] at hq ⊢
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
q : P
hq : q ∈ ↑(affineSpan k (Set.range Subtype.val))
⊢ q ∈ ↑(affineSpan k (Set.range fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q)))
[PROOFSTEP]
erw [mem_affineSpan_iff_eq_weightedVSubOfPoint_vadd k V _ (⟨p, hp⟩ : s) q] at hq ⊢
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
q : P
hq :
∃ s_1 w_1,
q =
↑(Finset.weightedVSubOfPoint s_1 (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
w_1 +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })
⊢ ∃ s_1 w,
q = ↑(Finset.weightedVSubOfPoint s_1 Subtype.val ↑{ val := p, property := hp }) w +ᵥ ↑{ val := p, property := hp }
[PROOFSTEP]
obtain ⟨t, μ, rfl⟩ := hq
[GOAL]
case a
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
q : P
hq :
∃ s_1 w,
q = ↑(Finset.weightedVSubOfPoint s_1 Subtype.val ↑{ val := p, property := hp }) w +ᵥ ↑{ val := p, property := hp }
⊢ ∃ s_1 w_1,
q =
↑(Finset.weightedVSubOfPoint s_1 (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
w_1 +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })
[PROOFSTEP]
obtain ⟨t, μ, rfl⟩ := hq
[GOAL]
case a.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
t : Finset { x // x ∈ s }
μ : { x // x ∈ s } → k
⊢ ∃ s_1 w_1,
↑(Finset.weightedVSubOfPoint t (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
μ +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp }) =
↑(Finset.weightedVSubOfPoint s_1 Subtype.val ↑{ val := p, property := hp }) w_1 +ᵥ ↑{ val := p, property := hp }
[PROOFSTEP]
use t
[GOAL]
case a.intro.intro
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
t : Finset { x // x ∈ s }
μ : { x // x ∈ s } → k
⊢ ∃ s_1 w_1,
↑(Finset.weightedVSubOfPoint t Subtype.val ↑{ val := p, property := hp }) μ +ᵥ ↑{ val := p, property := hp } =
↑(Finset.weightedVSubOfPoint s_1 (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
w_1 +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })
[PROOFSTEP]
use t
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
t : Finset { x // x ∈ s }
μ : { x // x ∈ s } → k
⊢ ∃ w_1,
↑(Finset.weightedVSubOfPoint t (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
μ +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp }) =
↑(Finset.weightedVSubOfPoint t Subtype.val ↑{ val := p, property := hp }) w_1 +ᵥ ↑{ val := p, property := hp }
[PROOFSTEP]
use fun x => μ x * ↑(w x)
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
t : Finset { x // x ∈ s }
μ : { x // x ∈ s } → k
⊢ ∃ w_1,
↑(Finset.weightedVSubOfPoint t Subtype.val ↑{ val := p, property := hp }) μ +ᵥ ↑{ val := p, property := hp } =
↑(Finset.weightedVSubOfPoint t (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
w_1 +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })
[PROOFSTEP]
use fun x => μ x * ↑(w x)⁻¹
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
t : Finset { x // x ∈ s }
μ : { x // x ∈ s } → k
⊢ ↑(Finset.weightedVSubOfPoint t (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
μ +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp }) =
(↑(Finset.weightedVSubOfPoint t Subtype.val ↑{ val := p, property := hp }) fun x => μ x * ↑(w x)) +ᵥ
↑{ val := p, property := hp }
[PROOFSTEP]
simp [smul_smul]
[GOAL]
case h
k : Type u_1
V : Type u_2
P : Type u_3
inst✝⁴ : Ring k
inst✝³ : AddCommGroup V
inst✝² : Module k V
inst✝¹ : AffineSpace V P
inst✝ : Nontrivial k
s : Set P
p : P
hp : p ∈ s
w : ↑s → kˣ
this : s = Set.range Subtype.val
t : Finset { x // x ∈ s }
μ : { x // x ∈ s } → k
⊢ ↑(Finset.weightedVSubOfPoint t Subtype.val ↑{ val := p, property := hp }) μ +ᵥ ↑{ val := p, property := hp } =
(↑(Finset.weightedVSubOfPoint t (fun q => ↑(AffineMap.lineMap p ↑q) ↑(w q))
(↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })))
fun x => μ x * ↑(w x)⁻¹) +ᵥ
↑(AffineMap.lineMap p ↑{ val := p, property := hp }) ↑(w { val := p, property := hp })
[PROOFSTEP]
simp [smul_smul]
[GOAL]
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : CommRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
⊢ ∀ (p : (ι → P) × P) (v : (ι → V) × V),
(fun p => ↑(Finset.weightedVSubOfPoint s p.fst p.snd) w) (v +ᵥ p) =
↑(∑ i in s, w i • (LinearMap.comp (LinearMap.proj i) (LinearMap.fst k (ι → V) V) - LinearMap.snd k (ι → V) V))
v +ᵥ
(fun p => ↑(Finset.weightedVSubOfPoint s p.fst p.snd) w) p
[PROOFSTEP]
rintro ⟨p, b⟩
⟨v, b'⟩
-- Porting note: needed to give `Prod.mk_vadd_mk` a hint
[GOAL]
case mk.mk
k : Type u_1
V : Type u_2
P : Type u_3
inst✝³ : CommRing k
inst✝² : AddCommGroup V
inst✝¹ : Module k V
inst✝ : AffineSpace V P
ι : Type u_4
s : Finset ι
w : ι → k
p : ι → P
b : P
v : ι → V
b' : V
⊢ (fun p => ↑(Finset.weightedVSubOfPoint s p.fst p.snd) w) ((v, b') +ᵥ (p, b)) =
↑(∑ i in s, w i • (LinearMap.comp (LinearMap.proj i) (LinearMap.fst k (ι → V) V) - LinearMap.snd k (ι → V) V))
(v, b') +ᵥ
(fun p => ↑(Finset.weightedVSubOfPoint s p.fst p.snd) w) (p, b)
[PROOFSTEP]
simp [LinearMap.sum_apply, Finset.weightedVSubOfPoint, vsub_vadd_eq_vsub_sub, vadd_vsub_assoc, add_sub, ←
sub_add_eq_add_sub, smul_add, Finset.sum_add_distrib, Prod.mk_vadd_mk v]
| {"mathlib_filename": "Mathlib.LinearAlgebra.AffineSpace.Combination", "llama_tokens": 81666} |
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ eigenvectorMatrix hA * eigenvectorMatrixInv hA = 1
[PROOFSTEP]
apply Basis.toMatrix_mul_toMatrix_flip
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
⊢ eigenvectorMatrix hA i j = ↑(eigenvectorBasis hA) j i
[PROOFSTEP]
simp_rw [eigenvectorMatrix, Basis.toMatrix_apply, OrthonormalBasis.coe_toBasis, PiLp.basisFun_repr]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
⊢ eigenvectorMatrixInv hA i j = star (↑(eigenvectorBasis hA) i j)
[PROOFSTEP]
rw [eigenvectorMatrixInv, Basis.toMatrix_apply, OrthonormalBasis.coe_toBasis_repr_apply,
OrthonormalBasis.repr_apply_apply, PiLp.basisFun_apply, PiLp.equiv_symm_single, EuclideanSpace.inner_single_right,
one_mul, IsROrC.star_def]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ (eigenvectorMatrixInv hA)ᴴ = eigenvectorMatrix hA
[PROOFSTEP]
ext i j
[GOAL]
case a.h
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
⊢ (eigenvectorMatrixInv hA)ᴴ i j = eigenvectorMatrix hA i j
[PROOFSTEP]
rw [conjTranspose_apply, eigenvectorMatrixInv_apply, eigenvectorMatrix_apply, star_star]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ (eigenvectorMatrix hA)ᴴ = eigenvectorMatrixInv hA
[PROOFSTEP]
rw [← conjTranspose_eigenvectorMatrixInv, conjTranspose_conjTranspose]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ eigenvectorMatrixInv hA * A = diagonal (IsROrC.ofReal ∘ eigenvalues hA) * eigenvectorMatrixInv hA
[PROOFSTEP]
rw [eigenvectorMatrixInv, PiLp.basis_toMatrix_basisFun_mul]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ (↑of fun i j =>
↑(↑(OrthonormalBasis.toBasis (eigenvectorBasis hA)).repr (↑(PiLp.equiv 2 fun i => 𝕜).symm (Aᵀ j))) i) =
diagonal (IsROrC.ofReal ∘ eigenvalues hA) *
Basis.toMatrix (OrthonormalBasis.toBasis (eigenvectorBasis hA)) ↑(PiLp.basisFun 2 𝕜 n)
[PROOFSTEP]
ext i j
[GOAL]
case a.h
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
⊢ ↑of (fun i j => ↑(↑(OrthonormalBasis.toBasis (eigenvectorBasis hA)).repr (↑(PiLp.equiv 2 fun i => 𝕜).symm (Aᵀ j))) i)
i j =
(diagonal (IsROrC.ofReal ∘ eigenvalues hA) *
Basis.toMatrix (OrthonormalBasis.toBasis (eigenvectorBasis hA)) ↑(PiLp.basisFun 2 𝕜 n))
i j
[PROOFSTEP]
have := isHermitian_iff_isSymmetric.1 hA
[GOAL]
case a.h
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
this : LinearMap.IsSymmetric (↑toEuclideanLin A)
⊢ ↑of (fun i j => ↑(↑(OrthonormalBasis.toBasis (eigenvectorBasis hA)).repr (↑(PiLp.equiv 2 fun i => 𝕜).symm (Aᵀ j))) i)
i j =
(diagonal (IsROrC.ofReal ∘ eigenvalues hA) *
Basis.toMatrix (OrthonormalBasis.toBasis (eigenvectorBasis hA)) ↑(PiLp.basisFun 2 𝕜 n))
i j
[PROOFSTEP]
convert
this.eigenvectorBasis_apply_self_apply finrank_euclideanSpace (EuclideanSpace.single j 1)
((Fintype.equivOfCardEq (Fintype.card_fin _)).symm i) using
1
[GOAL]
case h.e'_2
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
this : LinearMap.IsSymmetric (↑toEuclideanLin A)
⊢ ↑of (fun i j => ↑(↑(OrthonormalBasis.toBasis (eigenvectorBasis hA)).repr (↑(PiLp.equiv 2 fun i => 𝕜).symm (Aᵀ j))) i)
i j =
↑(LinearMap.IsSymmetric.eigenvectorBasis this
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)).repr
(↑(↑toEuclideanLin A) (EuclideanSpace.single j 1))
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)
[PROOFSTEP]
dsimp only [EuclideanSpace.single, toEuclideanLin_piLp_equiv_symm, toLin'_apply, Matrix.of_apply,
IsHermitian.eigenvectorBasis]
[GOAL]
case h.e'_2
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
this : LinearMap.IsSymmetric (↑toEuclideanLin A)
⊢ ↑(↑(OrthonormalBasis.toBasis
(OrthonormalBasis.reindex
(LinearMap.IsSymmetric.eigenvectorBasis (_ : LinearMap.IsSymmetric (↑toEuclideanLin A))
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n))
(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)))).repr
(↑(PiLp.equiv 2 fun i => 𝕜).symm (Aᵀ j)))
i =
↑(LinearMap.IsSymmetric.eigenvectorBasis this
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)).repr
(↑(PiLp.equiv 2 fun i => 𝕜).symm (mulVec A (Pi.single j 1)))
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)
[PROOFSTEP]
simp_rw [mulVec_single, mul_one, OrthonormalBasis.coe_toBasis_repr_apply, OrthonormalBasis.repr_reindex]
[GOAL]
case h.e'_2
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
this : LinearMap.IsSymmetric (↑toEuclideanLin A)
⊢ ↑(LinearMap.IsSymmetric.eigenvectorBasis (_ : LinearMap.IsSymmetric (↑toEuclideanLin A))
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)).repr
(↑(PiLp.equiv 2 fun i => 𝕜).symm (Aᵀ j))
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i) =
↑(LinearMap.IsSymmetric.eigenvectorBasis this
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)).repr
(↑(PiLp.equiv 2 fun i => 𝕜).symm fun i => A i j)
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)
[PROOFSTEP]
rfl
[GOAL]
case h.e'_3
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
this : LinearMap.IsSymmetric (↑toEuclideanLin A)
⊢ (diagonal (IsROrC.ofReal ∘ eigenvalues hA) *
Basis.toMatrix (OrthonormalBasis.toBasis (eigenvectorBasis hA)) ↑(PiLp.basisFun 2 𝕜 n))
i j =
↑(LinearMap.IsSymmetric.eigenvalues this (_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)) *
↑(LinearMap.IsSymmetric.eigenvectorBasis this
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)).repr
(EuclideanSpace.single j 1)
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)
[PROOFSTEP]
simp only [diagonal_mul, (· ∘ ·), eigenvalues]
[GOAL]
case h.e'_3
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i j : n
this : LinearMap.IsSymmetric (↑toEuclideanLin A)
⊢ ↑(eigenvalues₀ hA (↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)) *
Basis.toMatrix (OrthonormalBasis.toBasis (eigenvectorBasis hA)) (↑(PiLp.basisFun 2 𝕜 n)) i j =
↑(LinearMap.IsSymmetric.eigenvalues this (_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)) *
↑(LinearMap.IsSymmetric.eigenvectorBasis this
(_ : FiniteDimensional.finrank 𝕜 (EuclideanSpace 𝕜 n) = Fintype.card n)).repr
(EuclideanSpace.single j 1)
(↑(Fintype.equivOfCardEq (_ : Fintype.card (Fin (Fintype.card n)) = Fintype.card n)).symm i)
[PROOFSTEP]
rw [eigenvectorBasis, Basis.toMatrix_apply, OrthonormalBasis.coe_toBasis_repr_apply, OrthonormalBasis.repr_reindex,
eigenvalues₀, PiLp.basisFun_apply, PiLp.equiv_symm_single]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i : n
⊢ eigenvalues hA i = ↑IsROrC.re (star ((eigenvectorMatrix hA)ᵀ i) ⬝ᵥ mulVec A ((eigenvectorMatrix hA)ᵀ i))
[PROOFSTEP]
have := hA.spectral_theorem
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i : n
this : eigenvectorMatrixInv hA * A = diagonal (IsROrC.ofReal ∘ eigenvalues hA) * eigenvectorMatrixInv hA
⊢ eigenvalues hA i = ↑IsROrC.re (star ((eigenvectorMatrix hA)ᵀ i) ⬝ᵥ mulVec A ((eigenvectorMatrix hA)ᵀ i))
[PROOFSTEP]
rw [← @Matrix.mul_inv_eq_iff_eq_mul_of_invertible (A := hA.eigenvectorMatrixInv)] at this
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i : n
this : eigenvectorMatrixInv hA * A * (eigenvectorMatrixInv hA)⁻¹ = diagonal (IsROrC.ofReal ∘ eigenvalues hA)
⊢ eigenvalues hA i = ↑IsROrC.re (star ((eigenvectorMatrix hA)ᵀ i) ⬝ᵥ mulVec A ((eigenvectorMatrix hA)ᵀ i))
[PROOFSTEP]
have := congr_arg IsROrC.re (congr_fun (congr_fun this i) i)
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i : n
this✝ : eigenvectorMatrixInv hA * A * (eigenvectorMatrixInv hA)⁻¹ = diagonal (IsROrC.ofReal ∘ eigenvalues hA)
this :
↑IsROrC.re ((eigenvectorMatrixInv hA * A * (eigenvectorMatrixInv hA)⁻¹) i i) =
↑IsROrC.re (diagonal (IsROrC.ofReal ∘ eigenvalues hA) i i)
⊢ eigenvalues hA i = ↑IsROrC.re (star ((eigenvectorMatrix hA)ᵀ i) ⬝ᵥ mulVec A ((eigenvectorMatrix hA)ᵀ i))
[PROOFSTEP]
rw [diagonal_apply_eq, Function.comp_apply, IsROrC.ofReal_re, inv_eq_left_inv hA.eigenvectorMatrix_mul_inv, ←
conjTranspose_eigenvectorMatrix, mul_mul_apply] at this
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
i : n
this✝ : eigenvectorMatrixInv hA * A * (eigenvectorMatrixInv hA)⁻¹ = diagonal (IsROrC.ofReal ∘ eigenvalues hA)
this : ↑IsROrC.re ((eigenvectorMatrix hA)ᴴ i ⬝ᵥ mulVec A ((eigenvectorMatrix hA)ᵀ i)) = eigenvalues hA i
⊢ eigenvalues hA i = ↑IsROrC.re (star ((eigenvectorMatrix hA)ᵀ i) ⬝ᵥ mulVec A ((eigenvectorMatrix hA)ᵀ i))
[PROOFSTEP]
exact this.symm
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ det A = ∏ i : n, ↑(eigenvalues hA i)
[PROOFSTEP]
apply mul_left_cancel₀ (det_ne_zero_of_left_inverse (eigenvectorMatrix_mul_inv hA))
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ det (eigenvectorMatrixInv hA) * det A = det (eigenvectorMatrixInv hA) * ∏ i : n, ↑(eigenvalues hA i)
[PROOFSTEP]
rw [← det_mul, spectral_theorem, det_mul, mul_comm, det_diagonal]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ det (eigenvectorMatrixInv hA) * ∏ i : n, (IsROrC.ofReal ∘ eigenvalues hA) i =
det (eigenvectorMatrixInv hA) * ∏ i : n, ↑(eigenvalues hA i)
[PROOFSTEP]
simp_rw [Function.comp_apply]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ A = eigenvectorMatrix hA * diagonal (IsROrC.ofReal ∘ eigenvalues hA) * eigenvectorMatrixInv hA
[PROOFSTEP]
simpa [← Matrix.mul_assoc, hA.eigenvectorMatrix_mul_inv, Matrix.one_mul] using
congr_arg (hA.eigenvectorMatrix * ·) hA.spectral_theorem
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ rank A = rank (diagonal (eigenvalues hA))
[PROOFSTEP]
conv_lhs => rw [hA.spectral_theorem']
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
| rank A
[PROOFSTEP]
rw [hA.spectral_theorem']
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
| rank A
[PROOFSTEP]
rw [hA.spectral_theorem']
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
| rank A
[PROOFSTEP]
rw [hA.spectral_theorem']
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ rank (eigenvectorMatrix hA * diagonal (IsROrC.ofReal ∘ eigenvalues hA) * eigenvectorMatrixInv hA) =
rank (diagonal (eigenvalues hA))
[PROOFSTEP]
have hE := isUnit_det_of_invertible (hA.eigenvectorMatrix)
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
hE : IsUnit (det (eigenvectorMatrix hA))
⊢ rank (eigenvectorMatrix hA * diagonal (IsROrC.ofReal ∘ eigenvalues hA) * eigenvectorMatrixInv hA) =
rank (diagonal (eigenvalues hA))
[PROOFSTEP]
have hiE := isUnit_det_of_invertible (hA.eigenvectorMatrixInv)
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
hE : IsUnit (det (eigenvectorMatrix hA))
hiE : IsUnit (det (eigenvectorMatrixInv hA))
⊢ rank (eigenvectorMatrix hA * diagonal (IsROrC.ofReal ∘ eigenvalues hA) * eigenvectorMatrixInv hA) =
rank (diagonal (eigenvalues hA))
[PROOFSTEP]
simp only [rank_mul_eq_right_of_isUnit_det hA.eigenvectorMatrix _ hE,
rank_mul_eq_left_of_isUnit_det hA.eigenvectorMatrixInv _ hiE, rank_diagonal, Function.comp_apply, ne_eq,
algebraMap.lift_map_eq_zero_iff]
[GOAL]
𝕜 : Type u_1
inst✝³ : IsROrC 𝕜
inst✝² : DecidableEq 𝕜
n : Type u_2
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n 𝕜
hA : IsHermitian A
⊢ rank A = Fintype.card { i // eigenvalues hA i ≠ 0 }
[PROOFSTEP]
rw [rank_eq_rank_diagonal hA, Matrix.rank_diagonal]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Spectrum", "llama_tokens": 6930} |
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
cases isEmpty_or_nonempty n
[GOAL]
case inl
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : IsEmpty n
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
exfalso
[GOAL]
case inl.h
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : IsEmpty n
⊢ False
[PROOFSTEP]
exact hμ (Submodule.eq_bot_of_subsingleton _)
[GOAL]
case inr
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
obtain ⟨v, h_eg, h_nz⟩ := hμ.exists_hasEigenvector
[GOAL]
case inr.intro.intro
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz : v ≠ 0
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
obtain ⟨i, -, h_i⟩ := Finset.exists_mem_eq_sup' Finset.univ_nonempty (fun i => ‖v i‖)
[GOAL]
case inr.intro.intro.intro.intro
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
have h_nz : v i ≠ 0 := by
contrapose! h_nz
ext j
rw [Pi.zero_apply, ← norm_le_zero_iff]
refine (h_i ▸ Finset.le_sup' (fun i => ‖v i‖) (Finset.mem_univ j)).trans ?_
exact norm_le_zero_iff.mpr h_nz
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
⊢ v i ≠ 0
[PROOFSTEP]
contrapose! h_nz
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i = 0
⊢ v = 0
[PROOFSTEP]
ext j
[GOAL]
case h
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i = 0
j : n
⊢ v j = OfNat.ofNat 0 j
[PROOFSTEP]
rw [Pi.zero_apply, ← norm_le_zero_iff]
[GOAL]
case h
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i = 0
j : n
⊢ ‖v j‖ ≤ 0
[PROOFSTEP]
refine (h_i ▸ Finset.le_sup' (fun i => ‖v i‖) (Finset.mem_univ j)).trans ?_
[GOAL]
case h
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i = 0
j : n
⊢ ‖v i‖ ≤ 0
[PROOFSTEP]
exact norm_le_zero_iff.mpr h_nz
[GOAL]
case inr.intro.intro.intro.intro
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
have h_le : ∀ j, ‖v j * (v i)⁻¹‖ ≤ 1 := fun j =>
by
rw [norm_mul, norm_inv, mul_inv_le_iff' (norm_pos_iff.mpr h_nz), one_mul]
exact h_i ▸ Finset.le_sup' (fun i => ‖v i‖) (Finset.mem_univ j)
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
j : n
⊢ ‖v j * (v i)⁻¹‖ ≤ 1
[PROOFSTEP]
rw [norm_mul, norm_inv, mul_inv_le_iff' (norm_pos_iff.mpr h_nz), one_mul]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
j : n
⊢ ‖v j‖ ≤ ‖v i‖
[PROOFSTEP]
exact h_i ▸ Finset.le_sup' (fun i => ‖v i‖) (Finset.mem_univ j)
[GOAL]
case inr.intro.intro.intro.intro
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ∃ k, μ ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
simp_rw [mem_closedBall_iff_norm']
[GOAL]
case inr.intro.intro.intro.intro
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ∃ k, ‖A k k - μ‖ ≤ ∑ j in Finset.erase Finset.univ k, ‖A k j‖
[PROOFSTEP]
refine ⟨i, ?_⟩
[GOAL]
case inr.intro.intro.intro.intro
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ‖A i i - μ‖ ≤ ∑ j in Finset.erase Finset.univ i, ‖A i j‖
[PROOFSTEP]
calc
_ = ‖(A i i * v i - μ * v i) * (v i)⁻¹‖ := by congr; field_simp [h_nz]; ring
_ = ‖(A i i * v i - ∑ j, A i j * v j) * (v i)⁻¹‖ := by
rw [show μ * v i = ∑ x : n, A i x * v x
by
rw [← Matrix.dotProduct, ← Matrix.mulVec]
exact (congrFun (Module.End.mem_eigenspace_iff.mp h_eg) i).symm]
_ = ‖(∑ j in Finset.univ.erase i, A i j * v j) * (v i)⁻¹‖ := by
rw [Finset.sum_erase_eq_sub (Finset.mem_univ i), ← neg_sub, neg_mul, norm_neg]
_ ≤ ∑ j in Finset.univ.erase i, ‖A i j‖ * ‖v j * (v i)⁻¹‖ :=
by
rw [Finset.sum_mul]
exact (norm_sum_le _ _).trans (le_of_eq (by simp_rw [mul_assoc, norm_mul]))
_ ≤ ∑ j in Finset.univ.erase i, ‖A i j‖ :=
(Finset.sum_le_sum fun j _ => mul_le_of_le_one_right (norm_nonneg _) (h_le j))
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ‖A i i - μ‖ = ‖(A i i * v i - μ * v i) * (v i)⁻¹‖
[PROOFSTEP]
congr
[GOAL]
case e_a
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ A i i - μ = (A i i * v i - μ * v i) * (v i)⁻¹
[PROOFSTEP]
field_simp [h_nz]
[GOAL]
case e_a
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ (A i i - μ) * v i = A i i * v i - μ * v i
[PROOFSTEP]
ring
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ‖(A i i * v i - μ * v i) * (v i)⁻¹‖ = ‖(A i i * v i - ∑ j : n, A i j * v j) * (v i)⁻¹‖
[PROOFSTEP]
rw [show μ * v i = ∑ x : n, A i x * v x by
rw [← Matrix.dotProduct, ← Matrix.mulVec]
exact (congrFun (Module.End.mem_eigenspace_iff.mp h_eg) i).symm]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ μ * v i = ∑ x : n, A i x * v x
[PROOFSTEP]
rw [← Matrix.dotProduct, ← Matrix.mulVec]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ μ * v i = Matrix.mulVec A (fun x => v x) i
[PROOFSTEP]
exact (congrFun (Module.End.mem_eigenspace_iff.mp h_eg) i).symm
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ‖(A i i * v i - ∑ j : n, A i j * v j) * (v i)⁻¹‖ = ‖(∑ j in Finset.erase Finset.univ i, A i j * v j) * (v i)⁻¹‖
[PROOFSTEP]
rw [Finset.sum_erase_eq_sub (Finset.mem_univ i), ← neg_sub, neg_mul, norm_neg]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ‖(∑ j in Finset.erase Finset.univ i, A i j * v j) * (v i)⁻¹‖ ≤
∑ j in Finset.erase Finset.univ i, ‖A i j‖ * ‖v j * (v i)⁻¹‖
[PROOFSTEP]
rw [Finset.sum_mul]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ‖∑ x in Finset.erase Finset.univ i, A i x * v x * (v i)⁻¹‖ ≤
∑ j in Finset.erase Finset.univ i, ‖A i j‖ * ‖v j * (v i)⁻¹‖
[PROOFSTEP]
exact (norm_sum_le _ _).trans (le_of_eq (by simp_rw [mul_assoc, norm_mul]))
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
μ : K
hμ : Module.End.HasEigenvalue (↑Matrix.toLin' A) μ
h✝ : Nonempty n
v : n → K
h_eg : v ∈ Module.End.eigenspace (↑Matrix.toLin' A) μ
h_nz✝ : v ≠ 0
i : n
h_i : (Finset.sup' Finset.univ (_ : Finset.Nonempty Finset.univ) fun i => ‖v i‖) = ‖v i‖
h_nz : v i ≠ 0
h_le : ∀ (j : n), ‖v j * (v i)⁻¹‖ ≤ 1
⊢ ∑ i_1 in Finset.erase Finset.univ i, ‖A i i_1 * v i_1 * (v i)⁻¹‖ =
∑ j in Finset.erase Finset.univ i, ‖A i j‖ * ‖v j * (v i)⁻¹‖
[PROOFSTEP]
simp_rw [mul_assoc, norm_mul]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : ∀ (k : n), ∑ j in Finset.erase Finset.univ k, ‖A k j‖ < ‖A k k‖
⊢ Matrix.det A ≠ 0
[PROOFSTEP]
contrapose! h
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : Matrix.det A = 0
⊢ ∃ k, ‖A k k‖ ≤ ∑ j in Finset.erase Finset.univ k, ‖A k j‖
[PROOFSTEP]
suffices ∃ k, 0 ∈ Metric.closedBall (A k k) (∑ j in Finset.univ.erase k, ‖A k j‖) by
exact this.imp (fun a h ↦ by rwa [mem_closedBall_iff_norm', sub_zero] at h )
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : Matrix.det A = 0
this : ∃ k, 0 ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
⊢ ∃ k, ‖A k k‖ ≤ ∑ j in Finset.erase Finset.univ k, ‖A k j‖
[PROOFSTEP]
exact this.imp (fun a h ↦ by rwa [mem_closedBall_iff_norm', sub_zero] at h )
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h✝ : Matrix.det A = 0
this : ∃ k, 0 ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
a : n
h : 0 ∈ Metric.closedBall (A a a) (∑ j in Finset.erase Finset.univ a, ‖A a j‖)
⊢ ‖A a a‖ ≤ ∑ j in Finset.erase Finset.univ a, ‖A a j‖
[PROOFSTEP]
rwa [mem_closedBall_iff_norm', sub_zero] at h
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : Matrix.det A = 0
⊢ ∃ k, 0 ∈ Metric.closedBall (A k k) (∑ j in Finset.erase Finset.univ k, ‖A k j‖)
[PROOFSTEP]
refine eigenvalue_mem_ball ?_
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : Matrix.det A = 0
⊢ Module.End.HasEigenvalue (↑Matrix.toLin' fun k => A k) 0
[PROOFSTEP]
rw [Module.End.HasEigenvalue, Module.End.eigenspace_zero, ne_comm]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : Matrix.det A = 0
⊢ ⊥ ≠ LinearMap.ker (↑Matrix.toLin' fun k => A k)
[PROOFSTEP]
exact ne_of_lt (LinearMap.bot_lt_ker_of_det_eq_zero (by rwa [LinearMap.det_toLin']))
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : Matrix.det A = 0
⊢ ↑LinearMap.det (↑Matrix.toLin' fun k => A k) = 0
[PROOFSTEP]
rwa [LinearMap.det_toLin']
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : ∀ (k : n), ∑ i in Finset.erase Finset.univ k, ‖A i k‖ < ‖A k k‖
⊢ Matrix.det A ≠ 0
[PROOFSTEP]
rw [← Matrix.det_transpose]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : ∀ (k : n), ∑ i in Finset.erase Finset.univ k, ‖A i k‖ < ‖A k k‖
⊢ Matrix.det (Matrix.transpose A) ≠ 0
[PROOFSTEP]
exact det_ne_zero_of_sum_row_lt_diag (by simp_rw [Matrix.transpose_apply]; exact h)
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : ∀ (k : n), ∑ i in Finset.erase Finset.univ k, ‖A i k‖ < ‖A k k‖
⊢ ∀ (k : n), ∑ j in Finset.erase Finset.univ k, ‖Matrix.transpose A k j‖ < ‖Matrix.transpose A k k‖
[PROOFSTEP]
simp_rw [Matrix.transpose_apply]
[GOAL]
K : Type u_1
n : Type u_2
inst✝² : NormedField K
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n K
h : ∀ (k : n), ∑ i in Finset.erase Finset.univ k, ‖A i k‖ < ‖A k k‖
⊢ ∀ (k : n), ∑ x in Finset.erase Finset.univ k, ‖A x k‖ < ‖A k k‖
[PROOFSTEP]
exact h
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Gershgorin", "llama_tokens": 9424} |
[GOAL]
R : Type u_1
inst✝² : CommRing R
M : Type u_2
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ℕ
m : M
⊢ ↑(ι Q) m * ↑(ι Q) m = ↑(algebraMap R (CliffordAlgebra Q)) (↑Q m)
[PROOFSTEP]
erw [← AlgHom.map_mul, RingQuot.mkAlgHom_rel R (Rel.of m), AlgHom.commutes]
[GOAL]
R : Type u_1
inst✝² : CommRing R
M : Type u_2
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ℕ
m : M
⊢ ↑(algebraMap R (RingQuot (Rel Q))) (↑Q m) = ↑(algebraMap R (CliffordAlgebra Q)) (↑Q m)
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
g : CliffordAlgebra Q →ₐ[R] A
m : M
⊢ ↑g (↑(ι Q) m) * ↑g (↑(ι Q) m) = ↑(algebraMap R A) (↑Q m)
[PROOFSTEP]
rw [← AlgHom.map_mul, ι_sq_scalar, AlgHom.commutes]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m) }
x y : TensorAlgebra R M
h : Rel Q x y
⊢ ↑(↑(TensorAlgebra.lift R) ↑f) x = ↑(↑(TensorAlgebra.lift R) ↑f) y
[PROOFSTEP]
induction h
[GOAL]
case of
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m) }
x y : TensorAlgebra R M
m✝ : M
⊢ ↑(↑(TensorAlgebra.lift R) ↑f) (↑(TensorAlgebra.ι R) m✝ * ↑(TensorAlgebra.ι R) m✝) =
↑(↑(TensorAlgebra.lift R) ↑f) (↑(algebraMap R (TensorAlgebra R M)) (↑Q m✝))
[PROOFSTEP]
rw [AlgHom.commutes, AlgHom.map_mul, TensorAlgebra.lift_ι_apply, f.prop]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
F : CliffordAlgebra Q →ₐ[R] A
m : M
⊢ ↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m * ↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m =
↑(algebraMap R A) (↑Q m)
[PROOFSTEP]
rw [LinearMap.comp_apply, AlgHom.toLinearMap_apply, comp_ι_sq_scalar]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m) }
⊢ (fun F =>
{ val := LinearMap.comp (AlgHom.toLinearMap F) (ι Q),
property :=
(_ :
∀ (m : M),
↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m * ↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m =
↑(algebraMap R A) (↑Q m)) })
((fun f =>
↑(RingQuot.liftAlgHom R)
{ val := ↑(TensorAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : TensorAlgebra R M),
Rel Q x y → ↑(↑(TensorAlgebra.lift R) ↑f) x = ↑(↑(TensorAlgebra.lift R) ↑f) y) })
f) =
f
[PROOFSTEP]
ext x
[GOAL]
case a.h
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m) }
x : M
⊢ ↑↑((fun F =>
{ val := LinearMap.comp (AlgHom.toLinearMap F) (ι Q),
property :=
(_ :
∀ (m : M),
↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m *
↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m =
↑(algebraMap R A) (↑Q m)) })
((fun f =>
↑(RingQuot.liftAlgHom R)
{ val := ↑(TensorAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : TensorAlgebra R M),
Rel Q x y → ↑(↑(TensorAlgebra.lift R) ↑f) x = ↑(↑(TensorAlgebra.lift R) ↑f) y) })
f))
x =
↑↑f x
[PROOFSTEP]
exact (RingQuot.liftAlgHom_mkAlgHom_apply _ _ _ _).trans (TensorAlgebra.lift_ι_apply _ x)
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
F : CliffordAlgebra Q →ₐ[R] A
x : M
⊢ ↑(LinearMap.comp
(AlgHom.toLinearMap
(AlgHom.comp
((fun f =>
↑(RingQuot.liftAlgHom R)
{ val := ↑(TensorAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : TensorAlgebra R M),
Rel Q x y → ↑(↑(TensorAlgebra.lift R) ↑f) x = ↑(↑(TensorAlgebra.lift R) ↑f) y) })
((fun F =>
{ val := LinearMap.comp (AlgHom.toLinearMap F) (ι Q),
property :=
(_ :
∀ (m : M),
↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m *
↑(LinearMap.comp (AlgHom.toLinearMap F) (ι Q)) m =
↑(algebraMap R A) (↑Q m)) })
F))
(RingQuot.mkAlgHom R fun x y => Rel Q x y)))
(TensorAlgebra.ι R))
x =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.comp F (RingQuot.mkAlgHom R fun x y => Rel Q x y)))
(TensorAlgebra.ι R))
x
[PROOFSTEP]
exact (RingQuot.liftAlgHom_mkAlgHom_apply _ _ _ _).trans (TensorAlgebra.lift_ι_apply _ _)
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
cond : ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m)
g : CliffordAlgebra Q →ₐ[R] A
⊢ LinearMap.comp (AlgHom.toLinearMap g) (ι Q) = f ↔ g = ↑(lift Q) { val := f, property := cond }
[PROOFSTEP]
convert (lift Q : _ ≃ (CliffordAlgebra Q →ₐ[R] A)).symm_apply_eq
[GOAL]
case h.e'_1.a
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
cond : ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m)
g : CliffordAlgebra Q →ₐ[R] A
⊢ LinearMap.comp (AlgHom.toLinearMap g) (ι Q) = f ↔ ↑(lift Q).symm g = { val := f, property := cond }
[PROOFSTEP]
rw [lift_symm_apply, Subtype.mk_eq_mk]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
g : CliffordAlgebra Q →ₐ[R] A
⊢ ↑(lift Q)
{ val := LinearMap.comp (AlgHom.toLinearMap g) (ι Q),
property := (_ : ∀ (m : M), ↑g (↑(ι Q) m) * ↑g (↑(ι Q) m) = ↑(algebraMap R A) (↑Q m)) } =
g
[PROOFSTEP]
exact (lift Q : _ ≃ (CliffordAlgebra Q →ₐ[R] A)).apply_symm_apply g
[GOAL]
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A✝ : Type u_3
inst✝³ : Semiring A✝
inst✝² : Algebra R A✝
A : Type u_4
inst✝¹ : Semiring A
inst✝ : Algebra R A
f g : CliffordAlgebra Q →ₐ[R] A
⊢ LinearMap.comp (AlgHom.toLinearMap f) (ι Q) = LinearMap.comp (AlgHom.toLinearMap g) (ι Q) → f = g
[PROOFSTEP]
intro h
[GOAL]
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A✝ : Type u_3
inst✝³ : Semiring A✝
inst✝² : Algebra R A✝
A : Type u_4
inst✝¹ : Semiring A
inst✝ : Algebra R A
f g : CliffordAlgebra Q →ₐ[R] A
h : LinearMap.comp (AlgHom.toLinearMap f) (ι Q) = LinearMap.comp (AlgHom.toLinearMap g) (ι Q)
⊢ f = g
[PROOFSTEP]
apply (lift Q).symm.injective
[GOAL]
case a
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A✝ : Type u_3
inst✝³ : Semiring A✝
inst✝² : Algebra R A✝
A : Type u_4
inst✝¹ : Semiring A
inst✝ : Algebra R A
f g : CliffordAlgebra Q →ₐ[R] A
h : LinearMap.comp (AlgHom.toLinearMap f) (ι Q) = LinearMap.comp (AlgHom.toLinearMap g) (ι Q)
⊢ ↑(lift Q).symm f = ↑(lift Q).symm g
[PROOFSTEP]
rw [lift_symm_apply, lift_symm_apply]
[GOAL]
case a
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A✝ : Type u_3
inst✝³ : Semiring A✝
inst✝² : Algebra R A✝
A : Type u_4
inst✝¹ : Semiring A
inst✝ : Algebra R A
f g : CliffordAlgebra Q →ₐ[R] A
h : LinearMap.comp (AlgHom.toLinearMap f) (ι Q) = LinearMap.comp (AlgHom.toLinearMap g) (ι Q)
⊢ { val := LinearMap.comp (AlgHom.toLinearMap f) (ι Q),
property :=
(_ :
∀ (m : M),
↑(LinearMap.comp (AlgHom.toLinearMap f) (ι Q)) m * ↑(LinearMap.comp (AlgHom.toLinearMap f) (ι Q)) m =
↑(algebraMap R A) (↑Q m)) } =
{ val := LinearMap.comp (AlgHom.toLinearMap g) (ι Q),
property :=
(_ :
∀ (m : M),
↑(LinearMap.comp (AlgHom.toLinearMap g) (ι Q)) m * ↑(LinearMap.comp (AlgHom.toLinearMap g) (ι Q)) m =
↑(algebraMap R A) (↑Q m)) }
[PROOFSTEP]
simp only [h]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
⊢ C a
[PROOFSTEP]
let s : Subalgebra R (CliffordAlgebra Q) :=
{ carrier := C
mul_mem' := @h_mul
add_mem' := @h_add
algebraMap_mem' := h_grade0 }
-- porting note: Added `h`. `h` is needed for `of`.
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
⊢ C a
[PROOFSTEP]
letI h : AddCommMonoid s := inferInstanceAs (AddCommMonoid (Subalgebra.toSubmodule s))
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
⊢ C a
[PROOFSTEP]
let of : { f : M →ₗ[R] s // ∀ m, f m * f m = algebraMap _ _ (Q m) } :=
⟨(ι Q).codRestrict (Subalgebra.toSubmodule s) h_grade1, fun m => Subtype.eq <| ι_sq_scalar Q m⟩
-- the mapping through the subalgebra is the identity
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R { x // x ∈ s }) (↑Q m) } :=
{ val := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1,
property :=
(_ :
∀ (m : M),
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m *
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m =
↑(algebraMap R { x // x ∈ s }) (↑Q m)) }
⊢ C a
[PROOFSTEP]
have of_id : AlgHom.id R (CliffordAlgebra Q) = s.val.comp (lift Q of) :=
by
ext
simp
-- porting note: `simp` can't apply this
erw [LinearMap.codRestrict_apply]
-- finding a proof is finding an element of the subalgebra
-- porting note: was `convert Subtype.prop (lift Q of a); exact AlgHom.congr_fun of_id a`
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R { x // x ∈ s }) (↑Q m) } :=
{ val := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1,
property :=
(_ :
∀ (m : M),
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m *
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m =
↑(algebraMap R { x // x ∈ s }) (↑Q m)) }
⊢ AlgHom.id R (CliffordAlgebra Q) = AlgHom.comp (Subalgebra.val s) (↑(lift Q) of)
[PROOFSTEP]
ext
[GOAL]
case a.h
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R { x // x ∈ s }) (↑Q m) } :=
{ val := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1,
property :=
(_ :
∀ (m : M),
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m *
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m =
↑(algebraMap R { x // x ∈ s }) (↑Q m)) }
x✝ : M
⊢ ↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (CliffordAlgebra Q))) (ι Q)) x✝ =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.comp (Subalgebra.val s) (↑(lift Q) of))) (ι Q)) x✝
[PROOFSTEP]
simp
-- porting note: `simp` can't apply this
[GOAL]
case a.h
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R { x // x ∈ s }) (↑Q m) } :=
{ val := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1,
property :=
(_ :
∀ (m : M),
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m *
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m =
↑(algebraMap R { x // x ∈ s }) (↑Q m)) }
x✝ : M
⊢ ↑(ι Q) x✝ = ↑(↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) x✝)
[PROOFSTEP]
erw [LinearMap.codRestrict_apply]
-- finding a proof is finding an element of the subalgebra
-- porting note: was `convert Subtype.prop (lift Q of a); exact AlgHom.congr_fun of_id a`
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R { x // x ∈ s }) (↑Q m) } :=
{ val := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1,
property :=
(_ :
∀ (m : M),
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m *
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m =
↑(algebraMap R { x // x ∈ s }) (↑Q m)) }
of_id : AlgHom.id R (CliffordAlgebra Q) = AlgHom.comp (Subalgebra.val s) (↑(lift Q) of)
⊢ C a
[PROOFSTEP]
rw [← AlgHom.id_apply (R := R) a, of_id]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
C : CliffordAlgebra Q → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (CliffordAlgebra Q)) r)
h_grade1 : ∀ (x : M), C (↑(ι Q) x)
h_mul : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a * b)
h_add : ∀ (a b : CliffordAlgebra Q), C a → C b → C (a + b)
a : CliffordAlgebra Q
s : Subalgebra R (CliffordAlgebra Q) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : { f // ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R { x // x ∈ s }) (↑Q m) } :=
{ val := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1,
property :=
(_ :
∀ (m : M),
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m *
↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι Q) h_grade1) m =
↑(algebraMap R { x // x ∈ s }) (↑Q m)) }
of_id : AlgHom.id R (CliffordAlgebra Q) = AlgHom.comp (Subalgebra.val s) (↑(lift Q) of)
⊢ C (↑(AlgHom.comp (Subalgebra.val s) (↑(lift Q) of)) a)
[PROOFSTEP]
exact Subtype.prop (lift Q of a)
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
a b : M
⊢ ↑(ι Q) a * ↑(ι Q) b + ↑(ι Q) b * ↑(ι Q) a =
↑(ι Q) (a + b) * ↑(ι Q) (a + b) - ↑(ι Q) a * ↑(ι Q) a - ↑(ι Q) b * ↑(ι Q) b
[PROOFSTEP]
rw [(ι Q).map_add, mul_add, add_mul, add_mul]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
a b : M
⊢ ↑(ι Q) a * ↑(ι Q) b + ↑(ι Q) b * ↑(ι Q) a =
↑(ι Q) a * ↑(ι Q) a + ↑(ι Q) b * ↑(ι Q) a + (↑(ι Q) a * ↑(ι Q) b + ↑(ι Q) b * ↑(ι Q) b) - ↑(ι Q) a * ↑(ι Q) a -
↑(ι Q) b * ↑(ι Q) b
[PROOFSTEP]
abel
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
a b : M
⊢ ↑(ι Q) a * ↑(ι Q) b + ↑(ι Q) b * ↑(ι Q) a =
↑(ι Q) a * ↑(ι Q) a + ↑(ι Q) b * ↑(ι Q) a + (↑(ι Q) a * ↑(ι Q) b + ↑(ι Q) b * ↑(ι Q) b) - ↑(ι Q) a * ↑(ι Q) a -
↑(ι Q) b * ↑(ι Q) b
[PROOFSTEP]
abel
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
a b : M
⊢ ↑(ι Q) (a + b) * ↑(ι Q) (a + b) - ↑(ι Q) a * ↑(ι Q) a - ↑(ι Q) b * ↑(ι Q) b =
↑(algebraMap R (CliffordAlgebra Q)) (↑Q (a + b)) - ↑(algebraMap R (CliffordAlgebra Q)) (↑Q a) -
↑(algebraMap R (CliffordAlgebra Q)) (↑Q b)
[PROOFSTEP]
rw [ι_sq_scalar, ι_sq_scalar, ι_sq_scalar]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
a b : M
⊢ ↑(algebraMap R (CliffordAlgebra Q)) (↑Q (a + b)) - ↑(algebraMap R (CliffordAlgebra Q)) (↑Q a) -
↑(algebraMap R (CliffordAlgebra Q)) (↑Q b) =
↑(algebraMap R (CliffordAlgebra Q)) (↑Q (a + b) - ↑Q a - ↑Q b)
[PROOFSTEP]
rw [← RingHom.map_sub, ← RingHom.map_sub]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
a b : M
⊢ ↑(ι Q) a * ↑(ι Q) b * ↑(ι Q) a = ↑(ι Q) (QuadraticForm.polar (↑Q) a b • a - ↑Q a • b)
[PROOFSTEP]
rw [ι_mul_comm, sub_mul, mul_assoc, ι_sq_scalar, ← Algebra.smul_def, ← Algebra.commutes, ← Algebra.smul_def, ← map_smul,
← map_smul, ← map_sub]
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
cond : ∀ (m : M), ↑f m * ↑f m = ↑(algebraMap R A) (↑Q m)
⊢ Submodule.map (AlgHom.toLinearMap (↑(lift Q) { val := f, property := cond })) (LinearMap.range (ι Q)) =
LinearMap.range f
[PROOFSTEP]
rw [← LinearMap.range_comp, ι_comp_lift]
[GOAL]
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
⊢ map Q₁ Q₁ LinearMap.id (_ : ∀ (m : M₁), ↑Q₁ (↑LinearMap.id m) = ↑Q₁ (↑LinearMap.id m)) =
AlgHom.id R (CliffordAlgebra Q₁)
[PROOFSTEP]
ext m
[GOAL]
case a.h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
m : M₁
⊢ ↑(LinearMap.comp
(AlgHom.toLinearMap (map Q₁ Q₁ LinearMap.id (_ : ∀ (m : M₁), ↑Q₁ (↑LinearMap.id m) = ↑Q₁ (↑LinearMap.id m))))
(ι Q₁))
m =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (CliffordAlgebra Q₁))) (ι Q₁)) m
[PROOFSTEP]
exact map_apply_ι _ _ _ _ m
[GOAL]
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
f : M₂ →ₗ[R] M₃
hf : ∀ (m : M₂), ↑Q₃ (↑f m) = ↑Q₂ m
g : M₁ →ₗ[R] M₂
hg : ∀ (m : M₁), ↑Q₂ (↑g m) = ↑Q₁ m
⊢ AlgHom.comp (map Q₂ Q₃ f hf) (map Q₁ Q₂ g hg) =
map Q₁ Q₃ (LinearMap.comp f g) (_ : ∀ (m : M₁), ↑Q₃ (↑f (↑g m)) = ↑Q₁ m)
[PROOFSTEP]
ext m
[GOAL]
case a.h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
f : M₂ →ₗ[R] M₃
hf : ∀ (m : M₂), ↑Q₃ (↑f m) = ↑Q₂ m
g : M₁ →ₗ[R] M₂
hg : ∀ (m : M₁), ↑Q₂ (↑g m) = ↑Q₁ m
m : M₁
⊢ ↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.comp (map Q₂ Q₃ f hf) (map Q₁ Q₂ g hg))) (ι Q₁)) m =
↑(LinearMap.comp (AlgHom.toLinearMap (map Q₁ Q₃ (LinearMap.comp f g) (_ : ∀ (m : M₁), ↑Q₃ (↑f (↑g m)) = ↑Q₁ m)))
(ι Q₁))
m
[PROOFSTEP]
dsimp only [LinearMap.comp_apply, AlgHom.comp_apply, AlgHom.toLinearMap_apply, AlgHom.id_apply]
[GOAL]
case a.h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
f : M₂ →ₗ[R] M₃
hf : ∀ (m : M₂), ↑Q₃ (↑f m) = ↑Q₂ m
g : M₁ →ₗ[R] M₂
hg : ∀ (m : M₁), ↑Q₂ (↑g m) = ↑Q₁ m
m : M₁
⊢ ↑(map Q₂ Q₃ f hf) (↑(map Q₁ Q₂ g hg) (↑(ι Q₁) m)) =
↑(map Q₁ Q₃ (LinearMap.comp f g) (_ : ∀ (m : M₁), ↑Q₃ (↑f (↑g m)) = ↑Q₁ m)) (↑(ι Q₁) m)
[PROOFSTEP]
rw [map_apply_ι, map_apply_ι, map_apply_ι, LinearMap.comp_apply]
[GOAL]
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e : QuadraticForm.IsometryEquiv Q₁ Q₂
⊢ map Q₂ Q₂ (LinearMap.comp ↑↑e ↑↑(QuadraticForm.IsometryEquiv.symm e))
(_ : ∀ (m : M₂), ↑Q₂ (↑↑↑e (↑↑↑(QuadraticForm.IsometryEquiv.symm e) m)) = ↑Q₂ m) =
AlgHom.id R (CliffordAlgebra Q₂)
[PROOFSTEP]
convert map_id Q₂ using 2
-- porting note: replaced `_` with `Q₂`
[GOAL]
case h.e'_2.h.e'_11
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e : QuadraticForm.IsometryEquiv Q₁ Q₂
⊢ LinearMap.comp ↑↑e ↑↑(QuadraticForm.IsometryEquiv.symm e) = LinearMap.id
[PROOFSTEP]
ext m
[GOAL]
case h.e'_2.h.e'_11.h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e : QuadraticForm.IsometryEquiv Q₁ Q₂
m : M₂
⊢ ↑(LinearMap.comp ↑↑e ↑↑(QuadraticForm.IsometryEquiv.symm e)) m = ↑LinearMap.id m
[PROOFSTEP]
exact e.toLinearEquiv.apply_symm_apply m
[GOAL]
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e : QuadraticForm.IsometryEquiv Q₁ Q₂
⊢ map Q₁ Q₁ (LinearMap.comp ↑↑(QuadraticForm.IsometryEquiv.symm e) ↑↑e)
(_ : ∀ (m : M₁), ↑Q₁ (↑↑↑(QuadraticForm.IsometryEquiv.symm e) (↑↑↑e m)) = ↑Q₁ m) =
AlgHom.id R (CliffordAlgebra Q₁)
[PROOFSTEP]
convert map_id Q₁ using 2
-- porting note: replaced `_` with `Q₁`
[GOAL]
case h.e'_2.h.e'_11
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e : QuadraticForm.IsometryEquiv Q₁ Q₂
⊢ LinearMap.comp ↑↑(QuadraticForm.IsometryEquiv.symm e) ↑↑e = LinearMap.id
[PROOFSTEP]
ext m
[GOAL]
case h.e'_2.h.e'_11.h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e : QuadraticForm.IsometryEquiv Q₁ Q₂
m : M₁
⊢ ↑(LinearMap.comp ↑↑(QuadraticForm.IsometryEquiv.symm e) ↑↑e) m = ↑LinearMap.id m
[PROOFSTEP]
exact e.toLinearEquiv.symm_apply_apply m
[GOAL]
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e₁₂ : QuadraticForm.IsometryEquiv Q₁ Q₂
e₂₃ : QuadraticForm.IsometryEquiv Q₂ Q₃
⊢ AlgEquiv.trans (equivOfIsometry e₁₂) (equivOfIsometry e₂₃) =
equivOfIsometry (QuadraticForm.IsometryEquiv.trans e₁₂ e₂₃)
[PROOFSTEP]
ext x
[GOAL]
case h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
e₁₂ : QuadraticForm.IsometryEquiv Q₁ Q₂
e₂₃ : QuadraticForm.IsometryEquiv Q₂ Q₃
x : CliffordAlgebra Q₁
⊢ ↑(AlgEquiv.trans (equivOfIsometry e₁₂) (equivOfIsometry e₂₃)) x =
↑(equivOfIsometry (QuadraticForm.IsometryEquiv.trans e₁₂ e₂₃)) x
[PROOFSTEP]
exact AlgHom.congr_fun (map_comp_map Q₁ Q₂ Q₃ _ _ _ _) x
[GOAL]
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
⊢ equivOfIsometry (QuadraticForm.IsometryEquiv.refl Q₁) = AlgEquiv.refl
[PROOFSTEP]
ext x
[GOAL]
case h
R : Type u_1
inst✝¹⁰ : CommRing R
M : Type u_2
inst✝⁹ : AddCommGroup M
inst✝⁸ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝⁷ : Semiring A
inst✝⁶ : Algebra R A
M₁ : Type u_4
M₂ : Type u_5
M₃ : Type u_6
inst✝⁵ : AddCommGroup M₁
inst✝⁴ : AddCommGroup M₂
inst✝³ : AddCommGroup M₃
inst✝² : Module R M₁
inst✝¹ : Module R M₂
inst✝ : Module R M₃
Q₁ : QuadraticForm R M₁
Q₂ : QuadraticForm R M₂
Q₃ : QuadraticForm R M₃
x : CliffordAlgebra Q₁
⊢ ↑(equivOfIsometry (QuadraticForm.IsometryEquiv.refl Q₁)) x = ↑AlgEquiv.refl x
[PROOFSTEP]
exact AlgHom.congr_fun (map_id Q₁) x
[GOAL]
R : Type u_1
inst✝⁵ : CommRing R
M : Type u_2
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝² : Semiring A
inst✝¹ : Algebra R A
m : M
inst✝ : Invertible (↑Q m)
⊢ ↑(ι Q) (⅟(↑Q m) • m) * ↑(ι Q) m = 1
[PROOFSTEP]
rw [map_smul, smul_mul_assoc, ι_sq_scalar, Algebra.smul_def, ← map_mul, invOf_mul_self, map_one]
[GOAL]
R : Type u_1
inst✝⁵ : CommRing R
M : Type u_2
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝² : Semiring A
inst✝¹ : Algebra R A
m : M
inst✝ : Invertible (↑Q m)
⊢ ↑(ι Q) m * ↑(ι Q) (⅟(↑Q m) • m) = 1
[PROOFSTEP]
rw [map_smul, mul_smul_comm, ι_sq_scalar, Algebra.smul_def, ← map_mul, invOf_mul_self, map_one]
[GOAL]
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝³ : Semiring A
inst✝² : Algebra R A
m : M
inst✝¹ : Invertible (↑Q m)
inst✝ : Invertible (↑(ι Q) m)
⊢ ⅟(↑(ι Q) m) = ↑(ι Q) (⅟(↑Q m) • m)
[PROOFSTEP]
letI := invertibleιOfInvertible Q m
[GOAL]
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝³ : Semiring A
inst✝² : Algebra R A
m : M
inst✝¹ : Invertible (↑Q m)
inst✝ : Invertible (↑(ι Q) m)
this : Invertible (↑(ι Q) m) := invertibleιOfInvertible Q m
⊢ ⅟(↑(ι Q) m) = ↑(ι Q) (⅟(↑Q m) • m)
[PROOFSTEP]
convert (rfl : ⅟(ι Q m) = _)
[GOAL]
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
m : M
h : IsUnit (↑Q m)
⊢ IsUnit (↑(ι Q) m)
[PROOFSTEP]
cases h.nonempty_invertible
[GOAL]
case intro
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
m : M
h : IsUnit (↑Q m)
val✝ : Invertible (↑Q m)
⊢ IsUnit (↑(ι Q) m)
[PROOFSTEP]
letI := invertibleιOfInvertible Q m
[GOAL]
case intro
R : Type u_1
inst✝⁴ : CommRing R
M : Type u_2
inst✝³ : AddCommGroup M
inst✝² : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
m : M
h : IsUnit (↑Q m)
val✝ : Invertible (↑Q m)
this : Invertible (↑(ι Q) m) := invertibleιOfInvertible Q m
⊢ IsUnit (↑(ι Q) m)
[PROOFSTEP]
exact isUnit_of_invertible (ι Q m)
[GOAL]
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝³ : Semiring A
inst✝² : Algebra R A
a b : M
inst✝¹ : Invertible (↑(ι Q) a)
inst✝ : Invertible (↑Q a)
⊢ ↑(ι Q) a * ↑(ι Q) b * ⅟(↑(ι Q) a) = ↑(ι Q) ((⅟(↑Q a) * QuadraticForm.polar (↑Q) a b) • a - b)
[PROOFSTEP]
rw [invOf_ι, map_smul, mul_smul_comm, ι_mul_ι_mul_ι, ← map_smul, smul_sub, smul_smul, smul_smul, invOf_mul_self,
one_smul]
[GOAL]
R : Type u_1
inst✝⁶ : CommRing R
M : Type u_2
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
Q : QuadraticForm R M
n : ℕ
A : Type u_3
inst✝³ : Semiring A
inst✝² : Algebra R A
a b : M
inst✝¹ : Invertible (↑(ι Q) a)
inst✝ : Invertible (↑Q a)
⊢ ⅟(↑(ι Q) a) * ↑(ι Q) b * ↑(ι Q) a = ↑(ι Q) ((⅟(↑Q a) * QuadraticForm.polar (↑Q) a b) • a - b)
[PROOFSTEP]
rw [invOf_ι, map_smul, smul_mul_assoc, smul_mul_assoc, ι_mul_ι_mul_ι, ← map_smul, smul_sub, smul_smul, smul_smul,
invOf_mul_self, one_smul]
[GOAL]
R : Type u_1
inst✝² : CommRing R
M : Type u_2
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ℕ
m : M
⊢ ↑toClifford (↑(ι R) m) = ↑(CliffordAlgebra.ι Q) m
[PROOFSTEP]
simp [toClifford]
| {"mathlib_filename": "Mathlib.LinearAlgebra.CliffordAlgebra.Basic", "llama_tokens": 17852} |
{"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.InvariantBasisNumber", "llama_tokens": 0} |
|
[GOAL]
m : Type u_1
n : Type u_2
R : Type u_3
S : Type u_4
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing R
inst✝ : Nontrivial R
⊢ det (mvPolynomialX m m R) ≠ 0
[PROOFSTEP]
intro h_det
[GOAL]
m : Type u_1
n : Type u_2
R : Type u_3
S : Type u_4
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing R
inst✝ : Nontrivial R
h_det : det (mvPolynomialX m m R) = 0
⊢ False
[PROOFSTEP]
have := congr_arg Matrix.det (mvPolynomialX_mapMatrix_eval (1 : Matrix m m R))
[GOAL]
m : Type u_1
n : Type u_2
R : Type u_3
S : Type u_4
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing R
inst✝ : Nontrivial R
h_det : det (mvPolynomialX m m R) = 0
this : det (↑(RingHom.mapMatrix (MvPolynomial.eval fun p => OfNat.ofNat 1 p.fst p.snd)) (mvPolynomialX m m R)) = det 1
⊢ False
[PROOFSTEP]
rw [det_one, ← RingHom.map_det, h_det, RingHom.map_zero] at this
[GOAL]
m : Type u_1
n : Type u_2
R : Type u_3
S : Type u_4
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing R
inst✝ : Nontrivial R
h_det : det (mvPolynomialX m m R) = 0
this : 0 = 1
⊢ False
[PROOFSTEP]
exact zero_ne_one this
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.MvPolynomial", "llama_tokens": 549} |
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
⊢ ker (↑toLin' (diagonal w)) = ⨆ (i : m) (_ : i ∈ {i | w i = 0}), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
rw [← comap_bot, ← iInf_ker_proj, comap_iInf]
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
⊢ ⨅ (i : m), comap (↑toLin' (diagonal w)) (ker (proj i)) =
⨆ (i : m) (_ : i ∈ {i | w i = 0}), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
have := fun i : m => ker_comp (toLin' (diagonal w)) (proj i)
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
this : ∀ (i : m), ker (comp (proj i) (↑toLin' (diagonal w))) = comap (↑toLin' (diagonal w)) (ker (proj i))
⊢ ⨅ (i : m), comap (↑toLin' (diagonal w)) (ker (proj i)) =
⨆ (i : m) (_ : i ∈ {i | w i = 0}), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
simp only [comap_iInf, ← this, proj_diagonal, ker_smul']
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
this : ∀ (i : m), ker (comp (proj i) (↑toLin' (diagonal w))) = comap (↑toLin' (diagonal w)) (ker (proj i))
⊢ ⨅ (i : m) (_ : w i ≠ 0), ker (proj i) =
⨆ (i : m) (_ : i ∈ {i | w i = 0}), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
have : univ ⊆ {i : m | w i = 0} ∪ {i : m | w i = 0}ᶜ := by rw [Set.union_compl_self]
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
this : ∀ (i : m), ker (comp (proj i) (↑toLin' (diagonal w))) = comap (↑toLin' (diagonal w)) (ker (proj i))
⊢ univ ⊆ {i | w i = 0} ∪ {i | w i = 0}ᶜ
[PROOFSTEP]
rw [Set.union_compl_self]
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
this✝ : ∀ (i : m), ker (comp (proj i) (↑toLin' (diagonal w))) = comap (↑toLin' (diagonal w)) (ker (proj i))
this : univ ⊆ {i | w i = 0} ∪ {i | w i = 0}ᶜ
⊢ ⨅ (i : m) (_ : w i ≠ 0), ker (proj i) =
⨆ (i : m) (_ : i ∈ {i | w i = 0}), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
exact (iSup_range_stdBasis_eq_iInf_ker_proj K (fun _ : m => K) disjoint_compl_right this (Set.toFinite _)).symm
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
⊢ LinearMap.range (↑toLin' (diagonal w)) =
⨆ (i : m) (_ : i ∈ {i | w i ≠ 0}), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
dsimp only [mem_setOf_eq]
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
⊢ LinearMap.range (↑toLin' (diagonal w)) =
⨆ (i : m) (_ : w i ≠ 0), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
rw [← Submodule.map_top, ← iSup_range_stdBasis, Submodule.map_iSup]
[GOAL]
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
⊢ ⨆ (i : m), Submodule.map (↑toLin' (diagonal w)) (LinearMap.range (LinearMap.stdBasis K (fun a => K) i)) =
⨆ (i : m) (_ : w i ≠ 0), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
congr
[GOAL]
case e_s
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
⊢ (fun i => Submodule.map (↑toLin' (diagonal w)) (LinearMap.range (LinearMap.stdBasis K (fun a => K) i))) = fun i =>
⨆ (_ : w i ≠ 0), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
funext i
[GOAL]
case e_s.h
m : Type u_1
n : Type u_2
inst✝³ : Fintype m
inst✝² : Fintype n
K : Type u
inst✝¹ : Semifield K
inst✝ : DecidableEq m
w : m → K
i : m
⊢ Submodule.map (↑toLin' (diagonal w)) (LinearMap.range (LinearMap.stdBasis K (fun a => K) i)) =
⨆ (_ : w i ≠ 0), LinearMap.range (LinearMap.stdBasis K (fun x => K) i)
[PROOFSTEP]
rw [← LinearMap.range_comp, diagonal_comp_stdBasis, ← range_smul']
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
⊢ rank (↑toLin' (Matrix.diagonal w)) = ↑(Fintype.card { i // w i ≠ 0 })
[PROOFSTEP]
have hu : univ ⊆ {i : m | w i = 0}ᶜ ∪ {i : m | w i = 0} := by rw [Set.compl_union_self]
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
⊢ univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
[PROOFSTEP]
rw [Set.compl_union_self]
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
hu : univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
⊢ rank (↑toLin' (Matrix.diagonal w)) = ↑(Fintype.card { i // w i ≠ 0 })
[PROOFSTEP]
have hd : Disjoint {i : m | w i ≠ 0} {i : m | w i = 0} := disjoint_compl_left
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
hu : univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
hd : Disjoint {i | w i ≠ 0} {i | w i = 0}
⊢ rank (↑toLin' (Matrix.diagonal w)) = ↑(Fintype.card { i // w i ≠ 0 })
[PROOFSTEP]
have B₁ := iSup_range_stdBasis_eq_iInf_ker_proj K (fun _ : m => K) hd hu (Set.toFinite _)
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
hu : univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
hd : Disjoint {i | w i ≠ 0} {i | w i = 0}
B₁ :
⨆ (i : m) (_ : i ∈ {i | w i ≠ 0}), range (stdBasis K (fun x => K) i) = ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i)
⊢ rank (↑toLin' (Matrix.diagonal w)) = ↑(Fintype.card { i // w i ≠ 0 })
[PROOFSTEP]
have B₂ := iInfKerProjEquiv K (fun _ ↦ K) hd hu
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
hu : univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
hd : Disjoint {i | w i ≠ 0} {i | w i = 0}
B₁ :
⨆ (i : m) (_ : i ∈ {i | w i ≠ 0}), range (stdBasis K (fun x => K) i) = ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i)
B₂ : { x // x ∈ ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i) } ≃ₗ[K] (i : ↑{i | w i ≠ 0}) → (fun x => K) ↑i
⊢ rank (↑toLin' (Matrix.diagonal w)) = ↑(Fintype.card { i // w i ≠ 0 })
[PROOFSTEP]
rw [LinearMap.rank, range_diagonal, B₁, ← @rank_fun' K]
[GOAL]
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
hu : univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
hd : Disjoint {i | w i ≠ 0} {i | w i = 0}
B₁ :
⨆ (i : m) (_ : i ∈ {i | w i ≠ 0}), range (stdBasis K (fun x => K) i) = ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i)
B₂ : { x // x ∈ ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i) } ≃ₗ[K] (i : ↑{i | w i ≠ 0}) → (fun x => K) ↑i
⊢ Module.rank K { x // x ∈ ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i) } = Module.rank K ({ i // w i ≠ 0 } → K)
[PROOFSTEP]
apply LinearEquiv.rank_eq
[GOAL]
case f
m : Type u_1
n : Type u_2
inst✝⁴ : Fintype m
inst✝³ : Fintype n
K : Type u
inst✝² : Field K
inst✝¹ : DecidableEq m
inst✝ : DecidableEq K
w : m → K
hu : univ ⊆ {i | w i = 0}ᶜ ∪ {i | w i = 0}
hd : Disjoint {i | w i ≠ 0} {i | w i = 0}
B₁ :
⨆ (i : m) (_ : i ∈ {i | w i ≠ 0}), range (stdBasis K (fun x => K) i) = ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i)
B₂ : { x // x ∈ ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i) } ≃ₗ[K] (i : ↑{i | w i ≠ 0}) → (fun x => K) ↑i
⊢ { x // x ∈ ⨅ (i : m) (_ : i ∈ {i | w i = 0}), ker (proj i) } ≃ₗ[K] { i // w i ≠ 0 } → K
[PROOFSTEP]
apply B₂
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Diagonal", "llama_tokens": 4183} |
[GOAL]
R : Type u_1
S : Type u_2
inst✝⁴ : CommRing R
inst✝³ : Nontrivial R
inst✝² : LinearOrderedCommRing S
n : Type u_3
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n R
abv : AbsoluteValue R S
x : S
hx : ∀ (i j : n), ↑abv (A i j) ≤ x
σ : Perm n
x✝ : σ ∈ univ
⊢ ↑abv (↑Perm.sign σ • ∏ i : n, A (↑σ i) i) = ∏ i : n, ↑abv (A (↑σ i) i)
[PROOFSTEP]
rw [abv.map_units_int_smul, abv.map_prod]
[GOAL]
R : Type u_1
S : Type u_2
inst✝⁴ : CommRing R
inst✝³ : Nontrivial R
inst✝² : LinearOrderedCommRing S
n : Type u_3
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n R
abv : AbsoluteValue R S
x : S
hx : ∀ (i j : n), ↑abv (A i j) ≤ x
x✝¹ : Perm n
x✝ : x✝¹ ∈ univ
⊢ ∏ _i : n, x = x ^ Fintype.card n
[PROOFSTEP]
rw [prod_const, Finset.card_univ]
[GOAL]
R : Type u_1
S : Type u_2
inst✝⁴ : CommRing R
inst✝³ : Nontrivial R
inst✝² : LinearOrderedCommRing S
n : Type u_3
inst✝¹ : Fintype n
inst✝ : DecidableEq n
A : Matrix n n R
abv : AbsoluteValue R S
x : S
hx : ∀ (i j : n), ↑abv (A i j) ≤ x
⊢ ∑ _σ : Perm n, x ^ Fintype.card n = Nat.factorial (Fintype.card n) • x ^ Fintype.card n
[PROOFSTEP]
rw [sum_const, Finset.card_univ, Fintype.card_perm]
[GOAL]
R : Type u_1
S : Type u_2
inst✝⁴ : CommRing R
inst✝³ : Nontrivial R
inst✝² : LinearOrderedCommRing S
n : Type u_3
inst✝¹ : Fintype n
inst✝ : DecidableEq n
ι : Type u_4
s : Finset ι
A : ι → Matrix n n R
abv : AbsoluteValue R S
x : S
hx : ∀ (k : ι) (i j : n), ↑abv (A k i j) ≤ x
i j : n
⊢ ↑abv (Finset.sum s (fun k => A k) i j) = ↑abv (∑ k in s, A k i j)
[PROOFSTEP]
simp only [sum_apply]
[GOAL]
R : Type u_1
S : Type u_2
inst✝⁴ : CommRing R
inst✝³ : Nontrivial R
inst✝² : LinearOrderedCommRing S
n : Type u_3
inst✝¹ : Fintype n
inst✝ : DecidableEq n
ι : Type u_4
s : Finset ι
c : ι → R
A : ι → Matrix n n R
abv : AbsoluteValue R S
x : S
hx : ∀ (k : ι) (i j : n), ↑abv (A k i j) ≤ x
y : S
hy : ∀ (k : ι), ↑abv (c k) ≤ y
⊢ ↑abv (det (∑ k in s, c k • A k)) ≤ Nat.factorial (Fintype.card n) • (card s • y * x) ^ Fintype.card n
[PROOFSTEP]
simpa only [smul_mul_assoc] using
det_sum_le s fun k i j =>
calc
abv (c k * A k i j) = abv (c k) * abv (A k i j) := abv.map_mul _ _
_ ≤ y * x := mul_le_mul (hy k) (hx k i j) (abv.nonneg _) ((abv.nonneg _).trans (hy k))
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.AbsoluteValue", "llama_tokens": 1186} |
{"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.FiniteDimensional", "llama_tokens": 0} |
|
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝⁴ : Fintype m
inst✝³ : Fintype n
inst✝² : Fintype p
inst✝¹ : DecidableEq n
inst✝ : AddCommMonoidWithOne R
⊢ trace 1 = ↑(Fintype.card n)
[PROOFSTEP]
simp_rw [trace, diag_one, Pi.one_def, Finset.sum_const, nsmul_one, Finset.card_univ]
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝⁴ : Fintype m
inst✝³ : Fintype n
inst✝² : Fintype p
inst✝¹ : AddCommMonoid R
inst✝ : CommSemigroup R
A : Matrix m n R
B : Matrix n m R
⊢ trace (A * B) = trace (B * A)
[PROOFSTEP]
rw [← trace_transpose, ← trace_transpose_mul, transpose_mul]
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : NonUnitalCommSemiring R
A : Matrix m n R
B : Matrix n p R
C : Matrix p m R
⊢ trace (A * B * C) = trace (C * A * B)
[PROOFSTEP]
rw [trace_mul_comm, Matrix.mul_assoc]
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : NonUnitalCommSemiring R
A : Matrix m n R
B : Matrix n p R
C : Matrix p m R
⊢ trace (A * (B * C)) = trace (C * (A * B))
[PROOFSTEP]
rw [← Matrix.mul_assoc, trace_mul_comm]
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : NonUnitalNonAssocSemiring R
a b : n → R
⊢ trace (col a * row b) = a ⬝ᵥ b
[PROOFSTEP]
apply Finset.sum_congr rfl
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : NonUnitalNonAssocSemiring R
a b : n → R
⊢ ∀ (x : n), x ∈ Finset.univ → diag (col a * row b) x = a x * b x
[PROOFSTEP]
simp [mul_apply]
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : AddCommMonoid R
A : Matrix (Fin 3) (Fin 3) R
⊢ trace A = A 0 0 + A 1 1 + A 2 2
[PROOFSTEP]
rw [← add_zero (A 2 2), add_assoc]
[GOAL]
ι : Type u_1
m : Type u_2
n : Type u_3
p : Type u_4
α : Type u_5
R : Type u_6
S : Type u_7
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : AddCommMonoid R
A : Matrix (Fin 3) (Fin 3) R
⊢ trace A = A 0 0 + (A 1 1 + (A 2 2 + 0))
[PROOFSTEP]
rfl
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Trace", "llama_tokens": 1287} |
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
⊢ eigenspace f 0 = LinearMap.ker f
[PROOFSTEP]
simp [eigenspace]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
x : M
h : HasEigenvector f μ x
⊢ HasEigenvalue f μ
[PROOFSTEP]
rw [HasEigenvalue, Submodule.ne_bot_iff]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
x : M
h : HasEigenvector f μ x
⊢ ∃ x, x ∈ eigenspace f μ ∧ x ≠ 0
[PROOFSTEP]
use x
[GOAL]
case h
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
x : M
h : HasEigenvector f μ x
⊢ x ∈ eigenspace f μ ∧ x ≠ 0
[PROOFSTEP]
exact h
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
x : M
⊢ x ∈ eigenspace f μ ↔ ↑f x = μ • x
[PROOFSTEP]
rw [eigenspace, LinearMap.mem_ker, LinearMap.sub_apply, algebraMap_end_apply, sub_eq_zero]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
hμ : HasEigenvalue f μ
⊢ μ ∈ spectrum R f
[PROOFSTEP]
refine' spectrum.mem_iff.mpr fun h_unit => _
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
hμ : HasEigenvalue f μ
h_unit : IsUnit (↑(algebraMap R (End R M)) μ - f)
⊢ False
[PROOFSTEP]
set f' := LinearMap.GeneralLinearGroup.toLinearEquiv h_unit.unit
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
hμ : HasEigenvalue f μ
h_unit : IsUnit (↑(algebraMap R (End R M)) μ - f)
f' : M ≃ₗ[R] M := LinearMap.GeneralLinearGroup.toLinearEquiv (IsUnit.unit h_unit)
⊢ False
[PROOFSTEP]
rcases hμ.exists_hasEigenvector with ⟨v, hv⟩
[GOAL]
case intro
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
hμ : HasEigenvalue f μ
h_unit : IsUnit (↑(algebraMap R (End R M)) μ - f)
f' : M ≃ₗ[R] M := LinearMap.GeneralLinearGroup.toLinearEquiv (IsUnit.unit h_unit)
v : M
hv : HasEigenvector f μ v
⊢ False
[PROOFSTEP]
refine' hv.2 ((LinearMap.ker_eq_bot'.mp f'.ker) v (_ : μ • v - f v = 0))
[GOAL]
case intro
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
hμ : HasEigenvalue f μ
h_unit : IsUnit (↑(algebraMap R (End R M)) μ - f)
f' : M ≃ₗ[R] M := LinearMap.GeneralLinearGroup.toLinearEquiv (IsUnit.unit h_unit)
v : M
hv : HasEigenvector f μ v
⊢ μ • v - ↑f v = 0
[PROOFSTEP]
rw [hv.apply_eq_smul, sub_self]
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
h : μ ∈ spectrum K f
⊢ HasEigenvalue f μ
[PROOFSTEP]
rwa [spectrum.mem_iff, IsUnit.sub_iff, LinearMap.isUnit_iff_ker_eq_bot] at h
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
a b : K
hb : b ≠ 0
⊢ eigenspace f (a / b) = eigenspace f (b⁻¹ * a)
[PROOFSTEP]
rw [div_eq_mul_inv, mul_comm]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
a b : K
hb : b ≠ 0
⊢ eigenspace f (b⁻¹ * a) = LinearMap.ker (f - (b⁻¹ * a) • LinearMap.id)
[PROOFSTEP]
rw [eigenspace]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
a b : K
hb : b ≠ 0
⊢ LinearMap.ker (f - ↑(algebraMap K (End K V)) (b⁻¹ * a)) = LinearMap.ker (f - (b⁻¹ * a) • LinearMap.id)
[PROOFSTEP]
rfl
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
a b : K
hb : b ≠ 0
⊢ LinearMap.ker (f - (b⁻¹ * a) • LinearMap.id) = LinearMap.ker (f - b⁻¹ • a • LinearMap.id)
[PROOFSTEP]
rw [smul_smul]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
a b : K
hb : b ≠ 0
⊢ LinearMap.ker (f - b⁻¹ • ↑(algebraMap K (End K V)) a) = LinearMap.ker (b • (f - b⁻¹ • ↑(algebraMap K (End K V)) a))
[PROOFSTEP]
rw [LinearMap.ker_smul _ b hb]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
a b : K
hb : b ≠ 0
⊢ LinearMap.ker (b • (f - b⁻¹ • ↑(algebraMap K (End K V)) a)) = LinearMap.ker (b • f - ↑(algebraMap K (End K V)) a)
[PROOFSTEP]
rw [smul_sub, smul_inv_smul₀ hb]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
⊢ CompleteLattice.Independent (eigenspace f)
[PROOFSTEP]
classical
-- Define an operation from `Π₀ μ : K, f.eigenspace μ`, the vector space of finitely-supported
-- choices of an eigenvector from each eigenspace, to `V`, by sending a collection to its sum.
let S :
@LinearMap K K _ _ (RingHom.id K) (Π₀ μ : K, f.eigenspace μ) V (@DFinsupp.addCommMonoid K (fun μ => f.eigenspace μ) _)
_ (@DFinsupp.module K _ (fun μ => f.eigenspace μ) _ _ _) _ :=
@DFinsupp.lsum K K ℕ _ V _ _ _ _ _ _ _ _ _ fun μ => (f.eigenspace μ).subtype
suffices ∀ l : Π₀ μ, f.eigenspace μ, S l = 0 → l = 0
by
rw [CompleteLattice.independent_iff_dfinsupp_lsum_injective]
change Function.Injective S
rw [← @LinearMap.ker_eq_bot K K (Π₀ μ, f.eigenspace μ) V _ _ (@DFinsupp.addCommGroup K (fun μ => f.eigenspace μ) _)]
rw [eq_bot_iff]
exact this
intro l hl
induction' h_l_support : l.support using Finset.induction with μ₀ l_support' hμ₀ ih generalizing l
· exact DFinsupp.support_eq_empty.1 h_l_support
· let l' := DFinsupp.mapRange.linearMap (fun μ => (μ - μ₀) • @LinearMap.id K (f.eigenspace μ) _ _ _) l
have h_l_support' : l'.support = l_support' :=
by
rw [← Finset.erase_insert hμ₀, ← h_l_support]
ext a
have : ¬(a = μ₀ ∨ l a = 0) ↔ ¬a = μ₀ ∧ ¬l a = 0 := not_or
simp only [DFinsupp.mapRange.linearMap_apply, DFinsupp.mapRange_apply, DFinsupp.mem_support_iff, Finset.mem_erase,
id.def, LinearMap.id_coe, LinearMap.smul_apply, Ne.def, smul_eq_zero, sub_eq_zero, this]
-- The entries of `l'` add up to `0`.
have total_l' : S l' = 0 := by
let g := f - algebraMap K (End K V) μ₀
let a : Π₀ _ : K, V := DFinsupp.mapRange.linearMap (fun μ => (f.eigenspace μ).subtype) l
calc
S l' = DFinsupp.lsum ℕ (fun μ => (f.eigenspace μ).subtype.comp ((μ - μ₀) • LinearMap.id)) l := ?_
_ = DFinsupp.lsum ℕ (fun μ => g.comp (f.eigenspace μ).subtype) l := ?_
_ = DFinsupp.lsum ℕ (fun _ => g) a := ?_
_ = g (DFinsupp.lsum ℕ (fun _ => (LinearMap.id : V →ₗ[K] V)) a) := ?_
_ = g (S l) := ?_
_ = 0 := by rw [hl, g.map_zero]
· exact DFinsupp.sum_mapRange_index.linearMap
· congr
ext μ v
simp only [LinearMap.coe_comp, Function.comp_apply, LinearMap.smul_apply, LinearMap.id_coe, id.def, sub_smul,
Submodule.subtype_apply, Submodule.coe_sub, Submodule.coe_smul_of_tower, LinearMap.sub_apply,
mem_eigenspace_iff.1 v.prop, algebraMap_end_apply]
· rw [DFinsupp.sum_mapRange_index.linearMap]
·
simp only [DFinsupp.sumAddHom_apply, LinearMap.id_coe, LinearMap.map_dfinsupp_sum, id.def,
LinearMap.toAddMonoidHom_coe, DFinsupp.lsum_apply_apply]
·
simp only [DFinsupp.sum_mapRange_index.linearMap, LinearMap.id_comp]
-- Therefore, by the induction hypothesis, all entries of `l'` are zero.
have l'_eq_0 := ih l' total_l' h_l_support'
have h_smul_eq_0 : ∀ μ, (μ - μ₀) • l μ = 0 := by
intro μ
calc
(μ - μ₀) • l μ = l' μ := by
simp only [LinearMap.id_coe, id.def, LinearMap.smul_apply, DFinsupp.mapRange_apply,
DFinsupp.mapRange.linearMap_apply]
_ = 0 := by rw [l'_eq_0];
rfl
-- Thus, the eigenspace-representatives in `l` for all `μ ≠ μ₀` are `0`.
have h_lμ_eq_0 : ∀ μ : K, μ ≠ μ₀ → l μ = 0 := by
intro μ hμ
apply or_iff_not_imp_left.1 (smul_eq_zero.1 (h_smul_eq_0 μ))
rwa [sub_eq_zero]
-- So if we sum over all these representatives, we obtain `0`.
have h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => (l μ : V)) = 0 :=
by
rw [← Finset.sum_const_zero]
apply Finset.sum_congr rfl
intro μ hμ
rw [Submodule.coe_eq_zero, h_lμ_eq_0]
rintro rfl
exact hμ₀ hμ
have : l μ₀ = 0 :=
by
simp only [DFinsupp.lsum_apply_apply, DFinsupp.sumAddHom_apply, LinearMap.toAddMonoidHom_coe, DFinsupp.sum,
h_l_support, Submodule.subtype_apply, Submodule.coe_eq_zero, Finset.sum_insert hμ₀, h_sum_l_support'_eq_0,
add_zero] at hl
exact hl
show l = 0
· ext μ
by_cases h_cases : μ = μ₀
· rwa [h_cases, SetLike.coe_eq_coe, DFinsupp.coe_zero, Pi.zero_apply]
· exact congr_arg _ (h_lμ_eq_0 μ h_cases)
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
⊢ CompleteLattice.Independent (eigenspace f)
[PROOFSTEP]
let S :
@LinearMap K K _ _ (RingHom.id K) (Π₀ μ : K, f.eigenspace μ) V (@DFinsupp.addCommMonoid K (fun μ => f.eigenspace μ) _)
_ (@DFinsupp.module K _ (fun μ => f.eigenspace μ) _ _ _) _ :=
@DFinsupp.lsum K K ℕ _ V _ _ _ _ _ _ _ _ _ fun μ => (f.eigenspace μ).subtype
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
⊢ CompleteLattice.Independent (eigenspace f)
[PROOFSTEP]
suffices ∀ l : Π₀ μ, f.eigenspace μ, S l = 0 → l = 0
by
rw [CompleteLattice.independent_iff_dfinsupp_lsum_injective]
change Function.Injective S
rw [← @LinearMap.ker_eq_bot K K (Π₀ μ, f.eigenspace μ) V _ _ (@DFinsupp.addCommGroup K (fun μ => f.eigenspace μ) _)]
rw [eq_bot_iff]
exact this
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
this : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → l = 0
⊢ CompleteLattice.Independent (eigenspace f)
[PROOFSTEP]
rw [CompleteLattice.independent_iff_dfinsupp_lsum_injective]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
this : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → l = 0
⊢ Function.Injective ↑(↑(DFinsupp.lsum ℕ) fun i => Submodule.subtype (eigenspace f i))
[PROOFSTEP]
change Function.Injective S
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
this : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → l = 0
⊢ Function.Injective ↑S
[PROOFSTEP]
rw [← @LinearMap.ker_eq_bot K K (Π₀ μ, f.eigenspace μ) V _ _ (@DFinsupp.addCommGroup K (fun μ => f.eigenspace μ) _)]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
this : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → l = 0
⊢ LinearMap.ker S = ⊥
[PROOFSTEP]
rw [eq_bot_iff]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
this : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → l = 0
⊢ LinearMap.ker S ≤ ⊥
[PROOFSTEP]
exact this
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
⊢ ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → l = 0
[PROOFSTEP]
intro l hl
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
⊢ l = 0
[PROOFSTEP]
induction' h_l_support : l.support using Finset.induction with μ₀ l_support' hμ₀ ih generalizing l
[GOAL]
case empty
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = ∅
⊢ l = 0
[PROOFSTEP]
exact DFinsupp.support_eq_empty.1 h_l_support
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
⊢ l = 0
[PROOFSTEP]
let l' := DFinsupp.mapRange.linearMap (fun μ => (μ - μ₀) • @LinearMap.id K (f.eigenspace μ) _ _ _) l
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
⊢ l = 0
[PROOFSTEP]
have h_l_support' : l'.support = l_support' :=
by
rw [← Finset.erase_insert hμ₀, ← h_l_support]
ext a
have : ¬(a = μ₀ ∨ l a = 0) ↔ ¬a = μ₀ ∧ ¬l a = 0 := not_or
simp only [DFinsupp.mapRange.linearMap_apply, DFinsupp.mapRange_apply, DFinsupp.mem_support_iff, Finset.mem_erase,
id.def, LinearMap.id_coe, LinearMap.smul_apply, Ne.def, smul_eq_zero, sub_eq_zero, this]
-- The entries of `l'` add up to `0`.
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
⊢ DFinsupp.support l' = l_support'
[PROOFSTEP]
rw [← Finset.erase_insert hμ₀, ← h_l_support]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
⊢ DFinsupp.support l' = Finset.erase (DFinsupp.support l) μ₀
[PROOFSTEP]
ext a
[GOAL]
case a
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
a : K
⊢ a ∈ DFinsupp.support l' ↔ a ∈ Finset.erase (DFinsupp.support l) μ₀
[PROOFSTEP]
have : ¬(a = μ₀ ∨ l a = 0) ↔ ¬a = μ₀ ∧ ¬l a = 0 := not_or
[GOAL]
case a
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
a : K
this : ¬(a = μ₀ ∨ ↑l a = 0) ↔ ¬a = μ₀ ∧ ¬↑l a = 0
⊢ a ∈ DFinsupp.support l' ↔ a ∈ Finset.erase (DFinsupp.support l) μ₀
[PROOFSTEP]
simp only [DFinsupp.mapRange.linearMap_apply, DFinsupp.mapRange_apply, DFinsupp.mem_support_iff, Finset.mem_erase,
id.def, LinearMap.id_coe, LinearMap.smul_apply, Ne.def, smul_eq_zero, sub_eq_zero, this]
-- The entries of `l'` add up to `0`.
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
⊢ l = 0
[PROOFSTEP]
have total_l' : S l' = 0 := by
let g := f - algebraMap K (End K V) μ₀
let a : Π₀ _ : K, V := DFinsupp.mapRange.linearMap (fun μ => (f.eigenspace μ).subtype) l
calc
S l' = DFinsupp.lsum ℕ (fun μ => (f.eigenspace μ).subtype.comp ((μ - μ₀) • LinearMap.id)) l := ?_
_ = DFinsupp.lsum ℕ (fun μ => g.comp (f.eigenspace μ).subtype) l := ?_
_ = DFinsupp.lsum ℕ (fun _ => g) a := ?_
_ = g (DFinsupp.lsum ℕ (fun _ => (LinearMap.id : V →ₗ[K] V)) a) := ?_
_ = g (S l) := ?_
_ = 0 := by rw [hl, g.map_zero]
· exact DFinsupp.sum_mapRange_index.linearMap
· congr
ext μ v
simp only [LinearMap.coe_comp, Function.comp_apply, LinearMap.smul_apply, LinearMap.id_coe, id.def, sub_smul,
Submodule.subtype_apply, Submodule.coe_sub, Submodule.coe_smul_of_tower, LinearMap.sub_apply,
mem_eigenspace_iff.1 v.prop, algebraMap_end_apply]
· rw [DFinsupp.sum_mapRange_index.linearMap]
·
simp only [DFinsupp.sumAddHom_apply, LinearMap.id_coe, LinearMap.map_dfinsupp_sum, id.def,
LinearMap.toAddMonoidHom_coe, DFinsupp.lsum_apply_apply]
·
simp only [DFinsupp.sum_mapRange_index.linearMap, LinearMap.id_comp]
-- Therefore, by the induction hypothesis, all entries of `l'` are zero.
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
⊢ ↑S l' = 0
[PROOFSTEP]
let g := f - algebraMap K (End K V) μ₀
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
⊢ ↑S l' = 0
[PROOFSTEP]
let a : Π₀ _ : K, V := DFinsupp.mapRange.linearMap (fun μ => (f.eigenspace μ).subtype) l
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑S l' = 0
[PROOFSTEP]
calc
S l' = DFinsupp.lsum ℕ (fun μ => (f.eigenspace μ).subtype.comp ((μ - μ₀) • LinearMap.id)) l := ?_
_ = DFinsupp.lsum ℕ (fun μ => g.comp (f.eigenspace μ).subtype) l := ?_
_ = DFinsupp.lsum ℕ (fun _ => g) a := ?_
_ = g (DFinsupp.lsum ℕ (fun _ => (LinearMap.id : V →ₗ[K] V)) a) := ?_
_ = g (S l) := ?_
_ = 0 := by rw [hl, g.map_zero]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑g (↑S l) = 0
[PROOFSTEP]
rw [hl, g.map_zero]
[GOAL]
case calc_1
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑S l' = ↑(↑(DFinsupp.lsum ℕ) fun μ => LinearMap.comp (Submodule.subtype (eigenspace f μ)) ((μ - μ₀) • LinearMap.id)) l
[PROOFSTEP]
exact DFinsupp.sum_mapRange_index.linearMap
[GOAL]
case calc_2
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑(↑(DFinsupp.lsum ℕ) fun μ => LinearMap.comp (Submodule.subtype (eigenspace f μ)) ((μ - μ₀) • LinearMap.id)) l =
↑(↑(DFinsupp.lsum ℕ) fun μ => LinearMap.comp g (Submodule.subtype (eigenspace f μ))) l
[PROOFSTEP]
congr
[GOAL]
case calc_2.e_a.h.e_6.h
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ (fun μ => LinearMap.comp (Submodule.subtype (eigenspace f μ)) ((μ - μ₀) • LinearMap.id)) = fun μ =>
LinearMap.comp g (Submodule.subtype (eigenspace f μ))
[PROOFSTEP]
ext μ v
[GOAL]
case calc_2.e_a.h.e_6.h.h.h
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
μ : K
v : { x // x ∈ eigenspace f μ }
⊢ ↑(LinearMap.comp (Submodule.subtype (eigenspace f μ)) ((μ - μ₀) • LinearMap.id)) v =
↑(LinearMap.comp g (Submodule.subtype (eigenspace f μ))) v
[PROOFSTEP]
simp only [LinearMap.coe_comp, Function.comp_apply, LinearMap.smul_apply, LinearMap.id_coe, id.def, sub_smul,
Submodule.subtype_apply, Submodule.coe_sub, Submodule.coe_smul_of_tower, LinearMap.sub_apply,
mem_eigenspace_iff.1 v.prop, algebraMap_end_apply]
[GOAL]
case calc_3
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑(↑(DFinsupp.lsum ℕ) fun μ => LinearMap.comp g (Submodule.subtype (eigenspace f μ))) l =
↑(↑(DFinsupp.lsum ℕ) fun x => g) a
[PROOFSTEP]
rw [DFinsupp.sum_mapRange_index.linearMap]
[GOAL]
case calc_4
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑(↑(DFinsupp.lsum ℕ) fun x => g) a = ↑g (↑(↑(DFinsupp.lsum ℕ) fun x => LinearMap.id) a)
[PROOFSTEP]
simp only [DFinsupp.sumAddHom_apply, LinearMap.id_coe, LinearMap.map_dfinsupp_sum, id.def, LinearMap.toAddMonoidHom_coe,
DFinsupp.lsum_apply_apply]
[GOAL]
case calc_5
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
g : End K V := f - ↑(algebraMap K (End K V)) μ₀
a : Π₀ (x : K), V := ↑(DFinsupp.mapRange.linearMap fun μ => Submodule.subtype (eigenspace f μ)) l
⊢ ↑g (↑(↑(DFinsupp.lsum ℕ) fun x => LinearMap.id) a) = ↑g (↑S l)
[PROOFSTEP]
simp only [DFinsupp.sum_mapRange_index.linearMap, LinearMap.id_comp]
-- Therefore, by the induction hypothesis, all entries of `l'` are zero.
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
⊢ l = 0
[PROOFSTEP]
have l'_eq_0 := ih l' total_l' h_l_support'
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
⊢ l = 0
[PROOFSTEP]
have h_smul_eq_0 : ∀ μ, (μ - μ₀) • l μ = 0 := by
intro μ
calc
(μ - μ₀) • l μ = l' μ := by
simp only [LinearMap.id_coe, id.def, LinearMap.smul_apply, DFinsupp.mapRange_apply,
DFinsupp.mapRange.linearMap_apply]
_ = 0 := by rw [l'_eq_0];
rfl
-- Thus, the eigenspace-representatives in `l` for all `μ ≠ μ₀` are `0`.
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
⊢ ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
[PROOFSTEP]
intro μ
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
μ : K
⊢ (μ - μ₀) • ↑l μ = 0
[PROOFSTEP]
calc
(μ - μ₀) • l μ = l' μ := by
simp only [LinearMap.id_coe, id.def, LinearMap.smul_apply, DFinsupp.mapRange_apply,
DFinsupp.mapRange.linearMap_apply]
_ = 0 := by rw [l'_eq_0];
rfl
-- Thus, the eigenspace-representatives in `l` for all `μ ≠ μ₀` are `0`.
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
μ : K
⊢ (μ - μ₀) • ↑l μ = ↑l' μ
[PROOFSTEP]
simp only [LinearMap.id_coe, id.def, LinearMap.smul_apply, DFinsupp.mapRange_apply, DFinsupp.mapRange.linearMap_apply]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
μ : K
⊢ ↑l' μ = 0
[PROOFSTEP]
rw [l'_eq_0]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
μ : K
⊢ ↑0 μ = 0
[PROOFSTEP]
rfl
-- Thus, the eigenspace-representatives in `l` for all `μ ≠ μ₀` are `0`.
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
⊢ l = 0
[PROOFSTEP]
have h_lμ_eq_0 : ∀ μ : K, μ ≠ μ₀ → l μ = 0 := by
intro μ hμ
apply or_iff_not_imp_left.1 (smul_eq_zero.1 (h_smul_eq_0 μ))
rwa [sub_eq_zero]
-- So if we sum over all these representatives, we obtain `0`.
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
⊢ ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
[PROOFSTEP]
intro μ hμ
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
μ : K
hμ : μ ≠ μ₀
⊢ ↑l μ = 0
[PROOFSTEP]
apply or_iff_not_imp_left.1 (smul_eq_zero.1 (h_smul_eq_0 μ))
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
μ : K
hμ : μ ≠ μ₀
⊢ ¬μ - μ₀ = 0
[PROOFSTEP]
rwa [sub_eq_zero]
-- So if we sum over all these representatives, we obtain `0`.
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
⊢ l = 0
[PROOFSTEP]
have h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => (l μ : V)) = 0 :=
by
rw [← Finset.sum_const_zero]
apply Finset.sum_congr rfl
intro μ hμ
rw [Submodule.coe_eq_zero, h_lμ_eq_0]
rintro rfl
exact hμ₀ hμ
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
⊢ (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
[PROOFSTEP]
rw [← Finset.sum_const_zero]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
⊢ (Finset.sum l_support' fun μ => ↑(↑l μ)) = Finset.sum ?m.347048 fun _x => 0
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
⊢ Type ?u.347044
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
⊢ Finset ?m.347047
[PROOFSTEP]
apply Finset.sum_congr rfl
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
⊢ ∀ (x : K), x ∈ l_support' → ↑(↑l x) = 0
[PROOFSTEP]
intro μ hμ
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
μ : K
hμ : μ ∈ l_support'
⊢ ↑(↑l μ) = 0
[PROOFSTEP]
rw [Submodule.coe_eq_zero, h_lμ_eq_0]
[GOAL]
case a
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
μ : K
hμ : μ ∈ l_support'
⊢ μ ≠ μ₀
[PROOFSTEP]
rintro rfl
[GOAL]
case a
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
l_support' : Finset K
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
μ : K
hμ : μ ∈ l_support'
hμ₀ : ¬μ ∈ l_support'
h_l_support : DFinsupp.support l = insert μ l_support'
l' : Π₀ (i : K), { x // x ∈ eigenspace f i } := ↑(DFinsupp.mapRange.linearMap fun μ_1 => (μ_1 - μ) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ_1 : K), (μ_1 - μ) • ↑l μ_1 = 0
h_lμ_eq_0 : ∀ (μ_1 : K), μ_1 ≠ μ → ↑l μ_1 = 0
⊢ False
[PROOFSTEP]
exact hμ₀ hμ
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
⊢ l = 0
[PROOFSTEP]
have : l μ₀ = 0 :=
by
simp only [DFinsupp.lsum_apply_apply, DFinsupp.sumAddHom_apply, LinearMap.toAddMonoidHom_coe, DFinsupp.sum,
h_l_support, Submodule.subtype_apply, Submodule.coe_eq_zero, Finset.sum_insert hμ₀, h_sum_l_support'_eq_0,
add_zero] at hl
exact hl
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
⊢ ↑l μ₀ = 0
[PROOFSTEP]
simp only [DFinsupp.lsum_apply_apply, DFinsupp.sumAddHom_apply, LinearMap.toAddMonoidHom_coe, DFinsupp.sum, h_l_support,
Submodule.subtype_apply, Submodule.coe_eq_zero, Finset.sum_insert hμ₀, h_sum_l_support'_eq_0, add_zero] at hl
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
hl : ↑l μ₀ = 0
⊢ ↑l μ₀ = 0
[PROOFSTEP]
exact hl
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
this : ↑l μ₀ = 0
⊢ l = 0
[PROOFSTEP]
show l = 0
[GOAL]
case insert
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
this : ↑l μ₀ = 0
⊢ l = 0
[PROOFSTEP]
ext μ
[GOAL]
case insert.h.a
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
this : ↑l μ₀ = 0
μ : K
⊢ ↑(↑l μ) = ↑(↑0 μ)
[PROOFSTEP]
by_cases h_cases : μ = μ₀
[GOAL]
case pos
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
this : ↑l μ₀ = 0
μ : K
h_cases : μ = μ₀
⊢ ↑(↑l μ) = ↑(↑0 μ)
[PROOFSTEP]
rwa [h_cases, SetLike.coe_eq_coe, DFinsupp.coe_zero, Pi.zero_apply]
[GOAL]
case neg
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
S : (Π₀ (μ : K), { x // x ∈ eigenspace f μ }) →ₗ[K] V := ↑(DFinsupp.lsum ℕ) fun μ => Submodule.subtype (eigenspace f μ)
l✝ : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl✝ : ↑S l✝ = 0
x✝ : Finset K
h_l_support✝ : DFinsupp.support l✝ = x✝
μ₀ : K
l_support' : Finset K
hμ₀ : ¬μ₀ ∈ l_support'
ih : ∀ (l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }), ↑S l = 0 → DFinsupp.support l = l_support' → l = 0
l : Π₀ (μ : K), { x // x ∈ eigenspace f μ }
hl : ↑S l = 0
h_l_support : DFinsupp.support l = insert μ₀ l_support'
l' : (fun x => Π₀ (i : K), { x // x ∈ eigenspace f i }) l :=
↑(DFinsupp.mapRange.linearMap fun μ => (μ - μ₀) • LinearMap.id) l
h_l_support' : DFinsupp.support l' = l_support'
total_l' : ↑S l' = 0
l'_eq_0 : l' = 0
h_smul_eq_0 : ∀ (μ : K), (μ - μ₀) • ↑l μ = 0
h_lμ_eq_0 : ∀ (μ : K), μ ≠ μ₀ → ↑l μ = 0
h_sum_l_support'_eq_0 : (Finset.sum l_support' fun μ => ↑(↑l μ)) = 0
this : ↑l μ₀ = 0
μ : K
h_cases : ¬μ = μ₀
⊢ ↑(↑l μ) = ↑(↑0 μ)
[PROOFSTEP]
exact congr_arg _ (h_lμ_eq_0 μ h_cases)
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k m : ℕ
hm : k ≤ m
⊢ (fun k => LinearMap.ker ((f - ↑(algebraMap R (End R M)) μ) ^ k)) k ≤
(fun k => LinearMap.ker ((f - ↑(algebraMap R (End R M)) μ) ^ k)) m
[PROOFSTEP]
simp only [← pow_sub_mul_pow _ hm]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k m : ℕ
hm : k ≤ m
⊢ LinearMap.ker ((f - ↑(algebraMap R (End R M)) μ) ^ k) ≤
LinearMap.ker ((f - ↑(algebraMap R (End R M)) μ) ^ (m - k) * (f - ↑(algebraMap R (End R M)) μ) ^ k)
[PROOFSTEP]
exact LinearMap.ker_le_ker_comp ((f - algebraMap R (End R M) μ) ^ k) ((f - algebraMap R (End R M) μ) ^ (m - k))
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
k : ℕ
⊢ ↑(generalizedEigenspace f 0) k = LinearMap.ker (f ^ k)
[PROOFSTEP]
simp [Module.End.generalizedEigenspace]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
h : HasGeneralizedEigenvalue f μ k
⊢ k ≠ 0
[PROOFSTEP]
rintro rfl
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
h : HasGeneralizedEigenvalue f μ 0
⊢ False
[PROOFSTEP]
exact h LinearMap.ker_id
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
m : M
⊢ m ∈ maximalGeneralizedEigenspace f μ ↔ ∃ k, ↑((f - μ • 1) ^ k) m = 0
[PROOFSTEP]
simp only [maximalGeneralizedEigenspace, ← mem_generalizedEigenspace, Submodule.mem_iSup_of_chain]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
h : IsNoetherian R M
f : End R M
μ : R
⊢ maximalGeneralizedEigenspace f μ = ↑(generalizedEigenspace f μ) (maximalGeneralizedEigenspaceIndex f μ)
[PROOFSTEP]
rw [isNoetherian_iff_wellFounded] at h
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
h : WellFounded fun x x_1 => x > x_1
f : End R M
μ : R
⊢ maximalGeneralizedEigenspace f μ = ↑(generalizedEigenspace f μ) (maximalGeneralizedEigenspaceIndex f μ)
[PROOFSTEP]
exact (WellFounded.iSup_eq_monotonicSequenceLimit h (f.generalizedEigenspace μ) : _)
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k m : ℕ
hm : k ≤ m
hk : HasGeneralizedEigenvalue f μ k
⊢ HasGeneralizedEigenvalue f μ m
[PROOFSTEP]
unfold HasGeneralizedEigenvalue at *
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k m : ℕ
hm : k ≤ m
hk : ↑(generalizedEigenspace f μ) k ≠ ⊥
⊢ ↑(generalizedEigenspace f μ) m ≠ ⊥
[PROOFSTEP]
contrapose! hk
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k m : ℕ
hm : k ≤ m
hk : ↑(generalizedEigenspace f μ) m = ⊥
⊢ ↑(generalizedEigenspace f μ) k = ⊥
[PROOFSTEP]
rw [← le_bot_iff, ← hk]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k m : ℕ
hm : k ≤ m
hk : ↑(generalizedEigenspace f μ) m = ⊥
⊢ ↑(generalizedEigenspace f μ) k ≤ ↑(generalizedEigenspace f μ) m
[PROOFSTEP]
exact (f.generalizedEigenspace μ).monotone hm
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hk : 0 < k
hμ : HasEigenvalue f μ
⊢ HasGeneralizedEigenvalue f μ k
[PROOFSTEP]
apply hasGeneralizedEigenvalue_of_hasGeneralizedEigenvalue_of_le hk
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hk : 0 < k
hμ : HasEigenvalue f μ
⊢ HasGeneralizedEigenvalue f μ (Nat.succ 0)
[PROOFSTEP]
rw [HasGeneralizedEigenvalue, generalizedEigenspace, OrderHom.coe_mk, pow_one]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hk : 0 < k
hμ : HasEigenvalue f μ
⊢ LinearMap.ker (f - ↑(algebraMap R (End R M)) μ) ≠ ⊥
[PROOFSTEP]
exact hμ
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hμ : HasGeneralizedEigenvalue f μ k
⊢ HasEigenvalue f μ
[PROOFSTEP]
intro contra
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hμ : HasGeneralizedEigenvalue f μ k
contra : eigenspace f μ = ⊥
⊢ False
[PROOFSTEP]
apply hμ
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hμ : HasGeneralizedEigenvalue f μ k
contra : eigenspace f μ = ⊥
⊢ ↑(generalizedEigenspace f μ) k = ⊥
[PROOFSTEP]
erw [LinearMap.ker_eq_bot] at contra ⊢
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hμ : HasGeneralizedEigenvalue f μ k
contra : Function.Injective ↑(f - ↑(algebraMap R (End R M)) μ)
⊢ Function.Injective ↑((f - ↑(algebraMap R (End R M)) μ) ^ k)
[PROOFSTEP]
rw [LinearMap.coe_pow]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
μ : R
k : ℕ
hμ : HasGeneralizedEigenvalue f μ k
contra : Function.Injective ↑(f - ↑(algebraMap R (End R M)) μ)
⊢ Function.Injective (↑(f - ↑(algebraMap R (End R M)) μ))^[k]
[PROOFSTEP]
exact Function.Injective.iterate contra k
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
k : ℕ
μ : R
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
⊢ ↑(generalizedEigenspace (LinearMap.restrict f hfp) μ) k =
Submodule.comap (Submodule.subtype p) (↑(generalizedEigenspace f μ) k)
[PROOFSTEP]
simp only [generalizedEigenspace, OrderHom.coe_mk, ← LinearMap.ker_comp]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
k : ℕ
μ : R
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
⊢ LinearMap.ker ((LinearMap.restrict f hfp - ↑(algebraMap R (End R { x // x ∈ p })) μ) ^ k) =
LinearMap.ker (LinearMap.comp ((f - ↑(algebraMap R (End R M)) μ) ^ k) (Submodule.subtype p))
[PROOFSTEP]
induction' k with k ih
[GOAL]
case zero
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
μ : R
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
⊢ LinearMap.ker ((LinearMap.restrict f hfp - ↑(algebraMap R (End R { x // x ∈ p })) μ) ^ Nat.zero) =
LinearMap.ker (LinearMap.comp ((f - ↑(algebraMap R (End R M)) μ) ^ Nat.zero) (Submodule.subtype p))
[PROOFSTEP]
rw [pow_zero, pow_zero, LinearMap.one_eq_id]
[GOAL]
case zero
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
μ : R
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
⊢ LinearMap.ker LinearMap.id = LinearMap.ker (LinearMap.comp 1 (Submodule.subtype p))
[PROOFSTEP]
apply (Submodule.ker_subtype _).symm
[GOAL]
case succ
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
μ : R
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
k : ℕ
ih :
LinearMap.ker ((LinearMap.restrict f hfp - ↑(algebraMap R (End R { x // x ∈ p })) μ) ^ k) =
LinearMap.ker (LinearMap.comp ((f - ↑(algebraMap R (End R M)) μ) ^ k) (Submodule.subtype p))
⊢ LinearMap.ker ((LinearMap.restrict f hfp - ↑(algebraMap R (End R { x // x ∈ p })) μ) ^ Nat.succ k) =
LinearMap.ker (LinearMap.comp ((f - ↑(algebraMap R (End R M)) μ) ^ Nat.succ k) (Submodule.subtype p))
[PROOFSTEP]
erw [pow_succ', pow_succ', LinearMap.ker_comp, LinearMap.ker_comp, ih, ← LinearMap.ker_comp, LinearMap.comp_assoc]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
μ : R
⊢ Submodule.map (Submodule.subtype p) (eigenspace (LinearMap.restrict f hfp) μ) ≤ eigenspace f μ
[PROOFSTEP]
rintro a ⟨x, hx, rfl⟩
[GOAL]
case intro.intro
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
μ : R
x : { x // x ∈ p }
hx : x ∈ ↑(eigenspace (LinearMap.restrict f hfp) μ)
⊢ ↑(Submodule.subtype p) x ∈ eigenspace f μ
[PROOFSTEP]
simp only [SetLike.mem_coe, mem_eigenspace_iff, LinearMap.restrict_apply] at hx ⊢
[GOAL]
case intro.intro
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
μ : R
x : { x // x ∈ p }
hx : { val := ↑f ↑x, property := (_ : ↑f ↑x ∈ p) } = μ • x
⊢ ↑f (↑(Submodule.subtype p) x) = μ • ↑(Submodule.subtype p) x
[PROOFSTEP]
exact congr_arg Subtype.val hx
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ Disjoint (generalizedEigenrange f μ (finrank K V)) (↑(generalizedEigenspace f μ) (finrank K V))
[PROOFSTEP]
have h :=
calc
Submodule.comap ((f - algebraMap _ _ μ) ^ finrank K V) (f.generalizedEigenspace μ (finrank K V)) =
LinearMap.ker ((f - algebraMap _ _ μ) ^ finrank K V * (f - algebraMap K (End K V) μ) ^ finrank K V) :=
by rw [generalizedEigenspace, OrderHom.coe_mk, ← LinearMap.ker_comp]; rfl
_ = f.generalizedEigenspace μ (finrank K V + finrank K V) := by rw [← pow_add]; rfl
_ = f.generalizedEigenspace μ (finrank K V) := by rw [generalizedEigenspace_eq_generalizedEigenspace_finrank_of_le];
linarith
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ Submodule.comap ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V) (↑(generalizedEigenspace f μ) (finrank K V)) =
LinearMap.ker ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V * (f - ↑(algebraMap K (End K V)) μ) ^ finrank K V)
[PROOFSTEP]
rw [generalizedEigenspace, OrderHom.coe_mk, ← LinearMap.ker_comp]
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ LinearMap.ker
(LinearMap.comp ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V)
((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V)) =
LinearMap.ker ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V * (f - ↑(algebraMap K (End K V)) μ) ^ finrank K V)
[PROOFSTEP]
rfl
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ LinearMap.ker ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V * (f - ↑(algebraMap K (End K V)) μ) ^ finrank K V) =
↑(generalizedEigenspace f μ) (finrank K V + finrank K V)
[PROOFSTEP]
rw [← pow_add]
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ LinearMap.ker ((f - ↑(algebraMap K (End K V)) μ) ^ (finrank K V + finrank K V)) =
↑(generalizedEigenspace f μ) (finrank K V + finrank K V)
[PROOFSTEP]
rfl
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ ↑(generalizedEigenspace f μ) (finrank K V + finrank K V) = ↑(generalizedEigenspace f μ) (finrank K V)
[PROOFSTEP]
rw [generalizedEigenspace_eq_generalizedEigenspace_finrank_of_le]
[GOAL]
case hk
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
⊢ finrank K V ≤ finrank K V + finrank K V
[PROOFSTEP]
linarith
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
h :
Submodule.comap ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V) (↑(generalizedEigenspace f μ) (finrank K V)) =
↑(generalizedEigenspace f μ) (finrank K V)
⊢ Disjoint (generalizedEigenrange f μ (finrank K V)) (↑(generalizedEigenspace f μ) (finrank K V))
[PROOFSTEP]
rw [disjoint_iff_inf_le, generalizedEigenrange, LinearMap.range_eq_map, Submodule.map_inf_eq_map_inf_comap, top_inf_eq,
h]
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
μ : K
h :
Submodule.comap ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V) (↑(generalizedEigenspace f μ) (finrank K V)) =
↑(generalizedEigenspace f μ) (finrank K V)
⊢ Submodule.map ((f - ↑(algebraMap K (End K V)) μ) ^ finrank K V) (↑(generalizedEigenspace f μ) (finrank K V)) ≤ ⊥
[PROOFSTEP]
apply Submodule.map_comap_le
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
μ : R
hμp : Disjoint (eigenspace f μ) p
⊢ eigenspace (LinearMap.restrict f hfp) μ = ⊥
[PROOFSTEP]
rw [eq_bot_iff]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
μ : R
hμp : Disjoint (eigenspace f μ) p
⊢ eigenspace (LinearMap.restrict f hfp) μ ≤ ⊥
[PROOFSTEP]
intro x hx
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End R M
p : Submodule R M
hfp : ∀ (x : M), x ∈ p → ↑f x ∈ p
μ : R
hμp : Disjoint (eigenspace f μ) p
x : { x // x ∈ p }
hx : x ∈ eigenspace (LinearMap.restrict f hfp) μ
⊢ x ∈ ⊥
[PROOFSTEP]
simpa using hμp.le_bot ⟨eigenspace_restrict_le_eigenspace f hfp μ ⟨x, hx, rfl⟩, x.prop⟩
[GOAL]
K R : Type v
V M : Type w
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R M
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : FiniteDimensional K V
f : End K V
k : ℕ
μ : K
hx : HasEigenvalue f μ
hk : 0 < k
⊢ 0 = finrank K { x // x ∈ ⊥ }
[PROOFSTEP]
rw [finrank_bot]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
μ : K
n : ℕ
⊢ Submodule.map f (generalizedEigenrange f μ n) = LinearMap.range (f * (f - ↑(algebraMap K (End K V)) μ) ^ n)
[PROOFSTEP]
rw [generalizedEigenrange]
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
μ : K
n : ℕ
⊢ Submodule.map f (LinearMap.range ((f - ↑(algebraMap K (End K V)) μ) ^ n)) =
LinearMap.range (f * (f - ↑(algebraMap K (End K V)) μ) ^ n)
[PROOFSTEP]
exact (LinearMap.range_comp _ _).symm
[GOAL]
K R : Type v
V M : Type w
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
f : End K V
μ : K
n : ℕ
⊢ LinearMap.range (f * (f - ↑(algebraMap K (End K V)) μ) ^ n) =
LinearMap.range ((f - ↑(algebraMap K (End K V)) μ) ^ n * f)
[PROOFSTEP]
rw [Algebra.mul_sub_algebraMap_pow_commutes]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Eigenspace.Basic", "llama_tokens": 42678} |
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ 1 ≤ evenOdd Q 0
[PROOFSTEP]
refine' le_trans _ (le_iSup _ ⟨0, Nat.cast_zero⟩)
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ 1 ≤ LinearMap.range (ι Q) ^ ↑{ val := 0, property := (_ : ↑0 = 0) }
[PROOFSTEP]
exact (pow_zero _).ge
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ LinearMap.range (ι Q) ≤ evenOdd Q 1
[PROOFSTEP]
refine' le_trans _ (le_iSup _ ⟨1, Nat.cast_one⟩)
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ LinearMap.range (ι Q) ≤ LinearMap.range (ι Q) ^ ↑{ val := 1, property := (_ : ↑1 = 1) }
[PROOFSTEP]
exact (pow_one _).ge
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁ m₂ : M
⊢ ↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) ^ ↑{ val := 2, property := (_ : ↑2 = ↑2) }
[PROOFSTEP]
rw [Subtype.coe_mk, pow_two]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁ m₂ : M
⊢ ↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
[PROOFSTEP]
exact Submodule.mul_mem_mul (LinearMap.mem_range_self (ι Q) m₁) (LinearMap.mem_range_self (ι Q) m₂)
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
⊢ evenOdd Q i * evenOdd Q j ≤ evenOdd Q (i + j)
[PROOFSTEP]
simp_rw [evenOdd, Submodule.iSup_eq_span, Submodule.span_mul_span]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
⊢ Submodule.span R
((⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)) *
⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)) ≤
Submodule.span R (⋃ (i_1 : { n // ↑n = i + j }), ↑(LinearMap.range (ι Q) ^ ↑i_1))
[PROOFSTEP]
apply Submodule.span_mono
[GOAL]
case h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
⊢ (⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)) *
⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i) ⊆
⋃ (i_1 : { n // ↑n = i + j }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
[PROOFSTEP]
intro z hz
[GOAL]
case h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
z : CliffordAlgebra Q
hz :
z ∈
(⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)) *
⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
⊢ z ∈ ⋃ (i_1 : { n // ↑n = i + j }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
[PROOFSTEP]
obtain ⟨x, y, hx, hy, rfl⟩ := hz
[GOAL]
case h.intro.intro.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
x y : CliffordAlgebra Q
hx : x ∈ ⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
hy : y ∈ ⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
⊢ (fun x x_1 => x * x_1) x y ∈ ⋃ (i_1 : { n // ↑n = i + j }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
[PROOFSTEP]
obtain ⟨xi, hx'⟩ := Set.mem_iUnion.mp hx
[GOAL]
case h.intro.intro.intro.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
x y : CliffordAlgebra Q
hx : x ∈ ⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
hy : y ∈ ⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
xi : { n // ↑n = i }
hx' : x ∈ ↑(LinearMap.range (ι Q) ^ ↑xi)
⊢ (fun x x_1 => x * x_1) x y ∈ ⋃ (i_1 : { n // ↑n = i + j }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
[PROOFSTEP]
obtain ⟨yi, hy'⟩ := Set.mem_iUnion.mp hy
[GOAL]
case h.intro.intro.intro.intro.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
x y : CliffordAlgebra Q
hx : x ∈ ⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
hy : y ∈ ⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
xi : { n // ↑n = i }
hx' : x ∈ ↑(LinearMap.range (ι Q) ^ ↑xi)
yi : { n // ↑n = j }
hy' : y ∈ ↑(LinearMap.range (ι Q) ^ ↑yi)
⊢ (fun x x_1 => x * x_1) x y ∈ ⋃ (i_1 : { n // ↑n = i + j }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
[PROOFSTEP]
refine' Set.mem_iUnion.mpr ⟨⟨xi + yi, by simp only [Nat.cast_add, xi.prop, yi.prop]⟩, _⟩
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
x y : CliffordAlgebra Q
hx : x ∈ ⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
hy : y ∈ ⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
xi : { n // ↑n = i }
hx' : x ∈ ↑(LinearMap.range (ι Q) ^ ↑xi)
yi : { n // ↑n = j }
hy' : y ∈ ↑(LinearMap.range (ι Q) ^ ↑yi)
⊢ ↑(↑xi + ↑yi) = i + j
[PROOFSTEP]
simp only [Nat.cast_add, xi.prop, yi.prop]
[GOAL]
case h.intro.intro.intro.intro.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
x y : CliffordAlgebra Q
hx : x ∈ ⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
hy : y ∈ ⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
xi : { n // ↑n = i }
hx' : x ∈ ↑(LinearMap.range (ι Q) ^ ↑xi)
yi : { n // ↑n = j }
hy' : y ∈ ↑(LinearMap.range (ι Q) ^ ↑yi)
⊢ (fun x x_1 => x * x_1) x y ∈ ↑(LinearMap.range (ι Q) ^ ↑{ val := ↑xi + ↑yi, property := (_ : ↑(↑xi + ↑yi) = i + j) })
[PROOFSTEP]
simp only [Subtype.coe_mk, Nat.cast_add, pow_add]
[GOAL]
case h.intro.intro.intro.intro.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i j : ZMod 2
x y : CliffordAlgebra Q
hx : x ∈ ⋃ (i_1 : { n // ↑n = i }), ↑(LinearMap.range (ι Q) ^ ↑i_1)
hy : y ∈ ⋃ (i : { n // ↑n = j }), ↑(LinearMap.range (ι Q) ^ ↑i)
xi : { n // ↑n = i }
hx' : x ∈ ↑(LinearMap.range (ι Q) ^ ↑xi)
yi : { n // ↑n = j }
hy' : y ∈ ↑(LinearMap.range (ι Q) ^ ↑yi)
⊢ x * y ∈ ↑(LinearMap.range (ι Q) ^ ↑xi * LinearMap.range (ι Q) ^ ↑yi)
[PROOFSTEP]
exact Submodule.mul_mem_mul hx' hy'
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m = ↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)
[PROOFSTEP]
rw [GradedAlgebra.ι_apply Q, DirectSum.of_mul_of, DirectSum.algebraMap_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) (1 + 1))
(GradedMonoid.GMul.mul { val := ↑(ι Q) m, property := (_ : ↑(ι Q) m ∈ evenOdd Q 1) }
{ val := ↑(ι Q) m, property := (_ : ↑(ι Q) m ∈ evenOdd Q 1) }) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) 0) (↑DirectSum.GAlgebra.toFun (↑Q m))
[PROOFSTEP]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext rfl <| ι_sq_scalar _ _)
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : { x // x ∈ evenOdd Q i' }
⊢ M →ₗ[R] ⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i }
[PROOFSTEP]
apply GradedAlgebra.ι Q
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : { x // x ∈ evenOdd Q i' }
⊢ ∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m = ↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)
[PROOFSTEP]
apply GradedAlgebra.ι_sq_scalar Q
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : { x // x ∈ evenOdd Q i' }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
↑x' =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') x'
[PROOFSTEP]
cases' x' with x' hx'
[GOAL]
case mk
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
hx' : x' ∈ evenOdd Q i'
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
↑{ val := x', property := hx' } =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := x', property := hx' }
[PROOFSTEP]
dsimp only [Subtype.coe_mk, DirectSum.lof_eq_of]
[GOAL]
case mk
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
hx' : x' ∈ evenOdd Q i'
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x' =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := x', property := hx' }
[PROOFSTEP]
induction hx' using Submodule.iSup_induction' with
| hp i x hx =>
obtain ⟨i, rfl⟩ := i
change x ∈ LinearMap.range (ι Q) ^ i at hx
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy =>
rw [AlgHom.map_add, ihx, ihy, ← map_add]
rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _) <;> dsimp only [GradedMonoid.mk, Subtype.coe_mk]
· rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
rfl
| h0 =>
rw [AlgHom.map_zero]
apply Eq.symm
apply DFinsupp.single_eq_zero.mpr; rfl
| hadd x y hx hy ihx ihy => rw [AlgHom.map_add, ihx, ihy, ← map_add]; rfl
[GOAL]
case mk
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
hx' : x' ∈ evenOdd Q i'
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x' =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := x', property := hx' }
[PROOFSTEP]
induction hx' using Submodule.iSup_induction' with
| hp i x hx =>
obtain ⟨i, rfl⟩ := i
change x ∈ LinearMap.range (ι Q) ^ i at hx
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy =>
rw [AlgHom.map_add, ihx, ihy, ← map_add]
rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _) <;> dsimp only [GradedMonoid.mk, Subtype.coe_mk]
· rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
rfl
| h0 =>
rw [AlgHom.map_zero]
apply Eq.symm
apply DFinsupp.single_eq_zero.mpr; rfl
| hadd x y hx hy ihx ihy => rw [AlgHom.map_add, ihx, ihy, ← map_add]; rfl
[GOAL]
case mk.hp
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
i : { n // ↑n = i' }
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ ↑i
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := x, property := (_ : x ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
| hp i x hx =>
obtain ⟨i, rfl⟩ := i
change x ∈ LinearMap.range (ι Q) ^ i at hx
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy =>
rw [AlgHom.map_add, ihx, ihy, ← map_add]
rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _) <;> dsimp only [GradedMonoid.mk, Subtype.coe_mk]
· rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
rfl
[GOAL]
case mk.hp
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
i : { n // ↑n = i' }
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ ↑i
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := x, property := (_ : x ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
obtain ⟨i, rfl⟩ := i
[GOAL]
case mk.hp.mk
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x : CliffordAlgebra Q
i : ℕ
hx : x ∈ LinearMap.range (ι Q) ^ ↑{ val := i, property := (_ : ↑i = ↑i) }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
change x ∈ LinearMap.range (ι Q) ^ i at hx
[GOAL]
case mk.hp.mk
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x : CliffordAlgebra Q
i : ℕ
hx : x ∈ LinearMap.range (ι Q) ^ i
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy =>
rw [AlgHom.map_add, ihx, ihy, ← map_add]
rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _) <;> dsimp only [GradedMonoid.mk, Subtype.coe_mk]
· rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
rfl
[GOAL]
case mk.hp.mk
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x : CliffordAlgebra Q
i : ℕ
hx : x ∈ LinearMap.range (ι Q) ^ i
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy =>
rw [AlgHom.map_add, ihx, ihy, ← map_add]
rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _) <;> dsimp only [GradedMonoid.mk, Subtype.coe_mk]
· rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
rfl
[GOAL]
case mk.hp.mk.hr
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x : CliffordAlgebra Q
i : ℕ
r : R
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(↑(algebraMap R (CliffordAlgebra Q)) r) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑0)
{ val := ↑(algebraMap R (CliffordAlgebra Q)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ ⨆ (i : { n // ↑n = ↑0 }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
[GOAL]
case mk.hp.mk.hr
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x : CliffordAlgebra Q
i : ℕ
r : R
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(↑(algebraMap R (CliffordAlgebra Q)) r) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑0)
{ val := ↑(algebraMap R (CliffordAlgebra Q)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ ⨆ (i : { n // ↑n = ↑0 }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
rw [AlgHom.commutes, DirectSum.algebraMap_apply]
[GOAL]
case mk.hp.mk.hr
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x : CliffordAlgebra Q
i : ℕ
r : R
⊢ ↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) 0) (↑DirectSum.GAlgebra.toFun r) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑0)
{ val := ↑(algebraMap R (CliffordAlgebra Q)) r,
property := (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ ⨆ (i : { n // ↑n = ↑0 }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
rfl
[GOAL]
case mk.hp.mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ : ℕ
x y : CliffordAlgebra Q
i : ℕ
hx : x ∈ LinearMap.range (ι Q) ^ i
hy : y ∈ LinearMap.range (ι Q) ^ i
ihx :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
ihy :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
y =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := y, property := (_ : y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(x + y) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x + y, property := (_ : x + y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
| hadd x y i hx hy ihx ihy =>
rw [AlgHom.map_add, ihx, ihy, ← map_add]
rfl
[GOAL]
case mk.hp.mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ : ℕ
x y : CliffordAlgebra Q
i : ℕ
hx : x ∈ LinearMap.range (ι Q) ^ i
hy : y ∈ LinearMap.range (ι Q) ^ i
ihx :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
ihy :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
y =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := y, property := (_ : y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(x + y) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x + y, property := (_ : x + y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
rw [AlgHom.map_add, ihx, ihy, ← map_add]
[GOAL]
case mk.hp.mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ : ℕ
x y : CliffordAlgebra Q
i : ℕ
hx : x ∈ LinearMap.range (ι Q) ^ i
hy : y ∈ LinearMap.range (ι Q) ^ i
ihx :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
ihy :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
y =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := y, property := (_ : y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
⊢ ↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
({ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) } +
{ val := y, property := (_ : y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x + y, property := (_ : x + y ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
rfl
[GOAL]
case mk.hp.mk.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ : ℕ
m : CliffordAlgebra Q
hm : m ∈ LinearMap.range (ι Q)
i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(m * x) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑(Nat.succ i))
{ val := m * x, property := (_ : m * x ∈ ⨆ (i_1 : { n // ↑n = ↑(Nat.succ i) }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _) <;> dsimp only [GradedMonoid.mk, Subtype.coe_mk]
· rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
rfl
[GOAL]
case mk.hp.mk.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ : ℕ
m : CliffordAlgebra Q
hm : m ∈ LinearMap.range (ι Q)
i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(m * x) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑(Nat.succ i))
{ val := m * x, property := (_ : m * x ∈ ⨆ (i_1 : { n // ↑n = ↑(Nat.succ i) }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
obtain ⟨_, rfl⟩ := hm
[GOAL]
case mk.hp.mk.hmul.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
w✝ : M
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(↑(ι Q) w✝ * x) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑(Nat.succ i))
{ val := ↑(ι Q) w✝ * x,
property := (_ : ↑(ι Q) w✝ * x ∈ ⨆ (i_1 : { n // ↑n = ↑(Nat.succ i) }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.of_mul_of]
[GOAL]
case mk.hp.mk.hmul.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
w✝ : M
⊢ ↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) (1 + ↑i))
(GradedMonoid.GMul.mul { val := ↑(ι Q) w✝, property := (_ : ↑(ι Q) w✝ ∈ evenOdd Q 1) }
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑(Nat.succ i))
{ val := ↑(ι Q) w✝ * x,
property := (_ : ↑(ι Q) w✝ * x ∈ ⨆ (i_1 : { n // ↑n = ↑(Nat.succ i) }), LinearMap.range (ι Q) ^ ↑i_1) }
[PROOFSTEP]
refine' DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext _ _)
[GOAL]
case mk.hp.mk.hmul.intro.refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
w✝ : M
⊢ (GradedMonoid.mk (1 + ↑i)
(GradedMonoid.GMul.mul { val := ↑(ι Q) w✝, property := (_ : ↑(ι Q) w✝ ∈ evenOdd Q 1) }
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) })).fst =
(GradedMonoid.mk ↑(Nat.succ i)
{ val := ↑(ι Q) w✝ * x,
property := (_ : ↑(ι Q) w✝ * x ∈ ⨆ (i_1 : { n // ↑n = ↑(Nat.succ i) }), LinearMap.range (ι Q) ^ ↑i_1) }).fst
[PROOFSTEP]
dsimp only [GradedMonoid.mk, Subtype.coe_mk]
[GOAL]
case mk.hp.mk.hmul.intro.refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
w✝ : M
⊢ ↑(GradedMonoid.mk (1 + ↑i)
(GradedMonoid.GMul.mul { val := ↑(ι Q) w✝, property := (_ : ↑(ι Q) w✝ ∈ evenOdd Q 1) }
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) })).snd =
↑(GradedMonoid.mk ↑(Nat.succ i)
{ val := ↑(ι Q) w✝ * x,
property := (_ : ↑(ι Q) w✝ * x ∈ ⨆ (i_1 : { n // ↑n = ↑(Nat.succ i) }), LinearMap.range (ι Q) ^ ↑i_1) }).snd
[PROOFSTEP]
dsimp only [GradedMonoid.mk, Subtype.coe_mk]
[GOAL]
case mk.hp.mk.hmul.intro.refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
w✝ : M
⊢ 1 + ↑i = ↑(Nat.succ i)
[PROOFSTEP]
rw [Nat.succ_eq_add_one, add_comm, Nat.cast_add, Nat.cast_one]
[GOAL]
case mk.hp.mk.hmul.intro.refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x' x✝ : CliffordAlgebra Q
i✝ i : ℕ
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ i
ih :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) ↑i)
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }
w✝ : M
⊢ ↑(GradedMonoid.GMul.mul { val := ↑(ι Q) w✝, property := (_ : ↑(ι Q) w✝ ∈ evenOdd Q 1) }
{ val := x, property := (_ : x ∈ ⨆ (i_1 : { n // ↑n = ↑i }), LinearMap.range (ι Q) ^ ↑i_1) }) =
↑(ι Q) w✝ * x
[PROOFSTEP]
rfl
[GOAL]
case mk.h0
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
0 =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := 0, property := (_ : 0 ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
| h0 =>
rw [AlgHom.map_zero]
apply Eq.symm
apply DFinsupp.single_eq_zero.mpr; rfl
[GOAL]
case mk.h0
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
0 =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := 0, property := (_ : 0 ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
rw [AlgHom.map_zero]
[GOAL]
case mk.h0
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
⊢ 0 =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := 0, property := (_ : 0 ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
apply Eq.symm
[GOAL]
case mk.h0.h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
⊢ ↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := 0, property := (_ : 0 ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) } =
0
[PROOFSTEP]
apply DFinsupp.single_eq_zero.mpr
[GOAL]
case mk.h0.h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' : CliffordAlgebra Q
⊢ { val := 0, property := (_ : 0 ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) } = 0
[PROOFSTEP]
rfl
[GOAL]
case mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' x y : CliffordAlgebra Q
hx : x ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i
hy : y ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i
ihx :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := x, property := hx }
ihy :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
y =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := y, property := hy }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(x + y) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := x + y, property := (_ : x + y ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
| hadd x y hx hy ihx ihy => rw [AlgHom.map_add, ihx, ihy, ← map_add]; rfl
[GOAL]
case mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' x y : CliffordAlgebra Q
hx : x ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i
hy : y ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i
ihx :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := x, property := hx }
ihy :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
y =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := y, property := hy }
⊢ ↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(x + y) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := x + y, property := (_ : x + y ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
rw [AlgHom.map_add, ihx, ihy, ← map_add]
[GOAL]
case mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
i' : ZMod 2
x' x y : CliffordAlgebra Q
hx : x ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i
hy : y ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i
ihx :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := x, property := hx }
ihy :
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
y =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') { val := y, property := hy }
⊢ ↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i') ({ val := x, property := hx } + { val := y, property := hy }) =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i')
{ val := x + y, property := (_ : x + y ∈ ⨆ (i : { n // ↑n = i' }), LinearMap.range (ι Q) ^ ↑i) }
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ M →ₗ[R] ⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i }
[PROOFSTEP]
apply GradedAlgebra.ι Q
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ ∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m = ↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)
[PROOFSTEP]
apply GradedAlgebra.ι_sq_scalar Q
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ AlgHom.comp (DirectSum.coeAlgHom (evenOdd Q))
(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) }) =
AlgHom.id R (CliffordAlgebra Q)
[PROOFSTEP]
ext m
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(LinearMap.comp
(AlgHom.toLinearMap
(AlgHom.comp (DirectSum.coeAlgHom (evenOdd Q))
(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })))
(ι Q))
m =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (CliffordAlgebra Q))) (ι Q)) m
[PROOFSTEP]
dsimp only [LinearMap.comp_apply, AlgHom.toLinearMap_apply, AlgHom.comp_apply, AlgHom.id_apply]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(DirectSum.coeAlgHom (evenOdd Q))
(↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
(↑(ι Q) m)) =
↑(ι Q) m
[PROOFSTEP]
rw [lift_ι_apply, GradedAlgebra.ι_apply Q, DirectSum.coeAlgHom_of, Subtype.coe_mk]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ ∀ (i : ZMod 2) (x : { x // x ∈ evenOdd Q i }),
↑(↑(lift Q)
{ val := GradedAlgebra.ι Q,
property :=
(_ :
∀ (m : M),
↑(GradedAlgebra.ι Q) m * ↑(GradedAlgebra.ι Q) m =
↑(algebraMap R (⨁ (i : ZMod 2), { x // x ∈ evenOdd Q i })) (↑Q m)) })
↑x =
↑(DirectSum.of (fun i => { x // x ∈ evenOdd Q i }) i) x
[PROOFSTEP]
apply GradedAlgebra.lift_ι_eq Q
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ ⨆ (i : ℕ), LinearMap.range (ι Q) ^ i = ⊤
[PROOFSTEP]
rw [← (DirectSum.Decomposition.isInternal (evenOdd Q)).submodule_iSup_eq_top, eq_comm]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ iSup (evenOdd Q) = ⨆ (i : ℕ), LinearMap.range (ι Q) ^ i
[PROOFSTEP]
calc
-- porting note: needs extra annotations, no longer unifies against the goal in the face of
-- ambiguity
⨆ (i : ZMod 2) (j : { n : ℕ // ↑n = i }), LinearMap.range (ι Q) ^ (j : ℕ) =
⨆ i : Σ i : ZMod 2, { n : ℕ // ↑n = i }, LinearMap.range (ι Q) ^ (i.2 : ℕ) :=
by rw [iSup_sigma]
_ = ⨆ i : ℕ, LinearMap.range (ι Q) ^ i :=
Function.Surjective.iSup_congr (fun i => i.2) (fun i => ⟨⟨_, i, rfl⟩, rfl⟩) fun _ => rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ ⨆ (i : ZMod 2) (j : { n // ↑n = i }), LinearMap.range (ι Q) ^ ↑j =
⨆ (i : (i : ZMod 2) × { n // ↑n = i }), LinearMap.range (ι Q) ^ ↑i.snd
[PROOFSTEP]
rw [iSup_sigma]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ Set.univ = {0, 1}
[PROOFSTEP]
have : (Finset.univ : Finset (ZMod 2)) = {0, 1} := rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
this : Finset.univ = {0, 1}
⊢ Set.univ = {0, 1}
[PROOFSTEP]
simpa using congr_arg ((↑) : Finset (ZMod 2) → Set (ZMod 2)) this
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
⊢ P x hx
[PROOFSTEP]
apply Submodule.iSup_induction' (C := P) _ (hr 0 (Submodule.zero_mem _)) @hadd
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
⊢ ∀ (i : { n_1 // ↑n_1 = n }) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ ↑i),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
refine'
Subtype.rec
_
-- porting note: was `simp_rw [Subtype.coe_mk, ZMod.nat_coe_zmod_eq_iff, add_comm n.val]`
-- leanprover/lean4#1926 is to blame.
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
⊢ ∀ (val : ℕ) (property : ↑val = n) (x : CliffordAlgebra Q)
(hx : x ∈ LinearMap.range (ι Q) ^ ↑{ val := val, property := property }),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
dsimp only [Subtype.coe_mk]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
⊢ ∀ (val : ℕ) (property : ↑val = n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
let hlean1926 : ∀ val : ℕ, ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
by
intro val
simp_rw [ZMod.nat_coe_zmod_eq_iff, add_comm n.val]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
⊢ ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n
[PROOFSTEP]
intro val
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
val : ℕ
⊢ ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n
[PROOFSTEP]
simp_rw [ZMod.nat_coe_zmod_eq_iff, add_comm n.val]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
⊢ ∀ (val : ℕ) (property : ↑val = n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
have := fun val : ℕ =>
forall_prop_congr' (q := fun property =>
∀ x (hx : x ∈ LinearMap.range (ι Q) ^ val), P x (Submodule.mem_iSup_of_mem { val := val, property := property } hx))
(hq := fun property => Iff.rfl) (hp := hlean1926 val)
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
this :
∀ (val : ℕ),
(∀ (h : ↑val = n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)) =
∀ (h : ∃ k, val = 2 * k + ZMod.val n),
(fun property =>
∀ (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i))
(_ : ↑val = n)
⊢ ∀ (val : ℕ) (property : ↑val = n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
simp_rw [this]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
this :
∀ (val : ℕ),
(∀ (h : ↑val = n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)) =
∀ (h : ∃ k, val = 2 * k + ZMod.val n),
(fun property =>
∀ (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i))
(_ : ↑val = n)
⊢ ∀ (val : ℕ) (h : ∃ k, val = 2 * k + ZMod.val n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
clear this
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
⊢ ∀ (val : ℕ) (h : ∃ k, val = 2 * k + ZMod.val n) (x : CliffordAlgebra Q) (hx : x ∈ LinearMap.range (ι Q) ^ val),
P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
rintro n' ⟨k, rfl⟩ xv
[GOAL]
case intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv : CliffordAlgebra Q
⊢ ∀ (hx : xv ∈ LinearMap.range (ι Q) ^ (2 * k + ZMod.val n)),
P xv (_ : xv ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl)
(show
xv ∈ LinearMap.range (ι Q) ^ (2 * k + ZMod.val n) ↔
xv ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
by simp_rw [pow_add, pow_mul])).mpr
?_
-- end porting note
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv : CliffordAlgebra Q
⊢ xv ∈ LinearMap.range (ι Q) ^ (2 * k + ZMod.val n) ↔
xv ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
[PROOFSTEP]
simp_rw [pow_add, pow_mul]
[GOAL]
case intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv : CliffordAlgebra Q
⊢ ∀ (h : xv ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n),
P xv (_ : xv ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
intro hxv
[GOAL]
case intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv : CliffordAlgebra Q
hxv : xv ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
⊢ P xv (_ : xv ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
induction hxv using Submodule.mul_induction_on' with
| hm a ha b hb =>
induction ha using Submodule.pow_induction_on_left' with
| hr r =>
simp_rw [← Algebra.smul_def]
exact hr _ (Submodule.smul_mem _ _ hb)
| hadd x y n hx hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| hmul x hx n'' y hy ihy =>
revert hx
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by
rw [pow_two]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
intro hx2
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| ha x y hx hy ihx ihy => apply hadd ihx ihy
[GOAL]
case intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv : CliffordAlgebra Q
hxv : xv ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
⊢ P xv (_ : xv ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
induction hxv using Submodule.mul_induction_on' with
| hm a ha b hb =>
induction ha using Submodule.pow_induction_on_left' with
| hr r =>
simp_rw [← Algebra.smul_def]
exact hr _ (Submodule.smul_mem _ _ hb)
| hadd x y n hx hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| hmul x hx n'' y hy ihy =>
revert hx
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by
rw [pow_two]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
intro hx2
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| ha x y hx hy ihx ihy => apply hadd ihx ihy
[GOAL]
case intro.hm
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a : CliffordAlgebra Q
ha : a ∈ (LinearMap.range (ι Q) ^ 2) ^ k
b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
⊢ P (a * b) (_ : a * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| hm a ha b hb =>
induction ha using Submodule.pow_induction_on_left' with
| hr r =>
simp_rw [← Algebra.smul_def]
exact hr _ (Submodule.smul_mem _ _ hb)
| hadd x y n hx hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| hmul x hx n'' y hy ihy =>
revert hx
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by
rw [pow_two]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
intro hx2
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a : CliffordAlgebra Q
ha : a ∈ (LinearMap.range (ι Q) ^ 2) ^ k
b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
⊢ P (a * b) (_ : a * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
induction ha using Submodule.pow_induction_on_left' with
| hr r =>
simp_rw [← Algebra.smul_def]
exact hr _ (Submodule.smul_mem _ _ hb)
| hadd x y n hx hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| hmul x hx n'' y hy ihy =>
revert hx
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by rw [pow_two]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
intro hx2
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a : CliffordAlgebra Q
ha : a ∈ (LinearMap.range (ι Q) ^ 2) ^ k
b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
⊢ P (a * b) (_ : a * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
induction ha using Submodule.pow_induction_on_left' with
| hr r =>
simp_rw [← Algebra.smul_def]
exact hr _ (Submodule.smul_mem _ _ hb)
| hadd x y n hx hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
| hmul x hx n'' y hy ihy =>
revert hx
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by rw [pow_two]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
intro hx2
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm.hr
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
r : R
⊢ P (↑(algebraMap R (CliffordAlgebra Q)) r * b)
(_ : ↑(algebraMap R (CliffordAlgebra Q)) r * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| hr r =>
simp_rw [← Algebra.smul_def]
exact hr _ (Submodule.smul_mem _ _ hb)
[GOAL]
case intro.hm.hr
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
r : R
⊢ P (↑(algebraMap R (CliffordAlgebra Q)) r * b)
(_ : ↑(algebraMap R (CliffordAlgebra Q)) r * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
simp_rw [← Algebra.smul_def]
[GOAL]
case intro.hm.hr
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
r : R
⊢ P (r • b) (_ : r • b ∈ evenOdd Q n)
[PROOFSTEP]
exact hr _ (Submodule.smul_mem _ _ hb)
[GOAL]
case intro.hm.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x y : CliffordAlgebra Q
n : ℕ
hx : x ∈ (LinearMap.range (ι Q) ^ 2) ^ n
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n
ihx : P (x * b) (_ : x * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
⊢ P ((x + y) * b) (_ : (x + y) * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| hadd x y n hx hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x y : CliffordAlgebra Q
n : ℕ
hx : x ∈ (LinearMap.range (ι Q) ^ 2) ^ n
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n
ihx : P (x * b) (_ : x * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
⊢ P ((x + y) * b) (_ : (x + y) * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
simp_rw [add_mul]
[GOAL]
case intro.hm.hadd
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x y : CliffordAlgebra Q
n : ℕ
hx : x ∈ (LinearMap.range (ι Q) ^ 2) ^ n
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n
ihx : P (x * b) (_ : x * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
⊢ P (x * b + y * b) (_ : x * b + y * b ∈ evenOdd Q n✝)
[PROOFSTEP]
apply hadd ihx ihy
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ 2
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
⊢ P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| hmul x hx n'' y hy ihy =>
revert hx
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by rw [pow_two]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
intro hx2
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) ^ 2
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
⊢ P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
revert hx
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
⊢ ∀ (hx : x ∈ LinearMap.range (ι Q) ^ 2),
P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
let hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) := by rw [pow_two]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
⊢ x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
[PROOFSTEP]
rw [pow_two]
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ ∀ (hx : x ∈ LinearMap.range (ι Q) ^ 2),
P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
refine
(forall_prop_congr' (hq := fun property => Iff.rfl) hlean1926'').mpr
?_
-- end porting note
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ ∀ (h : x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)),
P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
intro hx2
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
hx2 : x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
⊢ P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm.hmul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
hx2 : x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
⊢ P (x * y * b) (_ : x * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
induction hx2 using Submodule.mul_induction_on' with
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm.hmul.hm
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
m : CliffordAlgebra Q
hm : m ∈ LinearMap.range (ι Q)
n : CliffordAlgebra Q
hn : n ∈ LinearMap.range (ι Q)
hlean1926'' : m * n ∈ LinearMap.range (ι Q) ^ 2 ↔ m * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (m * n ∈ LinearMap.range (ι Q) ^ 2 ↔ m * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P (m * n * y * b) (_ : m * n * y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| hm m hm n hn =>
simp_rw [LinearMap.mem_range] at hm hn
obtain ⟨m₁, rfl⟩ := hm; obtain ⟨m₂, rfl⟩ := hn
simp_rw [mul_assoc _ y b]
refine' hιι_mul _ _ ihy
[GOAL]
case intro.hm.hmul.hm
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
m : CliffordAlgebra Q
hm : m ∈ LinearMap.range (ι Q)
n : CliffordAlgebra Q
hn : n ∈ LinearMap.range (ι Q)
hlean1926'' : m * n ∈ LinearMap.range (ι Q) ^ 2 ↔ m * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (m * n ∈ LinearMap.range (ι Q) ^ 2 ↔ m * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P (m * n * y * b) (_ : m * n * y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
simp_rw [LinearMap.mem_range] at hm hn
[GOAL]
case intro.hm.hmul.hm
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
m : CliffordAlgebra Q
hm✝ : m ∈ LinearMap.range (ι Q)
n : CliffordAlgebra Q
hn✝ : n ∈ LinearMap.range (ι Q)
hlean1926'' : m * n ∈ LinearMap.range (ι Q) ^ 2 ↔ m * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (m * n ∈ LinearMap.range (ι Q) ^ 2 ↔ m * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
hm : ∃ y, ↑(ι Q) y = m
hn : ∃ y, ↑(ι Q) y = n
⊢ P (m * n * y * b) (_ : m * n * y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
obtain ⟨m₁, rfl⟩ := hm
[GOAL]
case intro.hm.hmul.hm.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n✝ : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n✝ → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n✝),
P v (_ : v ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝} {hy : y ∈ evenOdd Q n✝},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n✝)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n✝},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n✝)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n✝
hlean1926 : ∀ (val : ℕ), ↑val = n✝ ↔ ∃ k, val = 2 * k + ZMod.val n✝ :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n✝)) (∃ k, val = 2 * k + ZMod.val n✝)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n✝) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n✝))
(iff_self (∃ k, val = 2 * k + ZMod.val n✝))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n✝
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
n : CliffordAlgebra Q
hn✝ : n ∈ LinearMap.range (ι Q)
hn : ∃ y, ↑(ι Q) y = n
m₁ : M
hm : ↑(ι Q) m₁ ∈ LinearMap.range (ι Q)
hlean1926'' : ↑(ι Q) m₁ * n ∈ LinearMap.range (ι Q) ^ 2 ↔
↑(ι Q) m₁ * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl
(↑(ι Q) m₁ * n ∈ LinearMap.range (ι Q) ^ 2 ↔ ↑(ι Q) m₁ * n ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P (↑(ι Q) m₁ * n * y * b) (_ : ↑(ι Q) m₁ * n * y * b ∈ ⨆ (i : { n // ↑n = n✝ }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
obtain ⟨m₂, rfl⟩ := hn
[GOAL]
case intro.hm.hmul.hm.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
m₁ : M
hm : ↑(ι Q) m₁ ∈ LinearMap.range (ι Q)
m₂ : M
hn : ↑(ι Q) m₂ ∈ LinearMap.range (ι Q)
hlean1926'' : ↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) ^ 2 ↔
↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl
(↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) ^ 2 ↔
↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P (↑(ι Q) m₁ * ↑(ι Q) m₂ * y * b)
(_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
simp_rw [mul_assoc _ y b]
[GOAL]
case intro.hm.hmul.hm.intro.intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x : CliffordAlgebra Q
n'' : ℕ
y : CliffordAlgebra Q
hy : y ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy : P (y * b) (_ : y * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
m₁ : M
hm : ↑(ι Q) m₁ ∈ LinearMap.range (ι Q)
m₂ : M
hn : ↑(ι Q) m₂ ∈ LinearMap.range (ι Q)
hlean1926'' : ↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) ^ 2 ↔
↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl
(↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) ^ 2 ↔
↑(ι Q) m₁ * ↑(ι Q) m₂ ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P (↑(ι Q) m₁ * ↑(ι Q) m₂ * (y * b)) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * (y * b) ∈ evenOdd Q n)
[PROOFSTEP]
refine' hιι_mul _ _ ihy
[GOAL]
case intro.hm.hmul.ha
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝¹ : CliffordAlgebra Q
hx✝ : x✝¹ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x✝ : CliffordAlgebra Q
n'' : ℕ
y✝ : CliffordAlgebra Q
hy✝ : y✝ ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy✝ : P (y✝ * b) (_ : y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
y : CliffordAlgebra Q
hy : y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
ihx :
let hlean1926'' := (_ : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q));
P (x * y✝ * b) (_ : x * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
ihy :
let hlean1926'' := (_ : y ∈ LinearMap.range (ι Q) ^ 2 ↔ y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q));
P (y * y✝ * b) (_ : y * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x + y ∈ LinearMap.range (ι Q) ^ 2 ↔ x + y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x + y ∈ LinearMap.range (ι Q) ^ 2 ↔ x + y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P ((x + y) * y✝ * b) (_ : (x + y) * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| ha x hx y hy ihx ihy =>
simp_rw [add_mul]
apply hadd ihx ihy
[GOAL]
case intro.hm.hmul.ha
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝¹ : CliffordAlgebra Q
hx✝ : x✝¹ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x✝ : CliffordAlgebra Q
n'' : ℕ
y✝ : CliffordAlgebra Q
hy✝ : y✝ ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy✝ : P (y✝ * b) (_ : y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
y : CliffordAlgebra Q
hy : y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
ihx :
let hlean1926'' := (_ : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q));
P (x * y✝ * b) (_ : x * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
ihy :
let hlean1926'' := (_ : y ∈ LinearMap.range (ι Q) ^ 2 ↔ y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q));
P (y * y✝ * b) (_ : y * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x + y ∈ LinearMap.range (ι Q) ^ 2 ↔ x + y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x + y ∈ LinearMap.range (ι Q) ^ 2 ↔ x + y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P ((x + y) * y✝ * b) (_ : (x + y) * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
simp_rw [add_mul]
[GOAL]
case intro.hm.hmul.ha
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝¹ : CliffordAlgebra Q
hx✝ : x✝¹ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv a b : CliffordAlgebra Q
hb : b ∈ LinearMap.range (ι Q) ^ ZMod.val n
x✝ : CliffordAlgebra Q
n'' : ℕ
y✝ : CliffordAlgebra Q
hy✝ : y✝ ∈ (LinearMap.range (ι Q) ^ 2) ^ n''
ihy✝ : P (y✝ * b) (_ : y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
x : CliffordAlgebra Q
hx : x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
y : CliffordAlgebra Q
hy : y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q)
ihx :
let hlean1926'' := (_ : x ∈ LinearMap.range (ι Q) ^ 2 ↔ x ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q));
P (x * y✝ * b) (_ : x * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
ihy :
let hlean1926'' := (_ : y ∈ LinearMap.range (ι Q) ^ 2 ↔ y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q));
P (y * y✝ * b) (_ : y * y✝ * b ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hlean1926'' : x + y ∈ LinearMap.range (ι Q) ^ 2 ↔ x + y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q) :=
Eq.mpr
(id
(pow_two (LinearMap.range (ι Q)) ▸
Eq.refl (x + y ∈ LinearMap.range (ι Q) ^ 2 ↔ x + y ∈ LinearMap.range (ι Q) * LinearMap.range (ι Q))))
Iff.rfl
⊢ P (x * y✝ * b + y * y✝ * b) (_ : x * y✝ * b + y * y✝ * b ∈ evenOdd Q n)
[PROOFSTEP]
apply hadd ihx ihy
[GOAL]
case intro.ha
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv x : CliffordAlgebra Q
y : x ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
hx : CliffordAlgebra Q
hy : hx ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
ihx : P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
ihy : P hx (_ : hx ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
⊢ P (x + hx) (_ : x + hx ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
| ha x y hx hy ihx ihy => apply hadd ihx ihy
[GOAL]
case intro.ha
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
n : ZMod 2
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q n → Prop
hr :
∀ (v : CliffordAlgebra Q) (h : v ∈ LinearMap.range (ι Q) ^ ZMod.val n),
P v (_ : v ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n} {hy : y ∈ evenOdd Q n},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q n)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q n},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q n)
x✝ : CliffordAlgebra Q
hx✝ : x✝ ∈ evenOdd Q n
hlean1926 : ∀ (val : ℕ), ↑val = n ↔ ∃ k, val = 2 * k + ZMod.val n :=
fun val =>
Eq.mpr (id (congrFun (congrArg Iff (_auxLemma.1 2 val n)) (∃ k, val = 2 * k + ZMod.val n)))
(of_eq_true
(Eq.trans
(congrFun
(congrArg Iff
(congrArg Exists (funext fun k => congrArg (Eq val) ((fun b => add_comm (ZMod.val n) b) (2 * k)))))
(∃ k, val = 2 * k + ZMod.val n))
(iff_self (∃ k, val = 2 * k + ZMod.val n))))
k : ℕ
xv x : CliffordAlgebra Q
y : x ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
hx : CliffordAlgebra Q
hy : hx ∈ (LinearMap.range (ι Q) ^ 2) ^ k * LinearMap.range (ι Q) ^ ZMod.val n
ihx : P x (_ : x ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
ihy : P hx (_ : hx ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
⊢ P (x + hx) (_ : x + hx ∈ ⨆ (i : { n_1 // ↑n_1 = n }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
apply hadd ihx ihy
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 0 → Prop
hr : ∀ (r : R), P (↑(algebraMap R (CliffordAlgebra Q)) r) (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ evenOdd Q 0)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0} {hy : y ∈ evenOdd Q 0},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 0)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 0)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
⊢ P x hx
[PROOFSTEP]
refine' evenOdd_induction Q 0 (fun rx => _) (@hadd) hιι_mul x hx
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 0 → Prop
hr : ∀ (r : R), P (↑(algebraMap R (CliffordAlgebra Q)) r) (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ evenOdd Q 0)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0} {hy : y ∈ evenOdd Q 0},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 0)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 0)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
rx : CliffordAlgebra Q
⊢ ∀ (h : rx ∈ LinearMap.range (ι Q) ^ ZMod.val 0), P rx (_ : rx ∈ ⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
rintro ⟨r, rfl⟩
[GOAL]
case intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 0 → Prop
hr : ∀ (r : R), P (↑(algebraMap R (CliffordAlgebra Q)) r) (_ : ↑(algebraMap R (CliffordAlgebra Q)) r ∈ evenOdd Q 0)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0} {hy : y ∈ evenOdd Q 0},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 0)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 0},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 0)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 0
r : R
⊢ P (↑(Algebra.linearMap R (CliffordAlgebra Q)) r)
(_ : ↑(Algebra.linearMap R (CliffordAlgebra Q)) r ∈ ⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
exact hr r
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 1 → Prop
hι : ∀ (v : M), P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ evenOdd Q 1)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1} {hy : y ∈ evenOdd Q 1},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 1)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 1)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 1
⊢ P x hx
[PROOFSTEP]
refine' evenOdd_induction Q 1 (fun ιv => _) (@hadd) hιι_mul x hx
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 1 → Prop
hι : ∀ (v : M), P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ evenOdd Q 1)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1} {hy : y ∈ evenOdd Q 1},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 1)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 1)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 1
ιv : CliffordAlgebra Q
⊢ ∀ (h : ιv ∈ LinearMap.range (ι Q) ^ ZMod.val 1), P ιv (_ : ιv ∈ ⨆ (i : { n // ↑n = 1 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
intro h
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 1 → Prop
hι : ∀ (v : M), P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ evenOdd Q 1)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1} {hy : y ∈ evenOdd Q 1},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 1)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 1)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 1
ιv : CliffordAlgebra Q
h : ιv ∈ LinearMap.range (ι Q) ^ ZMod.val 1
⊢ P ιv (_ : ιv ∈ ⨆ (i : { n // ↑n = 1 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
rw [ZMod.val_one, pow_one] at h
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 1 → Prop
hι : ∀ (v : M), P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ evenOdd Q 1)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1} {hy : y ∈ evenOdd Q 1},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 1)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 1)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 1
ιv : CliffordAlgebra Q
h✝ : ιv ∈ LinearMap.range (ι Q) ^ ZMod.val 1
h : ιv ∈ LinearMap.range (ι Q)
⊢ P ιv (_ : ιv ∈ ⨆ (i : { n // ↑n = 1 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
revert h
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 1 → Prop
hι : ∀ (v : M), P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ evenOdd Q 1)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1} {hy : y ∈ evenOdd Q 1},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 1)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 1)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 1
ιv : CliffordAlgebra Q
h : ιv ∈ LinearMap.range (ι Q) ^ ZMod.val 1
⊢ ιv ∈ LinearMap.range (ι Q) → P ιv (_ : ιv ∈ ⨆ (i : { n // ↑n = 1 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
rintro ⟨v, rfl⟩
[GOAL]
case intro
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
P : (x : CliffordAlgebra Q) → x ∈ evenOdd Q 1 → Prop
hι : ∀ (v : M), P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ evenOdd Q 1)
hadd :
∀ {x y : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1} {hy : y ∈ evenOdd Q 1},
P x hx → P y hy → P (x + y) (_ : x + y ∈ evenOdd Q 1)
hιι_mul :
∀ (m₁ m₂ : M) {x : CliffordAlgebra Q} {hx : x ∈ evenOdd Q 1},
P x hx → P (↑(ι Q) m₁ * ↑(ι Q) m₂ * x) (_ : ↑(ι Q) m₁ * ↑(ι Q) m₂ * x ∈ evenOdd Q 1)
x : CliffordAlgebra Q
hx : x ∈ evenOdd Q 1
v : M
h : ↑(ι Q) v ∈ LinearMap.range (ι Q) ^ ZMod.val 1
⊢ P (↑(ι Q) v) (_ : ↑(ι Q) v ∈ ⨆ (i : { n // ↑n = 1 }), LinearMap.range (ι Q) ^ ↑i)
[PROOFSTEP]
exact hι v
| {"mathlib_filename": "Mathlib.LinearAlgebra.CliffordAlgebra.Grading", "llama_tokens": 62381} |
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝² : Semiring R
inst✝¹ : Fintype n
inst✝ : DecidableEq n
v : n → R
c : R
i : n
⊢ v ⬝ᵥ ↑(LinearMap.stdBasis R (fun x => R) i) c = v i * c
[PROOFSTEP]
rw [dotProduct, Finset.sum_eq_single i, LinearMap.stdBasis_same]
[GOAL]
case h₀
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝² : Semiring R
inst✝¹ : Fintype n
inst✝ : DecidableEq n
v : n → R
c : R
i : n
⊢ ∀ (b : n), b ∈ Finset.univ → b ≠ i → v b * ↑(LinearMap.stdBasis R (fun x => R) i) c b = 0
case h₁
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝² : Semiring R
inst✝¹ : Fintype n
inst✝ : DecidableEq n
v : n → R
c : R
i : n
⊢ ¬i ∈ Finset.univ → v i * ↑(LinearMap.stdBasis R (fun x => R) i) c i = 0
[PROOFSTEP]
exact fun _ _ hb => by rw [LinearMap.stdBasis_ne _ _ _ _ hb, mul_zero]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝² : Semiring R
inst✝¹ : Fintype n
inst✝ : DecidableEq n
v : n → R
c : R
i x✝¹ : n
x✝ : x✝¹ ∈ Finset.univ
hb : x✝¹ ≠ i
⊢ v x✝¹ * ↑(LinearMap.stdBasis R (fun x => R) i) c x✝¹ = 0
[PROOFSTEP]
rw [LinearMap.stdBasis_ne _ _ _ _ hb, mul_zero]
[GOAL]
case h₁
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝² : Semiring R
inst✝¹ : Fintype n
inst✝ : DecidableEq n
v : n → R
c : R
i : n
⊢ ¬i ∈ Finset.univ → v i * ↑(LinearMap.stdBasis R (fun x => R) i) c i = 0
[PROOFSTEP]
exact fun hi => False.elim (hi <| Finset.mem_univ _)
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝² : Semiring R
inst✝¹ : Fintype n
inst✝ : DecidableEq n
v : n → R
i : n
⊢ v ⬝ᵥ ↑(LinearMap.stdBasis R (fun x => R) i) 1 = v i
[PROOFSTEP]
rw [dotProduct_stdBasis_eq_mul, mul_one]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝¹ : Semiring R
inst✝ : Fintype n
v w : n → R
h : ∀ (u : n → R), v ⬝ᵥ u = w ⬝ᵥ u
⊢ v = w
[PROOFSTEP]
funext x
[GOAL]
case h
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝¹ : Semiring R
inst✝ : Fintype n
v w : n → R
h : ∀ (u : n → R), v ⬝ᵥ u = w ⬝ᵥ u
x : n
⊢ v x = w x
[PROOFSTEP]
classical rw [← dotProduct_stdBasis_one v x, ← dotProduct_stdBasis_one w x, h]
[GOAL]
case h
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝¹ : Semiring R
inst✝ : Fintype n
v w : n → R
h : ∀ (u : n → R), v ⬝ᵥ u = w ⬝ᵥ u
x : n
⊢ v x = w x
[PROOFSTEP]
rw [← dotProduct_stdBasis_one v x, ← dotProduct_stdBasis_one w x, h]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝³ : Fintype m
inst✝² : Fintype n
inst✝¹ : Fintype p
inst✝ : LinearOrderedRing R
v : n → R
⊢ (∀ (i : n), i ∈ Finset.univ → v i * v i = 0) ↔ v = 0
[PROOFSTEP]
simp [Function.funext_iff]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
v : n → R
⊢ (∀ (i : n), i ∈ Finset.univ → star (v i) * v i = 0) ↔ v = 0
[PROOFSTEP]
simp [Function.funext_iff, mul_eq_zero]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
v : n → R
⊢ (∀ (i : n), i ∈ Finset.univ → v i * star (v i) = 0) ↔ v = 0
[PROOFSTEP]
simp [Function.funext_iff, mul_eq_zero]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix n p R
⊢ Aᴴ * A * B = 0 ↔ A * B = 0
[PROOFSTEP]
refine ⟨fun h => ?_, fun h => by simp only [Matrix.mul_assoc, h, Matrix.mul_zero]⟩
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix n p R
h : A * B = 0
⊢ Aᴴ * A * B = 0
[PROOFSTEP]
simp only [Matrix.mul_assoc, h, Matrix.mul_zero]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix n p R
h : Aᴴ * A * B = 0
⊢ A * B = 0
[PROOFSTEP]
apply_fun (Bᴴ * ·) at h
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix n p R
h : Bᴴ * (Aᴴ * A * B) = Bᴴ * 0
⊢ A * B = 0
[PROOFSTEP]
rwa [Matrix.mul_zero, Matrix.mul_assoc, ← Matrix.mul_assoc, ← conjTranspose_mul, conjTranspose_mul_self_eq_zero] at h
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix m p R
⊢ A * Aᴴ * B = 0 ↔ Aᴴ * B = 0
[PROOFSTEP]
simpa only [conjTranspose_conjTranspose] using conjTranspose_mul_self_mul_eq_zero Aᴴ _
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix p m R
⊢ B * (A * Aᴴ) = 0 ↔ B * A = 0
[PROOFSTEP]
rw [← conjTranspose_eq_zero, conjTranspose_mul, conjTranspose_mul, conjTranspose_conjTranspose,
self_mul_conjTranspose_mul_eq_zero, ← conjTranspose_mul, conjTranspose_eq_zero]
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
B : Matrix p n R
⊢ B * (Aᴴ * A) = 0 ↔ B * Aᴴ = 0
[PROOFSTEP]
simpa only [conjTranspose_conjTranspose] using mul_self_mul_conjTranspose_eq_zero Aᴴ _
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
v : n → R
⊢ mulVec (Aᴴ * A) v = 0 ↔ mulVec A v = 0
[PROOFSTEP]
simpa only [← Matrix.col_mulVec, col_eq_zero] using conjTranspose_mul_self_mul_eq_zero A (col v)
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
v : m → R
⊢ mulVec (A * Aᴴ) v = 0 ↔ mulVec Aᴴ v = 0
[PROOFSTEP]
simpa only [conjTranspose_conjTranspose] using conjTranspose_mul_self_mulVec_eq_zero Aᴴ _
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
v : n → R
⊢ vecMul v (Aᴴ * A) = 0 ↔ vecMul v Aᴴ = 0
[PROOFSTEP]
simpa only [← Matrix.row_vecMul, row_eq_zero] using mul_conjTranspose_mul_self_eq_zero A (row v)
[GOAL]
m : Type u_1
n : Type u_2
p : Type u_3
R : Type u_4
inst✝⁶ : Fintype m
inst✝⁵ : Fintype n
inst✝⁴ : Fintype p
inst✝³ : PartialOrder R
inst✝² : NonUnitalRing R
inst✝¹ : StarOrderedRing R
inst✝ : NoZeroDivisors R
A : Matrix m n R
v : m → R
⊢ vecMul v (A * Aᴴ) = 0 ↔ vecMul v A = 0
[PROOFSTEP]
simpa only [conjTranspose_conjTranspose] using vecMul_conjTranspose_mul_self_eq_zero Aᴴ _
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.DotProduct", "llama_tokens": 3955} |
[GOAL]
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
R : Type u_2
inst✝ : Field R
A : Matrix n n R
hAps : Splits (RingHom.id R) (charpoly A)
⊢ det A = Multiset.prod (roots (charpoly A))
[PROOFSTEP]
rw [det_eq_sign_charpoly_coeff, ← charpoly_natDegree_eq_dim A,
Polynomial.prod_roots_eq_coeff_zero_of_monic_of_split A.charpoly_monic hAps, ← mul_assoc, ← pow_two, pow_right_comm,
neg_one_sq, one_pow, one_mul]
[GOAL]
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
R : Type u_2
inst✝ : Field R
A : Matrix n n R
hAps : Splits (RingHom.id R) (charpoly A)
⊢ trace A = Multiset.sum (roots (charpoly A))
[PROOFSTEP]
cases' isEmpty_or_nonempty n with h
[GOAL]
case inl
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
R : Type u_2
inst✝ : Field R
A : Matrix n n R
hAps : Splits (RingHom.id R) (charpoly A)
h : IsEmpty n
⊢ trace A = Multiset.sum (roots (charpoly A))
[PROOFSTEP]
rw [Matrix.trace, Fintype.sum_empty, Matrix.charpoly, det_eq_one_of_card_eq_zero (Fintype.card_eq_zero_iff.2 h),
Polynomial.roots_one, Multiset.empty_eq_zero, Multiset.sum_zero]
[GOAL]
case inr
n : Type u_1
inst✝² : Fintype n
inst✝¹ : DecidableEq n
R : Type u_2
inst✝ : Field R
A : Matrix n n R
hAps : Splits (RingHom.id R) (charpoly A)
h✝ : Nonempty n
⊢ trace A = Multiset.sum (roots (charpoly A))
[PROOFSTEP]
rw [trace_eq_neg_charpoly_coeff, neg_eq_iff_eq_neg, ←
Polynomial.sum_roots_eq_nextCoeff_of_monic_of_split A.charpoly_monic hAps, nextCoeff, charpoly_natDegree_eq_dim,
if_neg (Fintype.card_ne_zero : Fintype.card n ≠ 0)]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Charpoly.Eigs", "llama_tokens": 732} |
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ IsLinearMap α (cramerMap A)
[PROOFSTEP]
constructor
[GOAL]
case map_add
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ ∀ (x y : n → α), cramerMap A (x + y) = cramerMap A x + cramerMap A y
[PROOFSTEP]
intros
[GOAL]
case map_smul
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ ∀ (c : α) (x : n → α), cramerMap A (c • x) = c • cramerMap A x
[PROOFSTEP]
intros
[GOAL]
case map_add
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b x✝ y✝ : n → α
⊢ cramerMap A (x✝ + y✝) = cramerMap A x✝ + cramerMap A y✝
[PROOFSTEP]
ext i
[GOAL]
case map_smul
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
c✝ : α
x✝ : n → α
⊢ cramerMap A (c✝ • x✝) = c✝ • cramerMap A x✝
[PROOFSTEP]
ext i
[GOAL]
case map_add.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b x✝ y✝ : n → α
i : n
⊢ cramerMap A (x✝ + y✝) i = (cramerMap A x✝ + cramerMap A y✝) i
[PROOFSTEP]
apply (cramerMap_is_linear A i).1
[GOAL]
case map_smul.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
c✝ : α
x✝ : n → α
i : n
⊢ cramerMap A (c✝ • x✝) i = (c✝ • cramerMap A x✝) i
[PROOFSTEP]
apply (cramerMap_is_linear A i).2
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i : n
⊢ ↑(cramer Aᵀ) b i = det (updateRow A i b)
[PROOFSTEP]
rw [cramer_apply, updateColumn_transpose, det_transpose]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i : n
⊢ ↑(cramer Aᵀ) (A i) = Pi.single i (det A)
[PROOFSTEP]
ext j
[GOAL]
case h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
⊢ ↑(cramer Aᵀ) (A i) j = Pi.single i (det A) j
[PROOFSTEP]
rw [cramer_apply, Pi.single_apply]
[GOAL]
case h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
⊢ det (updateColumn Aᵀ j (A i)) = if j = i then det A else 0
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
h : j = i
⊢ det (updateColumn Aᵀ j (A i)) = det A
[PROOFSTEP]
subst h
[GOAL]
case pos
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
j : n
⊢ det (updateColumn Aᵀ j (A j)) = det A
[PROOFSTEP]
simp only [updateColumn_transpose, det_transpose, updateRow_eq_self]
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
h : ¬j = i
⊢ det (updateColumn Aᵀ j (A i)) = 0
[PROOFSTEP]
rw [updateColumn_transpose, det_transpose]
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
h : ¬j = i
⊢ det (updateRow A j (A i)) = 0
[PROOFSTEP]
apply det_zero_of_row_eq h
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
h : ¬j = i
⊢ updateRow A j (A i) j = updateRow A j (A i) i
[PROOFSTEP]
rw [updateRow_self, updateRow_ne (Ne.symm h)]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i : n
h : ∀ (j : n), b j = A j i
⊢ ↑(cramer A) b = Pi.single i (det A)
[PROOFSTEP]
rw [← transpose_transpose A, det_transpose]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i : n
h : ∀ (j : n), b j = A j i
⊢ ↑(cramer Aᵀᵀ) b = Pi.single i (det Aᵀ)
[PROOFSTEP]
convert cramer_transpose_row_self Aᵀ i
[GOAL]
case h.e'_2.h.e'_6
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i : n
h : ∀ (j : n), b j = A j i
⊢ b = Aᵀ i
[PROOFSTEP]
exact funext h
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ cramer 1 = 1
[PROOFSTEP]
refine LinearMap.pi_ext' (fun (i : n) => LinearMap.ext_ring (funext (fun (j : n) => ?_)))
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
⊢ ↑(LinearMap.comp (cramer 1) (LinearMap.single i)) 1 j = ↑(LinearMap.comp 1 (LinearMap.single i)) 1 j
[PROOFSTEP]
convert congr_fun (cramer_row_self (1 : Matrix n n α) (Pi.single i 1) i _) j
[GOAL]
case h.e'_3.h.e'_1
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
⊢ 1 = det 1
[PROOFSTEP]
simp
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j : n
⊢ ∀ (j : n), Pi.single i 1 j = OfNat.ofNat 1 j i
[PROOFSTEP]
intro j
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
i j✝ j : n
⊢ Pi.single i 1 j = OfNat.ofNat 1 j i
[PROOFSTEP]
rw [Matrix.one_eq_pi_single, Pi.single_comm]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
A✝ : Matrix n n α
b✝ : n → α
inst✝ : Subsingleton n
A : Matrix n n α
b : n → α
i : n
⊢ ↑(cramer A) b i = b i
[PROOFSTEP]
rw [cramer_apply, det_eq_elem_of_subsingleton _ i, updateColumn_self]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
A : Matrix n n α
b : n → α
inst✝ : Nontrivial n
⊢ cramer 0 = 0
[PROOFSTEP]
ext i j
[GOAL]
case h.h.h
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
A : Matrix n n α
b : n → α
inst✝ : Nontrivial n
i j : n
⊢ ↑(LinearMap.comp (cramer 0) (LinearMap.single i)) 1 j = ↑(LinearMap.comp 0 (LinearMap.single i)) 1 j
[PROOFSTEP]
obtain ⟨j', hj'⟩ : ∃ j', j' ≠ j := exists_ne j
[GOAL]
case h.h.h.intro
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
A : Matrix n n α
b : n → α
inst✝ : Nontrivial n
i j j' : n
hj' : j' ≠ j
⊢ ↑(LinearMap.comp (cramer 0) (LinearMap.single i)) 1 j = ↑(LinearMap.comp 0 (LinearMap.single i)) 1 j
[PROOFSTEP]
apply det_eq_zero_of_column_eq_zero j'
[GOAL]
case h.h.h.intro
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
A : Matrix n n α
b : n → α
inst✝ : Nontrivial n
i j j' : n
hj' : j' ≠ j
⊢ ∀ (i_1 : n), updateColumn 0 j (↑(LinearMap.single i) 1) i_1 j' = 0
[PROOFSTEP]
intro j''
[GOAL]
case h.h.h.intro
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
A : Matrix n n α
b : n → α
inst✝ : Nontrivial n
i j j' : n
hj' : j' ≠ j
j'' : n
⊢ updateColumn 0 j (↑(LinearMap.single i) 1) j'' j' = 0
[PROOFSTEP]
simp [updateColumn_ne hj']
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
β : Type u_1
s : Finset β
f : n → β → α
i : n
⊢ Finset.sum s (fun x => ↑(cramer A) fun j => f j x) i = ↑(cramer A) (fun j => ∑ x in s, f j x) i
[PROOFSTEP]
rw [sum_cramer, cramer_apply, cramer_apply]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
β : Type u_1
s : Finset β
f : n → β → α
i : n
⊢ det (updateColumn A i (∑ x in s, fun j => f j x)) = det (updateColumn A i fun j => ∑ x in s, f j x)
[PROOFSTEP]
simp only [updateColumn]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
β : Type u_1
s : Finset β
f : n → β → α
i : n
⊢ det (↑of fun i_1 => Function.update (A i_1) i (Finset.sum s (fun x j => f j x) i_1)) =
det (↑of fun i_1 => Function.update (A i_1) i (∑ x in s, f i_1 x))
[PROOFSTEP]
congr with j
[GOAL]
case e_M.h.e_6.h.h.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
β : Type u_1
s : Finset β
f : n → β → α
i j x✝ : n
⊢ Function.update (A j) i (Finset.sum s (fun x j => f j x) j) x✝ = Function.update (A j) i (∑ x in s, f j x) x✝
[PROOFSTEP]
congr
[GOAL]
case e_M.h.e_6.h.h.h.e_v
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
β : Type u_1
s : Finset β
f : n → β → α
i j x✝ : n
⊢ Finset.sum s (fun x j => f j x) j = ∑ x in s, f j x
[PROOFSTEP]
apply Finset.sum_apply
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A✝ : Matrix n n α
b✝ : n → α
A : Matrix m m α
e : n ≃ m
b : n → α
⊢ ↑(cramer (submatrix A ↑e ↑e)) b = ↑(cramer A) (b ∘ ↑e.symm) ∘ ↑e
[PROOFSTEP]
ext i
[GOAL]
case h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A✝ : Matrix n n α
b✝ : n → α
A : Matrix m m α
e : n ≃ m
b : n → α
i : n
⊢ ↑(cramer (submatrix A ↑e ↑e)) b i = (↑(cramer A) (b ∘ ↑e.symm) ∘ ↑e) i
[PROOFSTEP]
simp_rw [Function.comp_apply, cramer_apply, updateColumn_submatrix_equiv, det_submatrix_equiv_self e, Function.comp]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ adjugate A i j = det (updateRow A j (Pi.single i 1))
[PROOFSTEP]
rw [adjugate_def, of_apply, cramer_apply, updateColumn_transpose, det_transpose]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ (adjugate A)ᵀ = adjugate Aᵀ
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ (adjugate A)ᵀ i j = adjugate Aᵀ i j
[PROOFSTEP]
rw [transpose_apply, adjugate_apply, adjugate_apply, updateRow_transpose, det_transpose]
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ det (updateRow A i (Pi.single j 1)) = det (updateColumn A j (Pi.single i 1))
[PROOFSTEP]
rw [det_apply', det_apply']
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ ∑ σ : Perm n, ↑↑(↑sign σ) * ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 =
∑ σ : Perm n, ↑↑(↑sign σ) * ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
apply Finset.sum_congr rfl
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ ∀ (x : Perm n),
x ∈ univ →
↑↑(↑sign x) * ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑x i_1) i_1 =
↑↑(↑sign x) * ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑x i_1) i_1
[PROOFSTEP]
intro σ _
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
⊢ ↑↑(↑sign σ) * ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 =
↑↑(↑sign σ) * ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
congr 1
[GOAL]
case a.h.e_a
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
⊢ ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 = ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
by_cases i = σ j
[GOAL]
case a.h.e_a
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
⊢ ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 = ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
by_cases i = σ j
[GOAL]
case pos
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : i = ↑σ j
⊢ ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 = ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
congr
[GOAL]
case pos.e_f
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : i = ↑σ j
⊢ (fun i_1 => updateRow A i (Pi.single j 1) (↑σ i_1) i_1) = fun i_1 => updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
ext j'
[GOAL]
case pos.e_f.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : i = ↑σ j
j' : n
⊢ updateRow A i (Pi.single j 1) (↑σ j') j' = updateColumn A j (Pi.single i 1) (↑σ j') j'
[PROOFSTEP]
subst h
[GOAL]
case pos.e_f.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
j : n
σ : Perm n
a✝ : σ ∈ univ
j' : n
⊢ updateRow A (↑σ j) (Pi.single j 1) (↑σ j') j' = updateColumn A j (Pi.single (↑σ j) 1) (↑σ j') j'
[PROOFSTEP]
have : σ j' = σ j ↔ j' = j := σ.injective.eq_iff
[GOAL]
case pos.e_f.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
j : n
σ : Perm n
a✝ : σ ∈ univ
j' : n
this : ↑σ j' = ↑σ j ↔ j' = j
⊢ updateRow A (↑σ j) (Pi.single j 1) (↑σ j') j' = updateColumn A j (Pi.single (↑σ j) 1) (↑σ j') j'
[PROOFSTEP]
rw [updateRow_apply, updateColumn_apply]
[GOAL]
case pos.e_f.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
j : n
σ : Perm n
a✝ : σ ∈ univ
j' : n
this : ↑σ j' = ↑σ j ↔ j' = j
⊢ (if ↑σ j' = ↑σ j then Pi.single j 1 j' else A (↑σ j') j') =
if j' = j then Pi.single (↑σ j) 1 (↑σ j') else A (↑σ j') j'
[PROOFSTEP]
simp_rw [this]
[GOAL]
case pos.e_f.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
j : n
σ : Perm n
a✝ : σ ∈ univ
j' : n
this : ↑σ j' = ↑σ j ↔ j' = j
⊢ (if j' = j then Pi.single j 1 j' else A (↑σ j') j') = if j' = j then Pi.single (↑σ j) 1 (↑σ j') else A (↑σ j') j'
[PROOFSTEP]
rw [← dite_eq_ite, ← dite_eq_ite]
[GOAL]
case pos.e_f.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
j : n
σ : Perm n
a✝ : σ ∈ univ
j' : n
this : ↑σ j' = ↑σ j ↔ j' = j
⊢ (if x : j' = j then Pi.single j 1 j' else A (↑σ j') j') =
if x : j' = j then Pi.single (↑σ j) 1 (↑σ j') else A (↑σ j') j'
[PROOFSTEP]
congr 1 with rfl
[GOAL]
case pos.e_f.h.e_t.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
σ : Perm n
a✝ : σ ∈ univ
j' : n
this : ↑σ j' = ↑σ j' ↔ j' = j'
⊢ Pi.single j' 1 j' = Pi.single (↑σ j') 1 (↑σ j')
[PROOFSTEP]
rw [Pi.single_eq_same, Pi.single_eq_same]
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
⊢ ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 = ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
have : (∏ j' : n, updateColumn A j (Pi.single i 1) (σ j') j') = 0 :=
by
apply prod_eq_zero (mem_univ j)
rw [updateColumn_self, Pi.single_eq_of_ne' h]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
⊢ ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
[PROOFSTEP]
apply prod_eq_zero (mem_univ j)
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
⊢ updateColumn A j (Pi.single i 1) (↑σ j) j = 0
[PROOFSTEP]
rw [updateColumn_self, Pi.single_eq_of_ne' h]
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
this : ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
⊢ ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 = ∏ i_1 : n, updateColumn A j (Pi.single i 1) (↑σ i_1) i_1
[PROOFSTEP]
rw [this]
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
this : ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
⊢ ∏ i_1 : n, updateRow A i (Pi.single j 1) (↑σ i_1) i_1 = 0
[PROOFSTEP]
apply prod_eq_zero (mem_univ (σ⁻¹ i))
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
this : ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
⊢ updateRow A i (Pi.single j 1) (↑σ (↑σ⁻¹ i)) (↑σ⁻¹ i) = 0
[PROOFSTEP]
erw [apply_symm_apply σ i, updateRow_self]
[GOAL]
case neg
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
this : ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
⊢ Pi.single j 1 (↑σ⁻¹ i) = 0
[PROOFSTEP]
apply Pi.single_eq_of_ne
[GOAL]
case neg.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
this : ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
⊢ ↑σ⁻¹ i ≠ j
[PROOFSTEP]
intro h'
[GOAL]
case neg.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
σ : Perm n
a✝ : σ ∈ univ
h : ¬i = ↑σ j
this : ∏ j' : n, updateColumn A j (Pi.single i 1) (↑σ j') j' = 0
h' : ↑σ⁻¹ i = j
⊢ False
[PROOFSTEP]
exact h ((symm_apply_eq σ).mp h')
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
e : n ≃ m
A : Matrix m m α
⊢ adjugate (submatrix A ↑e ↑e) = submatrix (adjugate A) ↑e ↑e
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
e : n ≃ m
A : Matrix m m α
i j : n
⊢ adjugate (submatrix A ↑e ↑e) i j = submatrix (adjugate A) (↑e) (↑e) i j
[PROOFSTEP]
rw [adjugate_apply, submatrix_apply, adjugate_apply, ← det_submatrix_equiv_self e, updateRow_submatrix_equiv]
-- Porting note: added
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
e : n ≃ m
A : Matrix m m α
i j : n
⊢ det (submatrix (updateRow A (↑e j) fun j => Pi.single i 1 (↑e.symm j)) ↑e ↑e) =
det (submatrix (updateRow A (↑e j) (Pi.single (↑e i) 1)) ↑e ↑e)
[PROOFSTEP]
suffices (fun j => Pi.single i 1 (e.symm j)) = Pi.single (e i) 1 by erw [this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
e : n ≃ m
A : Matrix m m α
i j : n
this : (fun j => Pi.single i 1 (↑e.symm j)) = Pi.single (↑e i) 1
⊢ det (submatrix (updateRow A (↑e j) fun j => Pi.single i 1 (↑e.symm j)) ↑e ↑e) =
det (submatrix (updateRow A (↑e j) (Pi.single (↑e i) 1)) ↑e ↑e)
[PROOFSTEP]
erw [this]
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
e : n ≃ m
A : Matrix m m α
i j : n
⊢ (fun j => Pi.single i 1 (↑e.symm j)) = Pi.single (↑e i) 1
[PROOFSTEP]
exact Function.update_comp_equiv _ e.symm _ _
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ ↑(cramer A) b = mulVec (adjugate A) b
[PROOFSTEP]
nth_rw 2 [← A.transpose_transpose]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ ↑(cramer A) b = mulVec (adjugate Aᵀᵀ) b
[PROOFSTEP]
rw [← adjugate_transpose, adjugate_def]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ ↑(cramer A) b = mulVec (↑of fun i => ↑(cramer Aᵀᵀ) (Pi.single i 1))ᵀ b
[PROOFSTEP]
have : b = ∑ i, b i • Pi.single i 1 := by
refine' (pi_eq_sum_univ b).trans _
congr with j
simp [Pi.single_apply, eq_comm, Pi.smul_apply (b j)]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ b = ∑ i : n, b i • Pi.single i 1
[PROOFSTEP]
refine' (pi_eq_sum_univ b).trans _
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ (∑ i : n, b i • fun j => if i = j then 1 else 0) = ∑ i : n, b i • Pi.single i 1
[PROOFSTEP]
congr with j
[GOAL]
case e_f.h.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
j x✝ : n
⊢ (b j • fun j_1 => if j = j_1 then 1 else 0) x✝ = (b j • Pi.single j 1) x✝
[PROOFSTEP]
simp [Pi.single_apply, eq_comm, Pi.smul_apply (b j)]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
this : b = ∑ i : n, b i • Pi.single i 1
⊢ ↑(cramer A) b = mulVec (↑of fun i => ↑(cramer Aᵀᵀ) (Pi.single i 1))ᵀ b
[PROOFSTEP]
conv_lhs => rw [this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
this : b = ∑ i : n, b i • Pi.single i 1
| ↑(cramer A) b
[PROOFSTEP]
rw [this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
this : b = ∑ i : n, b i • Pi.single i 1
| ↑(cramer A) b
[PROOFSTEP]
rw [this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
this : b = ∑ i : n, b i • Pi.single i 1
| ↑(cramer A) b
[PROOFSTEP]
rw [this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
this : b = ∑ i : n, b i • Pi.single i 1
⊢ ↑(cramer A) (∑ i : n, b i • Pi.single i 1) = mulVec (↑of fun i => ↑(cramer Aᵀᵀ) (Pi.single i 1))ᵀ b
[PROOFSTEP]
ext k
[GOAL]
case h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
this : b = ∑ i : n, b i • Pi.single i 1
k : n
⊢ ↑(cramer A) (∑ i : n, b i • Pi.single i 1) k = mulVec (↑of fun i => ↑(cramer Aᵀᵀ) (Pi.single i 1))ᵀ b k
[PROOFSTEP]
simp [mulVec, dotProduct, mul_comm]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j k : n
⊢ A i k * adjugate A k j = ↑(cramer Aᵀ) (Pi.single k (A i k)) j
[PROOFSTEP]
erw [← smul_eq_mul, adjugate, of_apply, ← Pi.smul_apply, ← LinearMap.map_smul, ← Pi.single_smul', smul_eq_mul, mul_one]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ A * adjugate A = det A • 1
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ (A * adjugate A) i j = (det A • 1) i j
[PROOFSTEP]
rw [mul_apply, Pi.smul_apply, Pi.smul_apply, one_apply, smul_eq_mul, mul_boole]
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i j : n
⊢ ∑ j_1 : n, A i j_1 * adjugate A j_1 j = if i = j then det A else 0
[PROOFSTEP]
simp [mul_adjugate_apply, sum_cramer_apply, cramer_transpose_row_self, Pi.single_apply, eq_comm]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ adjugate A * A = (Aᵀ * adjugate Aᵀ)ᵀ
[PROOFSTEP]
rw [← adjugate_transpose, ← transpose_mul, transpose_transpose]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ (Aᵀ * adjugate Aᵀ)ᵀ = det A • 1
[PROOFSTEP]
rw [mul_adjugate Aᵀ, det_transpose, transpose_smul, transpose_one]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
r : α
A : Matrix n n α
⊢ adjugate (r • A) = r ^ (Fintype.card n - 1) • adjugate A
[PROOFSTEP]
rw [adjugate, adjugate, transpose_smul, cramer_smul]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
r : α
A : Matrix n n α
⊢ (↑of fun i => ↑(r ^ (Fintype.card n - 1) • cramer Aᵀ) (Pi.single i 1)) =
r ^ (Fintype.card n - 1) • ↑of fun i => ↑(cramer Aᵀ) (Pi.single i 1)
[PROOFSTEP]
rfl
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
b : n → α
⊢ mulVec A (↑(cramer A) b) = det A • b
[PROOFSTEP]
rw [cramer_eq_adjugate_mulVec, mulVec_mulVec, mul_adjugate, smul_mulVec_assoc, one_mulVec]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Subsingleton n
A : Matrix n n α
⊢ adjugate A = 1
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Subsingleton n
A : Matrix n n α
i j : n
⊢ adjugate A i j = OfNat.ofNat 1 i j
[PROOFSTEP]
simp [Subsingleton.elim i j, adjugate_apply, det_eq_elem_of_subsingleton _ i]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Nontrivial n
⊢ adjugate 0 = 0
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Nontrivial n
i j : n
⊢ adjugate 0 i j = OfNat.ofNat 0 i j
[PROOFSTEP]
obtain ⟨j', hj'⟩ : ∃ j', j' ≠ j := exists_ne j
[GOAL]
case a.h.intro
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Nontrivial n
i j j' : n
hj' : j' ≠ j
⊢ adjugate 0 i j = OfNat.ofNat 0 i j
[PROOFSTEP]
apply det_eq_zero_of_column_eq_zero j'
[GOAL]
case a.h.intro
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Nontrivial n
i j j' : n
hj' : j' ≠ j
⊢ ∀ (i_1 : n), updateColumn 0ᵀ j (Pi.single i 1) i_1 j' = 0
[PROOFSTEP]
intro j''
[GOAL]
case a.h.intro
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : Nontrivial n
i j j' : n
hj' : j' ≠ j
j'' : n
⊢ updateColumn 0ᵀ j (Pi.single i 1) j'' j' = 0
[PROOFSTEP]
simp [updateColumn_ne hj']
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
⊢ adjugate 1 = 1
[PROOFSTEP]
ext
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
i✝ x✝ : n
⊢ adjugate 1 i✝ x✝ = OfNat.ofNat 1 i✝ x✝
[PROOFSTEP]
simp [adjugate_def, Matrix.one_apply, Pi.single_apply, eq_comm]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
⊢ adjugate (diagonal v) = diagonal fun i => ∏ j in Finset.erase univ i, v j
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i j : n
⊢ adjugate (diagonal v) i j = diagonal (fun i => ∏ j in Finset.erase univ i, v j) i j
[PROOFSTEP]
simp only [adjugate_def, cramer_apply, diagonal_transpose, of_apply]
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i j : n
⊢ det (updateColumn (diagonal v) j (Pi.single i 1)) = diagonal (fun i => ∏ j in Finset.erase univ i, v j) i j
[PROOFSTEP]
obtain rfl | hij := eq_or_ne i j
[GOAL]
case a.h.inl
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i : n
⊢ det (updateColumn (diagonal v) i (Pi.single i 1)) = diagonal (fun i => ∏ j in Finset.erase univ i, v j) i i
[PROOFSTEP]
rw [diagonal_apply_eq, diagonal_updateColumn_single, det_diagonal, prod_update_of_mem (Finset.mem_univ _),
sdiff_singleton_eq_erase, one_mul]
[GOAL]
case a.h.inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i j : n
hij : i ≠ j
⊢ det (updateColumn (diagonal v) j (Pi.single i 1)) = diagonal (fun i => ∏ j in Finset.erase univ i, v j) i j
[PROOFSTEP]
rw [diagonal_apply_ne _ hij]
[GOAL]
case a.h.inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i j : n
hij : i ≠ j
⊢ det (updateColumn (diagonal v) j (Pi.single i 1)) = 0
[PROOFSTEP]
refine' det_eq_zero_of_row_eq_zero j fun k => _
[GOAL]
case a.h.inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i j : n
hij : i ≠ j
k : n
⊢ updateColumn (diagonal v) j (Pi.single i 1) j k = 0
[PROOFSTEP]
obtain rfl | hjk := eq_or_ne k j
[GOAL]
case a.h.inr.inl
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i k : n
hij : i ≠ k
⊢ updateColumn (diagonal v) k (Pi.single i 1) k k = 0
[PROOFSTEP]
rw [updateColumn_self, Pi.single_eq_of_ne' hij]
[GOAL]
case a.h.inr.inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
v : n → α
i j : n
hij : i ≠ j
k : n
hjk : k ≠ j
⊢ updateColumn (diagonal v) j (Pi.single i 1) j k = 0
[PROOFSTEP]
rw [updateColumn_ne hjk, diagonal_apply_ne' _ hjk]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : CommRing α
R : Type u_1
S : Type u_2
inst✝¹ : CommRing R
inst✝ : CommRing S
f : R →+* S
M : Matrix n n R
⊢ ↑(RingHom.mapMatrix f) (adjugate M) = adjugate (↑(RingHom.mapMatrix f) M)
[PROOFSTEP]
ext i k
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : CommRing α
R : Type u_1
S : Type u_2
inst✝¹ : CommRing R
inst✝ : CommRing S
f : R →+* S
M : Matrix n n R
i k : n
⊢ ↑(RingHom.mapMatrix f) (adjugate M) i k = adjugate (↑(RingHom.mapMatrix f) M) i k
[PROOFSTEP]
have : Pi.single i (1 : S) = f ∘ Pi.single i 1 := by
rw [← f.map_one]
exact Pi.single_op (fun _ => f) (fun _ => f.map_zero) i (1 : R)
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : CommRing α
R : Type u_1
S : Type u_2
inst✝¹ : CommRing R
inst✝ : CommRing S
f : R →+* S
M : Matrix n n R
i k : n
⊢ Pi.single i 1 = ↑f ∘ Pi.single i 1
[PROOFSTEP]
rw [← f.map_one]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : CommRing α
R : Type u_1
S : Type u_2
inst✝¹ : CommRing R
inst✝ : CommRing S
f : R →+* S
M : Matrix n n R
i k : n
⊢ Pi.single i (↑f 1) = ↑f ∘ Pi.single i 1
[PROOFSTEP]
exact Pi.single_op (fun _ => f) (fun _ => f.map_zero) i (1 : R)
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : CommRing α
R : Type u_1
S : Type u_2
inst✝¹ : CommRing R
inst✝ : CommRing S
f : R →+* S
M : Matrix n n R
i k : n
this : Pi.single i 1 = ↑f ∘ Pi.single i 1
⊢ ↑(RingHom.mapMatrix f) (adjugate M) i k = adjugate (↑(RingHom.mapMatrix f) M) i k
[PROOFSTEP]
rw [adjugate_apply, RingHom.mapMatrix_apply, map_apply, RingHom.mapMatrix_apply, this, ← map_updateRow, ←
RingHom.mapMatrix_apply, ← RingHom.map_det, ← adjugate_apply]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
cases' (Fintype.card n).eq_zero_or_pos with h_card h_card
[GOAL]
case inl
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n = 0
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
haveI : IsEmpty n := Fintype.card_eq_zero_iff.mp h_card
[GOAL]
case inl
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n = 0
this : IsEmpty n
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
rw [h_card, Nat.zero_sub, pow_zero, adjugate_subsingleton, det_one]
[GOAL]
case inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n > 0
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
replace h_card := tsub_add_cancel_of_le h_card.nat_succ_le
[GOAL]
case inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
let A' := mvPolynomialX n n ℤ
[GOAL]
case inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
suffices A'.adjugate.det = A'.det ^ (Fintype.card n - 1) by
rw [← mvPolynomialX_mapMatrix_aeval ℤ A, ← AlgHom.map_adjugate, ← AlgHom.map_det, ← AlgHom.map_det, ← AlgHom.map_pow,
this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
this : det (adjugate A') = det A' ^ (Fintype.card n - 1)
⊢ det (adjugate A) = det A ^ (Fintype.card n - 1)
[PROOFSTEP]
rw [← mvPolynomialX_mapMatrix_aeval ℤ A, ← AlgHom.map_adjugate, ← AlgHom.map_det, ← AlgHom.map_det, ← AlgHom.map_pow,
this]
[GOAL]
case inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ det (adjugate A') = det A' ^ (Fintype.card n - 1)
[PROOFSTEP]
apply mul_left_cancel₀ (show A'.det ≠ 0 from det_mvPolynomialX_ne_zero n ℤ)
[GOAL]
case inr
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ det A' * det (adjugate A') = det A' * det A' ^ (Fintype.card n - 1)
[PROOFSTEP]
calc
A'.det * A'.adjugate.det = (A' * adjugate A').det := (det_mul _ _).symm
_ = A'.det ^ Fintype.card n := by rw [mul_adjugate, det_smul, det_one, mul_one]
_ = A'.det * A'.det ^ (Fintype.card n - 1) := by rw [← pow_succ, h_card]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ det (A' * adjugate A') = det A' ^ Fintype.card n
[PROOFSTEP]
rw [mul_adjugate, det_smul, det_one, mul_one]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h_card : Fintype.card n - Nat.succ 0 + Nat.succ 0 = Fintype.card n
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ det A' ^ Fintype.card n = det A' * det A' ^ (Fintype.card n - 1)
[PROOFSTEP]
rw [← pow_succ, h_card]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
⊢ adjugate A = ↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]]
[PROOFSTEP]
ext i j
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
i j : Fin 2
⊢ adjugate A i j = ↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] i j
[PROOFSTEP]
rw [adjugate_apply, det_fin_two]
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
i j : Fin 2
⊢ updateRow A j (Pi.single i 1) 0 0 * updateRow A j (Pi.single i 1) 1 1 -
updateRow A j (Pi.single i 1) 0 1 * updateRow A j (Pi.single i 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] i j
[PROOFSTEP]
fin_cases i
[GOAL]
case a.h.head
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
j : Fin 2
⊢ updateRow A j (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 0 0 *
updateRow A j (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 1 1 -
updateRow A j (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 0 1 *
updateRow A j (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] { val := 0, isLt := (_ : 0 < 2) } j
[PROOFSTEP]
fin_cases j
[GOAL]
case a.h.tail.head
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
j : Fin 2
⊢ updateRow A j (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 0 0 *
updateRow A j (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 1 1 -
updateRow A j (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 0 1 *
updateRow A j (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] { val := 1, isLt := (_ : (fun a => a < 2) 1) } j
[PROOFSTEP]
fin_cases j
[GOAL]
case a.h.head.head
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
⊢ updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 0 0 *
updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 1 1 -
updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 0 1 *
updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] { val := 0, isLt := (_ : 0 < 2) } { val := 0, isLt := (_ : 0 < 2) }
[PROOFSTEP]
simp [one_mul, Fin.one_eq_zero_iff, Pi.single_eq_same, mul_zero, sub_zero, Pi.single_eq_of_ne, Ne.def, not_false_iff,
updateRow_self, updateRow_ne, cons_val_zero, of_apply, Nat.succ_succ_ne_one, Pi.single_eq_of_ne, updateRow_self,
Pi.single_eq_of_ne, Ne.def, Fin.zero_eq_one_iff, Nat.succ_succ_ne_one, not_false_iff, updateRow_ne,
Fin.one_eq_zero_iff, zero_mul, Pi.single_eq_same, one_mul, zero_sub, of_apply, cons_val', cons_val_fin_one,
cons_val_one, head_fin_const, neg_inj, eq_self_iff_true, cons_val_zero, head_cons, mul_one]
[GOAL]
case a.h.head.tail.head
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
⊢ updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 0 0 *
updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 1 1 -
updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 0 1 *
updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) } (Pi.single { val := 0, isLt := (_ : 0 < 2) } 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] { val := 0, isLt := (_ : 0 < 2) }
{ val := 1, isLt := (_ : (fun a => a < 2) 1) }
[PROOFSTEP]
simp [one_mul, Fin.one_eq_zero_iff, Pi.single_eq_same, mul_zero, sub_zero, Pi.single_eq_of_ne, Ne.def, not_false_iff,
updateRow_self, updateRow_ne, cons_val_zero, of_apply, Nat.succ_succ_ne_one, Pi.single_eq_of_ne, updateRow_self,
Pi.single_eq_of_ne, Ne.def, Fin.zero_eq_one_iff, Nat.succ_succ_ne_one, not_false_iff, updateRow_ne,
Fin.one_eq_zero_iff, zero_mul, Pi.single_eq_same, one_mul, zero_sub, of_apply, cons_val', cons_val_fin_one,
cons_val_one, head_fin_const, neg_inj, eq_self_iff_true, cons_val_zero, head_cons, mul_one]
[GOAL]
case a.h.tail.head.head
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
⊢ updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 0 0 *
updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 1 1 -
updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 0 1 *
updateRow A { val := 0, isLt := (_ : 0 < 2) } (Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] { val := 1, isLt := (_ : (fun a => a < 2) 1) }
{ val := 0, isLt := (_ : 0 < 2) }
[PROOFSTEP]
simp [one_mul, Fin.one_eq_zero_iff, Pi.single_eq_same, mul_zero, sub_zero, Pi.single_eq_of_ne, Ne.def, not_false_iff,
updateRow_self, updateRow_ne, cons_val_zero, of_apply, Nat.succ_succ_ne_one, Pi.single_eq_of_ne, updateRow_self,
Pi.single_eq_of_ne, Ne.def, Fin.zero_eq_one_iff, Nat.succ_succ_ne_one, not_false_iff, updateRow_ne,
Fin.one_eq_zero_iff, zero_mul, Pi.single_eq_same, one_mul, zero_sub, of_apply, cons_val', cons_val_fin_one,
cons_val_one, head_fin_const, neg_inj, eq_self_iff_true, cons_val_zero, head_cons, mul_one]
[GOAL]
case a.h.tail.head.tail.head
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix (Fin 2) (Fin 2) α
⊢ updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) }
(Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 0 0 *
updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) }
(Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 1 1 -
updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) }
(Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 0 1 *
updateRow A { val := 1, isLt := (_ : (fun a => a < 2) 1) }
(Pi.single { val := 1, isLt := (_ : (fun a => a < 2) 1) } 1) 1 0 =
↑of ![![A 1 1, -A 0 1], ![-A 1 0, A 0 0]] { val := 1, isLt := (_ : (fun a => a < 2) 1) }
{ val := 1, isLt := (_ : (fun a => a < 2) 1) }
[PROOFSTEP]
simp [one_mul, Fin.one_eq_zero_iff, Pi.single_eq_same, mul_zero, sub_zero, Pi.single_eq_of_ne, Ne.def, not_false_iff,
updateRow_self, updateRow_ne, cons_val_zero, of_apply, Nat.succ_succ_ne_one, Pi.single_eq_of_ne, updateRow_self,
Pi.single_eq_of_ne, Ne.def, Fin.zero_eq_one_iff, Nat.succ_succ_ne_one, not_false_iff, updateRow_ne,
Fin.one_eq_zero_iff, zero_mul, Pi.single_eq_same, one_mul, zero_sub, of_apply, cons_val', cons_val_fin_one,
cons_val_one, head_fin_const, neg_inj, eq_self_iff_true, cons_val_zero, head_cons, mul_one]
[GOAL]
m : Type u
n✝ : Type v
α : Type w
inst✝⁴ : DecidableEq n✝
inst✝³ : Fintype n✝
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
n : ℕ
A : Matrix (Fin (Nat.succ n)) (Fin (Nat.succ n)) α
i j : Fin (Nat.succ n)
⊢ adjugate A i j = (-1) ^ (↑j + ↑i) * det (submatrix A (Fin.succAbove j) (Fin.succAbove i))
[PROOFSTEP]
simp_rw [adjugate_apply, det_succ_row _ j, updateRow_self, submatrix_updateRow_succAbove]
[GOAL]
m : Type u
n✝ : Type v
α : Type w
inst✝⁴ : DecidableEq n✝
inst✝³ : Fintype n✝
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
n : ℕ
A : Matrix (Fin (Nat.succ n)) (Fin (Nat.succ n)) α
i j : Fin (Nat.succ n)
⊢ ∑ x : Fin (Nat.succ n), (-1) ^ (↑j + ↑x) * Pi.single i 1 x * det (submatrix A (Fin.succAbove j) (Fin.succAbove x)) =
(-1) ^ (↑j + ↑i) * det (submatrix A (Fin.succAbove j) (Fin.succAbove i))
[PROOFSTEP]
rw [Fintype.sum_eq_single i fun h hjk => ?_, Pi.single_eq_same, mul_one]
[GOAL]
m : Type u
n✝ : Type v
α : Type w
inst✝⁴ : DecidableEq n✝
inst✝³ : Fintype n✝
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
n : ℕ
A : Matrix (Fin (Nat.succ n)) (Fin (Nat.succ n)) α
i j h : Fin (Nat.succ n)
hjk : h ≠ i
⊢ (-1) ^ (↑j + ↑h) * Pi.single i 1 h * det (submatrix A (Fin.succAbove j) (Fin.succAbove h)) = 0
[PROOFSTEP]
rw [Pi.single_eq_of_ne hjk, mul_zero, zero_mul]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
haveI : Nonempty n := ⟨i⟩
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this : Nonempty n
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
obtain ⟨n', hn'⟩ := Nat.exists_eq_succ_of_ne_zero (Fintype.card_ne_zero : Fintype.card n ≠ 0)
[GOAL]
case intro
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
obtain ⟨e⟩ := Fintype.truncEquivFinOfCardEq hn'
[GOAL]
case intro.mk
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
x✝ : Trunc (n ≃ Fin (Nat.succ n'))
e : n ≃ Fin (Nat.succ n')
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
let A' := reindex e e A
[GOAL]
case intro.mk
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
x✝ : Trunc (n ≃ Fin (Nat.succ n'))
e : n ≃ Fin (Nat.succ n')
A' : (fun x => Matrix (Fin (Nat.succ n')) (Fin (Nat.succ n')) α) A := ↑(reindex e e) A
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
suffices det A' = ∑ j : Fin n'.succ, A' (e i) j * adjugate A' j (e i)
by
simp_rw [det_reindex_self, adjugate_reindex, reindex_apply, submatrix_apply, ← e.sum_comp, Equiv.symm_apply_apply] at
this
exact this
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this✝ : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
x✝ : Trunc (n ≃ Fin (Nat.succ n'))
e : n ≃ Fin (Nat.succ n')
A' : (fun x => Matrix (Fin (Nat.succ n')) (Fin (Nat.succ n')) α) A := ↑(reindex e e) A
this : det A' = ∑ j : Fin (Nat.succ n'), A' (↑e i) j * adjugate A' j (↑e i)
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
simp_rw [det_reindex_self, adjugate_reindex, reindex_apply, submatrix_apply, ← e.sum_comp, Equiv.symm_apply_apply] at
this
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this✝ : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
x✝ : Trunc (n ≃ Fin (Nat.succ n'))
e : n ≃ Fin (Nat.succ n')
A' : (fun x => Matrix (Fin (Nat.succ n')) (Fin (Nat.succ n')) α) A := ↑(reindex e e) A
this : det A = ∑ x : n, A i x * adjugate A x i
⊢ det A = ∑ j : n, A i j * adjugate A j i
[PROOFSTEP]
exact this
[GOAL]
case intro.mk
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
x✝ : Trunc (n ≃ Fin (Nat.succ n'))
e : n ≃ Fin (Nat.succ n')
A' : (fun x => Matrix (Fin (Nat.succ n')) (Fin (Nat.succ n')) α) A := ↑(reindex e e) A
⊢ det A' = ∑ j : Fin (Nat.succ n'), A' (↑e i) j * adjugate A' j (↑e i)
[PROOFSTEP]
rw [det_succ_row A' (e i)]
[GOAL]
case intro.mk
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
i : n
this : Nonempty n
n' : ℕ
hn' : Fintype.card n = Nat.succ n'
x✝ : Trunc (n ≃ Fin (Nat.succ n'))
e : n ≃ Fin (Nat.succ n')
A' : (fun x => Matrix (Fin (Nat.succ n')) (Fin (Nat.succ n')) α) A := ↑(reindex e e) A
⊢ ∑ j : Fin (Nat.succ n'),
(-1) ^ (↑(↑e i) + ↑j) * A' (↑e i) j * det (submatrix A' (Fin.succAbove (↑e i)) (Fin.succAbove j)) =
∑ j : Fin (Nat.succ n'), A' (↑e i) j * adjugate A' j (↑e i)
[PROOFSTEP]
simp_rw [mul_assoc, mul_left_comm _ (A' _ _), ← adjugate_fin_succ_eq_det_submatrix]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
j : n
⊢ det A = ∑ i : n, A i j * adjugate A j i
[PROOFSTEP]
simpa only [det_transpose, ← adjugate_transpose] using det_eq_sum_mul_adjugate_row Aᵀ j
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : StarRing α
A : Matrix n n α
⊢ (adjugate A)ᴴ = adjugate Aᴴ
[PROOFSTEP]
dsimp only [conjTranspose]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : StarRing α
A : Matrix n n α
⊢ map (adjugate A)ᵀ star = adjugate (map Aᵀ star)
[PROOFSTEP]
have : Aᵀ.adjugate.map star = adjugate (Aᵀ.map star) := (starRingEnd α).map_adjugate Aᵀ
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq m
inst✝² : Fintype m
inst✝¹ : CommRing α
inst✝ : StarRing α
A : Matrix n n α
this : map (adjugate Aᵀ) star = adjugate (map Aᵀ star)
⊢ map (adjugate A)ᵀ star = adjugate (map Aᵀ star)
[PROOFSTEP]
rw [A.adjugate_transpose, this]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
⊢ IsRegular A
[PROOFSTEP]
constructor
[GOAL]
case left
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
⊢ IsLeftRegular A
[PROOFSTEP]
intro B C h
[GOAL]
case left
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
B C : Matrix n n α
h : (fun x => A * x) B = (fun x => A * x) C
⊢ B = C
[PROOFSTEP]
refine' hA.matrix _
[GOAL]
case left
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
B C : Matrix n n α
h : (fun x => A * x) B = (fun x => A * x) C
⊢ (fun x => det A • x) B = (fun x => det A • x) C
[PROOFSTEP]
simp only at h ⊢
[GOAL]
case left
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
B C : Matrix n n α
h : A * B = A * C
⊢ det A • B = det A • C
[PROOFSTEP]
rw [← Matrix.one_mul B, ← Matrix.one_mul C, ← Matrix.smul_mul, ← Matrix.smul_mul, ← adjugate_mul, Matrix.mul_assoc,
Matrix.mul_assoc, h]
[GOAL]
case right
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
⊢ IsRightRegular A
[PROOFSTEP]
intro B C (h : B * A = C * A)
[GOAL]
case right
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
B C : Matrix n n α
h : B * A = C * A
⊢ B = C
[PROOFSTEP]
refine' hA.matrix _
[GOAL]
case right
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
B C : Matrix n n α
h : B * A = C * A
⊢ (fun x => det A • x) B = (fun x => det A • x) C
[PROOFSTEP]
simp only
[GOAL]
case right
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
hA : IsLeftRegular (det A)
B C : Matrix n n α
h : B * A = C * A
⊢ det A • B = det A • C
[PROOFSTEP]
rw [← Matrix.mul_one B, ← Matrix.mul_one C, ← Matrix.mul_smul, ← Matrix.mul_smul, ← mul_adjugate, ← Matrix.mul_assoc, ←
Matrix.mul_assoc, h]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
hA : IsLeftRegular (det A)
hB : IsLeftRegular (det B)
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
have hAB : IsLeftRegular (A * B).det := by
rw [det_mul]
exact hA.mul hB
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
hA : IsLeftRegular (det A)
hB : IsLeftRegular (det B)
⊢ IsLeftRegular (det (A * B))
[PROOFSTEP]
rw [det_mul]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
hA : IsLeftRegular (det A)
hB : IsLeftRegular (det B)
⊢ IsLeftRegular (det A * det B)
[PROOFSTEP]
exact hA.mul hB
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
hA : IsLeftRegular (det A)
hB : IsLeftRegular (det B)
hAB : IsLeftRegular (det (A * B))
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
refine' (isRegular_of_isLeftRegular_det hAB).left _
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
hA : IsLeftRegular (det A)
hB : IsLeftRegular (det B)
hAB : IsLeftRegular (det (A * B))
⊢ (fun x => A * B * x) (adjugate (A * B)) = (fun x => A * B * x) (adjugate B * adjugate A)
[PROOFSTEP]
simp only
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
hA : IsLeftRegular (det A)
hB : IsLeftRegular (det B)
hAB : IsLeftRegular (det (A * B))
⊢ A * B * adjugate (A * B) = A * B * (adjugate B * adjugate A)
[PROOFSTEP]
rw [mul_adjugate, Matrix.mul_assoc, ← Matrix.mul_assoc B, mul_adjugate, smul_mul, Matrix.one_mul, mul_smul,
mul_adjugate, smul_smul, mul_comm, ← det_mul]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
let g : Matrix n n α → Matrix n n α[X] := fun M => M.map Polynomial.C + (Polynomial.X : α[X]) • (1 : Matrix n n α[X])
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
let f' : Matrix n n α[X] →+* Matrix n n α := (Polynomial.evalRingHom 0).mapMatrix
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
have f'_inv : ∀ M, f' (g M) = M := by
intro
ext
simp
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
⊢ ∀ (M : Matrix n n α), ↑f' (g M) = M
[PROOFSTEP]
intro
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
M✝ : Matrix n n α
⊢ ↑f' (g M✝) = M✝
[PROOFSTEP]
ext
[GOAL]
case a.h
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
M✝ : Matrix n n α
i✝ x✝ : n
⊢ ↑f' (g M✝) i✝ x✝ = M✝ i✝ x✝
[PROOFSTEP]
simp
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
have f'_adj : ∀ M : Matrix n n α, f' (adjugate (g M)) = adjugate M :=
by
intro
rw [RingHom.map_adjugate, f'_inv]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
⊢ ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
[PROOFSTEP]
intro
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
M✝ : Matrix n n α
⊢ ↑f' (adjugate (g M✝)) = adjugate M✝
[PROOFSTEP]
rw [RingHom.map_adjugate, f'_inv]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
have f'_g_mul : ∀ M N : Matrix n n α, f' (g M * g N) = M * N :=
by
intros M N
rw [RingHom.map_mul, f'_inv, f'_inv]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
⊢ ∀ (M N : Matrix n n α), ↑f' (g M * g N) = M * N
[PROOFSTEP]
intros M N
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
M N : Matrix n n α
⊢ ↑f' (g M * g N) = M * N
[PROOFSTEP]
rw [RingHom.map_mul, f'_inv, f'_inv]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
f'_g_mul : ∀ (M N : Matrix n n α), ↑f' (g M * g N) = M * N
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
have hu : ∀ M : Matrix n n α, IsRegular (g M).det := by
intro M
refine' Polynomial.Monic.isRegular _
simp only [Polynomial.Monic.def, ← Polynomial.leadingCoeff_det_X_one_add_C M, add_comm]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
f'_g_mul : ∀ (M N : Matrix n n α), ↑f' (g M * g N) = M * N
⊢ ∀ (M : Matrix n n α), IsRegular (det (g M))
[PROOFSTEP]
intro M
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
f'_g_mul : ∀ (M N : Matrix n n α), ↑f' (g M * g N) = M * N
M : Matrix n n α
⊢ IsRegular (det (g M))
[PROOFSTEP]
refine' Polynomial.Monic.isRegular _
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
f'_g_mul : ∀ (M N : Matrix n n α), ↑f' (g M * g N) = M * N
M : Matrix n n α
⊢ Monic (det (g M))
[PROOFSTEP]
simp only [Polynomial.Monic.def, ← Polynomial.leadingCoeff_det_X_one_add_C M, add_comm]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A B : Matrix n n α
g : Matrix n n α → Matrix n n α[X] := fun M => map M ↑C + X • 1
f' : Matrix n n α[X] →+* Matrix n n α := RingHom.mapMatrix (evalRingHom 0)
f'_inv : ∀ (M : Matrix n n α), ↑f' (g M) = M
f'_adj : ∀ (M : Matrix n n α), ↑f' (adjugate (g M)) = adjugate M
f'_g_mul : ∀ (M N : Matrix n n α), ↑f' (g M * g N) = M * N
hu : ∀ (M : Matrix n n α), IsRegular (det (g M))
⊢ adjugate (A * B) = adjugate B * adjugate A
[PROOFSTEP]
rw [← f'_adj, ← f'_adj, ← f'_adj, ← f'.map_mul, ← adjugate_mul_distrib_aux _ _ (hu A).left (hu B).left,
RingHom.map_adjugate, RingHom.map_adjugate, f'_inv, f'_g_mul]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
k : ℕ
⊢ adjugate (A ^ k) = adjugate A ^ k
[PROOFSTEP]
induction' k with k IH
[GOAL]
case zero
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ adjugate (A ^ Nat.zero) = adjugate A ^ Nat.zero
[PROOFSTEP]
simp
[GOAL]
case succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
k : ℕ
IH : adjugate (A ^ k) = adjugate A ^ k
⊢ adjugate (A ^ Nat.succ k) = adjugate A ^ Nat.succ k
[PROOFSTEP]
rw [pow_succ', adjugate_mul_distrib, IH, pow_succ]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ det A • adjugate (adjugate A) = det A ^ (Fintype.card n - 1) • A
[PROOFSTEP]
have : A * (A.adjugate * A.adjugate.adjugate) = A * (A.det ^ (Fintype.card n - 1) • (1 : Matrix n n α)) := by
rw [← adjugate_mul_distrib, adjugate_mul, adjugate_smul, adjugate_one]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
⊢ A * (adjugate A * adjugate (adjugate A)) = A * det A ^ (Fintype.card n - 1) • 1
[PROOFSTEP]
rw [← adjugate_mul_distrib, adjugate_mul, adjugate_smul, adjugate_one]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
this : A * (adjugate A * adjugate (adjugate A)) = A * det A ^ (Fintype.card n - 1) • 1
⊢ det A • adjugate (adjugate A) = det A ^ (Fintype.card n - 1) • A
[PROOFSTEP]
rwa [← Matrix.mul_assoc, mul_adjugate, Matrix.mul_smul, Matrix.mul_one, Matrix.smul_mul, Matrix.one_mul] at this
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
⊢ adjugate (adjugate A) = det A ^ (Fintype.card n - 2) • A
[PROOFSTEP]
cases' h_card : Fintype.card n with n'
[GOAL]
case zero
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
h_card : Fintype.card n = Nat.zero
⊢ adjugate (adjugate A) = det A ^ (Nat.zero - 2) • A
[PROOFSTEP]
haveI : IsEmpty n := Fintype.card_eq_zero_iff.mp h_card
[GOAL]
case zero
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
h_card : Fintype.card n = Nat.zero
this : IsEmpty n
⊢ adjugate (adjugate A) = det A ^ (Nat.zero - 2) • A
[PROOFSTEP]
apply Subsingleton.elim
[GOAL]
case succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n' : ℕ
h_card : Fintype.card n = Nat.succ n'
⊢ adjugate (adjugate A) = det A ^ (Nat.succ n' - 2) • A
[PROOFSTEP]
cases n'
[GOAL]
case succ.zero
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
h_card : Fintype.card n = Nat.succ Nat.zero
⊢ adjugate (adjugate A) = det A ^ (Nat.succ Nat.zero - 2) • A
[PROOFSTEP]
exact (h h_card).elim
[GOAL]
case succ.succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
⊢ adjugate (adjugate A) = det A ^ (Nat.succ (Nat.succ n✝) - 2) • A
[PROOFSTEP]
rw [← h_card]
-- express `A` as an evaluation of a polynomial in n^2 variables, and solve in the polynomial ring
-- where `A'.det` is non-zero.
[GOAL]
case succ.succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
⊢ adjugate (adjugate A) = det A ^ (Fintype.card n - 2) • A
[PROOFSTEP]
let A' := mvPolynomialX n n ℤ
[GOAL]
case succ.succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ adjugate (adjugate A) = det A ^ (Fintype.card n - 2) • A
[PROOFSTEP]
suffices adjugate (adjugate A') = det A' ^ (Fintype.card n - 2) • A' by
rw [← mvPolynomialX_mapMatrix_aeval ℤ A, ← AlgHom.map_adjugate, ← AlgHom.map_adjugate, this, ← AlgHom.map_det, ←
AlgHom.map_pow, AlgHom.mapMatrix_apply, AlgHom.mapMatrix_apply, Matrix.map_smul' _ _ _ (_root_.map_mul _)]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
this : adjugate (adjugate A') = det A' ^ (Fintype.card n - 2) • A'
⊢ adjugate (adjugate A) = det A ^ (Fintype.card n - 2) • A
[PROOFSTEP]
rw [← mvPolynomialX_mapMatrix_aeval ℤ A, ← AlgHom.map_adjugate, ← AlgHom.map_adjugate, this, ← AlgHom.map_det, ←
AlgHom.map_pow, AlgHom.mapMatrix_apply, AlgHom.mapMatrix_apply, Matrix.map_smul' _ _ _ (_root_.map_mul _)]
[GOAL]
case succ.succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ adjugate (adjugate A') = det A' ^ (Fintype.card n - 2) • A'
[PROOFSTEP]
have h_card' : Fintype.card n - 2 + 1 = Fintype.card n - 1 := by simp [h_card]
[GOAL]
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
⊢ Fintype.card n - 2 + 1 = Fintype.card n - 1
[PROOFSTEP]
simp [h_card]
[GOAL]
case succ.succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
h_card' : Fintype.card n - 2 + 1 = Fintype.card n - 1
⊢ adjugate (adjugate A') = det A' ^ (Fintype.card n - 2) • A'
[PROOFSTEP]
have is_reg : IsSMulRegular (MvPolynomial (n × n) ℤ) (det A') := fun x y =>
mul_left_cancel₀ (det_mvPolynomialX_ne_zero n ℤ)
[GOAL]
case succ.succ
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
h_card' : Fintype.card n - 2 + 1 = Fintype.card n - 1
is_reg : IsSMulRegular (MvPolynomial (n × n) ℤ) (det A')
⊢ adjugate (adjugate A') = det A' ^ (Fintype.card n - 2) • A'
[PROOFSTEP]
apply is_reg.matrix
[GOAL]
case succ.succ.a
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
h_card' : Fintype.card n - 2 + 1 = Fintype.card n - 1
is_reg : IsSMulRegular (MvPolynomial (n × n) ℤ) (det A')
⊢ (fun x => det A' • x) (adjugate (adjugate A')) = (fun x => det A' • x) (det A' ^ (Fintype.card n - 2) • A')
[PROOFSTEP]
simp only
[GOAL]
case succ.succ.a
m : Type u
n : Type v
α : Type w
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : CommRing α
A : Matrix n n α
h : Fintype.card n ≠ 1
n✝ : ℕ
h_card : Fintype.card n = Nat.succ (Nat.succ n✝)
A' : Matrix n n (MvPolynomial (n × n) ℤ) := mvPolynomialX n n ℤ
h_card' : Fintype.card n - 2 + 1 = Fintype.card n - 1
is_reg : IsSMulRegular (MvPolynomial (n × n) ℤ) (det A')
⊢ det (mvPolynomialX n n ℤ) • adjugate (adjugate (mvPolynomialX n n ℤ)) =
det (mvPolynomialX n n ℤ) • det (mvPolynomialX n n ℤ) ^ (Fintype.card n - 2) • mvPolynomialX n n ℤ
[PROOFSTEP]
rw [smul_smul, ← pow_succ, h_card', det_smul_adjugate_adjugate]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Adjugate", "llama_tokens": 39596} |
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
⊢ Monoid M
[PROOFSTEP]
infer_instance
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
src✝ : Monoid M :=
let_fun this := inferInstance;
this
⊢ Inv M
[PROOFSTEP]
infer_instance
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ A⁻¹ ^ n = (A ^ n)⁻¹
[PROOFSTEP]
induction' n with n ih
[GOAL]
case zero
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
⊢ A⁻¹ ^ Nat.zero = (A ^ Nat.zero)⁻¹
[PROOFSTEP]
simp
[GOAL]
case succ
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
ih : A⁻¹ ^ n = (A ^ n)⁻¹
⊢ A⁻¹ ^ Nat.succ n = (A ^ Nat.succ n)⁻¹
[PROOFSTEP]
rw [pow_succ A, mul_inv_rev, ← ih, ← pow_succ']
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℕ
ha : IsUnit (det A)
h : n ≤ m
⊢ A ^ (m - n) = A ^ m * (A ^ n)⁻¹
[PROOFSTEP]
rw [← tsub_add_cancel_of_le h, pow_add, Matrix.mul_assoc, mul_nonsing_inv, tsub_add_cancel_of_le h, Matrix.mul_one]
[GOAL]
case h
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℕ
ha : IsUnit (det A)
h : n ≤ m
⊢ IsUnit (det (A ^ n))
[PROOFSTEP]
simpa using ha.pow n
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℕ
⊢ A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
[PROOFSTEP]
induction' n with n IH generalizing m
[GOAL]
case zero
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ m : ℕ
⊢ A⁻¹ ^ m * A ^ Nat.zero = A ^ Nat.zero * A⁻¹ ^ m
[PROOFSTEP]
simp
[GOAL]
case succ
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
⊢ A⁻¹ ^ m * A ^ Nat.succ n = A ^ Nat.succ n * A⁻¹ ^ m
[PROOFSTEP]
cases' m with m m
[GOAL]
case succ.zero
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
⊢ A⁻¹ ^ Nat.zero * A ^ Nat.succ n = A ^ Nat.succ n * A⁻¹ ^ Nat.zero
[PROOFSTEP]
simp
[GOAL]
case succ.succ
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
⊢ A⁻¹ ^ Nat.succ m * A ^ Nat.succ n = A ^ Nat.succ n * A⁻¹ ^ Nat.succ m
[PROOFSTEP]
rcases nonsing_inv_cancel_or_zero A with (⟨h, h'⟩ | h)
[GOAL]
case succ.succ.inl.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ * A = 1
h' : A * A⁻¹ = 1
⊢ A⁻¹ ^ Nat.succ m * A ^ Nat.succ n = A ^ Nat.succ n * A⁻¹ ^ Nat.succ m
[PROOFSTEP]
simp only [Nat.succ_eq_add_one]
[GOAL]
case succ.succ.inl.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ * A = 1
h' : A * A⁻¹ = 1
⊢ A⁻¹ ^ (m + 1) * A ^ (n + 1) = A ^ (n + 1) * A⁻¹ ^ (m + 1)
[PROOFSTEP]
calc
A⁻¹ ^ (m + 1) * A ^ (n + 1) = A⁻¹ ^ m * (A⁻¹ * A) * A ^ n := by
simp only [pow_succ' A⁻¹, pow_succ A, Matrix.mul_assoc]
_ = A ^ n * A⁻¹ ^ m := by simp only [h, Matrix.mul_one, Matrix.one_mul, IH m]
_ = A ^ n * (A * A⁻¹) * A⁻¹ ^ m := by simp only [h', Matrix.mul_one, Matrix.one_mul]
_ = A ^ (n + 1) * A⁻¹ ^ (m + 1) := by simp only [pow_succ' A, pow_succ A⁻¹, Matrix.mul_assoc]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ * A = 1
h' : A * A⁻¹ = 1
⊢ A⁻¹ ^ (m + 1) * A ^ (n + 1) = A⁻¹ ^ m * (A⁻¹ * A) * A ^ n
[PROOFSTEP]
simp only [pow_succ' A⁻¹, pow_succ A, Matrix.mul_assoc]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ * A = 1
h' : A * A⁻¹ = 1
⊢ A⁻¹ ^ m * (A⁻¹ * A) * A ^ n = A ^ n * A⁻¹ ^ m
[PROOFSTEP]
simp only [h, Matrix.mul_one, Matrix.one_mul, IH m]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ * A = 1
h' : A * A⁻¹ = 1
⊢ A ^ n * A⁻¹ ^ m = A ^ n * (A * A⁻¹) * A⁻¹ ^ m
[PROOFSTEP]
simp only [h', Matrix.mul_one, Matrix.one_mul]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ * A = 1
h' : A * A⁻¹ = 1
⊢ A ^ n * (A * A⁻¹) * A⁻¹ ^ m = A ^ (n + 1) * A⁻¹ ^ (m + 1)
[PROOFSTEP]
simp only [pow_succ' A, pow_succ A⁻¹, Matrix.mul_assoc]
[GOAL]
case succ.succ.inr
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m✝ n : ℕ
IH : ∀ (m : ℕ), A⁻¹ ^ m * A ^ n = A ^ n * A⁻¹ ^ m
m : ℕ
h : A⁻¹ = 0
⊢ A⁻¹ ^ Nat.succ m * A ^ Nat.succ n = A ^ Nat.succ n * A⁻¹ ^ Nat.succ m
[PROOFSTEP]
simp [h]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℕ
⊢ 1 ^ ↑n = 1
[PROOFSTEP]
rw [zpow_ofNat, one_pow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℕ
⊢ 1 ^ -[n+1] = 1
[PROOFSTEP]
rw [zpow_negSucc, one_pow, inv_one]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℕ
h : ↑n ≠ 0
⊢ 0 ^ ↑n = 0
[PROOFSTEP]
rw [zpow_ofNat, zero_pow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℕ
h : ↑n ≠ 0
⊢ 0 < n
[PROOFSTEP]
refine' lt_of_le_of_ne n.zero_le (Ne.symm _)
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℕ
h : ↑n ≠ 0
⊢ n ≠ 0
[PROOFSTEP]
simpa using h
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℕ
x✝ : -[n+1] ≠ 0
⊢ 0 ^ -[n+1] = 0
[PROOFSTEP]
simp [zero_pow n.zero_lt_succ]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℤ
⊢ 0 ^ n = if n = 0 then 1 else 0
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℤ
h : n = 0
⊢ 0 ^ n = 1
[PROOFSTEP]
rw [h, zpow_zero]
[GOAL]
case neg
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℤ
h : ¬n = 0
⊢ 0 ^ n = 0
[PROOFSTEP]
rw [zero_zpow _ h]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ A⁻¹ ^ ↑n = (A ^ ↑n)⁻¹
[PROOFSTEP]
rw [zpow_ofNat, zpow_ofNat, inv_pow']
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ A⁻¹ ^ -[n+1] = (A ^ -[n+1])⁻¹
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, inv_pow']
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
⊢ A ^ (-1) = A⁻¹
[PROOFSTEP]
convert DivInvMonoid.zpow_neg' 0 A
[GOAL]
case h.e'_3.h.e'_3
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
⊢ A = DivInvMonoid.zpow (↑(Nat.succ 0)) A
[PROOFSTEP]
simp only [zpow_one, Int.ofNat_zero, Int.ofNat_succ, zpow_eq_pow, zero_add]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ A ^ (-↑n) = (A ^ n)⁻¹
[PROOFSTEP]
cases n
[GOAL]
case zero
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
⊢ A ^ (-↑Nat.zero) = (A ^ Nat.zero)⁻¹
[PROOFSTEP]
simp
[GOAL]
case succ
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n✝ : ℕ
⊢ A ^ (-↑(Nat.succ n✝)) = (A ^ Nat.succ n✝)⁻¹
[PROOFSTEP]
exact DivInvMonoid.zpow_neg' _ _
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℤ
⊢ IsUnit (det (A ^ n))
[PROOFSTEP]
cases' n with n n
[GOAL]
case ofNat
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ IsUnit (det (A ^ ofNat n))
[PROOFSTEP]
simpa using h.pow n
[GOAL]
case negSucc
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ IsUnit (det (A ^ -[n+1]))
[PROOFSTEP]
simpa using h.pow n.succ
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
z : ℤ
⊢ IsUnit (det (A ^ z)) ↔ IsUnit (det A) ∨ z = 0
[PROOFSTEP]
induction' z using Int.induction_on with z _ z _
[GOAL]
case hz
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
⊢ IsUnit (det (A ^ 0)) ↔ IsUnit (det A) ∨ 0 = 0
[PROOFSTEP]
simp
[GOAL]
case hp
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
z : ℕ
a✝ : IsUnit (det (A ^ ↑z)) ↔ IsUnit (det A) ∨ ↑z = 0
⊢ IsUnit (det (A ^ (↑z + 1))) ↔ IsUnit (det A) ∨ ↑z + 1 = 0
[PROOFSTEP]
rw [← Int.ofNat_succ, zpow_ofNat, det_pow, isUnit_pow_succ_iff, ← Int.ofNat_zero, Int.ofNat_inj]
[GOAL]
case hp
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
z : ℕ
a✝ : IsUnit (det (A ^ ↑z)) ↔ IsUnit (det A) ∨ ↑z = 0
⊢ IsUnit (det A) ↔ IsUnit (det A) ∨ Nat.succ z = 0
[PROOFSTEP]
simp
[GOAL]
case hn
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
z : ℕ
a✝ : IsUnit (det (A ^ (-↑z))) ↔ IsUnit (det A) ∨ -↑z = 0
⊢ IsUnit (det (A ^ (-↑z - 1))) ↔ IsUnit (det A) ∨ -↑z - 1 = 0
[PROOFSTEP]
rw [← neg_add', ← Int.ofNat_succ, zpow_neg_coe_nat, isUnit_nonsing_inv_det_iff, det_pow, isUnit_pow_succ_iff,
neg_eq_zero, ← Int.ofNat_zero, Int.ofNat_inj]
[GOAL]
case hn
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
z : ℕ
a✝ : IsUnit (det (A ^ (-↑z))) ↔ IsUnit (det A) ∨ -↑z = 0
⊢ IsUnit (det A) ↔ IsUnit (det A) ∨ Nat.succ z = 0
[PROOFSTEP]
simp
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ A ^ (- -[n+1]) = (A ^ -[n+1])⁻¹
[PROOFSTEP]
rw [zpow_negSucc, neg_negSucc, zpow_ofNat, nonsing_inv_nonsing_inv]
[GOAL]
case h
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ IsUnit (det (A ^ (n + 1)))
[PROOFSTEP]
rw [det_pow]
[GOAL]
case h
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ IsUnit (det A ^ (n + 1))
[PROOFSTEP]
exact h.pow _
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℤ
⊢ A⁻¹ ^ n = A ^ (-n)
[PROOFSTEP]
rw [zpow_neg h, inv_zpow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ A ^ (↑n + 1) = A ^ ↑n * A
[PROOFSTEP]
simp only [← Nat.cast_succ, pow_succ', zpow_ofNat]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ A ^ (-(↑n + 1) + 1) = (A ^ n)⁻¹
[PROOFSTEP]
rw [neg_add, neg_add_cancel_right, zpow_neg h, zpow_ofNat]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ (A ^ n)⁻¹ = (A * A ^ n)⁻¹ * A
[PROOFSTEP]
rw [mul_inv_rev, Matrix.mul_assoc, nonsing_inv_mul _ h, Matrix.mul_one]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℕ
⊢ (A * A ^ n)⁻¹ * A = A ^ (-(↑n + 1)) * A
[PROOFSTEP]
rw [zpow_neg h, ← Int.ofNat_succ, zpow_ofNat, pow_succ]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℤ
⊢ A ^ (n - 1) = A ^ (n - 1) * A * A⁻¹
[PROOFSTEP]
rw [mul_assoc, mul_nonsing_inv _ h, mul_one]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
n : ℤ
⊢ A ^ (n - 1) * A * A⁻¹ = A ^ n * A⁻¹
[PROOFSTEP]
rw [← zpow_add_one h, sub_add_cancel]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m n : ℤ
⊢ A ^ (m + n) = A ^ m * A ^ n
[PROOFSTEP]
induction n using Int.induction_on with
| hz => simp
| hp n ihn => simp only [← add_assoc, zpow_add_one ha, ihn, mul_assoc]
| hn n ihn => rw [zpow_sub_one ha, ← mul_assoc, ← ihn, ← zpow_sub_one ha, add_sub_assoc]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m n : ℤ
⊢ A ^ (m + n) = A ^ m * A ^ n
[PROOFSTEP]
induction n using Int.induction_on with
| hz => simp
| hp n ihn => simp only [← add_assoc, zpow_add_one ha, ihn, mul_assoc]
| hn n ihn => rw [zpow_sub_one ha, ← mul_assoc, ← ihn, ← zpow_sub_one ha, add_sub_assoc]
[GOAL]
case hz
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m : ℤ
⊢ A ^ (m + 0) = A ^ m * A ^ 0
[PROOFSTEP]
| hz => simp
[GOAL]
case hz
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m : ℤ
⊢ A ^ (m + 0) = A ^ m * A ^ 0
[PROOFSTEP]
simp
[GOAL]
case hp
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m : ℤ
n : ℕ
ihn : A ^ (m + ↑n) = A ^ m * A ^ ↑n
⊢ A ^ (m + (↑n + 1)) = A ^ m * A ^ (↑n + 1)
[PROOFSTEP]
| hp n ihn => simp only [← add_assoc, zpow_add_one ha, ihn, mul_assoc]
[GOAL]
case hp
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m : ℤ
n : ℕ
ihn : A ^ (m + ↑n) = A ^ m * A ^ ↑n
⊢ A ^ (m + (↑n + 1)) = A ^ m * A ^ (↑n + 1)
[PROOFSTEP]
simp only [← add_assoc, zpow_add_one ha, ihn, mul_assoc]
[GOAL]
case hn
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m : ℤ
n : ℕ
ihn : A ^ (m + -↑n) = A ^ m * A ^ (-↑n)
⊢ A ^ (m + (-↑n - 1)) = A ^ m * A ^ (-↑n - 1)
[PROOFSTEP]
| hn n ihn => rw [zpow_sub_one ha, ← mul_assoc, ← ihn, ← zpow_sub_one ha, add_sub_assoc]
[GOAL]
case hn
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
m : ℤ
n : ℕ
ihn : A ^ (m + -↑n) = A ^ m * A ^ (-↑n)
⊢ A ^ (m + (-↑n - 1)) = A ^ m * A ^ (-↑n - 1)
[PROOFSTEP]
rw [zpow_sub_one ha, ← mul_assoc, ← ihn, ← zpow_sub_one ha, add_sub_assoc]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℤ
hm : m ≤ 0
hn : n ≤ 0
⊢ A ^ (m + n) = A ^ m * A ^ n
[PROOFSTEP]
rcases nonsing_inv_cancel_or_zero A with (⟨h, _⟩ | h)
[GOAL]
case inl.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℤ
hm : m ≤ 0
hn : n ≤ 0
h : A⁻¹ * A = 1
right✝ : A * A⁻¹ = 1
⊢ A ^ (m + n) = A ^ m * A ^ n
[PROOFSTEP]
exact zpow_add (isUnit_det_of_left_inverse h) m n
[GOAL]
case inr
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℤ
hm : m ≤ 0
hn : n ≤ 0
h : A⁻¹ = 0
⊢ A ^ (m + n) = A ^ m * A ^ n
[PROOFSTEP]
obtain ⟨k, rfl⟩ := exists_eq_neg_ofNat hm
[GOAL]
case inr.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
hn : n ≤ 0
h : A⁻¹ = 0
k : ℕ
hm : -↑k ≤ 0
⊢ A ^ (-↑k + n) = A ^ (-↑k) * A ^ n
[PROOFSTEP]
obtain ⟨l, rfl⟩ := exists_eq_neg_ofNat hn
[GOAL]
case inr.intro.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : A⁻¹ = 0
k : ℕ
hm : -↑k ≤ 0
l : ℕ
hn : -↑l ≤ 0
⊢ A ^ (-↑k + -↑l) = A ^ (-↑k) * A ^ (-↑l)
[PROOFSTEP]
simp_rw [← neg_add, ← Int.ofNat_add, zpow_neg_coe_nat, ← inv_pow', h, pow_add]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
m n : ℤ
hm : 0 ≤ m
hn : 0 ≤ n
⊢ A ^ (m + n) = A ^ m * A ^ n
[PROOFSTEP]
obtain ⟨k, rfl⟩ := eq_ofNat_of_zero_le hm
[GOAL]
case intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
hn : 0 ≤ n
k : ℕ
hm : 0 ≤ ↑k
⊢ A ^ (↑k + n) = A ^ ↑k * A ^ n
[PROOFSTEP]
obtain ⟨l, rfl⟩ := eq_ofNat_of_zero_le hn
[GOAL]
case intro.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
k : ℕ
hm : 0 ≤ ↑k
l : ℕ
hn : 0 ≤ ↑l
⊢ A ^ (↑k + ↑l) = A ^ ↑k * A ^ ↑l
[PROOFSTEP]
rw [← Int.ofNat_add, zpow_ofNat, zpow_ofNat, zpow_ofNat, pow_add]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
i : ℤ
⊢ A ^ (1 + i) = A * A ^ i
[PROOFSTEP]
rw [zpow_add h, zpow_one]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
⊢ SemiconjBy A (X ^ ↑n) (Y ^ ↑n)
[PROOFSTEP]
simp [h.pow_right n]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
⊢ SemiconjBy A (X ^ -[n+1]) (Y ^ -[n+1])
[PROOFSTEP]
have hx' : IsUnit (X ^ n.succ).det := by
rw [det_pow]
exact hx.pow n.succ
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
⊢ IsUnit (det (X ^ Nat.succ n))
[PROOFSTEP]
rw [det_pow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
⊢ IsUnit (det X ^ Nat.succ n)
[PROOFSTEP]
exact hx.pow n.succ
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
⊢ SemiconjBy A (X ^ -[n+1]) (Y ^ -[n+1])
[PROOFSTEP]
have hy' : IsUnit (Y ^ n.succ).det := by
rw [det_pow]
exact hy.pow n.succ
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
⊢ IsUnit (det (Y ^ Nat.succ n))
[PROOFSTEP]
rw [det_pow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
⊢ IsUnit (det Y ^ Nat.succ n)
[PROOFSTEP]
exact hy.pow n.succ
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
hy' : IsUnit (det (Y ^ Nat.succ n))
⊢ SemiconjBy A (X ^ -[n+1]) (Y ^ -[n+1])
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, nonsing_inv_apply _ hx', nonsing_inv_apply _ hy', SemiconjBy]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
hy' : IsUnit (det (Y ^ Nat.succ n))
⊢ A * ↑(IsUnit.unit hx')⁻¹ • adjugate (X ^ Nat.succ n) = ↑(IsUnit.unit hy')⁻¹ • adjugate (Y ^ Nat.succ n) * A
[PROOFSTEP]
refine' (isRegular_of_isLeftRegular_det hy'.isRegular.left).left _
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
hy' : IsUnit (det (Y ^ Nat.succ n))
⊢ (fun x => Y ^ Nat.succ n * x) (A * ↑(IsUnit.unit hx')⁻¹ • adjugate (X ^ Nat.succ n)) =
(fun x => Y ^ Nat.succ n * x) (↑(IsUnit.unit hy')⁻¹ • adjugate (Y ^ Nat.succ n) * A)
[PROOFSTEP]
dsimp only
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A X Y : M
hx : IsUnit (det X)
hy : IsUnit (det Y)
h : SemiconjBy A X Y
n : ℕ
hx' : IsUnit (det (X ^ Nat.succ n))
hy' : IsUnit (det (Y ^ Nat.succ n))
⊢ Y ^ Nat.succ n * (A * ↑(IsUnit.unit hx')⁻¹ • adjugate (X ^ Nat.succ n)) =
Y ^ Nat.succ n * (↑(IsUnit.unit hy')⁻¹ • adjugate (Y ^ Nat.succ n) * A)
[PROOFSTEP]
rw [← mul_assoc, ← (h.pow_right n.succ).eq, mul_assoc, mul_smul, mul_adjugate, ← Matrix.mul_assoc,
mul_smul (Y ^ _) (↑hy'.unit⁻¹ : R), mul_adjugate, smul_smul, smul_smul, hx'.val_inv_mul, hy'.val_inv_mul, one_smul,
Matrix.mul_one, Matrix.one_mul]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
m : ℤ
⊢ Commute A (B ^ m)
[PROOFSTEP]
rcases nonsing_inv_cancel_or_zero B with (⟨hB, _⟩ | hB)
[GOAL]
case inl.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
m : ℤ
hB : B⁻¹ * B = 1
right✝ : B * B⁻¹ = 1
⊢ Commute A (B ^ m)
[PROOFSTEP]
refine' SemiconjBy.zpow_right _ _ h _
[GOAL]
case inl.intro.refine'_1
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
m : ℤ
hB : B⁻¹ * B = 1
right✝ : B * B⁻¹ = 1
⊢ IsUnit (det B)
[PROOFSTEP]
exact isUnit_det_of_left_inverse hB
[GOAL]
case inl.intro.refine'_2
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
m : ℤ
hB : B⁻¹ * B = 1
right✝ : B * B⁻¹ = 1
⊢ IsUnit (det B)
[PROOFSTEP]
exact isUnit_det_of_left_inverse hB
[GOAL]
case inr
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
m : ℤ
hB : B⁻¹ = 0
⊢ Commute A (B ^ m)
[PROOFSTEP]
cases m
[GOAL]
case inr.ofNat
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
hB : B⁻¹ = 0
a✝ : ℕ
⊢ Commute A (B ^ ofNat a✝)
[PROOFSTEP]
simpa using h.pow_right _
[GOAL]
case inr.negSucc
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
hB : B⁻¹ = 0
a✝ : ℕ
⊢ Commute A (B ^ -[a✝+1])
[PROOFSTEP]
simp [← inv_pow', hB]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
⊢ A ^ bit0 n = A ^ n * A ^ n
[PROOFSTEP]
cases' le_total 0 n with nonneg nonpos
[GOAL]
case inl
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
nonneg : 0 ≤ n
⊢ A ^ bit0 n = A ^ n * A ^ n
[PROOFSTEP]
exact zpow_add_of_nonneg nonneg nonneg
[GOAL]
case inr
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
nonpos : n ≤ 0
⊢ A ^ bit0 n = A ^ n * A ^ n
[PROOFSTEP]
exact zpow_add_of_nonpos nonpos nonpos
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
x✝ : ↑n ≠ -1
⊢ A ^ (↑n + 1) = A ^ ↑n * A
[PROOFSTEP]
simp only [pow_succ', ← Nat.cast_succ, zpow_ofNat]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
x✝ : -(↑n + 2) ≠ -1
⊢ A ^ (-(↑n + 2) + 1) = A ^ (-(↑n + 2)) * A
[PROOFSTEP]
rcases nonsing_inv_cancel_or_zero A with (⟨h, _⟩ | h)
[GOAL]
case inl.intro
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
x✝ : -(↑n + 2) ≠ -1
h : A⁻¹ * A = 1
right✝ : A * A⁻¹ = 1
⊢ A ^ (-(↑n + 2) + 1) = A ^ (-(↑n + 2)) * A
[PROOFSTEP]
apply zpow_add_one (isUnit_det_of_left_inverse h)
[GOAL]
case inr
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
x✝ : -(↑n + 2) ≠ -1
h : A⁻¹ = 0
⊢ A ^ (-(↑n + 2) + 1) = A ^ (-(↑n + 2)) * A
[PROOFSTEP]
show A ^ (-((n + 1 : ℕ) : ℤ)) = A ^ (-((n + 2 : ℕ) : ℤ)) * A
[GOAL]
case inr
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
x✝ : -(↑n + 2) ≠ -1
h : A⁻¹ = 0
⊢ A ^ (-↑(n + 1)) = A ^ (-↑(n + 2)) * A
[PROOFSTEP]
simp_rw [zpow_neg_coe_nat, ← inv_pow', h, zero_pow Nat.succ_pos', zero_mul]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
⊢ A ^ bit1 n = A ^ n * A ^ n * A
[PROOFSTEP]
rw [bit1, zpow_add_one_of_ne_neg_one, zpow_bit0]
[GOAL]
case a
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
⊢ bit0 n ≠ -1
[PROOFSTEP]
intro h
[GOAL]
case a
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
h : bit0 n = -1
⊢ False
[PROOFSTEP]
simpa using congr_arg bodd h
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℕ
⊢ A ^ (↑m * ↑n) = (A ^ ↑m) ^ ↑n
[PROOFSTEP]
rw [zpow_ofNat, zpow_ofNat, ← pow_mul, ← zpow_ofNat, Int.ofNat_mul]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℕ
⊢ A ^ (↑m * -[n+1]) = (A ^ ↑m) ^ -[n+1]
[PROOFSTEP]
rw [zpow_ofNat, zpow_negSucc, ← pow_mul, ofNat_mul_negSucc, zpow_neg_coe_nat]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℕ
⊢ A ^ (-[m+1] * ↑n) = (A ^ -[m+1]) ^ ↑n
[PROOFSTEP]
rw [zpow_ofNat, zpow_negSucc, ← inv_pow', ← pow_mul, negSucc_mul_ofNat, zpow_neg_coe_nat, inv_pow']
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℕ
⊢ A ^ (-[m+1] * -[n+1]) = (A ^ -[m+1]) ^ -[n+1]
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, negSucc_mul_negSucc, ← Int.ofNat_mul, zpow_ofNat, inv_pow', ← pow_mul,
nonsing_inv_nonsing_inv]
[GOAL]
case h
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℕ
⊢ IsUnit (det (A ^ ((m + 1) * (n + 1))))
[PROOFSTEP]
rw [det_pow]
[GOAL]
case h
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℕ
⊢ IsUnit (det A ^ ((m + 1) * (n + 1)))
[PROOFSTEP]
exact h.pow _
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
h : IsUnit (det A)
m n : ℤ
⊢ A ^ (m * n) = (A ^ n) ^ m
[PROOFSTEP]
rw [mul_comm, zpow_mul _ h]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
u : Mˣ
n : ℕ
⊢ ↑(u ^ ↑n) = ↑u ^ ↑n
[PROOFSTEP]
rw [_root_.zpow_coe_nat, zpow_ofNat, Units.val_pow_eq_pow_val]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
u : Mˣ
k : ℕ
⊢ ↑(u ^ -[k+1]) = ↑u ^ -[k+1]
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, ← inv_pow, u⁻¹.val_pow_eq_pow_val, ← inv_pow', coe_units_inv]
[GOAL]
n' : Type u_1
inst✝⁴ : DecidableEq n'
inst✝³ : Fintype n'
R : Type u_2
inst✝² : CommRing R
inst✝¹ : Nonempty n'
inst✝ : Nontrivial R
A : M
ha : IsUnit (det A)
z : ℤ
⊢ A ^ z ≠ 0
[PROOFSTEP]
have := ha.det_zpow z
[GOAL]
n' : Type u_1
inst✝⁴ : DecidableEq n'
inst✝³ : Fintype n'
R : Type u_2
inst✝² : CommRing R
inst✝¹ : Nonempty n'
inst✝ : Nontrivial R
A : M
ha : IsUnit (det A)
z : ℤ
this : IsUnit (det (A ^ z))
⊢ A ^ z ≠ 0
[PROOFSTEP]
contrapose! this
[GOAL]
n' : Type u_1
inst✝⁴ : DecidableEq n'
inst✝³ : Fintype n'
R : Type u_2
inst✝² : CommRing R
inst✝¹ : Nonempty n'
inst✝ : Nontrivial R
A : M
ha : IsUnit (det A)
z : ℤ
this : A ^ z = 0
⊢ ¬IsUnit (det (A ^ z))
[PROOFSTEP]
rw [this, det_zero ‹_›]
[GOAL]
n' : Type u_1
inst✝⁴ : DecidableEq n'
inst✝³ : Fintype n'
R : Type u_2
inst✝² : CommRing R
inst✝¹ : Nonempty n'
inst✝ : Nontrivial R
A : M
ha : IsUnit (det A)
z : ℤ
this : A ^ z = 0
⊢ ¬IsUnit 0
[PROOFSTEP]
exact not_isUnit_zero
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
ha : IsUnit (det A)
z1 z2 : ℤ
⊢ A ^ (z1 - z2) = A ^ z1 / A ^ z2
[PROOFSTEP]
rw [sub_eq_add_neg, zpow_add ha, zpow_neg ha, div_eq_mul_inv]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
n : ℕ
⊢ (A * B) ^ ↑n = A ^ ↑n * B ^ ↑n
[PROOFSTEP]
simp [h.mul_pow n]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A B : M
h : Commute A B
n : ℕ
⊢ (A * B) ^ -[n+1] = A ^ -[n+1] * B ^ -[n+1]
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, zpow_negSucc, ← mul_inv_rev, h.mul_pow n.succ, (h.pow_pow _ _).eq]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
⊢ A ^ bit1 n = (A * A) ^ n * A
[PROOFSTEP]
rw [zpow_bit1, Commute.mul_zpow (Commute.refl A)]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
n : ℤ
A : M
h : IsUnit (det A)
⊢ A ^ (-n) * A ^ n = 1
[PROOFSTEP]
rw [zpow_neg h, nonsing_inv_mul _ (h.det_zpow _)]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ (1 / A) ^ n = 1 / A ^ n
[PROOFSTEP]
simp only [one_div, inv_pow']
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℤ
⊢ (1 / A) ^ n = 1 / A ^ n
[PROOFSTEP]
simp only [one_div, inv_zpow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ (A ^ ↑n)ᵀ = Aᵀ ^ ↑n
[PROOFSTEP]
rw [zpow_ofNat, zpow_ofNat, transpose_pow]
[GOAL]
n' : Type u_1
inst✝² : DecidableEq n'
inst✝¹ : Fintype n'
R : Type u_2
inst✝ : CommRing R
A : M
n : ℕ
⊢ (A ^ -[n+1])ᵀ = Aᵀ ^ -[n+1]
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, transpose_nonsing_inv, transpose_pow]
[GOAL]
n' : Type u_1
inst✝³ : DecidableEq n'
inst✝² : Fintype n'
R : Type u_2
inst✝¹ : CommRing R
inst✝ : StarRing R
A : M
n : ℕ
⊢ (A ^ ↑n)ᴴ = Aᴴ ^ ↑n
[PROOFSTEP]
rw [zpow_ofNat, zpow_ofNat, conjTranspose_pow]
[GOAL]
n' : Type u_1
inst✝³ : DecidableEq n'
inst✝² : Fintype n'
R : Type u_2
inst✝¹ : CommRing R
inst✝ : StarRing R
A : M
n : ℕ
⊢ (A ^ -[n+1])ᴴ = Aᴴ ^ -[n+1]
[PROOFSTEP]
rw [zpow_negSucc, zpow_negSucc, conjTranspose_nonsing_inv, conjTranspose_pow]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.ZPow", "llama_tokens": 17068} |
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ natDegree (det (X • Matrix.map A ↑C + Matrix.map B ↑C)) ≤ Fintype.card n
[PROOFSTEP]
rw [det_apply]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ natDegree (∑ σ : Equiv.Perm n, ↑sign σ • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑σ i) i) ≤ Fintype.card n
[PROOFSTEP]
refine' (natDegree_sum_le _ _).trans _
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ Finset.fold max 0 (natDegree ∘ fun σ => ↑sign σ • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑σ i) i)
Finset.univ ≤
Fintype.card n
[PROOFSTEP]
refine' Multiset.max_nat_le_of_forall_le _ _ _
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∀ (x : ℕ),
x ∈
Multiset.map (natDegree ∘ fun σ => ↑sign σ • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑σ i) i)
Finset.univ.val →
x ≤ Fintype.card n
[PROOFSTEP]
simp only [forall_apply_eq_imp_iff', true_and_iff, Function.comp_apply, Multiset.map_map, Multiset.mem_map, exists_imp,
Finset.mem_univ_val]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∀ (a : Equiv.Perm n), natDegree (↑sign a • ∏ x : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑a x) x) ≤ Fintype.card n
[PROOFSTEP]
intro g
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ natDegree (↑sign g • ∏ x : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g x) x) ≤ Fintype.card n
[PROOFSTEP]
calc
natDegree (sign g • ∏ i : n, (X • A.map C + B.map C) (g i) i) ≤
natDegree (∏ i : n, (X • A.map C + B.map C) (g i) i) :=
by
cases' Int.units_eq_one_or (sign g) with sg sg
· rw [sg, one_smul]
· rw [sg, Units.neg_smul, one_smul, natDegree_neg]
_ ≤ ∑ i : n, natDegree (((X : α[X]) • A.map C + B.map C) (g i) i) :=
(natDegree_prod_le (Finset.univ : Finset n) fun i : n => (X • A.map C + B.map C) (g i) i)
_ ≤ Finset.univ.card • 1 := (Finset.sum_le_card_nsmul _ _ 1 fun (i : n) _ => ?_)
_ ≤ Fintype.card n := by simp [mul_one, Algebra.id.smul_eq_mul, Finset.card_univ]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ natDegree (↑sign g • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) ≤
natDegree (∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i)
[PROOFSTEP]
cases' Int.units_eq_one_or (sign g) with sg sg
[GOAL]
case inl
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
sg : ↑sign g = 1
⊢ natDegree (↑sign g • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) ≤
natDegree (∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i)
[PROOFSTEP]
rw [sg, one_smul]
[GOAL]
case inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
sg : ↑sign g = -1
⊢ natDegree (↑sign g • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) ≤
natDegree (∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i)
[PROOFSTEP]
rw [sg, Units.neg_smul, one_smul, natDegree_neg]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ Finset.card Finset.univ • 1 ≤ Fintype.card n
[PROOFSTEP]
simp [mul_one, Algebra.id.smul_eq_mul, Finset.card_univ]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
i : n
x✝ : i ∈ Finset.univ
⊢ natDegree ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) ≤ 1
[PROOFSTEP]
calc
natDegree (((X : α[X]) • A.map C + B.map C) (g i) i) = natDegree ((X : α[X]) * C (A (g i) i) + C (B (g i) i)) := by
simp
_ ≤ max (natDegree ((X : α[X]) * C (A (g i) i))) (natDegree (C (B (g i) i))) := (natDegree_add_le _ _)
_ = natDegree ((X : α[X]) * C (A (g i) i)) := (max_eq_left ((natDegree_C _).le.trans (zero_le _)))
_ ≤ natDegree (X : α[X]) := (natDegree_mul_C_le _ _)
_ ≤ 1 := natDegree_X_le
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
i : n
x✝ : i ∈ Finset.univ
⊢ natDegree ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) = natDegree (X * ↑C (A (↑g i) i) + ↑C (B (↑g i) i))
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ coeff (det (X • Matrix.map A ↑C + Matrix.map B ↑C)) 0 = det B
[PROOFSTEP]
rw [det_apply, finset_sum_coeff, det_apply]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∑ b : Equiv.Perm n, coeff (↑sign b • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑b i) i) 0 =
∑ σ : Equiv.Perm n, ↑sign σ • ∏ i : n, B (↑σ i) i
[PROOFSTEP]
refine' Finset.sum_congr rfl _
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∀ (x : Equiv.Perm n),
x ∈ Finset.univ →
coeff (↑sign x • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑x i) i) 0 = ↑sign x • ∏ i : n, B (↑x i) i
[PROOFSTEP]
rintro g -
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ coeff (↑sign g • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) 0 = ↑sign g • ∏ i : n, B (↑g i) i
[PROOFSTEP]
convert coeff_smul (R := α) (sign g) _ 0
[GOAL]
case h.e'_3.h.e'_6
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ ∏ i : n, B (↑g i) i = coeff (∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) 0
[PROOFSTEP]
rw [coeff_zero_prod]
[GOAL]
case h.e'_3.h.e'_6
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ ∏ i : n, B (↑g i) i = ∏ i : n, coeff ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g i) i) 0
[PROOFSTEP]
refine' Finset.prod_congr rfl _
[GOAL]
case h.e'_3.h.e'_6
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ ∀ (x : n), x ∈ Finset.univ → B (↑g x) x = coeff ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g x) x) 0
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ coeff (det (X • Matrix.map A ↑C + Matrix.map B ↑C)) (Fintype.card n) = det A
[PROOFSTEP]
rw [det_apply, det_apply, finset_sum_coeff]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∑ b : Equiv.Perm n, coeff (↑sign b • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑b i) i) (Fintype.card n) =
∑ σ : Equiv.Perm n, ↑sign σ • ∏ i : n, A (↑σ i) i
[PROOFSTEP]
refine' Finset.sum_congr rfl _
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∀ (x : Equiv.Perm n),
x ∈ Finset.univ →
coeff (↑sign x • ∏ i : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑x i) i) (Fintype.card n) =
↑sign x • ∏ i : n, A (↑x i) i
[PROOFSTEP]
simp only [Algebra.id.smul_eq_mul, Finset.mem_univ, RingHom.mapMatrix_apply, forall_true_left, map_apply, Pi.smul_apply]
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
⊢ ∀ (x : Equiv.Perm n),
coeff (↑sign x • ∏ x_1 : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑x x_1) x_1) (Fintype.card n) =
↑sign x • ∏ x_1 : n, A (↑x x_1) x_1
[PROOFSTEP]
intro g
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ coeff (↑sign g • ∏ x : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g x) x) (Fintype.card n) =
↑sign g • ∏ x : n, A (↑g x) x
[PROOFSTEP]
convert coeff_smul (R := α) (sign g) _ _
[GOAL]
case h.e'_3.h.e'_6
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ ∏ x : n, A (↑g x) x = coeff (∏ x : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g x) x) (Fintype.card n)
[PROOFSTEP]
rw [← mul_one (Fintype.card n)]
[GOAL]
case h.e'_3.h.e'_6
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ ∏ x : n, A (↑g x) x = coeff (∏ x : n, (X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g x) x) (Fintype.card n * 1)
[PROOFSTEP]
convert (coeff_prod_of_natDegree_le (R := α) _ _ _ _).symm
[GOAL]
case h.e'_2.a
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
x✝ : n
a✝ : x✝ ∈ Finset.univ
⊢ A (↑g x✝) x✝ = coeff ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g x✝) x✝) 1
[PROOFSTEP]
simp [coeff_C]
[GOAL]
case h.e'_3.h.e'_6.convert_5
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
⊢ ∀ (p : n), p ∈ Finset.univ → natDegree ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g p) p) ≤ 1
[PROOFSTEP]
rintro p -
[GOAL]
case h.e'_3.h.e'_6.convert_5
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
p : n
⊢ natDegree ((X • Matrix.map A ↑C + Matrix.map B ↑C) (↑g p) p) ≤ 1
[PROOFSTEP]
refine' (natDegree_add_le _ _).trans _
[GOAL]
case h.e'_3.h.e'_6.convert_5
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A B : Matrix n n α
g : Equiv.Perm n
p : n
⊢ max (natDegree ((X • Matrix.map A ↑C) (↑g p) p)) (natDegree (Matrix.map B (↑C) (↑g p) p)) ≤ 1
[PROOFSTEP]
simpa [Pi.smul_apply, map_apply, Algebra.id.smul_eq_mul, X_mul_C, natDegree_C, max_eq_left, zero_le'] using
(natDegree_C_mul_le _ _).trans (natDegree_X_le (R := α))
[GOAL]
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
⊢ leadingCoeff (det (X • 1 + Matrix.map A ↑C)) = 1
[PROOFSTEP]
cases subsingleton_or_nontrivial α
[GOAL]
case inl
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Subsingleton α
⊢ leadingCoeff (det (X • 1 + Matrix.map A ↑C)) = 1
[PROOFSTEP]
simp
[GOAL]
case inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
⊢ leadingCoeff (det (X • 1 + Matrix.map A ↑C)) = 1
[PROOFSTEP]
rw [← @det_one n, ← coeff_det_X_add_C_card _ A, leadingCoeff]
[GOAL]
case inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • Matrix.map 1 ↑C + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
simp only [Matrix.map_one, C_eq_zero, RingHom.map_one]
[GOAL]
case inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • 1 + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
cases' (natDegree_det_X_add_C_le 1 A).eq_or_lt with h h
[GOAL]
case inr.inl
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
h : natDegree (det (X • Matrix.map 1 ↑C + Matrix.map A ↑C)) = Fintype.card n
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • 1 + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
simp only [RingHom.map_one, Matrix.map_one, C_eq_zero] at h
[GOAL]
case inr.inl
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
h : natDegree (det (X • 1 + Matrix.map A ↑C)) = Fintype.card n
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • 1 + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
rw [h]
[GOAL]
case inr.inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
h : natDegree (det (X • Matrix.map 1 ↑C + Matrix.map A ↑C)) < Fintype.card n
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • 1 + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
have H := coeff_eq_zero_of_natDegree_lt h
[GOAL]
case inr.inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
h : natDegree (det (X • Matrix.map 1 ↑C + Matrix.map A ↑C)) < Fintype.card n
H : coeff (det (X • Matrix.map 1 ↑C + Matrix.map A ↑C)) (Fintype.card n) = 0
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • 1 + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
rw [coeff_det_X_add_C_card] at H
[GOAL]
case inr.inr
n : Type u_1
α : Type u_2
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : CommRing α
A : Matrix n n α
h✝ : Nontrivial α
h : natDegree (det (X • Matrix.map 1 ↑C + Matrix.map A ↑C)) < Fintype.card n
H : det 1 = 0
⊢ coeff (det (X • 1 + Matrix.map A ↑C)) (natDegree (det (X • 1 + Matrix.map A ↑C))) =
coeff (det (X • 1 + Matrix.map A ↑C)) (Fintype.card n)
[PROOFSTEP]
simp at H
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Polynomial", "llama_tokens": 7140} |
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : LT α
b : n → α
e : m ≃ n
⊢ BlockTriangular (↑(reindex e e) M) b ↔ BlockTriangular M (b ∘ ↑e)
[PROOFSTEP]
refine' ⟨fun h => _, fun h => _⟩
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : LT α
b : n → α
e : m ≃ n
h : BlockTriangular (↑(reindex e e) M) b
⊢ BlockTriangular M (b ∘ ↑e)
[PROOFSTEP]
convert h.submatrix
[GOAL]
case h.e'_6
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : LT α
b : n → α
e : m ≃ n
h : BlockTriangular (↑(reindex e e) M) b
⊢ M = submatrix (↑(reindex e e) M) ↑e ↑e
[PROOFSTEP]
simp only [reindex_apply, submatrix_submatrix, submatrix_id_id, Equiv.symm_comp_self]
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : LT α
b : n → α
e : m ≃ n
h : BlockTriangular M (b ∘ ↑e)
⊢ BlockTriangular (↑(reindex e e) M) b
[PROOFSTEP]
convert h.submatrix
[GOAL]
case h.e'_7
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : LT α
b : n → α
e : m ≃ n
h : BlockTriangular M (b ∘ ↑e)
⊢ b = (b ∘ ↑e) ∘ fun i => ↑e.symm i
[PROOFSTEP]
simp only [comp.assoc b e e.symm, Equiv.self_comp_symm, comp.right_id]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b : m → α
inst✝ : LT α
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
h : b j < b i
⊢ (M + N) i j = 0
[PROOFSTEP]
simp_rw [Matrix.add_apply, hM h, hN h, zero_add]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b : m → α
inst✝ : LT α
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
h : b j < b i
⊢ (M - N) i j = 0
[PROOFSTEP]
simp_rw [Matrix.sub_apply, hM h, hN h, sub_zero]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M N : Matrix m m R
b : m → α
inst✝¹ : Preorder α
inst✝ : DecidableEq α
d : (i : α) → Matrix (m' i) (m' i) R
⊢ BlockTriangular (blockDiagonal' d) Sigma.fst
[PROOFSTEP]
rintro ⟨i, i'⟩ ⟨j, j'⟩ h
[GOAL]
case mk.mk
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M N : Matrix m m R
b : m → α
inst✝¹ : Preorder α
inst✝ : DecidableEq α
d : (i : α) → Matrix (m' i) (m' i) R
i : α
i' : m' i
j : α
j' : m' j
h : { fst := j, snd := j' }.fst < { fst := i, snd := i' }.fst
⊢ blockDiagonal' d { fst := i, snd := i' } { fst := j, snd := j' } = 0
[PROOFSTEP]
apply blockDiagonal'_apply_ne d i' j' fun h' => ne_of_lt h h'.symm
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M N : Matrix m m R
b : m → α
inst✝¹ : Preorder α
inst✝ : DecidableEq α
d : α → Matrix m m R
⊢ BlockTriangular (blockDiagonal d) Prod.snd
[PROOFSTEP]
rintro ⟨i, i'⟩ ⟨j, j'⟩ h
[GOAL]
case mk.mk
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M N : Matrix m m R
b : m → α
inst✝¹ : Preorder α
inst✝ : DecidableEq α
d : α → Matrix m m R
i : m
i' : α
j : m
j' : α
h : (j, j').snd < (i, i').snd
⊢ blockDiagonal d (i, i') (j, j') = 0
[PROOFSTEP]
rw [blockDiagonal'_eq_blockDiagonal, blockTriangular_blockDiagonal']
[GOAL]
case mk.mk.a
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M N : Matrix m m R
b : m → α
inst✝¹ : Preorder α
inst✝ : DecidableEq α
d : α → Matrix m m R
i : m
i' : α
j : m
j' : α
h : (j, j').snd < (i, i').snd
⊢ { fst := j', snd := j }.fst < { fst := i', snd := i }.fst
[PROOFSTEP]
exact h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M✝ N✝ : Matrix m m R
b : m → α
inst✝¹ : LinearOrder α
inst✝ : Fintype m
M N : Matrix m m R
hM : BlockTriangular M b
hN : BlockTriangular N b
⊢ BlockTriangular (M * N) b
[PROOFSTEP]
intro i j hij
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M✝ N✝ : Matrix m m R
b : m → α
inst✝¹ : LinearOrder α
inst✝ : Fintype m
M N : Matrix m m R
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
hij : b j < b i
⊢ (M * N) i j = 0
[PROOFSTEP]
apply Finset.sum_eq_zero
[GOAL]
case h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M✝ N✝ : Matrix m m R
b : m → α
inst✝¹ : LinearOrder α
inst✝ : Fintype m
M N : Matrix m m R
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
hij : b j < b i
⊢ ∀ (x : m), x ∈ univ → (fun j => M i j) x * (fun j_1 => N j_1 j) x = 0
[PROOFSTEP]
intro k _
[GOAL]
case h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M✝ N✝ : Matrix m m R
b : m → α
inst✝¹ : LinearOrder α
inst✝ : Fintype m
M N : Matrix m m R
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
hij : b j < b i
k : m
a✝ : k ∈ univ
⊢ (fun j => M i j) k * (fun j_1 => N j_1 j) k = 0
[PROOFSTEP]
by_cases hki : b k < b i
[GOAL]
case pos
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M✝ N✝ : Matrix m m R
b : m → α
inst✝¹ : LinearOrder α
inst✝ : Fintype m
M N : Matrix m m R
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
hij : b j < b i
k : m
a✝ : k ∈ univ
hki : b k < b i
⊢ (fun j => M i j) k * (fun j_1 => N j_1 j) k = 0
[PROOFSTEP]
simp_rw [hM hki, zero_mul]
[GOAL]
case neg
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝² : CommRing R
M✝ N✝ : Matrix m m R
b : m → α
inst✝¹ : LinearOrder α
inst✝ : Fintype m
M N : Matrix m m R
hM : BlockTriangular M b
hN : BlockTriangular N b
i j : m
hij : b j < b i
k : m
a✝ : k ∈ univ
hki : ¬b k < b i
⊢ (fun j => M i j) k * (fun j_1 => N j_1 j) k = 0
[PROOFSTEP]
simp_rw [hN (lt_of_lt_of_le hij (le_of_not_lt hki)), mul_zero]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
⊢ BlockTriangular (fromBlocks A B 0 D) (Sum.elim (fun x => a) fun x => b)
[PROOFSTEP]
rintro (c | c) (d | d) hcd
[GOAL]
case inl.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c d : m
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inl d) < Sum.elim (fun x => a) (fun x => b) (Sum.inl c)
⊢ fromBlocks A B 0 D (Sum.inl c) (Sum.inl d) = 0
[PROOFSTEP]
first
| simp [hab.not_lt] at hcd ⊢
[GOAL]
case inl.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c d : m
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inl d) < Sum.elim (fun x => a) (fun x => b) (Sum.inl c)
⊢ fromBlocks A B 0 D (Sum.inl c) (Sum.inl d) = 0
[PROOFSTEP]
simp [hab.not_lt] at hcd ⊢
[GOAL]
case inl.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c : m
d : n
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inr d) < Sum.elim (fun x => a) (fun x => b) (Sum.inl c)
⊢ fromBlocks A B 0 D (Sum.inl c) (Sum.inr d) = 0
[PROOFSTEP]
first
| simp [hab.not_lt] at hcd ⊢
[GOAL]
case inl.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c : m
d : n
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inr d) < Sum.elim (fun x => a) (fun x => b) (Sum.inl c)
⊢ fromBlocks A B 0 D (Sum.inl c) (Sum.inr d) = 0
[PROOFSTEP]
simp [hab.not_lt] at hcd ⊢
[GOAL]
case inr.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c : n
d : m
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inl d) < Sum.elim (fun x => a) (fun x => b) (Sum.inr c)
⊢ fromBlocks A B 0 D (Sum.inr c) (Sum.inl d) = 0
[PROOFSTEP]
first
| simp [hab.not_lt] at hcd ⊢
[GOAL]
case inr.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c : n
d : m
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inl d) < Sum.elim (fun x => a) (fun x => b) (Sum.inr c)
⊢ fromBlocks A B 0 D (Sum.inr c) (Sum.inl d) = 0
[PROOFSTEP]
simp [hab.not_lt] at hcd ⊢
[GOAL]
case inr.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c d : n
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inr d) < Sum.elim (fun x => a) (fun x => b) (Sum.inr c)
⊢ fromBlocks A B 0 D (Sum.inr c) (Sum.inr d) = 0
[PROOFSTEP]
first
| simp [hab.not_lt] at hcd ⊢
[GOAL]
case inr.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝¹ : CommRing R
M N : Matrix m m R
b✝ : m → α
inst✝ : Preorder α
A : Matrix m m R
B : Matrix m n R
D : Matrix n n R
a b : α
hab : a < b
c d : n
hcd : Sum.elim (fun x => a) (fun x => b) (Sum.inr d) < Sum.elim (fun x => a) (fun x => b) (Sum.inr c)
⊢ fromBlocks A B 0 D (Sum.inr c) (Sum.inr d) = 0
[PROOFSTEP]
simp [hab.not_lt] at hcd ⊢
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
M : Matrix m m R
p q : m → Prop
inst✝¹ : DecidablePred p
inst✝ : DecidablePred q
e : ∀ (x : m), q x ↔ p x
⊢ det (toSquareBlockProp M p) = det (toSquareBlockProp M q)
[PROOFSTEP]
convert Matrix.det_reindex_self (Equiv.subtypeEquivRight e) (toSquareBlockProp M q)
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
⊢ det M =
det
(fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j))
[PROOFSTEP]
rw [← Matrix.det_reindex_self (Equiv.sumCompl p).symm M]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
⊢ det (↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M) =
det
(fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j))
[PROOFSTEP]
rw [det_apply', det_apply']
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
⊢ ∑ σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a }),
↑↑(↑Equiv.Perm.sign σ) *
∏ i : { a // p a } ⊕ { a // ¬p a }, ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (↑σ i) i =
∑ σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a }),
↑↑(↑Equiv.Perm.sign σ) *
∏ i : { a // p a } ⊕ { a // ¬p a },
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (↑σ i) i
[PROOFSTEP]
congr
[GOAL]
case e_f
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
⊢ (fun σ =>
↑↑(↑Equiv.Perm.sign σ) *
∏ i : { a // p a } ⊕ { a // ¬p a }, ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (↑σ i) i) =
fun σ =>
↑↑(↑Equiv.Perm.sign σ) *
∏ i : { a // p a } ⊕ { a // ¬p a },
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (↑σ i) i
[PROOFSTEP]
ext σ
[GOAL]
case e_f.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
⊢ ↑↑(↑Equiv.Perm.sign σ) *
∏ i : { a // p a } ⊕ { a // ¬p a }, ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (↑σ i) i =
↑↑(↑Equiv.Perm.sign σ) *
∏ i : { a // p a } ⊕ { a // ¬p a },
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (↑σ i) i
[PROOFSTEP]
congr
[GOAL]
case e_f.h.e_a.e_f
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
⊢ (fun i => ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (↑σ i) i) = fun i =>
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (↑σ i) i
[PROOFSTEP]
ext x
[GOAL]
case e_f.h.e_a.e_f.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
x : { a // p a } ⊕ { a // ¬p a }
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (↑σ x) x =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (↑σ x) x
[PROOFSTEP]
generalize hy : σ x = y
[GOAL]
case e_f.h.e_a.e_f.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
x y : { a // p a } ⊕ { a // ¬p a }
hy : ↑σ x = y
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M y x =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) y x
[PROOFSTEP]
cases x
[GOAL]
case e_f.h.e_a.e_f.h.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
y : { a // p a } ⊕ { a // ¬p a }
val✝ : { a // p a }
hy : ↑σ (Sum.inl val✝) = y
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M y (Sum.inl val✝) =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) y (Sum.inl val✝)
[PROOFSTEP]
cases y
[GOAL]
case e_f.h.e_a.e_f.h.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
y : { a // p a } ⊕ { a // ¬p a }
val✝ : { a // ¬p a }
hy : ↑σ (Sum.inr val✝) = y
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M y (Sum.inr val✝) =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) y (Sum.inr val✝)
[PROOFSTEP]
cases y
[GOAL]
case e_f.h.e_a.e_f.h.inl.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
val✝¹ val✝ : { a // p a }
hy : ↑σ (Sum.inl val✝¹) = Sum.inl val✝
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (Sum.inl val✝) (Sum.inl val✝¹) =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (Sum.inl val✝) (Sum.inl val✝¹)
[PROOFSTEP]
simp only [Matrix.reindex_apply, toBlock_apply, Equiv.symm_symm, Equiv.sumCompl_apply_inr, Equiv.sumCompl_apply_inl,
fromBlocks_apply₁₁, fromBlocks_apply₁₂, fromBlocks_apply₂₁, fromBlocks_apply₂₂, Matrix.submatrix_apply]
[GOAL]
case e_f.h.e_a.e_f.h.inl.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
val✝¹ : { a // p a }
val✝ : { a // ¬p a }
hy : ↑σ (Sum.inl val✝¹) = Sum.inr val✝
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (Sum.inr val✝) (Sum.inl val✝¹) =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (Sum.inr val✝) (Sum.inl val✝¹)
[PROOFSTEP]
simp only [Matrix.reindex_apply, toBlock_apply, Equiv.symm_symm, Equiv.sumCompl_apply_inr, Equiv.sumCompl_apply_inl,
fromBlocks_apply₁₁, fromBlocks_apply₁₂, fromBlocks_apply₂₁, fromBlocks_apply₂₂, Matrix.submatrix_apply]
[GOAL]
case e_f.h.e_a.e_f.h.inr.inl
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
val✝¹ : { a // ¬p a }
val✝ : { a // p a }
hy : ↑σ (Sum.inr val✝¹) = Sum.inl val✝
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (Sum.inl val✝) (Sum.inr val✝¹) =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (Sum.inl val✝) (Sum.inr val✝¹)
[PROOFSTEP]
simp only [Matrix.reindex_apply, toBlock_apply, Equiv.symm_symm, Equiv.sumCompl_apply_inr, Equiv.sumCompl_apply_inl,
fromBlocks_apply₁₁, fromBlocks_apply₁₂, fromBlocks_apply₂₁, fromBlocks_apply₂₂, Matrix.submatrix_apply]
[GOAL]
case e_f.h.e_a.e_f.h.inr.inr
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
σ : Equiv.Perm ({ a // p a } ⊕ { a // ¬p a })
val✝¹ val✝ : { a // ¬p a }
hy : ↑σ (Sum.inr val✝¹) = Sum.inr val✝
⊢ ↑(reindex (Equiv.sumCompl p).symm (Equiv.sumCompl p).symm) M (Sum.inr val✝) (Sum.inr val✝¹) =
fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j) (Sum.inr val✝) (Sum.inr val✝¹)
[PROOFSTEP]
simp only [Matrix.reindex_apply, toBlock_apply, Equiv.symm_symm, Equiv.sumCompl_apply_inr, Equiv.sumCompl_apply_inl,
fromBlocks_apply₁₁, fromBlocks_apply₁₂, fromBlocks_apply₂₁, fromBlocks_apply₂₂, Matrix.submatrix_apply]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), ¬p i → ∀ (j : m), p j → M i j = 0
⊢ det M = det (toSquareBlockProp M p) * det (toSquareBlockProp M fun i => ¬p i)
[PROOFSTEP]
rw [det_toBlock M p]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), ¬p i → ∀ (j : m), p j → M i j = 0
⊢ det
(fromBlocks (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) p)
(toBlock M (fun j => ¬p j) fun j => ¬p j)) =
det (toSquareBlockProp M p) * det (toSquareBlockProp M fun i => ¬p i)
[PROOFSTEP]
convert det_fromBlocks_zero₂₁ (toBlock M p p) (toBlock M p fun j => ¬p j) (toBlock M (fun j => ¬p j) fun j => ¬p j)
[GOAL]
case h.e'_2.h.e'_6.h.e'_8
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), ¬p i → ∀ (j : m), p j → M i j = 0
⊢ toBlock M (fun j => ¬p j) p = 0
[PROOFSTEP]
ext i j
[GOAL]
case h.e'_2.h.e'_6.h.e'_8.a.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), ¬p i → ∀ (j : m), p j → M i j = 0
i : { a // ¬p a }
j : { a // p a }
⊢ toBlock M (fun j => ¬p j) p i j = OfNat.ofNat 0 i j
[PROOFSTEP]
exact h (↑i) i.2 (↑j) j.2
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), p i → ∀ (j : m), ¬p j → M i j = 0
⊢ det M = det (toSquareBlockProp M p) * det (toSquareBlockProp M fun i => ¬p i)
[PROOFSTEP]
rw [M.twoBlockTriangular_det fun i => ¬p i, mul_comm]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), p i → ∀ (j : m), ¬p j → M i j = 0
⊢ det (toSquareBlockProp M fun i => ¬¬p i) * det (toSquareBlockProp M fun i => ¬p i) =
det (toSquareBlockProp M p) * det (toSquareBlockProp M fun i => ¬p i)
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), p i → ∀ (j : m), ¬p j → M i j = 0
⊢ ∀ (i : m), ¬¬p i → ∀ (j : m), ¬p j → M i j = 0
[PROOFSTEP]
congr 1
[GOAL]
case e_a
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), p i → ∀ (j : m), ¬p j → M i j = 0
⊢ det (toSquareBlockProp M fun i => ¬¬p i) = det (toSquareBlockProp M p)
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), p i → ∀ (j : m), ¬p j → M i j = 0
⊢ ∀ (i : m), ¬¬p i → ∀ (j : m), ¬p j → M i j = 0
[PROOFSTEP]
exact equiv_block_det _ fun _ => not_not.symm
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
M : Matrix m m R
p : m → Prop
inst✝ : DecidablePred p
h : ∀ (i : m), p i → ∀ (j : m), ¬p j → M i j = 0
⊢ ∀ (i : m), ¬¬p i → ∀ (j : m), ¬p j → M i j = 0
[PROOFSTEP]
simpa only [Classical.not_not] using h
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : DecidableEq α
inst✝ : LinearOrder α
hM : BlockTriangular M b
⊢ det M = ∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
clear N
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : DecidableEq α
inst✝ : LinearOrder α
hM : BlockTriangular M b
⊢ det M = ∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
induction' hs : univ.image b using Finset.strongInduction with s ih generalizing m
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs✝ : image b✝ univ = x✝
s : Finset α
ih :
∀ (t : Finset α),
t ⊂ s →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
hs : image b univ = s
⊢ det M = ∏ a in s, det (toSquareBlock M b a)
[PROOFSTEP]
subst hs
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
⊢ det M = ∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
cases isEmpty_or_nonempty m
[GOAL]
case H.inl
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : IsEmpty m
⊢ det M = ∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
simp
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
⊢ det M = ∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
let k := (univ.image b).max' (univ_nonempty.image _)
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
⊢ det M = ∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
rw [twoBlockTriangular_det' M fun i => b i = k]
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
⊢ det (toSquareBlockProp M fun i => b i = k) * det (toSquareBlockProp M fun i => ¬b i = k) =
∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
have : univ.image b = insert k ((univ.image b).erase k) :=
by
rw [insert_erase]
apply max'_mem
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
⊢ image b univ = insert k (erase (image b univ) k)
[PROOFSTEP]
rw [insert_erase]
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
⊢ k ∈ image b univ
[PROOFSTEP]
apply max'_mem
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
⊢ det (toSquareBlockProp M fun i => b i = k) * det (toSquareBlockProp M fun i => ¬b i = k) =
∏ a in image b univ, det (toSquareBlock M b a)
[PROOFSTEP]
rw [this, prod_insert (not_mem_erase _ _)]
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
⊢ det (toSquareBlockProp M fun i => b i = k) * det (toSquareBlockProp M fun i => ¬b i = k) =
det (toSquareBlock M b k) * ∏ x in erase (image b univ) k, det (toSquareBlock M b x)
[PROOFSTEP]
refine' congr_arg _ _
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
⊢ det (toSquareBlockProp M fun i => ¬b i = k) = ∏ x in erase (image b univ) k, det (toSquareBlock M b x)
[PROOFSTEP]
let b' := fun i : { a // b a ≠ k } => b ↑i
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
⊢ det (toSquareBlockProp M fun i => ¬b i = k) = ∏ x in erase (image b univ) k, det (toSquareBlock M b x)
[PROOFSTEP]
have h' : BlockTriangular (M.toSquareBlockProp fun i => b i ≠ k) b' := hM.submatrix
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
⊢ det (toSquareBlockProp M fun i => ¬b i = k) = ∏ x in erase (image b univ) k, det (toSquareBlock M b x)
[PROOFSTEP]
have hb' : image b' univ = (image b univ).erase k := by convert image_subtype_ne_univ_eq_image_erase k b
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
⊢ image b' univ = erase (image b univ) k
[PROOFSTEP]
convert image_subtype_ne_univ_eq_image_erase k b
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
hb' : image b' univ = erase (image b univ) k
⊢ det (toSquareBlockProp M fun i => ¬b i = k) = ∏ x in erase (image b univ) k, det (toSquareBlock M b x)
[PROOFSTEP]
rw [ih _ (erase_ssubset <| max'_mem _ _) h' hb']
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
hb' : image b' univ = erase (image b univ) k
⊢ ∏ a in erase (image b univ) (max' (image b univ) (_ : Finset.Nonempty (image b univ))),
det (toSquareBlock (toSquareBlockProp M fun i => b i ≠ k) b' a) =
∏ x in erase (image b univ) k, det (toSquareBlock M b x)
[PROOFSTEP]
refine' Finset.prod_congr rfl fun l hl => _
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
hb' : image b' univ = erase (image b univ) k
l : α
hl : l ∈ erase (image b univ) k
⊢ det (toSquareBlock (toSquareBlockProp M fun i => b i ≠ k) b' l) = det (toSquareBlock M b l)
[PROOFSTEP]
let he : { a // b' a = l } ≃ { a // b a = l } :=
haveI hc : ∀ i, b i = l → b i ≠ k := fun i hi => ne_of_eq_of_ne hi (ne_of_mem_erase hl)
Equiv.subtypeSubtypeEquivSubtype @(hc)
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
hb' : image b' univ = erase (image b univ) k
l : α
hl : l ∈ erase (image b univ) k
he : { a // b' a = l } ≃ { a // b a = l } := Equiv.subtypeSubtypeEquivSubtype (_ : ∀ (i : m), b i = l → b i ≠ k)
⊢ det (toSquareBlock (toSquareBlockProp M fun i => b i ≠ k) b' l) = det (toSquareBlock M b l)
[PROOFSTEP]
simp only [toSquareBlock_def]
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
hb' : image b' univ = erase (image b univ) k
l : α
hl : l ∈ erase (image b univ) k
he : { a // b' a = l } ≃ { a // b a = l } := Equiv.subtypeSubtypeEquivSubtype (_ : ∀ (i : m), b i = l → b i ≠ k)
⊢ det
(↑of fun i j =>
toSquareBlockProp M (fun i => b i ≠ max' (image b univ) (_ : Finset.Nonempty (image b univ))) ↑i ↑j) =
det (↑of fun i j => M ↑i ↑j)
[PROOFSTEP]
erw [← Matrix.det_reindex_self he.symm fun i j : { a // b a = l } => M ↑i ↑j]
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
this : image b univ = insert k (erase (image b univ) k)
b' : { a // b a ≠ k } → α := fun i => b ↑i
h' : BlockTriangular (toSquareBlockProp M fun i => b i ≠ k) b'
hb' : image b' univ = erase (image b univ) k
l : α
hl : l ∈ erase (image b univ) k
he : { a // b' a = l } ≃ { a // b a = l } := Equiv.subtypeSubtypeEquivSubtype (_ : ∀ (i : m), b i = l → b i ≠ k)
⊢ det
(↑of fun i j =>
toSquareBlockProp M (fun i => b i ≠ max' (image b univ) (_ : Finset.Nonempty (image b univ))) ↑i ↑j) =
det (↑(reindex he.symm he.symm) fun i j => M ↑i ↑j)
[PROOFSTEP]
rfl
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
⊢ ∀ (i : m), b i = k → ∀ (j : m), ¬b j = k → M i j = 0
[PROOFSTEP]
intro i hi j hj
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
i : m
hi : b i = k
j : m
hj : ¬b j = k
⊢ M i j = 0
[PROOFSTEP]
apply hM
[GOAL]
case H.inr.a
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
i : m
hi : b i = k
j : m
hj : ¬b j = k
⊢ b j < b i
[PROOFSTEP]
rw [hi]
[GOAL]
case H.inr.a
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
i : m
hi : b i = k
j : m
hj : ¬b j = k
⊢ b j < k
[PROOFSTEP]
apply lt_of_le_of_ne _ hj
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁸ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁷ : DecidableEq m✝
inst✝⁶ : Fintype m✝
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
inst✝³ : DecidableEq α
inst✝² : LinearOrder α
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝¹ : DecidableEq m
inst✝ : Fintype m
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m],
BlockTriangular M b → image b univ = t → det M = ∏ a in t, det (toSquareBlock M b a)
h✝ : Nonempty m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
i : m
hi : b i = k
j : m
hj : ¬b j = k
⊢ b j ≤ k
[PROOFSTEP]
exact Finset.le_max' (univ.image b) _ (mem_image_of_mem _ (mem_univ _))
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁷ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁶ : DecidableEq m
inst✝⁵ : Fintype m
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq α
inst✝¹ : Fintype α
inst✝ : LinearOrder α
h : BlockTriangular M b
⊢ det M = ∏ k : α, det (toSquareBlock M b k)
[PROOFSTEP]
refine' h.det.trans (prod_subset (subset_univ _) fun a _ ha => _)
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁷ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁶ : DecidableEq m
inst✝⁵ : Fintype m
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq α
inst✝¹ : Fintype α
inst✝ : LinearOrder α
h : BlockTriangular M b
a : α
x✝ : a ∈ univ
ha : ¬a ∈ image b univ
⊢ det (toSquareBlock M b a) = 1
[PROOFSTEP]
have : IsEmpty { i // b i = a } := ⟨fun i => ha <| mem_image.2 ⟨i, mem_univ _, i.2⟩⟩
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁷ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁶ : DecidableEq m
inst✝⁵ : Fintype m
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
inst✝² : DecidableEq α
inst✝¹ : Fintype α
inst✝ : LinearOrder α
h : BlockTriangular M b
a : α
x✝ : a ∈ univ
ha : ¬a ∈ image b univ
this : IsEmpty { i // b i = a }
⊢ det (toSquareBlock M b a) = 1
[PROOFSTEP]
exact det_isEmpty
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : LinearOrder m
h : BlockTriangular M id
⊢ det M = ∏ i : m, M i i
[PROOFSTEP]
haveI : DecidableEq R := Classical.decEq _
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : LinearOrder m
h : BlockTriangular M id
this : DecidableEq R
⊢ det M = ∏ i : m, M i i
[PROOFSTEP]
simp_rw [h.det, image_id, det_toSquareBlock_id]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : LinearOrder m
M : Matrix m m R
h : BlockTriangular M ↑toDual
⊢ det M = ∏ i : m, M i i
[PROOFSTEP]
rw [← det_transpose]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁵ : CommRing R
M✝ N : Matrix m m R
b : m → α
inst✝⁴ : DecidableEq m
inst✝³ : Fintype m
inst✝² : DecidableEq n
inst✝¹ : Fintype n
inst✝ : LinearOrder m
M : Matrix m m R
h : BlockTriangular M ↑toDual
⊢ det Mᵀ = ∏ i : m, M i i
[PROOFSTEP]
exact det_of_upperTriangular h.transpose
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
⊢ ((toBlock M⁻¹ (fun i => b i < k) fun i => b i < k) * toBlock M (fun i => b i < k) fun i => b i < k) = 1
[PROOFSTEP]
let p i := b i < k
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
⊢ ((toBlock M⁻¹ (fun i => b i < k) fun i => b i < k) * toBlock M (fun i => b i < k) fun i => b i < k) = 1
[PROOFSTEP]
have h_sum : M⁻¹.toBlock p p * M.toBlock p p + (M⁻¹.toBlock p fun i => ¬p i) * M.toBlock (fun i => ¬p i) p = 1 := by
rw [← toBlock_mul_eq_add, inv_mul_of_invertible M, toBlock_one_self]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
⊢ toBlock M⁻¹ p p * toBlock M p p + (toBlock M⁻¹ p fun i => ¬p i) * toBlock M (fun i => ¬p i) p = 1
[PROOFSTEP]
rw [← toBlock_mul_eq_add, inv_mul_of_invertible M, toBlock_one_self]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
h_sum : toBlock M⁻¹ p p * toBlock M p p + (toBlock M⁻¹ p fun i => ¬p i) * toBlock M (fun i => ¬p i) p = 1
⊢ ((toBlock M⁻¹ (fun i => b i < k) fun i => b i < k) * toBlock M (fun i => b i < k) fun i => b i < k) = 1
[PROOFSTEP]
have h_zero : M.toBlock (fun i => ¬p i) p = 0 := by
ext i j
simpa using hM (lt_of_lt_of_le j.2 (le_of_not_lt i.2))
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
h_sum : toBlock M⁻¹ p p * toBlock M p p + (toBlock M⁻¹ p fun i => ¬p i) * toBlock M (fun i => ¬p i) p = 1
⊢ toBlock M (fun i => ¬p i) p = 0
[PROOFSTEP]
ext i j
[GOAL]
case a.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
h_sum : toBlock M⁻¹ p p * toBlock M p p + (toBlock M⁻¹ p fun i => ¬p i) * toBlock M (fun i => ¬p i) p = 1
i : { a // ¬p a }
j : { a // p a }
⊢ toBlock M (fun i => ¬p i) p i j = OfNat.ofNat 0 i j
[PROOFSTEP]
simpa using hM (lt_of_lt_of_le j.2 (le_of_not_lt i.2))
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
h_sum : toBlock M⁻¹ p p * toBlock M p p + (toBlock M⁻¹ p fun i => ¬p i) * toBlock M (fun i => ¬p i) p = 1
h_zero : toBlock M (fun i => ¬p i) p = 0
⊢ ((toBlock M⁻¹ (fun i => b i < k) fun i => b i < k) * toBlock M (fun i => b i < k) fun i => b i < k) = 1
[PROOFSTEP]
simpa [h_zero] using h_sum
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
⊢ ((toBlock (⅟M) (fun i => b i < k) fun i => b i < k) * toBlock M (fun i => b i < k) fun i => b i < k) = 1
[PROOFSTEP]
simpa only [invOf_eq_nonsing_inv] using hM.toBlock_inverse_mul_toBlock_eq_one k
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
let p i := b i < k
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
let q i := ¬b i < k
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
have h_sum : M⁻¹.toBlock q p * M.toBlock p p + M⁻¹.toBlock q q * M.toBlock q p = 0 :=
by
rw [← toBlock_mul_eq_add, inv_mul_of_invertible M, toBlock_one_disjoint]
rw [disjoint_iff_inf_le]
exact fun i h => h.1 h.2
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
⊢ toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
[PROOFSTEP]
rw [← toBlock_mul_eq_add, inv_mul_of_invertible M, toBlock_one_disjoint]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
⊢ Disjoint q p
[PROOFSTEP]
rw [disjoint_iff_inf_le]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
⊢ q ⊓ p ≤ ⊥
[PROOFSTEP]
exact fun i h => h.1 h.2
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
have h_zero : M.toBlock q p = 0 := by
ext i j
simpa using hM (lt_of_lt_of_le j.2 <| le_of_not_lt i.2)
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
⊢ toBlock M q p = 0
[PROOFSTEP]
ext i j
[GOAL]
case a.h
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
i : { a // q a }
j : { a // p a }
⊢ toBlock M q p i j = OfNat.ofNat 0 i j
[PROOFSTEP]
simpa using hM (lt_of_lt_of_le j.2 <| le_of_not_lt i.2)
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
have h_mul_eq_zero : M⁻¹.toBlock q p * M.toBlock p p = 0 := by simpa [h_zero] using h_sum
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
⊢ toBlock M⁻¹ q p * toBlock M p p = 0
[PROOFSTEP]
simpa [h_zero] using h_sum
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
h_mul_eq_zero : toBlock M⁻¹ q p * toBlock M p p = 0
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
haveI : Invertible (M.toBlock p p) := hM.invertibleToBlock k
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
h_mul_eq_zero : toBlock M⁻¹ q p * toBlock M p p = 0
this : Invertible (toBlock M p p)
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
have : (fun i => k ≤ b i) = q := by
ext
exact not_lt.symm
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
h_mul_eq_zero : toBlock M⁻¹ q p * toBlock M p p = 0
this : Invertible (toBlock M p p)
⊢ (fun i => k ≤ b i) = q
[PROOFSTEP]
ext
[GOAL]
case h.a
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
h_mul_eq_zero : toBlock M⁻¹ q p * toBlock M p p = 0
this : Invertible (toBlock M p p)
x✝ : m
⊢ k ≤ b x✝ ↔ q x✝
[PROOFSTEP]
exact not_lt.symm
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
k : α
p : m → Prop := fun i => b i < k
q : m → Prop := fun i => ¬b i < k
h_sum : toBlock M⁻¹ q p * toBlock M p p + toBlock M⁻¹ q q * toBlock M q p = 0
h_zero : toBlock M q p = 0
h_mul_eq_zero : toBlock M⁻¹ q p * toBlock M p p = 0
this✝ : Invertible (toBlock M p p)
this : (fun i => k ≤ b i) = q
⊢ (toBlock M⁻¹ (fun i => k ≤ b i) fun i => b i < k) = 0
[PROOFSTEP]
rw [this, ← Matrix.zero_mul (M.toBlock p p)⁻¹, ← h_mul_eq_zero, mul_inv_cancel_right_of_invertible]
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M N : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
⊢ BlockTriangular M⁻¹ b
[PROOFSTEP]
clear N
[GOAL]
α : Type u_1
β : Type u_2
m : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁶ : CommRing R
M : Matrix m m R
b : m → α
inst✝⁵ : DecidableEq m
inst✝⁴ : Fintype m
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrder α
inst✝ : Invertible M
hM : BlockTriangular M b
⊢ BlockTriangular M⁻¹ b
[PROOFSTEP]
induction' hs : univ.image b using Finset.strongInduction with s ih generalizing m
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs✝ : image b✝ univ = x✝
s : Finset α
ih :
∀ (t : Finset α),
t ⊂ s →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
hs : image b univ = s
⊢ BlockTriangular M⁻¹ b
[PROOFSTEP]
subst hs
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
⊢ BlockTriangular M⁻¹ b
[PROOFSTEP]
intro i j hij
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
⊢ M⁻¹ i j = 0
[PROOFSTEP]
haveI : Inhabited m := ⟨i⟩
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
⊢ M⁻¹ i j = 0
[PROOFSTEP]
let k := (univ.image b).max' (univ_nonempty.image _)
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
⊢ M⁻¹ i j = 0
[PROOFSTEP]
let b' := fun i : { a // b a < k } => b ↑i
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
⊢ M⁻¹ i j = 0
[PROOFSTEP]
let A := M.toBlock (fun i => b i < k) fun j => b j < k
[GOAL]
case H
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
⊢ M⁻¹ i j = 0
[PROOFSTEP]
obtain hbi | hi : b i = k ∨ _ := (le_max' _ (b i) <| mem_image_of_mem _ <| mem_univ _).eq_or_lt
[GOAL]
case H.inl
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hbi : b i = k
⊢ M⁻¹ i j = 0
[PROOFSTEP]
have : M⁻¹.toBlock (fun i => k ≤ b i) (fun i => b i < k) ⟨i, hbi.ge⟩ ⟨j, hbi ▸ hij⟩ = 0 := by
simp only [toBlock_inverse_eq_zero hM k, Matrix.zero_apply]
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hbi : b i = k
⊢ toBlock M⁻¹ (fun i => k ≤ b i) (fun i => b i < k) { val := i, property := (_ : k ≤ b i) }
{ val := j, property := (_ : (fun i => b i < k) j) } =
0
[PROOFSTEP]
simp only [toBlock_inverse_eq_zero hM k, Matrix.zero_apply]
[GOAL]
case H.inl
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hbi : b i = k
this :
toBlock M⁻¹ (fun i => k ≤ b i) (fun i => b i < k) { val := i, property := (_ : k ≤ b i) }
{ val := j, property := (_ : (fun i => b i < k) j) } =
0
⊢ M⁻¹ i j = 0
[PROOFSTEP]
simp [this.symm]
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
⊢ M⁻¹ i j = 0
[PROOFSTEP]
haveI : Invertible A := hM.invertibleToBlock _
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
⊢ M⁻¹ i j = 0
[PROOFSTEP]
have hA : A.BlockTriangular b' := hM.submatrix
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
hA : BlockTriangular A b'
⊢ M⁻¹ i j = 0
[PROOFSTEP]
have hb' : image b' univ ⊂ image b univ :=
by
convert image_subtype_univ_ssubset_image_univ k b _ (fun a => a < k) (lt_irrefl _)
convert max'_mem (α := α) _ _
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
hA : BlockTriangular A b'
⊢ image b' univ ⊂ image b univ
[PROOFSTEP]
convert image_subtype_univ_ssubset_image_univ k b _ (fun a => a < k) (lt_irrefl _)
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
hA : BlockTriangular A b'
⊢ k ∈ image b univ
[PROOFSTEP]
convert max'_mem (α := α) _ _
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
hA : BlockTriangular A b'
hb' : image b' univ ⊂ image b univ
⊢ M⁻¹ i j = 0
[PROOFSTEP]
have hij' : b' ⟨j, hij.trans hi⟩ < b' ⟨i, hi⟩ := by simp_rw [hij]
[GOAL]
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
hA : BlockTriangular A b'
hb' : image b' univ ⊂ image b univ
⊢ b' { val := j, property := (_ : b j < k) } < b' { val := i, property := hi }
[PROOFSTEP]
simp_rw [hij]
[GOAL]
case H.inr
α : Type u_1
β : Type u_2
m✝ : Type u_3
n : Type u_4
o : Type u_5
m' : α → Type u_6
n' : α → Type u_7
R : Type v
inst✝⁹ : CommRing R
M✝ : Matrix m✝ m✝ R
b✝ : m✝ → α
inst✝⁸ : DecidableEq m✝
inst✝⁷ : Fintype m✝
inst✝⁶ : DecidableEq n
inst✝⁵ : Fintype n
inst✝⁴ : LinearOrder α
inst✝³ : Invertible M✝
hM✝ : BlockTriangular M✝ b✝
x✝ : Finset α
hs : image b✝ univ = x✝
m : Type u_3
M : Matrix m m R
b : m → α
inst✝² : DecidableEq m
inst✝¹ : Fintype m
inst✝ : Invertible M
hM : BlockTriangular M b
ih :
∀ (t : Finset α),
t ⊂ image b univ →
∀ {m : Type u_3} {M : Matrix m m R} {b : m → α} [inst : DecidableEq m] [inst_1 : Fintype m]
[inst_2 : Invertible M], BlockTriangular M b → image b univ = t → BlockTriangular M⁻¹ b
i j : m
hij : b j < b i
this✝ : Inhabited m
k : α := max' (image b univ) (_ : Finset.Nonempty (image b univ))
b' : { a // b a < k } → α := fun i => b ↑i
A : Matrix { a // b a < k } { a // b a < k } R := toBlock M (fun i => b i < k) fun j => b j < k
hi : b i < max' (image b univ) (_ : ∃ x, x ∈ image b univ)
this : Invertible A
hA : BlockTriangular A b'
hb' : image b' univ ⊂ image b univ
hij' : b' { val := j, property := (_ : b j < k) } < b' { val := i, property := hi }
⊢ M⁻¹ i j = 0
[PROOFSTEP]
simp [hM.inv_toBlock k, (ih (image b' univ) hb' hA rfl hij').symm]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Block", "llama_tokens": 46464} |
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j : n
⊢ transvection i j 0 = 1
[PROOFSTEP]
simp [transvection]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) = transvection i j c
[PROOFSTEP]
cases nonempty_fintype n
[GOAL]
case intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) = transvection i j c
[PROOFSTEP]
ext a b
[GOAL]
case intro.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
a b : n
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) a b = transvection i j c a b
[PROOFSTEP]
by_cases ha : i = a
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
a b : n
ha : i = a
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) a b = transvection i j c a b
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
a b : n
ha : ¬i = a
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) a b = transvection i j c a b
[PROOFSTEP]
by_cases hb : j = b
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
a b : n
ha : i = a
hb : j = b
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) a b = transvection i j c a b
[PROOFSTEP]
simp only [updateRow_self, transvection, ha, hb, Pi.add_apply, StdBasisMatrix.apply_same, one_apply_eq, Pi.smul_apply,
mul_one, Algebra.id.smul_eq_mul, add_apply]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
a b : n
ha : i = a
hb : ¬j = b
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) a b = transvection i j c a b
[PROOFSTEP]
simp only [updateRow_self, transvection, ha, hb, StdBasisMatrix.apply_of_ne, Pi.add_apply, Ne.def, not_false_iff,
Pi.smul_apply, and_false_iff, one_apply_ne, Algebra.id.smul_eq_mul, mul_zero, add_apply]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Finite n
c : R
val✝ : Fintype n
a b : n
ha : ¬i = a
⊢ updateRow 1 i (OfNat.ofNat 1 i + c • OfNat.ofNat 1 j) a b = transvection i j c a b
[PROOFSTEP]
simp only [updateRow_ne, transvection, ha, Ne.symm ha, StdBasisMatrix.apply_of_ne, add_zero, Algebra.id.smul_eq_mul,
Ne.def, not_false_iff, DMatrix.add_apply, Pi.smul_apply, mul_zero, false_and_iff, add_apply]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
h : i ≠ j
c d : R
⊢ transvection i j c * transvection i j d = transvection i j (c + d)
[PROOFSTEP]
simp [transvection, Matrix.add_mul, Matrix.mul_add, h, h.symm, add_smul, add_assoc, stdBasisMatrix_add]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
b : n
c : R
M : Matrix n n R
⊢ (transvection i j c * M) i b = M i b + c * M j b
[PROOFSTEP]
simp [transvection, Matrix.add_mul]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
a : n
c : R
M : Matrix n n R
⊢ (M * transvection i j c) a j = M a j + c * M a i
[PROOFSTEP]
simp [transvection, Matrix.mul_add, mul_comm]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
a b : n
ha : a ≠ i
c : R
M : Matrix n n R
⊢ (transvection i j c * M) a b = M a b
[PROOFSTEP]
simp [transvection, Matrix.add_mul, ha]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
a b : n
hb : b ≠ j
c : R
M : Matrix n n R
⊢ (M * transvection i j c) a b = M a b
[PROOFSTEP]
simp [transvection, Matrix.mul_add, hb]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
h : i ≠ j
c : R
⊢ det (transvection i j c) = 1
[PROOFSTEP]
rw [← updateRow_eq_transvection i j, det_updateRow_add_smul_self _ h, det_one]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Nontrivial n
⊢ Nonempty (TransvectionStruct n R)
[PROOFSTEP]
choose x y hxy using exists_pair_ne n
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Nontrivial n
x y : n
hxy : x ≠ y
⊢ Nonempty (TransvectionStruct n R)
[PROOFSTEP]
exact ⟨⟨x, y, hxy, 0⟩⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
L : List (TransvectionStruct n 𝕜)
⊢ det (List.prod (List.map toMatrix L)) = 1
[PROOFSTEP]
induction' L with t L IH
[GOAL]
case nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
⊢ det (List.prod (List.map toMatrix [])) = 1
[PROOFSTEP]
simp
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n 𝕜
L : List (TransvectionStruct n 𝕜)
IH : det (List.prod (List.map toMatrix L)) = 1
⊢ det (List.prod (List.map toMatrix (t :: L))) = 1
[PROOFSTEP]
simp [IH]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
⊢ toMatrix (TransvectionStruct.inv t) * toMatrix t = 1
[PROOFSTEP]
rcases t with ⟨_, _, t_hij⟩
[GOAL]
case mk
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
i✝ j✝ : n
t_hij : i✝ ≠ j✝
c✝ : R
⊢ toMatrix (TransvectionStruct.inv { i := i✝, j := j✝, hij := t_hij, c := c✝ }) *
toMatrix { i := i✝, j := j✝, hij := t_hij, c := c✝ } =
1
[PROOFSTEP]
simp [toMatrix, transvection_mul_transvection_same, t_hij]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
⊢ toMatrix t * toMatrix (TransvectionStruct.inv t) = 1
[PROOFSTEP]
rcases t with ⟨_, _, t_hij⟩
[GOAL]
case mk
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
i✝ j✝ : n
t_hij : i✝ ≠ j✝
c✝ : R
⊢ toMatrix { i := i✝, j := j✝, hij := t_hij, c := c✝ } *
toMatrix (TransvectionStruct.inv { i := i✝, j := j✝, hij := t_hij, c := c✝ }) =
1
[PROOFSTEP]
simp [toMatrix, transvection_mul_transvection_same, t_hij]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
L : List (TransvectionStruct n R)
⊢ List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) * List.prod (List.map toMatrix L) = 1
[PROOFSTEP]
induction' L with t L IH
[GOAL]
case nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
⊢ List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse [])) * List.prod (List.map toMatrix []) = 1
[PROOFSTEP]
simp
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) * List.prod (List.map toMatrix L) = 1
⊢ List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse (t :: L))) *
List.prod (List.map toMatrix (t :: L)) =
1
[PROOFSTEP]
suffices
(L.reverse.map (toMatrix ∘ TransvectionStruct.inv)).prod * (t.inv.toMatrix * t.toMatrix) * (L.map toMatrix).prod = 1
by simpa [Matrix.mul_assoc]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) * List.prod (List.map toMatrix L) = 1
this :
List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) *
(toMatrix (TransvectionStruct.inv t) * toMatrix t) *
List.prod (List.map toMatrix L) =
1
⊢ List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse (t :: L))) *
List.prod (List.map toMatrix (t :: L)) =
1
[PROOFSTEP]
simpa [Matrix.mul_assoc]
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) * List.prod (List.map toMatrix L) = 1
⊢ List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) *
(toMatrix (TransvectionStruct.inv t) * toMatrix t) *
List.prod (List.map toMatrix L) =
1
[PROOFSTEP]
simpa [inv_mul] using IH
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
L : List (TransvectionStruct n R)
⊢ List.prod (List.map toMatrix L) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) = 1
[PROOFSTEP]
induction' L with t L IH
[GOAL]
case nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
⊢ List.prod (List.map toMatrix []) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse [])) = 1
[PROOFSTEP]
simp
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map toMatrix L) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) = 1
⊢ List.prod (List.map toMatrix (t :: L)) *
List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse (t :: L))) =
1
[PROOFSTEP]
suffices
t.toMatrix * ((L.map toMatrix).prod * (L.reverse.map (toMatrix ∘ TransvectionStruct.inv)).prod) * t.inv.toMatrix = 1
by simpa [Matrix.mul_assoc]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map toMatrix L) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) = 1
this :
toMatrix t *
(List.prod (List.map toMatrix L) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L))) *
toMatrix (TransvectionStruct.inv t) =
1
⊢ List.prod (List.map toMatrix (t :: L)) *
List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse (t :: L))) =
1
[PROOFSTEP]
simpa [Matrix.mul_assoc]
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
i j : n
inst✝ : Fintype n
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map toMatrix L) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) = 1
⊢ toMatrix t *
(List.prod (List.map toMatrix L) * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L))) *
toMatrix (TransvectionStruct.inv t) =
1
[PROOFSTEP]
simp_rw [IH, Matrix.mul_one, t.mul_inv]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j : n
t : TransvectionStruct n R
⊢ inl t.i ≠ inl t.j
[PROOFSTEP]
simp [t.hij]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j : n
t : TransvectionStruct n R
⊢ toMatrix (sumInl p t) = fromBlocks (toMatrix t) 0 0 1
[PROOFSTEP]
cases t
[GOAL]
case mk
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1
[PROOFSTEP]
ext a b
[GOAL]
case mk.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : n ⊕ p
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) a b =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 a b
[PROOFSTEP]
cases' a with a a
[GOAL]
case mk.a.h.inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
b : n ⊕ p
a : n
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inl a) b =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inl a) b
[PROOFSTEP]
cases' b with b b
[GOAL]
case mk.a.h.inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
b : n ⊕ p
a : p
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inr a) b =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inr a) b
[PROOFSTEP]
cases' b with b b
[GOAL]
case mk.a.h.inl.inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : n
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inl a) (inl b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inl a) (inl b)
[PROOFSTEP]
by_cases h : a = b
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : n
h : a = b
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inl a) (inl b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inl a) (inl b)
[PROOFSTEP]
simp [TransvectionStruct.sumInl, transvection, h, stdBasisMatrix]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : n
h : ¬a = b
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inl a) (inl b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inl a) (inl b)
[PROOFSTEP]
simp [TransvectionStruct.sumInl, transvection, h, stdBasisMatrix]
[GOAL]
case mk.a.h.inl.inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a : n
b : p
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inl a) (inr b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inl a) (inr b)
[PROOFSTEP]
simp [TransvectionStruct.sumInl, transvection]
[GOAL]
case mk.a.h.inr.inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a : p
b : n
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inr a) (inl b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inr a) (inl b)
[PROOFSTEP]
simp [TransvectionStruct.sumInl, transvection]
[GOAL]
case mk.a.h.inr.inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : p
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inr a) (inr b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inr a) (inr b)
[PROOFSTEP]
by_cases h : a = b
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : p
h : a = b
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inr a) (inr b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inr a) (inr b)
[PROOFSTEP]
simp [TransvectionStruct.sumInl, transvection, h]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j i✝ j✝ : n
hij✝ : i✝ ≠ j✝
c✝ : R
a b : p
h : ¬a = b
⊢ toMatrix (sumInl p { i := i✝, j := j✝, hij := hij✝, c := c✝ }) (inr a) (inr b) =
fromBlocks (toMatrix { i := i✝, j := j✝, hij := hij✝, c := c✝ }) 0 0 1 (inr a) (inr b)
[PROOFSTEP]
simp [TransvectionStruct.sumInl, transvection, h]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n R
L : List (TransvectionStruct n R)
N : Matrix p p R
⊢ List.prod (List.map (toMatrix ∘ sumInl p) L) * fromBlocks M 0 0 N =
fromBlocks (List.prod (List.map toMatrix L) * M) 0 0 N
[PROOFSTEP]
induction' L with t L IH
[GOAL]
case nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n R
N : Matrix p p R
⊢ List.prod (List.map (toMatrix ∘ sumInl p) []) * fromBlocks M 0 0 N =
fromBlocks (List.prod (List.map toMatrix []) * M) 0 0 N
[PROOFSTEP]
simp
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n R
N : Matrix p p R
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH :
List.prod (List.map (toMatrix ∘ sumInl p) L) * fromBlocks M 0 0 N =
fromBlocks (List.prod (List.map toMatrix L) * M) 0 0 N
⊢ List.prod (List.map (toMatrix ∘ sumInl p) (t :: L)) * fromBlocks M 0 0 N =
fromBlocks (List.prod (List.map toMatrix (t :: L)) * M) 0 0 N
[PROOFSTEP]
simp [Matrix.mul_assoc, IH, toMatrix_sumInl, fromBlocks_multiply]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n R
L : List (TransvectionStruct n R)
N : Matrix p p R
⊢ fromBlocks M 0 0 N * List.prod (List.map (toMatrix ∘ sumInl p) L) =
fromBlocks (M * List.prod (List.map toMatrix L)) 0 0 N
[PROOFSTEP]
induction' L with t L IH generalizing M N
[GOAL]
case nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
M✝ : Matrix n n R
N✝ : Matrix p p R
M : Matrix n n R
N : Matrix p p R
⊢ fromBlocks M 0 0 N * List.prod (List.map (toMatrix ∘ sumInl p) []) =
fromBlocks (M * List.prod (List.map toMatrix [])) 0 0 N
[PROOFSTEP]
simp
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
M✝ : Matrix n n R
N✝ : Matrix p p R
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH :
∀ (M : Matrix n n R) (N : Matrix p p R),
fromBlocks M 0 0 N * List.prod (List.map (toMatrix ∘ sumInl p) L) =
fromBlocks (M * List.prod (List.map toMatrix L)) 0 0 N
M : Matrix n n R
N : Matrix p p R
⊢ fromBlocks M 0 0 N * List.prod (List.map (toMatrix ∘ sumInl p) (t :: L)) =
fromBlocks (M * List.prod (List.map toMatrix (t :: L))) 0 0 N
[PROOFSTEP]
simp [IH, toMatrix_sumInl, fromBlocks_multiply]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
i j : n
e : n ≃ p
t : TransvectionStruct n R
⊢ ↑e t.i ≠ ↑e t.j
[PROOFSTEP]
simp [t.hij]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t : TransvectionStruct n R
⊢ toMatrix (reindexEquiv e t) = ↑(reindexAlgEquiv R e) (toMatrix t)
[PROOFSTEP]
rcases t with ⟨t_i, t_j, _⟩
[GOAL]
case mk
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
⊢ toMatrix (reindexEquiv e { i := t_i, j := t_j, hij := hij✝, c := c✝ }) =
↑(reindexAlgEquiv R e) (toMatrix { i := t_i, j := t_j, hij := hij✝, c := c✝ })
[PROOFSTEP]
ext a b
[GOAL]
case mk.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
⊢ toMatrix (reindexEquiv e { i := t_i, j := t_j, hij := hij✝, c := c✝ }) a b =
↑(reindexAlgEquiv R e) (toMatrix { i := t_i, j := t_j, hij := hij✝, c := c✝ }) a b
[PROOFSTEP]
simp only [reindexEquiv, transvection, mul_boole, Algebra.id.smul_eq_mul, toMatrix_mk, submatrix_apply, reindex_apply,
DMatrix.add_apply, Pi.smul_apply, reindexAlgEquiv_apply]
[GOAL]
case mk.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases ha : e t_i = a
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases hb : e t_j = b
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases hb : e t_j = b
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
hb : ↑e t_j = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases hab : a = b
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
hb : ¬↑e t_j = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases hab : a = b
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
hb : ↑e t_j = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases hab : a = b
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
hb : ¬↑e t_j = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
by_cases hab : a = b
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
hb : ↑e t_j = b
hab : a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
hb : ↑e t_j = b
hab : ¬a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
hb : ¬↑e t_j = b
hab : a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ↑e t_i = a
hb : ¬↑e t_j = b
hab : ¬a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
hb : ↑e t_j = b
hab : a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
hb : ↑e t_j = b
hab : ¬a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
hb : ¬↑e t_j = b
hab : a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t_i t_j : n
hij✝ : t_i ≠ t_j
c✝ : R
a b : p
ha : ¬↑e t_i = a
hb : ¬↑e t_j = b
hab : ¬a = b
⊢ (1 + stdBasisMatrix (↑e t_i) (↑e t_j) c✝) a b = (1 + stdBasisMatrix t_i t_j c✝) (↑e.symm a) (↑e.symm b)
[PROOFSTEP]
simp [ha, hb, hab, ← e.apply_eq_iff_eq_symm_apply, stdBasisMatrix]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
L : List (TransvectionStruct n R)
⊢ List.prod (List.map (toMatrix ∘ reindexEquiv e) L) = ↑(reindexAlgEquiv R e) (List.prod (List.map toMatrix L))
[PROOFSTEP]
induction' L with t L IH
[GOAL]
case nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
⊢ List.prod (List.map (toMatrix ∘ reindexEquiv e) []) = ↑(reindexAlgEquiv R e) (List.prod (List.map toMatrix []))
[PROOFSTEP]
simp
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map (toMatrix ∘ reindexEquiv e) L) = ↑(reindexAlgEquiv R e) (List.prod (List.map toMatrix L))
⊢ List.prod (List.map (toMatrix ∘ reindexEquiv e) (t :: L)) =
↑(reindexAlgEquiv R e) (List.prod (List.map toMatrix (t :: L)))
[PROOFSTEP]
simp only [toMatrix_reindexEquiv, IH, Function.comp_apply, List.prod_cons, reindexAlgEquiv_apply, List.map]
[GOAL]
case cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
i j : n
inst✝¹ : Fintype n
inst✝ : Fintype p
e : n ≃ p
t : TransvectionStruct n R
L : List (TransvectionStruct n R)
IH : List.prod (List.map (toMatrix ∘ reindexEquiv e) L) = ↑(reindexAlgEquiv R e) (List.prod (List.map toMatrix L))
⊢ ↑(reindex e e) (toMatrix t) * ↑(reindex e e) (List.prod (List.map toMatrix L)) =
↑(reindex e e) (toMatrix t * List.prod (List.map toMatrix L))
[PROOFSTEP]
exact (reindexAlgEquiv_mul _ _ _ _).symm
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
⊢ (List.prod (List.drop k (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
[PROOFSTEP]
refine' Nat.decreasingInduction' _ hk _
[GOAL]
case refine'_1
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
⊢ ∀ (k_1 : ℕ),
k_1 < r →
k ≤ k_1 →
(List.prod (List.drop (k_1 + 1) (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i →
(List.prod (List.drop k_1 (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
[PROOFSTEP]
intro n hn _ IH
[GOAL]
case refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
n : ℕ
hn : n < r
a✝ : k ≤ n
IH : (List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
⊢ (List.prod (List.drop n (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
[PROOFSTEP]
have hn' : n < (listTransvecCol M).length := by simpa [listTransvecCol] using hn
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
n : ℕ
hn : n < r
a✝ : k ≤ n
IH : (List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
⊢ n < List.length (listTransvecCol M)
[PROOFSTEP]
simpa [listTransvecCol] using hn
[GOAL]
case refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
n : ℕ
hn : n < r
a✝ : k ≤ n
IH : (List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
hn' : n < List.length (listTransvecCol M)
⊢ (List.prod (List.drop n (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
[PROOFSTEP]
rw [← @List.cons_get_drop_succ _ _ ⟨n, hn'⟩]
[GOAL]
case refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
n : ℕ
hn : n < r
a✝ : k ≤ n
IH : (List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
hn' : n < List.length (listTransvecCol M)
⊢ (List.prod
(List.get (listTransvecCol M) { val := n, isLt := hn' } ::
List.drop (↑{ val := n, isLt := hn' } + 1) (listTransvecCol M)) *
M)
(inr ()) i =
M (inr ()) i
[PROOFSTEP]
simpa [listTransvecCol, Matrix.mul_assoc]
[GOAL]
case refine'_2
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
⊢ (List.prod (List.drop r (listTransvecCol M)) * M) (inr ()) i = M (inr ()) i
[PROOFSTEP]
simp only [listTransvecCol, List.length_ofFn, le_refl, List.drop_eq_nil_of_le, List.prod_nil, Matrix.one_mul]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
⊢ (List.prod (listTransvecCol M) * M) (inr ()) i = M (inr ()) i
[PROOFSTEP]
simpa using listTransvecCol_mul_last_row_drop M i (zero_le _)
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ (List.prod (listTransvecCol M) * M) (inl i) (inr ()) = 0
[PROOFSTEP]
suffices H :
∀ k : ℕ,
k ≤ r → (((listTransvecCol M).drop k).prod * M) (inl i) (inr unit) = if k ≤ i then 0 else M (inl i) (inr unit)
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(List.prod (List.drop k (listTransvecCol M)) * M) (inl i) (inr ()) = if k ≤ ↑i then 0 else M (inl i) (inr ())
⊢ (List.prod (listTransvecCol M) * M) (inl i) (inr ()) = 0
[PROOFSTEP]
simpa only [List.drop, _root_.zero_le, ite_true] using H 0 (zero_le _)
[GOAL]
case H
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ ∀ (k : ℕ),
k ≤ r →
(List.prod (List.drop k (listTransvecCol M)) * M) (inl i) (inr ()) = if k ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
intro k hk
[GOAL]
case H
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk : k ≤ r
⊢ (List.prod (List.drop k (listTransvecCol M)) * M) (inl i) (inr ()) = if k ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
refine' Nat.decreasingInduction' _ hk _
[GOAL]
case H.refine'_1
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk : k ≤ r
⊢ ∀ (k_1 : ℕ),
k_1 < r →
k ≤ k_1 →
((List.prod (List.drop (k_1 + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if k_1 + 1 ≤ ↑i then 0 else M (inl i) (inr ())) →
(List.prod (List.drop k_1 (listTransvecCol M)) * M) (inl i) (inr ()) =
if k_1 ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
intro n hn hk IH
[GOAL]
case H.refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
⊢ (List.prod (List.drop n (listTransvecCol M)) * M) (inl i) (inr ()) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
have hn' : n < (listTransvecCol M).length := by simpa [listTransvecCol] using hn
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
⊢ n < List.length (listTransvecCol M)
[PROOFSTEP]
simpa [listTransvecCol] using hn
[GOAL]
case H.refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
⊢ (List.prod (List.drop n (listTransvecCol M)) * M) (inl i) (inr ()) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
let n' : Fin r :=
⟨n, hn⟩
-- porting note: after changing from `nthLe` to `get`, we need to provide all arguments
[GOAL]
case H.refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
⊢ (List.prod (List.drop n (listTransvecCol M)) * M) (inl i) (inr ()) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
rw [← @List.cons_get_drop_succ _ _ ⟨n, hn'⟩]
[GOAL]
case H.refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
⊢ (List.prod
(List.get (listTransvecCol M) { val := n, isLt := hn' } ::
List.drop (↑{ val := n, isLt := hn' } + 1) (listTransvecCol M)) *
M)
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
have A :
(listTransvecCol M).get ⟨n, hn'⟩ =
transvection (inl n') (inr unit) (-M (inl n') (inr unit) / M (inr unit) (inr unit)) :=
by simp [listTransvecCol]
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
⊢ List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
[PROOFSTEP]
simp [listTransvecCol]
[GOAL]
case H.refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
⊢ (List.prod
(List.get (listTransvecCol M) { val := n, isLt := hn' } ::
List.drop (↑{ val := n, isLt := hn' } + 1) (listTransvecCol M)) *
M)
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
simp only [Matrix.mul_assoc, A, List.prod_cons]
[GOAL]
case H.refine'_1
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
⊢ (transvection (inl { val := n, isLt := hn }) (inr ())
(-M (inl { val := n, isLt := hn }) (inr ()) / M (inr ()) (inr ())) *
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M))
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
by_cases h : n' = i
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : n' = i
⊢ (transvection (inl { val := n, isLt := hn }) (inr ())
(-M (inl { val := n, isLt := hn }) (inr ()) / M (inr ()) (inr ())) *
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M))
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
have hni : n = i := by
cases i
simp only [Fin.mk_eq_mk] at h
simp [h]
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : n' = i
⊢ n = ↑i
[PROOFSTEP]
cases i
[GOAL]
case mk
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
val✝ : ℕ
isLt✝ : val✝ < r
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl { val := val✝, isLt := isLt✝ }) (inr ()) =
if n + 1 ≤ ↑{ val := val✝, isLt := isLt✝ } then 0 else M (inl { val := val✝, isLt := isLt✝ }) (inr ())
h : n' = { val := val✝, isLt := isLt✝ }
⊢ n = ↑{ val := val✝, isLt := isLt✝ }
[PROOFSTEP]
simp only [Fin.mk_eq_mk] at h
[GOAL]
case mk
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
val✝ : ℕ
isLt✝ : val✝ < r
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl { val := val✝, isLt := isLt✝ }) (inr ()) =
if n + 1 ≤ ↑{ val := val✝, isLt := isLt✝ } then 0 else M (inl { val := val✝, isLt := isLt✝ }) (inr ())
h : n = val✝
⊢ n = ↑{ val := val✝, isLt := isLt✝ }
[PROOFSTEP]
simp [h]
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : n' = i
hni : n = ↑i
⊢ (transvection (inl { val := n, isLt := hn }) (inr ())
(-M (inl { val := n, isLt := hn }) (inr ()) / M (inr ()) (inr ())) *
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M))
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
simp only [h, transvection_mul_apply_same, IH, ← hni, add_le_iff_nonpos_right, listTransvecCol_mul_last_row_drop _ _ hn]
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : n' = i
hni : n = ↑i
⊢ (if False then 0 else M (inl i) (inr ())) + -M (inl i) (inr ()) / M (inr ()) (inr ()) * M (inr ()) (inr ()) =
if n ≤ n then 0 else M (inl i) (inr ())
[PROOFSTEP]
field_simp [hM]
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
⊢ (transvection (inl { val := n, isLt := hn }) (inr ())
(-M (inl { val := n, isLt := hn }) (inr ()) / M (inr ()) (inr ())) *
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M))
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
have hni : n ≠ i := by
rintro rfl
cases i
simp at h
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
⊢ n ≠ ↑i
[PROOFSTEP]
rintro rfl
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
hn : ↑i < r
hk : k ≤ ↑i
IH :
(List.prod (List.drop (↑i + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if ↑i + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : ↑i < List.length (listTransvecCol M)
n' : Fin r := { val := ↑i, isLt := hn }
A :
List.get (listTransvecCol M) { val := ↑i, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
⊢ False
[PROOFSTEP]
cases i
[GOAL]
case mk
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
k : ℕ
hk✝ : k ≤ r
val✝ : ℕ
isLt✝ : val✝ < r
hn : ↑{ val := val✝, isLt := isLt✝ } < r
hk : k ≤ ↑{ val := val✝, isLt := isLt✝ }
IH :
(List.prod (List.drop (↑{ val := val✝, isLt := isLt✝ } + 1) (listTransvecCol M)) * M)
(inl { val := val✝, isLt := isLt✝ }) (inr ()) =
if ↑{ val := val✝, isLt := isLt✝ } + 1 ≤ ↑{ val := val✝, isLt := isLt✝ } then 0
else M (inl { val := val✝, isLt := isLt✝ }) (inr ())
hn' : ↑{ val := val✝, isLt := isLt✝ } < List.length (listTransvecCol M)
n' : Fin r := { val := ↑{ val := val✝, isLt := isLt✝ }, isLt := hn }
A :
List.get (listTransvecCol M) { val := ↑{ val := val✝, isLt := isLt✝ }, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = { val := val✝, isLt := isLt✝ }
⊢ False
[PROOFSTEP]
simp at h
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
⊢ (transvection (inl { val := n, isLt := hn }) (inr ())
(-M (inl { val := n, isLt := hn }) (inr ()) / M (inr ()) (inr ())) *
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M))
(inl i) (inr ()) =
if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
simp only [ne_eq, inl.injEq, Ne.symm h, not_false_eq_true, transvection_mul_apply_of_ne]
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
⊢ (List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
rw [IH]
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
⊢ (if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
rcases le_or_lt (n + 1) i with (hi | hi)
[GOAL]
case neg.inl
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
hi : n + 1 ≤ ↑i
⊢ (if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
simp only [hi, n.le_succ.trans hi, if_true]
[GOAL]
case neg.inr
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
hi : ↑i < n + 1
⊢ (if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())) = if n ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
rw [if_neg, if_neg]
[GOAL]
case neg.inr.hnc
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
hi : ↑i < n + 1
⊢ ¬n ≤ ↑i
[PROOFSTEP]
simpa only [hni.symm, not_le, or_false_iff] using Nat.lt_succ_iff_lt_or_eq.1 hi
[GOAL]
case neg.inr.hnc
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
hn : n < r
hk : k ≤ n
IH :
(List.prod (List.drop (n + 1) (listTransvecCol M)) * M) (inl i) (inr ()) =
if n + 1 ≤ ↑i then 0 else M (inl i) (inr ())
hn' : n < List.length (listTransvecCol M)
n' : Fin r := { val := n, isLt := hn }
A :
List.get (listTransvecCol M) { val := n, isLt := hn' } =
transvection (inl n') (inr ()) (-M (inl n') (inr ()) / M (inr ()) (inr ()))
h : ¬n' = i
hni : n ≠ ↑i
hi : ↑i < n + 1
⊢ ¬n + 1 ≤ ↑i
[PROOFSTEP]
simpa only [not_le] using hi
[GOAL]
case H.refine'_2
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk : k ≤ r
⊢ (List.prod (List.drop r (listTransvecCol M)) * M) (inl i) (inr ()) = if r ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
simp only [listTransvecCol, List.length_ofFn, le_refl, List.drop_eq_nil_of_le, List.prod_nil, Matrix.one_mul]
[GOAL]
case H.refine'_2
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk : k ≤ r
⊢ M (inl i) (inr ()) = if r ≤ ↑i then 0 else M (inl i) (inr ())
[PROOFSTEP]
rw [if_neg]
[GOAL]
case H.refine'_2.hnc
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk : k ≤ r
⊢ ¬r ≤ ↑i
[PROOFSTEP]
simpa only [not_le] using i.2
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk : k ≤ r
⊢ (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
induction' k with k IH
[GOAL]
case zero
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k : ℕ
hk✝ : k ≤ r
hk : Nat.zero ≤ r
⊢ (M * List.prod (List.take Nat.zero (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
simp only [Matrix.mul_one, List.take_zero, List.prod_nil, List.take, Matrix.mul_one]
[GOAL]
case succ
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
⊢ (M * List.prod (List.take (Nat.succ k) (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
have hkr : k < r := hk
[GOAL]
case succ
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
hkr : k < r
⊢ (M * List.prod (List.take (Nat.succ k) (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
let k' : Fin r := ⟨k, hkr⟩
[GOAL]
case succ
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
hkr : k < r
k' : Fin r := { val := k, isLt := hkr }
⊢ (M * List.prod (List.take (Nat.succ k) (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
have :
(listTransvecRow M).get? k =
↑(transvection (inr Unit.unit) (inl k') (-M (inr Unit.unit) (inl k') / M (inr Unit.unit) (inr Unit.unit))) :=
by simp only [listTransvecRow, List.ofFnNthVal, hkr, dif_pos, List.get?_ofFn]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
hkr : k < r
k' : Fin r := { val := k, isLt := hkr }
⊢ List.get? (listTransvecRow M) k = some (transvection (inr ()) (inl k') (-M (inr ()) (inl k') / M (inr ()) (inr ())))
[PROOFSTEP]
simp only [listTransvecRow, List.ofFnNthVal, hkr, dif_pos, List.get?_ofFn]
[GOAL]
case succ
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
hkr : k < r
k' : Fin r := { val := k, isLt := hkr }
this :
List.get? (listTransvecRow M) k = some (transvection (inr ()) (inl k') (-M (inr ()) (inl k') / M (inr ()) (inr ())))
⊢ (M * List.prod (List.take (Nat.succ k) (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
simp only [List.take_succ, ← Matrix.mul_assoc, this, List.prod_append, Matrix.mul_one, List.prod_cons, List.prod_nil,
Option.to_list_some]
[GOAL]
case succ
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
hkr : k < r
k' : Fin r := { val := k, isLt := hkr }
this :
List.get? (listTransvecRow M) k = some (transvection (inr ()) (inl k') (-M (inr ()) (inl k') / M (inr ()) (inr ())))
⊢ (M * List.prod (List.take k (listTransvecRow M)) *
transvection (inr ()) (inl { val := k, isLt := hkr })
(-M (inr ()) (inl { val := k, isLt := hkr }) / M (inr ()) (inr ())))
i (inr ()) =
M i (inr ())
[PROOFSTEP]
rw [mul_transvection_apply_of_ne, IH hkr.le]
[GOAL]
case succ.hb
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
k✝ : ℕ
hk✝ : k✝ ≤ r
k : ℕ
IH : k ≤ r → (M * List.prod (List.take k (listTransvecRow M))) i (inr ()) = M i (inr ())
hk : Nat.succ k ≤ r
hkr : k < r
k' : Fin r := { val := k, isLt := hkr }
this :
List.get? (listTransvecRow M) k = some (transvection (inr ()) (inl k') (-M (inr ()) (inl k') / M (inr ()) (inr ())))
⊢ inr () ≠ inl { val := k, isLt := hkr }
[PROOFSTEP]
simp only [Ne.def, not_false_iff]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
⊢ (M * List.prod (listTransvecRow M)) i (inr ()) = M i (inr ())
[PROOFSTEP]
have A : (listTransvecRow M).length = r := by simp [listTransvecRow]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
⊢ List.length (listTransvecRow M) = r
[PROOFSTEP]
simp [listTransvecRow]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
A : List.length (listTransvecRow M) = r
⊢ (M * List.prod (listTransvecRow M)) i (inr ()) = M i (inr ())
[PROOFSTEP]
rw [← List.take_length (listTransvecRow M), A]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
i : Fin r ⊕ Unit
A : List.length (listTransvecRow M) = r
⊢ (M * List.prod (List.take r (listTransvecRow M))) i (inr ()) = M i (inr ())
[PROOFSTEP]
simpa using mul_listTransvecRow_last_col_take M i le_rfl
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ (M * List.prod (listTransvecRow M)) (inr ()) (inl i) = 0
[PROOFSTEP]
suffices H :
∀ k : ℕ,
k ≤ r → (M * ((listTransvecRow M).take k).prod) (inr unit) (inl i) = if k ≤ i then M (inr unit) (inl i) else 0
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
⊢ (M * List.prod (listTransvecRow M)) (inr ()) (inl i) = 0
[PROOFSTEP]
have A : (listTransvecRow M).length = r := by simp [listTransvecRow]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
⊢ List.length (listTransvecRow M) = r
[PROOFSTEP]
simp [listTransvecRow]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
A : List.length (listTransvecRow M) = r
⊢ (M * List.prod (listTransvecRow M)) (inr ()) (inl i) = 0
[PROOFSTEP]
rw [← List.take_length (listTransvecRow M), A]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
A : List.length (listTransvecRow M) = r
⊢ (M * List.prod (List.take r (listTransvecRow M))) (inr ()) (inl i) = 0
[PROOFSTEP]
have : ¬r ≤ i := by simp
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
A : List.length (listTransvecRow M) = r
⊢ ¬r ≤ ↑i
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
H :
∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
A : List.length (listTransvecRow M) = r
this : ¬r ≤ ↑i
⊢ (M * List.prod (List.take r (listTransvecRow M))) (inr ()) (inl i) = 0
[PROOFSTEP]
simpa only [this, ite_eq_right_iff] using H r le_rfl
[GOAL]
case H
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ ∀ (k : ℕ),
k ≤ r →
(M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
intro k hk
[GOAL]
case H
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk : k ≤ r
⊢ (M * List.prod (List.take k (listTransvecRow M))) (inr ()) (inl i) = if k ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
induction' k with n IH
[GOAL]
case H.zero
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
hk : Nat.zero ≤ r
⊢ (M * List.prod (List.take Nat.zero (listTransvecRow M))) (inr ()) (inl i) =
if Nat.zero ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
simp only [if_true, Matrix.mul_one, List.take_zero, zero_le', List.prod_nil, Nat.zero_eq]
[GOAL]
case H.succ
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
⊢ (M * List.prod (List.take (Nat.succ n) (listTransvecRow M))) (inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
have hnr : n < r := hk
[GOAL]
case H.succ
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
⊢ (M * List.prod (List.take (Nat.succ n) (listTransvecRow M))) (inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
let n' : Fin r := ⟨n, hnr⟩
[GOAL]
case H.succ
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
⊢ (M * List.prod (List.take (Nat.succ n) (listTransvecRow M))) (inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
have A :
(listTransvecRow M).get? n = ↑(transvection (inr unit) (inl n') (-M (inr unit) (inl n') / M (inr unit) (inr unit))) :=
by simp only [listTransvecRow, List.ofFnNthVal, hnr, dif_pos, List.get?_ofFn]
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
⊢ List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
[PROOFSTEP]
simp only [listTransvecRow, List.ofFnNthVal, hnr, dif_pos, List.get?_ofFn]
[GOAL]
case H.succ
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
⊢ (M * List.prod (List.take (Nat.succ n) (listTransvecRow M))) (inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
simp only [List.take_succ, A, ← Matrix.mul_assoc, List.prod_append, Matrix.mul_one, List.prod_cons, List.prod_nil,
Option.to_list_some]
[GOAL]
case H.succ
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
⊢ (M * List.prod (List.take n (listTransvecRow M)) *
transvection (inr ()) (inl { val := n, isLt := hnr })
(-M (inr ()) (inl { val := n, isLt := hnr }) / M (inr ()) (inr ())))
(inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
by_cases h : n' = i
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : n' = i
⊢ (M * List.prod (List.take n (listTransvecRow M)) *
transvection (inr ()) (inl { val := n, isLt := hnr })
(-M (inr ()) (inl { val := n, isLt := hnr }) / M (inr ()) (inr ())))
(inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
have hni : n = i := by
cases i
simp only [Fin.mk_eq_mk] at h
simp only [h]
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : n' = i
⊢ n = ↑i
[PROOFSTEP]
cases i
[GOAL]
case mk
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
k : ℕ
hk✝ : k ≤ r
n : ℕ
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
val✝ : ℕ
isLt✝ : val✝ < r
IH :
n ≤ r →
(M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl { val := val✝, isLt := isLt✝ }) =
if n ≤ ↑{ val := val✝, isLt := isLt✝ } then M (inr ()) (inl { val := val✝, isLt := isLt✝ }) else 0
h : n' = { val := val✝, isLt := isLt✝ }
⊢ n = ↑{ val := val✝, isLt := isLt✝ }
[PROOFSTEP]
simp only [Fin.mk_eq_mk] at h
[GOAL]
case mk
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
k : ℕ
hk✝ : k ≤ r
n : ℕ
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
val✝ : ℕ
isLt✝ : val✝ < r
IH :
n ≤ r →
(M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl { val := val✝, isLt := isLt✝ }) =
if n ≤ ↑{ val := val✝, isLt := isLt✝ } then M (inr ()) (inl { val := val✝, isLt := isLt✝ }) else 0
h : n = val✝
⊢ n = ↑{ val := val✝, isLt := isLt✝ }
[PROOFSTEP]
simp only [h]
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : n' = i
hni : n = ↑i
⊢ (M * List.prod (List.take n (listTransvecRow M)) *
transvection (inr ()) (inl { val := n, isLt := hnr })
(-M (inr ()) (inl { val := n, isLt := hnr }) / M (inr ()) (inr ())))
(inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
have : ¬n.succ ≤ i := by simp only [← hni, n.lt_succ_self, not_le]
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : n' = i
hni : n = ↑i
⊢ ¬Nat.succ n ≤ ↑i
[PROOFSTEP]
simp only [← hni, n.lt_succ_self, not_le]
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : n' = i
hni : n = ↑i
this : ¬Nat.succ n ≤ ↑i
⊢ (M * List.prod (List.take n (listTransvecRow M)) *
transvection (inr ()) (inl { val := n, isLt := hnr })
(-M (inr ()) (inl { val := n, isLt := hnr }) / M (inr ()) (inr ())))
(inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
simp only [h, mul_transvection_apply_same, List.take, if_false, mul_listTransvecRow_last_col_take _ _ hnr.le, hni.le,
this, if_true, IH hnr.le]
[GOAL]
case pos
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : n' = i
hni : n = ↑i
this : ¬Nat.succ n ≤ ↑i
⊢ M (inr ()) (inl i) + -M (inr ()) (inl i) / M (inr ()) (inr ()) * M (inr ()) (inr ()) = 0
[PROOFSTEP]
field_simp [hM]
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
⊢ (M * List.prod (List.take n (listTransvecRow M)) *
transvection (inr ()) (inl { val := n, isLt := hnr })
(-M (inr ()) (inl { val := n, isLt := hnr }) / M (inr ()) (inr ())))
(inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
have hni : n ≠ i := by
rintro rfl
cases i
tauto
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
⊢ n ≠ ↑i
[PROOFSTEP]
rintro rfl
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
IH :
↑i ≤ r →
(M * List.prod (List.take (↑i) (listTransvecRow M))) (inr ()) (inl i) = if ↑i ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ ↑i ≤ r
hnr : ↑i < r
n' : Fin r := { val := ↑i, isLt := hnr }
A :
List.get? (listTransvecRow M) ↑i = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
⊢ False
[PROOFSTEP]
cases i
[GOAL]
case mk
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
k : ℕ
hk✝ : k ≤ r
val✝ : ℕ
isLt✝ : val✝ < r
IH :
↑{ val := val✝, isLt := isLt✝ } ≤ r →
(M * List.prod (List.take (↑{ val := val✝, isLt := isLt✝ }) (listTransvecRow M))) (inr ())
(inl { val := val✝, isLt := isLt✝ }) =
if ↑{ val := val✝, isLt := isLt✝ } ≤ ↑{ val := val✝, isLt := isLt✝ } then
M (inr ()) (inl { val := val✝, isLt := isLt✝ })
else 0
hk : Nat.succ ↑{ val := val✝, isLt := isLt✝ } ≤ r
hnr : ↑{ val := val✝, isLt := isLt✝ } < r
n' : Fin r := { val := ↑{ val := val✝, isLt := isLt✝ }, isLt := hnr }
A :
List.get? (listTransvecRow M) ↑{ val := val✝, isLt := isLt✝ } =
some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = { val := val✝, isLt := isLt✝ }
⊢ False
[PROOFSTEP]
tauto
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
hni : n ≠ ↑i
⊢ (M * List.prod (List.take n (listTransvecRow M)) *
transvection (inr ()) (inl { val := n, isLt := hnr })
(-M (inr ()) (inl { val := n, isLt := hnr }) / M (inr ()) (inr ())))
(inr ()) (inl i) =
if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
simp only [IH hnr.le, Ne.def, mul_transvection_apply_of_ne, Ne.symm h, inl.injEq]
[GOAL]
case neg
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
hni : n ≠ ↑i
⊢ (if n ≤ ↑i then M (inr ()) (inl i) else 0) = if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
rcases le_or_lt (n + 1) i with (hi | hi)
[GOAL]
case neg.inl
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
hni : n ≠ ↑i
hi : n + 1 ≤ ↑i
⊢ (if n ≤ ↑i then M (inr ()) (inl i) else 0) = if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
simp [hi, n.le_succ.trans hi, if_true]
[GOAL]
case neg.inr
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
hni : n ≠ ↑i
hi : ↑i < n + 1
⊢ (if n ≤ ↑i then M (inr ()) (inl i) else 0) = if Nat.succ n ≤ ↑i then M (inr ()) (inl i) else 0
[PROOFSTEP]
rw [if_neg, if_neg]
[GOAL]
case neg.inr.hnc
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
hni : n ≠ ↑i
hi : ↑i < n + 1
⊢ ¬Nat.succ n ≤ ↑i
[PROOFSTEP]
simpa only [not_le] using hi
[GOAL]
case neg.inr.hnc
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n✝
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
k : ℕ
hk✝ : k ≤ r
n : ℕ
IH :
n ≤ r → (M * List.prod (List.take n (listTransvecRow M))) (inr ()) (inl i) = if n ≤ ↑i then M (inr ()) (inl i) else 0
hk : Nat.succ n ≤ r
hnr : n < r
n' : Fin r := { val := n, isLt := hnr }
A : List.get? (listTransvecRow M) n = some (transvection (inr ()) (inl n') (-M (inr ()) (inl n') / M (inr ()) (inr ())))
h : ¬n' = i
hni : n ≠ ↑i
hi : ↑i < n + 1
⊢ ¬n ≤ ↑i
[PROOFSTEP]
simpa only [hni.symm, not_le, or_false_iff] using Nat.lt_succ_iff_lt_or_eq.1 hi
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) (inr ()) (inl i) = 0
[PROOFSTEP]
have : listTransvecRow M = listTransvecRow ((listTransvecCol M).prod * M) := by
simp [listTransvecRow, listTransvecCol_mul_last_row]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ listTransvecRow M = listTransvecRow (List.prod (listTransvecCol M) * M)
[PROOFSTEP]
simp [listTransvecRow, listTransvecCol_mul_last_row]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
this : listTransvecRow M = listTransvecRow (List.prod (listTransvecCol M) * M)
⊢ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) (inr ()) (inl i) = 0
[PROOFSTEP]
rw [this]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
this : listTransvecRow M = listTransvecRow (List.prod (listTransvecCol M) * M)
⊢ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow (List.prod (listTransvecCol M) * M))) (inr ())
(inl i) =
0
[PROOFSTEP]
apply mul_listTransvecRow_last_row
[GOAL]
case hM
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
this : listTransvecRow M = listTransvecRow (List.prod (listTransvecCol M) * M)
⊢ (List.prod (listTransvecCol M) * M) (inr ()) (inr ()) ≠ 0
[PROOFSTEP]
simpa [listTransvecCol_mul_last_row] using hM
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) (inl i) (inr ()) = 0
[PROOFSTEP]
have : listTransvecCol M = listTransvecCol (M * (listTransvecRow M).prod) := by
simp [listTransvecCol, mul_listTransvecRow_last_col]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ listTransvecCol M = listTransvecCol (M * List.prod (listTransvecRow M))
[PROOFSTEP]
simp [listTransvecCol, mul_listTransvecRow_last_col]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
this : listTransvecCol M = listTransvecCol (M * List.prod (listTransvecRow M))
⊢ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) (inl i) (inr ()) = 0
[PROOFSTEP]
rw [this, Matrix.mul_assoc]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
this : listTransvecCol M = listTransvecCol (M * List.prod (listTransvecRow M))
⊢ (List.prod (listTransvecCol (M * List.prod (listTransvecRow M))) * (M * List.prod (listTransvecRow M))) (inl i)
(inr ()) =
0
[PROOFSTEP]
apply listTransvecCol_mul_last_col
[GOAL]
case hM
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
this : listTransvecCol M = listTransvecCol (M * List.prod (listTransvecRow M))
⊢ (M * List.prod (listTransvecRow M)) (inr ()) (inr ()) ≠ 0
[PROOFSTEP]
simpa [mul_listTransvecRow_last_col] using hM
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
⊢ IsTwoBlockDiagonal (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M))
[PROOFSTEP]
constructor
[GOAL]
case left
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
⊢ toBlocks₁₂ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) = 0
[PROOFSTEP]
ext i j
[GOAL]
case left.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
j : Unit
⊢ toBlocks₁₂ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) i j = OfNat.ofNat 0 i j
[PROOFSTEP]
have : j = unit := by simp only [eq_iff_true_of_subsingleton]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
j : Unit
⊢ j = ()
[PROOFSTEP]
simp only [eq_iff_true_of_subsingleton]
[GOAL]
case left.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
j : Unit
this : j = ()
⊢ toBlocks₁₂ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) i j = OfNat.ofNat 0 i j
[PROOFSTEP]
simp [toBlocks₁₂, this, listTransvecCol_mul_mul_listTransvecRow_last_row M hM]
[GOAL]
case right
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
⊢ toBlocks₂₁ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) = 0
[PROOFSTEP]
ext i j
[GOAL]
case right.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Unit
j : Fin r
⊢ toBlocks₂₁ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) i j = OfNat.ofNat 0 i j
[PROOFSTEP]
have : i = unit := by simp only [eq_iff_true_of_subsingleton]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Unit
j : Fin r
⊢ i = ()
[PROOFSTEP]
simp only [eq_iff_true_of_subsingleton]
[GOAL]
case right.a.h
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Unit
j : Fin r
this : i = ()
⊢ toBlocks₂₁ (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M)) i j = OfNat.ofNat 0 i j
[PROOFSTEP]
simp [toBlocks₂₁, this, listTransvecCol_mul_mul_listTransvecRow_last_col M hM]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
let L : List (TransvectionStruct (Sum (Fin r) Unit) 𝕜) :=
List.ofFn fun i : Fin r => ⟨inl i, inr unit, by simp, -M (inl i) (inr unit) / M (inr unit) (inr unit)⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
i : Fin r
⊢ inl i ≠ inr ()
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
let L' : List (TransvectionStruct (Sum (Fin r) Unit) 𝕜) :=
List.ofFn fun i : Fin r => ⟨inr unit, inl i, by simp, -M (inr unit) (inl i) / M (inr unit) (inr unit)⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
i : Fin r
⊢ inr () ≠ inl i
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
refine' ⟨L, L', _⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
⊢ IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
have A : L.map toMatrix = listTransvecCol M := by simp [listTransvecCol, (· ∘ ·)]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
⊢ List.map toMatrix L = listTransvecCol M
[PROOFSTEP]
simp [listTransvecCol, (· ∘ ·)]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
A : List.map toMatrix L = listTransvecCol M
⊢ IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
have B : L'.map toMatrix = listTransvecRow M := by simp [listTransvecRow, (· ∘ ·)]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
A : List.map toMatrix L = listTransvecCol M
⊢ List.map toMatrix L' = listTransvecRow M
[PROOFSTEP]
simp [listTransvecRow, (· ∘ ·)]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
A : List.map toMatrix L = listTransvecCol M
B : List.map toMatrix L' = listTransvecRow M
⊢ IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
rw [A, B]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) ≠ 0
L : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := -M (inl i) (inr ()) / M (inr ()) (inr ()) }
L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜) :=
List.ofFn fun i =>
{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := -M (inr ()) (inl i) / M (inr ()) (inr ()) }
A : List.map toMatrix L = listTransvecCol M
B : List.map toMatrix L' = listTransvecRow M
⊢ IsTwoBlockDiagonal (List.prod (listTransvecCol M) * M * List.prod (listTransvecRow M))
[PROOFSTEP]
exact isTwoBlockDiagonal_listTransvecCol_mul_mul_listTransvecRow M hM
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
by_cases H : IsTwoBlockDiagonal M
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
H : IsTwoBlockDiagonal M
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
refine'
⟨List.nil, List.nil, by simpa using H⟩
-- we have already proved this when the last coefficient is nonzero
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
H : IsTwoBlockDiagonal M
⊢ IsTwoBlockDiagonal (List.prod (List.map toMatrix []) * M * List.prod (List.map toMatrix []))
[PROOFSTEP]
simpa using H
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
H : ¬IsTwoBlockDiagonal M
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
by_cases hM : M (inr unit) (inr unit) ≠ 0
[GOAL]
case pos
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
H : ¬IsTwoBlockDiagonal M
hM : M (inr ()) (inr ()) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
exact exists_isTwoBlockDiagonal_of_ne_zero M hM
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
H : ¬IsTwoBlockDiagonal M
hM : ¬M (inr ()) (inr ()) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
push_neg at hM
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
H : ¬IsTwoBlockDiagonal M
hM : M (inr ()) (inr ()) = 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
simp only [not_and_or, IsTwoBlockDiagonal, toBlocks₁₂, toBlocks₂₁, ← Matrix.ext_iff] at H
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
have : ∃ i : Fin r, M (inl i) (inr unit) ≠ 0 ∨ M (inr unit) (inl i) ≠ 0 :=
by
cases' H with H H
· contrapose! H
rintro i ⟨⟩
exact (H i).1
· contrapose! H
rintro ⟨⟩ j
exact (H j).2
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
⊢ ∃ i, M (inl i) (inr ()) ≠ 0 ∨ M (inr ()) (inl i) ≠ 0
[PROOFSTEP]
cases' H with H H
[GOAL]
case inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H : ¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j
⊢ ∃ i, M (inl i) (inr ()) ≠ 0 ∨ M (inr ()) (inl i) ≠ 0
[PROOFSTEP]
contrapose! H
[GOAL]
case inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H : ∀ (i : Fin r), M (inl i) (inr ()) = 0 ∧ M (inr ()) (inl i) = 0
⊢ ∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j
[PROOFSTEP]
rintro i ⟨⟩
[GOAL]
case inl.unit
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H : ∀ (i : Fin r), M (inl i) (inr ()) = 0 ∧ M (inr ()) (inl i) = 0
i : Fin r
⊢ ↑of (fun i j => M (inl i) (inr j)) i PUnit.unit = OfNat.ofNat 0 i PUnit.unit
[PROOFSTEP]
exact (H i).1
[GOAL]
case inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H : ¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
⊢ ∃ i, M (inl i) (inr ()) ≠ 0 ∨ M (inr ()) (inl i) ≠ 0
[PROOFSTEP]
contrapose! H
[GOAL]
case inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H : ∀ (i : Fin r), M (inl i) (inr ()) = 0 ∧ M (inr ()) (inl i) = 0
⊢ ∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
[PROOFSTEP]
rintro ⟨⟩ j
[GOAL]
case inr.unit
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H : ∀ (i : Fin r), M (inl i) (inr ()) = 0 ∧ M (inr ()) (inl i) = 0
j : Fin r
⊢ ↑of (fun i j => M (inr i) (inl j)) PUnit.unit j = OfNat.ofNat 0 PUnit.unit j
[PROOFSTEP]
exact (H j).2
[GOAL]
case neg
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
this : ∃ i, M (inl i) (inr ()) ≠ 0 ∨ M (inr ()) (inl i) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
rcases this with ⟨i, h | h⟩
[GOAL]
case neg.intro.inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
let M' := transvection (inr Unit.unit) (inl i) 1 * M
[GOAL]
case neg.intro.inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
have hM' : M' (inr unit) (inr unit) ≠ 0 := by simpa [hM]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
⊢ M' (inr ()) (inr ()) ≠ 0
[PROOFSTEP]
simpa [hM]
[GOAL]
case neg.intro.inl
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
hM' : M' (inr ()) (inr ()) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
rcases exists_isTwoBlockDiagonal_of_ne_zero M' hM' with ⟨L, L', hLL'⟩
[GOAL]
case neg.intro.inl.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M' * List.prod (List.map toMatrix L'))
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
rw [Matrix.mul_assoc] at hLL'
[GOAL]
case neg.intro.inl.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * (M' * List.prod (List.map toMatrix L')))
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
refine' ⟨L ++ [⟨inr unit, inl i, by simp, 1⟩], L', _⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * (M' * List.prod (List.map toMatrix L')))
⊢ inr () ≠ inl i
[PROOFSTEP]
simp
[GOAL]
case neg.intro.inl.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * (M' * List.prod (List.map toMatrix L')))
⊢ IsTwoBlockDiagonal
(List.prod (List.map toMatrix (L ++ [{ i := inr (), j := inl i, hij := (_ : ¬inr () = inl i), c := 1 }])) * M *
List.prod (List.map toMatrix L'))
[PROOFSTEP]
simp only [List.map_append, List.prod_append, Matrix.mul_one, toMatrix_mk, List.prod_cons, List.prod_nil, List.map,
Matrix.mul_assoc (L.map toMatrix).prod]
[GOAL]
case neg.intro.inl.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inl i) (inr ()) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := transvection (inr ()) (inl i) 1 * M
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * (M' * List.prod (List.map toMatrix L')))
⊢ IsTwoBlockDiagonal
(List.prod (List.map toMatrix L) * (transvection (inr ()) (inl i) 1 * M * List.prod (List.map toMatrix L')))
[PROOFSTEP]
exact hLL'
[GOAL]
case neg.intro.inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
let M' := M * transvection (inl i) (inr unit) 1
[GOAL]
case neg.intro.inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
have hM' : M' (inr unit) (inr unit) ≠ 0 := by simpa [hM]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
⊢ M' (inr ()) (inr ()) ≠ 0
[PROOFSTEP]
simpa [hM]
[GOAL]
case neg.intro.inr
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
hM' : M' (inr ()) (inr ()) ≠ 0
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
rcases exists_isTwoBlockDiagonal_of_ne_zero M' hM' with ⟨L, L', hLL'⟩
[GOAL]
case neg.intro.inr.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M' * List.prod (List.map toMatrix L'))
⊢ ∃ L L', IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L'))
[PROOFSTEP]
refine' ⟨L, ⟨inl i, inr unit, by simp, 1⟩ :: L', _⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M' * List.prod (List.map toMatrix L'))
⊢ inl i ≠ inr ()
[PROOFSTEP]
simp
[GOAL]
case neg.intro.inr.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M' * List.prod (List.map toMatrix L'))
⊢ IsTwoBlockDiagonal
(List.prod (List.map toMatrix L) * M *
List.prod (List.map toMatrix ({ i := inl i, j := inr (), hij := (_ : ¬inl i = inr ()), c := 1 } :: L')))
[PROOFSTEP]
simp only [← Matrix.mul_assoc, toMatrix_mk, List.prod_cons, List.map]
[GOAL]
case neg.intro.inr.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M' * List.prod (List.map toMatrix L'))
⊢ IsTwoBlockDiagonal
(List.prod (List.map toMatrix L) * M * transvection (inl i) (inr ()) 1 * List.prod (List.map toMatrix L'))
[PROOFSTEP]
rw [Matrix.mul_assoc (L.map toMatrix).prod]
[GOAL]
case neg.intro.inr.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
hM : M (inr ()) (inr ()) = 0
H :
(¬∀ (i : Fin r) (j : Unit), ↑of (fun i j => M (inl i) (inr j)) i j = OfNat.ofNat 0 i j) ∨
¬∀ (i : Unit) (j : Fin r), ↑of (fun i j => M (inr i) (inl j)) i j = OfNat.ofNat 0 i j
i : Fin r
h : M (inr ()) (inl i) ≠ 0
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := M * transvection (inl i) (inr ()) 1
hM' : M' (inr ()) (inr ()) ≠ 0
L L' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hLL' : IsTwoBlockDiagonal (List.prod (List.map toMatrix L) * M' * List.prod (List.map toMatrix L'))
⊢ IsTwoBlockDiagonal
(List.prod (List.map toMatrix L) * (M * transvection (inl i) (inr ()) 1) * List.prod (List.map toMatrix L'))
[PROOFSTEP]
exact hLL'
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
rcases exists_isTwoBlockDiagonal_list_transvec_mul_mul_list_transvec M with ⟨L₁, L₁', hM⟩
[GOAL]
case intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
let M' := (L₁.map toMatrix).prod * M * (L₁'.map toMatrix).prod
[GOAL]
case intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
let M'' := toBlocks₁₁ M'
[GOAL]
case intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
rcases IH M'' with ⟨L₀, L₀', D₀, h₀⟩
[GOAL]
case intro.intro.intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
set c := M' (inr unit) (inr unit)
[GOAL]
case intro.intro.intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
refine' ⟨L₀.map (sumInl Unit) ++ L₁, L₁' ++ L₀'.map (sumInl Unit), Sum.elim D₀ fun _ => M' (inr unit) (inr unit), _⟩
[GOAL]
case intro.intro.intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
⊢ List.prod (List.map toMatrix (List.map (sumInl Unit) L₀ ++ L₁)) * M *
List.prod (List.map toMatrix (L₁' ++ List.map (sumInl Unit) L₀')) =
diagonal (Sum.elim D₀ fun x => M' (inr ()) (inr ()))
[PROOFSTEP]
suffices
(L₀.map (toMatrix ∘ sumInl Unit)).prod * M' * (L₀'.map (toMatrix ∘ sumInl Unit)).prod =
diagonal (Sum.elim D₀ fun _ => c)
by simpa [Matrix.mul_assoc]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
this :
List.prod (List.map (toMatrix ∘ sumInl Unit) L₀) * M' * List.prod (List.map (toMatrix ∘ sumInl Unit) L₀') =
diagonal (Sum.elim D₀ fun x => c)
⊢ List.prod (List.map toMatrix (List.map (sumInl Unit) L₀ ++ L₁)) * M *
List.prod (List.map toMatrix (L₁' ++ List.map (sumInl Unit) L₀')) =
diagonal (Sum.elim D₀ fun x => M' (inr ()) (inr ()))
[PROOFSTEP]
simpa [Matrix.mul_assoc]
[GOAL]
case intro.intro.intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
⊢ List.prod (List.map (toMatrix ∘ sumInl Unit) L₀) * M' * List.prod (List.map (toMatrix ∘ sumInl Unit) L₀') =
diagonal (Sum.elim D₀ fun x => c)
[PROOFSTEP]
have : M' = fromBlocks M'' 0 0 (diagonal fun _ => c) := by
-- porting note: simplified proof, because `congr` didn't work anymore
rw [← fromBlocks_toBlocks M', hM.1, hM.2]
rfl
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
⊢ M' = fromBlocks M'' 0 0 (diagonal fun x => c)
[PROOFSTEP]
rw [← fromBlocks_toBlocks M', hM.1, hM.2]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
⊢ fromBlocks (toBlocks₁₁ M') 0 0 (toBlocks₂₂ M') = fromBlocks M'' 0 0 (diagonal fun x => c)
[PROOFSTEP]
rfl
[GOAL]
case intro.intro.intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
this : M' = fromBlocks M'' 0 0 (diagonal fun x => c)
⊢ List.prod (List.map (toMatrix ∘ sumInl Unit) L₀) * M' * List.prod (List.map (toMatrix ∘ sumInl Unit) L₀') =
diagonal (Sum.elim D₀ fun x => c)
[PROOFSTEP]
rw [this]
[GOAL]
case intro.intro.intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝³ : Field 𝕜
inst✝² : DecidableEq n
inst✝¹ : DecidableEq p
inst✝ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
IH :
∀ (M : Matrix (Fin r) (Fin r) 𝕜),
∃ L₀ L₀' D₀, List.prod (List.map toMatrix L₀) * M * List.prod (List.map toMatrix L₀') = diagonal D₀
M : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
L₁ L₁' : List (TransvectionStruct (Fin r ⊕ Unit) 𝕜)
hM : IsTwoBlockDiagonal (List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁'))
M' : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜 := List.prod (List.map toMatrix L₁) * M * List.prod (List.map toMatrix L₁')
M'' : Matrix (Fin r) (Fin r) 𝕜 := toBlocks₁₁ M'
L₀ L₀' : List (TransvectionStruct (Fin r) 𝕜)
D₀ : Fin r → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * M'' * List.prod (List.map toMatrix L₀') = diagonal D₀
c : 𝕜 := M' (inr ()) (inr ())
this : M' = fromBlocks M'' 0 0 (diagonal fun x => c)
⊢ List.prod (List.map (toMatrix ∘ sumInl Unit) L₀) * fromBlocks M'' 0 0 (diagonal fun x => c) *
List.prod (List.map (toMatrix ∘ sumInl Unit) L₀') =
diagonal (Sum.elim D₀ fun x => c)
[PROOFSTEP]
simp [h₀]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
H : ∃ L L' D, List.prod (List.map toMatrix L) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L') = diagonal D
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
rcases H with ⟨L₀, L₀', D₀, h₀⟩
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
refine' ⟨L₀.map (reindexEquiv e.symm), L₀'.map (reindexEquiv e.symm), D₀ ∘ e, _⟩
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
⊢ List.prod (List.map toMatrix (List.map (reindexEquiv e.symm) L₀)) * M *
List.prod (List.map toMatrix (List.map (reindexEquiv e.symm) L₀')) =
diagonal (D₀ ∘ ↑e)
[PROOFSTEP]
have : M = reindexAlgEquiv 𝕜 e.symm (reindexAlgEquiv 𝕜 e M) := by
simp only [Equiv.symm_symm, submatrix_submatrix, reindex_apply, submatrix_id_id, Equiv.symm_comp_self,
reindexAlgEquiv_apply]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
⊢ M = ↑(reindexAlgEquiv 𝕜 e.symm) (↑(reindexAlgEquiv 𝕜 e) M)
[PROOFSTEP]
simp only [Equiv.symm_symm, submatrix_submatrix, reindex_apply, submatrix_id_id, Equiv.symm_comp_self,
reindexAlgEquiv_apply]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
this : M = ↑(reindexAlgEquiv 𝕜 e.symm) (↑(reindexAlgEquiv 𝕜 e) M)
⊢ List.prod (List.map toMatrix (List.map (reindexEquiv e.symm) L₀)) * M *
List.prod (List.map toMatrix (List.map (reindexEquiv e.symm) L₀')) =
diagonal (D₀ ∘ ↑e)
[PROOFSTEP]
rw [this]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
this : M = ↑(reindexAlgEquiv 𝕜 e.symm) (↑(reindexAlgEquiv 𝕜 e) M)
⊢ List.prod (List.map toMatrix (List.map (reindexEquiv e.symm) L₀)) *
↑(reindexAlgEquiv 𝕜 e.symm) (↑(reindexAlgEquiv 𝕜 e) M) *
List.prod (List.map toMatrix (List.map (reindexEquiv e.symm) L₀')) =
diagonal (D₀ ∘ ↑e)
[PROOFSTEP]
simp only [toMatrix_reindexEquiv_prod, List.map_map, reindexAlgEquiv_apply]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
this : M = ↑(reindexAlgEquiv 𝕜 e.symm) (↑(reindexAlgEquiv 𝕜 e) M)
⊢ ↑(reindex e.symm e.symm) (List.prod (List.map toMatrix L₀)) * ↑(reindex e.symm e.symm) (↑(reindex e e) M) *
↑(reindex e.symm e.symm) (List.prod (List.map toMatrix L₀')) =
diagonal (D₀ ∘ ↑e)
[PROOFSTEP]
simp only [← reindexAlgEquiv_apply, ← reindexAlgEquiv_mul, h₀]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix p p 𝕜
e : p ≃ n
L₀ L₀' : List (TransvectionStruct n 𝕜)
D₀ : n → 𝕜
h₀ : List.prod (List.map toMatrix L₀) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L₀') = diagonal D₀
this : M = ↑(reindexAlgEquiv 𝕜 e.symm) (↑(reindexAlgEquiv 𝕜 e) M)
⊢ ↑(reindexAlgEquiv 𝕜 e.symm) (diagonal D₀) = diagonal (D₀ ∘ ↑e)
[PROOFSTEP]
simp only [Equiv.symm_symm, reindex_apply, submatrix_diagonal_equiv, reindexAlgEquiv_apply]
[GOAL]
n✝ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁷ : Field 𝕜
inst✝⁶ : DecidableEq n✝
inst✝⁵ : DecidableEq p
inst✝⁴ : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝³ : Fintype n✝
inst✝² : Fintype p
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
induction' hn : Fintype.card n with r IH generalizing n M
[GOAL]
case zero
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r : ℕ
M✝¹ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.zero
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
refine' ⟨List.nil, List.nil, fun _ => 1, _⟩
[GOAL]
case zero
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r : ℕ
M✝¹ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.zero
⊢ List.prod (List.map toMatrix []) * M * List.prod (List.map toMatrix []) = diagonal fun x => 1
[PROOFSTEP]
ext i j
[GOAL]
case zero.a.h
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r : ℕ
M✝¹ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.zero
i j : n
⊢ (List.prod (List.map toMatrix []) * M * List.prod (List.map toMatrix [])) i j = diagonal (fun x => 1) i j
[PROOFSTEP]
rw [Fintype.card_eq_zero_iff] at hn
[GOAL]
case zero.a.h
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r : ℕ
M✝¹ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : IsEmpty n
i j : n
⊢ (List.prod (List.map toMatrix []) * M * List.prod (List.map toMatrix [])) i j = diagonal (fun x => 1) i j
[PROOFSTEP]
exact hn.elim' i
[GOAL]
case succ
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
have e : n ≃ Sum (Fin r) Unit := by
refine' Fintype.equivOfCardEq _
rw [hn]
rw [@Fintype.card_sum (Fin r) Unit _ _]
simp
[GOAL]
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
⊢ n ≃ Fin r ⊕ Unit
[PROOFSTEP]
refine' Fintype.equivOfCardEq _
[GOAL]
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
⊢ Fintype.card n = Fintype.card (Fin r ⊕ Unit)
[PROOFSTEP]
rw [hn]
[GOAL]
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
⊢ Nat.succ r = Fintype.card (Fin r ⊕ Unit)
[PROOFSTEP]
rw [@Fintype.card_sum (Fin r) Unit _ _]
[GOAL]
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
⊢ Nat.succ r = Fintype.card (Fin r) + Fintype.card Unit
[PROOFSTEP]
simp
[GOAL]
case succ
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
e : n ≃ Fin r ⊕ Unit
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
apply reindex_exists_list_transvec_mul_mul_list_transvec_eq_diagonal M e
[GOAL]
case succ
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
e : n ≃ Fin r ⊕ Unit
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
apply exists_list_transvec_mul_mul_list_transvec_eq_diagonal_induction fun N => IH (Fin r) N (by simp)
[GOAL]
n✝¹ : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁹ : Field 𝕜
inst✝⁸ : DecidableEq n✝¹
inst✝⁷ : DecidableEq p
inst✝⁶ : CommRing R
r✝ : ℕ
M✝¹ : Matrix (Fin r✝ ⊕ Unit) (Fin r✝ ⊕ Unit) 𝕜
inst✝⁵ : Fintype n✝¹
inst✝⁴ : Fintype p
n✝ : Type
inst✝³ : Fintype n✝
inst✝² : DecidableEq n✝
M✝ : Matrix n✝ n✝ 𝕜
x✝ : ℕ
hn✝ : Fintype.card n✝ = x✝
r : ℕ
IH :
∀ (n : Type) [inst : Fintype n] [inst_1 : DecidableEq n] (M : Matrix n n 𝕜),
Fintype.card n = r → ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
n : Type
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n 𝕜
hn : Fintype.card n = Nat.succ r
e : n ≃ Fin r ⊕ Unit
N : Matrix (Fin r) (Fin r) 𝕜
⊢ Fintype.card (Fin r) = r
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
have e : n ≃ Fin (Fintype.card n) := Fintype.equivOfCardEq (by simp)
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
⊢ Fintype.card n = Fintype.card (Fin (Fintype.card n))
[PROOFSTEP]
simp
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
e : n ≃ Fin (Fintype.card n)
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
apply reindex_exists_list_transvec_mul_mul_list_transvec_eq_diagonal M e
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
e : n ≃ Fin (Fintype.card n)
⊢ ∃ L L' D, List.prod (List.map toMatrix L) * ↑(reindexAlgEquiv 𝕜 e) M * List.prod (List.map toMatrix L') = diagonal D
[PROOFSTEP]
apply exists_list_transvec_mul_mul_list_transvec_eq_diagonal_aux
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
⊢ ∃ L L' D, M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
[PROOFSTEP]
rcases exists_list_transvec_mul_mul_list_transvec_eq_diagonal M with ⟨L, L', D, h⟩
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
⊢ ∃ L L' D, M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
[PROOFSTEP]
refine' ⟨L.reverse.map TransvectionStruct.inv, L'.reverse.map TransvectionStruct.inv, D, _⟩
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
⊢ M =
List.prod (List.map toMatrix (List.map TransvectionStruct.inv (List.reverse L))) * diagonal D *
List.prod (List.map toMatrix (List.map TransvectionStruct.inv (List.reverse L')))
[PROOFSTEP]
suffices
M =
(L.reverse.map (toMatrix ∘ TransvectionStruct.inv)).prod * (L.map toMatrix).prod * M *
((L'.map toMatrix).prod * (L'.reverse.map (toMatrix ∘ TransvectionStruct.inv)).prod)
by simpa [← h, Matrix.mul_assoc]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
this :
M =
List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) * List.prod (List.map toMatrix L) * M *
(List.prod (List.map toMatrix L') * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L')))
⊢ M =
List.prod (List.map toMatrix (List.map TransvectionStruct.inv (List.reverse L))) * diagonal D *
List.prod (List.map toMatrix (List.map TransvectionStruct.inv (List.reverse L')))
[PROOFSTEP]
simpa [← h, Matrix.mul_assoc]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁵ : Field 𝕜
inst✝⁴ : DecidableEq n
inst✝³ : DecidableEq p
inst✝² : CommRing R
r : ℕ
M✝ : Matrix (Fin r ⊕ Unit) (Fin r ⊕ Unit) 𝕜
inst✝¹ : Fintype n
inst✝ : Fintype p
M : Matrix n n 𝕜
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : List.prod (List.map toMatrix L) * M * List.prod (List.map toMatrix L') = diagonal D
⊢ M =
List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L)) * List.prod (List.map toMatrix L) * M *
(List.prod (List.map toMatrix L') * List.prod (List.map (toMatrix ∘ TransvectionStruct.inv) (List.reverse L')))
[PROOFSTEP]
rw [reverse_inv_prod_mul_prod, prod_mul_reverse_inv_prod, Matrix.one_mul, Matrix.mul_one]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
⊢ P M
[PROOFSTEP]
rcases exists_list_transvec_mul_diagonal_mul_list_transvec M with ⟨L, L', D, h⟩
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
⊢ P M
[PROOFSTEP]
have PD : P (diagonal D) := hdiag D (by simp [h])
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
⊢ det (diagonal D) = det M
[PROOFSTEP]
simp [h]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
⊢ P M
[PROOFSTEP]
suffices H :
∀ (L₁ L₂ : List (TransvectionStruct n 𝕜)) (E : Matrix n n 𝕜),
P E → P ((L₁.map toMatrix).prod * E * (L₂.map toMatrix).prod)
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
H :
∀ (L₁ L₂ : List (TransvectionStruct n 𝕜)) (E : Matrix n n 𝕜),
P E → P (List.prod (List.map toMatrix L₁) * E * List.prod (List.map toMatrix L₂))
⊢ P M
[PROOFSTEP]
rw [h]
[GOAL]
case intro.intro.intro
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
H :
∀ (L₁ L₂ : List (TransvectionStruct n 𝕜)) (E : Matrix n n 𝕜),
P E → P (List.prod (List.map toMatrix L₁) * E * List.prod (List.map toMatrix L₂))
⊢ P (List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L'))
[PROOFSTEP]
apply H L L'
[GOAL]
case intro.intro.intro.a
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
H :
∀ (L₁ L₂ : List (TransvectionStruct n 𝕜)) (E : Matrix n n 𝕜),
P E → P (List.prod (List.map toMatrix L₁) * E * List.prod (List.map toMatrix L₂))
⊢ P (diagonal D)
[PROOFSTEP]
exact PD
[GOAL]
case H
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
⊢ ∀ (L₁ L₂ : List (TransvectionStruct n 𝕜)) (E : Matrix n n 𝕜),
P E → P (List.prod (List.map toMatrix L₁) * E * List.prod (List.map toMatrix L₂))
[PROOFSTEP]
intro L₁ L₂ E PE
[GOAL]
case H
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
L₁ L₂ : List (TransvectionStruct n 𝕜)
E : Matrix n n 𝕜
PE : P E
⊢ P (List.prod (List.map toMatrix L₁) * E * List.prod (List.map toMatrix L₂))
[PROOFSTEP]
induction' L₁ with t L₁ IH
[GOAL]
case H.nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
L₂ : List (TransvectionStruct n 𝕜)
E : Matrix n n 𝕜
PE : P E
⊢ P (List.prod (List.map toMatrix []) * E * List.prod (List.map toMatrix L₂))
[PROOFSTEP]
simp only [Matrix.one_mul, List.prod_nil, List.map]
[GOAL]
case H.nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
L₂ : List (TransvectionStruct n 𝕜)
E : Matrix n n 𝕜
PE : P E
⊢ P (E * List.prod (List.map toMatrix L₂))
[PROOFSTEP]
induction' L₂ with t L₂ IH generalizing E
[GOAL]
case H.nil.nil
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
E✝ : Matrix n n 𝕜
PE✝ : P E✝
E : Matrix n n 𝕜
PE : P E
⊢ P (E * List.prod (List.map toMatrix []))
[PROOFSTEP]
simpa
[GOAL]
case H.nil.cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
E✝ : Matrix n n 𝕜
PE✝ : P E✝
t : TransvectionStruct n 𝕜
L₂ : List (TransvectionStruct n 𝕜)
IH : ∀ (E : Matrix n n 𝕜), P E → P (E * List.prod (List.map toMatrix L₂))
E : Matrix n n 𝕜
PE : P E
⊢ P (E * List.prod (List.map toMatrix (t :: L₂)))
[PROOFSTEP]
simp only [← Matrix.mul_assoc, List.prod_cons, List.map]
[GOAL]
case H.nil.cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
E✝ : Matrix n n 𝕜
PE✝ : P E✝
t : TransvectionStruct n 𝕜
L₂ : List (TransvectionStruct n 𝕜)
IH : ∀ (E : Matrix n n 𝕜), P E → P (E * List.prod (List.map toMatrix L₂))
E : Matrix n n 𝕜
PE : P E
⊢ P (E * toMatrix t * List.prod (List.map toMatrix L₂))
[PROOFSTEP]
apply IH
[GOAL]
case H.nil.cons.PE
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
E✝ : Matrix n n 𝕜
PE✝ : P E✝
t : TransvectionStruct n 𝕜
L₂ : List (TransvectionStruct n 𝕜)
IH : ∀ (E : Matrix n n 𝕜), P E → P (E * List.prod (List.map toMatrix L₂))
E : Matrix n n 𝕜
PE : P E
⊢ P (E * toMatrix t)
[PROOFSTEP]
exact hmul _ _ PE (htransvec _)
[GOAL]
case H.cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
L₂ : List (TransvectionStruct n 𝕜)
E : Matrix n n 𝕜
PE : P E
t : TransvectionStruct n 𝕜
L₁ : List (TransvectionStruct n 𝕜)
IH : P (List.prod (List.map toMatrix L₁) * E * List.prod (List.map toMatrix L₂))
⊢ P (List.prod (List.map toMatrix (t :: L₁)) * E * List.prod (List.map toMatrix L₂))
[PROOFSTEP]
simp only [Matrix.mul_assoc, List.prod_cons, List.map] at IH ⊢
[GOAL]
case H.cons
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hdiag : ∀ (D : n → 𝕜), det (diagonal D) = det M → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), P A → P B → P (A * B)
L L' : List (TransvectionStruct n 𝕜)
D : n → 𝕜
h : M = List.prod (List.map toMatrix L) * diagonal D * List.prod (List.map toMatrix L')
PD : P (diagonal D)
L₂ : List (TransvectionStruct n 𝕜)
E : Matrix n n 𝕜
PE : P E
t : TransvectionStruct n 𝕜
L₁ : List (TransvectionStruct n 𝕜)
IH : P (List.prod (List.map toMatrix L₁) * (E * List.prod (List.map toMatrix L₂)))
⊢ P (toMatrix t * (List.prod (List.map toMatrix L₁) * (E * List.prod (List.map toMatrix L₂))))
[PROOFSTEP]
exact hmul _ _ (htransvec _) IH
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
⊢ P M
[PROOFSTEP]
let Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
⊢ P M
[PROOFSTEP]
have : Q M := by
apply diagonal_transvection_induction Q M
· intro D hD
have detD : det (diagonal D) ≠ 0 := by
rw [hD]
exact hMdet
exact ⟨detD, hdiag _ detD⟩
· intro t
exact ⟨by simp, htransvec t⟩
· intro A B QA QB
exact ⟨by simp [QA.1, QB.1], hmul A B QA.1 QB.1 QA.2 QB.2⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
⊢ Q M
[PROOFSTEP]
apply diagonal_transvection_induction Q M
[GOAL]
case hdiag
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
⊢ ∀ (D : n → 𝕜), det (diagonal D) = det M → Q (diagonal D)
[PROOFSTEP]
intro D hD
[GOAL]
case hdiag
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
D : n → 𝕜
hD : det (diagonal D) = det M
⊢ Q (diagonal D)
[PROOFSTEP]
have detD : det (diagonal D) ≠ 0 := by
rw [hD]
exact hMdet
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
D : n → 𝕜
hD : det (diagonal D) = det M
⊢ det (diagonal D) ≠ 0
[PROOFSTEP]
rw [hD]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
D : n → 𝕜
hD : det (diagonal D) = det M
⊢ det M ≠ 0
[PROOFSTEP]
exact hMdet
[GOAL]
case hdiag
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
D : n → 𝕜
hD : det (diagonal D) = det M
detD : det (diagonal D) ≠ 0
⊢ Q (diagonal D)
[PROOFSTEP]
exact ⟨detD, hdiag _ detD⟩
[GOAL]
case htransvec
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
⊢ ∀ (t : TransvectionStruct n 𝕜), Q (toMatrix t)
[PROOFSTEP]
intro t
[GOAL]
case htransvec
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
t : TransvectionStruct n 𝕜
⊢ Q (toMatrix t)
[PROOFSTEP]
exact ⟨by simp, htransvec t⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
t : TransvectionStruct n 𝕜
⊢ det (toMatrix t) ≠ 0
[PROOFSTEP]
simp
[GOAL]
case hmul
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
⊢ ∀ (A B : Matrix n n 𝕜), Q A → Q B → Q (A * B)
[PROOFSTEP]
intro A B QA QB
[GOAL]
case hmul
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
A B : Matrix n n 𝕜
QA : Q A
QB : Q B
⊢ Q (A * B)
[PROOFSTEP]
exact ⟨by simp [QA.1, QB.1], hmul A B QA.1 QB.1 QA.2 QB.2⟩
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
A B : Matrix n n 𝕜
QA : Q A
QB : Q B
⊢ det (A * B) ≠ 0
[PROOFSTEP]
simp [QA.1, QB.1]
[GOAL]
n : Type u_1
p : Type u_2
R : Type u₂
𝕜 : Type u_3
inst✝⁴ : Field 𝕜
inst✝³ : DecidableEq n
inst✝² : DecidableEq p
inst✝¹ : CommRing R
inst✝ : Fintype n
P : Matrix n n 𝕜 → Prop
M : Matrix n n 𝕜
hMdet : det M ≠ 0
hdiag : ∀ (D : n → 𝕜), det (diagonal D) ≠ 0 → P (diagonal D)
htransvec : ∀ (t : TransvectionStruct n 𝕜), P (toMatrix t)
hmul : ∀ (A B : Matrix n n 𝕜), det A ≠ 0 → det B ≠ 0 → P A → P B → P (A * B)
Q : Matrix n n 𝕜 → Prop := fun N => det N ≠ 0 ∧ P N
this : Q M
⊢ P M
[PROOFSTEP]
exact this.2
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Transvection", "llama_tokens": 91700} |
[GOAL]
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
cases (isEmpty_or_nonempty n).symm
[GOAL]
case inl
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
cases' CharP.exists K with p hp
[GOAL]
case inl.intro
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp : CharP K p
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
letI := hp
[GOAL]
case inl.intro
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp : CharP K p
this : CharP K p := hp
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
rcases FiniteField.card K p with ⟨⟨k, kpos⟩, ⟨hp, hk⟩⟩
[GOAL]
case inl.intro.intro.mk.intro
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ ↑{ val := k, property := kpos }
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
haveI : Fact p.Prime := ⟨hp⟩
[GOAL]
case inl.intro.intro.mk.intro
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ ↑{ val := k, property := kpos }
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
dsimp at hk
[GOAL]
case inl.intro.intro.mk.intro
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
rw [hk]
[GOAL]
case inl.intro.intro.mk.intro
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ p ^ k) = charpoly M
[PROOFSTEP]
apply (frobenius_inj K[X] p).iterate k
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ (↑(frobenius K[X] p))^[k] (charpoly (M ^ p ^ k)) = (↑(frobenius K[X] p))^[k] (charpoly M)
[PROOFSTEP]
repeat' rw [iterate_frobenius (R := K[X])]; rw [← hk]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ (↑(frobenius K[X] p))^[k] (charpoly (M ^ p ^ k)) = (↑(frobenius K[X] p))^[k] (charpoly M)
[PROOFSTEP]
rw [iterate_frobenius (R := K[X])]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ p ^ k) ^ p ^ k = (↑(frobenius K[X] p))^[k] (charpoly M)
[PROOFSTEP]
rw [← hk]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ Fintype.card K) ^ Fintype.card K = (↑(frobenius K[X] p))^[k] (charpoly M)
[PROOFSTEP]
rw [iterate_frobenius (R := K[X])]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ Fintype.card K) ^ Fintype.card K = charpoly M ^ p ^ k
[PROOFSTEP]
rw [← hk]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ Fintype.card K) ^ Fintype.card K = charpoly M ^ Fintype.card K
[PROOFSTEP]
rw [iterate_frobenius (R := K[X])]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ charpoly (M ^ Fintype.card K) ^ Fintype.card K = charpoly M ^ Fintype.card K
[PROOFSTEP]
rw [← FiniteField.expand_card]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ ↑(expand K (Fintype.card K)) (charpoly (M ^ Fintype.card K)) = charpoly M ^ Fintype.card K
[PROOFSTEP]
unfold charpoly
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ ↑(expand K (Fintype.card K)) (det (charmatrix (M ^ Fintype.card K))) = det (charmatrix M) ^ Fintype.card K
[PROOFSTEP]
rw [AlgHom.map_det, ← coe_detMonoidHom, ← (detMonoidHom : Matrix n n K[X] →* K[X]).map_pow]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ ↑detMonoidHom (↑(AlgHom.mapMatrix (expand K (Fintype.card K))) (charmatrix (M ^ Fintype.card K))) =
↑detMonoidHom (charmatrix M ^ Fintype.card K)
[PROOFSTEP]
apply congr_arg det
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ ↑(AlgHom.mapMatrix (expand K (Fintype.card K))) (charmatrix (M ^ Fintype.card K)) = charmatrix M ^ Fintype.card K
[PROOFSTEP]
refine' matPolyEquiv.injective _
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ ↑matPolyEquiv (↑(AlgHom.mapMatrix (expand K (Fintype.card K))) (charmatrix (M ^ Fintype.card K))) =
↑matPolyEquiv (charmatrix M ^ Fintype.card K)
[PROOFSTEP]
rw [AlgEquiv.map_pow, matPolyEquiv_charmatrix, hk, sub_pow_char_pow_of_commute, ← C_pow]
[GOAL]
case inl.intro.intro.mk.intro.a
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ ↑matPolyEquiv (↑(AlgHom.mapMatrix (expand K (p ^ k))) (charmatrix (M ^ p ^ k))) = X ^ p ^ k - ↑C (M ^ p ^ k)
[PROOFSTEP]
exact (id (matPolyEquiv_eq_x_pow_sub_c (p ^ k) M) : _)
[GOAL]
case inl.intro.intro.mk.intro.a.h
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
p : ℕ
hp✝ : CharP K p
this✝ : CharP K p := hp✝
k : ℕ
kpos : 0 < k
hp : Nat.Prime p
hk : Fintype.card K = p ^ k
this : Fact (Nat.Prime p)
⊢ Commute X (↑C M)
[PROOFSTEP]
exact (C M).commute_X
[GOAL]
case inr
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : IsEmpty n
⊢ charpoly (M ^ Fintype.card K) = charpoly M
[PROOFSTEP]
exact congr_arg _ (Subsingleton.elim _ _)
[GOAL]
n : Type u_1
inst✝² : DecidableEq n
inst✝¹ : Fintype n
p : ℕ
inst✝ : Fact (Nat.Prime p)
M : Matrix n n (ZMod p)
⊢ charpoly (M ^ p) = charpoly M
[PROOFSTEP]
have h := FiniteField.Matrix.charpoly_pow_card M
[GOAL]
n : Type u_1
inst✝² : DecidableEq n
inst✝¹ : Fintype n
p : ℕ
inst✝ : Fact (Nat.Prime p)
M : Matrix n n (ZMod p)
h : charpoly (M ^ Fintype.card (ZMod p)) = charpoly M
⊢ charpoly (M ^ p) = charpoly M
[PROOFSTEP]
rwa [ZMod.card] at h
[GOAL]
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
⊢ trace (M ^ Fintype.card K) = trace M ^ Fintype.card K
[PROOFSTEP]
cases isEmpty_or_nonempty n
[GOAL]
case inl
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : IsEmpty n
⊢ trace (M ^ Fintype.card K) = trace M ^ Fintype.card K
[PROOFSTEP]
simp [Matrix.trace]
[GOAL]
case inl
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : IsEmpty n
⊢ 0 = 0 ^ Fintype.card K
[PROOFSTEP]
rw [zero_pow Fintype.card_pos]
[GOAL]
case inr
n : Type u_1
inst✝³ : DecidableEq n
inst✝² : Fintype n
K : Type u_2
inst✝¹ : Field K
inst✝ : Fintype K
M : Matrix n n K
h✝ : Nonempty n
⊢ trace (M ^ Fintype.card K) = trace M ^ Fintype.card K
[PROOFSTEP]
rw [Matrix.trace_eq_neg_charpoly_coeff, Matrix.trace_eq_neg_charpoly_coeff, FiniteField.Matrix.charpoly_pow_card,
FiniteField.pow_card]
[GOAL]
n : Type u_1
inst✝² : DecidableEq n
inst✝¹ : Fintype n
p : ℕ
inst✝ : Fact (Nat.Prime p)
M : Matrix n n (ZMod p)
⊢ trace (M ^ p) = trace M ^ p
[PROOFSTEP]
have h := FiniteField.trace_pow_card M
[GOAL]
n : Type u_1
inst✝² : DecidableEq n
inst✝¹ : Fintype n
p : ℕ
inst✝ : Fact (Nat.Prime p)
M : Matrix n n (ZMod p)
h : trace (M ^ Fintype.card (ZMod p)) = trace M ^ Fintype.card (ZMod p)
⊢ trace (M ^ p) = trace M ^ p
[PROOFSTEP]
rwa [ZMod.card] at h
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Charpoly.FiniteField", "llama_tokens": 5748} |
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁷ : CommSemiring R
inst✝⁶ : AddCommMonoid M
inst✝⁵ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁴ : CommRing R₂
inst✝³ : AddCommGroup M₂
inst✝² : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
inst✝¹ : Fintype ι
inst✝ : DecidableEq ι
v : ι → M
⊢ toMatrix e v = ↑(LinearMap.toMatrix e e) (↑(constr e ℕ) v)
[PROOFSTEP]
ext
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁷ : CommSemiring R
inst✝⁶ : AddCommMonoid M
inst✝⁵ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁴ : CommRing R₂
inst✝³ : AddCommGroup M₂
inst✝² : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
inst✝¹ : Fintype ι
inst✝ : DecidableEq ι
v : ι → M
i✝ x✝ : ι
⊢ toMatrix e v i✝ x✝ = ↑(LinearMap.toMatrix e e) (↑(constr e ℕ) v) i✝ x✝
[PROOFSTEP]
rw [Basis.toMatrix_apply, LinearMap.toMatrix_apply, Basis.constr_basis]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
⊢ toMatrix (Pi.basisFun R ι) = transpose
[PROOFSTEP]
ext M i j
[GOAL]
case h.a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M✝ : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M✝
inst✝⁴ : Module R M✝
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M✝
v : ι' → M✝
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
M : ι → ι → R
i j : ι
⊢ toMatrix (Pi.basisFun R ι) M i j = Mᵀ i j
[PROOFSTEP]
rfl
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι
⊢ toMatrix e ↑e = 1
[PROOFSTEP]
unfold Basis.toMatrix
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι
⊢ (fun i j => ↑(↑e.repr (↑e j)) i) = 1
[PROOFSTEP]
ext i j
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : DecidableEq ι
i j : ι
⊢ ↑(↑e.repr (↑e j)) i = OfNat.ofNat 1 i j
[PROOFSTEP]
simp [Basis.equivFun, Matrix.one_apply, Finsupp.single_apply, eq_comm]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι'
x : M
⊢ toMatrix e (update v j x) = updateColumn (toMatrix e v) j ↑(↑e.repr x)
[PROOFSTEP]
ext i' k
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι'
x : M
i' : ι
k : ι'
⊢ toMatrix e (update v j x) i' k = updateColumn (toMatrix e v) j (↑(↑e.repr x)) i' k
[PROOFSTEP]
rw [Basis.toMatrix, Matrix.updateColumn_apply, e.toMatrix_apply]
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι'
x : M
i' : ι
k : ι'
⊢ ↑(↑e.repr (update v j x k)) i' = if k = j then ↑(↑e.repr x) i' else ↑(↑e.repr (v k)) i'
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι'
x : M
i' : ι
k : ι'
h : k = j
⊢ ↑(↑e.repr (update v j x k)) i' = ↑(↑e.repr x) i'
[PROOFSTEP]
rw [h, update_same j x v]
[GOAL]
case neg
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι'
x : M
i' : ι
k : ι'
h : ¬k = j
⊢ ↑(↑e.repr (update v j x k)) i' = ↑(↑e.repr (v k)) i'
[PROOFSTEP]
rw [update_noteq h]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : DecidableEq ι
e : Basis ι R₂ M₂
w : ι → R₂ˣ
⊢ toMatrix e ↑(unitsSMul e w) = Matrix.diagonal (Units.val ∘ w)
[PROOFSTEP]
ext i j
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : DecidableEq ι
e : Basis ι R₂ M₂
w : ι → R₂ˣ
i j : ι
⊢ toMatrix e (↑(unitsSMul e w)) i j = Matrix.diagonal (Units.val ∘ w) i j
[PROOFSTEP]
by_cases h : i = j
[GOAL]
case pos
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : DecidableEq ι
e : Basis ι R₂ M₂
w : ι → R₂ˣ
i j : ι
h : i = j
⊢ toMatrix e (↑(unitsSMul e w)) i j = Matrix.diagonal (Units.val ∘ w) i j
[PROOFSTEP]
simp [h, toMatrix_apply, unitsSMul_apply, Units.smul_def]
[GOAL]
case neg
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : DecidableEq ι
e : Basis ι R₂ M₂
w : ι → R₂ˣ
i j : ι
h : ¬i = j
⊢ toMatrix e (↑(unitsSMul e w)) i j = Matrix.diagonal (Units.val ∘ w) i j
[PROOFSTEP]
simp [h, toMatrix_apply, unitsSMul_apply, Units.smul_def, Ne.symm h]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
⊢ ∑ i : ι, toMatrix e v i j • ↑e i = v j
[PROOFSTEP]
simp_rw [e.toMatrix_apply, e.sum_repr]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
S : Type u_9
inst✝² : Ring S
inst✝¹ : Algebra R S
inst✝ : Fintype ι
b : Basis ι R S
v : ι' → S
⊢ vecMul (↑b) (Matrix.map (toMatrix b v) ↑(algebraMap R S)) = v
[PROOFSTEP]
ext i
[GOAL]
case h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i✝ : ι
j : ι'
S : Type u_9
inst✝² : Ring S
inst✝¹ : Algebra R S
inst✝ : Fintype ι
b : Basis ι R S
v : ι' → S
i : ι'
⊢ vecMul (↑b) (Matrix.map (toMatrix b v) ↑(algebraMap R S)) i = v i
[PROOFSTEP]
simp_rw [vecMul, dotProduct, Matrix.map_apply, ← Algebra.commutes, ← Algebra.smul_def, sum_toMatrix_smul_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i✝ : ι
j : ι'
inst✝² : Fintype ι
inst✝¹ : Fintype ι'
inst✝ : DecidableEq ι'
v : Basis ι' R M
i : ι'
⊢ ↑(↑(toLin v e) (toMatrix e ↑v)) (↑v i) = ↑LinearMap.id (↑v i)
[PROOFSTEP]
rw [toLin_self, id_apply, e.sum_toMatrix_smul_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
v w : ι → M
⊢ toMatrix e (v + w) = toMatrix e v + toMatrix e w
[PROOFSTEP]
ext i j
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
v w : ι → M
i j : ι
⊢ toMatrix e (v + w) i j = (toMatrix e v + toMatrix e w) i j
[PROOFSTEP]
change _ = _ + _
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
v w : ι → M
i j : ι
⊢ toMatrix e (v + w) i j = toMatrix e v i j + toMatrix e w i j
[PROOFSTEP]
rw [e.toMatrix_apply, Pi.add_apply, LinearEquiv.map_add]
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
v w : ι → M
i j : ι
⊢ ↑(↑e.repr (v j) + ↑e.repr (w j)) i = toMatrix e v i j + toMatrix e w i j
[PROOFSTEP]
rfl
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
⊢ ∀ (r : R) (x : ι → M),
AddHom.toFun
{ toFun := toMatrix e, map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := toMatrix e, map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) } x
[PROOFSTEP]
intro c v
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
c : R
v : ι → M
⊢ AddHom.toFun
{ toFun := toMatrix e, map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e, map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) } v
[PROOFSTEP]
ext i j
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
c : R
v : ι → M
i j : ι
⊢ AddHom.toFun
{ toFun := toMatrix e, map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) i j =
(↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e, map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v)
i j
[PROOFSTEP]
dsimp only []
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
c : R
v : ι → M
i j : ι
⊢ toMatrix e (c • v) i j = (↑(RingHom.id R) c • toMatrix e v) i j
[PROOFSTEP]
rw [e.toMatrix_apply, Pi.smul_apply, LinearEquiv.map_smul]
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i✝ : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
c : R
v : ι → M
i j : ι
⊢ ↑(c • ↑e.repr (v j)) i = (↑(RingHom.id R) c • toMatrix e v) i j
[PROOFSTEP]
rfl
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
⊢ LeftInverse (fun m j => ∑ i : ι, m i j • ↑e i)
{
toAddHom :=
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) },
map_smul' :=
(_ :
∀ (c : R) (v : ι → M),
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v) }.toAddHom.toFun
[PROOFSTEP]
intro v
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
v : ι → M
⊢ (fun m j => ∑ i : ι, m i j • ↑e i)
(AddHom.toFun
{
toAddHom :=
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) },
map_smul' :=
(_ :
∀ (c : R) (v : ι → M),
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v) }.toAddHom
v) =
v
[PROOFSTEP]
ext j
[GOAL]
case h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j✝ : ι'
inst✝ : Fintype ι
e : Basis ι R M
v : ι → M
j : ι
⊢ (fun m j => ∑ i : ι, m i j • ↑e i)
(AddHom.toFun
{
toAddHom :=
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) },
map_smul' :=
(_ :
∀ (c : R) (v : ι → M),
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v) }.toAddHom
v)
j =
v j
[PROOFSTEP]
exact e.sum_toMatrix_smul_self v j
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
⊢ Function.RightInverse (fun m j => ∑ i : ι, m i j • ↑e i)
{
toAddHom :=
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) },
map_smul' :=
(_ :
∀ (c : R) (v : ι → M),
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v) }.toAddHom.toFun
[PROOFSTEP]
intro m
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
m : Matrix ι ι R
⊢ AddHom.toFun
{
toAddHom :=
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) },
map_smul' :=
(_ :
∀ (c : R) (v : ι → M),
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v) }.toAddHom
((fun m j => ∑ i : ι, m i j • ↑e i) m) =
m
[PROOFSTEP]
ext k l
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁶ : CommSemiring R
inst✝⁵ : AddCommMonoid M
inst✝⁴ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝³ : CommRing R₂
inst✝² : AddCommGroup M₂
inst✝¹ : Module R₂ M₂
e✝ : Basis ι R M
v : ι' → M
i : ι
j : ι'
inst✝ : Fintype ι
e : Basis ι R M
m : Matrix ι ι R
k l : ι
⊢ AddHom.toFun
{
toAddHom :=
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) },
map_smul' :=
(_ :
∀ (c : R) (v : ι → M),
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun
{ toFun := toMatrix e,
map_add' := (_ : ∀ (v w : ι → M), toMatrix e (v + w) = toMatrix e v + toMatrix e w) }
v) }.toAddHom
((fun m j => ∑ i : ι, m i j • ↑e i) m) k l =
m k l
[PROOFSTEP]
simp only [e.toMatrix_apply, ← e.equivFun_apply, ← e.equivFun_symm_apply, LinearEquiv.apply_symm_apply]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹¹ : CommSemiring R
inst✝¹⁰ : AddCommMonoid M
inst✝⁹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁸ : CommRing R₂
inst✝⁷ : AddCommGroup M₂
inst✝⁶ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁵ : AddCommMonoid N
inst✝⁴ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝³ : Fintype ι'
inst✝² : Fintype κ
inst✝¹ : Fintype κ'
inst✝ : DecidableEq ι'
⊢ ↑(toLin b' c) (Basis.toMatrix c ↑c' * ↑(toMatrix b' c') f) = ↑(toLin b' c) (↑(toMatrix b' c) f)
[PROOFSTEP]
haveI := Classical.decEq κ'
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹¹ : CommSemiring R
inst✝¹⁰ : AddCommMonoid M
inst✝⁹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁸ : CommRing R₂
inst✝⁷ : AddCommGroup M₂
inst✝⁶ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁵ : AddCommMonoid N
inst✝⁴ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝³ : Fintype ι'
inst✝² : Fintype κ
inst✝¹ : Fintype κ'
inst✝ : DecidableEq ι'
this : DecidableEq κ'
⊢ ↑(toLin b' c) (Basis.toMatrix c ↑c' * ↑(toMatrix b' c') f) = ↑(toLin b' c) (↑(toMatrix b' c) f)
[PROOFSTEP]
rw [toLin_toMatrix, toLin_mul b' c' c, toLin_toMatrix, c.toLin_toMatrix, id_comp]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹³ : CommSemiring R
inst✝¹² : AddCommMonoid M
inst✝¹¹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝¹⁰ : CommRing R₂
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁷ : AddCommMonoid N
inst✝⁶ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁵ : Fintype ι'
inst✝⁴ : Fintype κ
inst✝³ : Fintype κ'
inst✝² : Fintype ι
inst✝¹ : DecidableEq ι
inst✝ : DecidableEq ι'
⊢ ↑(toLin b c') (↑(toMatrix b' c') f * Basis.toMatrix b' ↑b) = ↑(toLin b c') (↑(toMatrix b c') f)
[PROOFSTEP]
rw [toLin_toMatrix, toLin_mul b b' c', toLin_toMatrix, b'.toLin_toMatrix, comp_id]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹³ : CommSemiring R
inst✝¹² : AddCommMonoid M
inst✝¹¹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝¹⁰ : CommRing R₂
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁷ : AddCommMonoid N
inst✝⁶ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁵ : Fintype ι'
inst✝⁴ : Fintype κ
inst✝³ : Fintype κ'
inst✝² : Fintype ι
inst✝¹ : DecidableEq ι
inst✝ : DecidableEq ι'
⊢ Basis.toMatrix c ↑c' * ↑(toMatrix b' c') f * Basis.toMatrix b' ↑b = ↑(toMatrix b c) f
[PROOFSTEP]
rw [basis_toMatrix_mul_linearMap_toMatrix, linearMap_toMatrix_mul_basis_toMatrix]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹² : CommSemiring R
inst✝¹¹ : AddCommMonoid M
inst✝¹⁰ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁹ : CommRing R₂
inst✝⁸ : AddCommGroup M₂
inst✝⁷ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁶ : AddCommMonoid N
inst✝⁵ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁴ : Fintype ι'
inst✝³ : Fintype κ
inst✝² : Fintype κ'
inst✝¹ : Fintype ι
inst✝ : DecidableEq κ
b₁ : Basis ι R M
b₂ : Basis ι' R M
b₃ : Basis κ R N
A : Matrix ι' κ R
⊢ Basis.toMatrix b₁ ↑b₂ * A = ↑(toMatrix b₃ b₁) (↑(toLin b₃ b₂) A)
[PROOFSTEP]
have := basis_toMatrix_mul_linearMap_toMatrix b₃ b₁ b₂ (Matrix.toLin b₃ b₂ A)
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹² : CommSemiring R
inst✝¹¹ : AddCommMonoid M
inst✝¹⁰ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁹ : CommRing R₂
inst✝⁸ : AddCommGroup M₂
inst✝⁷ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁶ : AddCommMonoid N
inst✝⁵ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁴ : Fintype ι'
inst✝³ : Fintype κ
inst✝² : Fintype κ'
inst✝¹ : Fintype ι
inst✝ : DecidableEq κ
b₁ : Basis ι R M
b₂ : Basis ι' R M
b₃ : Basis κ R N
A : Matrix ι' κ R
this : Basis.toMatrix b₁ ↑b₂ * ↑(toMatrix b₃ b₂) (↑(toLin b₃ b₂) A) = ↑(toMatrix b₃ b₁) (↑(toLin b₃ b₂) A)
⊢ Basis.toMatrix b₁ ↑b₂ * A = ↑(toMatrix b₃ b₁) (↑(toLin b₃ b₂) A)
[PROOFSTEP]
rwa [LinearMap.toMatrix_toLin] at this
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹³ : CommSemiring R
inst✝¹² : AddCommMonoid M
inst✝¹¹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝¹⁰ : CommRing R₂
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁷ : AddCommMonoid N
inst✝⁶ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁵ : Fintype ι'
inst✝⁴ : Fintype κ
inst✝³ : Fintype κ'
inst✝² : Fintype ι
inst✝¹ : DecidableEq ι
inst✝ : DecidableEq ι'
b₁ : Basis ι R M
b₂ : Basis ι' R M
b₃ : Basis κ R N
A : Matrix κ ι R
⊢ A * Basis.toMatrix b₁ ↑b₂ = ↑(toMatrix b₂ b₃) (↑(toLin b₁ b₃) A)
[PROOFSTEP]
have := linearMap_toMatrix_mul_basis_toMatrix b₂ b₁ b₃ (Matrix.toLin b₁ b₃ A)
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹³ : CommSemiring R
inst✝¹² : AddCommMonoid M
inst✝¹¹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝¹⁰ : CommRing R₂
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁷ : AddCommMonoid N
inst✝⁶ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁵ : Fintype ι'
inst✝⁴ : Fintype κ
inst✝³ : Fintype κ'
inst✝² : Fintype ι
inst✝¹ : DecidableEq ι
inst✝ : DecidableEq ι'
b₁ : Basis ι R M
b₂ : Basis ι' R M
b₃ : Basis κ R N
A : Matrix κ ι R
this : ↑(toMatrix b₁ b₃) (↑(toLin b₁ b₃) A) * Basis.toMatrix b₁ ↑b₂ = ↑(toMatrix b₂ b₃) (↑(toLin b₁ b₃) A)
⊢ A * Basis.toMatrix b₁ ↑b₂ = ↑(toMatrix b₂ b₃) (↑(toLin b₁ b₃) A)
[PROOFSTEP]
rwa [LinearMap.toMatrix_toLin] at this
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹¹ : CommSemiring R
inst✝¹⁰ : AddCommMonoid M
inst✝⁹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁸ : CommRing R₂
inst✝⁷ : AddCommGroup M₂
inst✝⁶ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁵ : AddCommMonoid N
inst✝⁴ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝³ : Fintype ι'
inst✝² : Fintype κ
inst✝¹ : Fintype κ'
inst✝ : Fintype ι
b : Basis ι R (ι → R)
A : Matrix ι ι R
⊢ Basis.toMatrix b ↑(Pi.basisFun R ι) * A = ↑of fun i j => ↑(↑b.repr (Aᵀ j)) i
[PROOFSTEP]
classical
simp only [basis_toMatrix_mul _ _ (Pi.basisFun R ι), Matrix.toLin_eq_toLin']
ext i j
rw [LinearMap.toMatrix_apply, Matrix.toLin'_apply, Pi.basisFun_apply, Matrix.mulVec_stdBasis_apply, Matrix.of_apply]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹¹ : CommSemiring R
inst✝¹⁰ : AddCommMonoid M
inst✝⁹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁸ : CommRing R₂
inst✝⁷ : AddCommGroup M₂
inst✝⁶ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁵ : AddCommMonoid N
inst✝⁴ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝³ : Fintype ι'
inst✝² : Fintype κ
inst✝¹ : Fintype κ'
inst✝ : Fintype ι
b : Basis ι R (ι → R)
A : Matrix ι ι R
⊢ Basis.toMatrix b ↑(Pi.basisFun R ι) * A = ↑of fun i j => ↑(↑b.repr (Aᵀ j)) i
[PROOFSTEP]
simp only [basis_toMatrix_mul _ _ (Pi.basisFun R ι), Matrix.toLin_eq_toLin']
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹¹ : CommSemiring R
inst✝¹⁰ : AddCommMonoid M
inst✝⁹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁸ : CommRing R₂
inst✝⁷ : AddCommGroup M₂
inst✝⁶ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁵ : AddCommMonoid N
inst✝⁴ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝³ : Fintype ι'
inst✝² : Fintype κ
inst✝¹ : Fintype κ'
inst✝ : Fintype ι
b : Basis ι R (ι → R)
A : Matrix ι ι R
⊢ ↑(toMatrix (Pi.basisFun R ι) b) (↑toLin' A) = ↑of fun i j => ↑(↑b.repr (Aᵀ j)) i
[PROOFSTEP]
ext i j
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹¹ : CommSemiring R
inst✝¹⁰ : AddCommMonoid M
inst✝⁹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁸ : CommRing R₂
inst✝⁷ : AddCommGroup M₂
inst✝⁶ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i✝ : ι
j✝ : ι'
N : Type u_9
inst✝⁵ : AddCommMonoid N
inst✝⁴ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝³ : Fintype ι'
inst✝² : Fintype κ
inst✝¹ : Fintype κ'
inst✝ : Fintype ι
b : Basis ι R (ι → R)
A : Matrix ι ι R
i j : ι
⊢ ↑(toMatrix (Pi.basisFun R ι) b) (↑toLin' A) i j = ↑of (fun i j => ↑(↑b.repr (Aᵀ j)) i) i j
[PROOFSTEP]
rw [LinearMap.toMatrix_apply, Matrix.toLin'_apply, Pi.basisFun_apply, Matrix.mulVec_stdBasis_apply, Matrix.of_apply]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹² : CommSemiring R
inst✝¹¹ : AddCommMonoid M
inst✝¹⁰ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁹ : CommRing R₂
inst✝⁸ : AddCommGroup M₂
inst✝⁷ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁶ : AddCommMonoid N
inst✝⁵ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁴ : Fintype ι'
inst✝³ : Fintype κ
inst✝² : Fintype κ'
inst✝¹ : Fintype ι
inst✝ : DecidableEq ι
⊢ ↑(toMatrix b b') id = Basis.toMatrix b' ↑b
[PROOFSTEP]
haveI := Classical.decEq ι'
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹² : CommSemiring R
inst✝¹¹ : AddCommMonoid M
inst✝¹⁰ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁹ : CommRing R₂
inst✝⁸ : AddCommGroup M₂
inst✝⁷ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁶ : AddCommMonoid N
inst✝⁵ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁴ : Fintype ι'
inst✝³ : Fintype κ
inst✝² : Fintype κ'
inst✝¹ : Fintype ι
inst✝ : DecidableEq ι
this : DecidableEq ι'
⊢ ↑(toMatrix b b') id = Basis.toMatrix b' ↑b
[PROOFSTEP]
rw [← @basis_toMatrix_mul_linearMap_toMatrix _ _ ι, toMatrix_id, Matrix.mul_one]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹³ : CommSemiring R
inst✝¹² : AddCommMonoid M
inst✝¹¹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝¹⁰ : CommRing R₂
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁷ : AddCommMonoid N
inst✝⁶ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁵ : Fintype ι'
inst✝⁴ : Fintype κ
inst✝³ : Fintype κ'
inst✝² : Fintype ι
inst✝¹ : DecidableEq ι
inst✝ : DecidableEq ι'
b : Basis ι R M
v : ι' → M
e : ι ≃ ι'
⊢ toMatrix (reindex b e) v = ↑(reindexAlgEquiv R e) (toMatrix b (v ∘ ↑e))
[PROOFSTEP]
ext
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝¹³ : CommSemiring R
inst✝¹² : AddCommMonoid M
inst✝¹¹ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝¹⁰ : CommRing R₂
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝⁷ : AddCommMonoid N
inst✝⁶ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝⁵ : Fintype ι'
inst✝⁴ : Fintype κ
inst✝³ : Fintype κ'
inst✝² : Fintype ι
inst✝¹ : DecidableEq ι
inst✝ : DecidableEq ι'
b : Basis ι R M
v : ι' → M
e : ι ≃ ι'
i✝ x✝ : ι'
⊢ toMatrix (reindex b e) v i✝ x✝ = ↑(reindexAlgEquiv R e) (toMatrix b (v ∘ ↑e)) i✝ x✝
[PROOFSTEP]
simp only [Basis.toMatrix_apply, Basis.repr_reindex, Matrix.reindexAlgEquiv_apply, Matrix.reindex_apply,
Matrix.submatrix_apply, Function.comp_apply, e.apply_symm_apply, Finsupp.mapDomain_equiv_apply]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝² : AddCommMonoid N
inst✝¹ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
ι'' : Type u_10
inst✝ : Fintype ι'
b'' : ι'' → M
⊢ toMatrix b ↑b' * toMatrix b' b'' = toMatrix b b''
[PROOFSTEP]
haveI := Classical.decEq ι
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝² : AddCommMonoid N
inst✝¹ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
ι'' : Type u_10
inst✝ : Fintype ι'
b'' : ι'' → M
this : DecidableEq ι
⊢ toMatrix b ↑b' * toMatrix b' b'' = toMatrix b b''
[PROOFSTEP]
haveI := Classical.decEq ι'
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝² : AddCommMonoid N
inst✝¹ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
ι'' : Type u_10
inst✝ : Fintype ι'
b'' : ι'' → M
this✝ : DecidableEq ι
this : DecidableEq ι'
⊢ toMatrix b ↑b' * toMatrix b' b'' = toMatrix b b''
[PROOFSTEP]
haveI := Classical.decEq ι''
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝² : AddCommMonoid N
inst✝¹ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
ι'' : Type u_10
inst✝ : Fintype ι'
b'' : ι'' → M
this✝¹ : DecidableEq ι
this✝ : DecidableEq ι'
this : DecidableEq ι''
⊢ toMatrix b ↑b' * toMatrix b' b'' = toMatrix b b''
[PROOFSTEP]
ext i j
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁸ : CommSemiring R
inst✝⁷ : AddCommMonoid M
inst✝⁶ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁵ : CommRing R₂
inst✝⁴ : AddCommGroup M₂
inst✝³ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i✝ : ι
j✝ : ι'
N : Type u_9
inst✝² : AddCommMonoid N
inst✝¹ : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
ι'' : Type u_10
inst✝ : Fintype ι'
b'' : ι'' → M
this✝¹ : DecidableEq ι
this✝ : DecidableEq ι'
this : DecidableEq ι''
i : ι
j : ι''
⊢ (toMatrix b ↑b' * toMatrix b' b'') i j = toMatrix b b'' i j
[PROOFSTEP]
simp only [Matrix.mul_apply, Basis.toMatrix_apply, Basis.sum_repr_mul_repr]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁹ : CommSemiring R
inst✝⁸ : AddCommMonoid M
inst✝⁷ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁶ : CommRing R₂
inst✝⁵ : AddCommGroup M₂
inst✝⁴ : Module R₂ M₂
e : Basis ι R M
v : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝³ : AddCommMonoid N
inst✝² : Module R N
b : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
inst✝¹ : DecidableEq ι
inst✝ : Fintype ι'
⊢ toMatrix b ↑b' * toMatrix b' ↑b = 1
[PROOFSTEP]
rw [Basis.toMatrix_mul_toMatrix, Basis.toMatrix_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁷ : CommSemiring R
inst✝⁶ : AddCommMonoid M
inst✝⁵ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁴ : CommRing R₂
inst✝³ : AddCommGroup M₂
inst✝² : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝¹ : AddCommMonoid N
inst✝ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
b : Basis ι R M
v : ι' → M
e : ι ≃ ι'
⊢ toMatrix (reindex b e) v = submatrix (toMatrix b v) (↑e.symm) _root_.id
[PROOFSTEP]
ext
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁷ : CommSemiring R
inst✝⁶ : AddCommMonoid M
inst✝⁵ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁴ : CommRing R₂
inst✝³ : AddCommGroup M₂
inst✝² : Module R₂ M₂
e✝ : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝¹ : AddCommMonoid N
inst✝ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f : M →ₗ[R] N
b : Basis ι R M
v : ι' → M
e : ι ≃ ι'
i✝ x✝ : ι'
⊢ toMatrix (reindex b e) v i✝ x✝ = submatrix (toMatrix b v) (↑e.symm) _root_.id i✝ x✝
[PROOFSTEP]
simp only [Basis.toMatrix_apply, Basis.repr_reindex, Matrix.submatrix_apply, id.def, Finsupp.mapDomain_equiv_apply]
[GOAL]
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁷ : CommSemiring R
inst✝⁶ : AddCommMonoid M
inst✝⁵ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁴ : CommRing R₂
inst✝³ : AddCommGroup M₂
inst✝² : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝¹ : AddCommMonoid N
inst✝ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f✝ : M →ₗ[R] N
b : Basis ι R M
f : M ≃ₗ[R] N
v : ι → N
⊢ toMatrix (Basis.map b f) v = toMatrix b (↑(LinearEquiv.symm f) ∘ v)
[PROOFSTEP]
ext
[GOAL]
case a.h
ι : Type u_1
ι' : Type u_2
κ : Type u_3
κ' : Type u_4
R : Type u_5
M : Type u_6
inst✝⁷ : CommSemiring R
inst✝⁶ : AddCommMonoid M
inst✝⁵ : Module R M
R₂ : Type u_7
M₂ : Type u_8
inst✝⁴ : CommRing R₂
inst✝³ : AddCommGroup M₂
inst✝² : Module R₂ M₂
e : Basis ι R M
v✝ : ι' → M
i : ι
j : ι'
N : Type u_9
inst✝¹ : AddCommMonoid N
inst✝ : Module R N
b✝ : Basis ι R M
b' : Basis ι' R M
c : Basis κ R N
c' : Basis κ' R N
f✝ : M →ₗ[R] N
b : Basis ι R M
f : M ≃ₗ[R] N
v : ι → N
i✝ x✝ : ι
⊢ toMatrix (Basis.map b f) v i✝ x✝ = toMatrix b (↑(LinearEquiv.symm f) ∘ v) i✝ x✝
[PROOFSTEP]
simp only [Basis.toMatrix_apply, Basis.map, LinearEquiv.trans_apply, (· ∘ ·)]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Basis", "llama_tokens": 20825} |
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
⊢ dualMap id = id
[PROOFSTEP]
ext
[GOAL]
case h.h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
x✝¹ : Dual R M₁
x✝ : M₁
⊢ ↑(↑(dualMap id) x✝¹) x✝ = ↑(↑id x✝¹) x✝
[PROOFSTEP]
rfl
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
hf : Function.Surjective ↑f
⊢ Function.Injective ↑(dualMap f)
[PROOFSTEP]
intro φ ψ h
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
hf : Function.Surjective ↑f
φ ψ : Dual R M₂
h : ↑(dualMap f) φ = ↑(dualMap f) ψ
⊢ φ = ψ
[PROOFSTEP]
ext x
[GOAL]
case h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
hf : Function.Surjective ↑f
φ ψ : Dual R M₂
h : ↑(dualMap f) φ = ↑(dualMap f) ψ
x : M₂
⊢ ↑φ x = ↑ψ x
[PROOFSTEP]
obtain ⟨y, rfl⟩ := hf x
[GOAL]
case h.intro
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
hf : Function.Surjective ↑f
φ ψ : Dual R M₂
h : ↑(dualMap f) φ = ↑(dualMap f) ψ
y : M₁
⊢ ↑φ (↑f y) = ↑ψ (↑f y)
[PROOFSTEP]
exact congr_arg (fun g : Module.Dual R M₁ => g y) h
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ ≃ₗ[R] M₂
src✝ : Dual R M₂ →ₗ[R] Dual R M₁ := LinearMap.dualMap ↑f
⊢ Function.LeftInverse ↑(LinearMap.dualMap ↑(symm f))
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R) (x : Dual R M₂),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom.toFun
[PROOFSTEP]
intro φ
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ ≃ₗ[R] M₂
src✝ : Dual R M₂ →ₗ[R] Dual R M₁ := LinearMap.dualMap ↑f
φ : Dual R M₂
⊢ ↑(LinearMap.dualMap ↑(symm f))
(AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R) (x : Dual R M₂),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
φ) =
φ
[PROOFSTEP]
ext x
[GOAL]
case h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ ≃ₗ[R] M₂
src✝ : Dual R M₂ →ₗ[R] Dual R M₁ := LinearMap.dualMap ↑f
φ : Dual R M₂
x : M₂
⊢ ↑(↑(LinearMap.dualMap ↑(symm f))
(AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R) (x : Dual R M₂),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
φ))
x =
↑φ x
[PROOFSTEP]
simp only [LinearMap.dualMap_apply, LinearEquiv.coe_toLinearMap, LinearMap.toFun_eq_coe, LinearEquiv.apply_symm_apply]
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ ≃ₗ[R] M₂
src✝ : Dual R M₂ →ₗ[R] Dual R M₁ := LinearMap.dualMap ↑f
⊢ Function.RightInverse ↑(LinearMap.dualMap ↑(symm f))
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R) (x : Dual R M₂),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom.toFun
[PROOFSTEP]
intro φ
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ ≃ₗ[R] M₂
src✝ : Dual R M₂ →ₗ[R] Dual R M₁ := LinearMap.dualMap ↑f
φ : Dual R M₁
⊢ AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R) (x : Dual R M₂),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
(↑(LinearMap.dualMap ↑(symm f)) φ) =
φ
[PROOFSTEP]
ext x
[GOAL]
case h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ ≃ₗ[R] M₂
src✝ : Dual R M₂ →ₗ[R] Dual R M₁ := LinearMap.dualMap ↑f
φ : Dual R M₁
x : M₁
⊢ ↑(AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R) (x : Dual R M₂),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
(↑(LinearMap.dualMap ↑(symm f)) φ))
x =
↑φ x
[PROOFSTEP]
simp only [LinearMap.dualMap_apply, LinearEquiv.coe_toLinearMap, LinearMap.toFun_eq_coe, LinearEquiv.symm_apply_apply]
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
⊢ dualMap (refl R M₁) = refl R (Dual R M₁)
[PROOFSTEP]
ext
[GOAL]
case h.h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
x✝¹ : Dual R M₁
x✝ : M₁
⊢ ↑(↑(dualMap (refl R M₁)) x✝¹) x✝ = ↑(↑(refl R (Dual R M₁)) x✝¹) x✝
[PROOFSTEP]
rfl
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
i j : ι
⊢ ↑(↑(toDual b) (↑b i)) (↑b j) = if i = j then 1 else 0
[PROOFSTEP]
erw [constr_basis b, constr_basis b]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
i j : ι
⊢ (if j = i then 1 else 0) = if i = j then 1 else 0
[PROOFSTEP]
simp only [eq_comm]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ ↑(↑(toDual b) (↑(Finsupp.total ι M R ↑b) f)) (↑b i) = ↑f i
[PROOFSTEP]
rw [Finsupp.total_apply, Finsupp.sum, LinearMap.map_sum, LinearMap.sum_apply]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ ∑ d in f.support, ↑(↑(toDual b) (↑f d • ↑b d)) (↑b i) = ↑f i
[PROOFSTEP]
simp_rw [LinearMap.map_smul, LinearMap.smul_apply, toDual_apply, smul_eq_mul, mul_boole, Finset.sum_ite_eq']
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ (if i ∈ f.support then ↑f i else 0) = ↑f i
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
h : i ∈ f.support
⊢ ↑f i = ↑f i
[PROOFSTEP]
rfl
[GOAL]
case neg
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
h : ¬i ∈ f.support
⊢ 0 = ↑f i
[PROOFSTEP]
rw [Finsupp.not_mem_support_iff.mp h]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ ↑(↑(toDual b) (↑b i)) (↑(Finsupp.total ι M R ↑b) f) = ↑f i
[PROOFSTEP]
rw [Finsupp.total_apply, Finsupp.sum, LinearMap.map_sum]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ ∑ i_1 in f.support, ↑(↑(toDual b) (↑b i)) (↑f i_1 • ↑b i_1) = ↑f i
[PROOFSTEP]
simp_rw [LinearMap.map_smul, toDual_apply, smul_eq_mul, mul_boole, Finset.sum_ite_eq]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ (if i ∈ f.support then ↑f i else 0) = ↑f i
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
h : i ∈ f.support
⊢ ↑f i = ↑f i
[PROOFSTEP]
rfl
[GOAL]
case neg
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
f : ι →₀ R
i : ι
h : ¬i ∈ f.support
⊢ 0 = ↑f i
[PROOFSTEP]
rw [Finsupp.not_mem_support_iff.mp h]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
m : M
i : ι
⊢ ↑(↑(toDual b) m) (↑b i) = ↑(↑b.repr m) i
[PROOFSTEP]
rw [← b.toDual_total_left, b.total_repr]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
i : ι
m : M
⊢ ↑(↑(toDual b) (↑b i)) m = ↑(↑b.repr m) i
[PROOFSTEP]
rw [← b.toDual_total_right, b.total_repr]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
i : ι
⊢ ↑(toDual b) (↑b i) = coord b i
[PROOFSTEP]
ext
[GOAL]
case h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
i : ι
x✝ : M
⊢ ↑(↑(toDual b) (↑b i)) x✝ = ↑(coord b i) x✝
[PROOFSTEP]
apply toDual_apply_right
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : Fintype ι
m : M
i : ι
⊢ ↑(↑(toDual b) m) (↑b i) = ↑(equivFun b) m i
[PROOFSTEP]
rw [b.equivFun_apply, toDual_eq_repr]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
m : M
a : ↑(toDual b) m = 0
⊢ m = 0
[PROOFSTEP]
rw [← mem_bot R, ← b.repr.ker, mem_ker, LinearEquiv.coe_coe]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
m : M
a : ↑(toDual b) m = 0
⊢ ↑b.repr m = 0
[PROOFSTEP]
apply Finsupp.ext
[GOAL]
case h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b : Basis ι R M
m : M
a : ↑(toDual b) m = 0
⊢ ∀ (a : ι), ↑(↑b.repr m) a = ↑0 a
[PROOFSTEP]
intro b
[GOAL]
case h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b✝ : Basis ι R M
m : M
a : ↑(toDual b✝) m = 0
b : ι
⊢ ↑(↑b✝.repr m) b = ↑0 b
[PROOFSTEP]
rw [← toDual_eq_repr, a]
[GOAL]
case h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : DecidableEq ι
b✝ : Basis ι R M
m : M
a : ↑(toDual b✝) m = 0
b : ι
⊢ ↑0 (↑b✝ b) = ↑0 b
[PROOFSTEP]
rfl
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
⊢ range (toDual b) = ⊤
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
val✝ : Fintype ι
⊢ range (toDual b) = ⊤
[PROOFSTEP]
refine' eq_top_iff'.2 fun f => _
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
val✝ : Fintype ι
f : Dual R M
⊢ f ∈ range (toDual b)
[PROOFSTEP]
rw [LinearMap.mem_range]
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
val✝ : Fintype ι
f : Dual R M
⊢ ∃ y, ↑(toDual b) y = f
[PROOFSTEP]
let lin_comb : ι →₀ R := Finsupp.equivFunOnFinite.symm fun i => f.toFun (b i)
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
val✝ : Fintype ι
f : Dual R M
lin_comb : ι →₀ R := ↑Finsupp.equivFunOnFinite.symm fun i => AddHom.toFun f.toAddHom (↑b i)
⊢ ∃ y, ↑(toDual b) y = f
[PROOFSTEP]
refine' ⟨Finsupp.total ι M R b lin_comb, b.ext fun i => _⟩
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
val✝ : Fintype ι
f : Dual R M
lin_comb : ι →₀ R := ↑Finsupp.equivFunOnFinite.symm fun i => AddHom.toFun f.toAddHom (↑b i)
i : ι
⊢ ↑(↑(toDual b) (↑(Finsupp.total ι M R ↑b) lin_comb)) (↑b i) = ↑f (↑b i)
[PROOFSTEP]
rw [b.toDual_eq_repr _ i, repr_total b]
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommSemiring R
inst✝³ : AddCommMonoid M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
val✝ : Fintype ι
f : Dual R M
lin_comb : ι →₀ R := ↑Finsupp.equivFunOnFinite.symm fun i => AddHom.toFun f.toAddHom (↑b i)
i : ι
⊢ ↑lin_comb i = ↑f (↑b i)
[PROOFSTEP]
rfl
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : Fintype ι
b : Basis ι R M
f : Dual R M
⊢ ∑ x : ι, ↑f (↑b x) • coord b x = f
[PROOFSTEP]
ext m
[GOAL]
case h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommSemiring R
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : Fintype ι
b : Basis ι R M
f : Dual R M
m : M
⊢ ↑(∑ x : ι, ↑f (↑b x) • coord b x) m = ↑f m
[PROOFSTEP]
simp_rw [LinearMap.sum_apply, LinearMap.smul_apply, smul_eq_mul, mul_comm (f _), ← smul_eq_mul, ← f.map_smul, ←
f.map_sum, Basis.coord_apply, Basis.sum_repr]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
i j : ι
⊢ ↑(↑(dualBasis b) i) (↑b j) = if j = i then 1 else 0
[PROOFSTEP]
convert b.toDual_apply i j using 2
[GOAL]
case h.e'_3.h₁.a
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
i j : ι
⊢ j = i ↔ i = j
[PROOFSTEP]
rw [@eq_comm _ j i]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
f : ι →₀ R
i : ι
⊢ ↑(↑(Finsupp.total ι (Dual R M) R ↑(dualBasis b)) f) (↑b i) = ↑f i
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
f : ι →₀ R
i : ι
val✝ : Fintype ι
⊢ ↑(↑(Finsupp.total ι (Dual R M) R ↑(dualBasis b)) f) (↑b i) = ↑f i
[PROOFSTEP]
rw [Finsupp.total_apply, Finsupp.sum_fintype, LinearMap.sum_apply]
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
f : ι →₀ R
i : ι
val✝ : Fintype ι
⊢ ∑ d : ι, ↑(↑f d • ↑(dualBasis b) d) (↑b i) = ↑f i
[PROOFSTEP]
simp_rw [LinearMap.smul_apply, smul_eq_mul, dualBasis_apply_self, mul_boole, Finset.sum_ite_eq,
if_pos (Finset.mem_univ i)]
[GOAL]
case intro.h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
f : ι →₀ R
i : ι
val✝ : Fintype ι
⊢ ∀ (i : ι), 0 • ↑(dualBasis b) i = 0
[PROOFSTEP]
intro
[GOAL]
case intro.h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
f : ι →₀ R
i : ι
val✝ : Fintype ι
i✝ : ι
⊢ 0 • ↑(dualBasis b) i✝ = 0
[PROOFSTEP]
rw [zero_smul]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
l : Dual R M
i : ι
⊢ ↑(↑(dualBasis b).repr l) i = ↑l (↑b i)
[PROOFSTEP]
rw [← total_dualBasis b, Basis.total_repr b.dualBasis l]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
⊢ ↑(dualBasis b) = coord b
[PROOFSTEP]
ext i x
[GOAL]
case h.h
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
i : ι
x : M
⊢ ↑(↑(dualBasis b) i) x = ↑(coord b i) x
[PROOFSTEP]
apply dualBasis_apply
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
⊢ LinearMap.comp (toDual (dualBasis b)) (toDual b) = Dual.eval R M
[PROOFSTEP]
refine' b.ext fun i => b.dualBasis.ext fun j => _
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : _root_.Finite ι
i j : ι
⊢ ↑(↑(LinearMap.comp (toDual (dualBasis b)) (toDual b)) (↑b i)) (↑(dualBasis b) j) =
↑(↑(Dual.eval R M) (↑b i)) (↑(dualBasis b) j)
[PROOFSTEP]
rw [LinearMap.comp_apply, toDual_apply_left, coe_toDual_self, ← coe_dualBasis, Dual.eval_apply, Basis.repr_self,
Finsupp.single_apply, dualBasis_apply_self]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι
b : Basis ι R M
inst✝ : Fintype ι
l : Dual R M
i : ι
⊢ ↑(equivFun (dualBasis b)) l i = ↑l (↑b i)
[PROOFSTEP]
rw [Basis.equivFun_apply, dualBasis_repr]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
inst✝ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
b : Basis ι R M
⊢ ker (Dual.eval R M) = ⊥
[PROOFSTEP]
rw [ker_eq_bot']
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
inst✝ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
b : Basis ι R M
⊢ ∀ (m : M), ↑(Dual.eval R M) m = 0 → m = 0
[PROOFSTEP]
intro m hm
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
inst✝ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
b : Basis ι R M
m : M
hm : ↑(Dual.eval R M) m = 0
⊢ m = 0
[PROOFSTEP]
simp_rw [LinearMap.ext_iff, Dual.eval_apply, zero_apply] at hm
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
inst✝ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
b : Basis ι R M
m : M
hm : ∀ (x : Dual R M), ↑x m = 0
⊢ m = 0
[PROOFSTEP]
exact (Basis.forall_coord_eq_zero_iff _).mp fun i => hm (b.coord i)
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
inst✝ : _root_.Finite ι
b : Basis ι R M
⊢ range (Dual.eval R M) = ⊤
[PROOFSTEP]
classical
cases nonempty_fintype ι
rw [← b.toDual_toDual, range_comp, b.toDual_range, Submodule.map_top, toDual_range _]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
inst✝ : _root_.Finite ι
b : Basis ι R M
⊢ range (Dual.eval R M) = ⊤
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι✝ : Type w
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : DecidableEq ι✝
b✝ : Basis ι✝ R M
ι : Type u_1
inst✝ : _root_.Finite ι
b : Basis ι R M
val✝ : Fintype ι
⊢ range (Dual.eval R M) = ⊤
[PROOFSTEP]
rw [← b.toDual_toDual, range_comp, b.toDual_range, Submodule.map_top, toDual_range _]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
inst✝ : _root_.Finite ι
b : Basis ι R M
f : ι →₀ R
i : ι
⊢ ↑(↑(Finsupp.total ι (Dual R M) R (coord b)) f) (↑b i) = ↑f i
[PROOFSTEP]
haveI := Classical.decEq ι
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
inst✝ : _root_.Finite ι
b : Basis ι R M
f : ι →₀ R
i : ι
this : DecidableEq ι
⊢ ↑(↑(Finsupp.total ι (Dual R M) R (coord b)) f) (↑b i) = ↑f i
[PROOFSTEP]
rw [← coe_dualBasis, total_dualBasis]
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : _root_.Finite ι
b : Basis ι K V
⊢ lift (Module.rank K V) = Module.rank K (Dual K V)
[PROOFSTEP]
classical
cases nonempty_fintype ι
have := LinearEquiv.lift_rank_eq b.toDualEquiv
rw [Cardinal.lift_umax.{u₂, u₁}] at this
rw [this, ← Cardinal.lift_umax]
apply Cardinal.lift_id
[GOAL]
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : _root_.Finite ι
b : Basis ι K V
⊢ lift (Module.rank K V) = Module.rank K (Dual K V)
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : _root_.Finite ι
b : Basis ι K V
val✝ : Fintype ι
⊢ lift (Module.rank K V) = Module.rank K (Dual K V)
[PROOFSTEP]
have := LinearEquiv.lift_rank_eq b.toDualEquiv
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : _root_.Finite ι
b : Basis ι K V
val✝ : Fintype ι
this : lift (Module.rank K V) = lift (Module.rank K (Dual K V))
⊢ lift (Module.rank K V) = Module.rank K (Dual K V)
[PROOFSTEP]
rw [Cardinal.lift_umax.{u₂, u₁}] at this
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : _root_.Finite ι
b : Basis ι K V
val✝ : Fintype ι
this : lift (Module.rank K V) = lift (Module.rank K (Dual K V))
⊢ lift (Module.rank K V) = Module.rank K (Dual K V)
[PROOFSTEP]
rw [this, ← Cardinal.lift_umax]
[GOAL]
case intro
R : Type u
M : Type v
K : Type u₁
V : Type u₂
ι : Type w
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : _root_.Finite ι
b : Basis ι K V
val✝ : Fintype ι
this : lift (Module.rank K V) = lift (Module.rank K (Dual K V))
⊢ lift (Module.rank K (Dual K V)) = Module.rank K (Dual K V)
[PROOFSTEP]
apply Cardinal.lift_id
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ ker (eval K V) = ⊥
[PROOFSTEP]
classical exact (Module.Free.chooseBasis K V).eval_ker
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ ker (eval K V) = ⊥
[PROOFSTEP]
exact (Module.Free.chooseBasis K V).eval_ker
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ Function.Injective (Submodule.map (eval K V))
[PROOFSTEP]
apply Submodule.map_injective_of_injective
[GOAL]
case hf
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ Function.Injective ↑(eval K V)
[PROOFSTEP]
rw [← LinearMap.ker_eq_bot]
[GOAL]
case hf
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ ker (eval K V) = ⊥
[PROOFSTEP]
apply eval_ker K V
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ Function.Surjective (Submodule.comap (eval K V))
[PROOFSTEP]
apply Submodule.comap_surjective_of_injective
[GOAL]
case hf
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ Function.Injective ↑(eval K V)
[PROOFSTEP]
rw [← LinearMap.ker_eq_bot]
[GOAL]
case hf
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
⊢ ker (eval K V) = ⊥
[PROOFSTEP]
apply eval_ker K V
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
v : V
⊢ ↑(eval K V) v = 0 ↔ v = 0
[PROOFSTEP]
simpa only using SetLike.ext_iff.mp (eval_ker K V) v
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
v : V
⊢ (∀ (φ : Dual K V), ↑φ v = 0) ↔ v = 0
[PROOFSTEP]
rw [← eval_apply_eq_zero_iff K v, LinearMap.ext_iff]
[GOAL]
K : Type u₁
V : Type u₂
inst✝³ : CommRing K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
inst✝ : Free K V
v : V
⊢ (∀ (φ : Dual K V), ↑φ v = 0) ↔ ∀ (x : Dual K V), ↑(↑(eval K V) v) x = ↑0 x
[PROOFSTEP]
rfl
[GOAL]
K : Type u₁
V : Type u₂
inst✝⁹ : CommRing K
inst✝⁸ : AddCommGroup V
inst✝⁷ : Module K V
inst✝⁶ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : AddCommGroup N
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : IsReflexive R M
f : Dual R M
g : Dual R (Dual R M)
⊢ ↑f (↑(LinearEquiv.symm (evalEquiv R M)) g) = ↑g f
[PROOFSTEP]
set m := (evalEquiv R M).symm g
[GOAL]
K : Type u₁
V : Type u₂
inst✝⁹ : CommRing K
inst✝⁸ : AddCommGroup V
inst✝⁷ : Module K V
inst✝⁶ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : AddCommGroup N
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : IsReflexive R M
f : Dual R M
g : Dual R (Dual R M)
m : M := ↑(LinearEquiv.symm (evalEquiv R M)) g
⊢ ↑f m = ↑g f
[PROOFSTEP]
rw [← (evalEquiv R M).apply_symm_apply g, evalEquiv_apply, Dual.eval_apply]
[GOAL]
K : Type u₁
V : Type u₂
inst✝⁹ : CommRing K
inst✝⁸ : AddCommGroup V
inst✝⁷ : Module K V
inst✝⁶ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : AddCommGroup N
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : IsReflexive R M
⊢ ↑(LinearEquiv.dualMap (LinearEquiv.symm (evalEquiv R M))) = Dual.eval R (Dual R M)
[PROOFSTEP]
ext
[GOAL]
case h.h
K : Type u₁
V : Type u₂
inst✝⁹ : CommRing K
inst✝⁸ : AddCommGroup V
inst✝⁷ : Module K V
inst✝⁶ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : AddCommGroup N
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : IsReflexive R M
x✝¹ : Dual R M
x✝ : Dual R (Dual R M)
⊢ ↑(↑↑(LinearEquiv.dualMap (LinearEquiv.symm (evalEquiv R M))) x✝¹) x✝ = ↑(↑(Dual.eval R (Dual R M)) x✝¹) x✝
[PROOFSTEP]
simp
[GOAL]
K : Type u₁
V : Type u₂
inst✝⁹ : CommRing K
inst✝⁸ : AddCommGroup V
inst✝⁷ : Module K V
inst✝⁶ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁵ : CommRing R
inst✝⁴ : AddCommGroup M
inst✝³ : AddCommGroup N
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : IsReflexive R M
⊢ Bijective ↑(eval R (Dual R M))
[PROOFSTEP]
simpa only [← symm_dualMap_evalEquiv] using (evalEquiv R M).dualMap.symm.bijective
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
⊢ Bijective ↑(Dual.eval R (M × N))
[PROOFSTEP]
let e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
(dualProdDualEquivDual R M N).dualMap.trans (dualProdDualEquivDual R (Dual R M) (Dual R N)).symm
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
LinearEquiv.trans (LinearEquiv.dualMap (dualProdDualEquivDual R M N))
(LinearEquiv.symm (dualProdDualEquivDual R (Dual R M) (Dual R N)))
⊢ Bijective ↑(Dual.eval R (M × N))
[PROOFSTEP]
have : Dual.eval R (M × N) = e.symm.comp ((Dual.eval R M).prodMap (Dual.eval R N)) := by ext m f <;> simp
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
LinearEquiv.trans (LinearEquiv.dualMap (dualProdDualEquivDual R M N))
(LinearEquiv.symm (dualProdDualEquivDual R (Dual R M) (Dual R N)))
⊢ Dual.eval R (M × N) = LinearMap.comp (↑(LinearEquiv.symm e)) (prodMap (Dual.eval R M) (Dual.eval R N))
[PROOFSTEP]
ext m f
[GOAL]
case hl.h.h
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
LinearEquiv.trans (LinearEquiv.dualMap (dualProdDualEquivDual R M N))
(LinearEquiv.symm (dualProdDualEquivDual R (Dual R M) (Dual R N)))
m : M
f : Dual R (M × N)
⊢ ↑(↑(LinearMap.comp (Dual.eval R (M × N)) (inl R M N)) m) f =
↑(↑(LinearMap.comp (LinearMap.comp (↑(LinearEquiv.symm e)) (prodMap (Dual.eval R M) (Dual.eval R N))) (inl R M N))
m)
f
[PROOFSTEP]
simp
[GOAL]
case hr.h.h
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
LinearEquiv.trans (LinearEquiv.dualMap (dualProdDualEquivDual R M N))
(LinearEquiv.symm (dualProdDualEquivDual R (Dual R M) (Dual R N)))
m : N
f : Dual R (M × N)
⊢ ↑(↑(LinearMap.comp (Dual.eval R (M × N)) (inr R M N)) m) f =
↑(↑(LinearMap.comp (LinearMap.comp (↑(LinearEquiv.symm e)) (prodMap (Dual.eval R M) (Dual.eval R N))) (inr R M N))
m)
f
[PROOFSTEP]
simp
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
LinearEquiv.trans (LinearEquiv.dualMap (dualProdDualEquivDual R M N))
(LinearEquiv.symm (dualProdDualEquivDual R (Dual R M) (Dual R N)))
this : Dual.eval R (M × N) = LinearMap.comp (↑(LinearEquiv.symm e)) (prodMap (Dual.eval R M) (Dual.eval R N))
⊢ Bijective ↑(Dual.eval R (M × N))
[PROOFSTEP]
simp only [this, LinearEquiv.trans_symm, LinearEquiv.symm_symm, LinearEquiv.dualMap_symm, coe_comp, LinearEquiv.coe_coe,
EquivLike.comp_bijective]
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ : IsReflexive R M
inst✝ : IsReflexive R N
e : Dual R (Dual R (M × N)) ≃ₗ[R] Dual R (Dual R M) × Dual R (Dual R N) :=
LinearEquiv.trans (LinearEquiv.dualMap (dualProdDualEquivDual R M N))
(LinearEquiv.symm (dualProdDualEquivDual R (Dual R M) (Dual R N)))
this : Dual.eval R (M × N) = LinearMap.comp (↑(LinearEquiv.symm e)) (prodMap (Dual.eval R M) (Dual.eval R N))
⊢ Bijective ↑(prodMap (Dual.eval R M) (Dual.eval R N))
[PROOFSTEP]
exact Bijective.Prod_map (bijective_dual_eval R M) (bijective_dual_eval R N)
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ inst✝ : IsReflexive R M
e : M ≃ₗ[R] N
⊢ Bijective ↑(Dual.eval R N)
[PROOFSTEP]
let ed : Dual R (Dual R N) ≃ₗ[R] Dual R (Dual R M) := e.symm.dualMap.dualMap
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ inst✝ : IsReflexive R M
e : M ≃ₗ[R] N
ed : Dual R (Dual R N) ≃ₗ[R] Dual R (Dual R M) := LinearEquiv.dualMap (LinearEquiv.dualMap (LinearEquiv.symm e))
⊢ Bijective ↑(Dual.eval R N)
[PROOFSTEP]
have : Dual.eval R N = ed.symm.comp ((Dual.eval R M).comp e.symm.toLinearMap) :=
by
ext m f
exact FunLike.congr_arg f (e.apply_symm_apply m).symm
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ inst✝ : IsReflexive R M
e : M ≃ₗ[R] N
ed : Dual R (Dual R N) ≃ₗ[R] Dual R (Dual R M) := LinearEquiv.dualMap (LinearEquiv.dualMap (LinearEquiv.symm e))
⊢ Dual.eval R N = LinearMap.comp (↑(LinearEquiv.symm ed)) (LinearMap.comp (Dual.eval R M) ↑(LinearEquiv.symm e))
[PROOFSTEP]
ext m f
[GOAL]
case h.h
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ inst✝ : IsReflexive R M
e : M ≃ₗ[R] N
ed : Dual R (Dual R N) ≃ₗ[R] Dual R (Dual R M) := LinearEquiv.dualMap (LinearEquiv.dualMap (LinearEquiv.symm e))
m : N
f : Dual R N
⊢ ↑(↑(Dual.eval R N) m) f =
↑(↑(LinearMap.comp (↑(LinearEquiv.symm ed)) (LinearMap.comp (Dual.eval R M) ↑(LinearEquiv.symm e))) m) f
[PROOFSTEP]
exact FunLike.congr_arg f (e.apply_symm_apply m).symm
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ inst✝ : IsReflexive R M
e : M ≃ₗ[R] N
ed : Dual R (Dual R N) ≃ₗ[R] Dual R (Dual R M) := LinearEquiv.dualMap (LinearEquiv.dualMap (LinearEquiv.symm e))
this : Dual.eval R N = LinearMap.comp (↑(LinearEquiv.symm ed)) (LinearMap.comp (Dual.eval R M) ↑(LinearEquiv.symm e))
⊢ Bijective ↑(Dual.eval R N)
[PROOFSTEP]
simp only [this, LinearEquiv.trans_symm, LinearEquiv.symm_symm, LinearEquiv.dualMap_symm, coe_comp, LinearEquiv.coe_coe,
EquivLike.comp_bijective]
[GOAL]
K : Type u₁
V : Type u₂
inst✝¹⁰ : CommRing K
inst✝⁹ : AddCommGroup V
inst✝⁸ : Module K V
inst✝⁷ : Free K V
R : Type u_1
M : Type u_2
N : Type u_3
inst✝⁶ : CommRing R
inst✝⁵ : AddCommGroup M
inst✝⁴ : AddCommGroup N
inst✝³ : Module R M
inst✝² : Module R N
inst✝¹ inst✝ : IsReflexive R M
e : M ≃ₗ[R] N
ed : Dual R (Dual R N) ≃ₗ[R] Dual R (Dual R M) := LinearEquiv.dualMap (LinearEquiv.dualMap (LinearEquiv.symm e))
this : Dual.eval R N = LinearMap.comp (↑(LinearEquiv.symm ed)) (LinearMap.comp (Dual.eval R M) ↑(LinearEquiv.symm e))
⊢ Bijective (↑(Dual.eval R M) ∘ ↑(LinearEquiv.symm e))
[PROOFSTEP]
refine Bijective.comp (bijective_dual_eval R M) (LinearEquiv.bijective _)
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
m : M
⊢ ∀ (a : ι), a ∈ Set.Finite.toFinset (_ : Set.Finite {i | ↑(ε i) m ≠ 0}) ↔ (fun i => ↑(ε i) m) a ≠ 0
[PROOFSTEP]
intro i
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
m : M
i : ι
⊢ i ∈ Set.Finite.toFinset (_ : Set.Finite {i | ↑(ε i) m ≠ 0}) ↔ (fun i => ↑(ε i) m) i ≠ 0
[PROOFSTEP]
rw [Set.Finite.mem_toFinset, Set.mem_setOf_eq]
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
⊢ ↑(ε i) (lc e l) = ↑l i
[PROOFSTEP]
erw [LinearMap.map_sum]
-- Porting note: cannot get at •
-- simp only [h.eval, map_smul, smul_eq_mul]
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
⊢ (Finset.sum l.support fun i_1 => ↑(ε i) ((fun i a => a • e i) i_1 (↑l i_1))) = ↑l i
[PROOFSTEP]
rw [Finset.sum_eq_single i]
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
⊢ ↑(ε i) ((fun i a => a • e i) i (↑l i)) = ↑l i
[PROOFSTEP]
simp [h.eval, smul_eq_mul]
[GOAL]
case h₀
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
⊢ ∀ (b : ι), b ∈ l.support → b ≠ i → ↑(ε i) ((fun i a => a • e i) b (↑l b)) = 0
[PROOFSTEP]
intro q _ q_ne
[GOAL]
case h₀
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i q : ι
a✝ : q ∈ l.support
q_ne : q ≠ i
⊢ ↑(ε i) ((fun i a => a • e i) q (↑l q)) = 0
[PROOFSTEP]
simp [q_ne.symm, h.eval, smul_eq_mul]
[GOAL]
case h₁
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
⊢ ¬i ∈ l.support → ↑(ε i) ((fun i a => a • e i) i (↑l i)) = 0
[PROOFSTEP]
intro p_not_in
[GOAL]
case h₁
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
p_not_in : ¬i ∈ l.support
⊢ ↑(ε i) ((fun i a => a • e i) i (↑l i)) = 0
[PROOFSTEP]
simp [Finsupp.not_mem_support_iff.1 p_not_in]
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
⊢ coeffs h (lc e l) = l
[PROOFSTEP]
ext i
[GOAL]
case h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
l : ι →₀ R
i : ι
⊢ ↑(coeffs h (lc e l)) i = ↑l i
[PROOFSTEP]
rw [h.coeffs_apply, h.dual_lc]
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
m : M
⊢ lc e (coeffs h m) = m
[PROOFSTEP]
refine' eq_of_sub_eq_zero (h.Total _)
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
m : M
⊢ ∀ (i : ι), ↑(ε i) (lc e (coeffs h m) - m) = 0
[PROOFSTEP]
intro i
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
m : M
i : ι
⊢ ↑(ε i) (lc e (coeffs h m) - m) = 0
[PROOFSTEP]
simp [LinearMap.map_sub, h.dual_lc, sub_eq_zero]
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
v w : M
⊢ coeffs h (v + w) = coeffs h v + coeffs h w
[PROOFSTEP]
ext i
[GOAL]
case h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
v w : M
i : ι
⊢ ↑(coeffs h (v + w)) i = ↑(coeffs h v + coeffs h w) i
[PROOFSTEP]
exact (ε i).map_add v w
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
c : R
v : M
⊢ AddHom.toFun { toFun := coeffs h, map_add' := (_ : ∀ (v w : M), coeffs h (v + w) = coeffs h v + coeffs h w) }
(c • v) =
↑(RingHom.id R) c •
AddHom.toFun { toFun := coeffs h, map_add' := (_ : ∀ (v w : M), coeffs h (v + w) = coeffs h v + coeffs h w) } v
[PROOFSTEP]
ext i
[GOAL]
case h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
c : R
v : M
i : ι
⊢ ↑(AddHom.toFun { toFun := coeffs h, map_add' := (_ : ∀ (v w : M), coeffs h (v + w) = coeffs h v + coeffs h w) }
(c • v))
i =
↑(↑(RingHom.id R) c •
AddHom.toFun { toFun := coeffs h, map_add' := (_ : ∀ (v w : M), coeffs h (v + w) = coeffs h v + coeffs h w) }
v)
i
[PROOFSTEP]
exact (ε i).map_smul c v
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
⊢ ↑(basis h) = e
[PROOFSTEP]
ext i
[GOAL]
case h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
i : ι
⊢ ↑(basis h) i = e i
[PROOFSTEP]
rw [Basis.apply_eq_iff]
[GOAL]
case h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
i : ι
⊢ ↑(basis h).repr (e i) = Finsupp.single i 1
[PROOFSTEP]
ext j
[GOAL]
case h.h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
i j : ι
⊢ ↑(↑(basis h).repr (e i)) j = ↑(Finsupp.single i 1) j
[PROOFSTEP]
rw [h.basis_repr_apply, coeffs_apply, h.eval, Finsupp.single_apply]
[GOAL]
case h.h
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
i j : ι
⊢ (if j = i then 1 else 0) = if i = j then 1 else 0
[PROOFSTEP]
convert if_congr (eq_comm (a := j) (b := i)) rfl rfl
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
H : Set ι
x : M
hmem : x ∈ Submodule.span R (e '' H)
⊢ ∀ (i : ι), ↑(ε i) x ≠ 0 → i ∈ H
[PROOFSTEP]
intro i hi
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
H : Set ι
x : M
hmem : x ∈ Submodule.span R (e '' H)
i : ι
hi : ↑(ε i) x ≠ 0
⊢ i ∈ H
[PROOFSTEP]
rcases(Finsupp.mem_span_image_iff_total _).mp hmem with ⟨l, supp_l, rfl⟩
[GOAL]
case intro.intro
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
H : Set ι
i : ι
l : ι →₀ R
supp_l : l ∈ Finsupp.supported R R H
hmem : ↑(Finsupp.total ι M R e) l ∈ Submodule.span R (e '' H)
hi : ↑(ε i) (↑(Finsupp.total ι M R e) l) ≠ 0
⊢ i ∈ H
[PROOFSTEP]
apply not_imp_comm.mp ((Finsupp.mem_supported' _ _).mp supp_l i)
[GOAL]
case intro.intro
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝³ : CommRing R
inst✝² : AddCommGroup M
inst✝¹ : Module R M
e : ι → M
ε : ι → Dual R M
inst✝ : DecidableEq ι
h : DualBases e ε
H : Set ι
i : ι
l : ι →₀ R
supp_l : l ∈ Finsupp.supported R R H
hmem : ↑(Finsupp.total ι M R e) l ∈ Submodule.span R (e '' H)
hi : ↑(ε i) (↑(Finsupp.total ι M R e) l) ≠ 0
⊢ ¬↑l i = 0
[PROOFSTEP]
rwa [← lc_def, h.dual_lc] at hi
[GOAL]
R : Type u_1
M : Type u_2
ι : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
e : ι → M
ε : ι → Dual R M
inst✝¹ : DecidableEq ι
h : DualBases e ε
inst✝ : Fintype ι
i j : ι
⊢ ↑(↑(Basis.dualBasis (basis h)) i) (↑(basis h) j) = ↑(ε i) (↑(basis h) j)
[PROOFSTEP]
rw [h.basis.dualBasis_apply_self, h.coe_basis, h.eval, if_congr eq_comm rfl rfl]
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
φ : Module.Dual R M
⊢ φ ∈ dualAnnihilator W ↔ ∀ (w : M), w ∈ W → ↑φ w = 0
[PROOFSTEP]
refine' LinearMap.mem_ker.trans _
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
φ : Module.Dual R M
⊢ ↑(dualRestrict W) φ = 0 ↔ ∀ (w : M), w ∈ W → ↑φ w = 0
[PROOFSTEP]
simp_rw [LinearMap.ext_iff, dualRestrict_apply]
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
φ : Module.Dual R M
⊢ (∀ (x : { x // x ∈ W }), ↑φ ↑x = ↑0 x) ↔ ∀ (w : M), w ∈ W → ↑φ w = 0
[PROOFSTEP]
exact ⟨fun h w hw => h ⟨w, hw⟩, fun h w => h w.1 w.2⟩
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
Φ : Submodule R (Module.Dual R M)
x : M
⊢ x ∈ dualCoannihilator Φ ↔ ∀ (φ : Module.Dual R M), φ ∈ Φ → ↑φ x = 0
[PROOFSTEP]
simp_rw [dualCoannihilator, mem_comap, mem_dualAnnihilator, Module.Dual.eval_apply]
[GOAL]
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ GaloisConnection (↑OrderDual.toDual ∘ dualAnnihilator) (dualCoannihilator ∘ ↑OrderDual.ofDual)
[PROOFSTEP]
intro a b
[GOAL]
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
b : (Submodule R (Module.Dual R M))ᵒᵈ
⊢ (↑OrderDual.toDual ∘ dualAnnihilator) a ≤ b ↔ a ≤ (dualCoannihilator ∘ ↑OrderDual.ofDual) b
[PROOFSTEP]
induction b using OrderDual.rec
[GOAL]
case h₂
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
⊢ (↑OrderDual.toDual ∘ dualAnnihilator) a ≤ ↑OrderDual.toDual a✝ ↔
a ≤ (dualCoannihilator ∘ ↑OrderDual.ofDual) (↑OrderDual.toDual a✝)
[PROOFSTEP]
simp only [Function.comp_apply, OrderDual.toDual_le_toDual, OrderDual.ofDual_toDual]
[GOAL]
case h₂
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
⊢ a✝ ≤ dualAnnihilator a ↔ a ≤ dualCoannihilator a✝
[PROOFSTEP]
constructor
[GOAL]
case h₂.mp
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
⊢ a✝ ≤ dualAnnihilator a → a ≤ dualCoannihilator a✝
[PROOFSTEP]
intro h x hx
[GOAL]
case h₂.mp
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a✝ ≤ dualAnnihilator a
x : M
hx : x ∈ a
⊢ x ∈ dualCoannihilator a✝
[PROOFSTEP]
simp only [mem_dualAnnihilator, mem_dualCoannihilator]
[GOAL]
case h₂.mp
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a✝ ≤ dualAnnihilator a
x : M
hx : x ∈ a
⊢ ∀ (φ : Module.Dual R M), φ ∈ a✝ → ↑φ x = 0
[PROOFSTEP]
intro y hy
[GOAL]
case h₂.mp
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a✝ ≤ dualAnnihilator a
x : M
hx : x ∈ a
y : Module.Dual R M
hy : y ∈ a✝
⊢ ↑y x = 0
[PROOFSTEP]
have := h hy
[GOAL]
case h₂.mp
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a✝ ≤ dualAnnihilator a
x : M
hx : x ∈ a
y : Module.Dual R M
hy : y ∈ a✝
this : y ∈ dualAnnihilator a
⊢ ↑y x = 0
[PROOFSTEP]
simp only [mem_dualAnnihilator, mem_dualCoannihilator] at this
[GOAL]
case h₂.mp
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a✝ ≤ dualAnnihilator a
x : M
hx : x ∈ a
y : Module.Dual R M
hy : y ∈ a✝
this : ∀ (w : M), w ∈ a → ↑y w = 0
⊢ ↑y x = 0
[PROOFSTEP]
exact this x hx
[GOAL]
case h₂.mpr
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
⊢ a ≤ dualCoannihilator a✝ → a✝ ≤ dualAnnihilator a
[PROOFSTEP]
intro h x hx
[GOAL]
case h₂.mpr
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a ≤ dualCoannihilator a✝
x : Module.Dual R M
hx : x ∈ a✝
⊢ x ∈ dualAnnihilator a
[PROOFSTEP]
simp only [mem_dualAnnihilator, mem_dualCoannihilator]
[GOAL]
case h₂.mpr
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a ≤ dualCoannihilator a✝
x : Module.Dual R M
hx : x ∈ a✝
⊢ ∀ (w : M), w ∈ a → ↑x w = 0
[PROOFSTEP]
intro y hy
[GOAL]
case h₂.mpr
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a ≤ dualCoannihilator a✝
x : Module.Dual R M
hx : x ∈ a✝
y : M
hy : y ∈ a
⊢ ↑x y = 0
[PROOFSTEP]
have := h hy
[GOAL]
case h₂.mpr
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a ≤ dualCoannihilator a✝
x : Module.Dual R M
hx : x ∈ a✝
y : M
hy : y ∈ a
this : y ∈ dualCoannihilator a✝
⊢ ↑x y = 0
[PROOFSTEP]
simp only [mem_dualAnnihilator, mem_dualCoannihilator] at this
[GOAL]
case h₂.mpr
R✝ : Type u
M✝ : Type v
inst✝⁵ : CommSemiring R✝
inst✝⁴ : AddCommMonoid M✝
inst✝³ : Module R✝ M✝
W : Submodule R✝ M✝
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
a : Submodule R M
a✝ : Submodule R (Module.Dual R M)
h : a ≤ dualCoannihilator a✝
x : Module.Dual R M
hx : x ∈ a✝
y : M
hy : y ∈ a
this : ∀ (φ : Module.Dual R M), φ ∈ a✝ → ↑φ y = 0
⊢ ↑x y = 0
[PROOFSTEP]
exact this x hx
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
⊢ dualAnnihilator ⊤ = ⊥
[PROOFSTEP]
rw [eq_bot_iff]
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
⊢ dualAnnihilator ⊤ ≤ ⊥
[PROOFSTEP]
intro v
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
v : Module.Dual R M
⊢ v ∈ dualAnnihilator ⊤ → v ∈ ⊥
[PROOFSTEP]
simp_rw [mem_dualAnnihilator, mem_bot, mem_top, forall_true_left]
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
v : Module.Dual R M
⊢ (∀ (w : M), ↑v w = 0) → v = 0
[PROOFSTEP]
exact fun h => LinearMap.ext h
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W U V : Submodule R M
⊢ dualAnnihilator U ⊔ dualAnnihilator V ≤ dualAnnihilator (U ⊓ V)
[PROOFSTEP]
rw [le_dualAnnihilator_iff_le_dualCoannihilator, dualCoannihilator_sup_eq]
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W U V : Submodule R M
⊢ U ⊓ V ≤ dualCoannihilator (dualAnnihilator U) ⊓ dualCoannihilator (dualAnnihilator V)
[PROOFSTEP]
apply inf_le_inf
[GOAL]
case h₁
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W U V : Submodule R M
⊢ U ≤ dualCoannihilator (dualAnnihilator U)
[PROOFSTEP]
exact le_dualAnnihilator_dualCoannihilator _
[GOAL]
case h₂
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W U V : Submodule R M
⊢ V ≤ dualCoannihilator (dualAnnihilator V)
[PROOFSTEP]
exact le_dualAnnihilator_dualCoannihilator _
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
ι : Type u_1
U : ι → Submodule R M
⊢ ⨆ (i : ι), dualAnnihilator (U i) ≤ dualAnnihilator (⨅ (i : ι), U i)
[PROOFSTEP]
rw [le_dualAnnihilator_iff_le_dualCoannihilator, dualCoannihilator_iSup_eq]
[GOAL]
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
ι : Type u_1
U : ι → Submodule R M
⊢ ⨅ (i : ι), U i ≤ ⨅ (i : ι), dualCoannihilator (dualAnnihilator (U i))
[PROOFSTEP]
apply iInf_mono
[GOAL]
case h
R : Type u
M : Type v
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
W : Submodule R M
ι : Type u_1
U : ι → Submodule R M
⊢ ∀ (i : ι), U i ≤ dualCoannihilator (dualAnnihilator (U i))
[PROOFSTEP]
exact fun i : ι => le_dualAnnihilator_dualCoannihilator (U i)
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
⊢ dualCoannihilator ⊤ = ⊥
[PROOFSTEP]
rw [dualCoannihilator, dualAnnihilator_top, comap_bot, Module.eval_ker]
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
⊢ dualCoannihilator (dualAnnihilator W) = W
[PROOFSTEP]
refine' le_antisymm _ (le_dualAnnihilator_dualCoannihilator _)
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
⊢ dualCoannihilator (dualAnnihilator W) ≤ W
[PROOFSTEP]
intro v
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
v : V
⊢ v ∈ dualCoannihilator (dualAnnihilator W) → v ∈ W
[PROOFSTEP]
simp only [mem_dualAnnihilator, mem_dualCoannihilator]
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
v : V
⊢ (∀ (φ : Module.Dual K V), (∀ (w : V), w ∈ W → ↑φ w = 0) → ↑φ v = 0) → v ∈ W
[PROOFSTEP]
contrapose!
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
v : V
⊢ ¬v ∈ W → ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ v ≠ 0
[PROOFSTEP]
intro hv
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
v : V
hv : ¬v ∈ W
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ v ≠ 0
[PROOFSTEP]
obtain ⟨W', hW⟩ := Submodule.exists_isCompl W
[GOAL]
case intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
v : V
hv : ¬v ∈ W
W' : Submodule K V
hW : IsCompl W W'
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ v ≠ 0
[PROOFSTEP]
obtain ⟨⟨w, w'⟩, rfl, -⟩ := existsUnique_add_of_isCompl_prod hW v
[GOAL]
case intro.intro.mk.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ (↑(w, w').fst + ↑(w, w').snd) ≠ 0
[PROOFSTEP]
have hw'n : (w' : V) ∉ W := by
contrapose! hv
exact Submodule.add_mem W w.2 hv
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
⊢ ¬↑w' ∈ W
[PROOFSTEP]
contrapose! hv
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ↑w' ∈ W
⊢ ↑w + ↑w' ∈ W
[PROOFSTEP]
exact Submodule.add_mem W w.2 hv
[GOAL]
case intro.intro.mk.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ (↑(w, w').fst + ↑(w, w').snd) ≠ 0
[PROOFSTEP]
have hw'nz : w' ≠ 0 := by
rintro rfl
exact hw'n (Submodule.zero_mem W)
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
⊢ w' ≠ 0
[PROOFSTEP]
rintro rfl
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
hv : ¬↑(w, 0).fst + ↑(w, 0).snd ∈ W
hw'n : ¬↑0 ∈ W
⊢ False
[PROOFSTEP]
exact hw'n (Submodule.zero_mem W)
[GOAL]
case intro.intro.mk.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
hw'nz : w' ≠ 0
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ (↑(w, w').fst + ↑(w, w').snd) ≠ 0
[PROOFSTEP]
rw [Ne.def, ← Module.forall_dual_apply_eq_zero_iff K w'] at hw'nz
[GOAL]
case intro.intro.mk.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
hw'nz : ¬∀ (φ : Module.Dual K { x // x ∈ W' }), ↑φ w' = 0
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ (↑(w, w').fst + ↑(w, w').snd) ≠ 0
[PROOFSTEP]
push_neg at hw'nz
[GOAL]
case intro.intro.mk.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
hw'nz : ∃ φ, ↑φ w' ≠ 0
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ (↑(w, w').fst + ↑(w, w').snd) ≠ 0
[PROOFSTEP]
obtain ⟨φ, hφ⟩ := hw'nz
[GOAL]
case intro.intro.mk.intro.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
φ : Module.Dual K { x // x ∈ W' }
hφ : ↑φ w' ≠ 0
⊢ ∃ φ, (∀ (w : V), w ∈ W → ↑φ w = 0) ∧ ↑φ (↑(w, w').fst + ↑(w, w').snd) ≠ 0
[PROOFSTEP]
exists ((LinearMap.ofIsComplProd hW).comp (LinearMap.inr _ _ _)) φ
[GOAL]
case intro.intro.mk.intro.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
φ : Module.Dual K { x // x ∈ W' }
hφ : ↑φ w' ≠ 0
⊢ (∀ (w : V),
w ∈ W → ↑(↑(comp (ofIsComplProd hW) (inr K ({ x // x ∈ W } →ₗ[K] K) ({ x // x ∈ W' } →ₗ[K] K))) φ) w = 0) ∧
↑(↑(comp (ofIsComplProd hW) (inr K ({ x // x ∈ W } →ₗ[K] K) ({ x // x ∈ W' } →ₗ[K] K))) φ)
(↑(w, w').fst + ↑(w, w').snd) ≠
0
[PROOFSTEP]
simp only [coe_comp, coe_inr, Function.comp_apply, ofIsComplProd_apply, map_add, ofIsCompl_left_apply, zero_apply,
ofIsCompl_right_apply, zero_add, Ne.def]
[GOAL]
case intro.intro.mk.intro.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
φ : Module.Dual K { x // x ∈ W' }
hφ : ↑φ w' ≠ 0
⊢ (∀ (w : V), w ∈ W → ↑(ofIsCompl hW 0 φ) w = 0) ∧ ¬↑φ w' = 0
[PROOFSTEP]
refine' ⟨_, hφ⟩
[GOAL]
case intro.intro.mk.intro.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
φ : Module.Dual K { x // x ∈ W' }
hφ : ↑φ w' ≠ 0
⊢ ∀ (w : V), w ∈ W → ↑(ofIsCompl hW 0 φ) w = 0
[PROOFSTEP]
intro v hv
[GOAL]
case intro.intro.mk.intro.intro
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
W' : Submodule K V
hW : IsCompl W W'
w : { x // x ∈ W }
w' : { x // x ∈ W' }
hv✝ : ¬↑(w, w').fst + ↑(w, w').snd ∈ W
hw'n : ¬↑w' ∈ W
φ : Module.Dual K { x // x ∈ W' }
hφ : ↑φ w' ≠ 0
v : V
hv : v ∈ W
⊢ ↑(ofIsCompl hW 0 φ) v = 0
[PROOFSTEP]
apply LinearMap.ofIsCompl_left_apply hW ⟨v, hv⟩
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
v : V
⊢ (∀ (φ : Module.Dual K V), φ ∈ dualAnnihilator W → ↑φ v = 0) ↔ v ∈ W
[PROOFSTEP]
rw [← SetLike.ext_iff.mp dualAnnihilator_dualCoannihilator_eq v, mem_dualCoannihilator]
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W W' : Subspace K V
⊢ dualAnnihilator W = dualAnnihilator W' ↔ W = W'
[PROOFSTEP]
constructor
[GOAL]
case mp
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W W' : Subspace K V
⊢ dualAnnihilator W = dualAnnihilator W' → W = W'
[PROOFSTEP]
apply (dualAnnihilatorGci K V).l_injective
[GOAL]
case mpr
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W W' : Subspace K V
⊢ W = W' → dualAnnihilator W = dualAnnihilator W'
[PROOFSTEP]
rintro rfl
[GOAL]
case mpr
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
⊢ dualAnnihilator W = dualAnnihilator W
[PROOFSTEP]
rfl
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
φ : Module.Dual K { x // x ∈ W }
w : { x // x ∈ W }
⊢ ↑(↑(dualLift W) φ) ↑w = ↑φ w
[PROOFSTEP]
erw [ofIsCompl_left_apply _ w]
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
φ : Module.Dual K { x // x ∈ W }
w : { x // x ∈ W }
⊢ ↑(↑(inl K (Module.Dual K { x // x ∈ W })
({ x // x ∈ ↑(Classical.indefiniteDescription (fun x => IsCompl W x) (_ : ∃ q, IsCompl W q)) } →ₗ[K] K))
φ).fst
w =
↑φ w
[PROOFSTEP]
rfl
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W : Subspace K V
φ : Module.Dual K { x // x ∈ W }
w : V
hw : w ∈ W
⊢ ↑(↑(dualLift W) φ) w = ↑φ { val := w, property := hw }
[PROOFSTEP]
convert dualLift_of_subtype ⟨w, hw⟩
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W✝ W : Subspace K V
⊢ comp (dualRestrict W) (dualLift W) = 1
[PROOFSTEP]
ext φ x
[GOAL]
case h.h
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W✝ W : Subspace K V
φ : Module.Dual K { x // x ∈ W }
x : { x // x ∈ W }
⊢ ↑(↑(comp (dualRestrict W) (dualLift W)) φ) x = ↑(↑1 φ) x
[PROOFSTEP]
simp
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W✝ W : Subspace K V
x : Module.Dual K { x // x ∈ W }
⊢ ↑(comp (dualRestrict W) (dualLift W)) x = x
[PROOFSTEP]
rw [dualRestrict_comp_dualLift]
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W✝ W : Subspace K V
x : Module.Dual K { x // x ∈ W }
⊢ ↑1 x = x
[PROOFSTEP]
rfl
[GOAL]
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W✝ W : Subspace K V
φ : Module.Dual K V
⊢ ↑(quotAnnihilatorEquiv W) (Submodule.Quotient.mk φ) = ↑(dualRestrict W) φ
[PROOFSTEP]
ext
[GOAL]
case h
K : Type u
V : Type v
inst✝² : Field K
inst✝¹ : AddCommGroup V
inst✝ : Module K V
W✝ W : Subspace K V
φ : Module.Dual K V
x✝ : { x // x ∈ W }
⊢ ↑(↑(quotAnnihilatorEquiv W) (Submodule.Quotient.mk φ)) x✝ = ↑(↑(dualRestrict W) φ) x✝
[PROOFSTEP]
rfl
[GOAL]
K : Type u
V : Type v
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
W : Subspace K V
V₁ : Type u_1
inst✝¹ : AddCommGroup V₁
inst✝ : Module K V₁
H : FiniteDimensional K V
⊢ FiniteDimensional K (Module.Dual K V)
[PROOFSTEP]
infer_instance
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K V
⊢ dualAnnihilator (dualAnnihilator W) = ↑(Module.mapEvalEquiv K V) W
[PROOFSTEP]
have : _ = W := Subspace.dualAnnihilator_dualCoannihilator_eq
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K V
this : dualCoannihilator (dualAnnihilator W) = W
⊢ dualAnnihilator (dualAnnihilator W) = ↑(Module.mapEvalEquiv K V) W
[PROOFSTEP]
rw [dualCoannihilator, ← Module.mapEvalEquiv_symm_apply] at this
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K V
this : ↑(OrderIso.symm (Module.mapEvalEquiv K V)) (dualAnnihilator (dualAnnihilator W)) = W
⊢ dualAnnihilator (dualAnnihilator W) = ↑(Module.mapEvalEquiv K V) W
[PROOFSTEP]
rwa [← OrderIso.symm_apply_eq]
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
⊢ finrank K (Module.Dual K V) = finrank K V
[PROOFSTEP]
classical exact LinearEquiv.finrank_eq (Basis.ofVectorSpace K V).toDualEquiv.symm
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
⊢ finrank K (Module.Dual K V) = finrank K V
[PROOFSTEP]
exact LinearEquiv.finrank_eq (Basis.ofVectorSpace K V).toDualEquiv.symm
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
Φ : Subspace K (Module.Dual K V)
⊢ finrank K { x // x ∈ dualCoannihilator Φ } = finrank K { x // x ∈ dualAnnihilator Φ }
[PROOFSTEP]
rw [Submodule.dualCoannihilator, ← Module.evalEquiv_toLinearMap]
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
Φ : Subspace K (Module.Dual K V)
⊢ finrank K { x // x ∈ comap (↑(Module.evalEquiv K V)) (dualAnnihilator Φ) } = finrank K { x // x ∈ dualAnnihilator Φ }
[PROOFSTEP]
exact LinearEquiv.finrank_eq (LinearEquiv.ofSubmodule' _ _)
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K (Module.Dual K V)
⊢ finrank K { x // x ∈ W } + finrank K { x // x ∈ dualCoannihilator W } = finrank K V
[PROOFSTEP]
rw [finrank_dualCoannihilator_eq]
-- Porting note: LinearEquiv.finrank_eq needs help
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K (Module.Dual K V)
⊢ finrank K { x // x ∈ W } + finrank K { x // x ∈ dualAnnihilator W } = finrank K V
[PROOFSTEP]
let equiv := W.quotEquivAnnihilator
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K (Module.Dual K V)
equiv : (Module.Dual K V ⧸ W) ≃ₗ[K] { x // x ∈ dualAnnihilator W } := quotEquivAnnihilator W
⊢ finrank K { x // x ∈ W } + finrank K { x // x ∈ dualAnnihilator W } = finrank K V
[PROOFSTEP]
have eq := LinearEquiv.finrank_eq (R := K) (M := (Module.Dual K V) ⧸ W) (M₂ := { x // x ∈ dualAnnihilator W }) equiv
[GOAL]
K : Type u
V : Type v
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
W✝ : Subspace K V
V₁ : Type u_1
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : FiniteDimensional K V
inst✝ : FiniteDimensional K V₁
W : Subspace K (Module.Dual K V)
equiv : (Module.Dual K V ⧸ W) ≃ₗ[K] { x // x ∈ dualAnnihilator W } := quotEquivAnnihilator W
eq : finrank K (Module.Dual K V ⧸ W) = finrank K { x // x ∈ dualAnnihilator W }
⊢ finrank K { x // x ∈ W } + finrank K { x // x ∈ dualAnnihilator W } = finrank K V
[PROOFSTEP]
rw [eq.symm, add_comm, Submodule.finrank_quotient_add_finrank, Subspace.dual_finrank_eq]
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
⊢ ker (dualMap f) = Submodule.dualAnnihilator (range f)
[PROOFSTEP]
ext φ
[GOAL]
case h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
⊢ φ ∈ ker (dualMap f) ↔ φ ∈ Submodule.dualAnnihilator (range f)
[PROOFSTEP]
constructor
[GOAL]
case h.mp
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
⊢ φ ∈ ker (dualMap f) → φ ∈ Submodule.dualAnnihilator (range f)
[PROOFSTEP]
intro hφ
[GOAL]
case h.mpr
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
⊢ φ ∈ Submodule.dualAnnihilator (range f) → φ ∈ ker (dualMap f)
[PROOFSTEP]
intro hφ
[GOAL]
case h.mp
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : φ ∈ ker (dualMap f)
⊢ φ ∈ Submodule.dualAnnihilator (range f)
[PROOFSTEP]
rw [mem_ker] at hφ
[GOAL]
case h.mp
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : ↑(dualMap f) φ = 0
⊢ φ ∈ Submodule.dualAnnihilator (range f)
[PROOFSTEP]
rw [Submodule.mem_dualAnnihilator]
[GOAL]
case h.mp
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : ↑(dualMap f) φ = 0
⊢ ∀ (w : M₂), w ∈ range f → ↑φ w = 0
[PROOFSTEP]
rintro y ⟨x, rfl⟩
[GOAL]
case h.mp.intro
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : ↑(dualMap f) φ = 0
x : M₁
⊢ ↑φ (↑f x) = 0
[PROOFSTEP]
rw [← dualMap_apply, hφ, zero_apply]
[GOAL]
case h.mpr
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : φ ∈ Submodule.dualAnnihilator (range f)
⊢ φ ∈ ker (dualMap f)
[PROOFSTEP]
ext x
[GOAL]
case h.mpr.h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : φ ∈ Submodule.dualAnnihilator (range f)
x : M₁
⊢ ↑(↑(dualMap f) φ) x = ↑0 x
[PROOFSTEP]
rw [dualMap_apply]
[GOAL]
case h.mpr.h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : φ ∈ Submodule.dualAnnihilator (range f)
x : M₁
⊢ ↑φ (↑f x) = ↑0 x
[PROOFSTEP]
rw [Submodule.mem_dualAnnihilator] at hφ
[GOAL]
case h.mpr.h
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
φ : Dual R M₂
hφ : ∀ (w : M₂), w ∈ range f → ↑φ w = 0
x : M₁
⊢ ↑φ (↑f x) = ↑0 x
[PROOFSTEP]
exact hφ (f x) ⟨x, rfl⟩
[GOAL]
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
⊢ range (dualMap f) ≤ Submodule.dualAnnihilator (ker f)
[PROOFSTEP]
rintro _ ⟨ψ, rfl⟩
[GOAL]
case intro
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
ψ : Dual R M₂
⊢ ↑(dualMap f) ψ ∈ Submodule.dualAnnihilator (ker f)
[PROOFSTEP]
simp_rw [Submodule.mem_dualAnnihilator, mem_ker]
[GOAL]
case intro
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
ψ : Dual R M₂
⊢ ∀ (w : M₁), ↑f w = 0 → ↑(↑(dualMap f) ψ) w = 0
[PROOFSTEP]
rintro x hx
[GOAL]
case intro
R : Type u
inst✝⁴ : CommSemiring R
M₁ : Type v
M₂ : Type v'
inst✝³ : AddCommMonoid M₁
inst✝² : Module R M₁
inst✝¹ : AddCommMonoid M₂
inst✝ : Module R M₂
f : M₁ →ₗ[R] M₂
ψ : Dual R M₂
x : M₁
hx : ↑f x = 0
⊢ ↑(↑(dualMap f) ψ) x = 0
[PROOFSTEP]
rw [dualMap_apply, hx, map_zero]
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
⊢ W ≤ LinearMap.ker (LinearMap.flip (LinearMap.domRestrict (dualPairing R M) (dualAnnihilator W)))
[PROOFSTEP]
intro w hw
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
w : M
hw : w ∈ W
⊢ w ∈ LinearMap.ker (LinearMap.flip (LinearMap.domRestrict (dualPairing R M) (dualAnnihilator W)))
[PROOFSTEP]
ext ⟨φ, hφ⟩
[GOAL]
case h.mk
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
w : M
hw : w ∈ W
φ : Dual R M
hφ : φ ∈ dualAnnihilator W
⊢ ↑(↑(LinearMap.flip (LinearMap.domRestrict (dualPairing R M) (dualAnnihilator W))) w) { val := φ, property := hφ } =
↑0 { val := φ, property := hφ }
[PROOFSTEP]
exact (mem_dualAnnihilator φ).mp hφ w hw
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ ψ : { x // x ∈ dualAnnihilator W }
h : (fun φ => ↑↑φ) φ = (fun φ => ↑↑φ) ψ
⊢ φ = ψ
[PROOFSTEP]
ext
[GOAL]
case a.h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ ψ : { x // x ∈ dualAnnihilator W }
h : (fun φ => ↑↑φ) φ = (fun φ => ↑↑φ) ψ
x✝ : M
⊢ ↑↑φ x✝ = ↑↑ψ x✝
[PROOFSTEP]
simp only [Function.funext_iff] at h
[GOAL]
case a.h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ ψ : { x // x ∈ dualAnnihilator W }
x✝ : M
h : ∀ (a : M), ↑↑φ a = ↑↑ψ a
⊢ ↑↑φ x✝ = ↑↑ψ x✝
[PROOFSTEP]
exact h _
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
⊢ LinearMap.range (LinearMap.dualMap (mkQ W)) = dualAnnihilator W
[PROOFSTEP]
ext φ
[GOAL]
case h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ : Dual R M
⊢ φ ∈ LinearMap.range (LinearMap.dualMap (mkQ W)) ↔ φ ∈ dualAnnihilator W
[PROOFSTEP]
rw [LinearMap.mem_range]
[GOAL]
case h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ : Dual R M
⊢ (∃ y, ↑(LinearMap.dualMap (mkQ W)) y = φ) ↔ φ ∈ dualAnnihilator W
[PROOFSTEP]
constructor
[GOAL]
case h.mp
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ : Dual R M
⊢ (∃ y, ↑(LinearMap.dualMap (mkQ W)) y = φ) → φ ∈ dualAnnihilator W
[PROOFSTEP]
rintro ⟨ψ, rfl⟩
[GOAL]
case h.mp.intro
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
ψ : Dual R (M ⧸ W)
⊢ ↑(LinearMap.dualMap (mkQ W)) ψ ∈ dualAnnihilator W
[PROOFSTEP]
have := LinearMap.mem_range_self W.mkQ.dualMap ψ
[GOAL]
case h.mp.intro
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
ψ : Dual R (M ⧸ W)
this : ↑(LinearMap.dualMap (mkQ W)) ψ ∈ LinearMap.range (LinearMap.dualMap (mkQ W))
⊢ ↑(LinearMap.dualMap (mkQ W)) ψ ∈ dualAnnihilator W
[PROOFSTEP]
simpa only [ker_mkQ] using LinearMap.range_dualMap_le_dualAnnihilator_ker W.mkQ this
[GOAL]
case h.mpr
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ : Dual R M
⊢ φ ∈ dualAnnihilator W → ∃ y, ↑(LinearMap.dualMap (mkQ W)) y = φ
[PROOFSTEP]
intro hφ
[GOAL]
case h.mpr
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
φ : Dual R M
hφ : φ ∈ dualAnnihilator W
⊢ ∃ y, ↑(LinearMap.dualMap (mkQ W)) y = φ
[PROOFSTEP]
exists W.dualCopairing ⟨φ, hφ⟩
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
⊢ LinearMap.comp
(LinearMap.codRestrict (dualAnnihilator W) (LinearMap.dualMap (mkQ W))
(_ : ∀ (φ : Dual R (M ⧸ W)), ↑(LinearMap.dualMap (mkQ W)) φ ∈ dualAnnihilator W))
(dualCopairing W) =
LinearMap.id
[PROOFSTEP]
ext
[GOAL]
case h.a.h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
x✝¹ : { x // x ∈ dualAnnihilator W }
x✝ : M
⊢ ↑↑(↑(LinearMap.comp
(LinearMap.codRestrict (dualAnnihilator W) (LinearMap.dualMap (mkQ W))
(_ : ∀ (φ : Dual R (M ⧸ W)), ↑(LinearMap.dualMap (mkQ W)) φ ∈ dualAnnihilator W))
(dualCopairing W))
x✝¹)
x✝ =
↑↑(↑LinearMap.id x✝¹) x✝
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
⊢ LinearMap.comp (dualCopairing W)
(LinearMap.codRestrict (dualAnnihilator W) (LinearMap.dualMap (mkQ W))
(_ : ∀ (φ : Dual R (M ⧸ W)), ↑(LinearMap.dualMap (mkQ W)) φ ∈ dualAnnihilator W)) =
LinearMap.id
[PROOFSTEP]
ext
[GOAL]
case h.h.h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
W : Submodule R M
x✝¹ : Dual R (M ⧸ W)
x✝ : M
⊢ ↑(LinearMap.comp
(↑(LinearMap.comp (dualCopairing W)
(LinearMap.codRestrict (dualAnnihilator W) (LinearMap.dualMap (mkQ W))
(_ : ∀ (φ : Dual R (M ⧸ W)), ↑(LinearMap.dualMap (mkQ W)) φ ∈ dualAnnihilator W)))
x✝¹)
(mkQ W))
x✝ =
↑(LinearMap.comp (↑LinearMap.id x✝¹) (mkQ W)) x✝
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
⊢ range (dualMap f) = dualAnnihilator (ker f)
[PROOFSTEP]
rw [← f.ker.range_dualMap_mkQ_eq]
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
⊢ range (dualMap f) = range (dualMap (mkQ (ker f)))
[PROOFSTEP]
let f' := LinearMap.quotKerEquivOfSurjective f hf
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
f' : (M ⧸ ker f) ≃ₗ[R] M' := quotKerEquivOfSurjective f hf
⊢ range (dualMap f) = range (dualMap (mkQ (ker f)))
[PROOFSTEP]
trans LinearMap.range (f.dualMap.comp f'.symm.dualMap.toLinearMap)
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
f' : (M ⧸ ker f) ≃ₗ[R] M' := quotKerEquivOfSurjective f hf
⊢ range (dualMap f) = range (comp (dualMap f) ↑(LinearEquiv.dualMap (LinearEquiv.symm f')))
[PROOFSTEP]
rw [LinearMap.range_comp_of_range_eq_top]
[GOAL]
case hf
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
f' : (M ⧸ ker f) ≃ₗ[R] M' := quotKerEquivOfSurjective f hf
⊢ range ↑(LinearEquiv.dualMap (LinearEquiv.symm f')) = ⊤
[PROOFSTEP]
apply LinearEquiv.range
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
f' : (M ⧸ ker f) ≃ₗ[R] M' := quotKerEquivOfSurjective f hf
⊢ range (comp (dualMap f) ↑(LinearEquiv.dualMap (LinearEquiv.symm f'))) = range (dualMap (mkQ (ker f)))
[PROOFSTEP]
apply congr_arg
[GOAL]
case h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
f' : (M ⧸ ker f) ≃ₗ[R] M' := quotKerEquivOfSurjective f hf
⊢ comp (dualMap f) ↑(LinearEquiv.dualMap (LinearEquiv.symm f')) = dualMap (mkQ (ker f))
[PROOFSTEP]
ext φ x
[GOAL]
case h.h.h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑f
f' : (M ⧸ ker f) ≃ₗ[R] M' := quotKerEquivOfSurjective f hf
φ : Dual R (M ⧸ ker f)
x : M
⊢ ↑(↑(comp (dualMap f) ↑(LinearEquiv.dualMap (LinearEquiv.symm f'))) φ) x = ↑(↑(dualMap (mkQ (ker f))) φ) x
[PROOFSTEP]
simp only [LinearMap.coe_comp, LinearEquiv.coe_toLinearMap, LinearMap.dualMap_apply, LinearEquiv.dualMap_apply,
mkQ_apply, LinearMap.quotKerEquivOfSurjective, LinearEquiv.trans_symm, LinearEquiv.trans_apply,
LinearEquiv.ofTop_symm_apply, LinearMap.quotKerEquivRange_symm_apply_image, mkQ_apply, Function.comp]
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
⊢ range (dualMap f) = dualAnnihilator (ker f)
[PROOFSTEP]
have rr_surj : Function.Surjective f.rangeRestrict := by rw [← LinearMap.range_eq_top, LinearMap.range_rangeRestrict]
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
⊢ Function.Surjective ↑(rangeRestrict f)
[PROOFSTEP]
rw [← LinearMap.range_eq_top, LinearMap.range_rangeRestrict]
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
⊢ range (dualMap f) = dualAnnihilator (ker f)
[PROOFSTEP]
have := range_dualMap_eq_dualAnnihilator_ker_of_surjective f.rangeRestrict rr_surj
[GOAL]
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
this : range (dualMap (rangeRestrict f)) = dualAnnihilator (ker (rangeRestrict f))
⊢ range (dualMap f) = dualAnnihilator (ker f)
[PROOFSTEP]
convert this using 1
-- Porting note: broken dot notation lean4#1910
[GOAL]
case h.e'_2
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
this : range (dualMap (rangeRestrict f)) = dualAnnihilator (ker (rangeRestrict f))
⊢ range (dualMap f) = range (dualMap (rangeRestrict f))
[PROOFSTEP]
change LinearMap.range ((Submodule.subtype <| LinearMap.range f).comp f.rangeRestrict).dualMap = _
[GOAL]
case h.e'_2
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
this : range (dualMap (rangeRestrict f)) = dualAnnihilator (ker (rangeRestrict f))
⊢ range (dualMap (comp (Submodule.subtype (range f)) (rangeRestrict f))) = range (dualMap (rangeRestrict f))
[PROOFSTEP]
rw [← LinearMap.dualMap_comp_dualMap, LinearMap.range_comp_of_range_eq_top]
[GOAL]
case h.e'_2.hf
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
this : range (dualMap (rangeRestrict f)) = dualAnnihilator (ker (rangeRestrict f))
⊢ range (dualMap (Submodule.subtype (range f))) = ⊤
[PROOFSTEP]
rwa [LinearMap.range_eq_top]
[GOAL]
case h.e'_3
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
this : range (dualMap (rangeRestrict f)) = dualAnnihilator (ker (rangeRestrict f))
⊢ dualAnnihilator (ker f) = dualAnnihilator (ker (rangeRestrict f))
[PROOFSTEP]
apply congr_arg
[GOAL]
case h.e'_3.h
R : Type u_1
M : Type u_2
M' : Type u_3
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup M'
inst✝ : Module R M'
f : M →ₗ[R] M'
hf : Function.Surjective ↑(dualMap (Submodule.subtype (range f)))
rr_surj : Function.Surjective ↑(rangeRestrict f)
this : range (dualMap (rangeRestrict f)) = dualAnnihilator (ker (rangeRestrict f))
⊢ ker f = ker (rangeRestrict f)
[PROOFSTEP]
exact (LinearMap.ker_rangeRestrict f).symm
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
⊢ Function.Surjective ↑(dualMap f)
[PROOFSTEP]
intro φ
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
φ : Dual K V₁
⊢ ∃ a, ↑(dualMap f) a = φ
[PROOFSTEP]
let f' := LinearEquiv.ofInjective f hf
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
φ : Dual K V₁
f' : V₁ ≃ₗ[K] { x // x ∈ range f } := LinearEquiv.ofInjective f hf
⊢ ∃ a, ↑(dualMap f) a = φ
[PROOFSTEP]
use Subspace.dualLift (range f) (f'.symm.dualMap φ)
[GOAL]
case h
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
φ : Dual K V₁
f' : V₁ ≃ₗ[K] { x // x ∈ range f } := LinearEquiv.ofInjective f hf
⊢ ↑(dualMap f) (↑(Subspace.dualLift (range f)) (↑(LinearEquiv.dualMap (LinearEquiv.symm f')) φ)) = φ
[PROOFSTEP]
ext x
[GOAL]
case h.h
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
φ : Dual K V₁
f' : V₁ ≃ₗ[K] { x // x ∈ range f } := LinearEquiv.ofInjective f hf
x : V₁
⊢ ↑(↑(dualMap f) (↑(Subspace.dualLift (range f)) (↑(LinearEquiv.dualMap (LinearEquiv.symm f')) φ))) x = ↑φ x
[PROOFSTEP]
rw [LinearMap.dualMap_apply, Subspace.dualLift_of_mem (mem_range_self f x), LinearEquiv.dualMap_apply]
[GOAL]
case h.h
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
φ : Dual K V₁
f' : V₁ ≃ₗ[K] { x // x ∈ range f } := LinearEquiv.ofInjective f hf
x : V₁
⊢ ↑φ (↑(LinearEquiv.symm f') { val := ↑f x, property := (_ : ↑f x ∈ range f) }) = ↑φ x
[PROOFSTEP]
congr 1
[GOAL]
case h.h.h.e_6.h
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
hf : Function.Injective ↑f
φ : Dual K V₁
f' : V₁ ≃ₗ[K] { x // x ∈ range f } := LinearEquiv.ofInjective f hf
x : V₁
⊢ ↑(LinearEquiv.symm f') { val := ↑f x, property := (_ : ↑f x ∈ range f) } = x
[PROOFSTEP]
exact LinearEquiv.symm_apply_apply f' x
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
f : V₁ →ₗ[K] V₂
⊢ Function.Surjective ↑(dualMap f) ↔ Function.Injective ↑f
[PROOFSTEP]
rw [← LinearMap.range_eq_top, range_dualMap_eq_dualAnnihilator_ker, ← Submodule.dualAnnihilator_bot,
Subspace.dualAnnihilator_inj, LinearMap.ker_eq_bot]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ Submodule.dualPairing W = ↑(quotAnnihilatorEquiv W)
[PROOFSTEP]
ext
[GOAL]
case h.h.h
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
x✝¹ : Dual K V₁
x✝ : { x // x ∈ W }
⊢ ↑(↑(LinearMap.comp (Submodule.dualPairing W) (mkQ (dualAnnihilator W))) x✝¹) x✝ =
↑(↑(LinearMap.comp (↑(quotAnnihilatorEquiv W)) (mkQ (dualAnnihilator W))) x✝¹) x✝
[PROOFSTEP]
rfl
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.Nondegenerate (Submodule.dualPairing W)
[PROOFSTEP]
constructor
[GOAL]
case left
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.SeparatingLeft (Submodule.dualPairing W)
[PROOFSTEP]
rw [LinearMap.separatingLeft_iff_ker_eq_bot, dualPairing_eq]
[GOAL]
case left
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.ker ↑(quotAnnihilatorEquiv W) = ⊥
[PROOFSTEP]
apply LinearEquiv.ker
[GOAL]
case right
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.SeparatingRight (Submodule.dualPairing W)
[PROOFSTEP]
intro x h
[GOAL]
case right
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
x : { x // x ∈ W }
h : ∀ (x_1 : Dual K V₁ ⧸ dualAnnihilator W), ↑(↑(Submodule.dualPairing W) x_1) x = 0
⊢ x = 0
[PROOFSTEP]
rw [← forall_dual_apply_eq_zero_iff K x]
[GOAL]
case right
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
x : { x // x ∈ W }
h : ∀ (x_1 : Dual K V₁ ⧸ dualAnnihilator W), ↑(↑(Submodule.dualPairing W) x_1) x = 0
⊢ ∀ (φ : Dual K { x // x ∈ W }), ↑φ x = 0
[PROOFSTEP]
intro φ
[GOAL]
case right
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
x : { x // x ∈ W }
h : ∀ (x_1 : Dual K V₁ ⧸ dualAnnihilator W), ↑(↑(Submodule.dualPairing W) x_1) x = 0
φ : Dual K { x // x ∈ W }
⊢ ↑φ x = 0
[PROOFSTEP]
simpa only [Submodule.dualPairing_apply, dualLift_of_subtype] using h (Submodule.Quotient.mk (W.dualLift φ))
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.Nondegenerate (dualCopairing W)
[PROOFSTEP]
constructor
[GOAL]
case left
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.SeparatingLeft (dualCopairing W)
[PROOFSTEP]
rw [LinearMap.separatingLeft_iff_ker_eq_bot, dualCopairing_eq]
[GOAL]
case left
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.ker ↑(LinearEquiv.symm (dualQuotEquivDualAnnihilator W)) = ⊥
[PROOFSTEP]
apply LinearEquiv.ker
[GOAL]
case right
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
⊢ LinearMap.SeparatingRight (dualCopairing W)
[PROOFSTEP]
rintro ⟨x⟩
[GOAL]
case right.mk
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
y✝ : V₁ ⧸ W
x : V₁
⊢ (∀ (x_1 : { x // x ∈ dualAnnihilator W }), ↑(↑(dualCopairing W) x_1) (Quot.mk Setoid.r x) = 0) →
Quot.mk Setoid.r x = 0
[PROOFSTEP]
simp only [Quotient.quot_mk_eq_mk, dualCopairing_apply, Quotient.mk_eq_zero]
[GOAL]
case right.mk
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
y✝ : V₁ ⧸ W
x : V₁
⊢ (∀ (x_1 : { x // x ∈ dualAnnihilator W }), ↑x_1 x = 0) → x ∈ W
[PROOFSTEP]
rw [← forall_mem_dualAnnihilator_apply_eq_zero_iff, SetLike.forall]
[GOAL]
case right.mk
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : Subspace K V₁
y✝ : V₁ ⧸ W
x : V₁
⊢ (∀ (x_1 : Dual K V₁) (h : x_1 ∈ dualAnnihilator W), ↑{ val := x_1, property := h } x = 0) →
∀ (φ : Dual K V₁), φ ∈ dualAnnihilator W → ↑φ x = 0
[PROOFSTEP]
exact id
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
⊢ dualAnnihilator (W ⊓ W') = dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
refine' le_antisymm _ (sup_dualAnnihilator_le_inf W W')
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
⊢ dualAnnihilator (W ⊓ W') ≤ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
let F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' :=
(Submodule.mkQ W).prod
(Submodule.mkQ W')
-- Porting note: broken dot notation lean4#1910 LinearMap.ker
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
⊢ dualAnnihilator (W ⊓ W') ≤ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
have : LinearMap.ker F = W ⊓ W' := by simp only [LinearMap.ker_prod, ker_mkQ]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
⊢ LinearMap.ker F = W ⊓ W'
[PROOFSTEP]
simp only [LinearMap.ker_prod, ker_mkQ]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
⊢ dualAnnihilator (W ⊓ W') ≤ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
rw [← this, ← LinearMap.range_dualMap_eq_dualAnnihilator_ker]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
⊢ LinearMap.range (LinearMap.dualMap F) ≤ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
intro φ
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
φ : Dual K V₁
⊢ φ ∈ LinearMap.range (LinearMap.dualMap F) → φ ∈ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
rw [LinearMap.mem_range]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
φ : Dual K V₁
⊢ (∃ y, ↑(LinearMap.dualMap F) y = φ) → φ ∈ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
rintro ⟨x, rfl⟩
[GOAL]
case intro
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
x : Dual K ((V₁ ⧸ W) × V₁ ⧸ W')
⊢ ↑(LinearMap.dualMap F) x ∈ dualAnnihilator W ⊔ dualAnnihilator W'
[PROOFSTEP]
rw [Submodule.mem_sup]
[GOAL]
case intro
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
x : Dual K ((V₁ ⧸ W) × V₁ ⧸ W')
⊢ ∃ y, y ∈ dualAnnihilator W ∧ ∃ z, z ∈ dualAnnihilator W' ∧ y + z = ↑(LinearMap.dualMap F) x
[PROOFSTEP]
obtain ⟨⟨a, b⟩, rfl⟩ := (dualProdDualEquivDual K (V₁ ⧸ W) (V₁ ⧸ W')).surjective x
[GOAL]
case intro.intro.mk
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
a : Dual K (V₁ ⧸ W)
b : Dual K (V₁ ⧸ W')
⊢ ∃ y,
y ∈ dualAnnihilator W ∧
∃ z,
z ∈ dualAnnihilator W' ∧ y + z = ↑(LinearMap.dualMap F) (↑(dualProdDualEquivDual K (V₁ ⧸ W) (V₁ ⧸ W')) (a, b))
[PROOFSTEP]
obtain ⟨a', rfl⟩ := (dualQuotEquivDualAnnihilator W).symm.surjective a
[GOAL]
case intro.intro.mk.intro
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
b : Dual K (V₁ ⧸ W')
a' : { x // x ∈ dualAnnihilator W }
⊢ ∃ y,
y ∈ dualAnnihilator W ∧
∃ z,
z ∈ dualAnnihilator W' ∧
y + z =
↑(LinearMap.dualMap F)
(↑(dualProdDualEquivDual K (V₁ ⧸ W) (V₁ ⧸ W'))
(↑(LinearEquiv.symm (dualQuotEquivDualAnnihilator W)) a', b))
[PROOFSTEP]
obtain ⟨b', rfl⟩ := (dualQuotEquivDualAnnihilator W').symm.surjective b
[GOAL]
case intro.intro.mk.intro.intro
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
a' : { x // x ∈ dualAnnihilator W }
b' : { x // x ∈ dualAnnihilator W' }
⊢ ∃ y,
y ∈ dualAnnihilator W ∧
∃ z,
z ∈ dualAnnihilator W' ∧
y + z =
↑(LinearMap.dualMap F)
(↑(dualProdDualEquivDual K (V₁ ⧸ W) (V₁ ⧸ W'))
(↑(LinearEquiv.symm (dualQuotEquivDualAnnihilator W)) a',
↑(LinearEquiv.symm (dualQuotEquivDualAnnihilator W')) b'))
[PROOFSTEP]
use a', a'.property, b', b'.property
[GOAL]
case right
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
F : V₁ →ₗ[K] (V₁ ⧸ W) × V₁ ⧸ W' := LinearMap.prod (mkQ W) (mkQ W')
this : LinearMap.ker F = W ⊓ W'
a' : { x // x ∈ dualAnnihilator W }
b' : { x // x ∈ dualAnnihilator W' }
⊢ ↑a' + ↑b' =
↑(LinearMap.dualMap F)
(↑(dualProdDualEquivDual K (V₁ ⧸ W) (V₁ ⧸ W'))
(↑(LinearEquiv.symm (dualQuotEquivDualAnnihilator W)) a',
↑(LinearEquiv.symm (dualQuotEquivDualAnnihilator W')) b'))
[PROOFSTEP]
rfl
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
ι : Type u_1
inst✝ : _root_.Finite ι
W : ι → Subspace K V₁
⊢ dualAnnihilator (⨅ (i : ι), W i) = ⨆ (i : ι), dualAnnihilator (W i)
[PROOFSTEP]
revert ι
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
⊢ ∀ {ι : Type u_1} [inst : _root_.Finite ι] (W : ι → Subspace K V₁),
dualAnnihilator (⨅ (i : ι), W i) = ⨆ (i : ι), dualAnnihilator (W i)
[PROOFSTEP]
refine' @Finite.induction_empty_option _ _ _ _
[GOAL]
case refine'_1
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
⊢ ∀ {α β : Type u_1},
α ≃ β →
(∀ (W : α → Subspace K V₁), dualAnnihilator (⨅ (i : α), W i) = ⨆ (i : α), dualAnnihilator (W i)) →
∀ (W : β → Subspace K V₁), dualAnnihilator (⨅ (i : β), W i) = ⨆ (i : β), dualAnnihilator (W i)
[PROOFSTEP]
intro α β h hyp W
[GOAL]
case refine'_1
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
α β : Type u_1
h : α ≃ β
hyp : ∀ (W : α → Subspace K V₁), dualAnnihilator (⨅ (i : α), W i) = ⨆ (i : α), dualAnnihilator (W i)
W : β → Subspace K V₁
⊢ dualAnnihilator (⨅ (i : β), W i) = ⨆ (i : β), dualAnnihilator (W i)
[PROOFSTEP]
rw [← h.iInf_comp, hyp _, ← h.iSup_comp]
[GOAL]
case refine'_2
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
⊢ ∀ (W : PEmpty → Subspace K V₁), dualAnnihilator (⨅ (i : PEmpty), W i) = ⨆ (i : PEmpty), dualAnnihilator (W i)
[PROOFSTEP]
intro W
[GOAL]
case refine'_2
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W : PEmpty → Subspace K V₁
⊢ dualAnnihilator (⨅ (i : PEmpty), W i) = ⨆ (i : PEmpty), dualAnnihilator (W i)
[PROOFSTEP]
rw [iSup_of_empty', iInf_of_empty', sInf_empty, sSup_empty, dualAnnihilator_top]
[GOAL]
case refine'_3
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
⊢ ∀ {α : Type u_1} [inst : Fintype α],
(∀ (W : α → Subspace K V₁), dualAnnihilator (⨅ (i : α), W i) = ⨆ (i : α), dualAnnihilator (W i)) →
∀ (W : Option α → Subspace K V₁),
dualAnnihilator (⨅ (i : Option α), W i) = ⨆ (i : Option α), dualAnnihilator (W i)
[PROOFSTEP]
intro α _ h W
[GOAL]
case refine'_3
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
α : Type u_1
inst✝ : Fintype α
h : ∀ (W : α → Subspace K V₁), dualAnnihilator (⨅ (i : α), W i) = ⨆ (i : α), dualAnnihilator (W i)
W : Option α → Subspace K V₁
⊢ dualAnnihilator (⨅ (i : Option α), W i) = ⨆ (i : Option α), dualAnnihilator (W i)
[PROOFSTEP]
rw [iInf_option, iSup_option, dualAnnihilator_inf_eq, h]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
h : IsCompl W W'
⊢ IsCompl (dualAnnihilator W) (dualAnnihilator W')
[PROOFSTEP]
rw [isCompl_iff, disjoint_iff, codisjoint_iff] at h ⊢
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
h : W ⊓ W' = ⊥ ∧ W ⊔ W' = ⊤
⊢ dualAnnihilator W ⊓ dualAnnihilator W' = ⊥ ∧ dualAnnihilator W ⊔ dualAnnihilator W' = ⊤
[PROOFSTEP]
rw [← dualAnnihilator_inf_eq, ← dualAnnihilator_sup_eq, h.1, h.2, dualAnnihilator_top, dualAnnihilator_bot]
[GOAL]
K : Type u
inst✝⁴ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝³ : AddCommGroup V₁
inst✝² : Module K V₁
inst✝¹ : AddCommGroup V₂
inst✝ : Module K V₂
W W' : Subspace K V₁
h : W ⊓ W' = ⊥ ∧ W ⊔ W' = ⊤
⊢ ⊥ = ⊥ ∧ ⊤ = ⊤
[PROOFSTEP]
exact ⟨rfl, rfl⟩
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
⊢ finrank K { x // x ∈ range (dualMap f) } = finrank K { x // x ∈ range f }
[PROOFSTEP]
have that :=
Submodule.finrank_quotient_add_finrank
(LinearMap.range f)
-- Porting note: Again LinearEquiv.finrank_eq needs help
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K (V₂ ⧸ range f) + finrank K { x // x ∈ range f } = finrank K V₂
⊢ finrank K { x // x ∈ range (dualMap f) } = finrank K { x // x ∈ range f }
[PROOFSTEP]
let equiv := (Subspace.quotEquivAnnihilator <| LinearMap.range f)
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K (V₂ ⧸ range f) + finrank K { x // x ∈ range f } = finrank K V₂
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
⊢ finrank K { x // x ∈ range (dualMap f) } = finrank K { x // x ∈ range f }
[PROOFSTEP]
have eq :=
LinearEquiv.finrank_eq (R := K) (M := (V₂ ⧸ range f)) (M₂ := { x // x ∈ Submodule.dualAnnihilator (range f) }) equiv
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K (V₂ ⧸ range f) + finrank K { x // x ∈ range f } = finrank K V₂
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
⊢ finrank K { x // x ∈ range (dualMap f) } = finrank K { x // x ∈ range f }
[PROOFSTEP]
rw [eq, ← ker_dualMap_eq_dualAnnihilator_range] at that
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K V₂
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
⊢ finrank K { x // x ∈ range (dualMap f) } = finrank K { x // x ∈ range f }
[PROOFSTEP]
conv_rhs at that => rw [← Subspace.dual_finrank_eq]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K V₂
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
| finrank K V₂
[PROOFSTEP]
rw [← Subspace.dual_finrank_eq]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K V₂
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
| finrank K V₂
[PROOFSTEP]
rw [← Subspace.dual_finrank_eq]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K V₂
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
| finrank K V₂
[PROOFSTEP]
rw [← Subspace.dual_finrank_eq]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K (Dual K V₂)
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
⊢ finrank K { x // x ∈ range (dualMap f) } = finrank K { x // x ∈ range f }
[PROOFSTEP]
refine' add_left_injective (finrank K <| LinearMap.ker f.dualMap) _
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K (Dual K V₂)
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
⊢ (fun x => x + finrank K { x // x ∈ ker (dualMap f) }) (finrank K { x // x ∈ range (dualMap f) }) =
(fun x => x + finrank K { x // x ∈ ker (dualMap f) }) (finrank K { x // x ∈ range f })
[PROOFSTEP]
change _ + _ = _ + _
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
that : finrank K { x // x ∈ ker (dualMap f) } + finrank K { x // x ∈ range f } = finrank K (Dual K V₂)
equiv : (V₂ ⧸ range f) ≃ₗ[K] { x // x ∈ Submodule.dualAnnihilator (range f) } := Subspace.quotEquivAnnihilator (range f)
eq : finrank K (V₂ ⧸ range f) = finrank K { x // x ∈ Submodule.dualAnnihilator (range f) }
⊢ finrank K { x // x ∈ range (dualMap f) } + finrank K { x // x ∈ ker (dualMap f) } =
finrank K { x // x ∈ range f } + finrank K { x // x ∈ ker (dualMap f) }
[PROOFSTEP]
rw [finrank_range_add_finrank_ker f.dualMap, add_comm, that]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
⊢ Function.Injective ↑(dualMap f) ↔ Function.Surjective ↑f
[PROOFSTEP]
refine' ⟨_, fun h => dualMap_injective_of_surjective h⟩
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
⊢ Function.Injective ↑(dualMap f) → Function.Surjective ↑f
[PROOFSTEP]
rw [← range_eq_top, ← ker_eq_bot]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
⊢ ker (dualMap f) = ⊥ → range f = ⊤
[PROOFSTEP]
intro h
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
h : ker (dualMap f) = ⊥
⊢ range f = ⊤
[PROOFSTEP]
apply Submodule.eq_top_of_finrank_eq
[GOAL]
case h
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
h : ker (dualMap f) = ⊥
⊢ finrank K { x // x ∈ range f } = finrank K V₂
[PROOFSTEP]
rw [← finrank_eq_zero] at h
[GOAL]
case h
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
h : finrank K { x // x ∈ ker (dualMap f) } = 0
⊢ finrank K { x // x ∈ range f } = finrank K V₂
[PROOFSTEP]
rw [← add_zero (FiniteDimensional.finrank K <| LinearMap.range f), ← h, ←
LinearMap.finrank_range_dualMap_eq_finrank_range, LinearMap.finrank_range_add_finrank_ker, Subspace.dual_finrank_eq]
[GOAL]
K : Type u
inst✝⁵ : Field K
V₁ : Type v'
V₂ : Type v''
inst✝⁴ : AddCommGroup V₁
inst✝³ : Module K V₁
inst✝² : AddCommGroup V₂
inst✝¹ : Module K V₂
inst✝ : FiniteDimensional K V₂
f : V₁ →ₗ[K] V₂
⊢ Function.Bijective ↑(dualMap f) ↔ Function.Bijective ↑f
[PROOFSTEP]
simp_rw [Function.Bijective, dualMap_surjective_iff, dualMap_injective_iff, and_comm]
[GOAL]
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
f : Dual R (M ⊗[R] N)
⊢ ↑(dualDistribInvOfBasis b c) f =
∑ i : ι, ∑ j : κ, ↑f (↑b i ⊗ₜ[R] ↑c j) • ↑(Basis.dualBasis b) i ⊗ₜ[R] ↑(Basis.dualBasis c) j
[PROOFSTEP]
simp [dualDistribInvOfBasis]
[GOAL]
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ comp (dualDistrib R M N) (dualDistribInvOfBasis b c) = LinearMap.id
[PROOFSTEP]
apply (b.tensorProduct c).dualBasis.ext
[GOAL]
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ ∀ (i : ι × κ),
↑(comp (dualDistrib R M N) (dualDistribInvOfBasis b c)) (↑(Basis.dualBasis (Basis.tensorProduct b c)) i) =
↑LinearMap.id (↑(Basis.dualBasis (Basis.tensorProduct b c)) i)
[PROOFSTEP]
rintro ⟨i, j⟩
[GOAL]
case mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ↑(comp (dualDistrib R M N) (dualDistribInvOfBasis b c)) (↑(Basis.dualBasis (Basis.tensorProduct b c)) (i, j)) =
↑LinearMap.id (↑(Basis.dualBasis (Basis.tensorProduct b c)) (i, j))
[PROOFSTEP]
apply (b.tensorProduct c).ext
[GOAL]
case mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (i_1 : ι × κ),
↑(↑(comp (dualDistrib R M N) (dualDistribInvOfBasis b c)) (↑(Basis.dualBasis (Basis.tensorProduct b c)) (i, j)))
(↑(Basis.tensorProduct b c) i_1) =
↑(↑LinearMap.id (↑(Basis.dualBasis (Basis.tensorProduct b c)) (i, j))) (↑(Basis.tensorProduct b c) i_1)
[PROOFSTEP]
rintro ⟨i', j'⟩
[GOAL]
case mk.mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ↑(↑(comp (dualDistrib R M N) (dualDistribInvOfBasis b c)) (↑(Basis.dualBasis (Basis.tensorProduct b c)) (i, j)))
(↑(Basis.tensorProduct b c) (i', j')) =
↑(↑LinearMap.id (↑(Basis.dualBasis (Basis.tensorProduct b c)) (i, j))) (↑(Basis.tensorProduct b c) (i', j'))
[PROOFSTEP]
simp only [dualDistrib, Basis.coe_dualBasis, coe_comp, Function.comp_apply, dualDistribInvOfBasis_apply,
Basis.coord_apply, Basis.tensorProduct_repr_tmul_apply, Basis.repr_self, ne_eq, LinearMap.map_sum, map_smul,
homTensorHomMap_apply, compRight_apply, Basis.tensorProduct_apply, coeFn_sum, Finset.sum_apply, smul_apply,
LinearEquiv.coe_coe, map_tmul, lid_tmul, smul_eq_mul, id_coe, id_eq]
[GOAL]
case mk.mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∑ x : ι,
∑ x_1 : κ,
↑(Finsupp.single x 1) i * ↑(Finsupp.single x_1 1) j * (↑(Finsupp.single i' 1) x * ↑(Finsupp.single j' 1) x_1) =
↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j
[PROOFSTEP]
rw [Finset.sum_eq_single i, Finset.sum_eq_single j]
[GOAL]
case mk.mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j) =
↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : κ),
b ∈ Finset.univ →
b ≠ j →
↑(Finsupp.single i 1) i * ↑(Finsupp.single b 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) b) = 0
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬j ∈ Finset.univ →
↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j) = 0
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : ι),
b ∈ Finset.univ →
b ≠ i →
∑ x : κ,
↑(Finsupp.single b 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) b * ↑(Finsupp.single j' 1) x) =
0
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, ↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
simp
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : κ),
b ∈ Finset.univ →
b ≠ j →
↑(Finsupp.single i 1) i * ↑(Finsupp.single b 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) b) = 0
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬j ∈ Finset.univ →
↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j) = 0
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : ι),
b ∈ Finset.univ →
b ≠ i →
∑ x : κ,
↑(Finsupp.single b 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) b * ↑(Finsupp.single j' 1) x) =
0
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, ↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
all_goals {intros; simp [*] at *
}
-- Porting note: introduced to help with timeout in dualDistribEquivOfBasis
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : κ),
b ∈ Finset.univ →
b ≠ j →
↑(Finsupp.single i 1) i * ↑(Finsupp.single b 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) b) = 0
[PROOFSTEP]
{intros; simp [*] at *
}
-- Porting note: introduced to help with timeout in dualDistribEquivOfBasis
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : κ),
b ∈ Finset.univ →
b ≠ j →
↑(Finsupp.single i 1) i * ↑(Finsupp.single b 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) b) = 0
[PROOFSTEP]
intros
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' b✝ : κ
a✝¹ : b✝ ∈ Finset.univ
a✝ : b✝ ≠ j
⊢ ↑(Finsupp.single i 1) i * ↑(Finsupp.single b✝ 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) b✝) = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬j ∈ Finset.univ →
↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j) = 0
[PROOFSTEP]
{intros; simp [*] at *
}
-- Porting note: introduced to help with timeout in dualDistribEquivOfBasis
[GOAL]
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬j ∈ Finset.univ →
↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j) = 0
[PROOFSTEP]
intros
[GOAL]
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
a✝ : ¬j ∈ Finset.univ
⊢ ↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) j) = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : ι),
b ∈ Finset.univ →
b ≠ i →
∑ x : κ,
↑(Finsupp.single b 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) b * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
{intros; simp [*] at *
}
-- Porting note: introduced to help with timeout in dualDistribEquivOfBasis
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ∀ (b : ι),
b ∈ Finset.univ →
b ≠ i →
∑ x : κ,
↑(Finsupp.single b 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) b * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
intros
[GOAL]
case mk.mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
b✝ : ι
a✝¹ : b✝ ∈ Finset.univ
a✝ : b✝ ≠ i
⊢ ∑ x : κ, ↑(Finsupp.single b✝ 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) b✝ * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
simp [*] at *
[GOAL]
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, ↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
{intros; simp [*] at *
}
-- Porting note: introduced to help with timeout in dualDistribEquivOfBasis
[GOAL]
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, ↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) x) =
0
[PROOFSTEP]
intros
[GOAL]
case mk.mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
i' : ι
j' : κ
a✝ : ¬i ∈ Finset.univ
⊢ ∑ x : κ, ↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j * (↑(Finsupp.single i' 1) i * ↑(Finsupp.single j' 1) x) = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ comp (dualDistribInvOfBasis b c) (dualDistrib R M N) = LinearMap.id
[PROOFSTEP]
apply (b.dualBasis.tensorProduct c.dualBasis).ext
[GOAL]
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ ∀ (i : ι × κ),
↑(comp (dualDistribInvOfBasis b c) (dualDistrib R M N))
(↑(Basis.tensorProduct (Basis.dualBasis b) (Basis.dualBasis c)) i) =
↑LinearMap.id (↑(Basis.tensorProduct (Basis.dualBasis b) (Basis.dualBasis c)) i)
[PROOFSTEP]
rintro ⟨i, j⟩
[GOAL]
case mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ↑(comp (dualDistribInvOfBasis b c) (dualDistrib R M N))
(↑(Basis.tensorProduct (Basis.dualBasis b) (Basis.dualBasis c)) (i, j)) =
↑LinearMap.id (↑(Basis.tensorProduct (Basis.dualBasis b) (Basis.dualBasis c)) (i, j))
[PROOFSTEP]
simp only [Basis.tensorProduct_apply, Basis.coe_dualBasis, coe_comp, Function.comp_apply, dualDistribInvOfBasis_apply,
dualDistrib_apply, Basis.coord_apply, Basis.repr_self, ne_eq, id_coe, id_eq]
[GOAL]
case mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∑ x : ι, ∑ x_1 : κ, (↑(Finsupp.single x 1) i * ↑(Finsupp.single x_1 1) j) • Basis.coord b x ⊗ₜ[R] Basis.coord c x_1 =
Basis.coord b i ⊗ₜ[R] Basis.coord c j
[PROOFSTEP]
rw [Finset.sum_eq_single i, Finset.sum_eq_single j]
[GOAL]
case mk
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ (↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c j =
Basis.coord b i ⊗ₜ[R] Basis.coord c j
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : κ),
b_1 ∈ Finset.univ →
b_1 ≠ j → (↑(Finsupp.single i 1) i * ↑(Finsupp.single b_1 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c b_1 = 0
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬j ∈ Finset.univ → (↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c j = 0
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : ι),
b_1 ∈ Finset.univ →
b_1 ≠ i →
∑ x : κ, (↑(Finsupp.single b_1 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b b_1 ⊗ₜ[R] Basis.coord c x = 0
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, (↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
simp
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : κ),
b_1 ∈ Finset.univ →
b_1 ≠ j → (↑(Finsupp.single i 1) i * ↑(Finsupp.single b_1 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c b_1 = 0
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬j ∈ Finset.univ → (↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c j = 0
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : ι),
b_1 ∈ Finset.univ →
b_1 ≠ i →
∑ x : κ, (↑(Finsupp.single b_1 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b b_1 ⊗ₜ[R] Basis.coord c x = 0
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, (↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
all_goals {intros; simp [*] at *
}
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : κ),
b_1 ∈ Finset.univ →
b_1 ≠ j → (↑(Finsupp.single i 1) i * ↑(Finsupp.single b_1 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c b_1 = 0
[PROOFSTEP]
{intros; simp [*] at *
}
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : κ),
b_1 ∈ Finset.univ →
b_1 ≠ j → (↑(Finsupp.single i 1) i * ↑(Finsupp.single b_1 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c b_1 = 0
[PROOFSTEP]
intros
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j b✝ : κ
a✝¹ : b✝ ∈ Finset.univ
a✝ : b✝ ≠ j
⊢ (↑(Finsupp.single i 1) i * ↑(Finsupp.single b✝ 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c b✝ = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬j ∈ Finset.univ → (↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c j = 0
[PROOFSTEP]
{intros; simp [*] at *
}
[GOAL]
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬j ∈ Finset.univ → (↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c j = 0
[PROOFSTEP]
intros
[GOAL]
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
a✝ : ¬j ∈ Finset.univ
⊢ (↑(Finsupp.single i 1) i * ↑(Finsupp.single j 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c j = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : ι),
b_1 ∈ Finset.univ →
b_1 ≠ i →
∑ x : κ, (↑(Finsupp.single b_1 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b b_1 ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
{intros; simp [*] at *
}
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ∀ (b_1 : ι),
b_1 ∈ Finset.univ →
b_1 ≠ i →
∑ x : κ, (↑(Finsupp.single b_1 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b b_1 ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
intros
[GOAL]
case mk.h₀
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
b✝ : ι
a✝¹ : b✝ ∈ Finset.univ
a✝ : b✝ ≠ i
⊢ ∑ x : κ, (↑(Finsupp.single b✝ 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b b✝ ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, (↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
{intros; simp [*] at *
}
[GOAL]
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
⊢ ¬i ∈ Finset.univ →
∑ x : κ, (↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
intros
[GOAL]
case mk.h₁
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
i : ι
j : κ
a✝ : ¬i ∈ Finset.univ
⊢ ∑ x : κ, (↑(Finsupp.single i 1) i * ↑(Finsupp.single x 1) j) • Basis.coord b i ⊗ₜ[R] Basis.coord c x = 0
[PROOFSTEP]
simp [*] at *
[GOAL]
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ Dual R M ⊗[R] Dual R N ≃ₗ[R] Dual R (M ⊗[R] N)
[PROOFSTEP]
refine' LinearEquiv.ofLinear (dualDistrib R M N) (dualDistribInvOfBasis b c) _ _
[GOAL]
case refine'_1
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ comp (dualDistrib R M N) (dualDistribInvOfBasis b c) = LinearMap.id
[PROOFSTEP]
exact dualDistrib_dualDistribInvOfBasis_left_inverse _ _
[GOAL]
case refine'_2
R : Type u_1
A : Type u_2
M : Type u_3
N : Type u_4
ι : Type u_5
κ : Type u_6
inst✝⁸ : DecidableEq ι
inst✝⁷ : DecidableEq κ
inst✝⁶ : Fintype ι
inst✝⁵ : Fintype κ
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : AddCommGroup N
inst✝¹ : Module R M
inst✝ : Module R N
b : Basis ι R M
c : Basis κ R N
⊢ comp (dualDistribInvOfBasis b c) (dualDistrib R M N) = LinearMap.id
[PROOFSTEP]
exact dualDistrib_dualDistribInvOfBasis_right_inverse _ _
| {"mathlib_filename": "Mathlib.LinearAlgebra.Dual", "llama_tokens": 76733} |
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
r : R
⊢ ↑(ι (Q' Q)) (m, r) = ↑(v Q) m + r • e0 Q
[PROOFSTEP]
rw [e0, v, LinearMap.comp_apply, LinearMap.inl_apply, ← LinearMap.map_smul, Prod.smul_mk, smul_zero, smul_eq_mul,
mul_one, ← LinearMap.map_add, Prod.mk_add_mk, zero_add, add_zero]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ ↑(algebraMap R (CliffordAlgebra (Q' Q))) (↑(Q' Q) (0, 1)) = -1
[PROOFSTEP]
simp
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(algebraMap R (CliffordAlgebra (Q' Q))) (↑(Q' Q) (↑(LinearMap.inl R M R) m)) =
↑(algebraMap R (CliffordAlgebra (Q' Q))) (↑Q m)
[PROOFSTEP]
simp
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ -(e0 Q * ↑(v Q) m) = ↑(v Q) m * e0 Q
[PROOFSTEP]
refine' neg_eq_of_add_eq_zero_right ((ι_mul_ι_add_swap _ _).trans _)
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(algebraMap R (CliffordAlgebra (Q' Q))) (QuadraticForm.polar ↑(Q' Q) (0, 1) (↑(LinearMap.inl R M R) m)) = 0
[PROOFSTEP]
dsimp [QuadraticForm.polar]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(algebraMap R (CliffordAlgebra (Q' Q))) (↑Q (0 + m) + -((1 + 0) * (1 + 0)) - (↑Q 0 + -(1 * 1)) - (↑Q m + -(0 * 0))) =
0
[PROOFSTEP]
simp only [add_zero, mul_zero, mul_one, zero_add, neg_zero, QuadraticForm.map_zero, add_sub_cancel, sub_self, map_zero,
zero_sub]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ -(↑(v Q) m * e0 Q) = e0 Q * ↑(v Q) m
[PROOFSTEP]
rw [neg_eq_iff_eq_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(v Q) m * e0 Q = -(e0 Q * ↑(v Q) m)
[PROOFSTEP]
exact (neg_e0_mul_v _ m).symm
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ e0 Q * ↑(v Q) m * e0 Q = ↑(v Q) m
[PROOFSTEP]
rw [← neg_v_mul_e0, ← neg_mul, mul_assoc, e0_mul_e0, mul_neg_one, neg_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ CliffordAlgebra Q →ₐ[R] { x // x ∈ even (Q' Q) }
[PROOFSTEP]
refine' CliffordAlgebra.lift Q ⟨_, fun m => _⟩
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ M →ₗ[R] { x // x ∈ even (Q' Q) }
[PROOFSTEP]
refine' LinearMap.codRestrict _ _ fun m => Submodule.mem_iSup_of_mem ⟨2, rfl⟩ _
[GOAL]
case refine'_1.refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ M →ₗ[R] CliffordAlgebra (Q' Q)
case refine'_1.refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑?refine'_1.refine'_1 m ∈ LinearMap.range (ι (Q' Q)) ^ ↑{ val := 2, property := (_ : ↑2 = ↑2) }
[PROOFSTEP]
exact (LinearMap.mulLeft R <| e0 Q).comp (v Q)
[GOAL]
case refine'_1.refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
LinearMap.range (ι (Q' Q)) ^ ↑{ val := 2, property := (_ : ↑2 = ↑2) }
[PROOFSTEP]
rw [Subtype.coe_mk, pow_two]
[GOAL]
case refine'_1.refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈ LinearMap.range (ι (Q' Q)) * LinearMap.range (ι (Q' Q))
[PROOFSTEP]
exact Submodule.mul_mem_mul (LinearMap.mem_range_self _ _) (LinearMap.mem_range_self _ _)
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m *
↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m =
↑(algebraMap R { x // x ∈ even (Q' Q) }) (↑Q m)
[PROOFSTEP]
ext1
[GOAL]
case refine'_2.a
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m *
↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m) =
↑(↑(algebraMap R { x // x ∈ even (Q' Q) }) (↑Q m))
[PROOFSTEP]
rw [Subalgebra.coe_mul]
-- porting note: was part of the `dsimp only` below
[GOAL]
case refine'_2.a
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m) *
↑(↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m) =
↑(↑(algebraMap R { x // x ∈ even (Q' Q) }) (↑Q m))
[PROOFSTEP]
erw [LinearMap.codRestrict_apply]
-- porting note: was part of the `dsimp only` below
[GOAL]
case refine'_2.a
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m * ↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m =
↑(↑(algebraMap R { x // x ∈ even (Q' Q) }) (↑Q m))
[PROOFSTEP]
dsimp only [LinearMap.comp_apply, LinearMap.mulLeft_apply, Subalgebra.coe_algebraMap]
[GOAL]
case refine'_2.a
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ e0 Q * ↑(v Q) m * (e0 Q * ↑(v Q) m) = ↑(algebraMap R (CliffordAlgebra (Q' Q))) (↑Q m)
[PROOFSTEP]
rw [← mul_assoc, e0_mul_v_mul_e0, v_sq_scalar]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(↑(toEven Q) (↑(ι Q) m)) = e0 Q * ↑(v Q) m
[PROOFSTEP]
rw [toEven, CliffordAlgebra.lift_ι_apply]
-- porting note: was `rw`
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(↑(LinearMap.codRestrict (⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i)
(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q))
(_ :
∀ (m : M),
↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m ∈
⨆ (i : { n // ↑n = 0 }), LinearMap.range (ι (Q' Q)) ^ ↑i))
m) =
e0 Q * ↑(v Q) m
[PROOFSTEP]
erw [LinearMap.codRestrict_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(LinearMap.comp (LinearMap.mulLeft R (e0 Q)) (v Q)) m = e0 Q * ↑(v Q) m
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
⊢ { x // x ∈ even (Q' Q) } →ₐ[R] CliffordAlgebra Q
[PROOFSTEP]
let f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
((Algebra.lmul R (CliffordAlgebra Q)).toLinearMap.comp <|
(ι Q).comp (LinearMap.fst _ _ _) + (Algebra.linearMap R _).comp (LinearMap.snd _ _ _)).compl₂
((ι Q).comp (LinearMap.fst _ _ _) - (Algebra.linearMap R _).comp (LinearMap.snd _ _ _))
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
⊢ { x // x ∈ even (Q' Q) } →ₐ[R] CliffordAlgebra Q
[PROOFSTEP]
haveI f_apply : ∀ x y, f x y = (ι Q x.1 + algebraMap R _ x.2) * (ι Q y.1 - algebraMap R _ y.2) := fun x y => by rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
x y : M × R
⊢ ↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
⊢ { x // x ∈ even (Q' Q) } →ₐ[R] CliffordAlgebra Q
[PROOFSTEP]
haveI hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (algebraMap _ _ r) x := Algebra.commutes
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
⊢ { x // x ∈ even (Q' Q) } →ₐ[R] CliffordAlgebra Q
[PROOFSTEP]
haveI hm : ∀ m : M × R, ι Q m.1 * ι Q m.1 - algebraMap R _ m.2 * algebraMap R _ m.2 = algebraMap R _ (Q' Q m) :=
by
intro m
rw [ι_sq_scalar, ← RingHom.map_mul, ← RingHom.map_sub, sub_eq_add_neg, Q'_apply, sub_eq_add_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
⊢ ∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
[PROOFSTEP]
intro m
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
m : M × R
⊢ ↑(ι Q) m.fst * ↑(ι Q) m.fst - ↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
[PROOFSTEP]
rw [ι_sq_scalar, ← RingHom.map_mul, ← RingHom.map_sub, sub_eq_add_neg, Q'_apply, sub_eq_add_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
⊢ { x // x ∈ even (Q' Q) } →ₐ[R] CliffordAlgebra Q
[PROOFSTEP]
refine' even.lift (Q' Q) ⟨f, _, _⟩
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
⊢ ∀ (m : M × R), ↑(↑f m) m = ↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
[PROOFSTEP]
simp_rw [f_apply]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
⊢ ∀ (m₁ m₂ m₃ : M × R), ↑(↑f m₁) m₂ * ↑(↑f m₂) m₃ = ↑(Q' Q) m₂ • ↑(↑f m₁) m₃
[PROOFSTEP]
simp_rw [f_apply]
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
⊢ ∀ (m : M × R),
(↑(ι Q) m.fst + ↑(algebraMap R (CliffordAlgebra Q)) m.snd) *
(↑(ι Q) m.fst - ↑(algebraMap R (CliffordAlgebra Q)) m.snd) =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
[PROOFSTEP]
intro m
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
m : M × R
⊢ (↑(ι Q) m.fst + ↑(algebraMap R (CliffordAlgebra Q)) m.snd) *
(↑(ι Q) m.fst - ↑(algebraMap R (CliffordAlgebra Q)) m.snd) =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
[PROOFSTEP]
rw [← (hc _ _).symm.mul_self_sub_mul_self_eq, hm]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
⊢ ∀ (m₁ m₂ m₃ : M × R),
(↑(ι Q) m₁.fst + ↑(algebraMap R (CliffordAlgebra Q)) m₁.snd) *
(↑(ι Q) m₂.fst - ↑(algebraMap R (CliffordAlgebra Q)) m₂.snd) *
((↑(ι Q) m₂.fst + ↑(algebraMap R (CliffordAlgebra Q)) m₂.snd) *
(↑(ι Q) m₃.fst - ↑(algebraMap R (CliffordAlgebra Q)) m₃.snd)) =
↑(Q' Q) m₂ •
((↑(ι Q) m₁.fst + ↑(algebraMap R (CliffordAlgebra Q)) m₁.snd) *
(↑(ι Q) m₃.fst - ↑(algebraMap R (CliffordAlgebra Q)) m₃.snd))
[PROOFSTEP]
intro m₁ m₂ m₃
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
f_apply :
∀ (x y : M × R),
↑(↑f x) y =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
hc : ∀ (r : R) (x : CliffordAlgebra Q), Commute (↑(algebraMap R (CliffordAlgebra Q)) r) x
hm :
∀ (m : M × R),
↑(ι Q) m.fst * ↑(ι Q) m.fst -
↑(algebraMap R (CliffordAlgebra Q)) m.snd * ↑(algebraMap R (CliffordAlgebra Q)) m.snd =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)
m₁ m₂ m₃ : M × R
⊢ (↑(ι Q) m₁.fst + ↑(algebraMap R (CliffordAlgebra Q)) m₁.snd) *
(↑(ι Q) m₂.fst - ↑(algebraMap R (CliffordAlgebra Q)) m₂.snd) *
((↑(ι Q) m₂.fst + ↑(algebraMap R (CliffordAlgebra Q)) m₂.snd) *
(↑(ι Q) m₃.fst - ↑(algebraMap R (CliffordAlgebra Q)) m₃.snd)) =
↑(Q' Q) m₂ •
((↑(ι Q) m₁.fst + ↑(algebraMap R (CliffordAlgebra Q)) m₁.snd) *
(↑(ι Q) m₃.fst - ↑(algebraMap R (CliffordAlgebra Q)) m₃.snd))
[PROOFSTEP]
rw [← mul_smul_comm, ← mul_assoc, mul_assoc (_ + _), ← (hc _ _).symm.mul_self_sub_mul_self_eq', Algebra.smul_def, ←
mul_assoc, hm]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : M × R
⊢ ↑(ofEven Q) (↑(↑(even.ι (Q' Q)).bilin x) y) =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
[PROOFSTEP]
unfold ofEven
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : M × R
⊢ ↑(let f :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R));
↑(even.lift (Q' Q))
{ bilin := f,
contract :=
(_ :
∀ (m : M × R),
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m)
m =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)),
contract_mid :=
(_ :
∀ (m₁ m₂ m₃ : M × R),
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₁)
m₂ *
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₂)
m₃ =
↑(Q' Q) m₂ •
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₁)
m₃) })
(↑(↑(even.ι (Q' Q)).bilin x) y) =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
[PROOFSTEP]
lift_lets
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : M × R
⊢ let f :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R));
↑(↑(even.lift (Q' Q))
{ bilin := f,
contract :=
(_ :
∀ (m : M × R),
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m)
m =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)),
contract_mid :=
(_ :
∀ (m₁ m₂ m₃ : M × R),
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₁)
m₂ *
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₂)
m₃ =
↑(Q' Q) m₂ •
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₁)
m₃) })
(↑(↑(even.ι (Q' Q)).bilin x) y) =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
[PROOFSTEP]
intro f
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : M × R
f : M × R →ₗ[R] M × R →ₗ[R] CliffordAlgebra Q :=
LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R))
⊢ ↑(↑(even.lift (Q' Q))
{ bilin := f,
contract :=
(_ :
∀ (m : M × R),
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m)
m =
↑(algebraMap R (CliffordAlgebra Q)) (↑(Q' Q) m)),
contract_mid :=
(_ :
∀ (m₁ m₂ m₃ : M × R),
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₁)
m₂ *
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₂)
m₃ =
↑(Q' Q) m₂ •
↑(↑(LinearMap.compl₂
(LinearMap.comp (AlgHom.toLinearMap (Algebra.lmul R (CliffordAlgebra Q)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) +
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
(LinearMap.comp (ι Q) (LinearMap.fst R M R) -
LinearMap.comp (Algebra.linearMap R (CliffordAlgebra Q)) (LinearMap.snd R M R)))
m₁)
m₃) })
(↑(↑(even.ι (Q' Q)).bilin x) y) =
(↑(ι Q) x.fst + ↑(algebraMap R (CliffordAlgebra Q)) x.snd) *
(↑(ι Q) y.fst - ↑(algebraMap R (CliffordAlgebra Q)) y.snd)
[PROOFSTEP]
refine @even.lift_ι R (M × R) _ _ _ (Q' Q) _ _ _ ⟨f, ?_, ?_⟩ x y
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
⊢ ↑(↑(toEven Q) (↑(ofEven Q) (↑(↑(even.ι (Q' Q)).bilin (m₁, r₁)) (m₂, r₂)))) =
(e0 Q * ↑(v Q) m₁ + ↑(algebraMap R (CliffordAlgebra (Q' Q))) r₁) *
(e0 Q * ↑(v Q) m₂ - ↑(algebraMap R (CliffordAlgebra (Q' Q))) r₂)
[PROOFSTEP]
rw [ofEven_ι, AlgHom.map_mul, AlgHom.map_add, AlgHom.map_sub, AlgHom.commutes, AlgHom.commutes, Subalgebra.coe_mul,
Subalgebra.coe_add, Subalgebra.coe_sub, toEven_ι, toEven_ι, Subalgebra.coe_algebraMap, Subalgebra.coe_algebraMap]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
⊢ (e0 Q * ↑(v Q) m₁ + ↑(algebraMap R (CliffordAlgebra (Q' Q))) r₁) *
(e0 Q * ↑(v Q) m₂ - ↑(algebraMap R (CliffordAlgebra (Q' Q))) r₂) =
e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) + r₁ • e0 Q * ↑(v Q) m₂ - r₂ • e0 Q * ↑(v Q) m₁ -
↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂)
[PROOFSTEP]
rw [mul_sub, add_mul, add_mul, ← Algebra.commutes, ← Algebra.smul_def, ← map_mul, ← Algebra.smul_def,
sub_add_eq_sub_sub, smul_mul_assoc, smul_mul_assoc]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
⊢ e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) + r₁ • e0 Q * ↑(v Q) m₂ - r₂ • e0 Q * ↑(v Q) m₁ -
↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂) =
↑(v Q) m₁ * ↑(v Q) m₂ + r₁ • e0 Q * ↑(v Q) m₂ + ↑(v Q) m₁ * r₂ • e0 Q + r₁ • e0 Q * r₂ • e0 Q
[PROOFSTEP]
have h1 : e0 Q * v Q m₁ * (e0 Q * v Q m₂) = v Q m₁ * v Q m₂ := by rw [← mul_assoc, e0_mul_v_mul_e0]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
⊢ e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) = ↑(v Q) m₁ * ↑(v Q) m₂
[PROOFSTEP]
rw [← mul_assoc, e0_mul_v_mul_e0]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
h1 : e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) = ↑(v Q) m₁ * ↑(v Q) m₂
⊢ e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) + r₁ • e0 Q * ↑(v Q) m₂ - r₂ • e0 Q * ↑(v Q) m₁ -
↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂) =
↑(v Q) m₁ * ↑(v Q) m₂ + r₁ • e0 Q * ↑(v Q) m₂ + ↑(v Q) m₁ * r₂ • e0 Q + r₁ • e0 Q * r₂ • e0 Q
[PROOFSTEP]
have h2 : -(r₂ • e0 Q * v Q m₁) = v Q m₁ * r₂ • e0 Q := by rw [mul_smul_comm, smul_mul_assoc, ← smul_neg, neg_e0_mul_v]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
h1 : e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) = ↑(v Q) m₁ * ↑(v Q) m₂
⊢ -(r₂ • e0 Q * ↑(v Q) m₁) = ↑(v Q) m₁ * r₂ • e0 Q
[PROOFSTEP]
rw [mul_smul_comm, smul_mul_assoc, ← smul_neg, neg_e0_mul_v]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
h1 : e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) = ↑(v Q) m₁ * ↑(v Q) m₂
h2 : -(r₂ • e0 Q * ↑(v Q) m₁) = ↑(v Q) m₁ * r₂ • e0 Q
⊢ e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) + r₁ • e0 Q * ↑(v Q) m₂ - r₂ • e0 Q * ↑(v Q) m₁ -
↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂) =
↑(v Q) m₁ * ↑(v Q) m₂ + r₁ • e0 Q * ↑(v Q) m₂ + ↑(v Q) m₁ * r₂ • e0 Q + r₁ • e0 Q * r₂ • e0 Q
[PROOFSTEP]
have h3 : -algebraMap R _ (r₁ * r₂) = r₁ • e0 Q * r₂ • e0 Q := by
rw [Algebra.algebraMap_eq_smul_one, smul_mul_smul, e0_mul_e0, smul_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
h1 : e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) = ↑(v Q) m₁ * ↑(v Q) m₂
h2 : -(r₂ • e0 Q * ↑(v Q) m₁) = ↑(v Q) m₁ * r₂ • e0 Q
⊢ -↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂) = r₁ • e0 Q * r₂ • e0 Q
[PROOFSTEP]
rw [Algebra.algebraMap_eq_smul_one, smul_mul_smul, e0_mul_e0, smul_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
h1 : e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) = ↑(v Q) m₁ * ↑(v Q) m₂
h2 : -(r₂ • e0 Q * ↑(v Q) m₁) = ↑(v Q) m₁ * r₂ • e0 Q
h3 : -↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂) = r₁ • e0 Q * r₂ • e0 Q
⊢ e0 Q * ↑(v Q) m₁ * (e0 Q * ↑(v Q) m₂) + r₁ • e0 Q * ↑(v Q) m₂ - r₂ • e0 Q * ↑(v Q) m₁ -
↑(algebraMap R (CliffordAlgebra (Q' Q))) (r₁ * r₂) =
↑(v Q) m₁ * ↑(v Q) m₂ + r₁ • e0 Q * ↑(v Q) m₂ + ↑(v Q) m₁ * r₂ • e0 Q + r₁ • e0 Q * r₂ • e0 Q
[PROOFSTEP]
rw [sub_eq_add_neg, sub_eq_add_neg, h1, h2, h3]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m₁✝ m₂✝ : M × R
m₁ : M
r₁ : R
m₂ : M
r₂ : R
⊢ ↑(v Q) m₁ * ↑(v Q) m₂ + r₁ • e0 Q * ↑(v Q) m₂ + ↑(v Q) m₁ * r₂ • e0 Q + r₁ • e0 Q * r₂ • e0 Q =
↑(ι (Q' Q)) (m₁, r₁) * ↑(ι (Q' Q)) (m₂, r₂)
[PROOFSTEP]
rw [ι_eq_v_add_smul_e0, ι_eq_v_add_smul_e0, mul_add, add_mul, add_mul, add_assoc]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(ofEven Q) (↑(toEven Q) (↑(ι Q) m)) =
↑(ofEven Q) { val := ↑(↑(toEven Q) (↑(ι Q) m)), property := (_ : ↑(↑(toEven Q) (↑(ι Q) m)) ∈ even (Q' Q)) }
[PROOFSTEP]
rw [Subtype.coe_eta]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(ofEven Q) { val := ↑(↑(toEven Q) (↑(ι Q) m)), property := (_ : ↑(↑(toEven Q) (↑(ι Q) m)) ∈ even (Q' Q)) } =
(↑(ι Q) 0 + ↑(algebraMap R (CliffordAlgebra Q)) 1) * (↑(ι Q) m - ↑(algebraMap R (CliffordAlgebra Q)) 0)
[PROOFSTEP]
simp_rw [toEven_ι]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(ofEven Q) { val := e0 Q * ↑(v Q) m, property := (_ : (fun x => x ∈ even (Q' Q)) (e0 Q * ↑(v Q) m)) } =
(↑(ι Q) 0 + ↑(algebraMap R (CliffordAlgebra Q)) 1) * (↑(ι Q) m - ↑(algebraMap R (CliffordAlgebra Q)) 0)
[PROOFSTEP]
exact ofEven_ι Q _ _
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ (↑(ι Q) 0 + ↑(algebraMap R (CliffordAlgebra Q)) 1) * (↑(ι Q) m - ↑(algebraMap R (CliffordAlgebra Q)) 0) = ↑(ι Q) m
[PROOFSTEP]
rw [map_one, map_zero, map_zero, sub_zero, zero_add, one_mul]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x : CliffordAlgebra Q
⊢ ↑(↑(toEven Q) (↑reverse (↑involute x))) = ↑reverse ↑(↑(toEven Q) x)
[PROOFSTEP]
induction x using CliffordAlgebra.induction
[GOAL]
case h_grade0
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
r✝ : R
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(algebraMap R (CliffordAlgebra Q)) r✝)))) =
↑reverse ↑(↑(toEven Q) (↑(algebraMap R (CliffordAlgebra Q)) r✝))
case h_grade1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x✝ : M
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(ι Q) x✝)))) = ↑reverse ↑(↑(toEven Q) (↑(ι Q) x✝))
case h_mul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² * b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² * b✝))
case h_add
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² + b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² + b✝))
[PROOFSTEP]
case h_grade0 r => simp only [AlgHom.commutes, Subalgebra.coe_algebraMap, reverse.commutes]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
r : R
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(algebraMap R (CliffordAlgebra Q)) r)))) =
↑reverse ↑(↑(toEven Q) (↑(algebraMap R (CliffordAlgebra Q)) r))
[PROOFSTEP]
case h_grade0 r => simp only [AlgHom.commutes, Subalgebra.coe_algebraMap, reverse.commutes]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
r : R
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(algebraMap R (CliffordAlgebra Q)) r)))) =
↑reverse ↑(↑(toEven Q) (↑(algebraMap R (CliffordAlgebra Q)) r))
[PROOFSTEP]
simp only [AlgHom.commutes, Subalgebra.coe_algebraMap, reverse.commutes]
[GOAL]
case h_grade1
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x✝ : M
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(ι Q) x✝)))) = ↑reverse ↑(↑(toEven Q) (↑(ι Q) x✝))
case h_mul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² * b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² * b✝))
case h_add
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² + b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² + b✝))
[PROOFSTEP]
case h_grade1 m =>
-- porting note: added `letI`
letI : SubtractionMonoid (even (Q' Q)) := AddGroup.toSubtractionMonoid
simp only [involute_ι, Subalgebra.coe_neg, toEven_ι, reverse.map_mul, reverse_v, reverse_e0, reverse_ι, neg_e0_mul_v,
map_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(ι Q) m)))) = ↑reverse ↑(↑(toEven Q) (↑(ι Q) m))
[PROOFSTEP]
case h_grade1 m =>
-- porting note: added `letI`
letI : SubtractionMonoid (even (Q' Q)) := AddGroup.toSubtractionMonoid
simp only [involute_ι, Subalgebra.coe_neg, toEven_ι, reverse.map_mul, reverse_v, reverse_e0, reverse_ι, neg_e0_mul_v,
map_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(ι Q) m)))) = ↑reverse ↑(↑(toEven Q) (↑(ι Q) m))
[PROOFSTEP]
letI : SubtractionMonoid (even (Q' Q)) := AddGroup.toSubtractionMonoid
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
m : M
this : SubtractionMonoid { x // x ∈ even (Q' Q) } := AddGroup.toSubtractionMonoid
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (↑(ι Q) m)))) = ↑reverse ↑(↑(toEven Q) (↑(ι Q) m))
[PROOFSTEP]
simp only [involute_ι, Subalgebra.coe_neg, toEven_ι, reverse.map_mul, reverse_v, reverse_e0, reverse_ι, neg_e0_mul_v,
map_neg]
[GOAL]
case h_mul
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² * b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² * b✝))
case h_add
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² + b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² + b✝))
[PROOFSTEP]
case h_mul x y hx hy => simp only [map_mul, Subalgebra.coe_mul, reverse.map_mul, hx, hy]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : CliffordAlgebra Q
hx : ↑(↑(toEven Q) (↑reverse (↑involute x))) = ↑reverse ↑(↑(toEven Q) x)
hy : ↑(↑(toEven Q) (↑reverse (↑involute y))) = ↑reverse ↑(↑(toEven Q) y)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (x * y)))) = ↑reverse ↑(↑(toEven Q) (x * y))
[PROOFSTEP]
case h_mul x y hx hy => simp only [map_mul, Subalgebra.coe_mul, reverse.map_mul, hx, hy]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : CliffordAlgebra Q
hx : ↑(↑(toEven Q) (↑reverse (↑involute x))) = ↑reverse ↑(↑(toEven Q) x)
hy : ↑(↑(toEven Q) (↑reverse (↑involute y))) = ↑reverse ↑(↑(toEven Q) y)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (x * y)))) = ↑reverse ↑(↑(toEven Q) (x * y))
[PROOFSTEP]
simp only [map_mul, Subalgebra.coe_mul, reverse.map_mul, hx, hy]
[GOAL]
case h_add
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
a✝² b✝ : CliffordAlgebra Q
a✝¹ : ↑(↑(toEven Q) (↑reverse (↑involute a✝²))) = ↑reverse ↑(↑(toEven Q) a✝²)
a✝ : ↑(↑(toEven Q) (↑reverse (↑involute b✝))) = ↑reverse ↑(↑(toEven Q) b✝)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (a✝² + b✝)))) = ↑reverse ↑(↑(toEven Q) (a✝² + b✝))
[PROOFSTEP]
case h_add x y hx hy => simp only [map_add, Subalgebra.coe_add, hx, hy]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : CliffordAlgebra Q
hx : ↑(↑(toEven Q) (↑reverse (↑involute x))) = ↑reverse ↑(↑(toEven Q) x)
hy : ↑(↑(toEven Q) (↑reverse (↑involute y))) = ↑reverse ↑(↑(toEven Q) y)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (x + y)))) = ↑reverse ↑(↑(toEven Q) (x + y))
[PROOFSTEP]
case h_add x y hx hy => simp only [map_add, Subalgebra.coe_add, hx, hy]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q : QuadraticForm R M
x y : CliffordAlgebra Q
hx : ↑(↑(toEven Q) (↑reverse (↑involute x))) = ↑reverse ↑(↑(toEven Q) x)
hy : ↑(↑(toEven Q) (↑reverse (↑involute y))) = ↑reverse ↑(↑(toEven Q) y)
⊢ ↑(↑(toEven Q) (↑reverse (↑involute (x + y)))) = ↑reverse ↑(↑(toEven Q) (x + y))
[PROOFSTEP]
simp only [map_add, Subalgebra.coe_add, hx, hy]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q Q' : QuadraticForm R M
h : Q' = -Q
this✝ : AddCommGroup { x // x ∈ even Q' } := AddSubgroupClass.toAddCommGroup (even Q')
this : HasDistribNeg { x // x ∈ even Q' } := NonUnitalNonAssocRing.toHasDistribNeg
m : M
⊢ ↑(↑(-(even.ι Q').bilin) m) m = ↑(algebraMap R { x // x ∈ even Q' }) (↑Q m)
[PROOFSTEP]
simp_rw [LinearMap.neg_apply, EvenHom.contract, h, QuadraticForm.neg_apply, map_neg, neg_neg]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q Q' : QuadraticForm R M
h : Q' = -Q
this✝ : AddCommGroup { x // x ∈ even Q' } := AddSubgroupClass.toAddCommGroup (even Q')
this : HasDistribNeg { x // x ∈ even Q' } := NonUnitalNonAssocRing.toHasDistribNeg
m₁ m₂ m₃ : M
⊢ ↑(↑(-(even.ι Q').bilin) m₁) m₂ * ↑(↑(-(even.ι Q').bilin) m₂) m₃ = ↑Q m₂ • ↑(↑(-(even.ι Q').bilin) m₁) m₃
[PROOFSTEP]
simp_rw [LinearMap.neg_apply, neg_mul_neg, EvenHom.contract_mid, h, QuadraticForm.neg_apply, smul_neg, neg_smul]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q Q' : QuadraticForm R M
h : Q' = -Q
h' : Q = -Q'
⊢ AlgHom.comp (evenToNeg Q' Q h') (evenToNeg Q Q' h) = AlgHom.id R { x // x ∈ even Q }
[PROOFSTEP]
ext m₁ m₂ : 4
[GOAL]
case h.bilin.h.h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q Q' : QuadraticForm R M
h : Q' = -Q
h' : Q = -Q'
m₁ m₂ : M
⊢ ↑(↑(EvenHom.compr₂ (even.ι Q) (AlgHom.comp (evenToNeg Q' Q h') (evenToNeg Q Q' h))).bilin m₁) m₂ =
↑(↑(EvenHom.compr₂ (even.ι Q) (AlgHom.id R { x // x ∈ even Q })).bilin m₁) m₂
[PROOFSTEP]
dsimp only [EvenHom.compr₂_bilin, LinearMap.compr₂_apply, AlgHom.toLinearMap_apply, AlgHom.comp_apply, AlgHom.id_apply]
[GOAL]
case h.bilin.h.h
R : Type u_1
M : Type u_2
inst✝² : CommRing R
inst✝¹ : AddCommGroup M
inst✝ : Module R M
Q Q' : QuadraticForm R M
h : Q' = -Q
h' : Q = -Q'
m₁ m₂ : M
⊢ ↑(evenToNeg Q' Q h') (↑(evenToNeg Q Q' h) (↑(↑(even.ι Q).bilin m₁) m₂)) = ↑(↑(even.ι Q).bilin m₁) m₂
[PROOFSTEP]
rw [evenToNeg_ι, map_neg, evenToNeg_ι, neg_neg]
| {"mathlib_filename": "Mathlib.LinearAlgebra.CliffordAlgebra.EvenEquiv", "llama_tokens": 23647} |
[GOAL]
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
⊢ charpoly (↑(leftMulMatrix h.basis) h.gen) = minpoly R h.gen
[PROOFSTEP]
cases subsingleton_or_nontrivial R
[GOAL]
case inl
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Subsingleton R
⊢ charpoly (↑(leftMulMatrix h.basis) h.gen) = minpoly R h.gen
[PROOFSTEP]
apply Subsingleton.elim
[GOAL]
case inr
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
⊢ charpoly (↑(leftMulMatrix h.basis) h.gen) = minpoly R h.gen
[PROOFSTEP]
apply minpoly.unique' R h.gen (charpoly_monic _)
[GOAL]
case inr.hp
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
⊢ ↑(aeval h.gen) (charpoly (↑(leftMulMatrix h.basis) h.gen)) = 0
[PROOFSTEP]
apply (injective_iff_map_eq_zero (G := S) (leftMulMatrix _)).mp (leftMulMatrix_injective h.basis)
[GOAL]
case inr.hp.a
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
⊢ ↑(leftMulMatrix h.basis) (↑(aeval h.gen) (charpoly (↑(leftMulMatrix h.basis) h.gen))) = 0
[PROOFSTEP]
rw [← Polynomial.aeval_algHom_apply, aeval_self_charpoly]
[GOAL]
case inr.hl
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
⊢ ∀ (q : R[X]), degree q < degree (charpoly (↑(leftMulMatrix h.basis) h.gen)) → q = 0 ∨ ↑(aeval h.gen) q ≠ 0
[PROOFSTEP]
refine' fun q hq => or_iff_not_imp_left.2 fun h0 => _
[GOAL]
case inr.hl
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
q : R[X]
hq : degree q < degree (charpoly (↑(leftMulMatrix h.basis) h.gen))
h0 : ¬q = 0
⊢ ↑(aeval h.gen) q ≠ 0
[PROOFSTEP]
rw [Matrix.charpoly_degree_eq_dim, Fintype.card_fin] at hq
[GOAL]
case inr.hl
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
q : R[X]
hq : degree q < ↑h.dim
h0 : ¬q = 0
⊢ ↑(aeval h.gen) q ≠ 0
[PROOFSTEP]
contrapose! hq
[GOAL]
case inr.hl
R : Type u
inst✝⁶ : CommRing R
n : Type v
inst✝⁵ : DecidableEq n
inst✝⁴ : Fintype n
N : Type w
inst✝³ : AddCommGroup N
inst✝² : Module R N
S : Type u_1
inst✝¹ : Ring S
inst✝ : Algebra R S
h : PowerBasis R S
h✝ : Nontrivial R
q : R[X]
h0 : ¬q = 0
hq : ↑(aeval h.gen) q = 0
⊢ ↑h.dim ≤ degree q
[PROOFSTEP]
exact h.dim_le_degree_of_root h0 hq
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Charpoly.Minpoly", "llama_tokens": 1712} |
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
i : n
⊢ charmatrix M i i = X - ↑C (M i i)
[PROOFSTEP]
simp only [charmatrix, RingHom.mapMatrix_apply, sub_apply, scalar_apply_eq, map_apply]
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
i j : n
h : i ≠ j
⊢ charmatrix M i j = -↑C (M i j)
[PROOFSTEP]
simp only [charmatrix, RingHom.mapMatrix_apply, sub_apply, scalar_apply_ne _ _ _ h, map_apply, sub_eq_neg_self]
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
⊢ ↑matPolyEquiv (charmatrix M) = X - ↑C M
[PROOFSTEP]
ext k i j
[GOAL]
case a.a.h
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
⊢ coeff (↑matPolyEquiv (charmatrix M)) k i j = coeff (X - ↑C M) k i j
[PROOFSTEP]
simp only [matPolyEquiv_coeff_apply, coeff_sub, Pi.sub_apply]
[GOAL]
case a.a.h
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
⊢ coeff (charmatrix M i j) k = (coeff X k - coeff (↑C M) k) i j
[PROOFSTEP]
by_cases h : i = j
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : i = j
⊢ coeff (charmatrix M i j) k = (coeff X k - coeff (↑C M) k) i j
[PROOFSTEP]
subst h
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
⊢ coeff (charmatrix M i i) k = (coeff X k - coeff (↑C M) k) i i
[PROOFSTEP]
rw [charmatrix_apply_eq, coeff_sub]
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
⊢ coeff X k - coeff (↑C (M i i)) k = (coeff X k - coeff (↑C M) k) i i
[PROOFSTEP]
simp only [coeff_X, coeff_C]
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
⊢ ((if 1 = k then 1 else 0) - if k = 0 then M i i else 0) = ((if 1 = k then 1 else 0) - if k = 0 then M else 0) i i
[PROOFSTEP]
split_ifs
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
h✝¹ : 1 = k
h✝ : k = 0
⊢ 1 - M i i = (1 - M) i i
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
h✝¹ : 1 = k
h✝ : ¬k = 0
⊢ 1 - 0 = (1 - 0) i i
[PROOFSTEP]
simp
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
h✝¹ : ¬1 = k
h✝ : k = 0
⊢ 0 - M i i = (0 - M) i i
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i : n
h✝¹ : ¬1 = k
h✝ : ¬k = 0
⊢ 0 - 0 = (0 - 0) i i
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : ¬i = j
⊢ coeff (charmatrix M i j) k = (coeff X k - coeff (↑C M) k) i j
[PROOFSTEP]
rw [charmatrix_apply_ne _ _ _ h, coeff_X, coeff_neg, coeff_C, coeff_C]
[GOAL]
case neg
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : ¬i = j
⊢ (-if k = 0 then M i j else 0) = ((if 1 = k then 1 else 0) - if k = 0 then M else 0) i j
[PROOFSTEP]
split_ifs
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : ¬i = j
h✝¹ : k = 0
h✝ : 1 = k
⊢ -M i j = (1 - M) i j
[PROOFSTEP]
simp [h]
[GOAL]
case neg
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : ¬i = j
h✝¹ : k = 0
h✝ : ¬1 = k
⊢ -M i j = (0 - M) i j
[PROOFSTEP]
simp [h]
[GOAL]
case pos
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : ¬i = j
h✝¹ : ¬k = 0
h✝ : 1 = k
⊢ -0 = (1 - 0) i j
[PROOFSTEP]
simp [h]
[GOAL]
case neg
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
k : ℕ
i j : n
h : ¬i = j
h✝¹ : ¬k = 0
h✝ : ¬1 = k
⊢ -0 = (0 - 0) i j
[PROOFSTEP]
simp [h]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
⊢ charmatrix (↑(reindex e e) M) = ↑(reindex e e) (charmatrix M)
[PROOFSTEP]
ext i j x
[GOAL]
case a.h.a
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
i j : m
x : ℕ
⊢ coeff (charmatrix (↑(reindex e e) M) i j) x = coeff (↑(reindex e e) (charmatrix M) i j) x
[PROOFSTEP]
by_cases h : i = j
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
i j : m
x : ℕ
h : i = j
⊢ coeff (charmatrix (↑(reindex e e) M) i j) x = coeff (↑(reindex e e) (charmatrix M) i j) x
case neg
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
i j : m
x : ℕ
h : ¬i = j
⊢ coeff (charmatrix (↑(reindex e e) M) i j) x = coeff (↑(reindex e e) (charmatrix M) i j) x
[PROOFSTEP]
all_goals simp [h]
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
i j : m
x : ℕ
h : i = j
⊢ coeff (charmatrix (↑(reindex e e) M) i j) x = coeff (↑(reindex e e) (charmatrix M) i j) x
[PROOFSTEP]
simp [h]
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
i j : m
x : ℕ
h : ¬i = j
⊢ coeff (charmatrix (↑(reindex e e) M) i j) x = coeff (↑(reindex e e) (charmatrix M) i j) x
[PROOFSTEP]
simp [h]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
⊢ charpoly (↑(reindex e e) M) = charpoly M
[PROOFSTEP]
unfold Matrix.charpoly
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n : Type w
inst✝³ : DecidableEq n
inst✝² : Fintype n
m : Type v
inst✝¹ : DecidableEq m
inst✝ : Fintype m
e : n ≃ m
M : Matrix n n R
⊢ det (charmatrix (↑(reindex e e) M)) = det (charmatrix M)
[PROOFSTEP]
rw [charmatrix_reindex, Matrix.det_reindex_self]
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
have h : M.charpoly • (1 : Matrix n n R[X]) = adjugate (charmatrix M) * charmatrix M := (adjugate_mul _).symm
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
h : charpoly M • 1 = adjugate (charmatrix M) * charmatrix M
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
apply_fun matPolyEquiv at h
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
h : ↑matPolyEquiv (charpoly M • 1) = ↑matPolyEquiv (adjugate (charmatrix M) * charmatrix M)
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
simp only [matPolyEquiv.map_mul, matPolyEquiv_charmatrix] at h
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
h : ↑matPolyEquiv (charpoly M • 1) = ↑matPolyEquiv (adjugate (charmatrix M)) * (X - ↑C M)
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
apply_fun fun p => p.eval M at h
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
h : eval M (↑matPolyEquiv (charpoly M • 1)) = eval M (↑matPolyEquiv (adjugate (charmatrix M)) * (X - ↑C M))
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
rw [eval_mul_X_sub_C] at h
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
h : eval M (↑matPolyEquiv (charpoly M • 1)) = 0
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
rw [matPolyEquiv_smul_one, eval_map] at h
[GOAL]
R : Type u
inst✝² : CommRing R
n : Type w
inst✝¹ : DecidableEq n
inst✝ : Fintype n
M : Matrix n n R
h : eval₂ (algebraMap R (Matrix n n R)) M (charpoly M) = 0
⊢ ↑(aeval M) (charpoly M) = 0
[PROOFSTEP]
exact h
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Charpoly.Basic", "llama_tokens": 4455} |
[GOAL]
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
f : M →ₗ[R] M'
g : N →ₗ[R] N'
⊢ ↑(toMatrix (Basis.tensorProduct bM bN) (Basis.tensorProduct bM' bN')) (map f g) =
kroneckerMap (fun x x_1 => x * x_1) (↑(toMatrix bM bM') f) (↑(toMatrix bN bN') g)
[PROOFSTEP]
ext ⟨i, j⟩ ⟨i', j'⟩
[GOAL]
case a.mk.h.mk
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
f : M →ₗ[R] M'
g : N →ₗ[R] N'
i : ι'
j : κ'
i' : ι
j' : κ
⊢ ↑(toMatrix (Basis.tensorProduct bM bN) (Basis.tensorProduct bM' bN')) (map f g) (i, j) (i', j') =
kroneckerMap (fun x x_1 => x * x_1) (↑(toMatrix bM bM') f) (↑(toMatrix bN bN') g) (i, j) (i', j')
[PROOFSTEP]
simp_rw [Matrix.kroneckerMap_apply, toMatrix_apply, Basis.tensorProduct_apply, TensorProduct.map_tmul,
Basis.tensorProduct_repr_tmul_apply]
[GOAL]
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
A : Matrix ι' ι R
B : Matrix κ' κ R
⊢ ↑(toLin (Basis.tensorProduct bM bN) (Basis.tensorProduct bM' bN')) (kroneckerMap (fun x x_1 => x * x_1) A B) =
TensorProduct.map (↑(toLin bM bM') A) (↑(toLin bN bN') B)
[PROOFSTEP]
rw [← LinearEquiv.eq_symm_apply, toLin_symm, TensorProduct.toMatrix_map, toMatrix_toLin, toMatrix_toLin]
[GOAL]
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
⊢ ↑(toMatrix (Basis.tensorProduct bM bN) (Basis.tensorProduct bN bM)) ↑(TensorProduct.comm R M N) =
submatrix 1 Prod.swap _root_.id
[PROOFSTEP]
ext ⟨i, j⟩ ⟨i', j'⟩
[GOAL]
case a.mk.h.mk
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : κ
j i' : ι
j' : κ
⊢ ↑(toMatrix (Basis.tensorProduct bM bN) (Basis.tensorProduct bN bM)) ↑(TensorProduct.comm R M N) (i, j) (i', j') =
submatrix 1 Prod.swap _root_.id (i, j) (i', j')
[PROOFSTEP]
simp_rw [toMatrix_apply, Basis.tensorProduct_apply, LinearEquiv.coe_coe, TensorProduct.comm_tmul,
Basis.tensorProduct_repr_tmul_apply, Matrix.submatrix_apply, Prod.swap_prod_mk, id.def, Basis.repr_self_apply,
Matrix.one_apply, Prod.ext_iff, ite_and, @eq_comm _ i', @eq_comm _ j']
[GOAL]
case a.mk.h.mk
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : κ
j i' : ι
j' : κ
⊢ ((if i = j' then 1 else 0) * if j = i' then 1 else 0) = if j = i' then if i = j' then 1 else 0 else 0
[PROOFSTEP]
split_ifs
[GOAL]
case pos
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : κ
j i' : ι
j' : κ
h✝¹ : i = j'
h✝ : j = i'
⊢ 1 * 1 = 1
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : κ
j i' : ι
j' : κ
h✝¹ : i = j'
h✝ : ¬j = i'
⊢ 1 * 0 = 0
[PROOFSTEP]
simp
[GOAL]
case pos
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : κ
j i' : ι
j' : κ
h✝¹ : ¬i = j'
h✝ : j = i'
⊢ 0 * 1 = 0
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : κ
j i' : ι
j' : κ
h✝¹ : ¬i = j'
h✝ : ¬j = i'
⊢ 0 * 0 = 0
[PROOFSTEP]
simp
[GOAL]
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
⊢ ↑(toMatrix (Basis.tensorProduct (Basis.tensorProduct bM bN) bP) (Basis.tensorProduct bM (Basis.tensorProduct bN bP)))
↑(TensorProduct.assoc R M N P) =
submatrix 1 _root_.id ↑(Equiv.prodAssoc ι κ τ)
[PROOFSTEP]
ext ⟨i, j, k⟩ ⟨⟨i', j'⟩, k'⟩
[GOAL]
case a.mk.mk.h.mk.mk
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
⊢ ↑(toMatrix (Basis.tensorProduct (Basis.tensorProduct bM bN) bP) (Basis.tensorProduct bM (Basis.tensorProduct bN bP)))
↑(TensorProduct.assoc R M N P) (i, j, k) ((i', j'), k') =
submatrix 1 _root_.id ↑(Equiv.prodAssoc ι κ τ) (i, j, k) ((i', j'), k')
[PROOFSTEP]
simp_rw [toMatrix_apply, Basis.tensorProduct_apply, LinearEquiv.coe_coe, TensorProduct.assoc_tmul,
Basis.tensorProduct_repr_tmul_apply, Matrix.submatrix_apply, Equiv.prodAssoc_apply, id.def, Basis.repr_self_apply,
Matrix.one_apply, Prod.ext_iff, ite_and, @eq_comm _ i', @eq_comm _ j', @eq_comm _ k']
[GOAL]
case a.mk.mk.h.mk.mk
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
⊢ (if i = i' then 1 else 0) * ((if j = j' then 1 else 0) * if k = k' then 1 else 0) =
if i = i' then if j = j' then if k = k' then 1 else 0 else 0 else 0
[PROOFSTEP]
split_ifs
[GOAL]
case pos
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : i = i'
h✝¹ : j = j'
h✝ : k = k'
⊢ 1 * (1 * 1) = 1
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : i = i'
h✝¹ : j = j'
h✝ : ¬k = k'
⊢ 1 * (1 * 0) = 0
[PROOFSTEP]
simp
[GOAL]
case pos
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : i = i'
h✝¹ : ¬j = j'
h✝ : k = k'
⊢ 1 * (0 * 1) = 0
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : i = i'
h✝¹ : ¬j = j'
h✝ : ¬k = k'
⊢ 1 * (0 * 0) = 0
[PROOFSTEP]
simp
[GOAL]
case pos
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : ¬i = i'
h✝¹ : j = j'
h✝ : k = k'
⊢ 0 * (1 * 1) = 0
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : ¬i = i'
h✝¹ : j = j'
h✝ : ¬k = k'
⊢ 0 * (1 * 0) = 0
[PROOFSTEP]
simp
[GOAL]
case pos
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : ¬i = i'
h✝¹ : ¬j = j'
h✝ : k = k'
⊢ 0 * (0 * 1) = 0
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u_1
M : Type u_2
N : Type u_3
P : Type u_4
M' : Type u_5
N' : Type u_6
ι : Type u_7
κ : Type u_8
τ : Type u_9
ι' : Type u_10
κ' : Type u_11
inst✝¹⁸ : DecidableEq ι
inst✝¹⁷ : DecidableEq κ
inst✝¹⁶ : DecidableEq τ
inst✝¹⁵ : Fintype ι
inst✝¹⁴ : Fintype κ
inst✝¹³ : Fintype τ
inst✝¹² : Fintype ι'
inst✝¹¹ : Fintype κ'
inst✝¹⁰ : CommRing R
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : AddCommGroup P
inst✝⁶ : AddCommGroup M'
inst✝⁵ : AddCommGroup N'
inst✝⁴ : Module R M
inst✝³ : Module R N
inst✝² : Module R P
inst✝¹ : Module R M'
inst✝ : Module R N'
bM : Basis ι R M
bN : Basis κ R N
bP : Basis τ R P
bM' : Basis ι' R M'
bN' : Basis κ' R N'
i : ι
j : κ
k k' : τ
i' : ι
j' : κ
h✝² : ¬i = i'
h✝¹ : ¬j = j'
h✝ : ¬k = k'
⊢ 0 * (0 * 0) = 0
[PROOFSTEP]
simp
| {"mathlib_filename": "Mathlib.LinearAlgebra.TensorProduct.Matrix", "llama_tokens": 10216} |
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : M →ₛₗ[ρ₁₂] N →ₛₗ[σ₁₂] P
x : M
y : N
⊢ (Finsupp.sum (↑b₁.repr x) fun i xi =>
Finsupp.sum (↑b₂.repr y) fun j yj => ↑ρ₁₂ xi • ↑σ₁₂ yj • ↑(↑B (↑b₁ i)) (↑b₂ j)) =
↑(↑B x) y
[PROOFSTEP]
conv_rhs => rw [← b₁.total_repr x, ← b₂.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : M →ₛₗ[ρ₁₂] N →ₛₗ[σ₁₂] P
x : M
y : N
| ↑(↑B x) y
[PROOFSTEP]
rw [← b₁.total_repr x, ← b₂.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : M →ₛₗ[ρ₁₂] N →ₛₗ[σ₁₂] P
x : M
y : N
| ↑(↑B x) y
[PROOFSTEP]
rw [← b₁.total_repr x, ← b₂.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : M →ₛₗ[ρ₁₂] N →ₛₗ[σ₁₂] P
x : M
y : N
| ↑(↑B x) y
[PROOFSTEP]
rw [← b₁.total_repr x, ← b₂.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : M →ₛₗ[ρ₁₂] N →ₛₗ[σ₁₂] P
x : M
y : N
⊢ (Finsupp.sum (↑b₁.repr x) fun i xi =>
Finsupp.sum (↑b₂.repr y) fun j yj => ↑ρ₁₂ xi • ↑σ₁₂ yj • ↑(↑B (↑b₁ i)) (↑b₂ j)) =
↑(↑B (↑(Finsupp.total ι₁ M R ↑b₁) (↑b₁.repr x))) (↑(Finsupp.total ι₂ N S ↑b₂) (↑b₂.repr y))
[PROOFSTEP]
simp_rw [Finsupp.total_apply, Finsupp.sum, map_sum₂, map_sum, LinearMap.map_smulₛₗ₂, LinearMap.map_smulₛₗ]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : Mₗ →ₗ[R] Nₗ →ₗ[R] Pₗ
x : Mₗ
y : Nₗ
⊢ (Finsupp.sum (↑b₁'.repr x) fun i xi => Finsupp.sum (↑b₂'.repr y) fun j yj => xi • yj • ↑(↑B (↑b₁' i)) (↑b₂' j)) =
↑(↑B x) y
[PROOFSTEP]
conv_rhs => rw [← b₁'.total_repr x, ← b₂'.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : Mₗ →ₗ[R] Nₗ →ₗ[R] Pₗ
x : Mₗ
y : Nₗ
| ↑(↑B x) y
[PROOFSTEP]
rw [← b₁'.total_repr x, ← b₂'.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : Mₗ →ₗ[R] Nₗ →ₗ[R] Pₗ
x : Mₗ
y : Nₗ
| ↑(↑B x) y
[PROOFSTEP]
rw [← b₁'.total_repr x, ← b₂'.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : Mₗ →ₗ[R] Nₗ →ₗ[R] Pₗ
x : Mₗ
y : Nₗ
| ↑(↑B x) y
[PROOFSTEP]
rw [← b₁'.total_repr x, ← b₂'.total_repr y]
[GOAL]
ι₁ : Type u_1
ι₂ : Type u_2
R : Type u_3
R₂ : Type u_4
S : Type u_5
S₂ : Type u_6
M : Type u_7
N : Type u_8
P : Type u_9
Mₗ : Type u_10
Nₗ : Type u_11
Pₗ : Type u_12
inst✝¹⁷ : CommSemiring R
inst✝¹⁶ : CommSemiring S
inst✝¹⁵ : CommSemiring R₂
inst✝¹⁴ : CommSemiring S₂
inst✝¹³ : AddCommMonoid M
inst✝¹² : AddCommMonoid N
inst✝¹¹ : AddCommMonoid P
inst✝¹⁰ : AddCommMonoid Mₗ
inst✝⁹ : AddCommMonoid Nₗ
inst✝⁸ : AddCommMonoid Pₗ
inst✝⁷ : Module R M
inst✝⁶ : Module S N
inst✝⁵ : Module R₂ P
inst✝⁴ : Module S₂ P
inst✝³ : Module R Mₗ
inst✝² : Module R Nₗ
inst✝¹ : Module R Pₗ
inst✝ : SMulCommClass S₂ R₂ P
ρ₁₂ : R →+* R₂
σ₁₂ : S →+* S₂
b₁ : Basis ι₁ R M
b₂ : Basis ι₂ S N
b₁' : Basis ι₁ R Mₗ
b₂' : Basis ι₂ R Nₗ
B : Mₗ →ₗ[R] Nₗ →ₗ[R] Pₗ
x : Mₗ
y : Nₗ
⊢ (Finsupp.sum (↑b₁'.repr x) fun i xi => Finsupp.sum (↑b₂'.repr y) fun j yj => xi • yj • ↑(↑B (↑b₁' i)) (↑b₂' j)) =
↑(↑B (↑(Finsupp.total ι₁ Mₗ R ↑b₁') (↑b₁'.repr x))) (↑(Finsupp.total ι₂ Nₗ R ↑b₂') (↑b₂'.repr y))
[PROOFSTEP]
simp_rw [Finsupp.total_apply, Finsupp.sum, map_sum₂, map_sum, LinearMap.map_smul₂, LinearMap.map_smul]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Basis.Bilinear", "llama_tokens": 5115} |
[GOAL]
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
r : Rel β α
l : Filter β
a : α
⊢ RTendsto' r l (𝓝 a) ↔ ∀ (s : Set α), IsOpen s → a ∈ s → Rel.preimage r s ∈ l
[PROOFSTEP]
rw [rtendsto'_def]
[GOAL]
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
r : Rel β α
l : Filter β
a : α
⊢ (∀ (s : Set α), s ∈ 𝓝 a → Rel.preimage r s ∈ l) ↔ ∀ (s : Set α), IsOpen s → a ∈ s → Rel.preimage r s ∈ l
[PROOFSTEP]
apply all_mem_nhds_filter
[GOAL]
case hf
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
r : Rel β α
l : Filter β
a : α
⊢ ∀ (s t : Set α), s ⊆ t → Rel.preimage r s ⊆ Rel.preimage r t
[PROOFSTEP]
apply Rel.preimage_mono
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
h : PContinuous f
⊢ IsOpen (PFun.Dom f)
[PROOFSTEP]
rw [← PFun.preimage_univ]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
h : PContinuous f
⊢ IsOpen (PFun.preimage f Set.univ)
[PROOFSTEP]
exact h _ isOpen_univ
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
⊢ PContinuous f ↔ ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
⊢ PContinuous f → ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
[PROOFSTEP]
intro h x y h'
[GOAL]
case mp
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
h : PContinuous f
x : α
y : β
h' : y ∈ f x
⊢ PTendsto' f (𝓝 x) (𝓝 y)
[PROOFSTEP]
simp only [ptendsto'_def, mem_nhds_iff]
[GOAL]
case mp
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
h : PContinuous f
x : α
y : β
h' : y ∈ f x
⊢ ∀ (s : Set β), (∃ t, t ⊆ s ∧ IsOpen t ∧ y ∈ t) → ∃ t, t ⊆ PFun.preimage f s ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
rintro s ⟨t, tsubs, opent, yt⟩
[GOAL]
case mp.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
h : PContinuous f
x : α
y : β
h' : y ∈ f x
s t : Set β
tsubs : t ⊆ s
opent : IsOpen t
yt : y ∈ t
⊢ ∃ t, t ⊆ PFun.preimage f s ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
exact ⟨f.preimage t, PFun.preimage_mono _ tsubs, h _ opent, ⟨y, yt, h'⟩⟩
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
⊢ (∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)) → PContinuous f
[PROOFSTEP]
intro hf s os
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
⊢ IsOpen (PFun.preimage f s)
[PROOFSTEP]
rw [isOpen_iff_nhds]
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
⊢ ∀ (a : α), a ∈ PFun.preimage f s → 𝓝 a ≤ 𝓟 (PFun.preimage f s)
[PROOFSTEP]
rintro x ⟨y, ys, fxy⟩ t
[GOAL]
case mpr.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
⊢ t ∈ 𝓟 (PFun.preimage f s) → t ∈ 𝓝 x
[PROOFSTEP]
rw [mem_principal]
[GOAL]
case mpr.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
⊢ PFun.preimage f s ⊆ t → t ∈ 𝓝 x
[PROOFSTEP]
intro (h : f.preimage s ⊆ t)
[GOAL]
case mpr.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
⊢ t ∈ 𝓝 x
[PROOFSTEP]
change t ∈ 𝓝 x
[GOAL]
case mpr.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
⊢ t ∈ 𝓝 x
[PROOFSTEP]
apply mem_of_superset _ h
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
⊢ PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
have h' : ∀ s ∈ 𝓝 y, f.preimage s ∈ 𝓝 x := by
intro s hs
have : PTendsto' f (𝓝 x) (𝓝 y) := hf fxy
rw [ptendsto'_def] at this
exact this s hs
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
⊢ ∀ (s : Set β), s ∈ 𝓝 y → PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s✝ : Set β
os : IsOpen s✝
x : α
y : β
ys : y ∈ s✝
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s✝ ⊆ t
s : Set β
hs : s ∈ 𝓝 y
⊢ PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
have : PTendsto' f (𝓝 x) (𝓝 y) := hf fxy
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s✝ : Set β
os : IsOpen s✝
x : α
y : β
ys : y ∈ s✝
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s✝ ⊆ t
s : Set β
hs : s ∈ 𝓝 y
this : PTendsto' f (𝓝 x) (𝓝 y)
⊢ PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
rw [ptendsto'_def] at this
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s✝ : Set β
os : IsOpen s✝
x : α
y : β
ys : y ∈ s✝
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s✝ ⊆ t
s : Set β
hs : s ∈ 𝓝 y
this : ∀ (s : Set β), s ∈ 𝓝 y → PFun.preimage f s ∈ 𝓝 x
⊢ PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
exact this s hs
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
h' : ∀ (s : Set β), s ∈ 𝓝 y → PFun.preimage f s ∈ 𝓝 x
⊢ PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
show f.preimage s ∈ 𝓝 x
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
h' : ∀ (s : Set β), s ∈ 𝓝 y → PFun.preimage f s ∈ 𝓝 x
⊢ PFun.preimage f s ∈ 𝓝 x
[PROOFSTEP]
apply h'
[GOAL]
case a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
h' : ∀ (s : Set β), s ∈ 𝓝 y → PFun.preimage f s ∈ 𝓝 x
⊢ s ∈ 𝓝 y
[PROOFSTEP]
rw [mem_nhds_iff]
[GOAL]
case a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α →. β
hf : ∀ {x : α} {y : β}, y ∈ f x → PTendsto' f (𝓝 x) (𝓝 y)
s : Set β
os : IsOpen s
x : α
y : β
ys : y ∈ s
fxy : y ∈ f x
t : Set α
h : PFun.preimage f s ⊆ t
h' : ∀ (s : Set β), s ∈ 𝓝 y → PFun.preimage f s ∈ 𝓝 x
⊢ ∃ t, t ⊆ s ∧ IsOpen t ∧ y ∈ t
[PROOFSTEP]
exact ⟨s, Set.Subset.refl _, os, ys⟩
| {"mathlib_filename": "Mathlib.Topology.Partial", "llama_tokens": 4179} |
[GOAL]
α : Type u
inst✝ : Preorder α
c : Chain α
x : α
⊢ IsωSup c x ↔ IsLUB (range ↑c) x
[PROOFSTEP]
simp [IsωSup, IsLUB, IsLeast, upperBounds, lowerBounds]
[GOAL]
α : Type u
inst✝ : OmegaCompletePartialOrder α
s : Set (Set α)
hs : ∀ (t : Set α), t ∈ s → IsOpen α t
⊢ IsOpen α (⋃₀ s)
[PROOFSTEP]
simp only [IsOpen] at hs ⊢
[GOAL]
α : Type u
inst✝ : OmegaCompletePartialOrder α
s : Set (Set α)
hs : ∀ (t : Set α), t ∈ s → Continuous' fun x => x ∈ t
⊢ Continuous' fun x => x ∈ ⋃₀ s
[PROOFSTEP]
convert CompleteLattice.sSup_continuous' (setOf ⁻¹' s) hs
[GOAL]
case h.e'_5.h.a
α : Type u
inst✝ : OmegaCompletePartialOrder α
s : Set (Set α)
hs : ∀ (t : Set α), t ∈ s → Continuous' fun x => x ∈ t
x✝ : α
⊢ x✝ ∈ ⋃₀ s ↔ sSup (setOf ⁻¹' s) x✝
[PROOFSTEP]
simp only [sSup_apply, setOf_bijective.surjective.exists, exists_prop, mem_preimage, SetCoe.exists, iSup_Prop_eq,
mem_setOf_eq, mem_sUnion]
[GOAL]
α : Type u_1
inst✝ : OmegaCompletePartialOrder α
y : Scott α
⊢ IsOpen (notBelow y)
[PROOFSTEP]
have h : Monotone (notBelow y) := fun x z hle ↦ mt hle.trans
[GOAL]
α : Type u_1
inst✝ : OmegaCompletePartialOrder α
y : Scott α
h : Monotone (notBelow y)
⊢ IsOpen (notBelow y)
[PROOFSTEP]
refine ⟨h, fun c ↦ eq_of_forall_ge_iff fun z ↦ ?_⟩
[GOAL]
α : Type u_1
inst✝ : OmegaCompletePartialOrder α
y : Scott α
h : Monotone (notBelow y)
c : Chain α
z : Prop
⊢ ↑{ toFun := fun x => x ∈ notBelow y, monotone' := h } (ωSup c) ≤ z ↔
ωSup (Chain.map c { toFun := fun x => x ∈ notBelow y, monotone' := h }) ≤ z
[PROOFSTEP]
simp only [ωSup_le_iff, notBelow, mem_setOf_eq, le_Prop_eq, OrderHom.coe_mk, Chain.map_coe, Function.comp_apply,
exists_imp, not_forall]
[GOAL]
α : Type u_1
inst✝ : OmegaCompletePartialOrder α
c : Chain α
⊢ IsωSup c (ωSup c)
[PROOFSTEP]
constructor
[GOAL]
case left
α : Type u_1
inst✝ : OmegaCompletePartialOrder α
c : Chain α
⊢ ∀ (i : ℕ), ↑c i ≤ ωSup c
[PROOFSTEP]
apply le_ωSup
[GOAL]
case right
α : Type u_1
inst✝ : OmegaCompletePartialOrder α
c : Chain α
⊢ ∀ (y : α), (∀ (i : ℕ), ↑c i ≤ y) → ωSup c ≤ y
[PROOFSTEP]
apply ωSup_le
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : _root_.Continuous f
⊢ Continuous' f
[PROOFSTEP]
have h : Monotone f := fun x y h ↦
by
have hf : IsUpperSet {x | ¬f x ≤ f y} := ((notBelow_isOpen (f y)).preimage hf).isUpperSet
simpa only [mem_setOf_eq, le_refl, not_true, imp_false, not_not] using hf h
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : _root_.Continuous f
x y : Scott α
h : x ≤ y
⊢ f x ≤ f y
[PROOFSTEP]
have hf : IsUpperSet {x | ¬f x ≤ f y} := ((notBelow_isOpen (f y)).preimage hf).isUpperSet
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf✝ : _root_.Continuous f
x y : Scott α
h : x ≤ y
hf : IsUpperSet {x | ¬f x ≤ f y}
⊢ f x ≤ f y
[PROOFSTEP]
simpa only [mem_setOf_eq, le_refl, not_true, imp_false, not_not] using hf h
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : _root_.Continuous f
h : Monotone f
⊢ Continuous' f
[PROOFSTEP]
refine ⟨h, fun c ↦ eq_of_forall_ge_iff fun z ↦ ?_⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : _root_.Continuous f
h : Monotone f
c : Chain (Scott α)
z : Scott β
⊢ ↑{ toFun := f, monotone' := h } (ωSup c) ≤ z ↔ ωSup (Chain.map c { toFun := f, monotone' := h }) ≤ z
[PROOFSTEP]
rcases(notBelow_isOpen z).preimage hf with ⟨hf, hf'⟩
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf✝ : _root_.Continuous f
h : Monotone f
c : Chain (Scott α)
z : Scott β
hf : Monotone fun x => x ∈ f ⁻¹' notBelow z
hf' : OmegaCompletePartialOrder.Continuous { toFun := fun x => x ∈ f ⁻¹' notBelow z, monotone' := hf }
⊢ ↑{ toFun := f, monotone' := h } (ωSup c) ≤ z ↔ ωSup (Chain.map c { toFun := f, monotone' := h }) ≤ z
[PROOFSTEP]
specialize hf' c
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf✝ : _root_.Continuous f
h : Monotone f
c : Chain (Scott α)
z : Scott β
hf : Monotone fun x => x ∈ f ⁻¹' notBelow z
hf' :
↑{ toFun := fun x => x ∈ f ⁻¹' notBelow z, monotone' := hf } (ωSup c) =
ωSup (Chain.map c { toFun := fun x => x ∈ f ⁻¹' notBelow z, monotone' := hf })
⊢ ↑{ toFun := f, monotone' := h } (ωSup c) ≤ z ↔ ωSup (Chain.map c { toFun := f, monotone' := h }) ≤ z
[PROOFSTEP]
simp only [OrderHom.coe_mk, mem_preimage, notBelow, mem_setOf_eq] at hf'
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf✝ : _root_.Continuous f
h : Monotone f
c : Chain (Scott α)
z : Scott β
hf : Monotone fun x => x ∈ f ⁻¹' notBelow z
hf' :
(¬f (ωSup c) ≤ z) = ωSup (Chain.map c { toFun := fun x => ¬f x ≤ z, monotone' := (_ : Monotone fun x => ¬f x ≤ z) })
⊢ ↑{ toFun := f, monotone' := h } (ωSup c) ≤ z ↔ ωSup (Chain.map c { toFun := f, monotone' := h }) ≤ z
[PROOFSTEP]
rw [← not_iff_not]
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf✝ : _root_.Continuous f
h : Monotone f
c : Chain (Scott α)
z : Scott β
hf : Monotone fun x => x ∈ f ⁻¹' notBelow z
hf' :
(¬f (ωSup c) ≤ z) = ωSup (Chain.map c { toFun := fun x => ¬f x ≤ z, monotone' := (_ : Monotone fun x => ¬f x ≤ z) })
⊢ ¬↑{ toFun := f, monotone' := h } (ωSup c) ≤ z ↔ ¬ωSup (Chain.map c { toFun := f, monotone' := h }) ≤ z
[PROOFSTEP]
simp only [ωSup_le_iff, hf', ωSup, iSup, sSup, mem_range, Chain.map_coe, Function.comp_apply, eq_iff_iff, not_forall,
OrderHom.coe_mk]
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf✝ : _root_.Continuous f
h : Monotone f
c : Chain (Scott α)
z : Scott β
hf : Monotone fun x => x ∈ f ⁻¹' notBelow z
hf' :
(¬f (ωSup c) ≤ z) = ωSup (Chain.map c { toFun := fun x => ¬f x ≤ z, monotone' := (_ : Monotone fun x => ¬f x ≤ z) })
⊢ (∃ a, (∃ y, ¬f (↑c y) ≤ z ↔ a) ∧ a) ↔ ∃ x, ¬f (↑c x) ≤ z
[PROOFSTEP]
tauto
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : Continuous' f
⊢ _root_.Continuous f
[PROOFSTEP]
rw [continuous_def]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : Continuous' f
⊢ ∀ (s : Set (Scott β)), IsOpen s → IsOpen (f ⁻¹' s)
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : Continuous' f
s : Set (Scott β)
hs : IsOpen s
⊢ IsOpen (f ⁻¹' s)
[PROOFSTEP]
change Continuous' (s ∘ f)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : Continuous' f
s : Set (Scott β)
hs : IsOpen s
⊢ Continuous' (s ∘ f)
[PROOFSTEP]
cases' hs with hs hs'
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
hf : Continuous' f
s : Set (Scott β)
hs : Monotone fun x => x ∈ s
hs' : OmegaCompletePartialOrder.Continuous { toFun := fun x => x ∈ s, monotone' := hs }
⊢ Continuous' (s ∘ f)
[PROOFSTEP]
cases' hf with hf hf'
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
s : Set (Scott β)
hs : Monotone fun x => x ∈ s
hs' : OmegaCompletePartialOrder.Continuous { toFun := fun x => x ∈ s, monotone' := hs }
hf : Monotone f
hf' : OmegaCompletePartialOrder.Continuous { toFun := f, monotone' := hf }
⊢ Continuous' (s ∘ f)
[PROOFSTEP]
apply Continuous.of_bundled
[GOAL]
case intro.intro.hf'
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
s : Set (Scott β)
hs : Monotone fun x => x ∈ s
hs' : OmegaCompletePartialOrder.Continuous { toFun := fun x => x ∈ s, monotone' := hs }
hf : Monotone f
hf' : OmegaCompletePartialOrder.Continuous { toFun := f, monotone' := hf }
⊢ OmegaCompletePartialOrder.Continuous { toFun := s ∘ f, monotone' := ?intro.intro.hf }
case intro.intro.hf
α : Type u_1
β : Type u_2
inst✝¹ : OmegaCompletePartialOrder α
inst✝ : OmegaCompletePartialOrder β
f : Scott α → Scott β
s : Set (Scott β)
hs : Monotone fun x => x ∈ s
hs' : OmegaCompletePartialOrder.Continuous { toFun := fun x => x ∈ s, monotone' := hs }
hf : Monotone f
hf' : OmegaCompletePartialOrder.Continuous { toFun := f, monotone' := hf }
⊢ Monotone (s ∘ f)
[PROOFSTEP]
apply continuous_comp _ _ hf' hs'
| {"mathlib_filename": "Mathlib.Topology.OmegaCompletePartialOrder", "llama_tokens": 4195} |
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
hs : LinearIndependent K Subtype.val
⊢ ↑⊤ ⊆ ↑(span K (range (restrict (LinearIndependent.extend hs (_ : s ⊆ univ)) id)))
[PROOFSTEP]
simpa using hs.subset_span_extend (subset_univ s)
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
hs : LinearIndependent K Subtype.val
⊢ range ↑(extend hs) = LinearIndependent.extend hs (_ : s ⊆ univ)
[PROOFSTEP]
rw [coe_extend, Subtype.range_coe_subtype, setOf_mem_eq]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x✝ y z : V
x : ↑(ofVectorSpaceIndex K V)
⊢ ↑(ofVectorSpace K V) x = ↑x
[PROOFSTEP]
unfold ofVectorSpace
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x✝ y z : V
x : ↑(ofVectorSpaceIndex K V)
⊢ ↑(extend (_ : LinearIndependent K fun x => ↑x)) x = ↑x
[PROOFSTEP]
exact Basis.mk_apply _ _ _
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
⊢ LinearIndependent K Subtype.val
[PROOFSTEP]
convert (ofVectorSpace K V).linearIndependent
[GOAL]
case h.e'_4
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
⊢ Subtype.val = ↑(ofVectorSpace K V)
[PROOFSTEP]
ext x
[GOAL]
case h.e'_4.h
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x✝ y z : V
x : { x // x ∈ ofVectorSpaceIndex K V }
⊢ ↑x = ↑(ofVectorSpace K V) x
[PROOFSTEP]
rw [ofVectorSpace_apply_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁶ : DivisionRing K
inst✝⁵ : AddCommGroup V
inst✝⁴ : AddCommGroup V'
inst✝³ : Module K V
inst✝² : Module K V'
v : ι → V
s t : Set V
x y z : V
inst✝¹ : Fintype K
inst✝ : Fintype V
⊢ ∃ n, card V = card K ^ n
[PROOFSTEP]
classical exact ⟨card (Basis.ofVectorSpaceIndex K V), Module.card_fintype (Basis.ofVectorSpace K V)⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁶ : DivisionRing K
inst✝⁵ : AddCommGroup V
inst✝⁴ : AddCommGroup V'
inst✝³ : Module K V
inst✝² : Module K V'
v : ι → V
s t : Set V
x y z : V
inst✝¹ : Fintype K
inst✝ : Fintype V
⊢ ∃ n, card V = card K ^ n
[PROOFSTEP]
exact ⟨card (Basis.ofVectorSpaceIndex K V), Module.card_fintype (Basis.ofVectorSpace K V)⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
⊢ IsAtom (span K {v})
[PROOFSTEP]
constructor
[GOAL]
case left
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
⊢ span K {v} ≠ ⊥
[PROOFSTEP]
rw [Submodule.ne_bot_iff]
[GOAL]
case left
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
⊢ ∃ x, x ∈ span K {v} ∧ x ≠ 0
[PROOFSTEP]
exact ⟨v, ⟨mem_span_singleton_self v, hv⟩⟩
[GOAL]
case right
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
⊢ ∀ (b : Submodule K V), b < span K {v} → b = ⊥
[PROOFSTEP]
intro T hT
[GOAL]
case right
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
⊢ T = ⊥
[PROOFSTEP]
by_contra h
[GOAL]
case right
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
h : ¬T = ⊥
⊢ False
[PROOFSTEP]
apply hT.2
[GOAL]
case right
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
h : ¬T = ⊥
⊢ ↑(span K {v}) ⊆ ↑T
[PROOFSTEP]
change span K { v } ≤ T
[GOAL]
case right
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
h : ¬T = ⊥
⊢ span K {v} ≤ T
[PROOFSTEP]
simp_rw [span_singleton_le_iff_mem, ← Ne.def, Submodule.ne_bot_iff] at *
[GOAL]
case right
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
h : ∃ x, x ∈ T ∧ x ≠ 0
⊢ v ∈ T
[PROOFSTEP]
rcases h with ⟨s, ⟨hs, hz⟩⟩
[GOAL]
case right.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s✝ t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
s : V
hs : s ∈ T
hz : s ≠ 0
⊢ v ∈ T
[PROOFSTEP]
rcases mem_span_singleton.1 (hT.1 hs) with ⟨a, rfl⟩
[GOAL]
case right.intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
a : K
hs : a • v ∈ T
hz : a • v ≠ 0
⊢ v ∈ T
[PROOFSTEP]
rcases eq_or_ne a 0 with rfl | h
[GOAL]
case right.intro.intro.intro.inl
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
hs : 0 • v ∈ T
hz : 0 • v ≠ 0
⊢ v ∈ T
[PROOFSTEP]
simp only [zero_smul, ne_eq, not_true] at hz
[GOAL]
case right.intro.intro.intro.inr
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
T : Submodule K V
hT : T < span K {v}
a : K
hs : a • v ∈ T
hz : a • v ≠ 0
h : a ≠ 0
⊢ v ∈ T
[PROOFSTEP]
rwa [T.smul_mem_iff h] at hs
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
⊢ IsAtom W ↔ ∃ v x, W = span K {v}
[PROOFSTEP]
refine' ⟨fun h => _, fun h => _⟩
[GOAL]
case refine'_1
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
h : IsAtom W
⊢ ∃ v x, W = span K {v}
[PROOFSTEP]
cases' h with hbot h
[GOAL]
case refine'_1.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
hbot : W ≠ ⊥
h : ∀ (b : Submodule K V), b < W → b = ⊥
⊢ ∃ v x, W = span K {v}
[PROOFSTEP]
rcases(Submodule.ne_bot_iff W).1 hbot with ⟨v, ⟨hW, hv⟩⟩
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
W : Submodule K V
hbot : W ≠ ⊥
h : ∀ (b : Submodule K V), b < W → b = ⊥
v : V
hW : v ∈ W
hv : v ≠ 0
⊢ ∃ v x, W = span K {v}
[PROOFSTEP]
refine' ⟨v, ⟨hv, _⟩⟩
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
W : Submodule K V
hbot : W ≠ ⊥
h : ∀ (b : Submodule K V), b < W → b = ⊥
v : V
hW : v ∈ W
hv : v ≠ 0
⊢ W = span K {v}
[PROOFSTEP]
by_contra heq
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
W : Submodule K V
hbot : W ≠ ⊥
h : ∀ (b : Submodule K V), b < W → b = ⊥
v : V
hW : v ∈ W
hv : v ≠ 0
heq : ¬W = span K {v}
⊢ False
[PROOFSTEP]
specialize h (span K { v })
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
W : Submodule K V
hbot : W ≠ ⊥
v : V
hW : v ∈ W
hv : v ≠ 0
heq : ¬W = span K {v}
h : span K {v} < W → span K {v} = ⊥
⊢ False
[PROOFSTEP]
rw [span_singleton_eq_bot, lt_iff_le_and_ne] at h
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
W : Submodule K V
hbot : W ≠ ⊥
v : V
hW : v ∈ W
hv : v ≠ 0
heq : ¬W = span K {v}
h : span K {v} ≤ W ∧ span K {v} ≠ W → v = 0
⊢ False
[PROOFSTEP]
exact hv (h ⟨(span_singleton_le_iff_mem v W).2 hW, Ne.symm heq⟩)
[GOAL]
case refine'_2
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
h : ∃ v x, W = span K {v}
⊢ IsAtom W
[PROOFSTEP]
rcases h with ⟨v, ⟨hv, rfl⟩⟩
[GOAL]
case refine'_2.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z v : V
hv : v ≠ 0
⊢ IsAtom (span K {v})
[PROOFSTEP]
exact nonzero_span_atom v hv
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
⊢ ∃ s, W = sSup s ∧ ∀ (a : Submodule K V), a ∈ s → IsAtom a
[PROOFSTEP]
refine ⟨_, submodule_eq_sSup_le_nonzero_spans W, ?_⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
⊢ ∀ (a : Submodule K V), a ∈ {T | ∃ m x x, T = span K {m}} → IsAtom a
[PROOFSTEP]
rintro _ ⟨w, ⟨_, ⟨hw, rfl⟩⟩⟩
[GOAL]
case intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
W : Submodule K V
w : V
w✝ : w ∈ W
hw : w ≠ 0
⊢ IsAtom (span K {w})
[PROOFSTEP]
exact nonzero_span_atom w hw
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
⊢ ∃ g, comp g f = id
[PROOFSTEP]
let B := Basis.ofVectorSpaceIndex K V
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
⊢ ∃ g, comp g f = id
[PROOFSTEP]
let hB := Basis.ofVectorSpace K V
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
⊢ ∃ g, comp g f = id
[PROOFSTEP]
have hB₀ : _ := hB.linearIndependent.to_subtype_range
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
⊢ ∃ g, comp g f = id
[PROOFSTEP]
have : LinearIndependent K (fun x => x : f '' B → V') :=
by
have h₁ : LinearIndependent K ((↑) : ↥(f '' Set.range (Basis.ofVectorSpace K V)) → V') :=
@LinearIndependent.image_subtype _ _ _ _ _ _ _ _ _ f hB₀ (show Disjoint _ _ by simp [hf_inj])
rwa [Basis.range_ofVectorSpace K V] at h₁
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
⊢ LinearIndependent K fun x => ↑x
[PROOFSTEP]
have h₁ : LinearIndependent K ((↑) : ↥(f '' Set.range (Basis.ofVectorSpace K V)) → V') :=
@LinearIndependent.image_subtype _ _ _ _ _ _ _ _ _ f hB₀ (show Disjoint _ _ by simp [hf_inj])
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
⊢ Disjoint (span K (Set.range ↑(Basis.ofVectorSpace K V))) (ker f)
[PROOFSTEP]
simp [hf_inj]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
h₁ : LinearIndependent K Subtype.val
⊢ LinearIndependent K fun x => ↑x
[PROOFSTEP]
rwa [Basis.range_ofVectorSpace K V] at h₁
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
⊢ ∃ g, comp g f = id
[PROOFSTEP]
let C := this.extend (subset_univ _)
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
⊢ ∃ g, comp g f = id
[PROOFSTEP]
have BC := this.subset_extend (subset_univ _)
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : ↑f '' B ⊆ LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
⊢ ∃ g, comp g f = id
[PROOFSTEP]
let hC := Basis.extend this
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : ↑f '' B ⊆ LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
⊢ ∃ g, comp g f = id
[PROOFSTEP]
haveI Vinh : Inhabited V := ⟨0⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : ↑f '' B ⊆ LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
⊢ ∃ g, comp g f = id
[PROOFSTEP]
refine' ⟨(hC.constr ℕ : _ → _) (C.restrict (invFun f)), hB.ext fun b => _⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : ↑f '' B ⊆ LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
⊢ ↑(comp (↑(Basis.constr hC ℕ) (Set.restrict C (invFun ↑f))) f) (↑hB b) = ↑id (↑hB b)
[PROOFSTEP]
rw [image_subset_iff] at BC
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : B ⊆ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
⊢ ↑(comp (↑(Basis.constr hC ℕ) (Set.restrict C (invFun ↑f))) f) (↑hB b) = ↑id (↑hB b)
[PROOFSTEP]
have fb_eq : f b = hC ⟨f b, BC b.2⟩ := by
change f b = Basis.extend this _
simp_rw [Basis.extend_apply_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : B ⊆ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
⊢ ↑f ↑b = ↑hC { val := ↑f ↑b, property := (_ : ↑b ∈ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)) }
[PROOFSTEP]
change f b = Basis.extend this _
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : B ⊆ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
⊢ ↑f ↑b =
↑(Basis.extend this)
{ val := ↑f ↑b, property := (_ : ↑b ∈ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)) }
[PROOFSTEP]
simp_rw [Basis.extend_apply_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : B ⊆ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
fb_eq : ↑f ↑b = ↑hC { val := ↑f ↑b, property := (_ : ↑b ∈ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)) }
⊢ ↑(comp (↑(Basis.constr hC ℕ) (Set.restrict C (invFun ↑f))) f) (↑hB b) = ↑id (↑hB b)
[PROOFSTEP]
dsimp []
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : B ⊆ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
fb_eq : ↑f ↑b = ↑hC { val := ↑f ↑b, property := (_ : ↑b ∈ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)) }
⊢ ↑(↑(Basis.constr (Basis.extend this) ℕ)
(Set.restrict (LinearIndependent.extend this (_ : ↑f '' Basis.ofVectorSpaceIndex K V ⊆ univ)) (invFun ↑f)))
(↑f (↑(Basis.ofVectorSpace K V) b)) =
↑(Basis.ofVectorSpace K V) b
[PROOFSTEP]
rw [Basis.ofVectorSpace_apply_self, fb_eq, hC.constr_basis]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_inj : ker f = ⊥
B : Set V := Basis.ofVectorSpaceIndex K V
hB : Basis (↑(Basis.ofVectorSpaceIndex K V)) K V := Basis.ofVectorSpace K V
hB₀ : LinearIndependent K Subtype.val
this : LinearIndependent K fun x => ↑x
C : Set V' := LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
BC : B ⊆ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)
hC : Basis (↑(LinearIndependent.extend this (_ : ↑f '' B ⊆ univ))) K V' := Basis.extend this
Vinh : Inhabited V
b : ↑(Basis.ofVectorSpaceIndex K V)
fb_eq : ↑f ↑b = ↑hC { val := ↑f ↑b, property := (_ : ↑b ∈ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)) }
⊢ Set.restrict (LinearIndependent.extend this (_ : ↑f '' Basis.ofVectorSpaceIndex K V ⊆ univ)) (invFun ↑f)
{ val := ↑f ↑b, property := (_ : ↑b ∈ ↑f ⁻¹' LinearIndependent.extend this (_ : ↑f '' B ⊆ univ)) } =
↑b
[PROOFSTEP]
exact leftInverse_invFun (LinearMap.ker_eq_bot.1 hf_inj) _
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_surj : range f = ⊤
⊢ ∃ g, comp f g = id
[PROOFSTEP]
let C := Basis.ofVectorSpaceIndex K V'
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_surj : range f = ⊤
C : Set V' := Basis.ofVectorSpaceIndex K V'
⊢ ∃ g, comp f g = id
[PROOFSTEP]
let hC := Basis.ofVectorSpace K V'
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_surj : range f = ⊤
C : Set V' := Basis.ofVectorSpaceIndex K V'
hC : Basis (↑(Basis.ofVectorSpaceIndex K V')) K V' := Basis.ofVectorSpace K V'
⊢ ∃ g, comp f g = id
[PROOFSTEP]
haveI : Inhabited V := ⟨0⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_surj : range f = ⊤
C : Set V' := Basis.ofVectorSpaceIndex K V'
hC : Basis (↑(Basis.ofVectorSpaceIndex K V')) K V' := Basis.ofVectorSpace K V'
this : Inhabited V
⊢ ∃ g, comp f g = id
[PROOFSTEP]
refine' ⟨(hC.constr ℕ : _ → _) (C.restrict (invFun f)), hC.ext fun c => _⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_surj : range f = ⊤
C : Set V' := Basis.ofVectorSpaceIndex K V'
hC : Basis (↑(Basis.ofVectorSpaceIndex K V')) K V' := Basis.ofVectorSpace K V'
this : Inhabited V
c : ↑(Basis.ofVectorSpaceIndex K V')
⊢ ↑(comp f (↑(Basis.constr hC ℕ) (Set.restrict C (invFun ↑f)))) (↑hC c) = ↑id (↑hC c)
[PROOFSTEP]
rw [LinearMap.comp_apply, hC.constr_basis]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
f : V →ₗ[K] V'
hf_surj : range f = ⊤
C : Set V' := Basis.ofVectorSpaceIndex K V'
hC : Basis (↑(Basis.ofVectorSpaceIndex K V')) K V' := Basis.ofVectorSpace K V'
this : Inhabited V
c : ↑(Basis.ofVectorSpaceIndex K V')
⊢ ↑f (Set.restrict C (invFun ↑f) c) = ↑id (↑hC c)
[PROOFSTEP]
simp [rightInverse_invFun (LinearMap.range_eq_top.1 hf_surj) c]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
p : Submodule K V
f : { x // x ∈ p } →ₗ[K] V'
g : V →ₗ[K] { x // x ∈ p }
hg : comp g (Submodule.subtype p) = id
⊢ comp (comp f g) (Submodule.subtype p) = f
[PROOFSTEP]
rw [LinearMap.comp_assoc, hg, f.comp_id]
[GOAL]
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v : ι → V
s t : Set V
x y z : V
p : Submodule K V
hp : p < ⊤
⊢ ∃ f, f ≠ 0 ∧ p ≤ ker f
[PROOFSTEP]
rcases SetLike.exists_of_lt hp with ⟨v, -, hpv⟩
[GOAL]
case intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
hp : p < ⊤
v : V
hpv : ¬v ∈ p
⊢ ∃ f, f ≠ 0 ∧ p ≤ ker f
[PROOFSTEP]
clear hp
[GOAL]
case intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
⊢ ∃ f, f ≠ 0 ∧ p ≤ ker f
[PROOFSTEP]
rcases(LinearPMap.supSpanSingleton ⟨p, 0⟩ v (1 : K) hpv).toFun.exists_extend with ⟨f, hf⟩
[GOAL]
case intro.intro.intro
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
f : V →ₗ[K] K
hf :
LinearMap.comp f (Submodule.subtype (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).domain) =
(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
⊢ ∃ f, f ≠ 0 ∧ p ≤ ker f
[PROOFSTEP]
refine' ⟨f, _, _⟩
[GOAL]
case intro.intro.intro.refine'_1
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
f : V →ₗ[K] K
hf :
LinearMap.comp f (Submodule.subtype (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).domain) =
(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
⊢ f ≠ 0
[PROOFSTEP]
rintro rfl
[GOAL]
case intro.intro.intro.refine'_1
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
hf :
LinearMap.comp 0 (Submodule.subtype (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).domain) =
(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
⊢ False
[PROOFSTEP]
rw [LinearMap.zero_comp] at hf
[GOAL]
case intro.intro.intro.refine'_1
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
hf : 0 = (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
⊢ False
[PROOFSTEP]
have := LinearPMap.supSpanSingleton_apply_mk ⟨p, 0⟩ v (1 : K) hpv 0 p.zero_mem 1
[GOAL]
case intro.intro.intro.refine'_1
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
hf : 0 = (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
this :
↑(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv)
{ val := 0 + 1 • v,
property :=
(_ :
0 + 1 • v ∈
{ domain := p, toFun := 0 }.domain ⊔ (LinearPMap.mkSpanSingleton v 1 (_ : v = 0 → False)).domain) } =
↑{ domain := p, toFun := 0 } { val := 0, property := (_ : 0 ∈ p) } + 1 • 1
⊢ False
[PROOFSTEP]
simpa using (LinearMap.congr_fun hf _).trans this
[GOAL]
case intro.intro.intro.refine'_2
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
f : V →ₗ[K] K
hf :
LinearMap.comp f (Submodule.subtype (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).domain) =
(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
⊢ p ≤ ker f
[PROOFSTEP]
refine' fun x hx => mem_ker.2 _
[GOAL]
case intro.intro.intro.refine'_2
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x✝ y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
f : V →ₗ[K] K
hf :
LinearMap.comp f (Submodule.subtype (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).domain) =
(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
x : V
hx : x ∈ p
⊢ ↑f x = 0
[PROOFSTEP]
have := LinearPMap.supSpanSingleton_apply_mk ⟨p, 0⟩ v (1 : K) hpv x hx 0
[GOAL]
case intro.intro.intro.refine'_2
ι : Type u_1
ι' : Type u_2
K : Type u_3
V : Type u_4
V' : Type u_5
inst✝⁴ : DivisionRing K
inst✝³ : AddCommGroup V
inst✝² : AddCommGroup V'
inst✝¹ : Module K V
inst✝ : Module K V'
v✝ : ι → V
s t : Set V
x✝ y z : V
p : Submodule K V
v : V
hpv : ¬v ∈ p
f : V →ₗ[K] K
hf :
LinearMap.comp f (Submodule.subtype (LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).domain) =
(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv).toFun
x : V
hx : x ∈ p
this :
↑(LinearPMap.supSpanSingleton { domain := p, toFun := 0 } v 1 hpv)
{ val := x + 0 • v,
property :=
(_ :
x + 0 • v ∈
{ domain := p, toFun := 0 }.domain ⊔ (LinearPMap.mkSpanSingleton v 1 (_ : v = 0 → False)).domain) } =
↑{ domain := p, toFun := 0 } { val := x, property := hx } + 0 • 1
⊢ ↑f x = 0
[PROOFSTEP]
simpa using (LinearMap.congr_fun hf _).trans this
| {"mathlib_filename": "Mathlib.LinearAlgebra.Basis.VectorSpace", "llama_tokens": 17519} |
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
j : ι
⊢ ↑(↑(fromMatrix R b) A) (Pi.single j 1) = ∑ i : ι, A i j • b i
[PROOFSTEP]
rw [PiToModule.fromMatrix_apply, Fintype.total_apply, Matrix.mulVec_single]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
j : ι
⊢ ∑ i : ι, (fun i => A i j * 1) i • b i = ∑ i : ι, A i j • b i
[PROOFSTEP]
simp_rw [mul_one]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
i : ι
⊢ ↑(↑(fromEnd R b) f) (Pi.single i 1) = ↑f (b i)
[PROOFSTEP]
rw [PiToModule.fromEnd_apply]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
i : ι
⊢ ↑f (↑(↑(Fintype.total R R) b) (Pi.single i 1)) = ↑f (b i)
[PROOFSTEP]
congr
[GOAL]
case h.e_6.h
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
i : ι
⊢ ↑(↑(Fintype.total R R) b) (Pi.single i 1) = b i
[PROOFSTEP]
convert Fintype.total_apply_single (S := R) R b i (1 : R)
[GOAL]
case h.e'_3
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
i : ι
⊢ b i = 1 • b i
[PROOFSTEP]
rw [one_smul]
[GOAL]
ι : Type u_1
inst✝³ : Fintype ι
M : Type u_2
inst✝² : AddCommGroup M
R : Type u_3
inst✝¹ : CommRing R
inst✝ : Module R M
I : Ideal R
b : ι → M
hb✝ hb : Submodule.span R (Set.range b) = ⊤
⊢ Function.Injective ↑(fromEnd R b)
[PROOFSTEP]
intro x y e
[GOAL]
ι : Type u_1
inst✝³ : Fintype ι
M : Type u_2
inst✝² : AddCommGroup M
R : Type u_3
inst✝¹ : CommRing R
inst✝ : Module R M
I : Ideal R
b : ι → M
hb✝ hb : Submodule.span R (Set.range b) = ⊤
x y : Module.End R M
e : ↑(fromEnd R b) x = ↑(fromEnd R b) y
⊢ x = y
[PROOFSTEP]
ext m
[GOAL]
case h
ι : Type u_1
inst✝³ : Fintype ι
M : Type u_2
inst✝² : AddCommGroup M
R : Type u_3
inst✝¹ : CommRing R
inst✝ : Module R M
I : Ideal R
b : ι → M
hb✝ hb : Submodule.span R (Set.range b) = ⊤
x y : Module.End R M
e : ↑(fromEnd R b) x = ↑(fromEnd R b) y
m : M
⊢ ↑x m = ↑y m
[PROOFSTEP]
obtain ⟨m, rfl⟩ : m ∈ LinearMap.range (Fintype.total R R b) :=
by
rw [(Fintype.range_total R b).trans hb]
exact Submodule.mem_top
[GOAL]
ι : Type u_1
inst✝³ : Fintype ι
M : Type u_2
inst✝² : AddCommGroup M
R : Type u_3
inst✝¹ : CommRing R
inst✝ : Module R M
I : Ideal R
b : ι → M
hb✝ hb : Submodule.span R (Set.range b) = ⊤
x y : Module.End R M
e : ↑(fromEnd R b) x = ↑(fromEnd R b) y
m : M
⊢ m ∈ LinearMap.range (↑(Fintype.total R R) b)
[PROOFSTEP]
rw [(Fintype.range_total R b).trans hb]
[GOAL]
ι : Type u_1
inst✝³ : Fintype ι
M : Type u_2
inst✝² : AddCommGroup M
R : Type u_3
inst✝¹ : CommRing R
inst✝ : Module R M
I : Ideal R
b : ι → M
hb✝ hb : Submodule.span R (Set.range b) = ⊤
x y : Module.End R M
e : ↑(fromEnd R b) x = ↑(fromEnd R b) y
m : M
⊢ m ∈ ⊤
[PROOFSTEP]
exact Submodule.mem_top
[GOAL]
case h.intro
ι : Type u_1
inst✝³ : Fintype ι
M : Type u_2
inst✝² : AddCommGroup M
R : Type u_3
inst✝¹ : CommRing R
inst✝ : Module R M
I : Ideal R
b : ι → M
hb✝ hb : Submodule.span R (Set.range b) = ⊤
x y : Module.End R M
e : ↑(fromEnd R b) x = ↑(fromEnd R b) y
m : ι → R
⊢ ↑x (↑(↑(Fintype.total R R) b) m) = ↑y (↑(↑(Fintype.total R R) b) m)
[PROOFSTEP]
exact (LinearMap.congr_fun e m : _)
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
⊢ Represents b A f ↔ ∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)
[PROOFSTEP]
constructor
[GOAL]
case mp
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
⊢ Represents b A f → ∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)
[PROOFSTEP]
intro h i
[GOAL]
case mp
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : Represents b A f
i : ι
⊢ ∑ i_1 : ι, A i_1 i • b i_1 = ↑f (b i)
[PROOFSTEP]
have := LinearMap.congr_fun h (Pi.single i 1)
[GOAL]
case mp
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : Represents b A f
i : ι
this : ↑(↑(PiToModule.fromMatrix R b) A) (Pi.single i 1) = ↑(↑(PiToModule.fromEnd R b) f) (Pi.single i 1)
⊢ ∑ i_1 : ι, A i_1 i • b i_1 = ↑f (b i)
[PROOFSTEP]
rwa [PiToModule.fromEnd_apply_single_one, PiToModule.fromMatrix_apply_single_one] at this
[GOAL]
case mpr
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
⊢ (∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)) → Represents b A f
[PROOFSTEP]
intro h
[GOAL]
case mpr
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : ∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)
⊢ Represents b A f
[PROOFSTEP]
refine LinearMap.pi_ext' (fun i => LinearMap.ext_ring ?_)
[GOAL]
case mpr
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : ∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)
i : ι
⊢ ↑(LinearMap.comp (↑(PiToModule.fromMatrix R b) A) (LinearMap.single i)) 1 =
↑(LinearMap.comp (↑(PiToModule.fromEnd R b) f) (LinearMap.single i)) 1
[PROOFSTEP]
simp_rw [LinearMap.comp_apply, LinearMap.coe_single, PiToModule.fromEnd_apply_single_one,
PiToModule.fromMatrix_apply_single_one]
[GOAL]
case mpr
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : ∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)
i : ι
⊢ ∑ i_1 : ι, A i_1 i • b i_1 = ↑f (b i)
[PROOFSTEP]
apply h
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
⊢ Represents b (A * A') (f * f')
[PROOFSTEP]
delta Matrix.Represents PiToModule.fromMatrix
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
⊢ ↑(LinearMap.comp (↑(LinearMap.llcomp R (ι → R) (ι → R) M) (↑(Fintype.total R R) b))
(AlgEquiv.toLinearMap (AlgEquiv.symm algEquivMatrix')))
(A * A') =
↑(PiToModule.fromEnd R b) (f * f')
[PROOFSTEP]
rw [LinearMap.comp_apply, AlgEquiv.toLinearMap_apply, _root_.map_mul]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
⊢ ↑(↑(LinearMap.llcomp R (ι → R) (ι → R) M) (↑(Fintype.total R R) b))
(↑(AlgEquiv.symm algEquivMatrix') A * ↑(AlgEquiv.symm algEquivMatrix') A') =
↑(PiToModule.fromEnd R b) (f * f')
[PROOFSTEP]
ext
[GOAL]
case h.h
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
i✝ : ι
⊢ ↑(LinearMap.comp
(↑(↑(LinearMap.llcomp R (ι → R) (ι → R) M) (↑(Fintype.total R R) b))
(↑(AlgEquiv.symm algEquivMatrix') A * ↑(AlgEquiv.symm algEquivMatrix') A'))
(LinearMap.single i✝))
1 =
↑(LinearMap.comp (↑(PiToModule.fromEnd R b) (f * f')) (LinearMap.single i✝)) 1
[PROOFSTEP]
dsimp [PiToModule.fromEnd]
[GOAL]
case h.h
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
i✝ : ι
⊢ ↑(↑(Fintype.total R R) b)
(↑(↑(AlgEquiv.symm algEquivMatrix') A) (↑(↑(AlgEquiv.symm algEquivMatrix') A') (Pi.single i✝ 1))) =
↑f (↑f' (↑(↑(Fintype.total R R) b) (Pi.single i✝ 1)))
[PROOFSTEP]
rw [← h'.congr_fun, ← h.congr_fun]
[GOAL]
case h.h
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
i✝ : ι
⊢ ↑(↑(Fintype.total R R) b)
(↑(↑(AlgEquiv.symm algEquivMatrix') A) (↑(↑(AlgEquiv.symm algEquivMatrix') A') (Pi.single i✝ 1))) =
↑(↑(Fintype.total R R) b) (mulVec A (mulVec A' (Pi.single i✝ 1)))
[PROOFSTEP]
rfl
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
⊢ Represents b 1 1
[PROOFSTEP]
delta Matrix.Represents PiToModule.fromMatrix
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
⊢ ↑(LinearMap.comp (↑(LinearMap.llcomp R (ι → R) (ι → R) M) (↑(Fintype.total R R) b))
(AlgEquiv.toLinearMap (AlgEquiv.symm algEquivMatrix')))
1 =
↑(PiToModule.fromEnd R b) 1
[PROOFSTEP]
rw [LinearMap.comp_apply, AlgEquiv.toLinearMap_apply, _root_.map_one]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
⊢ ↑(↑(LinearMap.llcomp R (ι → R) (ι → R) M) (↑(Fintype.total R R) b)) 1 = ↑(PiToModule.fromEnd R b) 1
[PROOFSTEP]
ext
[GOAL]
case h.h
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
i✝ : ι
⊢ ↑(LinearMap.comp (↑(↑(LinearMap.llcomp R (ι → R) (ι → R) M) (↑(Fintype.total R R) b)) 1) (LinearMap.single i✝)) 1 =
↑(LinearMap.comp (↑(PiToModule.fromEnd R b) 1) (LinearMap.single i✝)) 1
[PROOFSTEP]
rfl
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : Represents b A f
h' : Represents b A' f'
⊢ Represents b (A + A') (f + f')
[PROOFSTEP]
delta Matrix.Represents at h h' ⊢
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A A' : Matrix ι ι R
f f' : Module.End R M
h : ↑(PiToModule.fromMatrix R b) A = ↑(PiToModule.fromEnd R b) f
h' : ↑(PiToModule.fromMatrix R b) A' = ↑(PiToModule.fromEnd R b) f'
⊢ ↑(PiToModule.fromMatrix R b) (A + A') = ↑(PiToModule.fromEnd R b) (f + f')
[PROOFSTEP]
rw [map_add, map_add, h, h']
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
⊢ Represents b 0 0
[PROOFSTEP]
delta Matrix.Represents
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
⊢ ↑(PiToModule.fromMatrix R b) 0 = ↑(PiToModule.fromEnd R b) 0
[PROOFSTEP]
rw [map_zero, map_zero]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : Represents b A f
r : R
⊢ Represents b (r • A) (r • f)
[PROOFSTEP]
delta Matrix.Represents at h ⊢
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
A : Matrix ι ι R
f : Module.End R M
h : ↑(PiToModule.fromMatrix R b) A = ↑(PiToModule.fromEnd R b) f
r : R
⊢ ↑(PiToModule.fromMatrix R b) (r • A) = ↑(PiToModule.fromEnd R b) (r • f)
[PROOFSTEP]
rw [SMulHomClass.map_smul, SMulHomClass.map_smul, h]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
⊢ ∃ M_1, ↑(toEnd R b hb) M_1 = f ∧ ∀ (i j : ι), ↑M_1 i j ∈ I
[PROOFSTEP]
have : ∀ x, f x ∈ LinearMap.range (Ideal.finsuppTotal ι M I b) :=
by
rw [Ideal.range_finsuppTotal, hb]
exact fun x => hI (LinearMap.mem_range_self f x)
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
⊢ ∀ (x : M), ↑f x ∈ LinearMap.range (Ideal.finsuppTotal ι M I b)
[PROOFSTEP]
rw [Ideal.range_finsuppTotal, hb]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
⊢ ∀ (x : M), ↑f x ∈ I • ⊤
[PROOFSTEP]
exact fun x => hI (LinearMap.mem_range_self f x)
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
this : ∀ (x : M), ↑f x ∈ LinearMap.range (Ideal.finsuppTotal ι M I b)
⊢ ∃ M_1, ↑(toEnd R b hb) M_1 = f ∧ ∀ (i j : ι), ↑M_1 i j ∈ I
[PROOFSTEP]
choose bM' hbM' using this
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
⊢ ∃ M_1, ↑(toEnd R b hb) M_1 = f ∧ ∀ (i j : ι), ↑M_1 i j ∈ I
[PROOFSTEP]
let A : Matrix ι ι R := fun i j => bM' (b j) i
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
⊢ ∃ M_1, ↑(toEnd R b hb) M_1 = f ∧ ∀ (i j : ι), ↑M_1 i j ∈ I
[PROOFSTEP]
have : A.Represents b f := by
rw [Matrix.represents_iff']
dsimp
intro j
specialize hbM' (b j)
rwa [Ideal.finsuppTotal_apply_eq_of_fintype] at hbM'
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
⊢ Represents b A f
[PROOFSTEP]
rw [Matrix.represents_iff']
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
⊢ ∀ (j : ι), ∑ i : ι, A i j • b i = ↑f (b j)
[PROOFSTEP]
dsimp
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
⊢ ∀ (j : ι), ∑ i : ι, ↑(↑(bM' (b j)) i) • b i = ↑f (b j)
[PROOFSTEP]
intro j
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
j : ι
⊢ ∑ i : ι, ↑(↑(bM' (b j)) i) • b i = ↑f (b j)
[PROOFSTEP]
specialize hbM' (b j)
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
j : ι
hbM' : ↑(Ideal.finsuppTotal ι M I b) (bM' (b j)) = ↑f (b j)
⊢ ∑ i : ι, ↑(↑(bM' (b j)) i) • b i = ↑f (b j)
[PROOFSTEP]
rwa [Ideal.finsuppTotal_apply_eq_of_fintype] at hbM'
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
I : Ideal R
hI : LinearMap.range f ≤ I • ⊤
bM' : M → ι →₀ { x // x ∈ I }
hbM' : ∀ (x : M), ↑(Ideal.finsuppTotal ι M I b) (bM' x) = ↑f x
A : Matrix ι ι R := fun i j => ↑(↑(bM' (b j)) i)
this : Represents b A f
⊢ ∃ M_1, ↑(toEnd R b hb) M_1 = f ∧ ∀ (i j : ι), ↑M_1 i j ∈ I
[PROOFSTEP]
exact
⟨⟨A, f, this⟩, Matrix.isRepresentation.eq_toEnd_of_represents R b hb ⟨A, f, this⟩ this, fun i j => (bM' (b j) i).prop⟩
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
⊢ Function.Surjective ↑(toEnd R b hb)
[PROOFSTEP]
intro f
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
⊢ ∃ a, ↑(toEnd R b hb) a = f
[PROOFSTEP]
obtain ⟨M, e, -⟩ := Matrix.isRepresentation.toEnd_exists_mem_ideal R b hb f ⊤ (by simp)
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M
⊢ LinearMap.range f ≤ ⊤ • ⊤
[PROOFSTEP]
simp
[GOAL]
case intro.intro
ι : Type u_1
inst✝⁴ : Fintype ι
M✝ : Type u_2
inst✝³ : AddCommGroup M✝
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M✝
I : Ideal R
b : ι → M✝
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : DecidableEq ι
f : Module.End R M✝
M : { x // x ∈ isRepresentation R b }
e : ↑(toEnd R b hb) M = f
⊢ ∃ a, ↑(toEnd R b hb) a = f
[PROOFSTEP]
exact ⟨M, e⟩
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
⊢ ∃ p, Monic p ∧ (∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧ ↑(aeval f) p = 0
[PROOFSTEP]
classical
cases subsingleton_or_nontrivial R
· exact ⟨0, Polynomial.monic_of_subsingleton _, by simp⟩
obtain ⟨s : Finset M, hs : Submodule.span R (s : Set M) = ⊤⟩ :=
Module.Finite.out (R := R) (M := M)
-- Porting note: `H` was `rfl`
obtain ⟨A, H, h⟩ :=
Matrix.isRepresentation.toEnd_exists_mem_ideal R ((↑) : s → M)
(by rw [Subtype.range_coe_subtype, Finset.setOf_mem, hs]) f I hI
rw [← H]
refine' ⟨A.1.charpoly, A.1.charpoly_monic, _, _⟩
· rw [A.1.charpoly_natDegree_eq_dim]
exact coeff_charpoly_mem_ideal_pow h
· rw [Polynomial.aeval_algHom_apply, ← map_zero (Matrix.isRepresentation.toEnd R ((↑) : s → M) _)]
congr 1
ext1
rw [Polynomial.aeval_subalgebra_coe, Matrix.aeval_self_charpoly, Subalgebra.coe_zero]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
⊢ ∃ p, Monic p ∧ (∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧ ↑(aeval f) p = 0
[PROOFSTEP]
cases subsingleton_or_nontrivial R
[GOAL]
case inl
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Subsingleton R
⊢ ∃ p, Monic p ∧ (∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧ ↑(aeval f) p = 0
[PROOFSTEP]
exact ⟨0, Polynomial.monic_of_subsingleton _, by simp⟩
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Subsingleton R
⊢ (∀ (k : ℕ), coeff 0 k ∈ I ^ (natDegree 0 - k)) ∧ ↑(aeval f) 0 = 0
[PROOFSTEP]
simp
[GOAL]
case inr
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
⊢ ∃ p, Monic p ∧ (∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧ ↑(aeval f) p = 0
[PROOFSTEP]
obtain ⟨s : Finset M, hs : Submodule.span R (s : Set M) = ⊤⟩ :=
Module.Finite.out (R := R) (M := M)
-- Porting note: `H` was `rfl`
[GOAL]
case inr.intro
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
⊢ ∃ p, Monic p ∧ (∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧ ↑(aeval f) p = 0
[PROOFSTEP]
obtain ⟨A, H, h⟩ :=
Matrix.isRepresentation.toEnd_exists_mem_ideal R ((↑) : s → M)
(by rw [Subtype.range_coe_subtype, Finset.setOf_mem, hs]) f I hI
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
⊢ Submodule.span R (Set.range Subtype.val) = ⊤
[PROOFSTEP]
rw [Subtype.range_coe_subtype, Finset.setOf_mem, hs]
[GOAL]
case inr.intro.intro.intro
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ∃ p, Monic p ∧ (∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧ ↑(aeval f) p = 0
[PROOFSTEP]
rw [← H]
[GOAL]
case inr.intro.intro.intro
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ∃ p,
Monic p ∧
(∀ (k : ℕ), coeff p k ∈ I ^ (natDegree p - k)) ∧
↑(aeval (↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A))
p =
0
[PROOFSTEP]
refine' ⟨A.1.charpoly, A.1.charpoly_monic, _, _⟩
[GOAL]
case inr.intro.intro.intro.refine'_1
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ∀ (k : ℕ), coeff (Matrix.charpoly ↑A) k ∈ I ^ (natDegree (Matrix.charpoly ↑A) - k)
[PROOFSTEP]
rw [A.1.charpoly_natDegree_eq_dim]
[GOAL]
case inr.intro.intro.intro.refine'_1
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ∀ (k : ℕ), coeff (Matrix.charpoly ↑A) k ∈ I ^ (Fintype.card { x // x ∈ s } - k)
[PROOFSTEP]
exact coeff_charpoly_mem_ideal_pow h
[GOAL]
case inr.intro.intro.intro.refine'_2
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ↑(aeval (↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A))
(Matrix.charpoly ↑A) =
0
[PROOFSTEP]
rw [Polynomial.aeval_algHom_apply, ← map_zero (Matrix.isRepresentation.toEnd R ((↑) : s → M) _)]
[GOAL]
case inr.intro.intro.intro.refine'_2
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤))
(↑(aeval A) (Matrix.charpoly ↑A)) =
↑(Matrix.isRepresentation.toEnd R Subtype.val ?m.193133) 0
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ Submodule.span R (Set.range Subtype.val) = ⊤
[PROOFSTEP]
congr 1
[GOAL]
case inr.intro.intro.intro.refine'_2.h.e_6.h
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ↑(aeval A) (Matrix.charpoly ↑A) = 0
[PROOFSTEP]
ext1
[GOAL]
case inr.intro.intro.intro.refine'_2.h.e_6.h.a
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I✝ : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
I : Ideal R
hI : range f ≤ I • ⊤
h✝ : Nontrivial R
s : Finset M
hs : Submodule.span R ↑s = ⊤
A : { x // x ∈ Matrix.isRepresentation R Subtype.val }
H : ↑(Matrix.isRepresentation.toEnd R Subtype.val (_ : Submodule.span R (Set.range Subtype.val) = ⊤)) A = f
h : ∀ (i j : { x // x ∈ s }), ↑A i j ∈ I
⊢ ↑(↑(aeval A) (Matrix.charpoly ↑A)) = ↑0
[PROOFSTEP]
rw [Polynomial.aeval_subalgebra_coe, Matrix.aeval_self_charpoly, Subalgebra.coe_zero]
[GOAL]
ι : Type u_1
inst✝⁴ : Fintype ι
M : Type u_2
inst✝³ : AddCommGroup M
R : Type u_3
inst✝² : CommRing R
inst✝¹ : Module R M
I : Ideal R
b : ι → M
hb : Submodule.span R (Set.range b) = ⊤
inst✝ : Module.Finite R M
f : Module.End R M
⊢ range f ≤ ⊤ • ⊤
[PROOFSTEP]
simp
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Charpoly.LinearMap", "llama_tokens": 16626} |
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
⊢ ContinuousOn (extendFrom A f) B
[PROOFSTEP]
set φ := extendFrom A f
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
⊢ ContinuousOn φ B
[PROOFSTEP]
intro x x_in
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
⊢ ContinuousWithinAt φ B x
[PROOFSTEP]
suffices ∀ V' ∈ 𝓝 (φ x), IsClosed V' → φ ⁻¹' V' ∈ 𝓝[B] x by
simpa [ContinuousWithinAt, (closed_nhds_basis (φ x)).tendsto_right_iff]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
this : ∀ (V' : Set Y), V' ∈ 𝓝 (φ x) → IsClosed V' → φ ⁻¹' V' ∈ 𝓝[B] x
⊢ ContinuousWithinAt φ B x
[PROOFSTEP]
simpa [ContinuousWithinAt, (closed_nhds_basis (φ x)).tendsto_right_iff]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
⊢ ∀ (V' : Set Y), V' ∈ 𝓝 (φ x) → IsClosed V' → φ ⁻¹' V' ∈ 𝓝[B] x
[PROOFSTEP]
intro V' V'_in V'_closed
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
⊢ φ ⁻¹' V' ∈ 𝓝[B] x
[PROOFSTEP]
obtain ⟨V, V_in, V_op, hV⟩ : ∃ V ∈ 𝓝 x, IsOpen V ∧ V ∩ A ⊆ f ⁻¹' V' :=
by
have := tendsto_extendFrom (hf x x_in)
rcases(nhdsWithin_basis_open x A).tendsto_left_iff.mp this V' V'_in with ⟨V, ⟨hxV, V_op⟩, hV⟩
exact ⟨V, IsOpen.mem_nhds V_op hxV, V_op, hV⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
⊢ ∃ V, V ∈ 𝓝 x ∧ IsOpen V ∧ V ∩ A ⊆ f ⁻¹' V'
[PROOFSTEP]
have := tendsto_extendFrom (hf x x_in)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
this : Tendsto f (𝓝[A] x) (𝓝 (extendFrom A f x))
⊢ ∃ V, V ∈ 𝓝 x ∧ IsOpen V ∧ V ∩ A ⊆ f ⁻¹' V'
[PROOFSTEP]
rcases(nhdsWithin_basis_open x A).tendsto_left_iff.mp this V' V'_in with ⟨V, ⟨hxV, V_op⟩, hV⟩
[GOAL]
case intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
this : Tendsto f (𝓝[A] x) (𝓝 (extendFrom A f x))
V : Set X
hV : MapsTo f (V ∩ A) V'
hxV : x ∈ V
V_op : IsOpen V
⊢ ∃ V, V ∈ 𝓝 x ∧ IsOpen V ∧ V ∩ A ⊆ f ⁻¹' V'
[PROOFSTEP]
exact ⟨V, IsOpen.mem_nhds V_op hxV, V_op, hV⟩
[GOAL]
case intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
⊢ φ ⁻¹' V' ∈ 𝓝[B] x
[PROOFSTEP]
suffices : ∀ y ∈ V ∩ B, φ y ∈ V'
[GOAL]
case intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
this : ∀ (y : X), y ∈ V ∩ B → φ y ∈ V'
⊢ φ ⁻¹' V' ∈ 𝓝[B] x
case this
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
⊢ ∀ (y : X), y ∈ V ∩ B → φ y ∈ V'
[PROOFSTEP]
exact mem_of_superset (inter_mem_inf V_in <| mem_principal_self B) this
[GOAL]
case this
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
⊢ ∀ (y : X), y ∈ V ∩ B → φ y ∈ V'
[PROOFSTEP]
rintro y ⟨hyV, hyB⟩
[GOAL]
case this.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
y : X
hyV : y ∈ V
hyB : y ∈ B
⊢ φ y ∈ V'
[PROOFSTEP]
haveI := mem_closure_iff_nhdsWithin_neBot.mp (hB hyB)
[GOAL]
case this.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
y : X
hyV : y ∈ V
hyB : y ∈ B
this : NeBot (𝓝[A] y)
⊢ φ y ∈ V'
[PROOFSTEP]
have limy : Tendsto f (𝓝[A] y) (𝓝 <| φ y) := tendsto_extendFrom (hf y hyB)
[GOAL]
case this.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
y : X
hyV : y ∈ V
hyB : y ∈ B
this : NeBot (𝓝[A] y)
limy : Tendsto f (𝓝[A] y) (𝓝 (φ y))
⊢ φ y ∈ V'
[PROOFSTEP]
have hVy : V ∈ 𝓝 y := IsOpen.mem_nhds V_op hyV
[GOAL]
case this.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
y : X
hyV : y ∈ V
hyB : y ∈ B
this : NeBot (𝓝[A] y)
limy : Tendsto f (𝓝[A] y) (𝓝 (φ y))
hVy : V ∈ 𝓝 y
⊢ φ y ∈ V'
[PROOFSTEP]
have : V ∩ A ∈ 𝓝[A] y := by simpa only [inter_comm] using inter_mem_nhdsWithin A hVy
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
y : X
hyV : y ∈ V
hyB : y ∈ B
this : NeBot (𝓝[A] y)
limy : Tendsto f (𝓝[A] y) (𝓝 (φ y))
hVy : V ∈ 𝓝 y
⊢ V ∩ A ∈ 𝓝[A] y
[PROOFSTEP]
simpa only [inter_comm] using inter_mem_nhdsWithin A hVy
[GOAL]
case this.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A B : Set X
hB : B ⊆ closure A
hf : ∀ (x : X), x ∈ B → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
φ : X → Y := extendFrom A f
x : X
x_in : x ∈ B
V' : Set Y
V'_in : V' ∈ 𝓝 (φ x)
V'_closed : IsClosed V'
V : Set X
V_in : V ∈ 𝓝 x
V_op : IsOpen V
hV : V ∩ A ⊆ f ⁻¹' V'
y : X
hyV : y ∈ V
hyB : y ∈ B
this✝ : NeBot (𝓝[A] y)
limy : Tendsto f (𝓝[A] y) (𝓝 (φ y))
hVy : V ∈ 𝓝 y
this : V ∩ A ∈ 𝓝[A] y
⊢ φ y ∈ V'
[PROOFSTEP]
exact V'_closed.mem_of_tendsto limy (mem_of_superset this hV)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A : Set X
hA : Dense A
hf : ∀ (x : X), ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
⊢ Continuous (extendFrom A f)
[PROOFSTEP]
rw [continuous_iff_continuousOn_univ]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A : Set X
hA : Dense A
hf : ∀ (x : X), ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
⊢ ContinuousOn (extendFrom A f) univ
[PROOFSTEP]
exact continuousOn_extendFrom (fun x _ ↦ hA x) (by simpa using hf)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : RegularSpace Y
f : X → Y
A : Set X
hA : Dense A
hf : ∀ (x : X), ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
⊢ ∀ (x : X), x ∈ univ → ∃ y, Tendsto f (𝓝[A] x) (𝓝 y)
[PROOFSTEP]
simpa using hf
| {"mathlib_filename": "Mathlib.Topology.ExtendFrom", "llama_tokens": 5330} |
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α✝
x : α✝
α : Type u_3
inst✝ : TopologicalSpace (α × α)
⊢ 𝓝ˢ (diagonal α) = ⨆ (x : α), 𝓝 (x, x)
[PROOFSTEP]
rw [nhdsSet, ← range_diag, ← range_comp]
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α✝
x : α✝
α : Type u_3
inst✝ : TopologicalSpace (α × α)
⊢ sSup (range (𝓝 ∘ fun x => (x, x))) = ⨆ (x : α), 𝓝 (x, x)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ s ∈ 𝓝ˢ t ↔ ∀ (x : α), x ∈ t → s ∈ 𝓝 x
[PROOFSTEP]
simp_rw [nhdsSet, Filter.mem_sSup, ball_image_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ s ⊆ interior t ↔ t ∈ 𝓝ˢ s
[PROOFSTEP]
simp_rw [mem_nhdsSet_iff_forall, subset_interior_iff_nhds]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ Disjoint (𝓟 s) (𝓝ˢ t) ↔ Disjoint (closure s) t
[PROOFSTEP]
rw [disjoint_principal_left, ← subset_interior_iff_mem_nhdsSet, interior_compl, subset_compl_iff_disjoint_left]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ Disjoint (𝓝ˢ s) (𝓟 t) ↔ Disjoint s (closure t)
[PROOFSTEP]
rw [disjoint_comm, disjoint_principal_nhdsSet, disjoint_comm]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ s ∈ 𝓝ˢ t ↔ ∃ U, IsOpen U ∧ t ⊆ U ∧ U ⊆ s
[PROOFSTEP]
rw [← subset_interior_iff_mem_nhdsSet, subset_interior_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s₁ s₂ t₁ t₂ : Set α
x : α
s t : Set α
⊢ t ∈ 𝓝ˢ s ↔ ∃ i, (IsOpen i ∧ s ⊆ i) ∧ i ⊆ t
[PROOFSTEP]
simp [mem_nhdsSet_iff_exists, and_assoc]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
hU : IsOpen s
⊢ s ∈ 𝓝ˢ t ↔ t ⊆ s
[PROOFSTEP]
rw [← subset_interior_iff_mem_nhdsSet, hU.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ 𝓝ˢ s = 𝓟 s ↔ IsOpen s
[PROOFSTEP]
rw [← principal_le_nhdsSet.le_iff_eq, le_principal_iff, mem_nhdsSet_iff_forall, isOpen_iff_mem_nhds]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ 𝓝ˢ {x} = 𝓝 x
[PROOFSTEP]
simp [nhdsSet]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ 𝓝ˢ ∅ = ⊥
[PROOFSTEP]
rw [isOpen_empty.nhdsSet_eq, principal_empty]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ s ∈ 𝓝ˢ ∅
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
⊢ 𝓝ˢ univ = ⊤
[PROOFSTEP]
rw [isOpen_univ.nhdsSet_eq, principal_univ]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s₁ s₂ t₁ t₂ : Set α
x : α
s t : Set α
⊢ 𝓝ˢ (s ∪ t) = 𝓝ˢ s ⊔ 𝓝ˢ t
[PROOFSTEP]
simp only [nhdsSet, image_union, sSup_union]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
h₁ : s₁ ∈ 𝓝ˢ t₁
h₂ : s₂ ∈ 𝓝ˢ t₂
⊢ s₁ ∪ s₂ ∈ 𝓝ˢ (t₁ ∪ t₂)
[PROOFSTEP]
rw [nhdsSet_union]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t s₁ s₂ t₁ t₂ : Set α
x : α
h₁ : s₁ ∈ 𝓝ˢ t₁
h₂ : s₂ ∈ 𝓝ˢ t₂
⊢ s₁ ∪ s₂ ∈ 𝓝ˢ t₁ ⊔ 𝓝ˢ t₂
[PROOFSTEP]
exact union_mem_sup h₁ h₂
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s₁ s₂ t₁ t₂ : Set α
x✝ x : α
s : Set α
⊢ 𝓝ˢ (insert x s) = 𝓝 x ⊔ 𝓝ˢ s
[PROOFSTEP]
rw [insert_eq, nhdsSet_union, nhdsSet_singleton]
| {"mathlib_filename": "Mathlib.Topology.NhdsSet", "llama_tokens": 2136} |
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
a b : ℝ
hle : a ≤ b
f : X →ᵇ ℝ
hfs : EqOn (↑f) 0 s
hft : EqOn (↑f) 1 t
hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1
x : X
hx : x ∈ s
⊢ ↑(BoundedContinuousFunction.const X a + (b - a) • f) x = Function.const X a x
[PROOFSTEP]
simp [hfs hx]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
a b : ℝ
hle : a ≤ b
f : X →ᵇ ℝ
hfs : EqOn (↑f) 0 s
hft : EqOn (↑f) 1 t
hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1
x : X
hx : x ∈ t
⊢ ↑(BoundedContinuousFunction.const X a + (b - a) • f) x = Function.const X b x
[PROOFSTEP]
simp [hft hx]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
a b : ℝ
hle : a ≤ b
f : X →ᵇ ℝ
hfs : EqOn (↑f) 0 s
hft : EqOn (↑f) 1 t
hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1
x : X
⊢ a ≤ ↑(BoundedContinuousFunction.const X a + (b - a) • f) x
[PROOFSTEP]
dsimp
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
a b : ℝ
hle : a ≤ b
f : X →ᵇ ℝ
hfs : EqOn (↑f) 0 s
hft : EqOn (↑f) 1 t
hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1
x : X
⊢ a ≤ a + (b - a) * ↑f x
[PROOFSTEP]
nlinarith [(hf01 x).1]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
a b : ℝ
hle : a ≤ b
f : X →ᵇ ℝ
hfs : EqOn (↑f) 0 s
hft : EqOn (↑f) 1 t
hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1
x : X
⊢ ↑(BoundedContinuousFunction.const X a + (b - a) • f) x ≤ b
[PROOFSTEP]
dsimp
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
a b : ℝ
hle : a ≤ b
f : X →ᵇ ℝ
hfs : EqOn (↑f) 0 s
hft : EqOn (↑f) 1 t
hf01 : ∀ (x : X), ↑f x ∈ Icc 0 1
x : X
⊢ a + (b - a) * ↑f x ≤ b
[PROOFSTEP]
nlinarith [(hf01 x).2]
| {"mathlib_filename": "Mathlib.Topology.UrysohnsBounded", "llama_tokens": 1088} |
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
inst✝ : Nontrivial R
i j : n
⊢ natDegree (charmatrix M i j) = if i = j then 1 else 0
[PROOFSTEP]
by_cases i = j
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
inst✝ : Nontrivial R
i j : n
⊢ natDegree (charmatrix M i j) = if i = j then 1 else 0
[PROOFSTEP]
by_cases i = j
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
inst✝ : Nontrivial R
i j : n
h : i = j
⊢ natDegree (charmatrix M i j) = if i = j then 1 else 0
[PROOFSTEP]
simp [h, ← degree_eq_iff_natDegree_eq_of_pos (Nat.succ_pos 0)]
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
inst✝ : Nontrivial R
i j : n
h : ¬i = j
⊢ natDegree (charmatrix M i j) = if i = j then 1 else 0
[PROOFSTEP]
simp [h, ← degree_eq_iff_natDegree_eq_of_pos (Nat.succ_pos 0)]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
i j : n
⊢ natDegree (charmatrix M i j) ≤ if i = j then 1 else 0
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
i j : n
h : i = j
⊢ natDegree (charmatrix M i j) ≤ 1
[PROOFSTEP]
simp [h, natDegree_X_sub_C_le]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
i j : n
h : ¬i = j
⊢ natDegree (charmatrix M i j) ≤ 0
[PROOFSTEP]
simp [h, natDegree_X_sub_C_le]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i))) < ↑(Fintype.card n - 1)
[PROOFSTEP]
rw [charpoly, det_apply', ← insert_erase (mem_univ (Equiv.refl n)), sum_insert (not_mem_erase (Equiv.refl n) univ),
add_comm]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
⊢ degree
(∑ x in Finset.erase univ (Equiv.refl n), ↑↑(↑Equiv.Perm.sign x) * ∏ i : n, charmatrix M (↑x i) i +
↑↑(↑Equiv.Perm.sign (Equiv.refl n)) * ∏ i : n, charmatrix M (↑(Equiv.refl n) i) i -
∏ i : n, (X - ↑C (M i i))) <
↑(Fintype.card n - 1)
[PROOFSTEP]
simp only [charmatrix_apply_eq, one_mul, Equiv.Perm.sign_refl, id.def, Int.cast_one, Units.val_one, add_sub_cancel,
Equiv.coe_refl]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
⊢ degree (∑ x in Finset.erase univ (Equiv.refl n), ↑↑(↑Equiv.Perm.sign x) * ∏ x_1 : n, charmatrix M (↑x x_1) x_1) <
↑(Fintype.card n - 1)
[PROOFSTEP]
rw [← mem_degreeLT]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
⊢ ∑ x in Finset.erase univ (Equiv.refl n), ↑↑(↑Equiv.Perm.sign x) * ∏ x_1 : n, charmatrix M (↑x x_1) x_1 ∈
degreeLT R (Fintype.card n - 1)
[PROOFSTEP]
apply Submodule.sum_mem (degreeLT R (Fintype.card n - 1))
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
⊢ ∀ (c : n ≃ n),
c ∈ Finset.erase univ (Equiv.refl n) →
↑↑(↑Equiv.Perm.sign c) * ∏ x : n, charmatrix M (↑c x) x ∈ degreeLT R (Fintype.card n - 1)
[PROOFSTEP]
intro c hc
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ↑↑(↑Equiv.Perm.sign c) * ∏ x : n, charmatrix M (↑c x) x ∈ degreeLT R (Fintype.card n - 1)
[PROOFSTEP]
rw [← C_eq_int_cast, C_mul']
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ↑↑(↑Equiv.Perm.sign c) • ∏ x : n, charmatrix M (↑c x) x ∈ degreeLT R (Fintype.card n - 1)
[PROOFSTEP]
apply Submodule.smul_mem (degreeLT R (Fintype.card n - 1)) ↑↑(Equiv.Perm.sign c)
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ∏ x : n, charmatrix M (↑c x) x ∈ degreeLT R (Fintype.card n - 1)
[PROOFSTEP]
rw [mem_degreeLT]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ degree (∏ x : n, charmatrix M (↑c x) x) < ↑(Fintype.card n - 1)
[PROOFSTEP]
apply lt_of_le_of_lt degree_le_natDegree _
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ↑(natDegree (∏ x : n, charmatrix M (↑c x) x)) < ↑(Fintype.card n - 1)
[PROOFSTEP]
rw [Nat.cast_withBot, Nat.cast_withBot]
-- porting note: added
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ↑(natDegree (∏ x : n, charmatrix M (↑c x) x)) < ↑(Fintype.card n - 1)
[PROOFSTEP]
rw [WithBot.coe_lt_coe]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ natDegree (∏ x : n, charmatrix M (↑c x) x) < Fintype.card n - 1
[PROOFSTEP]
apply lt_of_le_of_lt _ (Equiv.Perm.fixed_point_card_lt_of_ne_one (ne_of_mem_erase hc))
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ natDegree (∏ x : n, charmatrix M (↑c x) x) ≤ card (filter (fun x => ↑c x = x) univ)
[PROOFSTEP]
apply le_trans (Polynomial.natDegree_prod_le univ fun i : n => charmatrix M (c i) i) _
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ∑ i : n, natDegree (charmatrix M (↑c i) i) ≤ card (filter (fun x => ↑c x = x) univ)
[PROOFSTEP]
rw [card_eq_sum_ones]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ∑ i : n, natDegree (charmatrix M (↑c i) i) ≤ ∑ x in filter (fun x => ↑c x = x) univ, 1
[PROOFSTEP]
rw [sum_filter]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ∑ i : n, natDegree (charmatrix M (↑c i) i) ≤ ∑ a : n, if ↑c a = a then 1 else 0
[PROOFSTEP]
apply sum_le_sum
[GOAL]
case h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
⊢ ∀ (i : n), i ∈ univ → natDegree (charmatrix M (↑c i) i) ≤ if ↑c i = i then 1 else 0
[PROOFSTEP]
intros
[GOAL]
case h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
c : n ≃ n
hc : c ∈ Finset.erase univ (Equiv.refl n)
i✝ : n
a✝ : i✝ ∈ univ
⊢ natDegree (charmatrix M (↑c i✝) i✝) ≤ if ↑c i✝ = i✝ then 1 else 0
[PROOFSTEP]
apply charmatrix_apply_natDegree_le
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ coeff (charpoly M) k = coeff (∏ i : n, (X - ↑C (M i i))) k
[PROOFSTEP]
apply eq_of_sub_eq_zero
[GOAL]
case h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ coeff (charpoly M) k - coeff (∏ i : n, (X - ↑C (M i i))) k = 0
[PROOFSTEP]
rw [← coeff_sub]
[GOAL]
case h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ coeff (charpoly M - ∏ i : n, (X - ↑C (M i i))) k = 0
[PROOFSTEP]
apply Polynomial.coeff_eq_zero_of_degree_lt
[GOAL]
case h.h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i))) < ↑k
[PROOFSTEP]
apply lt_of_lt_of_le (charpoly_sub_diagonal_degree_lt M) ?_
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ ↑(Fintype.card n - 1) ≤ ↑k
[PROOFSTEP]
rw [Nat.cast_withBot, Nat.cast_withBot]
-- porting note: added
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ ↑(Fintype.card n - 1) ≤ ↑k
[PROOFSTEP]
rw [WithBot.coe_le_coe]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M : Matrix n n R
k : ℕ
h : Fintype.card n - 1 ≤ k
⊢ Fintype.card n - 1 ≤ k
[PROOFSTEP]
apply h
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
h : Fintype.card n = 0
M : Matrix n n R
⊢ det M = 1
[PROOFSTEP]
rw [Fintype.card_eq_zero_iff] at h
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
h : IsEmpty n
M : Matrix n n R
⊢ det M = 1
[PROOFSTEP]
suffices M = 1 by simp [this]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
h : IsEmpty n
M : Matrix n n R
this : M = 1
⊢ det M = 1
[PROOFSTEP]
simp [this]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
h : IsEmpty n
M : Matrix n n R
⊢ M = 1
[PROOFSTEP]
ext i
[GOAL]
case a.h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
h : IsEmpty n
M : Matrix n n R
i x✝ : n
⊢ M i x✝ = OfNat.ofNat 1 i x✝
[PROOFSTEP]
exact h.elim i
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
⊢ degree (charpoly M) = ↑(Fintype.card n)
[PROOFSTEP]
by_cases h : Fintype.card n = 0
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : Fintype.card n = 0
⊢ degree (charpoly M) = ↑(Fintype.card n)
[PROOFSTEP]
rw [h]
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : Fintype.card n = 0
⊢ degree (charpoly M) = ↑0
[PROOFSTEP]
unfold charpoly
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : Fintype.card n = 0
⊢ degree (det (charmatrix M)) = ↑0
[PROOFSTEP]
rw [det_of_card_zero]
[GOAL]
case pos
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : Fintype.card n = 0
⊢ degree 1 = ↑0
[PROOFSTEP]
simp
[GOAL]
case pos.h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : Fintype.card n = 0
⊢ Fintype.card n = 0
[PROOFSTEP]
assumption
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ degree (charpoly M) = ↑(Fintype.card n)
[PROOFSTEP]
rw [← sub_add_cancel M.charpoly (∏ i : n, (X - C (M i i)))]
-- porting note: added `↑` in front of `Fintype.card n`
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i)) + ∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
[PROOFSTEP]
have h1 : (∏ i : n, (X - C (M i i))).degree = ↑(Fintype.card n) :=
by
rw [degree_eq_iff_natDegree_eq_of_pos (Nat.pos_of_ne_zero h), natDegree_prod']
simp_rw [natDegree_X_sub_C]
rw [← Finset.card_univ, sum_const, smul_eq_mul, mul_one]
simp_rw [(monic_X_sub_C _).leadingCoeff]
simp
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
[PROOFSTEP]
rw [degree_eq_iff_natDegree_eq_of_pos (Nat.pos_of_ne_zero h), natDegree_prod']
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ ∑ i : n, natDegree (X - ↑C (M i i)) = Fintype.card n
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ ∏ i : n, leadingCoeff (X - ↑C (M i i)) ≠ 0
[PROOFSTEP]
simp_rw [natDegree_X_sub_C]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ ∑ x : n, 1 = Fintype.card n
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ ∏ i : n, leadingCoeff (X - ↑C (M i i)) ≠ 0
[PROOFSTEP]
rw [← Finset.card_univ, sum_const, smul_eq_mul, mul_one]
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ ∏ i : n, leadingCoeff (X - ↑C (M i i)) ≠ 0
[PROOFSTEP]
simp_rw [(monic_X_sub_C _).leadingCoeff]
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
⊢ ∏ x : n, 1 ≠ 0
[PROOFSTEP]
simp
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i)) + ∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
[PROOFSTEP]
rw [degree_add_eq_right_of_degree_lt]
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i))) < degree (∏ i : n, (X - ↑C (M i i)))
[PROOFSTEP]
exact h1
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i))) < degree (∏ i : n, (X - ↑C (M i i)))
[PROOFSTEP]
rw [h1]
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i))) < ↑(Fintype.card n)
[PROOFSTEP]
apply lt_trans (charpoly_sub_diagonal_degree_lt M)
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ ↑(Fintype.card n - 1) < ↑(Fintype.card n)
[PROOFSTEP]
rw [Nat.cast_withBot, Nat.cast_withBot]
-- porting note: added
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ ↑(Fintype.card n - 1) < ↑(Fintype.card n)
[PROOFSTEP]
rw [WithBot.coe_lt_coe]
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ Fintype.card n - 1 < Fintype.card n
[PROOFSTEP]
rw [← Nat.pred_eq_sub_one]
[GOAL]
case neg
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ Nat.pred (Fintype.card n) < Fintype.card n
[PROOFSTEP]
apply Nat.pred_lt
[GOAL]
case neg.a
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nontrivial R
M : Matrix n n R
h : ¬Fintype.card n = 0
h1 : degree (∏ i : n, (X - ↑C (M i i))) = ↑(Fintype.card n)
⊢ Fintype.card n ≠ 0
[PROOFSTEP]
apply h
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
⊢ Monic (charpoly M)
[PROOFSTEP]
nontriviality R
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
⊢ Monic (charpoly M)
[PROOFSTEP]
by_cases h : Fintype.card n = 0
[GOAL]
case pos
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : Fintype.card n = 0
⊢ Monic (charpoly M)
[PROOFSTEP]
rw [charpoly, det_of_card_zero h]
[GOAL]
case pos
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : Fintype.card n = 0
⊢ Monic 1
[PROOFSTEP]
apply monic_one
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
⊢ Monic (charpoly M)
[PROOFSTEP]
have mon : (∏ i : n, (X - C (M i i))).Monic :=
by
apply monic_prod_of_monic univ fun i : n => X - C (M i i)
simp [monic_X_sub_C]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
⊢ Monic (∏ i : n, (X - ↑C (M i i)))
[PROOFSTEP]
apply monic_prod_of_monic univ fun i : n => X - C (M i i)
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
⊢ ∀ (i : n), i ∈ univ → Monic (X - ↑C (M i i))
[PROOFSTEP]
simp [monic_X_sub_C]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : Monic (∏ i : n, (X - ↑C (M i i)))
⊢ Monic (charpoly M)
[PROOFSTEP]
rw [← sub_add_cancel (∏ i : n, (X - C (M i i))) M.charpoly] at mon
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : Monic (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M)
⊢ Monic (charpoly M)
[PROOFSTEP]
rw [Monic] at *
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ leadingCoeff (charpoly M) = 1
[PROOFSTEP]
rwa [leadingCoeff_add_of_degree_lt] at mon
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ degree (∏ i : n, (X - ↑C (M i i)) - charpoly M) < degree (charpoly M)
[PROOFSTEP]
rw [charpoly_degree_eq_dim]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ degree (∏ i : n, (X - ↑C (M i i)) - charpoly M) < ↑(Fintype.card n)
[PROOFSTEP]
rw [← neg_sub]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ degree (-(charpoly M - ∏ i : n, (X - ↑C (M i i)))) < ↑(Fintype.card n)
[PROOFSTEP]
rw [degree_neg]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ degree (charpoly M - ∏ i : n, (X - ↑C (M i i))) < ↑(Fintype.card n)
[PROOFSTEP]
apply lt_trans (charpoly_sub_diagonal_degree_lt M)
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ ↑(Fintype.card n - 1) < ↑(Fintype.card n)
[PROOFSTEP]
rw [Nat.cast_withBot, Nat.cast_withBot]
-- porting note: added
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ ↑(Fintype.card n - 1) < ↑(Fintype.card n)
[PROOFSTEP]
rw [WithBot.coe_lt_coe]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ Fintype.card n - 1 < Fintype.card n
[PROOFSTEP]
rw [← Nat.pred_eq_sub_one]
[GOAL]
case neg
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ Nat.pred (Fintype.card n) < Fintype.card n
[PROOFSTEP]
apply Nat.pred_lt
[GOAL]
case neg.a
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
✝ : Nontrivial R
h : ¬Fintype.card n = 0
mon : leadingCoeff (∏ i : n, (X - ↑C (M i i)) - charpoly M + charpoly M) = 1
⊢ Fintype.card n ≠ 0
[PROOFSTEP]
apply h
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nonempty n
M : Matrix n n R
⊢ trace M = -coeff (charpoly M) (Fintype.card n - 1)
[PROOFSTEP]
rw [charpoly_coeff_eq_prod_coeff_of_le _ le_rfl, Fintype.card,
prod_X_sub_C_coeff_card_pred univ (fun i : n => M i i) Fintype.card_pos, neg_neg, trace]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
inst✝ : Nonempty n
M : Matrix n n R
⊢ ∑ i : n, diag M i = ∑ i : n, M i i
[PROOFSTEP]
simp_rw [diag_apply]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ eval (↑(scalar n) r) (↑matPolyEquiv M) i j = eval r (M i j)
[PROOFSTEP]
unfold Polynomial.eval
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ eval₂ (RingHom.id ((fun x => Matrix n n R) r)) (↑(scalar n) r) (↑matPolyEquiv M) i j = eval₂ (RingHom.id R) r (M i j)
[PROOFSTEP]
rw [Polynomial.eval₂_def, Polynomial.eval₂_def]
-- porting note: was `unfold eval₂`
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ sum (↑matPolyEquiv M) (fun e a => ↑(RingHom.id ((fun x => Matrix n n R) r)) a * ↑(scalar n) r ^ e) i j =
sum (M i j) fun e a => ↑(RingHom.id R) a * r ^ e
[PROOFSTEP]
trans Polynomial.sum (matPolyEquiv M) fun (e : ℕ) (a : Matrix n n R) => (a * (scalar n) r ^ e) i j
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ sum (↑matPolyEquiv M) (fun e a => ↑(RingHom.id ((fun x => Matrix n n R) r)) a * ↑(scalar n) r ^ e) i j =
sum (↑matPolyEquiv M) fun e a => (a * ↑(scalar n) r ^ e) i j
[PROOFSTEP]
unfold Polynomial.sum
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ Finset.sum (support (↑matPolyEquiv M))
(fun n_1 =>
(fun e a => ↑(RingHom.id ((fun x => Matrix n n R) r)) a * ↑(scalar n) r ^ e) n_1 (coeff (↑matPolyEquiv M) n_1))
i j =
∑ n_1 in support (↑matPolyEquiv M), (fun e a => (a * ↑(scalar n) r ^ e) i j) n_1 (coeff (↑matPolyEquiv M) n_1)
[PROOFSTEP]
simp only [sum_apply]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ ∑ c in support (↑matPolyEquiv M), (↑(RingHom.id (Matrix n n R)) (coeff (↑matPolyEquiv M) c) * ↑(scalar n) r ^ c) i j =
∑ x in support (↑matPolyEquiv M), (coeff (↑matPolyEquiv M) x * ↑(scalar n) r ^ x) i j
[PROOFSTEP]
dsimp
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ (sum (↑matPolyEquiv M) fun e a => (a * ↑(scalar n) r ^ e) i j) = sum (M i j) fun e a => ↑(RingHom.id R) a * r ^ e
[PROOFSTEP]
simp_rw [← RingHom.map_pow, ← (scalar.commute _ _).eq]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ (sum (↑matPolyEquiv M) fun e a => (↑(scalar n) (r ^ e) * a) i j) = sum (M i j) fun e a => ↑(RingHom.id R) a * r ^ e
[PROOFSTEP]
simp only [coe_scalar, Matrix.one_mul, RingHom.id_apply, Pi.smul_apply, smul_eq_mul, Algebra.smul_mul_assoc]
-- porting note: the `have` was present and unused also in the original
--have h : ∀ x : ℕ, (fun (e : ℕ) (a : R) => r ^ e * a) x 0 = 0 := by simp
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ (sum (↑matPolyEquiv M) fun e a => (r ^ e • a) i j) = sum (M i j) fun e a => a * r ^ e
[PROOFSTEP]
simp only [Polynomial.sum, matPolyEquiv_coeff_apply, mul_comm]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ ∑ x in support (↑matPolyEquiv M), (r ^ x • coeff (↑matPolyEquiv M) x) i j =
∑ x in support (M i j), r ^ x * coeff (M i j) x
[PROOFSTEP]
simp only [smul_apply, matPolyEquiv_coeff_apply, smul_eq_mul]
-- porting note: added
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ ∑ x in support (↑matPolyEquiv M), r ^ x * coeff (M i j) x = ∑ x in support (M i j), r ^ x * coeff (M i j) x
[PROOFSTEP]
apply (Finset.sum_subset (support_subset_support_matPolyEquiv _ _ _) _).symm
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i j : n
⊢ ∀ (x : ℕ), x ∈ support (↑matPolyEquiv M) → ¬x ∈ support (M i j) → r ^ x * coeff (M i j) x = 0
[PROOFSTEP]
intro n _hn h'n
[GOAL]
R : Type u
inst✝³ : CommRing R
n✝ G : Type v
inst✝² : DecidableEq n✝
inst✝¹ : Fintype n✝
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n✝ n✝ R
M : Matrix n✝ n✝ R[X]
r : R
i j : n✝
n : ℕ
_hn : n ∈ support (↑matPolyEquiv M)
h'n : ¬n ∈ support (M i j)
⊢ r ^ n * coeff (M i j) n = 0
[PROOFSTEP]
rw [not_mem_support_iff] at h'n
[GOAL]
R : Type u
inst✝³ : CommRing R
n✝ G : Type v
inst✝² : DecidableEq n✝
inst✝¹ : Fintype n✝
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n✝ n✝ R
M : Matrix n✝ n✝ R[X]
r : R
i j : n✝
n : ℕ
_hn : n ∈ support (↑matPolyEquiv M)
h'n : coeff (M i j) n = 0
⊢ r ^ n * coeff (M i j) n = 0
[PROOFSTEP]
simp only [h'n, zero_mul]
[GOAL]
R : Type u
inst✝³ : CommRing R
n✝ G : Type v
inst✝² : DecidableEq n✝
inst✝¹ : Fintype n✝
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n✝ n✝ R
M : Matrix n✝ n✝ R[X]
r : R
i j : n✝
n : ℕ
_hn : n ∈ support (↑matPolyEquiv M)
h'n : coeff (M i j) n = 0
⊢ r ^ n * 0 = 0
[PROOFSTEP]
simp only [mul_zero]
-- porting note: added
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
⊢ eval r (det M) = det (eval (↑(scalar n) r) (↑matPolyEquiv M))
[PROOFSTEP]
rw [Polynomial.eval, ← coe_eval₂RingHom, RingHom.map_det]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
⊢ det (↑(RingHom.mapMatrix (eval₂RingHom (RingHom.id R) r)) M) = det (eval (↑(scalar n) r) (↑matPolyEquiv M))
[PROOFSTEP]
apply congr_arg det
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
⊢ ↑(RingHom.mapMatrix (eval₂RingHom (RingHom.id R) r)) M = eval (↑(scalar n) r) (↑matPolyEquiv M)
[PROOFSTEP]
ext
[GOAL]
case a.h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i✝ x✝ : n
⊢ ↑(RingHom.mapMatrix (eval₂RingHom (RingHom.id R) r)) M i✝ x✝ = eval (↑(scalar n) r) (↑matPolyEquiv M) i✝ x✝
[PROOFSTEP]
symm
-- porting note: `exact` was `convert`
[GOAL]
case a.h
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ : Matrix n n R
M : Matrix n n R[X]
r : R
i✝ x✝ : n
⊢ eval (↑(scalar n) r) (↑matPolyEquiv M) i✝ x✝ = ↑(RingHom.mapMatrix (eval₂RingHom (RingHom.id R) r)) M i✝ x✝
[PROOFSTEP]
exact matPolyEquiv_eval _ _ _ _
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
⊢ det M = (-1) ^ Fintype.card n * coeff (charpoly M) 0
[PROOFSTEP]
rw [coeff_zero_eq_eval_zero, charpoly, eval_det, matPolyEquiv_charmatrix, ← det_smul]
[GOAL]
R : Type u
inst✝³ : CommRing R
n G : Type v
inst✝² : DecidableEq n
inst✝¹ : Fintype n
α β : Type v
inst✝ : DecidableEq α
M✝ M : Matrix n n R
⊢ det M = det (-1 • eval (↑(scalar n) 0) (X - ↑C M))
[PROOFSTEP]
simp
[GOAL]
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
⊢ ↑matPolyEquiv (↑(RingHom.mapMatrix ↑(expand K k)) (charmatrix (M ^ k))) = X ^ k - ↑C (M ^ k)
[PROOFSTEP]
ext m i j
[GOAL]
case a.a.h
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
⊢ coeff (↑matPolyEquiv (↑(RingHom.mapMatrix ↑(expand K k)) (charmatrix (M ^ k)))) m i j =
coeff (X ^ k - ↑C (M ^ k)) m i j
[PROOFSTEP]
rw [coeff_sub, coeff_C, matPolyEquiv_coeff_apply, RingHom.mapMatrix_apply, Matrix.map_apply, AlgHom.coe_toRingHom,
DMatrix.sub_apply, coeff_X_pow]
[GOAL]
case a.a.h
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
⊢ coeff (↑(expand K k) (charmatrix (M ^ k) i j)) m = ite (m = k) 1 0 i j - ite (m = 0) (M ^ k) 0 i j
[PROOFSTEP]
by_cases hij : i = j
[GOAL]
case pos
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : i = j
⊢ coeff (↑(expand K k) (charmatrix (M ^ k) i j)) m = ite (m = k) 1 0 i j - ite (m = 0) (M ^ k) 0 i j
[PROOFSTEP]
rw [hij, charmatrix_apply_eq, AlgHom.map_sub, expand_C, expand_X, coeff_sub, coeff_X_pow, coeff_C]
-- porting note: the second `Matrix.` was `DMatrix.`
[GOAL]
case pos
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : i = j
⊢ ((if m = k then 1 else 0) - if m = 0 then (M ^ k) j j else 0) = ite (m = k) 1 0 j j - ite (m = 0) (M ^ k) 0 j j
[PROOFSTEP]
split_ifs with mp m0
[GOAL]
case pos
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : i = j
mp : m = k
m0 : m = 0
⊢ 1 - (M ^ k) j j = OfNat.ofNat 1 j j - (M ^ k) j j
[PROOFSTEP]
simp only [Matrix.one_apply_eq, Matrix.zero_apply]
[GOAL]
case neg
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : i = j
mp : m = k
m0 : ¬m = 0
⊢ 1 - 0 = OfNat.ofNat 1 j j - OfNat.ofNat 0 j j
[PROOFSTEP]
simp only [Matrix.one_apply_eq, Matrix.zero_apply]
[GOAL]
case pos
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : i = j
mp : ¬m = k
h✝ : m = 0
⊢ 0 - (M ^ k) j j = OfNat.ofNat 0 j j - (M ^ k) j j
[PROOFSTEP]
simp only [Matrix.one_apply_eq, Matrix.zero_apply]
[GOAL]
case neg
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : i = j
mp : ¬m = k
h✝ : ¬m = 0
⊢ 0 - 0 = OfNat.ofNat 0 j j - OfNat.ofNat 0 j j
[PROOFSTEP]
simp only [Matrix.one_apply_eq, Matrix.zero_apply]
[GOAL]
case neg
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : ¬i = j
⊢ coeff (↑(expand K k) (charmatrix (M ^ k) i j)) m = ite (m = k) 1 0 i j - ite (m = 0) (M ^ k) 0 i j
[PROOFSTEP]
rw [charmatrix_apply_ne _ _ _ hij, AlgHom.map_neg, expand_C, coeff_neg, coeff_C]
[GOAL]
case neg
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : ¬i = j
⊢ (-if m = 0 then (M ^ k) i j else 0) = ite (m = k) 1 0 i j - ite (m = 0) (M ^ k) 0 i j
[PROOFSTEP]
split_ifs with m0 mp
[GOAL]
case pos
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : ¬i = j
m0 : m = 0
mp : m = k
⊢ -(M ^ k) i j = OfNat.ofNat 1 i j - (M ^ k) i j
[PROOFSTEP]
simp only [hij, zero_sub, Matrix.zero_apply, sub_zero, neg_zero, Matrix.one_apply_ne, Ne.def, not_false_iff]
[GOAL]
case neg
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : ¬i = j
m0 : m = 0
mp : ¬m = k
⊢ -(M ^ k) i j = OfNat.ofNat 0 i j - (M ^ k) i j
[PROOFSTEP]
simp only [hij, zero_sub, Matrix.zero_apply, sub_zero, neg_zero, Matrix.one_apply_ne, Ne.def, not_false_iff]
[GOAL]
case pos
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : ¬i = j
m0 : ¬m = 0
h✝ : m = k
⊢ -0 = OfNat.ofNat 1 i j - OfNat.ofNat 0 i j
[PROOFSTEP]
simp only [hij, zero_sub, Matrix.zero_apply, sub_zero, neg_zero, Matrix.one_apply_ne, Ne.def, not_false_iff]
[GOAL]
case neg
R : Type u
inst✝⁵ : CommRing R
n G : Type v
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
α β : Type v
inst✝² : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝¹ : Fact (Nat.Prime p)
K : Type u_1
k : ℕ
inst✝ : Field K
M : Matrix n n K
m : ℕ
i j : n
hij : ¬i = j
m0 : ¬m = 0
h✝ : ¬m = k
⊢ -0 = OfNat.ofNat 0 i j - OfNat.ofNat 0 i j
[PROOFSTEP]
simp only [hij, zero_sub, Matrix.zero_apply, sub_zero, neg_zero, Matrix.one_apply_ne, Ne.def, not_false_iff]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M✝ : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
M : Matrix n n R
k : ℕ
⊢ M ^ k = ↑(aeval M) (X ^ k %ₘ charpoly M)
[PROOFSTEP]
rw [← aeval_eq_aeval_mod_charpoly, map_pow, aeval_X]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
⊢ coeff (charpoly M) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
delta charpoly
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
⊢ coeff (det (charmatrix M)) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
rw [Matrix.det_apply, finset_sum_coeff]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
⊢ ∑ b : Equiv.Perm n, coeff (↑Equiv.Perm.sign b • ∏ i : n, charmatrix M (↑b i) i) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
apply sum_mem
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
⊢ ∀ (c : Equiv.Perm n),
c ∈ univ → coeff (↑Equiv.Perm.sign c • ∏ i : n, charmatrix M (↑c i) i) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
rintro c -
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
⊢ coeff (↑Equiv.Perm.sign c • ∏ i : n, charmatrix M (↑c i) i) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
rw [coeff_smul, Submodule.smul_mem_iff']
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
⊢ coeff (∏ i : n, charmatrix M (↑c i) i) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
have : ∑ x : n, 1 = Fintype.card n := by rw [Finset.sum_const, card_univ, smul_eq_mul, mul_one]
[GOAL]
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
⊢ ∑ x : n, 1 = Fintype.card n
[PROOFSTEP]
rw [Finset.sum_const, card_univ, smul_eq_mul, mul_one]
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
⊢ coeff (∏ i : n, charmatrix M (↑c i) i) k ∈ I ^ (Fintype.card n - k)
[PROOFSTEP]
rw [← this]
[GOAL]
case h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
⊢ coeff (∏ i : n, charmatrix M (↑c i) i) k ∈ I ^ (∑ x : n, 1 - k)
[PROOFSTEP]
apply coeff_prod_mem_ideal_pow_tsub
[GOAL]
case h.h
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
⊢ ∀ (i : n), i ∈ univ → ∀ (k : ℕ), coeff (charmatrix M (↑c i) i) k ∈ I ^ (1 - k)
[PROOFSTEP]
rintro i - (_ | k)
[GOAL]
case h.h.zero
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
i : n
⊢ coeff (charmatrix M (↑c i) i) Nat.zero ∈ I ^ (1 - Nat.zero)
[PROOFSTEP]
rw [Nat.zero_eq]
-- porting note: `rw [Nat.zero_eq]` was not present
[GOAL]
case h.h.zero
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
i : n
⊢ coeff (charmatrix M (↑c i) i) 0 ∈ I ^ (1 - 0)
[PROOFSTEP]
rw [tsub_zero, pow_one, charmatrix_apply, coeff_sub, coeff_X_mul_zero, coeff_C_zero, zero_sub]
[GOAL]
case h.h.zero
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
i : n
⊢ -M (↑c i) i ∈ I
[PROOFSTEP]
apply neg_mem
[GOAL]
case h.h.zero.a
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
i : n
⊢ M (↑c i) i ∈ I
[PROOFSTEP]
exact h (c i) i
[GOAL]
case h.h.succ
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k✝ : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
i : n
k : ℕ
⊢ coeff (charmatrix M (↑c i) i) (Nat.succ k) ∈ I ^ (1 - Nat.succ k)
[PROOFSTEP]
rw [Nat.succ_eq_one_add, tsub_self_add, pow_zero, Ideal.one_eq_top]
[GOAL]
case h.h.succ
R : Type u
inst✝⁴ : CommRing R
n G : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
α β : Type v
inst✝¹ : DecidableEq α
M : Matrix n n R
p : ℕ
inst✝ : Fact (Nat.Prime p)
I : Ideal R
h : ∀ (i j : n), M i j ∈ I
k✝ : ℕ
c : Equiv.Perm n
this : ∑ x : n, 1 = Fintype.card n
i : n
k : ℕ
⊢ coeff (charmatrix M (↑c i) i) (1 + k) ∈ ⊤
[PROOFSTEP]
exact Submodule.mem_top
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.Charpoly.Coeff", "llama_tokens": 24926} |
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ negY W x₁ (negY W x₁ y₁) = y₁
[PROOFSTEP]
simp only [negY]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ -(-y₁ - W.a₁ * x₁ - W.a₃) - W.a₁ * x₁ - W.a₃ = y₁
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ negY (baseChange W A) (↑(algebraMap R A) x₁) (↑(algebraMap R A) y₁) = ↑(algebraMap R A) (negY W x₁ y₁)
[PROOFSTEP]
simp only [negY]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ -↑(algebraMap R A) y₁ - (baseChange W A).a₁ * ↑(algebraMap R A) x₁ - (baseChange W A).a₃ =
↑(algebraMap R A) (-y₁ - W.a₁ * x₁ - W.a₃)
[PROOFSTEP]
map_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ -↑(algebraMap R A) y₁ - (baseChange W A).a₁ * ↑(algebraMap R A) x₁ - (baseChange W A).a₃ =
-↑(algebraMap R A) y₁ - ↑(algebraMap R A) W.a₁ * ↑(algebraMap R A) x₁ - ↑(algebraMap R A) W.a₃
[PROOFSTEP]
rfl
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁✝ x₂ y₁✝ y₂ L : R
x₁ y₁ : A
⊢ negY (baseChange W B) (↑(algebraMap A B) x₁) (↑(algebraMap A B) y₁) = ↑(algebraMap A B) (negY (baseChange W A) x₁ y₁)
[PROOFSTEP]
rw [← baseChange_negY, baseChange_baseChange]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ eval x₁ (eval (↑C y₁) (negPolynomial W)) = negY W x₁ y₁
[PROOFSTEP]
rw [negY, sub_sub, negPolynomial]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ eval x₁ (eval (↑C y₁) (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) = -y₁ - (W.a₁ * x₁ + W.a₃)
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ XYIdeal W x₁ (↑C y₁) = XYIdeal W x₁ (linePolynomial x₁ y₁ L)
[PROOFSTEP]
simp only [XYIdeal, XClass, YClass, linePolynomial]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ span {↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁)), ↑(CoordinateRing.mk W) (Y - ↑C (↑C y₁))} =
span {↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁)), ↑(CoordinateRing.mk W) (Y - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁))}
[PROOFSTEP]
rw [← span_pair_add_mul_right <| CoordinateRing.mk W <| C <| C <| -L, ← _root_.map_mul, ← map_add]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁)),
↑(CoordinateRing.mk W) (Y - ↑C (↑C y₁) + ↑C (Y - ↑C x₁) * ↑C (↑C (-L)))} =
span {↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁)), ↑(CoordinateRing.mk W) (Y - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁))}
[PROOFSTEP]
apply congr_arg (_ ∘ _ ∘ _ ∘ _)
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ Y - ↑C (↑C y₁) + ↑C (Y - ↑C x₁) * ↑C (↑C (-L)) = Y - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁)
[PROOFSTEP]
C_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ Y - ↑C (↑C y₁) + (↑C Y - ↑C (↑C x₁)) * -↑C (↑C L) = Y - (↑C (↑C L) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁))
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑C (addPolynomial W x₁ y₁ L) =
(Y - ↑C (linePolynomial x₁ y₁ L)) * (negPolynomial W - ↑C (linePolynomial x₁ y₁ L)) + WeierstrassCurve.polynomial W
[PROOFSTEP]
rw [addPolynomial, linePolynomial, WeierstrassCurve.polynomial, negPolynomial]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑C
(eval (↑C L * (Y - ↑C x₁) + ↑C y₁)
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆))) =
(Y - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁)) * (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃) - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁)) +
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆))
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑C
((↑C L * (Y - ↑C x₁) + ↑C y₁) ^ 2 + (↑C W.a₁ * Y + ↑C W.a₃) * (↑C L * (Y - ↑C x₁) + ↑C y₁) -
(Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) =
(Y - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁)) * (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃) - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁)) +
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆))
[PROOFSTEP]
C_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ (↑C (↑C L) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁)) ^ 2 +
(↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)) * (↑C (↑C L) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁)) -
(↑C Y ^ 3 + ↑C (↑C W.a₂) * ↑C Y ^ 2 + ↑C (↑C W.a₄) * ↑C Y + ↑C (↑C W.a₆)) =
(Y - (↑C (↑C L) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁))) *
(-Y - (↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)) - (↑C (↑C L) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁))) +
(Y ^ 2 + (↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)) * Y -
(↑C Y ^ 3 + ↑C (↑C W.a₂) * ↑C Y ^ 2 + ↑C (↑C W.a₄) * ↑C Y + ↑C (↑C W.a₆)))
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑C (addPolynomial W x₁ y₁ L) - (Y - ↑C (linePolynomial x₁ y₁ L)) * (negPolynomial W - ↑C (linePolynomial x₁ y₁ L)) =
WeierstrassCurve.polynomial W * 1
[PROOFSTEP]
rw [W.C_addPolynomial, add_sub_cancel', mul_one]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ addPolynomial W x₁ y₁ L =
-Cubic.toPoly
{ a := 1, b := -L ^ 2 - W.a₁ * L + W.a₂,
c := 2 * x₁ * L ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * L + (-W.a₁ * y₁ + W.a₄),
d := -x₁ ^ 2 * L ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * L - (y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }
[PROOFSTEP]
rw [addPolynomial, linePolynomial, WeierstrassCurve.polynomial, Cubic.toPoly]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ eval (↑C L * (Y - ↑C x₁) + ↑C y₁)
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) =
-(↑C
{ a := 1, b := -L ^ 2 - W.a₁ * L + W.a₂,
c := 2 * x₁ * L ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * L + (-W.a₁ * y₁ + W.a₄),
d := -x₁ ^ 2 * L ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * L - (y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.a *
Y ^ 3 +
↑C
{ a := 1, b := -L ^ 2 - W.a₁ * L + W.a₂,
c := 2 * x₁ * L ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * L + (-W.a₁ * y₁ + W.a₄),
d := -x₁ ^ 2 * L ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * L - (y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.b *
Y ^ 2 +
↑C
{ a := 1, b := -L ^ 2 - W.a₁ * L + W.a₂,
c := 2 * x₁ * L ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * L + (-W.a₁ * y₁ + W.a₄),
d := -x₁ ^ 2 * L ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * L - (y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.c *
Y +
↑C
{ a := 1, b := -L ^ 2 - W.a₁ * L + W.a₂,
c := 2 * x₁ * L ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * L + (-W.a₁ * y₁ + W.a₄),
d := -x₁ ^ 2 * L ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * L - (y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.d)
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ (↑C L * (Y - ↑C x₁) + ↑C y₁) ^ 2 + (↑C W.a₁ * Y + ↑C W.a₃) * (↑C L * (Y - ↑C x₁) + ↑C y₁) -
(Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆) =
-(↑C 1 * Y ^ 3 + ↑C (-L ^ 2 - W.a₁ * L + W.a₂) * Y ^ 2 +
↑C (2 * x₁ * L ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * L + (-W.a₁ * y₁ + W.a₄)) * Y +
↑C (-x₁ ^ 2 * L ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * L - (y₁ ^ 2 + W.a₃ * y₁ - W.a₆)))
[PROOFSTEP]
C_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ (↑C L * (Y - ↑C x₁) + ↑C y₁) ^ 2 + (↑C W.a₁ * Y + ↑C W.a₃) * (↑C L * (Y - ↑C x₁) + ↑C y₁) -
(Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆) =
-(1 * Y ^ 3 + (-↑C L ^ 2 - ↑C W.a₁ * ↑C L + ↑C W.a₂) * Y ^ 2 +
(2 * ↑C x₁ * ↑C L ^ 2 + (↑C W.a₁ * ↑C x₁ - 2 * ↑C y₁ - ↑C W.a₃) * ↑C L + (-↑C W.a₁ * ↑C y₁ + ↑C W.a₄)) * Y +
(-↑C x₁ ^ 2 * ↑C L ^ 2 + (2 * ↑C x₁ * ↑C y₁ + ↑C W.a₃ * ↑C x₁) * ↑C L -
(↑C y₁ ^ 2 + ↑C W.a₃ * ↑C y₁ - ↑C W.a₆)))
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ addX (baseChange W A) (↑(algebraMap R A) x₁) (↑(algebraMap R A) x₂) (↑(algebraMap R A) L) =
↑(algebraMap R A) (addX W x₁ x₂ L)
[PROOFSTEP]
simp only [addX]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑(algebraMap R A) L ^ 2 + (baseChange W A).a₁ * ↑(algebraMap R A) L - (baseChange W A).a₂ - ↑(algebraMap R A) x₁ -
↑(algebraMap R A) x₂ =
↑(algebraMap R A) (L ^ 2 + W.a₁ * L - W.a₂ - x₁ - x₂)
[PROOFSTEP]
map_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑(algebraMap R A) L ^ 2 + (baseChange W A).a₁ * ↑(algebraMap R A) L - (baseChange W A).a₂ - ↑(algebraMap R A) x₁ -
↑(algebraMap R A) x₂ =
↑(algebraMap R A) L ^ 2 + ↑(algebraMap R A) W.a₁ * ↑(algebraMap R A) L - ↑(algebraMap R A) W.a₂ -
↑(algebraMap R A) x₁ -
↑(algebraMap R A) x₂
[PROOFSTEP]
rfl
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁✝ x₂✝ y₁ y₂ L✝ : R
x₁ x₂ L : A
⊢ addX (baseChange W B) (↑(algebraMap A B) x₁) (↑(algebraMap A B) x₂) (↑(algebraMap A B) L) =
↑(algebraMap A B) (addX (baseChange W A) x₁ x₂ L)
[PROOFSTEP]
rw [← baseChange_addX, baseChange_baseChange]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ addY' (baseChange W A) (↑(algebraMap R A) x₁) (↑(algebraMap R A) x₂) (↑(algebraMap R A) y₁) (↑(algebraMap R A) L) =
↑(algebraMap R A) (addY' W x₁ x₂ y₁ L)
[PROOFSTEP]
simp only [addY', baseChange_addX]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ↑(algebraMap R A) L * (↑(algebraMap R A) (addX W x₁ x₂ L) - ↑(algebraMap R A) x₁) + ↑(algebraMap R A) y₁ =
↑(algebraMap R A) (L * (addX W x₁ x₂ L - x₁) + y₁)
[PROOFSTEP]
map_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁✝ x₂✝ y₁✝ y₂ L✝ : R
x₁ x₂ y₁ L : A
⊢ addY' (baseChange W B) (↑(algebraMap A B) x₁) (↑(algebraMap A B) x₂) (↑(algebraMap A B) y₁) (↑(algebraMap A B) L) =
↑(algebraMap A B) (addY' (baseChange W A) x₁ x₂ y₁ L)
[PROOFSTEP]
rw [← baseChange_addY', baseChange_baseChange]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ addY (baseChange W A) (↑(algebraMap R A) x₁) (↑(algebraMap R A) x₂) (↑(algebraMap R A) y₁) (↑(algebraMap R A) L) =
↑(algebraMap R A) (addY W x₁ x₂ y₁ L)
[PROOFSTEP]
simp only [addY, baseChange_addY', baseChange_addX, baseChange_negY]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁✝ x₂✝ y₁✝ y₂ L✝ : R
x₁ x₂ y₁ L : A
⊢ addY (baseChange W B) (↑(algebraMap A B) x₁) (↑(algebraMap A B) x₂) (↑(algebraMap A B) y₁) (↑(algebraMap A B) L) =
↑(algebraMap A B) (addY (baseChange W A) x₁ x₂ y₁ L)
[PROOFSTEP]
rw [← baseChange_addY, baseChange_baseChange]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ XYIdeal W (addX W x₁ x₂ L) (↑C (addY W x₁ x₂ y₁ L)) =
span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ L))} ⊔ XIdeal W (addX W x₁ x₂ L)
[PROOFSTEP]
simp only [XYIdeal, XIdeal, XClass, YClass, addY, addY', negY, negPolynomial, linePolynomial]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C (addX W x₁ x₂ L))),
↑(CoordinateRing.mk W) (Y - ↑C (↑C (-(L * (addX W x₁ x₂ L - x₁) + y₁) - W.a₁ * addX W x₁ x₂ L - W.a₃)))} =
span {↑(CoordinateRing.mk W) (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃) - ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁))} ⊔
span {↑(CoordinateRing.mk W) (↑C (Y - ↑C (addX W x₁ x₂ L)))}
[PROOFSTEP]
rw [sub_sub <| -Y, neg_sub_left Y, map_neg, span_singleton_neg, sup_comm, ← span_insert, ←
span_pair_add_mul_right <| CoordinateRing.mk W <| C <| C <| W.a₁ + L, ← _root_.map_mul, ← map_add]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C (addX W x₁ x₂ L))),
↑(CoordinateRing.mk W)
(Y - ↑C (↑C (-(L * (addX W x₁ x₂ L - x₁) + y₁) - W.a₁ * addX W x₁ x₂ L - W.a₃)) +
↑C (Y - ↑C (addX W x₁ x₂ L)) * ↑C (↑C (W.a₁ + L)))} =
span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C (addX W x₁ x₂ L))),
↑(CoordinateRing.mk W) (↑C (↑C W.a₁ * Y + ↑C W.a₃) + ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁) + Y)}
[PROOFSTEP]
apply congr_arg (_ ∘ _ ∘ _ ∘ _)
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ Y - ↑C (↑C (-(L * (addX W x₁ x₂ L - x₁) + y₁) - W.a₁ * addX W x₁ x₂ L - W.a₃)) +
↑C (Y - ↑C (addX W x₁ x₂ L)) * ↑C (↑C (W.a₁ + L)) =
↑C (↑C W.a₁ * Y + ↑C W.a₃) + ↑C (↑C L * (Y - ↑C x₁) + ↑C y₁) + Y
[PROOFSTEP]
C_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ Y -
(-(↑C (↑C L) * (↑C (↑C (addX W x₁ x₂ L)) - ↑C (↑C x₁)) + ↑C (↑C y₁)) - ↑C (↑C W.a₁) * ↑C (↑C (addX W x₁ x₂ L)) -
↑C (↑C W.a₃)) +
(↑C Y - ↑C (↑C (addX W x₁ x₂ L))) * (↑C (↑C W.a₁) + ↑C (↑C L)) =
↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃) + (↑C (↑C L) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁)) + Y
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L) ↔
eval (addX W x₁ x₂ L) (addPolynomial W x₁ y₁ L) = 0
[PROOFSTEP]
rw [WeierstrassCurve.equation, addY', addPolynomial, linePolynomial, WeierstrassCurve.polynomial]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ eval (addX W x₁ x₂ L)
(eval (↑C (L * (addX W x₁ x₂ L - x₁) + y₁))
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆))) =
0 ↔
eval (addX W x₁ x₂ L)
(eval (↑C L * (Y - ↑C x₁) + ↑C y₁)
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆))) =
0
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx : eval (addX W x₁ x₂ L) (↑derivative (addPolynomial W x₁ y₁ L)) ≠ 0
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
[PROOFSTEP]
rw [WeierstrassCurve.nonsingular, and_iff_right hx', addY', WeierstrassCurve.polynomialX, WeierstrassCurve.polynomialY]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx : eval (addX W x₁ x₂ L) (↑derivative (addPolynomial W x₁ y₁ L)) ≠ 0
⊢ eval (addX W x₁ x₂ L)
(eval (↑C (L * (addX W x₁ x₂ L - x₁) + y₁))
(↑C (↑C W.a₁) * Y - ↑C (↑C 3 * Y ^ 2 + ↑C (2 * W.a₂) * Y + ↑C W.a₄))) ≠
0 ∨
eval (addX W x₁ x₂ L) (eval (↑C (L * (addX W x₁ x₂ L - x₁) + y₁)) (↑C (↑C 2) * Y + ↑C (↑C W.a₁ * Y + ↑C W.a₃))) ≠ 0
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx : eval (addX W x₁ x₂ L) (↑derivative (addPolynomial W x₁ y₁ L)) ≠ 0
⊢ W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) ≠ 0 ∨
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) ≠ 0
[PROOFSTEP]
contrapose! hx
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ eval (addX W x₁ x₂ L) (↑derivative (addPolynomial W x₁ y₁ L)) = 0
[PROOFSTEP]
rw [addPolynomial, linePolynomial, WeierstrassCurve.polynomial]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ eval (addX W x₁ x₂ L)
(↑derivative
(eval (↑C L * (Y - ↑C x₁) + ↑C y₁)
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)))) =
0
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ eval (addX W x₁ x₂ L)
(↑derivative
((↑C L * (Y - ↑C x₁) + ↑C y₁) ^ 2 + (↑C W.a₁ * Y + ↑C W.a₃) * (↑C L * (Y - ↑C x₁) + ↑C y₁) -
(Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆))) =
0
[PROOFSTEP]
derivative_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ eval (addX W x₁ x₂ L)
(↑C 2 * (↑C L * (Y - ↑C x₁) + ↑C y₁) * (0 * (Y - ↑C x₁) + ↑C L * (1 - 0) + 0) +
((0 * Y + ↑C W.a₁ * 1 + 0) * (↑C L * (Y - ↑C x₁) + ↑C y₁) +
(↑C W.a₁ * Y + ↑C W.a₃) * (0 * (Y - ↑C x₁) + ↑C L * (1 - 0) + 0)) -
(↑C ↑3 * Y ^ (3 - 1) + (0 * Y ^ 2 + ↑C W.a₂ * (↑C 2 * Y * 1)) + (0 * Y + ↑C W.a₄ * 1) + 0)) =
0
[PROOFSTEP]
simp only [zero_add, add_zero, sub_zero, zero_mul, mul_one]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ eval (addX W x₁ x₂ L)
(↑C 2 * (↑C L * (Y - ↑C x₁) + ↑C y₁) * ↑C L +
(↑C W.a₁ * (↑C L * (Y - ↑C x₁) + ↑C y₁) + (↑C W.a₁ * Y + ↑C W.a₃) * ↑C L) -
(↑C ↑3 * Y ^ (3 - 1) + ↑C W.a₂ * (↑C 2 * Y) + ↑C W.a₄)) =
0
[PROOFSTEP]
eval_simp
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ 2 * (L * (addX W x₁ x₂ L - x₁) + y₁) * L +
(W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) * L) -
(↑3 * addX W x₁ x₂ L ^ (3 - 1) + W.a₂ * (2 * addX W x₁ x₂ L) + W.a₄) =
0
[PROOFSTEP]
linear_combination (norm := (norm_num1; ring1)) hx.left + L * hx.right
[GOAL]
case a
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ 2 * (L * (addX W x₁ x₂ L - x₁) + y₁) * L +
(W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) * L) -
(↑3 * addX W x₁ x₂ L ^ (3 - 1) + W.a₂ * (2 * addX W x₁ x₂ L) + W.a₄) -
0 -
(W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) +
L * (2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃)) -
(0 + L * 0)) =
0
[PROOFSTEP]
norm_num1
[GOAL]
case a
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
hx' : WeierstrassCurve.equation W (addX W x₁ x₂ L) (addY' W x₁ x₂ y₁ L)
hx :
W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) = 0 ∧
2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) = 0
⊢ 2 * (L * (addX W x₁ x₂ L - x₁) + y₁) * L +
(W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃) * L) -
(3 * addX W x₁ x₂ L ^ 2 + W.a₂ * (2 * addX W x₁ x₂ L) + W.a₄) -
0 -
(W.a₁ * (L * (addX W x₁ x₂ L - x₁) + y₁) - (3 * addX W x₁ x₂ L ^ 2 + 2 * W.a₂ * addX W x₁ x₂ L + W.a₄) +
L * (2 * (L * (addX W x₁ x₂ L - x₁) + y₁) + (W.a₁ * addX W x₁ x₂ L + W.a₃)) -
(0 + L * 0)) =
0
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ WeierstrassCurve.equation W x₁ (negY W x₁ y₁) ↔ WeierstrassCurve.equation W x₁ y₁
[PROOFSTEP]
rw [equation_iff, equation_iff, negY]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ (-y₁ - W.a₁ * x₁ - W.a₃) ^ 2 + W.a₁ * x₁ * (-y₁ - W.a₁ * x₁ - W.a₃) + W.a₃ * (-y₁ - W.a₁ * x₁ - W.a₃) =
x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆ ↔
y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
[PROOFSTEP]
congr! 1
[GOAL]
case a.h.e'_2
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ (-y₁ - W.a₁ * x₁ - W.a₃) ^ 2 + W.a₁ * x₁ * (-y₁ - W.a₁ * x₁ - W.a₃) + W.a₃ * (-y₁ - W.a₁ * x₁ - W.a₃) =
y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁
[PROOFSTEP]
ring1
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ WeierstrassCurve.nonsingular W x₁ (negY W x₁ y₁) ↔ WeierstrassCurve.nonsingular W x₁ y₁
[PROOFSTEP]
rw [nonsingular_iff, equation_neg_iff, ← negY, negY_negY, ← @ne_comm _ y₁, nonsingular_iff]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ WeierstrassCurve.equation W x₁ y₁ ∧ (W.a₁ * negY W x₁ y₁ ≠ 3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ ∨ y₁ ≠ negY W x₁ y₁) ↔
WeierstrassCurve.equation W x₁ y₁ ∧ (W.a₁ * y₁ ≠ 3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ ∨ y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃)
[PROOFSTEP]
exact
and_congr_right' <|
(iff_congr not_and_or.symm not_and_or.symm).mpr <| not_congr <| and_congr_left fun h => by rw [← h]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
h : y₁ = negY W x₁ y₁
⊢ W.a₁ * negY W x₁ y₁ = 3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ ↔ W.a₁ * y₁ = 3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄
[PROOFSTEP]
rw [← h]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ ∀ (x : Point W), - -x = x
[PROOFSTEP]
rintro (_ | _)
[GOAL]
case zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L : R
⊢ - -zero = zero
[PROOFSTEP]
simp [zero_def]
[GOAL]
case some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L x✝ y✝ : R
h✝ : WeierstrassCurve.nonsingular W x✝ y✝
⊢ - -some h✝ = some h✝
[PROOFSTEP]
simp [zero_def]
[GOAL]
case some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
A : Type v
inst✝⁵ : CommRing A
inst✝⁴ : Algebra R A
B : Type w
inst✝³ : CommRing B
inst✝² : Algebra R B
inst✝¹ : Algebra A B
inst✝ : IsScalarTower R A B
x₁ x₂ y₁ y₂ L x✝ y✝ : R
h✝ : WeierstrassCurve.nonsingular W x✝ y✝
⊢ W.a₃ - (-y✝ - W.a₁ * x✝) - W.a₁ * x✝ - W.a₃ = y✝
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY W x₂ y₂
⊢ slope W x₁ x₂ y₁ y₂ = 0
[PROOFSTEP]
rw [slope, if_pos hx, if_pos hy]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ ≠ negY W x₂ y₂
⊢ slope W x₁ x₂ y₁ y₂ = (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)
[PROOFSTEP]
rw [slope, if_pos hx, if_neg hy]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ ≠ x₂
⊢ slope W x₁ x₂ y₁ y₂ = (y₁ - y₂) / (x₁ - x₂)
[PROOFSTEP]
rw [slope, if_neg hx]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ ≠ negY W x₂ y₂
⊢ slope W x₁ x₂ y₁ y₂ =
-eval x₁ (eval (↑C y₁) (WeierstrassCurve.polynomialX W)) / eval x₁ (eval (↑C y₁) (WeierstrassCurve.polynomialY W))
[PROOFSTEP]
rw [slope_of_Y_ne hx hy, eval_polynomialX, neg_sub]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ ≠ negY W x₂ y₂
⊢ (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁) =
(3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / eval x₁ (eval (↑C y₁) (WeierstrassCurve.polynomialY W))
[PROOFSTEP]
congr 1
[GOAL]
case e_a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ ≠ negY W x₂ y₂
⊢ y₁ - negY W x₁ y₁ = eval x₁ (eval (↑C y₁) (WeierstrassCurve.polynomialY W))
[PROOFSTEP]
rw [negY, eval_polynomialY]
[GOAL]
case e_a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ ≠ negY W x₂ y₂
⊢ y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) = 2 * y₁ + W.a₁ * x₁ + W.a₃
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁) (↑(algebraMap F K) y₂) =
↑(algebraMap F K) (slope W x₁ x₂ y₁ y₂)
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
⊢ slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁) (↑(algebraMap F K) y₂) =
↑(algebraMap F K) (slope W x₁ x₂ y₁ y₂)
[PROOFSTEP]
by_cases hy : y₁ = W.negY x₂ y₂
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY W x₂ y₂
⊢ slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁) (↑(algebraMap F K) y₂) =
↑(algebraMap F K) (slope W x₁ x₂ y₁ y₂)
[PROOFSTEP]
rw [slope_of_Y_eq hx hy, slope_of_Y_eq <| congr_arg _ hx, map_zero]
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY W x₂ y₂
⊢ ↑(algebraMap F K) y₁ = negY (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂)
[PROOFSTEP]
rw [hy, baseChange_negY]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁) (↑(algebraMap F K) y₂) =
↑(algebraMap F K) (slope W x₁ x₂ y₁ y₂)
[PROOFSTEP]
rw [slope_of_Y_ne hx hy, slope_of_Y_ne <| congr_arg _ hx]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ (3 * ↑(algebraMap F K) x₁ ^ 2 + 2 * (baseChange W K).a₂ * ↑(algebraMap F K) x₁ + (baseChange W K).a₄ -
(baseChange W K).a₁ * ↑(algebraMap F K) y₁) /
(↑(algebraMap F K) y₁ - negY (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) y₁)) =
↑(algebraMap F K) ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))
[PROOFSTEP]
map_simp
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ (3 * ↑(algebraMap F K) x₁ ^ 2 + 2 * (baseChange W K).a₂ * ↑(algebraMap F K) x₁ + (baseChange W K).a₄ -
(baseChange W K).a₁ * ↑(algebraMap F K) y₁) /
(↑(algebraMap F K) y₁ - negY (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) y₁)) =
(3 * ↑(algebraMap F K) x₁ ^ 2 + 2 * ↑(algebraMap F K) W.a₂ * ↑(algebraMap F K) x₁ + ↑(algebraMap F K) W.a₄ -
↑(algebraMap F K) W.a₁ * ↑(algebraMap F K) y₁) /
(↑(algebraMap F K) y₁ - ↑(algebraMap F K) (negY W x₁ y₁))
[PROOFSTEP]
simp only [baseChange_negY]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ (3 * ↑(algebraMap F K) x₁ ^ 2 + 2 * (baseChange W K).a₂ * ↑(algebraMap F K) x₁ + (baseChange W K).a₄ -
(baseChange W K).a₁ * ↑(algebraMap F K) y₁) /
(↑(algebraMap F K) y₁ - ↑(algebraMap F K) (negY W x₁ y₁)) =
(3 * ↑(algebraMap F K) x₁ ^ 2 + 2 * ↑(algebraMap F K) W.a₂ * ↑(algebraMap F K) x₁ + ↑(algebraMap F K) W.a₄ -
↑(algebraMap F K) W.a₁ * ↑(algebraMap F K) y₁) /
(↑(algebraMap F K) y₁ - ↑(algebraMap F K) (negY W x₁ y₁))
[PROOFSTEP]
rfl
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ ↑(algebraMap F K) y₁ ≠ negY (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂)
[PROOFSTEP]
rw [baseChange_negY]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ ↑(algebraMap F K) y₁ ≠ ↑(algebraMap F K) (negY W x₂ y₂)
[PROOFSTEP]
contrapose! hy
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : ↑(algebraMap F K) y₁ = ↑(algebraMap F K) (negY W x₂ y₂)
⊢ y₁ = negY W x₂ y₂
[PROOFSTEP]
exact NoZeroSMulDivisors.algebraMap_injective F K hy
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : ¬x₁ = x₂
⊢ slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁) (↑(algebraMap F K) y₂) =
↑(algebraMap F K) (slope W x₁ x₂ y₁ y₂)
[PROOFSTEP]
rw [slope_of_X_ne hx, slope_of_X_ne]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : ¬x₁ = x₂
⊢ (↑(algebraMap F K) y₁ - ↑(algebraMap F K) y₂) / (↑(algebraMap F K) x₁ - ↑(algebraMap F K) x₂) =
↑(algebraMap F K) ((y₁ - y₂) / (x₁ - x₂))
[PROOFSTEP]
map_simp
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : ¬x₁ = x₂
⊢ ↑(algebraMap F K) x₁ ≠ ↑(algebraMap F K) x₂
[PROOFSTEP]
contrapose! hx
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : ↑(algebraMap F K) x₁ = ↑(algebraMap F K) x₂
⊢ x₁ = x₂
[PROOFSTEP]
exact NoZeroSMulDivisors.algebraMap_injective F K hx
[GOAL]
F✝ : Type u
inst✝⁹ : Field F✝
W✝ : WeierstrassCurve F✝
K✝ : Type v
inst✝⁸ : Field K✝
inst✝⁷ : Algebra F✝ K✝
x₁✝ x₂✝ y₁✝ y₂✝ : F✝
h₁ : WeierstrassCurve.nonsingular W✝ x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W✝ x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W✝ x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W✝ x₂✝ y₂✝
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ x₂ y₁ y₂ : F
⊢ slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁) (↑(algebraMap F K) y₂) =
↑(algebraMap F K) (slope (baseChange W F) x₁ x₂ y₁ y₂)
[PROOFSTEP]
rw [← baseChange_slope, baseChange_baseChange]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
⊢ y₁ = y₂ ∨ y₁ = negY W x₂ y₂
[PROOFSTEP]
rw [equation_iff] at h₁' h₂'
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hx : x₁ = x₂
⊢ y₁ = y₂ ∨ y₁ = negY W x₂ y₂
[PROOFSTEP]
rw [← sub_eq_zero, ← @sub_eq_zero _ _ y₁, ← mul_eq_zero, negY]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hx : x₁ = x₂
⊢ (y₁ - y₂) * (y₁ - (-y₂ - W.a₁ * x₂ - W.a₃)) = 0
[PROOFSTEP]
linear_combination (norm := (rw [hx]; ring1)) h₁' - h₂'
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hx : x₁ = x₂
⊢ (y₁ - y₂) * (y₁ - (-y₂ - W.a₁ * x₂ - W.a₃)) - 0 -
(y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ - (y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂) -
(x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆ - (x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆))) =
0
[PROOFSTEP]
rw [hx]
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hx : x₁ = x₂
⊢ (y₁ - y₂) * (y₁ - (-y₂ - W.a₁ * x₂ - W.a₃)) - 0 -
(y₁ ^ 2 + W.a₁ * x₂ * y₁ + W.a₃ * y₁ - (y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂) -
(x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆ - (x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆))) =
0
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ XYIdeal W x₂ (↑C y₂) = XYIdeal W x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
clear h₂
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ XYIdeal W x₂ (↑C y₂) = XYIdeal W x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
have hy₂ : y₂ = (linePolynomial x₁ y₁ <| W.slope x₁ x₂ y₁ y₂).eval x₂ :=
by
by_cases hx : x₁ = x₂
· rcases hx, Y_eq_of_Y_ne h₁' h₂' hx <| hxy hx with ⟨rfl, rfl⟩
field_simp [linePolynomial, sub_ne_zero_of_ne (hxy rfl)]
· field_simp [linePolynomial, slope_of_X_ne hx, sub_ne_zero_of_ne hx]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : x₁ = x₂
⊢ y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
rcases hx, Y_eq_of_Y_ne h₁' h₂' hx <| hxy hx with ⟨rfl, rfl⟩
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₁
⊢ y₁ = eval x₁ (linePolynomial x₁ y₁ (slope W x₁ x₁ y₁ y₁))
[PROOFSTEP]
field_simp [linePolynomial, sub_ne_zero_of_ne (hxy rfl)]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : ¬x₁ = x₂
⊢ y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
field_simp [linePolynomial, slope_of_X_ne hx, sub_ne_zero_of_ne hx]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : ¬x₁ = x₂
⊢ y₂ * (x₁ - x₂) = (y₁ - y₂) * (x₂ - x₁) + y₁ * (x₁ - x₂)
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ XYIdeal W x₂ (↑C y₂) = XYIdeal W x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
nth_rw 1 [hy₂]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ XYIdeal W x₂ (↑C (eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))) =
XYIdeal W x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
simp only [XYIdeal, XClass, YClass, linePolynomial]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₂)),
↑(CoordinateRing.mk W) (Y - ↑C (↑C (eval x₂ (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁))))} =
span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₂)),
↑(CoordinateRing.mk W) (Y - ↑C (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁))}
[PROOFSTEP]
rw [← span_pair_add_mul_right <| CoordinateRing.mk W <| C <| C <| -W.slope x₁ x₂ y₁ y₂, ← _root_.map_mul, ← map_add]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₂)),
↑(CoordinateRing.mk W)
(Y - ↑C (↑C (eval x₂ (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁))) +
↑C (Y - ↑C x₂) * ↑C (↑C (-slope W x₁ x₂ y₁ y₂)))} =
span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₂)),
↑(CoordinateRing.mk W) (Y - ↑C (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁))}
[PROOFSTEP]
apply congr_arg (_ ∘ _ ∘ _ ∘ _)
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ Y - ↑C (↑C (eval x₂ (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁))) +
↑C (Y - ↑C x₂) * ↑C (↑C (-slope W x₁ x₂ y₁ y₂)) =
Y - ↑C (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁)
[PROOFSTEP]
eval_simp
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ Y - ↑C (↑C (slope W x₁ x₂ y₁ y₂ * (x₂ - x₁) + y₁)) + ↑C (Y - ↑C x₂) * ↑C (↑C (-slope W x₁ x₂ y₁ y₂)) =
Y - ↑C (↑C (slope W x₁ x₂ y₁ y₂) * (Y - ↑C x₁) + ↑C y₁)
[PROOFSTEP]
C_simp
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hy₂ : y₂ = eval x₂ (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))
⊢ Y - (↑C (↑C (slope W x₁ x₂ y₁ y₂)) * (↑C (↑C x₂) - ↑C (↑C x₁)) + ↑C (↑C y₁)) +
(↑C Y - ↑C (↑C x₂)) * -↑C (↑C (slope W x₁ x₂ y₁ y₂)) =
Y - (↑C (↑C (slope W x₁ x₂ y₁ y₂)) * (↑C Y - ↑C (↑C x₁)) + ↑C (↑C y₁))
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ addPolynomial W x₁ y₁ (slope W x₁ x₂ y₁ y₂) =
-((Y - ↑C x₁) * (Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
clear h₂
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ addPolynomial W x₁ y₁ (slope W x₁ x₂ y₁ y₂) =
-((Y - ↑C x₁) * (Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
rw [addPolynomial_eq, neg_inj, Cubic.prod_X_sub_C_eq, Cubic.toPoly_injective]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ { a := 1, b := -slope W x₁ x₂ y₁ y₂ ^ 2 - W.a₁ * slope W x₁ x₂ y₁ y₂ + W.a₂,
c := 2 * x₁ * slope W x₁ x₂ y₁ y₂ ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * slope W x₁ x₂ y₁ y₂ + (-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * slope W x₁ x₂ y₁ y₂ ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * slope W x₁ x₂ y₁ y₂ -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) + x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂),
d := -(x₁ * x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) }
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : x₁ = x₂
⊢ { a := 1, b := -slope W x₁ x₂ y₁ y₂ ^ 2 - W.a₁ * slope W x₁ x₂ y₁ y₂ + W.a₂,
c := 2 * x₁ * slope W x₁ x₂ y₁ y₂ ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * slope W x₁ x₂ y₁ y₂ + (-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * slope W x₁ x₂ y₁ y₂ ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * slope W x₁ x₂ y₁ y₂ -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) + x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂),
d := -(x₁ * x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) }
[PROOFSTEP]
rcases hx, Y_eq_of_Y_ne h₁' h₂' hx (hxy hx) with ⟨rfl, rfl⟩
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₁
⊢ { a := 1, b := -slope W x₁ x₁ y₁ y₁ ^ 2 - W.a₁ * slope W x₁ x₁ y₁ y₁ + W.a₂,
c := 2 * x₁ * slope W x₁ x₁ y₁ y₁ ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * slope W x₁ x₁ y₁ y₁ + (-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * slope W x₁ x₁ y₁ y₁ ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * slope W x₁ x₁ y₁ y₁ -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁)),
c := x₁ * x₁ + x₁ * addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁) + x₁ * addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁),
d := -(x₁ * x₁ * addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁)) }
[PROOFSTEP]
rw [equation_iff] at h₁' h₂'
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₁
⊢ { a := 1, b := -slope W x₁ x₁ y₁ y₁ ^ 2 - W.a₁ * slope W x₁ x₁ y₁ y₁ + W.a₂,
c := 2 * x₁ * slope W x₁ x₁ y₁ y₁ ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * slope W x₁ x₁ y₁ y₁ + (-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * slope W x₁ x₁ y₁ y₁ ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * slope W x₁ x₁ y₁ y₁ -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁)),
c := x₁ * x₁ + x₁ * addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁) + x₁ * addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁),
d := -(x₁ * x₁ * addX W x₁ x₁ (slope W x₁ x₁ y₁ y₁)) }
[PROOFSTEP]
rw [slope_of_Y_ne rfl <| hxy rfl]
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₁
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }
[PROOFSTEP]
rw [negY, ← sub_ne_zero] at hxy
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }
[PROOFSTEP]
ext
[GOAL]
case pos.a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.a =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }.a
[PROOFSTEP]
rfl
[GOAL]
case pos.b
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.b =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }.b
[PROOFSTEP]
simp only [addX]
[GOAL]
case pos.b
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ -((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂ =
-(x₁ + x₁ +
(((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
W.a₂ -
x₁ -
x₁))
[PROOFSTEP]
ring1
[GOAL]
case pos.c
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.c =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }.c
[PROOFSTEP]
field_simp [hxy rfl]
[GOAL]
case pos.c
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ 2 * x₁ * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) *
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 +
(-(W.a₁ * y₁) + W.a₄) * ((y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃))) =
x₁ * x₁ * ((y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃))) +
x₁ *
((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) +
W.a₁ * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * W.a₂ -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * x₁ -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * x₁) +
x₁ *
((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) +
W.a₁ * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * W.a₂ -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * x₁ -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * x₁)
[PROOFSTEP]
ring1
[GOAL]
case pos.d
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.d =
{ a := 1, b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }.d
[PROOFSTEP]
linear_combination (norm := (field_simp [hxy rfl]; ring1)) -h₁'
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ { a := 1,
b :=
-((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 -
W.a₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
W.a₂,
c :=
2 * x₁ * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(W.a₁ * x₁ - 2 * y₁ - W.a₃) *
((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) ^ 2 +
(2 * x₁ * y₁ + W.a₃ * x₁) * ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.d -
{ a := 1,
b := -(x₁ + x₁ + addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))),
c :=
x₁ * x₁ + x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)) +
x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁)),
d := -(x₁ * x₁ * addX W x₁ x₁ ((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) / (y₁ - negY W x₁ y₁))) }.d -
(-(y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁) - -(x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆)) =
0
[PROOFSTEP]
field_simp [hxy rfl]
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' h₂' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
hxy✝ : x₁ = x₁ → y₁ ≠ -y₁ - W.a₁ * x₁ - W.a₃
hxy : x₁ = x₁ → y₁ - (-y₁ - W.a₁ * x₁ - W.a₃) ≠ 0
⊢ -(x₁ ^ 2 * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃))) +
(2 * x₁ * y₁ + W.a₃ * x₁) * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) *
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * (y₁ ^ 2 + W.a₃ * y₁ - W.a₆) +
x₁ * x₁ *
((3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) +
W.a₁ * (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄ - W.a₁ * y₁) * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * W.a₂ -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * x₁ -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) * x₁) -
(y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2 * (y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) *
(-(W.a₃ * y₁) + (-(W.a₁ * x₁ * y₁) + -y₁ ^ 2) - (-W.a₆ + (-(W.a₄ * x₁) + (-(W.a₂ * x₁ ^ 2) + -x₁ ^ 3)))) =
0
[PROOFSTEP]
ring1
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : ¬x₁ = x₂
⊢ { a := 1, b := -slope W x₁ x₂ y₁ y₂ ^ 2 - W.a₁ * slope W x₁ x₂ y₁ y₂ + W.a₂,
c := 2 * x₁ * slope W x₁ x₂ y₁ y₂ ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * slope W x₁ x₂ y₁ y₂ + (-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * slope W x₁ x₂ y₁ y₂ ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * slope W x₁ x₂ y₁ y₂ -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) + x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂),
d := -(x₁ * x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) }
[PROOFSTEP]
rw [equation_iff] at h₁' h₂'
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : ¬x₁ = x₂
⊢ { a := 1, b := -slope W x₁ x₂ y₁ y₂ ^ 2 - W.a₁ * slope W x₁ x₂ y₁ y₂ + W.a₂,
c := 2 * x₁ * slope W x₁ x₂ y₁ y₂ ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * slope W x₁ x₂ y₁ y₂ + (-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * slope W x₁ x₂ y₁ y₂ ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * slope W x₁ x₂ y₁ y₂ -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) + x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂),
d := -(x₁ * x₂ * addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) }
[PROOFSTEP]
rw [slope_of_X_ne hx]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx : ¬x₁ = x₂
⊢ { a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }
[PROOFSTEP]
rw [← sub_eq_zero] at hx
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ { a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) } =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }
[PROOFSTEP]
ext
[GOAL]
case neg.a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ { a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.a =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.a
[PROOFSTEP]
rfl
[GOAL]
case neg.b
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ { a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.b =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.b
[PROOFSTEP]
simp only [addX]
[GOAL]
case neg.b
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂ =
-(x₁ + x₂ + (((y₁ - y₂) / (x₁ - x₂)) ^ 2 + W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) - W.a₂ - x₁ - x₂))
[PROOFSTEP]
ring1
[GOAL]
case neg.c
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ { a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.c =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.c
[PROOFSTEP]
apply mul_right_injective₀ hx
[GOAL]
case neg.c.a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ (fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.c =
(fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.c
[PROOFSTEP]
linear_combination (norm := (field_simp [hx]; ring1)) h₂' - h₁'
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ (fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.c -
(fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.c -
(y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ - (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁) -
(x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆ - (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆))) =
0
[PROOFSTEP]
field_simp [hx]
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ (x₁ - x₂) *
(2 * x₁ * (y₁ - y₂) ^ 2 * (x₁ - x₂) + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * (y₁ - y₂) * (x₁ - x₂) ^ 2 +
(-(W.a₁ * y₁) + W.a₄) * ((x₁ - x₂) ^ 2 * (x₁ - x₂))) -
(x₁ - x₂) *
(x₁ * x₂ * ((x₁ - x₂) ^ 2 * (x₁ - x₂)) +
x₁ *
((y₁ - y₂) ^ 2 * (x₁ - x₂) + W.a₁ * (y₁ - y₂) * (x₁ - x₂) ^ 2 - (x₁ - x₂) ^ 2 * (x₁ - x₂) * W.a₂ -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * x₁ -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * x₂) +
x₂ *
((y₁ - y₂) ^ 2 * (x₁ - x₂) + W.a₁ * (y₁ - y₂) * (x₁ - x₂) ^ 2 - (x₁ - x₂) ^ 2 * (x₁ - x₂) * W.a₂ -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * x₁ -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * x₂)) -
(x₁ - x₂) ^ 2 * (x₁ - x₂) *
(y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ - (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁) -
(x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ - (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁))) =
0
[PROOFSTEP]
ring1
[GOAL]
case neg.d
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ { a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.d =
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.d
[PROOFSTEP]
apply mul_right_injective₀ hx
[GOAL]
case neg.d.a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ (fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.d =
(fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.d
[PROOFSTEP]
linear_combination (norm := (field_simp [hx]; ring1)) x₂ * h₁' - x₁ * h₂'
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ (fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -((y₁ - y₂) / (x₁ - x₂)) ^ 2 - W.a₁ * ((y₁ - y₂) / (x₁ - x₂)) + W.a₂,
c :=
2 * x₁ * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (W.a₁ * x₁ - 2 * y₁ - W.a₃) * ((y₁ - y₂) / (x₁ - x₂)) +
(-W.a₁ * y₁ + W.a₄),
d :=
-x₁ ^ 2 * ((y₁ - y₂) / (x₁ - x₂)) ^ 2 + (2 * x₁ * y₁ + W.a₃ * x₁) * ((y₁ - y₂) / (x₁ - x₂)) -
(y₁ ^ 2 + W.a₃ * y₁ - W.a₆) }.d -
(fun x x_1 => x * x_1) (x₁ - x₂)
{ a := 1, b := -(x₁ + x₂ + addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))),
c := x₁ * x₂ + x₁ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)) + x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂)),
d := -(x₁ * x₂ * addX W x₁ x₂ ((y₁ - y₂) / (x₁ - x₂))) }.d -
(x₂ * (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁) - x₁ * (y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂) -
(x₂ * (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆) - x₁ * (x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆))) =
0
[PROOFSTEP]
field_simp [hx]
[GOAL]
case a
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁ = x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆
h₂' : y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂ = x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx✝ : ¬x₁ = x₂
hx : ¬x₁ - x₂ = 0
⊢ (x₁ - x₂) *
(-(x₁ ^ 2 * (y₁ - y₂) ^ 2 * (x₁ - x₂)) + (2 * x₁ * y₁ + W.a₃ * x₁) * (y₁ - y₂) * (x₁ - x₂) ^ 2 -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * (y₁ ^ 2 + W.a₃ * y₁ - W.a₆)) +
(x₁ - x₂) *
(x₁ * x₂ *
((y₁ - y₂) ^ 2 * (x₁ - x₂) + W.a₁ * (y₁ - y₂) * (x₁ - x₂) ^ 2 - (x₁ - x₂) ^ 2 * (x₁ - x₂) * W.a₂ -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * x₁ -
(x₁ - x₂) ^ 2 * (x₁ - x₂) * x₂)) -
(x₁ - x₂) ^ 2 * (x₁ - x₂) *
(x₂ * (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁) - x₁ * (y₂ ^ 2 + W.a₁ * x₂ * y₂ + W.a₃ * y₂) -
(x₂ * (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆) - x₁ * (x₂ ^ 3 + W.a₂ * x₂ ^ 2 + W.a₄ * x₂ + W.a₆))) =
0
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑(mk W) (↑C (addPolynomial W x₁ y₁ (slope W x₁ x₂ y₁ y₂))) =
-(XClass W x₁ * XClass W x₂ * XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)))
[PROOFSTEP]
simp only [addPolynomial_slope h₁' h₂' hxy, C_neg, mk, map_neg, neg_inj, _root_.map_mul]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) (↑C (Y - ↑C x₁)) *
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) (↑C (Y - ↑C x₂)) *
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) (↑C (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)))) =
XClass W x₁ * XClass W x₂ * XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
rfl
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑derivative (addPolynomial W x₁ y₁ (slope W x₁ x₂ y₁ y₂)) =
-((Y - ↑C x₁) * (Y - ↑C x₂) + (Y - ↑C x₁) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) +
(Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
rw [addPolynomial_slope h₁' h₂' hxy]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑derivative (-((Y - ↑C x₁) * (Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))) =
-((Y - ↑C x₁) * (Y - ↑C x₂) + (Y - ↑C x₁) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) +
(Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
derivative_simp
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ -(((1 - 0) * (Y - ↑C x₂) + (Y - ↑C x₁) * (1 - 0)) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) +
(Y - ↑C x₁) * (Y - ↑C x₂) * (1 - 0)) =
-((Y - ↑C x₁) * (Y - ↑C x₂) + (Y - ↑C x₁) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) +
(Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ WeierstrassCurve.equation W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
rw [equation_add_iff, addPolynomial_slope h₁' h₂' hxy]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ eval (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))
(-((Y - ↑C x₁) * (Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))) =
0
[PROOFSTEP]
eval_simp
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ -((addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - x₁) * (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - x₂) *
(addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) =
0
[PROOFSTEP]
rw [neg_eq_zero, sub_self, mul_zero]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
clear h₂'
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
by_cases hx₁ : W.addX x₁ x₂ (W.slope x₁ x₂ y₁ y₂) = x₁
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
rwa [addY', hx₁, sub_self, mul_zero, zero_add]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
by_cases hx₂ : W.addX x₁ x₂ (W.slope x₁ x₂ y₁ y₂) = x₂
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
hx : x₁ = x₂
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
subst hx
[GOAL]
case pos
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₁ y₂
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₂
hx₁ : ¬addX W x₁ x₁ (slope W x₁ x₁ y₁ y₂) = x₁
hx₂ : addX W x₁ x₁ (slope W x₁ x₁ y₁ y₂) = x₁
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₁ (slope W x₁ x₁ y₁ y₂)) (addY' W x₁ x₁ y₁ (slope W x₁ x₁ y₁ y₂))
[PROOFSTEP]
contradiction
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
hx : ¬x₁ = x₂
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
rwa [addY', ← neg_sub, mul_neg, hx₂, slope_of_X_ne hx, div_mul_cancel _ <| sub_ne_zero_of_ne hx, neg_sub,
sub_add_cancel]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
⊢ WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY' W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))
[PROOFSTEP]
apply W.nonsingular_add_of_eval_derivative_ne_zero _ _ _ _ (equation_add' h₁.1 h₂.1 hxy)
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
⊢ eval (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (↑derivative (addPolynomial W x₁ y₁ (slope W x₁ x₂ y₁ y₂))) ≠ 0
[PROOFSTEP]
rw [derivative_addPolynomial_slope h₁.left h₂.left hxy]
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
⊢ eval (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))
(-((Y - ↑C x₁) * (Y - ↑C x₂) + (Y - ↑C x₁) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) +
(Y - ↑C x₂) * (Y - ↑C (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))))) ≠
0
[PROOFSTEP]
eval_simp
[GOAL]
case neg
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
hx₁ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₁
hx₂ : ¬addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) = x₂
⊢ -((addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - x₁) * (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - x₂) +
(addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - x₁) *
(addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) +
(addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - x₂) *
(addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂) - addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))) ≠
0
[PROOFSTEP]
simpa only [neg_ne_zero, sub_self, mul_zero, add_zero] using mul_ne_zero (sub_ne_zero_of_ne hx₁) (sub_ne_zero_of_ne hx₂)
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ∀ (a : Point W), 0 + a = a
[PROOFSTEP]
rintro (_ | _)
[GOAL]
case zero
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ 0 + zero = zero
[PROOFSTEP]
rfl
[GOAL]
case some
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular W x✝ y✝
⊢ 0 + some h✝ = some h✝
[PROOFSTEP]
rfl
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ∀ (a : Point W), a + 0 = a
[PROOFSTEP]
rintro (_ | _)
[GOAL]
case zero
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ zero + 0 = zero
[PROOFSTEP]
rfl
[GOAL]
case some
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular W x✝ y✝
⊢ some h✝ + 0 = some h✝
[PROOFSTEP]
rfl
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY W x₂ y₂
⊢ some h₁ + some h₂ = 0
[PROOFSTEP]
simp only [← add_def, add, dif_pos hx, dif_pos hy]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ = x₂
hy : y₁ ≠ negY W x₂ y₂
⊢ some h₁ + some h₂ =
some
(_ : WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂)))
[PROOFSTEP]
simp only [← add_def, add, dif_pos hx, dif_neg hy]
[GOAL]
F : Type u
inst✝² : Field F
W : WeierstrassCurve F
K : Type v
inst✝¹ : Field K
inst✝ : Algebra F K
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hx : x₁ ≠ x₂
⊢ some h₁ + some h₂ =
some
(_ : WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂)))
[PROOFSTEP]
simp only [← add_def, add, dif_neg hx]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ XYIdeal W x₁ (↑C (negY W x₁ y₁)) * XYIdeal W x₁ (↑C y₁) = XIdeal W x₁
[PROOFSTEP]
have Y_rw :
(Y - C (C y₁)) * (Y - C (C (W.negY x₁ y₁))) -
C (X - C x₁) * (C (X ^ 2 + C (x₁ + W.a₂) * X + C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - C (C W.a₁) * Y) =
W.polynomial * 1 :=
by
linear_combination (norm := (rw [negY, WeierstrassCurve.polynomial]; C_simp; ring1))
congr_arg C (congr_arg C ((W.equation_iff _ _).mp h₁.left).symm)
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ (Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
[PROOFSTEP]
linear_combination (norm := (rw [negY, WeierstrassCurve.polynomial]; C_simp; ring1))
congr_arg C (congr_arg C ((W.equation_iff _ _).mp h₁.left).symm)
[GOAL]
case a
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ (Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) -
WeierstrassCurve.polynomial W * 1 -
(↑C (↑C (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆)) - ↑C (↑C (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁))) =
0
[PROOFSTEP]
rw [negY, WeierstrassCurve.polynomial]
[GOAL]
case a
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ (Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (-y₁ - W.a₁ * x₁ - W.a₃))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) -
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) * 1 -
(↑C (↑C (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆)) - ↑C (↑C (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁))) =
0
[PROOFSTEP]
C_simp
[GOAL]
case a
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ (Y - ↑C (↑C y₁)) * (Y - (-↑C (↑C y₁) - ↑C (↑C W.a₁) * ↑C (↑C x₁) - ↑C (↑C W.a₃))) -
(↑C Y - ↑C (↑C x₁)) *
(↑C Y ^ 2 + (↑C (↑C x₁) + ↑C (↑C W.a₂)) * ↑C Y +
(↑C (↑C x₁) ^ 2 + ↑C (↑C W.a₂) * ↑C (↑C x₁) + ↑C (↑C W.a₄)) -
↑C (↑C W.a₁) * Y) -
(Y ^ 2 + (↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)) * Y -
(↑C Y ^ 3 + ↑C (↑C W.a₂) * ↑C Y ^ 2 + ↑C (↑C W.a₄) * ↑C Y + ↑C (↑C W.a₆))) *
1 -
(↑C (↑C x₁) ^ 3 + ↑C (↑C W.a₂) * ↑C (↑C x₁) ^ 2 + ↑C (↑C W.a₄) * ↑C (↑C x₁) + ↑C (↑C W.a₆) -
(↑C (↑C y₁) ^ 2 + ↑C (↑C W.a₁) * ↑C (↑C x₁) * ↑C (↑C y₁) + ↑C (↑C W.a₃) * ↑C (↑C y₁))) =
0
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ XYIdeal W x₁ (↑C (negY W x₁ y₁)) * XYIdeal W x₁ (↑C y₁) = XIdeal W x₁
[PROOFSTEP]
simp_rw [XYIdeal, XClass, YClass, span_pair_mul_span_pair, mul_comm, ← _root_.map_mul,
AdjoinRoot.mk_eq_mk.mpr ⟨1, Y_rw⟩, _root_.map_mul, span_insert, ← span_singleton_mul_span_singleton, ← mul_sup, ←
span_insert]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ span {↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁))} *
span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁)), ↑(CoordinateRing.mk W) (Y - ↑C (↑C y₁)),
↑(CoordinateRing.mk W) (Y - ↑C (↑C (negY W x₁ y₁))),
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W))
(↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y)} =
XIdeal W x₁
[PROOFSTEP]
convert mul_top (_ : Ideal W.CoordinateRing) using 2
[GOAL]
case h.e'_2.h.e'_6
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ span
{↑(CoordinateRing.mk W) (↑C (Y - ↑C x₁)), ↑(CoordinateRing.mk W) (Y - ↑C (↑C y₁)),
↑(CoordinateRing.mk W) (Y - ↑C (↑C (negY W x₁ y₁))),
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W))
(↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y)} =
⊤
[PROOFSTEP]
simp_rw [← @Set.image_singleton _ _ <| CoordinateRing.mk W, ← Set.image_insert_eq, ← map_span]
[GOAL]
case h.e'_2.h.e'_6
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ Ideal.map (CoordinateRing.mk W)
(span
{↑C (Y - ↑C x₁), Y - ↑C (↑C y₁), Y - ↑C (↑C (negY W x₁ y₁)),
↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y}) =
⊤
[PROOFSTEP]
convert map_top (R := F[X][Y]) (CoordinateRing.mk W) using 1
[GOAL]
case h.e'_2
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ Ideal.map (CoordinateRing.mk W)
(span
{↑C (Y - ↑C x₁), Y - ↑C (↑C y₁), Y - ↑C (↑C (negY W x₁ y₁)),
↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y}) =
Ideal.map (CoordinateRing.mk W) ⊤
[PROOFSTEP]
apply congr_arg
[GOAL]
case h.e'_2.h
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ span
{↑C (Y - ↑C x₁), Y - ↑C (↑C y₁), Y - ↑C (↑C (negY W x₁ y₁)),
↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y} =
⊤
[PROOFSTEP]
simp_rw [eq_top_iff_one, mem_span_insert', mem_span_singleton']
[GOAL]
case h.e'_2.h
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
⊢ ∃ a a_1 a_2 a_3,
a_3 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + a * ↑C (Y - ↑C x₁) + a_1 * (Y - ↑C (↑C y₁)) + a_2 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
rcases((W.nonsingular_iff' _ _).mp h₁).right with hx | hy
[GOAL]
case h.e'_2.h.inl
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hx : W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄) ≠ 0
⊢ ∃ a a_1 a_2 a_3,
a_3 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + a * ↑C (Y - ↑C x₁) + a_1 * (Y - ↑C (↑C y₁)) + a_2 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
let W_X := W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄)
[GOAL]
case h.e'_2.h.inl
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hx : W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄) ≠ 0
W_X : F := W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄)
⊢ ∃ a a_1 a_2 a_3,
a_3 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + a * ↑C (Y - ↑C x₁) + a_1 * (Y - ↑C (↑C y₁)) + a_2 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
refine ⟨C (C W_X⁻¹ * -(X + C (2 * x₁ + W.a₂))), C (C <| W_X⁻¹ * W.a₁), 0, C (C <| W_X⁻¹ * -1), ?_⟩
[GOAL]
case h.e'_2.h.inl
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hx : W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄) ≠ 0
W_X : F := W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄)
⊢ ↑C (↑C (W_X⁻¹ * -1)) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + ↑C (↑C W_X⁻¹ * -(Y + ↑C (2 * x₁ + W.a₂))) * ↑C (Y - ↑C x₁) + ↑C (↑C (W_X⁻¹ * W.a₁)) * (Y - ↑C (↑C y₁)) +
0 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
rw [← mul_right_inj' <| C_ne_zero.mpr <| C_ne_zero.mpr hx]
[GOAL]
case h.e'_2.h.inl
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hx : W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄) ≠ 0
W_X : F := W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄)
⊢ ↑C (↑C (W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄))) *
(↑C (↑C (W_X⁻¹ * -1)) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y)) =
↑C (↑C (W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄))) *
(1 + ↑C (↑C W_X⁻¹ * -(Y + ↑C (2 * x₁ + W.a₂))) * ↑C (Y - ↑C x₁) + ↑C (↑C (W_X⁻¹ * W.a₁)) * (Y - ↑C (↑C y₁)) +
0 * (Y - ↑C (↑C (negY W x₁ y₁))))
[PROOFSTEP]
simp only [mul_add, ← mul_assoc, ← C_mul, mul_inv_cancel hx]
[GOAL]
case h.e'_2.h.inl
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hx : W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄) ≠ 0
W_X : F := W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄)
⊢ ↑C (↑C (1 * -1)) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
↑C (↑C (W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄))) * 1 +
↑C (↑C 1 * -(Y + ↑C (2 * x₁ + W.a₂)) * (Y - ↑C x₁)) +
↑C (↑C (1 * W.a₁)) * (Y - ↑C (↑C y₁)) +
↑C (↑C (W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄))) * 0 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
C_simp
[GOAL]
case h.e'_2.h.inl
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hx : W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄) ≠ 0
W_X : F := W.a₁ * y₁ - (3 * x₁ ^ 2 + 2 * W.a₂ * x₁ + W.a₄)
⊢ 1 * -1 *
(↑C Y ^ 2 + (↑C (↑C x₁) + ↑C (↑C W.a₂)) * ↑C Y + (↑C (↑C x₁) ^ 2 + ↑C (↑C W.a₂) * ↑C (↑C x₁) + ↑C (↑C W.a₄)) -
↑C (↑C W.a₁) * Y) =
(↑C (↑C W.a₁) * ↑C (↑C y₁) - (3 * ↑C (↑C x₁) ^ 2 + 2 * ↑C (↑C W.a₂) * ↑C (↑C x₁) + ↑C (↑C W.a₄))) * 1 +
1 * -(↑C Y + (2 * ↑C (↑C x₁) + ↑C (↑C W.a₂))) * (↑C Y - ↑C (↑C x₁)) +
1 * ↑C (↑C W.a₁) * (Y - ↑C (↑C y₁)) +
(↑C (↑C W.a₁) * ↑C (↑C y₁) - (3 * ↑C (↑C x₁) ^ 2 + 2 * ↑C (↑C W.a₂) * ↑C (↑C x₁) + ↑C (↑C W.a₄))) * 0 *
(Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
ring1
[GOAL]
case h.e'_2.h.inr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hy : 2 * y₁ + W.a₁ * x₁ + W.a₃ ≠ 0
⊢ ∃ a a_1 a_2 a_3,
a_3 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + a * ↑C (Y - ↑C x₁) + a_1 * (Y - ↑C (↑C y₁)) + a_2 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
let W_Y := 2 * y₁ + W.a₁ * x₁ + W.a₃
[GOAL]
case h.e'_2.h.inr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hy : 2 * y₁ + W.a₁ * x₁ + W.a₃ ≠ 0
W_Y : F := 2 * y₁ + W.a₁ * x₁ + W.a₃
⊢ ∃ a a_1 a_2 a_3,
a_3 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + a * ↑C (Y - ↑C x₁) + a_1 * (Y - ↑C (↑C y₁)) + a_2 * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
refine ⟨0, C (C W_Y⁻¹), C (C <| W_Y⁻¹ * -1), 0, ?_⟩
[GOAL]
case h.e'_2.h.inr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hy : 2 * y₁ + W.a₁ * x₁ + W.a₃ ≠ 0
W_Y : F := 2 * y₁ + W.a₁ * x₁ + W.a₃
⊢ 0 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
1 + 0 * ↑C (Y - ↑C x₁) + ↑C (↑C W_Y⁻¹) * (Y - ↑C (↑C y₁)) + ↑C (↑C (W_Y⁻¹ * -1)) * (Y - ↑C (↑C (negY W x₁ y₁)))
[PROOFSTEP]
rw [negY, ← mul_right_inj' <| C_ne_zero.mpr <| C_ne_zero.mpr hy]
[GOAL]
case h.e'_2.h.inr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hy : 2 * y₁ + W.a₁ * x₁ + W.a₃ ≠ 0
W_Y : F := 2 * y₁ + W.a₁ * x₁ + W.a₃
⊢ ↑C (↑C (2 * y₁ + W.a₁ * x₁ + W.a₃)) *
(0 * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y)) =
↑C (↑C (2 * y₁ + W.a₁ * x₁ + W.a₃)) *
(1 + 0 * ↑C (Y - ↑C x₁) + ↑C (↑C W_Y⁻¹) * (Y - ↑C (↑C y₁)) +
↑C (↑C (W_Y⁻¹ * -1)) * (Y - ↑C (↑C (-y₁ - W.a₁ * x₁ - W.a₃))))
[PROOFSTEP]
simp only [mul_add, ← mul_assoc, ← C_mul, mul_inv_cancel hy]
[GOAL]
case h.e'_2.h.inr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hy : 2 * y₁ + W.a₁ * x₁ + W.a₃ ≠ 0
W_Y : F := 2 * y₁ + W.a₁ * x₁ + W.a₃
⊢ ↑C (↑C (2 * y₁ + W.a₁ * x₁ + W.a₃)) * 0 *
(↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
↑C (↑C (2 * y₁ + W.a₁ * x₁ + W.a₃)) * 1 + ↑C (↑C (2 * y₁ + W.a₁ * x₁ + W.a₃)) * 0 * ↑C (Y - ↑C x₁) +
↑C (↑C 1) * (Y - ↑C (↑C y₁)) +
↑C (↑C (1 * -1)) * (Y - ↑C (↑C (-y₁ - W.a₁ * x₁ - W.a₃)))
[PROOFSTEP]
C_simp
[GOAL]
case h.e'_2.h.inr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
Y_rw :
(Y - ↑C (↑C y₁)) * (Y - ↑C (↑C (negY W x₁ y₁))) -
↑C (Y - ↑C x₁) * (↑C (Y ^ 2 + ↑C (x₁ + W.a₂) * Y + ↑C (x₁ ^ 2 + W.a₂ * x₁ + W.a₄)) - ↑C (↑C W.a₁) * Y) =
WeierstrassCurve.polynomial W * 1
hy : 2 * y₁ + W.a₁ * x₁ + W.a₃ ≠ 0
W_Y : F := 2 * y₁ + W.a₁ * x₁ + W.a₃
⊢ (2 * ↑C (↑C y₁) + ↑C (↑C W.a₁) * ↑C (↑C x₁) + ↑C (↑C W.a₃)) * 0 *
(↑C Y ^ 2 + (↑C (↑C x₁) + ↑C (↑C W.a₂)) * ↑C Y + (↑C (↑C x₁) ^ 2 + ↑C (↑C W.a₂) * ↑C (↑C x₁) + ↑C (↑C W.a₄)) -
↑C (↑C W.a₁) * Y) =
(2 * ↑C (↑C y₁) + ↑C (↑C W.a₁) * ↑C (↑C x₁) + ↑C (↑C W.a₃)) * 1 +
(2 * ↑C (↑C y₁) + ↑C (↑C W.a₁) * ↑C (↑C x₁) + ↑C (↑C W.a₃)) * 0 * (↑C Y - ↑C (↑C x₁)) +
1 * (Y - ↑C (↑C y₁)) +
1 * -1 * (Y - (-↑C (↑C y₁) - ↑C (↑C W.a₁) * ↑C (↑C x₁) - ↑C (↑C W.a₃)))
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ↑(XYIdeal W x₁ (↑C y₁)) * (↑(XYIdeal W x₁ (↑C (negY W x₁ y₁))) * (↑(XIdeal W x₁))⁻¹) = 1
[PROOFSTEP]
rw [← mul_assoc, ← FractionalIdeal.coeIdeal_mul, mul_comm <| XYIdeal W _ _, XYIdeal_neg_mul h₁, XIdeal,
FractionalIdeal.coe_ideal_span_singleton_mul_inv W.FunctionField <| XClass_ne_zero W x₁]
-- porting note: increased `maxHeartbeats` for `ring1`
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ XIdeal W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) * (XYIdeal W x₁ (↑C y₁) * XYIdeal W x₂ (↑C y₂)) =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
XYIdeal W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (↑C (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂)))
[PROOFSTEP]
clear h₂
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ XIdeal W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) * (XYIdeal W x₁ (↑C y₁) * XYIdeal W x₂ (↑C y₂)) =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
XYIdeal W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (↑C (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂)))
[PROOFSTEP]
have sup_rw : ∀ a b c d : Ideal W.CoordinateRing, a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c := fun _ _ c _ => by
rw [← sup_assoc, @sup_comm _ _ c, sup_sup_sup_comm, ← sup_assoc]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
x✝² x✝¹ c x✝ : Ideal (CoordinateRing W)
⊢ x✝² ⊔ (x✝¹ ⊔ (c ⊔ x✝)) = x✝² ⊔ x✝ ⊔ x✝¹ ⊔ c
[PROOFSTEP]
rw [← sup_assoc, @sup_comm _ _ c, sup_sup_sup_comm, ← sup_assoc]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ XIdeal W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) * (XYIdeal W x₁ (↑C y₁) * XYIdeal W x₂ (↑C y₂)) =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
XYIdeal W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (↑C (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂)))
[PROOFSTEP]
rw [XYIdeal_add_eq, XIdeal, mul_comm, W.XYIdeal_eq₁ x₁ y₁ <| W.slope x₁ x₂ y₁ y₂, XYIdeal, XYIdeal_eq₂ h₁' h₂' hxy,
XYIdeal, span_pair_mul_span_pair]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ span
{XClass W x₁ * XClass W x₂, XClass W x₁ * YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)),
YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) * XClass W x₂,
YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))} *
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))})
[PROOFSTEP]
simp_rw [span_insert, sup_rw, sup_mul, span_singleton_mul_span_singleton]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ span {XClass W x₁ * XClass W x₂ * XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span
{YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span
{XClass W x₁ * YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span
{YClass W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) * XClass W x₂ *
XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))})
[PROOFSTEP]
rw [← neg_eq_iff_eq_neg.mpr <| CoordinateRing.C_addPolynomial_slope h₁' h₂' hxy, span_singleton_neg,
CoordinateRing.C_addPolynomial, _root_.map_mul, YClass]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ span
{↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))) *
↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span
{↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))) *
↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))) *
XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span
{XClass W x₁ * ↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))) *
XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span
{↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂))) * XClass W x₂ *
XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))})
[PROOFSTEP]
simp_rw [mul_comm <| XClass W x₁, mul_assoc, ← span_singleton_mul_span_singleton, ← mul_sup]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ span {↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span {↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} *
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span {XClass W x₁} * span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} ⊔
span {XClass W x₂} * span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))}) =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))})
[PROOFSTEP]
rw [span_singleton_mul_span_singleton, ← span_insert, ←
span_pair_add_mul_right <| -(XClass W <| W.addX x₁ x₂ <| W.slope x₁ x₂ y₁ y₂), mul_neg, ← sub_eq_add_neg, ← sub_mul, ←
map_sub <| CoordinateRing.mk W, sub_sub_sub_cancel_right, span_insert, ← span_singleton_mul_span_singleton, ← sup_rw,
← sup_mul, ← sup_mul]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ span {↑(CoordinateRing.mk W) (Y - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
(span {XClass W x₁} ⊔ (span {XClass W x₂} ⊔ span {↑(CoordinateRing.mk W) (Y - negPolynomial W)})) *
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))}) =
YIdeal W (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)) *
(span {↑(CoordinateRing.mk W) (negPolynomial W - ↑C (linePolynomial x₁ y₁ (slope W x₁ x₂ y₁ y₂)))} ⊔
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))})
[PROOFSTEP]
apply congr_arg (_ ∘ _)
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ (span {XClass W x₁} ⊔ (span {XClass W x₂} ⊔ span {↑(CoordinateRing.mk W) (Y - negPolynomial W)})) *
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))} =
span {XClass W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂))}
[PROOFSTEP]
convert top_mul (_ : Ideal W.CoordinateRing)
[GOAL]
case h.e'_2.h.e'_5
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ span {XClass W x₁} ⊔ (span {XClass W x₂} ⊔ span {↑(CoordinateRing.mk W) (Y - negPolynomial W)}) = ⊤
[PROOFSTEP]
simp_rw [XClass, ← @Set.image_singleton _ _ <| CoordinateRing.mk W, ← map_span, ← Ideal.map_sup, eq_top_iff_one,
mem_map_iff_of_surjective _ <| AdjoinRoot.mk_surjective W.monic_polynomial, ← span_insert, mem_span_insert',
mem_span_singleton']
[GOAL]
case h.e'_2.h.e'_5
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₂)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : x₁ = x₂
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₂)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
rcases hx, Y_eq_of_Y_ne h₁' h₂' hx (hxy hx) with ⟨rfl, rfl⟩
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₁
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₁)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
let y := (y₁ - W.negY x₁ y₁) ^ 2
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
hxy : x₁ = x₁ → y₁ ≠ negY W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₁)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
replace hxy := pow_ne_zero 2 (sub_ne_zero_of_ne <| hxy rfl)
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₁)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
refine
⟨1 + C (C <| y⁻¹ * 4) * W.polynomial,
⟨C <| C y⁻¹ * (C 4 * X ^ 2 + C (4 * x₁ + W.b₂) * X + C (4 * x₁ ^ 2 + W.b₂ * x₁ + 2 * W.b₄)), 0,
C (C y⁻¹) * (Y - W.negPolynomial), ?_⟩,
by rw [map_add, map_one, _root_.map_mul <| CoordinateRing.mk W, AdjoinRoot.mk_self, mul_zero, add_zero]⟩
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) (1 + ↑C (↑C (y⁻¹ * 4)) * WeierstrassCurve.polynomial W) = 1
[PROOFSTEP]
rw [map_add, map_one, _root_.map_mul <| CoordinateRing.mk W, AdjoinRoot.mk_self, mul_zero, add_zero]
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ↑C (↑C y⁻¹) * (Y - negPolynomial W) * (Y - negPolynomial W) =
1 + ↑C (↑C (y⁻¹ * 4)) * WeierstrassCurve.polynomial W +
↑C (↑C y⁻¹ * (↑C 4 * Y ^ 2 + ↑C (4 * x₁ + b₂ W) * Y + ↑C (4 * x₁ ^ 2 + b₂ W * x₁ + 2 * b₄ W))) *
↑C (Y - ↑C x₁) +
0 * ↑C (Y - ↑C x₁)
[PROOFSTEP]
rw [WeierstrassCurve.polynomial, negPolynomial, ← mul_right_inj' <| C_ne_zero.mpr <| C_ne_zero.mpr hxy]
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ↑C (↑C ((y₁ - negY W x₁ y₁) ^ 2)) *
(↑C (↑C y⁻¹) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃)))) =
↑C (↑C ((y₁ - negY W x₁ y₁) ^ 2)) *
(1 +
↑C (↑C (y⁻¹ * 4)) *
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) +
↑C (↑C y⁻¹ * (↑C 4 * Y ^ 2 + ↑C (4 * x₁ + b₂ W) * Y + ↑C (4 * x₁ ^ 2 + b₂ W * x₁ + 2 * b₄ W))) *
↑C (Y - ↑C x₁) +
0 * ↑C (Y - ↑C x₁))
[PROOFSTEP]
simp only [mul_add, ← mul_assoc, ← C_mul, mul_inv_cancel hxy]
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ↑C (↑C 1) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) =
↑C (↑C ((y₁ - negY W x₁ y₁) ^ 2)) * 1 +
↑C (↑C (1 * 4)) *
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) +
↑C
((↑C (1 * 4) * Y ^ 2 + ↑C (1 * 4 * x₁ + 1 * b₂ W) * Y + ↑C (1 * 4 * x₁ ^ 2 + 1 * b₂ W * x₁ + 1 * 2 * b₄ W)) *
(Y - ↑C x₁)) +
↑C (↑C ((y₁ - negY W x₁ y₁) ^ 2)) * 0 * ↑C (Y - ↑C x₁)
[PROOFSTEP]
linear_combination (norm := (rw [b₂, b₄, negY]; C_simp; ring1))
-4 * congr_arg C (congr_arg C <| (W.equation_iff _ _).mp h₁')
[GOAL]
case a
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ↑C (↑C 1) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) -
(↑C (↑C ((y₁ - negY W x₁ y₁) ^ 2)) * 1 +
↑C (↑C (1 * 4)) *
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) +
↑C
((↑C (1 * 4) * Y ^ 2 + ↑C (1 * 4 * x₁ + 1 * b₂ W) * Y +
↑C (1 * 4 * x₁ ^ 2 + 1 * b₂ W * x₁ + 1 * 2 * b₄ W)) *
(Y - ↑C x₁)) +
↑C (↑C ((y₁ - negY W x₁ y₁) ^ 2)) * 0 * ↑C (Y - ↑C x₁)) -
(-4 * ↑C (↑C (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁)) - -4 * ↑C (↑C (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆))) =
0
[PROOFSTEP]
rw [b₂, b₄, negY]
[GOAL]
case a
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ ↑C (↑C 1) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) * (Y - (-Y - ↑C (↑C W.a₁ * Y + ↑C W.a₃))) -
(↑C (↑C ((y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2)) * 1 +
↑C (↑C (1 * 4)) *
(Y ^ 2 + ↑C (↑C W.a₁ * Y + ↑C W.a₃) * Y - ↑C (Y ^ 3 + ↑C W.a₂ * Y ^ 2 + ↑C W.a₄ * Y + ↑C W.a₆)) +
↑C
((↑C (1 * 4) * Y ^ 2 + ↑C (1 * 4 * x₁ + 1 * (W.a₁ ^ 2 + 4 * W.a₂)) * Y +
↑C (1 * 4 * x₁ ^ 2 + 1 * (W.a₁ ^ 2 + 4 * W.a₂) * x₁ + 1 * 2 * (2 * W.a₄ + W.a₁ * W.a₃))) *
(Y - ↑C x₁)) +
↑C (↑C ((y₁ - (-y₁ - W.a₁ * x₁ - W.a₃)) ^ 2)) * 0 * ↑C (Y - ↑C x₁)) -
(-4 * ↑C (↑C (y₁ ^ 2 + W.a₁ * x₁ * y₁ + W.a₃ * y₁)) - -4 * ↑C (↑C (x₁ ^ 3 + W.a₂ * x₁ ^ 2 + W.a₄ * x₁ + W.a₆))) =
0
[PROOFSTEP]
C_simp
[GOAL]
case a
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
h₂' : WeierstrassCurve.equation W x₁ y₁
y : F := (y₁ - negY W x₁ y₁) ^ 2
hxy : (y₁ - negY W x₁ y₁) ^ 2 ≠ 0
⊢ 1 * (Y - (-Y - (↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)))) * (Y - (-Y - (↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)))) -
((↑C (↑C y₁) - (-↑C (↑C y₁) - ↑C (↑C W.a₁) * ↑C (↑C x₁) - ↑C (↑C W.a₃))) ^ 2 * 1 +
1 * 4 *
(Y ^ 2 + (↑C (↑C W.a₁) * ↑C Y + ↑C (↑C W.a₃)) * Y -
(↑C Y ^ 3 + ↑C (↑C W.a₂) * ↑C Y ^ 2 + ↑C (↑C W.a₄) * ↑C Y + ↑C (↑C W.a₆))) +
(1 * 4 * ↑C Y ^ 2 + (1 * 4 * ↑C (↑C x₁) + 1 * (↑C (↑C W.a₁) ^ 2 + 4 * ↑C (↑C W.a₂))) * ↑C Y +
(1 * 4 * ↑C (↑C x₁) ^ 2 + 1 * (↑C (↑C W.a₁) ^ 2 + 4 * ↑C (↑C W.a₂)) * ↑C (↑C x₁) +
1 * 2 * (2 * ↑C (↑C W.a₄) + ↑C (↑C W.a₁) * ↑C (↑C W.a₃)))) *
(↑C Y - ↑C (↑C x₁)) +
(↑C (↑C y₁) - (-↑C (↑C y₁) - ↑C (↑C W.a₁) * ↑C (↑C x₁) - ↑C (↑C W.a₃))) ^ 2 * 0 * (↑C Y - ↑C (↑C x₁))) -
(-4 * (↑C (↑C y₁) ^ 2 + ↑C (↑C W.a₁) * ↑C (↑C x₁) * ↑C (↑C y₁) + ↑C (↑C W.a₃) * ↑C (↑C y₁)) -
-4 * (↑C (↑C x₁) ^ 3 + ↑C (↑C W.a₂) * ↑C (↑C x₁) ^ 2 + ↑C (↑C W.a₄) * ↑C (↑C x₁) + ↑C (↑C W.a₆))) =
0
[PROOFSTEP]
ring1
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : ¬x₁ = x₂
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₂)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
replace hx := sub_ne_zero_of_ne hx
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : x₁ - x₂ ≠ 0
⊢ ∃ x,
(∃ a a_1 a_2, a_2 * (Y - negPolynomial W) = x + a * ↑C (Y - ↑C x₁) + a_1 * ↑C (Y - ↑C x₂)) ∧
↑(AdjoinRoot.mk (WeierstrassCurve.polynomial W)) x = 1
[PROOFSTEP]
refine ⟨_, ⟨⟨C <| C (x₁ - x₂)⁻¹, C <| C <| (x₁ - x₂)⁻¹ * -1, 0, ?_⟩, map_one _⟩⟩
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : x₁ - x₂ ≠ 0
⊢ 0 * (Y - negPolynomial W) = 1 + ↑C (↑C (x₁ - x₂)⁻¹) * ↑C (Y - ↑C x₁) + ↑C (↑C ((x₁ - x₂)⁻¹ * -1)) * ↑C (Y - ↑C x₂)
[PROOFSTEP]
rw [← mul_right_inj' <| C_ne_zero.mpr <| C_ne_zero.mpr hx]
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : x₁ - x₂ ≠ 0
⊢ ↑C (↑C (x₁ - x₂)) * (0 * (Y - negPolynomial W)) =
↑C (↑C (x₁ - x₂)) * (1 + ↑C (↑C (x₁ - x₂)⁻¹) * ↑C (Y - ↑C x₁) + ↑C (↑C ((x₁ - x₂)⁻¹ * -1)) * ↑C (Y - ↑C x₂))
[PROOFSTEP]
simp only [← mul_assoc, mul_add, ← C_mul, mul_inv_cancel hx]
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : x₁ - x₂ ≠ 0
⊢ ↑C (↑C (x₁ - x₂)) * 0 * (Y - negPolynomial W) =
↑C (↑C (x₁ - x₂)) * 1 + ↑C (↑C 1 * (Y - ↑C x₁)) + ↑C (↑C (1 * -1) * (Y - ↑C x₂))
[PROOFSTEP]
C_simp
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
sup_rw : ∀ (a b c d : Ideal (CoordinateRing W)), a ⊔ (b ⊔ (c ⊔ d)) = a ⊔ d ⊔ b ⊔ c
hx : x₁ - x₂ ≠ 0
⊢ (↑C (↑C x₁) - ↑C (↑C x₂)) * 0 * (Y - negPolynomial W) =
(↑C (↑C x₁) - ↑C (↑C x₂)) * 1 + 1 * (↑C Y - ↑C (↑C x₁)) + 1 * -1 * (↑C Y - ↑C (↑C x₂))
[PROOFSTEP]
ring1
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ↑ClassGroup.mk (XYIdeal' (_ : WeierstrassCurve.nonsingular W x₁ (negY W x₁ y₁))) * ↑ClassGroup.mk (XYIdeal' h₁) = 1
[PROOFSTEP]
rw [← _root_.map_mul]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ↑ClassGroup.mk (XYIdeal' (_ : WeierstrassCurve.nonsingular W x₁ (negY W x₁ y₁)) * XYIdeal' h₁) = 1
[PROOFSTEP]
exact
(ClassGroup.mk_eq_one_of_coe_ideal <| by
exact
(FractionalIdeal.coeIdeal_mul _ _).symm.trans <| FractionalIdeal.coeIdeal_inj.mpr <| XYIdeal_neg_mul h₁).mpr
⟨_, XClass_ne_zero W _, rfl⟩
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ↑(XYIdeal' (_ : WeierstrassCurve.nonsingular W x₁ (negY W x₁ y₁)) * XYIdeal' h₁) = ↑(span {XClass W ?m.4456306})
[PROOFSTEP]
exact (FractionalIdeal.coeIdeal_mul _ _).symm.trans <| FractionalIdeal.coeIdeal_inj.mpr <| XYIdeal_neg_mul h₁
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑ClassGroup.mk (XYIdeal' h₁) * ↑ClassGroup.mk (XYIdeal' h₂) =
↑ClassGroup.mk
(XYIdeal'
(_ :
WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
rw [← _root_.map_mul]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑ClassGroup.mk (XYIdeal' h₁ * XYIdeal' h₂) =
↑ClassGroup.mk
(XYIdeal'
(_ :
WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))))
[PROOFSTEP]
exact
(ClassGroup.mk_eq_mk_of_coe_ideal (by exact (FractionalIdeal.coeIdeal_mul _ _).symm) <| XYIdeal'_eq _).mpr
⟨_, _, XClass_ne_zero W _, YClass_ne_zero W _, XYIdeal_mul_XYIdeal h₁.left h₂.left hxy⟩
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hxy : x₁ = x₂ → y₁ ≠ negY W x₂ y₂
⊢ ↑(XYIdeal' h₁ * XYIdeal' h₂) = ↑(XYIdeal W x₁ (↑C y₁) * XYIdeal W x₂ (↑C y₂))
[PROOFSTEP]
exact (FractionalIdeal.coeIdeal_mul _ _).symm
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ∀ (x y : Point W),
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (x + y) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } x +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } y
[PROOFSTEP]
rintro (_ | @⟨x₁, y₁, h₁⟩) (_ | @⟨x₂, y₂, h₂⟩)
[GOAL]
case zero.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (zero + zero) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero
case zero.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂✝ y₁ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (zero + some h₂) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₂)
case some.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂ y₁✝ y₂ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂ y₂
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁ + zero) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁) +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁ + some h₂) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁) +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₂)
[PROOFSTEP]
any_goals simp only [zero_def, toClassFun, _root_.zero_add, _root_.add_zero]
[GOAL]
case zero.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (zero + zero) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero
[PROOFSTEP]
simp only [zero_def, toClassFun, _root_.zero_add, _root_.add_zero]
[GOAL]
case zero.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂✝ y₁ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (zero + some h₂) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₂)
[PROOFSTEP]
simp only [zero_def, toClassFun, _root_.zero_add, _root_.add_zero]
[GOAL]
case some.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂ y₁✝ y₂ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂ y₂
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁ + zero) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁) +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } zero
[PROOFSTEP]
simp only [zero_def, toClassFun, _root_.zero_add, _root_.add_zero]
[GOAL]
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁ + some h₂) =
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₁) +
ZeroHom.toFun { toFun := toClassFun, map_zero' := (_ : toClassFun 0 = toClassFun 0) } (some h₂)
[PROOFSTEP]
simp only [zero_def, toClassFun, _root_.zero_add, _root_.add_zero]
[GOAL]
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ (match some h₁ + some h₂ with
| zero => 0
| some h => ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h))) =
↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₁)) + ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₂))
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
hx : x₁ = x₂
⊢ (match some h₁ + some h₂ with
| zero => 0
| some h => ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h))) =
↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₁)) + ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₂))
[PROOFSTEP]
by_cases hy : y₁ = W.negY x₂ y₂
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY W x₂ y₂
⊢ (match some h₁ + some h₂ with
| zero => 0
| some h => ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h))) =
↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₁)) + ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₂))
[PROOFSTEP]
substs hx hy
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂ y₁ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁
h₂✝ : WeierstrassCurve.nonsingular W x₂ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂✝
x₁ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₁ y₂
h₁ : WeierstrassCurve.nonsingular W x₁ (negY W x₁ y₂)
⊢ (match some h₁ + some h₂ with
| zero => 0
| some h => ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h))) =
↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₁)) + ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₂))
[PROOFSTEP]
simpa only [some_add_some_of_Y_eq rfl rfl] using (mk_XYIdeal'_mul_mk_XYIdeal'_of_Y_eq h₂).symm
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ (match some h₁ + some h₂ with
| zero => 0
| some h => ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h))) =
↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₁)) + ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₂))
[PROOFSTEP]
simpa only [some_add_some_of_Y_ne hx hy] using (mk_XYIdeal'_mul_mk_XYIdeal' h₁ h₂ fun _ => hy).symm
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁✝ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂✝ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
hx : ¬x₁ = x₂
⊢ (match some h₁ + some h₂ with
| zero => 0
| some h => ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h))) =
↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₁)) + ↑Additive.ofMul (↑ClassGroup.mk (XYIdeal' h₂))
[PROOFSTEP]
simpa only [some_add_some_of_X_ne hx] using (mk_XYIdeal'_mul_mk_XYIdeal' h₁ h₂ fun h => (hx h).elim).symm
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P Q : Point W
⊢ P + Q = 0 ↔ P = -Q
[PROOFSTEP]
rcases P, Q with ⟨_ | @⟨x₁, y₁, _⟩, _ | @⟨x₂, y₂, _⟩⟩
[GOAL]
case zero.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ zero + zero = 0 ↔ zero = -zero
case zero.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂✝ y₁ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ zero + some h✝ = 0 ↔ zero = -some h✝
case some.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂ y₁✝ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂ y₂
x₁ y₁ : F
h✝ : WeierstrassCurve.nonsingular W x₁ y₁
⊢ some h✝ + zero = 0 ↔ some h✝ = -zero
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ some h✝¹ + some h✝ = 0 ↔ some h✝¹ = -some h✝
[PROOFSTEP]
any_goals rfl
[GOAL]
case zero.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ zero + zero = 0 ↔ zero = -zero
[PROOFSTEP]
rfl
[GOAL]
case zero.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂✝ y₁ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ zero + some h✝ = 0 ↔ zero = -some h✝
[PROOFSTEP]
rfl
[GOAL]
case some.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂ y₁✝ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂ y₂
x₁ y₁ : F
h✝ : WeierstrassCurve.nonsingular W x₁ y₁
⊢ some h✝ + zero = 0 ↔ some h✝ = -zero
[PROOFSTEP]
rfl
[GOAL]
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ some h✝¹ + some h✝ = 0 ↔ some h✝¹ = -some h✝
[PROOFSTEP]
rfl
[GOAL]
case zero.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂✝ y₁ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ zero + some h✝ = 0 ↔ zero = -some h✝
[PROOFSTEP]
rw [zero_def, zero_add, ← neg_eq_iff_eq_neg, neg_zero, eq_comm]
[GOAL]
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ some h✝¹ + some h✝ = 0 ↔ some h✝¹ = -some h✝
[PROOFSTEP]
rw [neg_some, some.injEq]
[GOAL]
case some.some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ some h✝¹ + some h✝ = 0 ↔ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
constructor
[GOAL]
case some.some.mp
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ some h✝¹ + some h✝ = 0 → x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
intro h
[GOAL]
case some.some.mp
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
h : some h✝¹ + some h✝ = 0
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
h : some h✝¹ + some h✝ = 0
hx : x₁ = x₂
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
by_cases hy : y₁ = W.negY x₂ y₂
[GOAL]
case pos
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
h : some h✝¹ + some h✝ = 0
hx : x₁ = x₂
hy : y₁ = negY W x₂ y₂
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
exact ⟨hx, hy⟩
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
h : some h✝¹ + some h✝ = 0
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
rw [some_add_some_of_Y_ne hx hy] at h
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY W x₂ y₂
h :
some
(_ :
WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))) =
0
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
contradiction
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
h : some h✝¹ + some h✝ = 0
hx : ¬x₁ = x₂
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
rw [some_add_some_of_X_ne hx] at h
[GOAL]
case neg
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
hx : ¬x₁ = x₂
h :
some
(_ :
WeierstrassCurve.nonsingular W (addX W x₁ x₂ (slope W x₁ x₂ y₁ y₂)) (addY W x₁ x₂ y₁ (slope W x₁ x₂ y₁ y₂))) =
0
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂
[PROOFSTEP]
contradiction
[GOAL]
case some.some.mpr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁✝ x₂✝ y₁✝ y₂✝ : F
h₁ : WeierstrassCurve.nonsingular W x₁✝ y₁✝
h₂ : WeierstrassCurve.nonsingular W x₂✝ y₂✝
h₁' : WeierstrassCurve.equation W x₁✝ y₁✝
h₂' : WeierstrassCurve.equation W x₂✝ y₂✝
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular W x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular W x₂ y₂
⊢ x₁ = x₂ ∧ y₁ = negY W x₂ y₂ → some h✝¹ + some h✝ = 0
[PROOFSTEP]
exact fun ⟨hx, hy⟩ => some_add_some_of_Y_eq hx hy
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P : Point W
⊢ -P + P = 0
[PROOFSTEP]
rw [add_eq_zero]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P Q : Point W
⊢ -P + Q = 0 ↔ P = Q
[PROOFSTEP]
rw [add_eq_zero, neg_inj]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P : Point W
⊢ ↑toClass P = 0 ↔ P = 0
[PROOFSTEP]
constructor
[GOAL]
case mp
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P : Point W
⊢ ↑toClass P = 0 → P = 0
[PROOFSTEP]
intro hP
[GOAL]
case mp
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P : Point W
hP : ↑toClass P = 0
⊢ P = 0
[PROOFSTEP]
rcases P with (_ | @⟨_, _, ⟨h, _⟩⟩)
[GOAL]
case mp.zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
hP : ↑toClass zero = 0
⊢ zero = 0
[PROOFSTEP]
rfl
[GOAL]
case mp.some.intro
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.equation W x✝ y✝
right✝ :
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0
hP :
↑toClass
(some
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0))) =
0
⊢ some
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0)) =
0
[PROOFSTEP]
rcases(ClassGroup.mk_eq_one_of_coe_ideal <| by rfl).mp hP with ⟨p, h0, hp⟩
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.equation W x✝ y✝
right✝ :
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0
hP :
↑toClass
(some
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0))) =
0
⊢ ↑(XYIdeal'
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0))) =
↑?m.4705169
[PROOFSTEP]
rfl
[GOAL]
case mp.some.intro.intro.intro
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.equation W x✝ y✝
right✝ :
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0
hP :
↑toClass
(some
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0))) =
0
p : CoordinateRing W
h0 : p ≠ 0
hp : XYIdeal W x✝ (↑C y✝) = span {p}
⊢ some
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0)) =
0
[PROOFSTEP]
apply (p.natDegree_norm_ne_one _).elim
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.equation W x✝ y✝
right✝ :
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0
hP :
↑toClass
(some
(_ :
WeierstrassCurve.equation W x✝ y✝ ∧
(eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialX W)) ≠ 0 ∨
eval x✝ (eval (↑C y✝) (WeierstrassCurve.polynomialY W)) ≠ 0))) =
0
p : CoordinateRing W
h0 : p ≠ 0
hp : XYIdeal W x✝ (↑C y✝) = span {p}
⊢ natDegree (↑(Algebra.norm F[X]) p) = 1
[PROOFSTEP]
rw [← finrank_quotient_span_eq_natDegree_norm (CoordinateRing.basis W) h0, ←
(quotientEquivAlgOfEq F hp).toLinearEquiv.finrank_eq, (quotientXYIdealEquiv W h).toLinearEquiv.finrank_eq,
FiniteDimensional.finrank_self]
[GOAL]
case mpr
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P : Point W
⊢ P = 0 → ↑toClass P = 0
[PROOFSTEP]
exact congr_arg toClass
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
⊢ Function.Injective ↑toClass
[PROOFSTEP]
rintro (_ | h) _ hP
[GOAL]
case zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
a₂✝ : Point W
hP : ↑toClass zero = ↑toClass a₂✝
⊢ zero = a₂✝
case some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.nonsingular W x✝ y✝
a₂✝ : Point W
hP : ↑toClass (some h) = ↑toClass a₂✝
⊢ some h = a₂✝
[PROOFSTEP]
all_goals rw [← neg_add_eq_zero, ← toClass_eq_zero, map_add, ← hP]
[GOAL]
case zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
a₂✝ : Point W
hP : ↑toClass zero = ↑toClass a₂✝
⊢ zero = a₂✝
[PROOFSTEP]
rw [← neg_add_eq_zero, ← toClass_eq_zero, map_add, ← hP]
[GOAL]
case some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.nonsingular W x✝ y✝
a₂✝ : Point W
hP : ↑toClass (some h) = ↑toClass a₂✝
⊢ some h = a₂✝
[PROOFSTEP]
rw [← neg_add_eq_zero, ← toClass_eq_zero, map_add, ← hP]
[GOAL]
case zero
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
a₂✝ : Point W
hP : ↑toClass zero = ↑toClass a₂✝
⊢ ↑toClass (-zero) + ↑toClass zero = 0
[PROOFSTEP]
exact zero_add 0
[GOAL]
case some
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
x✝ y✝ : F
h : WeierstrassCurve.nonsingular W x✝ y✝
a₂✝ : Point W
hP : ↑toClass (some h) = ↑toClass a₂✝
⊢ ↑toClass (-some h) + ↑toClass (some h) = 0
[PROOFSTEP]
exact mk_XYIdeal'_mul_mk_XYIdeal'_of_Y_eq h
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P Q : Point W
⊢ ↑toClass (P + Q) = ↑toClass (Q + P)
[PROOFSTEP]
simp only [map_add, _root_.add_comm]
[GOAL]
F : Type u
inst✝ : Field F
W : WeierstrassCurve F
x₁ x₂ y₁ y₂ : F
h₁ : WeierstrassCurve.nonsingular W x₁ y₁
h₂ : WeierstrassCurve.nonsingular W x₂ y₂
h₁' : WeierstrassCurve.equation W x₁ y₁
h₂' : WeierstrassCurve.equation W x₂ y₂
P Q R : Point W
⊢ ↑toClass (P + Q + R) = ↑toClass (P + (Q + R))
[PROOFSTEP]
simp only [map_add, _root_.add_assoc]
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
⊢ ∀ (x y : W⟮F⟯),
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(x + y) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } x +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } y
[PROOFSTEP]
rintro (_ | @⟨x₁, y₁, _⟩) (_ | @⟨x₂, y₂, _⟩)
[GOAL]
case zero.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(zero + zero) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero
case zero.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(zero + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
case some.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝ + zero) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
any_goals rfl
[GOAL]
case zero.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(zero + zero) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero
[PROOFSTEP]
rfl
[GOAL]
case zero.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(zero + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
rfl
[GOAL]
case some.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝ + zero) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) } zero
[PROOFSTEP]
rfl
[GOAL]
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
rfl
[GOAL]
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
by_cases hx : x₁ = x₂
[GOAL]
case pos
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
by_cases hy : y₁ = (W.baseChange F).negY x₂ y₂
[GOAL]
case pos
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
simp only [some_add_some_of_Y_eq hx hy, ofBaseChangeFun]
[GOAL]
case pos
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY (baseChange W F) x₂ y₂
⊢ 0 =
some (_ : WeierstrassCurve.nonsingular (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) y₁)) +
some (_ : WeierstrassCurve.nonsingular (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂))
[PROOFSTEP]
rw [some_add_some_of_Y_eq <| congr_arg _ hx]
[GOAL]
case pos
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : y₁ = negY (baseChange W F) x₂ y₂
⊢ ↑(algebraMap F K) y₁ = negY (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂)
[PROOFSTEP]
rw [hy, baseChange_negY_of_baseChange]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY (baseChange W F) x₂ y₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
simp only [some_add_some_of_Y_ne hx hy, ofBaseChangeFun]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY (baseChange W F) x₂ y₂
⊢ some
(_ :
WeierstrassCurve.nonsingular (baseChange W K)
(↑(algebraMap F K) (addX (baseChange W F) x₁ x₂ (slope (baseChange W F) x₁ x₂ y₁ y₂)))
(↑(algebraMap F K) (addY (baseChange W F) x₁ x₂ y₁ (slope (baseChange W F) x₁ x₂ y₁ y₂)))) =
some (_ : WeierstrassCurve.nonsingular (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) y₁)) +
some (_ : WeierstrassCurve.nonsingular (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂))
[PROOFSTEP]
rw [some_add_some_of_Y_ne <| congr_arg _ hx]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY (baseChange W F) x₂ y₂
⊢ some
(_ :
WeierstrassCurve.nonsingular (baseChange W K)
(↑(algebraMap F K) (addX (baseChange W F) x₁ x₂ (slope (baseChange W F) x₁ x₂ y₁ y₂)))
(↑(algebraMap F K) (addY (baseChange W F) x₁ x₂ y₁ (slope (baseChange W F) x₁ x₂ y₁ y₂)))) =
some
(_ :
WeierstrassCurve.nonsingular (baseChange W K)
(addX (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂)
(slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁)
(↑(algebraMap F K) y₂)))
(addY (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁)
(slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁)
(↑(algebraMap F K) y₂))))
[PROOFSTEP]
simp only [baseChange_addX_of_baseChange, baseChange_addY_of_baseChange, baseChange_slope_of_baseChange]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY (baseChange W F) x₂ y₂
⊢ ↑(algebraMap F K) y₁ ≠ negY (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂)
[PROOFSTEP]
rw [baseChange_negY_of_baseChange]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : ¬y₁ = negY (baseChange W F) x₂ y₂
⊢ ↑(algebraMap F K) y₁ ≠ ↑(algebraMap F K) (negY (baseChange W F) x₂ y₂)
[PROOFSTEP]
contrapose! hy
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : x₁ = x₂
hy : ↑(algebraMap F K) y₁ = ↑(algebraMap F K) (negY (baseChange W F) x₂ y₂)
⊢ y₁ = negY (baseChange W F) x₂ y₂
[PROOFSTEP]
exact NoZeroSMulDivisors.algebraMap_injective F K hy
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : ¬x₁ = x₂
⊢ ZeroHom.toFun { toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹ + some h✝) =
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝¹) +
ZeroHom.toFun
{ toFun := ofBaseChangeFun W F K, map_zero' := (_ : ofBaseChangeFun W F K 0 = ofBaseChangeFun W F K 0) }
(some h✝)
[PROOFSTEP]
simp only [some_add_some_of_X_ne hx, ofBaseChangeFun]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : ¬x₁ = x₂
⊢ some
(_ :
WeierstrassCurve.nonsingular (baseChange W K)
(↑(algebraMap F K) (addX (baseChange W F) x₁ x₂ (slope (baseChange W F) x₁ x₂ y₁ y₂)))
(↑(algebraMap F K) (addY (baseChange W F) x₁ x₂ y₁ (slope (baseChange W F) x₁ x₂ y₁ y₂)))) =
some (_ : WeierstrassCurve.nonsingular (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) y₁)) +
some (_ : WeierstrassCurve.nonsingular (baseChange W K) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₂))
[PROOFSTEP]
rw [some_add_some_of_X_ne]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : ¬x₁ = x₂
⊢ some
(_ :
WeierstrassCurve.nonsingular (baseChange W K)
(↑(algebraMap F K) (addX (baseChange W F) x₁ x₂ (slope (baseChange W F) x₁ x₂ y₁ y₂)))
(↑(algebraMap F K) (addY (baseChange W F) x₁ x₂ y₁ (slope (baseChange W F) x₁ x₂ y₁ y₂)))) =
some
(_ :
WeierstrassCurve.nonsingular (baseChange W K)
(addX (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂)
(slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁)
(↑(algebraMap F K) y₂)))
(addY (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁)
(slope (baseChange W K) (↑(algebraMap F K) x₁) (↑(algebraMap F K) x₂) (↑(algebraMap F K) y₁)
(↑(algebraMap F K) y₂))))
[PROOFSTEP]
simp only [baseChange_addX_of_baseChange, baseChange_addY_of_baseChange, baseChange_slope_of_baseChange]
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : ¬x₁ = x₂
⊢ ↑(algebraMap F K) x₁ ≠ ↑(algebraMap F K) x₂
[PROOFSTEP]
contrapose! hx
[GOAL]
case neg
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x₁ y₁ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x₁ y₁
x₂ y₂ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x₂ y₂
hx : ↑(algebraMap F K) x₁ = ↑(algebraMap F K) x₂
⊢ x₁ = x₂
[PROOFSTEP]
exact NoZeroSMulDivisors.algebraMap_injective F K hx
[GOAL]
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
⊢ Function.Injective ↑(ofBaseChange W F K)
[PROOFSTEP]
rintro (_ | _) (_ | _) h
[GOAL]
case zero.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
h : ↑(ofBaseChange W F K) zero = ↑(ofBaseChange W F K) zero
⊢ zero = zero
case zero.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) zero = ↑(ofBaseChange W F K) (some h✝)
⊢ zero = some h✝
case some.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) (some h✝) = ↑(ofBaseChange W F K) zero
⊢ some h✝ = zero
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝¹ y✝¹ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x✝¹ y✝¹
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) (some h✝¹) = ↑(ofBaseChange W F K) (some h✝)
⊢ some h✝¹ = some h✝
[PROOFSTEP]
any_goals contradiction
[GOAL]
case zero.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
h : ↑(ofBaseChange W F K) zero = ↑(ofBaseChange W F K) zero
⊢ zero = zero
[PROOFSTEP]
contradiction
[GOAL]
case zero.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) zero = ↑(ofBaseChange W F K) (some h✝)
⊢ zero = some h✝
[PROOFSTEP]
contradiction
[GOAL]
case some.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) (some h✝) = ↑(ofBaseChange W F K) zero
⊢ some h✝ = zero
[PROOFSTEP]
contradiction
[GOAL]
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝¹ y✝¹ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x✝¹ y✝¹
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) (some h✝¹) = ↑(ofBaseChange W F K) (some h✝)
⊢ some h✝¹ = some h✝
[PROOFSTEP]
contradiction
[GOAL]
case zero.zero
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
h : ↑(ofBaseChange W F K) zero = ↑(ofBaseChange W F K) zero
⊢ zero = zero
[PROOFSTEP]
rfl
[GOAL]
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝¹ y✝¹ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x✝¹ y✝¹
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) (some h✝¹) = ↑(ofBaseChange W F K) (some h✝)
⊢ some h✝¹ = some h✝
[PROOFSTEP]
rw [some.injEq]
[GOAL]
case some.some
R : Type u
inst✝⁶ : CommRing R
W : WeierstrassCurve R
F : Type v
inst✝⁵ : Field F
inst✝⁴ : Algebra R F
K : Type w
inst✝³ : Field K
inst✝² : Algebra R K
inst✝¹ : Algebra F K
inst✝ : IsScalarTower R F K
x✝¹ y✝¹ : F
h✝¹ : WeierstrassCurve.nonsingular (baseChange W F) x✝¹ y✝¹
x✝ y✝ : F
h✝ : WeierstrassCurve.nonsingular (baseChange W F) x✝ y✝
h : ↑(ofBaseChange W F K) (some h✝¹) = ↑(ofBaseChange W F K) (some h✝)
⊢ x✝¹ = x✝ ∧ y✝¹ = y✝
[PROOFSTEP]
exact
⟨NoZeroSMulDivisors.algebraMap_injective F K (some.inj h).left,
NoZeroSMulDivisors.algebraMap_injective F K (some.inj h).right⟩
| {"mathlib_filename": "Mathlib.AlgebraicGeometry.EllipticCurve.Point", "llama_tokens": 110355} |
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible (det A)
⊢ ⅟(det A) • adjugate A * A = 1
[PROOFSTEP]
rw [smul_mul_assoc, adjugate_mul, smul_smul, invOf_mul_self, one_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible (det A)
⊢ A * ⅟(det A) • adjugate A = 1
[PROOFSTEP]
rw [mul_smul_comm, mul_adjugate, smul_smul, invOf_mul_self, one_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : Invertible (det A)
inst✝ : Invertible A
⊢ ⅟A = ⅟(det A) • adjugate A
[PROOFSTEP]
letI := invertibleOfDetInvertible A
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : Invertible (det A)
inst✝ : Invertible A
this : Invertible A := invertibleOfDetInvertible A
⊢ ⅟A = ⅟(det A) • adjugate A
[PROOFSTEP]
convert (rfl : ⅟A = _)
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : B * A = 1
⊢ det B * det A = 1
[PROOFSTEP]
rw [← det_mul, h, det_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : B * A = 1
⊢ det A * det B = 1
[PROOFSTEP]
rw [mul_comm, ← det_mul, h, det_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : A * B = 1
⊢ det B * det A = 1
[PROOFSTEP]
rw [mul_comm, ← det_mul, h, det_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : A * B = 1
⊢ det A * det B = 1
[PROOFSTEP]
rw [← det_mul, h, det_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : Invertible A
inst✝ : Invertible (det A)
⊢ det ⅟A = ⅟(det A)
[PROOFSTEP]
letI := detInvertibleOfInvertible A
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : Invertible A
inst✝ : Invertible (det A)
this : Invertible (det A) := detInvertibleOfInvertible A
⊢ det ⅟A = ⅟(det A)
[PROOFSTEP]
convert (rfl : _ = ⅟A.det)
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
h : A * B = 1
⊢ B * A = 1
[PROOFSTEP]
letI : Invertible B.det := detInvertibleOfLeftInverse _ _ h
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
h : A * B = 1
this : Invertible (det B) := detInvertibleOfLeftInverse B A h
⊢ B * A = 1
[PROOFSTEP]
letI : Invertible B := invertibleOfDetInvertible B
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
h : A * B = 1
this✝ : Invertible (det B) := detInvertibleOfLeftInverse B A h
this : Invertible B := invertibleOfDetInvertible B
⊢ B * A = 1
[PROOFSTEP]
calc
B * A = B * A * (B * ⅟B) := by rw [mul_invOf_self, Matrix.mul_one]
_ = B * (A * B * ⅟B) := by simp only [Matrix.mul_assoc]
_ = B * ⅟B := by rw [h, Matrix.one_mul]
_ = 1 := mul_invOf_self B
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
h : A * B = 1
this✝ : Invertible (det B) := detInvertibleOfLeftInverse B A h
this : Invertible B := invertibleOfDetInvertible B
⊢ B * A = B * A * (B * ⅟B)
[PROOFSTEP]
rw [mul_invOf_self, Matrix.mul_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
h : A * B = 1
this✝ : Invertible (det B) := detInvertibleOfLeftInverse B A h
this : Invertible B := invertibleOfDetInvertible B
⊢ B * A * (B * ⅟B) = B * (A * B * ⅟B)
[PROOFSTEP]
simp only [Matrix.mul_assoc]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
h : A * B = 1
this✝ : Invertible (det B) := detInvertibleOfLeftInverse B A h
this : Invertible B := invertibleOfDetInvertible B
⊢ B * (A * B * ⅟B) = B * ⅟B
[PROOFSTEP]
rw [h, Matrix.one_mul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
⊢ Invertible (det Aᵀ)
[PROOFSTEP]
simpa using detInvertibleOfInvertible A
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible Aᵀ
⊢ Invertible A
[PROOFSTEP]
rw [← transpose_transpose A]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible Aᵀ
⊢ Invertible Aᵀᵀ
[PROOFSTEP]
infer_instance
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : StarRing α
inst✝ : Invertible Aᴴ
⊢ Invertible A
[PROOFSTEP]
rw [← conjTranspose_conjTranspose A, ← star_eq_conjTranspose]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : StarRing α
inst✝ : Invertible Aᴴ
⊢ Invertible (star Aᴴ)
[PROOFSTEP]
infer_instance
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ IsUnit A ↔ IsUnit (det A)
[PROOFSTEP]
simp only [← nonempty_invertible_iff_isUnit, (invertibleEquivDetInvertible A).nonempty_congr]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ IsUnit (det Aᵀ)
[PROOFSTEP]
rw [det_transpose]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ IsUnit (det A)
[PROOFSTEP]
exact h
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : ¬IsUnit (det A)
⊢ A⁻¹ = 0
[PROOFSTEP]
rw [inv_def, Ring.inverse_non_unit _ h, zero_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ A⁻¹ = ↑(IsUnit.unit h)⁻¹ • adjugate A
[PROOFSTEP]
rw [inv_def, ← Ring.inverse_unit h.unit, IsUnit.unit_spec]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
⊢ ⅟A = A⁻¹
[PROOFSTEP]
letI := detInvertibleOfInvertible A
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
this : Invertible (det A) := detInvertibleOfInvertible A
⊢ ⅟A = A⁻¹
[PROOFSTEP]
rw [inv_def, Ring.inverse_invertible, invOf_eq]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B : Matrix n n α
A : (Matrix n n α)ˣ
⊢ ↑A⁻¹ = (↑A)⁻¹
[PROOFSTEP]
letI := A.invertible
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B : Matrix n n α
A : (Matrix n n α)ˣ
this : Invertible ↑A := Units.invertible A
⊢ ↑A⁻¹ = (↑A)⁻¹
[PROOFSTEP]
rw [← invOf_eq_nonsing_inv, invOf_units]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ A⁻¹ = Ring.inverse A
[PROOFSTEP]
by_cases h_det : IsUnit A.det
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h_det : IsUnit (det A)
⊢ A⁻¹ = Ring.inverse A
[PROOFSTEP]
cases (A.isUnit_iff_isUnit_det.mpr h_det).nonempty_invertible
[GOAL]
case pos.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h_det : IsUnit (det A)
val✝ : Invertible A
⊢ A⁻¹ = Ring.inverse A
[PROOFSTEP]
rw [← invOf_eq_nonsing_inv, Ring.inverse_invertible]
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h_det : ¬IsUnit (det A)
⊢ A⁻¹ = Ring.inverse A
[PROOFSTEP]
have h := mt A.isUnit_iff_isUnit_det.mp h_det
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h_det : ¬IsUnit (det A)
h : ¬IsUnit A
⊢ A⁻¹ = Ring.inverse A
[PROOFSTEP]
rw [Ring.inverse_non_unit _ h, nonsing_inv_apply_not_isUnit A h_det]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ A⁻¹ᵀ = Aᵀ⁻¹
[PROOFSTEP]
rw [inv_def, inv_def, transpose_smul, det_transpose, adjugate_transpose]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : StarRing α
⊢ A⁻¹ᴴ = Aᴴ⁻¹
[PROOFSTEP]
rw [inv_def, inv_def, conjTranspose_smul, det_conjTranspose, adjugate_conjTranspose, Ring.inverse_star]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ A * A⁻¹ = 1
[PROOFSTEP]
cases (A.isUnit_iff_isUnit_det.mpr h).nonempty_invertible
[GOAL]
case intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
val✝ : Invertible A
⊢ A * A⁻¹ = 1
[PROOFSTEP]
rw [← invOf_eq_nonsing_inv, mul_invOf_self]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ A⁻¹ * A = 1
[PROOFSTEP]
cases (A.isUnit_iff_isUnit_det.mpr h).nonempty_invertible
[GOAL]
case intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
val✝ : Invertible A
⊢ A⁻¹ * A = 1
[PROOFSTEP]
rw [← invOf_eq_nonsing_inv, invOf_mul_self]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
⊢ Invertible A⁻¹
[PROOFSTEP]
rw [← invOf_eq_nonsing_inv]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
⊢ Invertible ⅟A
[PROOFSTEP]
infer_instance
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
⊢ A⁻¹⁻¹ = A
[PROOFSTEP]
simp only [← invOf_eq_nonsing_inv, invOf_invOf]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B✝ : Matrix n n α
B : Matrix m n α
h : IsUnit (det A)
⊢ B * A * A⁻¹ = B
[PROOFSTEP]
simp [Matrix.mul_assoc, mul_nonsing_inv A h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B✝ : Matrix n n α
B : Matrix n m α
h : IsUnit (det A)
⊢ A * (A⁻¹ * B) = B
[PROOFSTEP]
simp [← Matrix.mul_assoc, mul_nonsing_inv A h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B✝ : Matrix n n α
B : Matrix m n α
h : IsUnit (det A)
⊢ B * A⁻¹ * A = B
[PROOFSTEP]
simp [Matrix.mul_assoc, nonsing_inv_mul A h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B✝ : Matrix n n α
B : Matrix n m α
h : IsUnit (det A)
⊢ A⁻¹ * (A * B) = B
[PROOFSTEP]
simp [← Matrix.mul_assoc, nonsing_inv_mul A h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A✝ B✝ A B C : Matrix n n α
inst✝ : Invertible A
h : A⁻¹ * B = C
⊢ B = A * C
[PROOFSTEP]
rw [← h, mul_inv_cancel_left_of_invertible]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A✝ B✝ A B C : Matrix n n α
inst✝ : Invertible A
h : B = A * C
⊢ A⁻¹ * B = C
[PROOFSTEP]
rw [h, inv_mul_cancel_left_of_invertible]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A✝ B✝ A B C : Matrix n n α
inst✝ : Invertible A
h : B * A⁻¹ = C
⊢ B = C * A
[PROOFSTEP]
rw [← h, inv_mul_cancel_right_of_invertible]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A✝ B✝ A B C : Matrix n n α
inst✝ : Invertible A
h : B = C * A
⊢ B * A⁻¹ = C
[PROOFSTEP]
rw [h, mul_inv_cancel_right_of_invertible]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
x✝¹ x✝ : Matrix n m α
h : (fun x => A * x) x✝¹ = (fun x => A * x) x✝
⊢ x✝¹ = x✝
[PROOFSTEP]
simpa only [inv_mul_cancel_left_of_invertible] using congr_arg (A⁻¹ * ·) h
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible A
a x : Matrix m n α
hax : (fun x => x * A) a = (fun x => x * A) x
⊢ a = x
[PROOFSTEP]
simpa only [mul_inv_cancel_right_of_invertible] using congr_arg (· * A⁻¹) hax
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ A⁻¹ * A = 1 ∧ A * A⁻¹ = 1 ∨ A⁻¹ = 0
[PROOFSTEP]
by_cases h : IsUnit A.det
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ A⁻¹ * A = 1 ∧ A * A⁻¹ = 1 ∨ A⁻¹ = 0
[PROOFSTEP]
exact Or.inl ⟨nonsing_inv_mul _ h, mul_nonsing_inv _ h⟩
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : ¬IsUnit (det A)
⊢ A⁻¹ * A = 1 ∧ A * A⁻¹ = 1 ∨ A⁻¹ = 0
[PROOFSTEP]
exact Or.inr (nonsing_inv_apply_not_isUnit _ h)
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ det A⁻¹ * det A = 1
[PROOFSTEP]
rw [← det_mul, A.nonsing_inv_mul h, det_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
by_cases h : IsUnit A.det
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
cases h.nonempty_invertible
[GOAL]
case pos.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
val✝ : Invertible (det A)
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
letI := invertibleOfDetInvertible A
[GOAL]
case pos.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
val✝ : Invertible (det A)
this : Invertible A := invertibleOfDetInvertible A
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
rw [Ring.inverse_invertible, ← invOf_eq_nonsing_inv, det_invOf]
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : ¬IsUnit (det A)
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
cases isEmpty_or_nonempty n
[GOAL]
case neg.inl
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : ¬IsUnit (det A)
h✝ : IsEmpty n
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
rw [det_isEmpty, det_isEmpty, Ring.inverse_one]
[GOAL]
case neg.inr
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : ¬IsUnit (det A)
h✝ : Nonempty n
⊢ det A⁻¹ = Ring.inverse (det A)
[PROOFSTEP]
rw [Ring.inverse_non_unit _ h, nonsing_inv_apply_not_isUnit _ h, det_zero ‹_›]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ A⁻¹⁻¹ = 1 * A⁻¹⁻¹
[PROOFSTEP]
rw [Matrix.one_mul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ 1 * A⁻¹⁻¹ = A * A⁻¹ * A⁻¹⁻¹
[PROOFSTEP]
rw [A.mul_nonsing_inv h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
h : IsUnit (det A)
⊢ A * A⁻¹ * A⁻¹⁻¹ = A
[PROOFSTEP]
rw [Matrix.mul_assoc, A⁻¹.mul_nonsing_inv (A.isUnit_nonsing_inv_det h), Matrix.mul_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
⊢ IsUnit (det A⁻¹) ↔ IsUnit (det A)
[PROOFSTEP]
rw [Matrix.det_nonsing_inv, isUnit_ring_inverse]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible (det A)
⊢ unitOfDetInvertible A = nonsingInvUnit A (_ : IsUnit (det A))
[PROOFSTEP]
ext
[GOAL]
case a.a.h
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
inst✝ : Invertible (det A)
i✝ x✝ : n
⊢ ↑(unitOfDetInvertible A) i✝ x✝ = ↑(nonsingInvUnit A (_ : IsUnit (det A))) i✝ x✝
[PROOFSTEP]
rfl
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : B * A = 1
g : C * A = 1
⊢ B = C
[PROOFSTEP]
rw [← inv_eq_left_inv h, ← inv_eq_left_inv g]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : A * B = 1
g : A * C = 1
⊢ B = C
[PROOFSTEP]
rw [← inv_eq_right_inv h, ← inv_eq_right_inv g]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : A * B = 1
g : C * A = 1
⊢ B = C
[PROOFSTEP]
rw [← inv_eq_right_inv h, ← inv_eq_left_inv g]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : A⁻¹ = B⁻¹
h' : IsUnit (det A)
⊢ A = B
[PROOFSTEP]
refine' left_inv_eq_left_inv (mul_nonsing_inv _ h') _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : A⁻¹ = B⁻¹
h' : IsUnit (det A)
⊢ B * A⁻¹ = 1
[PROOFSTEP]
rw [h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : A⁻¹ = B⁻¹
h' : IsUnit (det A)
⊢ B * B⁻¹ = 1
[PROOFSTEP]
refine' mul_nonsing_inv _ _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B C : Matrix n n α
h : A⁻¹ = B⁻¹
h' : IsUnit (det A)
⊢ IsUnit (det B)
[PROOFSTEP]
rwa [← isUnit_nonsing_inv_det_iff, ← h, isUnit_nonsing_inv_det_iff]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ 0⁻¹ = 0
[PROOFSTEP]
cases' subsingleton_or_nontrivial α with ht ht
[GOAL]
case inl
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Subsingleton α
⊢ 0⁻¹ = 0
[PROOFSTEP]
simp
[GOAL]
case inr
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
⊢ 0⁻¹ = 0
[PROOFSTEP]
cases' (Fintype.card n).zero_le.eq_or_lt with hc hc
[GOAL]
case inr.inl
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc : 0 = Fintype.card n
⊢ 0⁻¹ = 0
[PROOFSTEP]
rw [eq_comm, Fintype.card_eq_zero_iff] at hc
[GOAL]
case inr.inl
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc : IsEmpty n
⊢ 0⁻¹ = 0
[PROOFSTEP]
haveI := hc
[GOAL]
case inr.inl
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc this : IsEmpty n
⊢ 0⁻¹ = 0
[PROOFSTEP]
ext i
[GOAL]
case inr.inl.a.h
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc this : IsEmpty n
i x✝ : n
⊢ 0⁻¹ i x✝ = OfNat.ofNat 0 i x✝
[PROOFSTEP]
exact (IsEmpty.false i).elim
[GOAL]
case inr.inr
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc : 0 < Fintype.card n
⊢ 0⁻¹ = 0
[PROOFSTEP]
have hn : Nonempty n := Fintype.card_pos_iff.mp hc
[GOAL]
case inr.inr
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc : 0 < Fintype.card n
hn : Nonempty n
⊢ 0⁻¹ = 0
[PROOFSTEP]
refine' nonsing_inv_apply_not_isUnit _ _
[GOAL]
case inr.inr
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
ht : Nontrivial α
hc : 0 < Fintype.card n
hn : Nonempty n
⊢ ¬IsUnit (det 0)
[PROOFSTEP]
simp [hn]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
src✝¹ : One (Matrix n n α) := one
src✝ : Inv (Matrix n n α) := inv
⊢ 1 * 1 = 1
[PROOFSTEP]
simp
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
k : α
inst✝ : Invertible k
h : IsUnit (det A)
⊢ ⅟k • A⁻¹ * k • A = 1
[PROOFSTEP]
simp [h, smul_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
k : αˣ
h : IsUnit (det A)
⊢ k⁻¹ • A⁻¹ * k • A = 1
[PROOFSTEP]
simp [h, smul_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
h : IsUnit (det A)
⊢ (adjugate A)⁻¹ = (IsUnit.unit h)⁻¹ • A
[PROOFSTEP]
refine' inv_eq_left_inv _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
h : IsUnit (det A)
⊢ (IsUnit.unit h)⁻¹ • A * adjugate A = 1
[PROOFSTEP]
rw [smul_mul, mul_adjugate, Units.smul_def, smul_smul, h.val_inv_mul, one_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α✝ : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α✝
A B : Matrix n n α✝
α : Type u_2
inst✝² : Semiring α
v : n → α
inst✝¹ : Invertible v
inst✝ : Invertible (diagonal v)
⊢ ⅟(diagonal v) = diagonal ⅟v
[PROOFSTEP]
letI := diagonalInvertible v
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α✝ : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α✝
A B : Matrix n n α✝
α : Type u_2
inst✝² : Semiring α
v : n → α
inst✝¹ : Invertible v
inst✝ : Invertible (diagonal v)
this : Invertible (diagonal v) := diagonalInvertible v
⊢ ⅟(diagonal v) = diagonal ⅟v
[PROOFSTEP]
convert (rfl : ⅟(diagonal v) = _)
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
⊢ (diag ⅟(diagonal v) * v) i = OfNat.ofNat 1 i
[PROOFSTEP]
letI : Invertible (diagonal v).det := detInvertibleOfInvertible _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ (diag ⅟(diagonal v) * v) i = OfNat.ofNat 1 i
[PROOFSTEP]
rw [invOf_eq, diag_smul, adjugate_diagonal, diag_diagonal]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ ((⅟(det (diagonal v)) • fun i => ∏ j in erase univ i, v j) * v) i = OfNat.ofNat 1 i
[PROOFSTEP]
dsimp
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ (⅟(det (diagonal v)) * ∏ j in erase univ i, v j) * v i = 1
[PROOFSTEP]
rw [mul_assoc, prod_erase_mul _ _ (Finset.mem_univ _), ← det_diagonal]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ ⅟(det (diagonal v)) * det (diagonal fun x => v x) = 1
[PROOFSTEP]
exact mul_invOf_self _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
⊢ (v * diag ⅟(diagonal v)) i = OfNat.ofNat 1 i
[PROOFSTEP]
letI : Invertible (diagonal v).det := detInvertibleOfInvertible _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ (v * diag ⅟(diagonal v)) i = OfNat.ofNat 1 i
[PROOFSTEP]
rw [invOf_eq, diag_smul, adjugate_diagonal, diag_diagonal]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ (v * ⅟(det (diagonal v)) • fun i => ∏ j in erase univ i, v j) i = OfNat.ofNat 1 i
[PROOFSTEP]
dsimp
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ v i * (⅟(det (diagonal v)) * ∏ j in erase univ i, v j) = 1
[PROOFSTEP]
rw [mul_left_comm, mul_prod_erase _ _ (Finset.mem_univ _), ← det_diagonal]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝³ : Fintype n
inst✝² : DecidableEq n
inst✝¹ : CommRing α
A B : Matrix n n α
v : n → α
inst✝ : Invertible (diagonal v)
i : n
this : Invertible (det (diagonal v)) := detInvertibleOfInvertible (diagonal v)
⊢ ⅟(det (diagonal v)) * det (diagonal fun x => v x) = 1
[PROOFSTEP]
exact mul_invOf_self _
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
⊢ IsUnit (diagonal v) ↔ IsUnit v
[PROOFSTEP]
simp only [← nonempty_invertible_iff_isUnit, (diagonalInvertibleEquivInvertible v).nonempty_congr]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
⊢ (diagonal v)⁻¹ = diagonal (Ring.inverse v)
[PROOFSTEP]
rw [nonsing_inv_eq_ring_inverse]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
by_cases h : IsUnit v
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
h : IsUnit v
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
have := isUnit_diagonal.mpr h
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
h : IsUnit v
this : IsUnit (diagonal v)
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
cases this.nonempty_invertible
[GOAL]
case pos.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
h : IsUnit v
this : IsUnit (diagonal v)
val✝ : Invertible (diagonal v)
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
cases h.nonempty_invertible
[GOAL]
case pos.intro.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
h : IsUnit v
this : IsUnit (diagonal v)
val✝¹ : Invertible (diagonal v)
val✝ : Invertible v
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
rw [Ring.inverse_invertible, Ring.inverse_invertible, invOf_diagonal_eq]
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
h : ¬IsUnit v
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
have := isUnit_diagonal.not.mpr h
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
v : n → α
h : ¬IsUnit v
this : ¬IsUnit (diagonal v)
⊢ Ring.inverse (diagonal v) = diagonal (Ring.inverse v)
[PROOFSTEP]
rw [Ring.inverse_non_unit _ h, Pi.zero_def, diagonal_zero, Ring.inverse_non_unit _ this]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
⊢ A⁻¹⁻¹⁻¹ = A⁻¹
[PROOFSTEP]
by_cases h : IsUnit A.det
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
h : IsUnit (det A)
⊢ A⁻¹⁻¹⁻¹ = A⁻¹
[PROOFSTEP]
rw [nonsing_inv_nonsing_inv _ h]
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
h : ¬IsUnit (det A)
⊢ A⁻¹⁻¹⁻¹ = A⁻¹
[PROOFSTEP]
simp [nonsing_inv_apply_not_isUnit _ h]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
⊢ (A * B)⁻¹ = B⁻¹ * A⁻¹
[PROOFSTEP]
simp only [inv_def]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B✝ A B : Matrix n n α
⊢ Ring.inverse (det (A * B)) • adjugate (A * B) = Ring.inverse (det B) • adjugate B * Ring.inverse (det A) • adjugate A
[PROOFSTEP]
rw [Matrix.smul_mul, Matrix.mul_smul, smul_smul, det_mul, adjugate_mul_distrib, Ring.mul_inverse_rev]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A B : Matrix n n α
⊢ (List.prod [])⁻¹ = List.prod (List.map Inv.inv (List.reverse []))
[PROOFSTEP]
rw [List.reverse_nil, List.map_nil, List.prod_nil, inv_one]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
Xs : List (Matrix n n α)
⊢ (List.prod (A :: Xs))⁻¹ = List.prod (List.map Inv.inv (List.reverse (A :: Xs)))
[PROOFSTEP]
rw [List.reverse_cons', List.map_concat, List.prod_concat, List.prod_cons, mul_inv_rev, list_prod_inv_reverse Xs]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
b : n → α
h : IsUnit (det A)
⊢ det A • mulVec A⁻¹ b = ↑(cramer A) b
[PROOFSTEP]
rw [cramer_eq_adjugate_mulVec, A.nonsing_inv_apply h, ← smul_mulVec_assoc, smul_smul, h.mul_val_inv, one_smul]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝² : Fintype n
inst✝¹ : DecidableEq n
inst✝ : CommRing α
A✝ B A : Matrix n n α
b : n → α
h : IsUnit (det A)
⊢ det A • vecMul b A⁻¹ = ↑(cramer Aᵀ) b
[PROOFSTEP]
rw [← A⁻¹.transpose_transpose, vecMul_transpose, transpose_nonsing_inv, ← det_transpose,
Aᵀ.det_smul_inv_mulVec_eq_cramer _ (isUnit_det_transpose A h)]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α
A✝ B : Matrix n n α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝ : Invertible A
⊢ submatrix A ↑e₁ ↑e₂ * submatrix ⅟A ↑e₂ ↑e₁ = 1
[PROOFSTEP]
rw [Matrix.submatrix_mul_equiv, mul_invOf_self, submatrix_one_equiv]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α
A✝ B : Matrix n n α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝ : Invertible (submatrix A ↑e₁ ↑e₂)
⊢ A * submatrix ⅟(submatrix A ↑e₁ ↑e₂) ↑e₂.symm ↑e₁.symm = 1
[PROOFSTEP]
have : A = (A.submatrix e₁ e₂).submatrix e₁.symm e₂.symm := by
simp
-- Porting note: was
-- conv in _ * _ =>
-- congr
-- rw [this]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α
A✝ B : Matrix n n α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝ : Invertible (submatrix A ↑e₁ ↑e₂)
⊢ A = submatrix (submatrix A ↑e₁ ↑e₂) ↑e₁.symm ↑e₂.symm
[PROOFSTEP]
simp
-- Porting note: was
-- conv in _ * _ =>
-- congr
-- rw [this]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α
A✝ B : Matrix n n α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝ : Invertible (submatrix A ↑e₁ ↑e₂)
this : A = submatrix (submatrix A ↑e₁ ↑e₂) ↑e₁.symm ↑e₂.symm
⊢ A * submatrix ⅟(submatrix A ↑e₁ ↑e₂) ↑e₂.symm ↑e₁.symm = 1
[PROOFSTEP]
rw [congr_arg₂ (· * ·) this rfl]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁵ : Fintype n
inst✝⁴ : DecidableEq n
inst✝³ : CommRing α
A✝ B : Matrix n n α
inst✝² : Fintype m
inst✝¹ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝ : Invertible (submatrix A ↑e₁ ↑e₂)
this : A = submatrix (submatrix A ↑e₁ ↑e₂) ↑e₁.symm ↑e₂.symm
⊢ submatrix (submatrix A ↑e₁ ↑e₂) ↑e₁.symm ↑e₂.symm * submatrix ⅟(submatrix A ↑e₁ ↑e₂) ↑e₂.symm ↑e₁.symm = 1
[PROOFSTEP]
rw [Matrix.submatrix_mul_equiv, mul_invOf_self, submatrix_one_equiv]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁶ : Fintype n
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing α
A✝ B : Matrix n n α
inst✝³ : Fintype m
inst✝² : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝¹ : Invertible A
inst✝ : Invertible (submatrix A ↑e₁ ↑e₂)
⊢ ⅟(submatrix A ↑e₁ ↑e₂) = submatrix ⅟A ↑e₂ ↑e₁
[PROOFSTEP]
letI := submatrixEquivInvertible A e₁ e₂
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁶ : Fintype n
inst✝⁵ : DecidableEq n
inst✝⁴ : CommRing α
A✝ B : Matrix n n α
inst✝³ : Fintype m
inst✝² : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
inst✝¹ : Invertible A
inst✝ : Invertible (submatrix A ↑e₁ ↑e₂)
this : Invertible (submatrix A ↑e₁ ↑e₂) := submatrixEquivInvertible A e₁ e₂
⊢ ⅟(submatrix A ↑e₁ ↑e₂) = submatrix ⅟A ↑e₂ ↑e₁
[PROOFSTEP]
convert (rfl : ⅟(A.submatrix e₁ e₂) = _)
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
⊢ IsUnit (submatrix A ↑e₁ ↑e₂) ↔ IsUnit A
[PROOFSTEP]
simp only [← nonempty_invertible_iff_isUnit, (submatrixEquivInvertibleEquivInvertible A _ _).nonempty_congr]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
⊢ (submatrix A ↑e₁ ↑e₂)⁻¹ = submatrix A⁻¹ ↑e₂ ↑e₁
[PROOFSTEP]
by_cases h : IsUnit A
[GOAL]
case pos
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
h : IsUnit A
⊢ (submatrix A ↑e₁ ↑e₂)⁻¹ = submatrix A⁻¹ ↑e₂ ↑e₁
[PROOFSTEP]
cases h.nonempty_invertible
[GOAL]
case pos.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
h : IsUnit A
val✝ : Invertible A
⊢ (submatrix A ↑e₁ ↑e₂)⁻¹ = submatrix A⁻¹ ↑e₂ ↑e₁
[PROOFSTEP]
letI := submatrixEquivInvertible A e₁ e₂
[GOAL]
case pos.intro
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
h : IsUnit A
val✝ : Invertible A
this : Invertible (submatrix A ↑e₁ ↑e₂) := submatrixEquivInvertible A e₁ e₂
⊢ (submatrix A ↑e₁ ↑e₂)⁻¹ = submatrix A⁻¹ ↑e₂ ↑e₁
[PROOFSTEP]
rw [← invOf_eq_nonsing_inv, ← invOf_eq_nonsing_inv, invOf_submatrix_equiv_eq A]
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
h : ¬IsUnit A
⊢ (submatrix A ↑e₁ ↑e₂)⁻¹ = submatrix A⁻¹ ↑e₂ ↑e₁
[PROOFSTEP]
have := (isUnit_submatrix_equiv e₁ e₂).not.mpr h
[GOAL]
case neg
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A✝ B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
A : Matrix m m α
e₁ e₂ : n ≃ m
h : ¬IsUnit A
this : ¬IsUnit (submatrix A ↑e₁ ↑e₂)
⊢ (submatrix A ↑e₁ ↑e₂)⁻¹ = submatrix A⁻¹ ↑e₂ ↑e₁
[PROOFSTEP]
simp_rw [nonsing_inv_eq_ring_inverse, Ring.inverse_non_unit _ h, Ring.inverse_non_unit _ this, submatrix_zero,
Pi.zero_apply]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
M : Matrix m m α
h : IsUnit M
N : Matrix m m α
⊢ det (M * N * M⁻¹) = det N
[PROOFSTEP]
rw [← h.unit_spec, ← coe_units_inv, det_units_conj]
[GOAL]
l : Type u_1
m : Type u
n : Type u'
α : Type v
inst✝⁴ : Fintype n
inst✝³ : DecidableEq n
inst✝² : CommRing α
A B : Matrix n n α
inst✝¹ : Fintype m
inst✝ : DecidableEq m
M : Matrix m m α
h : IsUnit M
N : Matrix m m α
⊢ det (M⁻¹ * N * M) = det N
[PROOFSTEP]
rw [← h.unit_spec, ← coe_units_inv, det_units_conj']
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.NonsingularInverse", "llama_tokens": 19973} |
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x y : α
S U Z : Set α
⊢ IsGenericPoint x S ↔ ∀ (y : α), x ⤳ y ↔ y ∈ S
[PROOFSTEP]
simp only [specializes_iff_mem_closure, IsGenericPoint, Set.ext_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x y : α
S U Z : Set α
h : IsGenericPoint x S
hU : IsOpen U
⊢ Disjoint S U ↔ ¬x ∈ U
[PROOFSTEP]
rw [h.mem_open_set_iff hU, ← not_disjoint_iff_nonempty_inter, Classical.not_not]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x y : α
S U Z : Set α
h : IsGenericPoint x S
hZ : IsClosed Z
⊢ x ∈ Z ↔ S ⊆ Z
[PROOFSTEP]
rw [← h.def, hZ.closure_subset_iff, singleton_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x y : α
S U Z : Set α
h : IsGenericPoint x S
f : α → β
hf : Continuous f
⊢ IsGenericPoint (f x) (closure (f '' S))
[PROOFSTEP]
rw [isGenericPoint_def, ← h.def, ← image_singleton, closure_image_closure hf]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x y : α
S U Z : Set α
hS : IsClosed S
hxS : x ∈ S
⊢ IsGenericPoint x S ↔ ∀ (Z : Set α), IsClosed Z → x ∈ Z → S ⊆ Z
[PROOFSTEP]
have : closure { x } ⊆ S := closure_minimal (singleton_subset_iff.2 hxS) hS
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x y : α
S U Z : Set α
hS : IsClosed S
hxS : x ∈ S
this : closure {x} ⊆ S
⊢ IsGenericPoint x S ↔ ∀ (Z : Set α), IsClosed Z → x ∈ Z → S ⊆ Z
[PROOFSTEP]
simp_rw [IsGenericPoint, subset_antisymm_iff, this, true_and_iff, closure, subset_sInter_iff, mem_setOf_eq, and_imp,
singleton_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : IrreducibleSpace α
⊢ IsGenericPoint (genericPoint α) ⊤
[PROOFSTEP]
simpa using (IrreducibleSpace.isIrreducible_univ α).genericPoint_spec
[GOAL]
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : IrreducibleSpace α
x : α
⊢ x ∈ closure univ
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : T0Space α
x : α
⊢ IsGenericPoint x (closure (closure {x}))
[PROOFSTEP]
rw [closure_closure]
[GOAL]
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : T0Space α
x : α
⊢ IsGenericPoint x (closure {x})
[PROOFSTEP]
exact isGenericPoint_closure
[GOAL]
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : T0Space α
⊢ ∀ {a b : ↑{s | IsIrreducible s ∧ IsClosed s}},
↑{ toFun := fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s),
invFun := fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) },
left_inv :=
(_ :
∀ (s : ↑{s | IsIrreducible s ∧ IsClosed s}),
(fun x =>
{ val := closure {x},
property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) })
((fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s)) s) =
s),
right_inv := (_ : ∀ (x : α), IsIrreducible.genericPoint (_ : IsIrreducible (closure {x})) = x) }
a ≤
↑{ toFun := fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s),
invFun := fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) },
left_inv :=
(_ :
∀ (s : ↑{s | IsIrreducible s ∧ IsClosed s}),
(fun x =>
{ val := closure {x},
property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) })
((fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s)) s) =
s),
right_inv := (_ : ∀ (x : α), IsIrreducible.genericPoint (_ : IsIrreducible (closure {x})) = x) }
b ↔
a ≤ b
[PROOFSTEP]
rintro ⟨s, hs⟩ ⟨t, ht⟩
[GOAL]
case mk.mk
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : T0Space α
s : Set α
hs : s ∈ {s | IsIrreducible s ∧ IsClosed s}
t : Set α
ht : t ∈ {s | IsIrreducible s ∧ IsClosed s}
⊢ ↑{ toFun := fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s),
invFun := fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) },
left_inv :=
(_ :
∀ (s : ↑{s | IsIrreducible s ∧ IsClosed s}),
(fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) })
((fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s)) s) =
s),
right_inv := (_ : ∀ (x : α), IsIrreducible.genericPoint (_ : IsIrreducible (closure {x})) = x) }
{ val := s, property := hs } ≤
↑{ toFun := fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s),
invFun := fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) },
left_inv :=
(_ :
∀ (s : ↑{s | IsIrreducible s ∧ IsClosed s}),
(fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) })
((fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s)) s) =
s),
right_inv := (_ : ∀ (x : α), IsIrreducible.genericPoint (_ : IsIrreducible (closure {x})) = x) }
{ val := t, property := ht } ↔
{ val := s, property := hs } ≤ { val := t, property := ht }
[PROOFSTEP]
refine specializes_iff_closure_subset.trans ?_
[GOAL]
case mk.mk
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : QuasiSober α
inst✝ : T0Space α
s : Set α
hs : s ∈ {s | IsIrreducible s ∧ IsClosed s}
t : Set α
ht : t ∈ {s | IsIrreducible s ∧ IsClosed s}
⊢ closure
{↑{ toFun := fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s),
invFun := fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) },
left_inv :=
(_ :
∀ (s : ↑{s | IsIrreducible s ∧ IsClosed s}),
(fun x =>
{ val := closure {x},
property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) })
((fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s)) s) =
s),
right_inv := (_ : ∀ (x : α), IsIrreducible.genericPoint (_ : IsIrreducible (closure {x})) = x) }
{ val := s, property := hs }} ⊆
closure
{↑{ toFun := fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s),
invFun := fun x =>
{ val := closure {x}, property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) },
left_inv :=
(_ :
∀ (s : ↑{s | IsIrreducible s ∧ IsClosed s}),
(fun x =>
{ val := closure {x},
property := (_ : IsIrreducible (closure {x}) ∧ IsClosed (closure {x})) })
((fun s => IsIrreducible.genericPoint (_ : IsIrreducible ↑s)) s) =
s),
right_inv := (_ : ∀ (x : α), IsIrreducible.genericPoint (_ : IsIrreducible (closure {x})) = x) }
{ val := t, property := ht }} ↔
{ val := s, property := hs } ≤ { val := t, property := ht }
[PROOFSTEP]
simp [hs.2.closure_eq, ht.2.closure_eq]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : ClosedEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
have hS'' := hS.image f hf.continuous.continuousOn
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : ClosedEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
obtain ⟨x, hx⟩ := QuasiSober.sober hS'' (hf.isClosedMap _ hS')
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : ClosedEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
x : β
hx : IsGenericPoint x (f '' S✝)
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
obtain ⟨y, -, rfl⟩ := hx.mem
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : ClosedEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
y : α
hx : IsGenericPoint (f y) (f '' S✝)
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
use y
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : ClosedEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
y : α
hx : IsGenericPoint (f y) (f '' S✝)
⊢ IsGenericPoint y S✝
[PROOFSTEP]
apply image_injective.mpr hf.inj
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : ClosedEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
y : α
hx : IsGenericPoint (f y) (f '' S✝)
⊢ f '' closure {y} = f '' S✝
[PROOFSTEP]
rw [← hx.def, ← hf.closure_image_eq, image_singleton]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
have hS'' := hS.image f hf.continuous.continuousOn
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
obtain ⟨x, hx⟩ := QuasiSober.sober hS''.closure isClosed_closure
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
S✝ : Set α
hS : IsIrreducible S✝
hS' : IsClosed S✝
hS'' : IsIrreducible (f '' S✝)
x : β
hx : IsGenericPoint x (closure (f '' S✝))
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
obtain ⟨T, hT, rfl⟩ := hf.toInducing.isClosed_iff.mp hS'
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (f '' (f ⁻¹' T))
hx : IsGenericPoint x (closure (f '' (f ⁻¹' T)))
⊢ ∃ x, IsGenericPoint x (f ⁻¹' T)
[PROOFSTEP]
rw [image_preimage_eq_inter_range] at hx hS''
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
⊢ ∃ x, IsGenericPoint x (f ⁻¹' T)
[PROOFSTEP]
have hxT : x ∈ T := by
rw [← hT.closure_eq]
exact closure_mono (inter_subset_left _ _) hx.mem
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
⊢ x ∈ T
[PROOFSTEP]
rw [← hT.closure_eq]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
⊢ x ∈ closure T
[PROOFSTEP]
exact closure_mono (inter_subset_left _ _) hx.mem
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
hxT : x ∈ T
⊢ ∃ x, IsGenericPoint x (f ⁻¹' T)
[PROOFSTEP]
obtain ⟨y, rfl⟩ : x ∈ range f := by
rw [hx.mem_open_set_iff hf.open_range]
refine' Nonempty.mono _ hS''.1
simpa using subset_closure
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
hxT : x ∈ T
⊢ x ∈ range f
[PROOFSTEP]
rw [hx.mem_open_set_iff hf.open_range]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
hxT : x ∈ T
⊢ Set.Nonempty (closure (T ∩ range f) ∩ range f)
[PROOFSTEP]
refine' Nonempty.mono _ hS''.1
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
x : β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
hx : IsGenericPoint x (closure (T ∩ range f))
hxT : x ∈ T
⊢ T ∩ range f ⊆ closure (T ∩ range f) ∩ range f
[PROOFSTEP]
simpa using subset_closure
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
⊢ ∃ x, IsGenericPoint x (f ⁻¹' T)
[PROOFSTEP]
use y
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
⊢ IsGenericPoint y (f ⁻¹' T)
[PROOFSTEP]
change _ = _
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
⊢ closure {y} = f ⁻¹' T
[PROOFSTEP]
rw [hf.toEmbedding.closure_eq_preimage_closure_image, image_singleton, show _ = _ from hx]
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
⊢ f ⁻¹' closure (T ∩ range f) = f ⁻¹' T
[PROOFSTEP]
apply image_injective.mpr hf.inj
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
⊢ f '' (f ⁻¹' closure (T ∩ range f)) = f '' (f ⁻¹' T)
[PROOFSTEP]
ext z
[GOAL]
case h.a.h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
z : β
⊢ z ∈ f '' (f ⁻¹' closure (T ∩ range f)) ↔ z ∈ f '' (f ⁻¹' T)
[PROOFSTEP]
simp only [image_preimage_eq_inter_range, mem_inter_iff, and_congr_left_iff]
[GOAL]
case h.a.h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
hf : OpenEmbedding f
inst✝ : QuasiSober β
T : Set β
hT : IsClosed T
hS : IsIrreducible (f ⁻¹' T)
hS' : IsClosed (f ⁻¹' T)
hS'' : IsIrreducible (T ∩ range f)
y : α
hx : IsGenericPoint (f y) (closure (T ∩ range f))
hxT : f y ∈ T
z : β
⊢ z ∈ range f → (z ∈ closure (T ∩ range f) ↔ z ∈ T)
[PROOFSTEP]
exact fun hy => ⟨fun h => hT.closure_eq ▸ closure_mono (inter_subset_left _ _) h, fun h => subset_closure ⟨h, hy⟩⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
⊢ QuasiSober α
[PROOFSTEP]
rw [quasiSober_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
⊢ ∀ {S : Set α}, IsIrreducible S → IsClosed S → ∃ x, IsGenericPoint x S
[PROOFSTEP]
intro t h h'
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
⊢ ∃ x, IsGenericPoint x t
[PROOFSTEP]
obtain ⟨x, hx⟩ := h.1
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
⊢ ∃ x, IsGenericPoint x t
[PROOFSTEP]
obtain ⟨U, hU, hU'⟩ : x ∈ ⋃₀ S := by
rw [hS'']
trivial
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
⊢ x ∈ ⋃₀ S
[PROOFSTEP]
rw [hS'']
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
⊢ x ∈ ⊤
[PROOFSTEP]
trivial
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
⊢ ∃ x, IsGenericPoint x t
[PROOFSTEP]
haveI : QuasiSober U := hS' ⟨U, hU⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this : QuasiSober ↑U
⊢ ∃ x, IsGenericPoint x t
[PROOFSTEP]
have H : IsPreirreducible ((↑) ⁻¹' t : Set U) := h.2.preimage (hS ⟨U, hU⟩).openEmbedding_subtype_val
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this : QuasiSober ↑U
H : IsPreirreducible (Subtype.val ⁻¹' t)
⊢ ∃ x, IsGenericPoint x t
[PROOFSTEP]
replace H : IsIrreducible ((↑) ⁻¹' t : Set U) := ⟨⟨⟨x, hU'⟩, by simpa using hx⟩, H⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this : QuasiSober ↑U
H : IsPreirreducible (Subtype.val ⁻¹' t)
⊢ { val := x, property := hU' } ∈ Subtype.val ⁻¹' t
[PROOFSTEP]
simpa using hx
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
⊢ ∃ x, IsGenericPoint x t
[PROOFSTEP]
use H.genericPoint
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
⊢ IsGenericPoint (↑(IsIrreducible.genericPoint H)) t
[PROOFSTEP]
have := continuous_subtype_val.closure_preimage_subset _ H.genericPoint_spec.mem
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' closure t
⊢ IsGenericPoint (↑(IsIrreducible.genericPoint H)) t
[PROOFSTEP]
rw [h'.closure_eq] at this
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ IsGenericPoint (↑(IsIrreducible.genericPoint H)) t
[PROOFSTEP]
apply le_antisymm
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ closure {↑(IsIrreducible.genericPoint H)} ≤ t
[PROOFSTEP]
apply h'.closure_subset_iff.mpr
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ {↑(IsIrreducible.genericPoint H)} ⊆ t
[PROOFSTEP]
simpa using this
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ t ≤ closure {↑(IsIrreducible.genericPoint H)}
[PROOFSTEP]
rw [← image_singleton, ← closure_image_closure continuous_subtype_val, H.genericPoint_spec.def]
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ t ≤ closure (Subtype.val '' closure (Subtype.val ⁻¹' t))
[PROOFSTEP]
refine' (subset_closure_inter_of_isPreirreducible_of_isOpen h.2 (hS ⟨U, hU⟩) ⟨x, hx, hU'⟩).trans (closure_mono _)
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ t ∩ ↑{ val := U, property := hU } ⊆ Subtype.val '' closure (Subtype.val ⁻¹' t)
[PROOFSTEP]
rw [← Subtype.image_preimage_coe]
[GOAL]
case h.a
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
S : Set (Set α)
hS : ∀ (s : ↑S), IsOpen ↑s
hS' : ∀ (s : ↑S), QuasiSober ↑↑s
hS'' : ⋃₀ S = ⊤
t : Set α
h : IsIrreducible t
h' : IsClosed t
x : α
hx : x ∈ t
U : Set α
hU : U ∈ S
hU' : x ∈ U
this✝ : QuasiSober ↑U
H : IsIrreducible (Subtype.val ⁻¹' t)
this : IsIrreducible.genericPoint H ∈ Subtype.val ⁻¹' t
⊢ Subtype.val '' (Subtype.val ⁻¹' t) ⊆ Subtype.val '' closure (Subtype.val ⁻¹' t)
[PROOFSTEP]
exact Set.image_subset _ subset_closure
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space α
S✝ : Set α
h : IsIrreducible S✝
x✝ : IsClosed S✝
⊢ ∃ x, IsGenericPoint x S✝
[PROOFSTEP]
obtain ⟨x, rfl⟩ := isIrreducible_iff_singleton.mp h
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space α
x : α
h : IsIrreducible {x}
x✝ : IsClosed {x}
⊢ ∃ x_1, IsGenericPoint x_1 {x}
[PROOFSTEP]
exact ⟨x, closure_singleton⟩
| {"mathlib_filename": "Mathlib.Topology.Sober", "llama_tokens": 12438} |
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
s : Set X
a : X
⊢ a ∈ closure s ↔ ∃ x, (∀ (n : ℕ), x n ∈ s) ∧ Tendsto x atTop (𝓝 a)
[PROOFSTEP]
rw [← seqClosure_eq_closure]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
s : Set X
a : X
⊢ a ∈ seqClosure s ↔ ∃ x, (∀ (n : ℕ), x n ∈ s) ∧ Tendsto x atTop (𝓝 a)
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
f : X → Y
a : X
b : Y
⊢ Tendsto f (𝓝 a) (𝓝 b) ↔ ∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 b)
[PROOFSTEP]
refine' ⟨fun hf u hu => hf.comp hu, fun h => ((nhds_basis_closeds _).tendsto_iff (nhds_basis_closeds _)).2 _⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
f : X → Y
a : X
b : Y
h : ∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 b)
⊢ ∀ (ib : Set Y), ¬b ∈ ib ∧ IsClosed ib → ∃ ia, (¬a ∈ ia ∧ IsClosed ia) ∧ ∀ (x : X), x ∈ iaᶜ → f x ∈ ibᶜ
[PROOFSTEP]
rintro s ⟨hbs, hsc⟩
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
f : X → Y
a : X
b : Y
h : ∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 b)
s : Set Y
hbs : ¬b ∈ s
hsc : IsClosed s
⊢ ∃ ia, (¬a ∈ ia ∧ IsClosed ia) ∧ ∀ (x : X), x ∈ iaᶜ → f x ∈ sᶜ
[PROOFSTEP]
refine' ⟨closure (f ⁻¹' s), ⟨mt _ hbs, isClosed_closure⟩, fun x => mt fun hx => subset_closure hx⟩
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
f : X → Y
a : X
b : Y
h : ∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 b)
s : Set Y
hbs : ¬b ∈ s
hsc : IsClosed s
⊢ a ∈ closure (f ⁻¹' s) → b ∈ s
[PROOFSTEP]
rw [← seqClosure_eq_closure]
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
f : X → Y
a : X
b : Y
h : ∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 b)
s : Set Y
hbs : ¬b ∈ s
hsc : IsClosed s
⊢ a ∈ seqClosure (f ⁻¹' s) → b ∈ s
[PROOFSTEP]
rintro ⟨u, hus, hu⟩
[GOAL]
case intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
f : X → Y
a : X
b : Y
h : ∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 b)
s : Set Y
hbs : ¬b ∈ s
hsc : IsClosed s
u : ℕ → X
hus : ∀ (n : ℕ), u n ∈ f ⁻¹' s
hu : Tendsto u atTop (𝓝 a)
⊢ b ∈ s
[PROOFSTEP]
exact hsc.mem_of_tendsto (h u hu) (eventually_of_forall hus)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
⊢ FrechetUrysohnSpace X
[PROOFSTEP]
refine ⟨fun s x hcx => ?_⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
s : Set X
x : X
hcx : x ∈ closure s
⊢ x ∈ seqClosure s
[PROOFSTEP]
by_cases hx : x ∈ s
[GOAL]
case pos
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
s : Set X
x : X
hcx : x ∈ closure s
hx : x ∈ s
⊢ x ∈ seqClosure s
[PROOFSTEP]
exact subset_seqClosure hx
[GOAL]
case neg
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
s : Set X
x : X
hcx : x ∈ closure s
hx : ¬x ∈ s
⊢ x ∈ seqClosure s
[PROOFSTEP]
obtain ⟨u, hux, hus⟩ : ∃ u : ℕ → X, Tendsto u atTop (𝓝 x) ∧ ∃ᶠ x in atTop, u x ∈ s
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
s : Set X
x : X
hcx : x ∈ closure s
hx : ¬x ∈ s
⊢ ∃ u, Tendsto u atTop (𝓝 x) ∧ ∃ᶠ (x : ℕ) in atTop, u x ∈ s
[PROOFSTEP]
simpa only [ContinuousAt, hx, tendsto_nhds_true, (· ∘ ·), ← not_frequently, exists_prop, ← mem_closure_iff_frequently,
hcx, imp_false, not_forall, not_not] using h (· ∉ s) x
[GOAL]
case neg.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
s : Set X
x : X
hcx : x ∈ closure s
hx : ¬x ∈ s
u : ℕ → X
hux : Tendsto u atTop (𝓝 x)
hus : ∃ᶠ (x : ℕ) in atTop, u x ∈ s
⊢ x ∈ seqClosure s
[PROOFSTEP]
rcases extraction_of_frequently_atTop hus with ⟨φ, φ_mono, hφ⟩
[GOAL]
case neg.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
h :
∀ (f : X → Prop) (a : X), (∀ (u : ℕ → X), Tendsto u atTop (𝓝 a) → Tendsto (f ∘ u) atTop (𝓝 (f a))) → ContinuousAt f a
s : Set X
x : X
hcx : x ∈ closure s
hx : ¬x ∈ s
u : ℕ → X
hux : Tendsto u atTop (𝓝 x)
hus : ∃ᶠ (x : ℕ) in atTop, u x ∈ s
φ : ℕ → ℕ
φ_mono : StrictMono φ
hφ : ∀ (n : ℕ), u (φ n) ∈ s
⊢ x ∈ seqClosure s
[PROOFSTEP]
exact ⟨u ∘ φ, hφ, hux.comp φ_mono.tendsto_atTop⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : FrechetUrysohnSpace X
s : Set X
hs : IsSeqClosed s
⊢ IsClosed s
[PROOFSTEP]
rw [← closure_eq_iff_isClosed, ← seqClosure_eq_closure, hs.seqClosure_eq]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
h : IsSeqCompact s
⊢ TotallyBounded s
[PROOFSTEP]
intro V V_in
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
h : IsSeqCompact s
V : Set (X × X)
V_in : V ∈ 𝓤 X
⊢ ∃ t, Set.Finite t ∧ s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
[PROOFSTEP]
unfold IsSeqCompact at h
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
h : ∀ ⦃x : ℕ → X⦄, (∀ (n : ℕ), x n ∈ s) → ∃ a, a ∈ s ∧ ∃ φ, StrictMono φ ∧ Tendsto (x ∘ φ) atTop (𝓝 a)
V : Set (X × X)
V_in : V ∈ 𝓤 X
⊢ ∃ t, Set.Finite t ∧ s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
[PROOFSTEP]
contrapose! h
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
⊢ Exists fun ⦃x⦄ => (∀ (n : ℕ), x n ∈ s) ∧ ∀ (a : X), a ∈ s → ∀ (φ : ℕ → ℕ), StrictMono φ → ¬Tendsto (x ∘ φ) atTop (𝓝 a)
[PROOFSTEP]
obtain ⟨u, u_in, hu⟩ : ∃ u : ℕ → X, (∀ n, u n ∈ s) ∧ ∀ n m, m < n → u m ∉ ball (u n) V :=
by
simp only [not_subset, mem_iUnion₂, not_exists, exists_prop] at h
simpa only [forall_and, ball_image_iff, not_and] using seq_of_forall_finite_exists h
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
⊢ ∃ u, (∀ (n : ℕ), u n ∈ s) ∧ ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
[PROOFSTEP]
simp only [not_subset, mem_iUnion₂, not_exists, exists_prop] at h
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ∃ a, a ∈ s ∧ ∀ (x : X), ¬(x ∈ t ∧ a ∈ {x_1 | (x_1, x) ∈ V})
⊢ ∃ u, (∀ (n : ℕ), u n ∈ s) ∧ ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
[PROOFSTEP]
simpa only [forall_and, ball_image_iff, not_and] using seq_of_forall_finite_exists h
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
u : ℕ → X
u_in : ∀ (n : ℕ), u n ∈ s
hu : ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
⊢ Exists fun ⦃x⦄ => (∀ (n : ℕ), x n ∈ s) ∧ ∀ (a : X), a ∈ s → ∀ (φ : ℕ → ℕ), StrictMono φ → ¬Tendsto (x ∘ φ) atTop (𝓝 a)
[PROOFSTEP]
refine' ⟨u, u_in, fun x _ φ hφ huφ => _⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
u : ℕ → X
u_in : ∀ (n : ℕ), u n ∈ s
hu : ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
x : X
x✝ : x ∈ s
φ : ℕ → ℕ
hφ : StrictMono φ
huφ : Tendsto (u ∘ φ) atTop (𝓝 x)
⊢ False
[PROOFSTEP]
obtain ⟨N, hN⟩ : ∃ N, ∀ p q, p ≥ N → q ≥ N → (u (φ p), u (φ q)) ∈ V
[GOAL]
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
u : ℕ → X
u_in : ∀ (n : ℕ), u n ∈ s
hu : ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
x : X
x✝ : x ∈ s
φ : ℕ → ℕ
hφ : StrictMono φ
huφ : Tendsto (u ∘ φ) atTop (𝓝 x)
⊢ ∃ N, ∀ (p q : ℕ), p ≥ N → q ≥ N → (u (φ p), u (φ q)) ∈ V
case intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
u : ℕ → X
u_in : ∀ (n : ℕ), u n ∈ s
hu : ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
x : X
x✝ : x ∈ s
φ : ℕ → ℕ
hφ : StrictMono φ
huφ : Tendsto (u ∘ φ) atTop (𝓝 x)
N : ℕ
hN : ∀ (p q : ℕ), p ≥ N → q ≥ N → (u (φ p), u (φ q)) ∈ V
⊢ False
[PROOFSTEP]
exact huφ.cauchySeq.mem_entourage V_in
[GOAL]
case intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝ : UniformSpace X
s : Set X
V : Set (X × X)
V_in : V ∈ 𝓤 X
h : ∀ (t : Set X), Set.Finite t → ¬s ⊆ ⋃ (y : X) (_ : y ∈ t), {x | (x, y) ∈ V}
u : ℕ → X
u_in : ∀ (n : ℕ), u n ∈ s
hu : ∀ (n m : ℕ), m < n → ¬u m ∈ ball (u n) V
x : X
x✝ : x ∈ s
φ : ℕ → ℕ
hφ : StrictMono φ
huφ : Tendsto (u ∘ φ) atTop (𝓝 x)
N : ℕ
hN : ∀ (p q : ℕ), p ≥ N → q ≥ N → (u (φ p), u (φ q)) ∈ V
⊢ False
[PROOFSTEP]
exact hu (φ <| N + 1) (φ N) (hφ <| lt_add_one N) (hN (N + 1) N N.le_succ le_rfl)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
have := hl.1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
rcases exists_antitone_basis (𝓤 X) with ⟨V, hV⟩
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
choose W hW hWV using fun n => comp_mem_uniformity_sets (hV.mem n)
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
have hWV' : ∀ n, W n ⊆ V n := fun n ⟨x, y⟩ hx => @hWV n (x, y) ⟨x, refl_mem_uniformity <| hW _, hx⟩
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
obtain ⟨t, ht_anti, htl, htW, hts⟩ :
∃ t : ℕ → Set X, Antitone t ∧ (∀ n, t n ∈ l) ∧ (∀ n, t n ×ˢ t n ⊆ W n) ∧ ∀ n, t n ⊆ s :=
by
have : ∀ n, ∃ t ∈ l, t ×ˢ t ⊆ W n ∧ t ⊆ s :=
by
rw [le_principal_iff] at hls
have : ∀ n, W n ∩ s ×ˢ s ∈ l ×ˢ l := fun n => inter_mem (hl.2 (hW n)) (prod_mem_prod hls hls)
simpa only [l.basis_sets.prod_self.mem_iff, true_imp_iff, subset_inter_iff, prod_self_subset_prod_self,
and_assoc] using this
choose t htl htW hts using this
have : ∀ n : ℕ, ⋂ k ≤ n, t k ⊆ t n := fun n => by apply iInter₂_subset; rfl
exact
⟨fun n => ⋂ k ≤ n, t k, fun m n h => biInter_subset_biInter_left fun k (hk : k ≤ m) => hk.trans h, fun n =>
(biInter_mem (finite_le_nat n)).2 fun k _ => htl k, fun n => (prod_mono (this n) (this n)).trans (htW n), fun n =>
(this n).trans (hts n)⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
⊢ ∃ t, Antitone t ∧ (∀ (n : ℕ), t n ∈ l) ∧ (∀ (n : ℕ), t n ×ˢ t n ⊆ W n) ∧ ∀ (n : ℕ), t n ⊆ s
[PROOFSTEP]
have : ∀ n, ∃ t ∈ l, t ×ˢ t ⊆ W n ∧ t ⊆ s := by
rw [le_principal_iff] at hls
have : ∀ n, W n ∩ s ×ˢ s ∈ l ×ˢ l := fun n => inter_mem (hl.2 (hW n)) (prod_mem_prod hls hls)
simpa only [l.basis_sets.prod_self.mem_iff, true_imp_iff, subset_inter_iff, prod_self_subset_prod_self,
and_assoc] using this
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
⊢ ∀ (n : ℕ), ∃ t, t ∈ l ∧ t ×ˢ t ⊆ W n ∧ t ⊆ s
[PROOFSTEP]
rw [le_principal_iff] at hls
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : s ∈ l
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
⊢ ∀ (n : ℕ), ∃ t, t ∈ l ∧ t ×ˢ t ⊆ W n ∧ t ⊆ s
[PROOFSTEP]
have : ∀ n, W n ∩ s ×ˢ s ∈ l ×ˢ l := fun n => inter_mem (hl.2 (hW n)) (prod_mem_prod hls hls)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : s ∈ l
this✝ : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
this : ∀ (n : ℕ), W n ∩ s ×ˢ s ∈ l ×ˢ l
⊢ ∀ (n : ℕ), ∃ t, t ∈ l ∧ t ×ˢ t ⊆ W n ∧ t ⊆ s
[PROOFSTEP]
simpa only [l.basis_sets.prod_self.mem_iff, true_imp_iff, subset_inter_iff, prod_self_subset_prod_self, and_assoc] using
this
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this✝ : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
this : ∀ (n : ℕ), ∃ t, t ∈ l ∧ t ×ˢ t ⊆ W n ∧ t ⊆ s
⊢ ∃ t, Antitone t ∧ (∀ (n : ℕ), t n ∈ l) ∧ (∀ (n : ℕ), t n ×ˢ t n ⊆ W n) ∧ ∀ (n : ℕ), t n ⊆ s
[PROOFSTEP]
choose t htl htW hts using this
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
⊢ ∃ t, Antitone t ∧ (∀ (n : ℕ), t n ∈ l) ∧ (∀ (n : ℕ), t n ×ˢ t n ⊆ W n) ∧ ∀ (n : ℕ), t n ⊆ s
[PROOFSTEP]
have : ∀ n : ℕ, ⋂ k ≤ n, t k ⊆ t n := fun n => by apply iInter₂_subset; rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
n : ℕ
⊢ ⋂ (k : ℕ) (_ : k ≤ n), t k ⊆ t n
[PROOFSTEP]
apply iInter₂_subset
[GOAL]
case j
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
n : ℕ
⊢ n ≤ n
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this✝ : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
this : ∀ (n : ℕ), ⋂ (k : ℕ) (_ : k ≤ n), t k ⊆ t n
⊢ ∃ t, Antitone t ∧ (∀ (n : ℕ), t n ∈ l) ∧ (∀ (n : ℕ), t n ×ˢ t n ⊆ W n) ∧ ∀ (n : ℕ), t n ⊆ s
[PROOFSTEP]
exact
⟨fun n => ⋂ k ≤ n, t k, fun m n h => biInter_subset_biInter_left fun k (hk : k ≤ m) => hk.trans h, fun n =>
(biInter_mem (finite_le_nat n)).2 fun k _ => htl k, fun n => (prod_mono (this n) (this n)).trans (htW n), fun n =>
(this n).trans (hts n)⟩
[GOAL]
case intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
choose u hu using fun n => Filter.nonempty_of_mem (htl n)
[GOAL]
case intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
have huc : CauchySeq u :=
hV.toHasBasis.cauchySeq_iff.2 fun N _ =>
⟨N, fun m hm n hn => hWV' _ <| @htW N (_, _) ⟨ht_anti hm (hu _), ht_anti hn (hu _)⟩⟩
[GOAL]
case intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
huc : CauchySeq u
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
rcases hs.exists_tendsto (fun n => hts n (hu n)) huc with ⟨x, hxs, hx⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
huc : CauchySeq u
x : X
hxs : x ∈ s
hx : Tendsto (fun n => u n) atTop (𝓝 x)
⊢ ∃ x, x ∈ s ∧ l ≤ 𝓝 x
[PROOFSTEP]
refine ⟨x, hxs, (nhds_basis_uniformity' hV.toHasBasis).ge_iff.2 fun N _ => ?_⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
huc : CauchySeq u
x : X
hxs : x ∈ s
hx : Tendsto (fun n => u n) atTop (𝓝 x)
N : ℕ
x✝ : True
⊢ ball x (V N) ∈ l
[PROOFSTEP]
obtain ⟨n, hNn, hn⟩ : ∃ n, N ≤ n ∧ u n ∈ ball x (W N)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
huc : CauchySeq u
x : X
hxs : x ∈ s
hx : Tendsto (fun n => u n) atTop (𝓝 x)
N : ℕ
x✝ : True
⊢ ∃ n, N ≤ n ∧ u n ∈ ball x (W N)
[PROOFSTEP]
exact ((eventually_ge_atTop N).and (hx <| ball_mem_nhds x (hW N))).exists
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
huc : CauchySeq u
x : X
hxs : x ∈ s
hx : Tendsto (fun n => u n) atTop (𝓝 x)
N : ℕ
x✝ : True
n : ℕ
hNn : N ≤ n
hn : u n ∈ ball x (W N)
⊢ ball x (V N) ∈ l
[PROOFSTEP]
refine mem_of_superset (htl n) fun y hy => hWV N ⟨u n, hn, htW N ?_⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
hs : IsSeqCompact s
l : Filter X
hl : Cauchy l
hls : l ≤ 𝓟 s
this : NeBot l
V : ℕ → Set (X × X)
hV : HasAntitoneBasis (𝓤 X) V
W : ℕ → Set (X × X)
hW : ∀ (n : ℕ), W n ∈ 𝓤 X
hWV : ∀ (n : ℕ), W n ○ W n ⊆ V n
hWV' : ∀ (n : ℕ), W n ⊆ V n
t : ℕ → Set X
ht_anti : Antitone t
htl : ∀ (n : ℕ), t n ∈ l
htW : ∀ (n : ℕ), t n ×ˢ t n ⊆ W n
hts : ∀ (n : ℕ), t n ⊆ s
u : ℕ → X
hu : ∀ (n : ℕ), u n ∈ t n
huc : CauchySeq u
x : X
hxs : x ∈ s
hx : Tendsto (fun n => u n) atTop (𝓝 x)
N : ℕ
x✝ : True
n : ℕ
hNn : N ≤ n
hn : u n ∈ ball x (W N)
y : X
hy : y ∈ t n
⊢ (u n, (x, y).snd) ∈ t N ×ˢ t N
[PROOFSTEP]
exact ⟨ht_anti hNn (hu n), ht_anti hNn hy⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : UniformSpace X
s : Set X
inst✝ : IsCountablyGenerated (𝓤 X)
⊢ CompactSpace X ↔ SeqCompactSpace X
[PROOFSTEP]
simp only [← isCompact_univ_iff, seqCompactSpace_iff, UniformSpace.isCompact_iff_isSeqCompact]
| {"mathlib_filename": "Mathlib.Topology.Sequences", "llama_tokens": 13198} |
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set α
h : IsOpen s
⊢ ∀ (t : Set α), t ∈ {s} → IsOpen t
[PROOFSTEP]
simp [h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
I : Set ι
hI : Set.Countable I
f : ι → Set α
hf : ∀ (i : ι), i ∈ I → IsOpen (f i)
⊢ ∀ (t : Set α), t ∈ f '' I → IsOpen t
[PROOFSTEP]
rwa [ball_image_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
I : Set ι
hI : Set.Countable I
f : ι → Set α
hf : ∀ (i : ι), i ∈ I → IsOpen (f i)
⊢ ⋂ (i : ι) (_ : i ∈ I), f i = ⋂₀ (f '' I)
[PROOFSTEP]
rw [sInter_image]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : Encodable ι
f : ι → Set α
hf : ∀ (i : ι), IsOpen (f i)
⊢ ∀ (t : Set α), t ∈ range f → IsOpen t
[PROOFSTEP]
rwa [forall_range_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : Encodable ι
f : ι → Set α
hf : ∀ (i : ι), IsOpen (f i)
⊢ ⋂ (i : ι), f i = ⋂₀ range f
[PROOFSTEP]
rw [sInter_range]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : Encodable ι
s : ι → Set α
hs : ∀ (i : ι), IsGδ (s i)
⊢ IsGδ (⋂ (i : ι), s i)
[PROOFSTEP]
choose T hTo hTc hTs using hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : Encodable ι
s : ι → Set α
T : ι → Set (Set α)
hTo : ∀ (i : ι) (t : Set α), t ∈ T i → IsOpen t
hTc : ∀ (i : ι), Set.Countable (T i)
hTs : ∀ (i : ι), s i = ⋂₀ T i
⊢ IsGδ (⋂ (i : ι), s i)
[PROOFSTEP]
obtain rfl : s = fun i => ⋂₀ T i := funext hTs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : Encodable ι
T : ι → Set (Set α)
hTo : ∀ (i : ι) (t : Set α), t ∈ T i → IsOpen t
hTc : ∀ (i : ι), Set.Countable (T i)
hTs : ∀ (i : ι), (fun i => ⋂₀ T i) i = ⋂₀ T i
⊢ IsGδ (⋂ (i : ι), (fun i => ⋂₀ T i) i)
[PROOFSTEP]
refine' ⟨⋃ i, T i, _, countable_iUnion hTc, (sInter_iUnion _).symm⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : Encodable ι
T : ι → Set (Set α)
hTo : ∀ (i : ι) (t : Set α), t ∈ T i → IsOpen t
hTc : ∀ (i : ι), Set.Countable (T i)
hTs : ∀ (i : ι), (fun i => ⋂₀ T i) i = ⋂₀ T i
⊢ ∀ (t : Set α), t ∈ ⋃ (i : ι), T i → IsOpen t
[PROOFSTEP]
simpa [@forall_swap ι] using hTo
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Countable s
t : (i : ι) → i ∈ s → Set α
ht : ∀ (i : ι) (hi : i ∈ s), IsGδ (t i hi)
⊢ IsGδ (⋂ (i : ι) (h : i ∈ s), t i h)
[PROOFSTEP]
rw [biInter_eq_iInter]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Countable s
t : (i : ι) → i ∈ s → Set α
ht : ∀ (i : ι) (hi : i ∈ s), IsGδ (t i hi)
⊢ IsGδ (⋂ (x : ↑s), t ↑x (_ : ↑x ∈ s))
[PROOFSTEP]
haveI := hs.toEncodable
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Countable s
t : (i : ι) → i ∈ s → Set α
ht : ∀ (i : ι) (hi : i ∈ s), IsGδ (t i hi)
this : Encodable ↑s
⊢ IsGδ (⋂ (x : ↑s), t ↑x (_ : ↑x ∈ s))
[PROOFSTEP]
exact isGδ_iInter fun x => ht x x.2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
S : Set (Set α)
h : ∀ (s : Set α), s ∈ S → IsGδ s
hS : Set.Countable S
⊢ IsGδ (⋂₀ S)
[PROOFSTEP]
simpa only [sInter_eq_biInter] using isGδ_biInter hS h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
hs : IsGδ s
ht : IsGδ t
⊢ IsGδ (s ∩ t)
[PROOFSTEP]
rw [inter_eq_iInter]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
hs : IsGδ s
ht : IsGδ t
⊢ IsGδ (⋂ (b : Bool), bif b then s else t)
[PROOFSTEP]
exact isGδ_iInter (Bool.forall_bool.2 ⟨ht, hs⟩)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
hs : IsGδ s
ht : IsGδ t
⊢ IsGδ (s ∪ t)
[PROOFSTEP]
rcases hs with ⟨S, Sopen, Scount, rfl⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
t : Set α
ht : IsGδ t
S : Set (Set α)
Sopen : ∀ (t : Set α), t ∈ S → IsOpen t
Scount : Set.Countable S
⊢ IsGδ (⋂₀ S ∪ t)
[PROOFSTEP]
rcases ht with ⟨T, Topen, Tcount, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
S : Set (Set α)
Sopen : ∀ (t : Set α), t ∈ S → IsOpen t
Scount : Set.Countable S
T : Set (Set α)
Topen : ∀ (t : Set α), t ∈ T → IsOpen t
Tcount : Set.Countable T
⊢ IsGδ (⋂₀ S ∪ ⋂₀ T)
[PROOFSTEP]
rw [sInter_union_sInter]
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
S : Set (Set α)
Sopen : ∀ (t : Set α), t ∈ S → IsOpen t
Scount : Set.Countable S
T : Set (Set α)
Topen : ∀ (t : Set α), t ∈ T → IsOpen t
Tcount : Set.Countable T
⊢ IsGδ (⋂ (p : Set α × Set α) (_ : p ∈ S ×ˢ T), p.fst ∪ p.snd)
[PROOFSTEP]
apply isGδ_biInter_of_open (Scount.prod Tcount)
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
S : Set (Set α)
Sopen : ∀ (t : Set α), t ∈ S → IsOpen t
Scount : Set.Countable S
T : Set (Set α)
Topen : ∀ (t : Set α), t ∈ T → IsOpen t
Tcount : Set.Countable T
⊢ ∀ (i : Set α × Set α), i ∈ S ×ˢ T → IsOpen (i.fst ∪ i.snd)
[PROOFSTEP]
rintro ⟨a, b⟩ ⟨ha, hb⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.mk.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
S : Set (Set α)
Sopen : ∀ (t : Set α), t ∈ S → IsOpen t
Scount : Set.Countable S
T : Set (Set α)
Topen : ∀ (t : Set α), t ∈ T → IsOpen t
Tcount : Set.Countable T
a b : Set α
ha : (a, b).fst ∈ S
hb : (a, b).snd ∈ T
⊢ IsOpen ((a, b).fst ∪ (a, b).snd)
[PROOFSTEP]
exact (Sopen a ha).union (Topen b hb)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Finite s
f : ι → Set α
h : ∀ (i : ι), i ∈ s → IsGδ (f i)
⊢ IsGδ (⋃ (i : ι) (_ : i ∈ s), f i)
[PROOFSTEP]
refine' Finite.induction_on hs (by simp) _ h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Finite s
f : ι → Set α
h : ∀ (i : ι), i ∈ s → IsGδ (f i)
⊢ (∀ (i : ι), i ∈ ∅ → IsGδ (f i)) → IsGδ (⋃ (i : ι) (_ : i ∈ ∅), f i)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Finite s
f : ι → Set α
h : ∀ (i : ι), i ∈ s → IsGδ (f i)
⊢ ∀ {a : ι} {s : Set ι},
¬a ∈ s →
Set.Finite s →
((∀ (i : ι), i ∈ s → IsGδ (f i)) → IsGδ (⋃ (i : ι) (_ : i ∈ s), f i)) →
(∀ (i : ι), i ∈ insert a s → IsGδ (f i)) → IsGδ (⋃ (i : ι) (_ : i ∈ insert a s), f i)
[PROOFSTEP]
simp only [ball_insert_iff, biUnion_insert]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set ι
hs : Set.Finite s
f : ι → Set α
h : ∀ (i : ι), i ∈ s → IsGδ (f i)
⊢ ∀ {a : ι} {s : Set ι},
¬a ∈ s →
Set.Finite s →
((∀ (i : ι), i ∈ s → IsGδ (f i)) → IsGδ (⋃ (i : ι) (_ : i ∈ s), f i)) →
(IsGδ (f a) ∧ ∀ (i : ι), i ∈ s → IsGδ (f i)) → IsGδ (f a ∪ ⋃ (i : ι) (_ : i ∈ s), f i)
[PROOFSTEP]
exact fun _ _ ihs H => H.1.union (ihs H.2)
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α✝
α : Type u_5
inst✝¹ : UniformSpace α
inst✝ : IsCountablyGenerated (uniformity α)
s : Set α
hs : IsClosed s
⊢ IsGδ s
[PROOFSTEP]
rcases(@uniformity_hasBasis_open α _).exists_antitone_subbasis with ⟨U, hUo, hU, -⟩
[GOAL]
case intro.intro.mk
α✝ : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α✝
α : Type u_5
inst✝¹ : UniformSpace α
inst✝ : IsCountablyGenerated (uniformity α)
s : Set α
hs : IsClosed s
U : ℕ → Set (α × α)
hUo : ∀ (i : ℕ), U i ∈ uniformity α ∧ IsOpen (U i)
hU : HasBasis (uniformity α) (fun x => True) fun i => id (U i)
⊢ IsGδ s
[PROOFSTEP]
rw [← hs.closure_eq, ← hU.biInter_biUnion_ball]
[GOAL]
case intro.intro.mk
α✝ : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α✝
α : Type u_5
inst✝¹ : UniformSpace α
inst✝ : IsCountablyGenerated (uniformity α)
s : Set α
hs : IsClosed s
U : ℕ → Set (α × α)
hUo : ∀ (i : ℕ), U i ∈ uniformity α ∧ IsOpen (U i)
hU : HasBasis (uniformity α) (fun x => True) fun i => id (U i)
⊢ IsGδ (⋂ (i : ℕ) (_ : True), ⋃ (x : α) (_ : x ∈ s), UniformSpace.ball x (id (U i)))
[PROOFSTEP]
refine' isGδ_biInter (to_countable _) fun n _ => IsOpen.isGδ _
[GOAL]
case intro.intro.mk
α✝ : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α✝
α : Type u_5
inst✝¹ : UniformSpace α
inst✝ : IsCountablyGenerated (uniformity α)
s : Set α
hs : IsClosed s
U : ℕ → Set (α × α)
hUo : ∀ (i : ℕ), U i ∈ uniformity α ∧ IsOpen (U i)
hU : HasBasis (uniformity α) (fun x => True) fun i => id (U i)
n : ℕ
x✝ : n ∈ fun i => True
⊢ IsOpen (⋃ (x : α) (_ : x ∈ s), UniformSpace.ball x (id (U n)))
[PROOFSTEP]
exact isOpen_biUnion fun x _ => UniformSpace.isOpen_ball _ (hUo _).2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
hs : Set.Countable s
⊢ IsGδ sᶜ
[PROOFSTEP]
rw [← biUnion_of_singleton s, compl_iUnion₂]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
hs : Set.Countable s
⊢ IsGδ (⋂ (i : α) (_ : i ∈ s), {i}ᶜ)
[PROOFSTEP]
exact isGδ_biInter hs fun x _ => isGδ_compl_singleton x
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : FirstCountableTopology α
a : α
⊢ IsGδ {a}
[PROOFSTEP]
rcases(nhds_basis_opens a).exists_antitone_subbasis with ⟨U, hU, h_basis⟩
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : FirstCountableTopology α
a : α
U : ℕ → Set α
hU : ∀ (i : ℕ), a ∈ U i ∧ IsOpen (U i)
h_basis : HasAntitoneBasis (𝓝 a) fun i => U i
⊢ IsGδ {a}
[PROOFSTEP]
rw [← biInter_basis_nhds h_basis.toHasBasis]
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : FirstCountableTopology α
a : α
U : ℕ → Set α
hU : ∀ (i : ℕ), a ∈ U i ∧ IsOpen (U i)
h_basis : HasAntitoneBasis (𝓝 a) fun i => U i
⊢ IsGδ (⋂ (i : ℕ) (_ : True), U i)
[PROOFSTEP]
exact isGδ_biInter (to_countable _) fun n _ => (hU n).2.isGδ
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : UniformSpace β
inst✝ : IsCountablyGenerated (uniformity β)
f : α → β
⊢ IsGδ {x | ContinuousAt f x}
[PROOFSTEP]
obtain ⟨U, _, hU⟩ := (@uniformity_hasBasis_open_symmetric β _).exists_antitone_subbasis
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : UniformSpace β
inst✝ : IsCountablyGenerated (uniformity β)
f : α → β
U : ℕ → Set (β × β)
left✝ : ∀ (i : ℕ), U i ∈ uniformity β ∧ IsOpen (U i) ∧ SymmetricRel (U i)
hU : HasAntitoneBasis (uniformity β) fun i => id (U i)
⊢ IsGδ {x | ContinuousAt f x}
[PROOFSTEP]
simp only [Uniform.continuousAt_iff_prod, nhds_prod_eq]
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : UniformSpace β
inst✝ : IsCountablyGenerated (uniformity β)
f : α → β
U : ℕ → Set (β × β)
left✝ : ∀ (i : ℕ), U i ∈ uniformity β ∧ IsOpen (U i) ∧ SymmetricRel (U i)
hU : HasAntitoneBasis (uniformity β) fun i => id (U i)
⊢ IsGδ {x | Tendsto (fun x => (f x.fst, f x.snd)) (𝓝 x ×ˢ 𝓝 x) (uniformity β)}
[PROOFSTEP]
simp only [(nhds_basis_opens _).prod_self.tendsto_iff hU.toHasBasis, forall_prop_of_true, setOf_forall, id]
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : UniformSpace β
inst✝ : IsCountablyGenerated (uniformity β)
f : α → β
U : ℕ → Set (β × β)
left✝ : ∀ (i : ℕ), U i ∈ uniformity β ∧ IsOpen (U i) ∧ SymmetricRel (U i)
hU : HasAntitoneBasis (uniformity β) fun i => id (U i)
⊢ IsGδ (⋂ (i : ℕ), {x | ∃ ia, (x ∈ ia ∧ IsOpen ia) ∧ ∀ (x : α × α), x ∈ ia ×ˢ ia → (f x.fst, f x.snd) ∈ U i})
[PROOFSTEP]
refine' isGδ_iInter fun k => IsOpen.isGδ <| isOpen_iff_mem_nhds.2 fun x => _
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : UniformSpace β
inst✝ : IsCountablyGenerated (uniformity β)
f : α → β
U : ℕ → Set (β × β)
left✝ : ∀ (i : ℕ), U i ∈ uniformity β ∧ IsOpen (U i) ∧ SymmetricRel (U i)
hU : HasAntitoneBasis (uniformity β) fun i => id (U i)
k : ℕ
x : α
⊢ x ∈ {x | ∃ ia, (x ∈ ia ∧ IsOpen ia) ∧ ∀ (x : α × α), x ∈ ia ×ˢ ia → (f x.fst, f x.snd) ∈ U k} →
{x | ∃ ia, (x ∈ ia ∧ IsOpen ia) ∧ ∀ (x : α × α), x ∈ ia ×ˢ ia → (f x.fst, f x.snd) ∈ U k} ∈ 𝓝 x
[PROOFSTEP]
rintro ⟨s, ⟨hsx, hso⟩, hsU⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : UniformSpace β
inst✝ : IsCountablyGenerated (uniformity β)
f : α → β
U : ℕ → Set (β × β)
left✝ : ∀ (i : ℕ), U i ∈ uniformity β ∧ IsOpen (U i) ∧ SymmetricRel (U i)
hU : HasAntitoneBasis (uniformity β) fun i => id (U i)
k : ℕ
x : α
s : Set α
hsU : ∀ (x : α × α), x ∈ s ×ˢ s → (f x.fst, f x.snd) ∈ U k
hsx : x ∈ s
hso : IsOpen s
⊢ {x | ∃ ia, (x ∈ ia ∧ IsOpen ia) ∧ ∀ (x : α × α), x ∈ ia ×ˢ ia → (f x.fst, f x.snd) ∈ U k} ∈ 𝓝 x
[PROOFSTEP]
filter_upwards [IsOpen.mem_nhds hso hsx] with _ hy using ⟨s, ⟨hy, hso⟩, hsU⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
⊢ CountableInterFilter (residual α)
[PROOFSTEP]
rw [residual]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
⊢ CountableInterFilter (countableGenerate {t | IsOpen t ∧ Dense t})
[PROOFSTEP]
infer_instance
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set α
ho : IsGδ s
hd : Dense s
⊢ s ∈ residual α
[PROOFSTEP]
rcases ho with ⟨T, To, Tct, rfl⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
T : Set (Set α)
To : ∀ (t : Set α), t ∈ T → IsOpen t
Tct : Set.Countable T
hd : Dense (⋂₀ T)
⊢ ⋂₀ T ∈ residual α
[PROOFSTEP]
exact (countable_sInter_mem Tct).mpr fun t tT => residual_of_dense_open (To t tT) (hd.mono (sInter_subset_of_mem tT))
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
ι : Type u_4
inst✝ : TopologicalSpace α
s : Set α
⊢ (∃ S, S ⊆ {t | IsOpen t ∧ Dense t} ∧ Set.Countable S ∧ ⋂₀ S ⊆ s) ↔
∃ S, (∀ (t : Set α), t ∈ S → IsOpen t) ∧ (∀ (t : Set α), t ∈ S → Dense t) ∧ Set.Countable S ∧ ⋂₀ S ⊆ s
[PROOFSTEP]
simp_rw [subset_def, mem_setOf, forall_and, and_assoc]
| {"mathlib_filename": "Mathlib.Topology.GDelta", "llama_tokens": 7599} |
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
⊢ find c ne i ∈ c
[PROOFSTEP]
rw [find]
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
⊢ (if hi : ∃ v, v ∈ c ∧ i ∈ v.carrier then Exists.choose hi else Set.Nonempty.some ne) ∈ c
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ∃ v, v ∈ c ∧ i ∈ v.carrier
⊢ Exists.choose h ∈ c
case neg
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ¬∃ v, v ∈ c ∧ i ∈ v.carrier
⊢ Set.Nonempty.some ne ∈ c
[PROOFSTEP]
exacts [h.choose_spec.1, ne.some_mem]
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
⊢ i ∈ (find c ne i).carrier ↔ i ∈ chainSupCarrier c
[PROOFSTEP]
rw [find]
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
⊢ i ∈ (if hi : ∃ v, v ∈ c ∧ i ∈ v.carrier then Exists.choose hi else Set.Nonempty.some ne).carrier ↔
i ∈ chainSupCarrier c
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ∃ v, v ∈ c ∧ i ∈ v.carrier
⊢ i ∈ (Exists.choose h).carrier ↔ i ∈ chainSupCarrier c
[PROOFSTEP]
have := h.choose_spec
[GOAL]
case pos
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ∃ v, v ∈ c ∧ i ∈ v.carrier
this : Exists.choose h ∈ c ∧ i ∈ (Exists.choose h).carrier
⊢ i ∈ (Exists.choose h).carrier ↔ i ∈ chainSupCarrier c
[PROOFSTEP]
exact iff_of_true this.2 (mem_iUnion₂.2 ⟨_, this.1, this.2⟩)
[GOAL]
case neg
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ¬∃ v, v ∈ c ∧ i ∈ v.carrier
⊢ i ∈ (Set.Nonempty.some ne).carrier ↔ i ∈ chainSupCarrier c
[PROOFSTEP]
push_neg at h
[GOAL]
case neg
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ∀ (v : PartialRefinement u s), v ∈ c → ¬i ∈ v.carrier
⊢ i ∈ (Set.Nonempty.some ne).carrier ↔ i ∈ chainSupCarrier c
[PROOFSTEP]
refine iff_of_false (h _ ne.some_mem) ?_
[GOAL]
case neg
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
i : ι
ne : Set.Nonempty c
h : ∀ (v : PartialRefinement u s), v ∈ c → ¬i ∈ v.carrier
⊢ ¬i ∈ chainSupCarrier c
[PROOFSTEP]
simpa only [chainSupCarrier, mem_iUnion₂, not_exists]
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
rcases em (∃ i, i ∉ chainSupCarrier c ∧ x ∈ u i) with (⟨i, hi, hxi⟩ | hx)
[GOAL]
case inl.intro.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
i : ι
hi : ¬i ∈ chainSupCarrier c
hxi : x ∈ u i
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
use i
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
i : ι
hi : ¬i ∈ chainSupCarrier c
hxi : x ∈ u i
⊢ x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
simpa only [(find c ne i).apply_eq (mt (mem_find_carrier_iff _).1 hi)]
[GOAL]
case inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
hx : ¬∃ i, ¬i ∈ chainSupCarrier c ∧ x ∈ u i
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
simp_rw [not_exists, not_and, not_imp_not, chainSupCarrier, mem_iUnion₂] at hx
[GOAL]
case inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
hx : ∀ (x_1 : ι), x ∈ u x_1 → ∃ i j, x_1 ∈ i.carrier
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
haveI : Nonempty (PartialRefinement u s) := ⟨ne.some⟩
[GOAL]
case inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
hx : ∀ (x_1 : ι), x ∈ u x_1 → ∃ i j, x_1 ∈ i.carrier
this : Nonempty (PartialRefinement u s)
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
choose! v hvc hiv using hx
[GOAL]
case inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
this : Nonempty (PartialRefinement u s)
v : ι → PartialRefinement u s
hvc : ∀ (x_1 : ι), x ∈ u x_1 → v x_1 ∈ c
hiv : ∀ (x_1 : ι), x ∈ u x_1 → x_1 ∈ (v x_1).carrier
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
rcases(hfin x hxs).exists_maximal_wrt v _ (mem_iUnion.1 (hU hxs)) with
⟨i, hxi : x ∈ u i, hmax : ∀ j, x ∈ u j → v i ≤ v j → v i = v j⟩
[GOAL]
case inr.intro.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
this : Nonempty (PartialRefinement u s)
v : ι → PartialRefinement u s
hvc : ∀ (x_1 : ι), x ∈ u x_1 → v x_1 ∈ c
hiv : ∀ (x_1 : ι), x ∈ u x_1 → x_1 ∈ (v x_1).carrier
i : ι
hxi : x ∈ u i
hmax : ∀ (j : ι), x ∈ u j → v i ≤ v j → v i = v j
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
rcases mem_iUnion.1 ((v i).subset_iUnion hxs) with ⟨j, hj⟩
[GOAL]
case inr.intro.intro.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
this : Nonempty (PartialRefinement u s)
v : ι → PartialRefinement u s
hvc : ∀ (x_1 : ι), x ∈ u x_1 → v x_1 ∈ c
hiv : ∀ (x_1 : ι), x ∈ u x_1 → x_1 ∈ (v x_1).carrier
i : ι
hxi : x ∈ u i
hmax : ∀ (j : ι), x ∈ u j → v i ≤ v j → v i = v j
j : ι
hj : x ∈ toFun (v i) j
⊢ ∃ i, x ∈ (fun i => toFun (find c ne i) i) i
[PROOFSTEP]
use j
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
this : Nonempty (PartialRefinement u s)
v : ι → PartialRefinement u s
hvc : ∀ (x_1 : ι), x ∈ u x_1 → v x_1 ∈ c
hiv : ∀ (x_1 : ι), x ∈ u x_1 → x_1 ∈ (v x_1).carrier
i : ι
hxi : x ∈ u i
hmax : ∀ (j : ι), x ∈ u j → v i ≤ v j → v i = v j
j : ι
hj : x ∈ toFun (v i) j
⊢ x ∈ (fun i => toFun (find c ne i) i) j
[PROOFSTEP]
have hj' : x ∈ u j := (v i).subset _ hj
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
this : Nonempty (PartialRefinement u s)
v : ι → PartialRefinement u s
hvc : ∀ (x_1 : ι), x ∈ u x_1 → v x_1 ∈ c
hiv : ∀ (x_1 : ι), x ∈ u x_1 → x_1 ∈ (v x_1).carrier
i : ι
hxi : x ∈ u i
hmax : ∀ (j : ι), x ∈ u j → v i ≤ v j → v i = v j
j : ι
hj : x ∈ toFun (v i) j
hj' : x ∈ u j
⊢ x ∈ (fun i => toFun (find c ne i) i) j
[PROOFSTEP]
have : v j ≤ v i := (hc.total (hvc _ hxi) (hvc _ hj')).elim (fun h => (hmax j hj' h).ge) id
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
c : Set (PartialRefinement u s)
hc : IsChain (fun x x_1 => x ≤ x_1) c
ne : Set.Nonempty c
hfin : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
hU : s ⊆ ⋃ (i : ι), u i
x : X
hxs : x ∈ s
this✝ : Nonempty (PartialRefinement u s)
v : ι → PartialRefinement u s
hvc : ∀ (x_1 : ι), x ∈ u x_1 → v x_1 ∈ c
hiv : ∀ (x_1 : ι), x ∈ u x_1 → x_1 ∈ (v x_1).carrier
i : ι
hxi : x ∈ u i
hmax : ∀ (j : ι), x ∈ u j → v i ≤ v j → v i = v j
j : ι
hj : x ∈ toFun (v i) j
hj' : x ∈ u j
this : v j ≤ v i
⊢ x ∈ (fun i => toFun (find c ne i) i) j
[PROOFSTEP]
simpa only [find_apply_of_mem hc ne (hvc _ hxi) (this.1 <| hiv _ hj')]
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
⊢ ∃ v', v < v'
[PROOFSTEP]
have I : (s ∩ ⋂ (j) (_ : j ≠ i), (v j)ᶜ) ⊆ v i :=
by
simp only [subset_def, mem_inter_iff, mem_iInter, and_imp]
intro x hxs H
rcases mem_iUnion.1 (v.subset_iUnion hxs) with ⟨j, hj⟩
exact (em (j = i)).elim (fun h => h ▸ hj) fun h => (H j h hj).elim
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
⊢ s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
[PROOFSTEP]
simp only [subset_def, mem_inter_iff, mem_iInter, and_imp]
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
⊢ ∀ (x : X), x ∈ s → (∀ (i_1 : ι), i_1 ≠ i → x ∈ (toFun v i_1)ᶜ) → x ∈ toFun v i
[PROOFSTEP]
intro x hxs H
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
x : X
hxs : x ∈ s
H : ∀ (i_1 : ι), i_1 ≠ i → x ∈ (toFun v i_1)ᶜ
⊢ x ∈ toFun v i
[PROOFSTEP]
rcases mem_iUnion.1 (v.subset_iUnion hxs) with ⟨j, hj⟩
[GOAL]
case intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
x : X
hxs : x ∈ s
H : ∀ (i_1 : ι), i_1 ≠ i → x ∈ (toFun v i_1)ᶜ
j : ι
hj : x ∈ toFun v j
⊢ x ∈ toFun v i
[PROOFSTEP]
exact (em (j = i)).elim (fun h => h ▸ hj) fun h => (H j h hj).elim
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
⊢ ∃ v', v < v'
[PROOFSTEP]
have C : IsClosed (s ∩ ⋂ (j) (_ : j ≠ i), (v j)ᶜ) :=
IsClosed.inter hs (isClosed_biInter fun _ _ => isClosed_compl_iff.2 <| v.isOpen _)
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
⊢ ∃ v', v < v'
[PROOFSTEP]
rcases normal_exists_closure_subset C (v.isOpen i) I with ⟨vi, ovi, hvi, cvi⟩
[GOAL]
case intro.intro.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ ∃ v', v < v'
[PROOFSTEP]
refine' ⟨⟨update v i vi, insert i v.carrier, _, _, _, _⟩, _, _⟩
[GOAL]
case intro.intro.intro.refine'_1
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ ∀ (i_1 : ι), IsOpen (update v.toFun i vi i_1)
[PROOFSTEP]
intro j
[GOAL]
case intro.intro.intro.refine'_1
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
⊢ IsOpen (update v.toFun i vi j)
[PROOFSTEP]
rcases eq_or_ne j i with (rfl | hne)
[GOAL]
case intro.intro.intro.refine'_1.inl
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
vi : Set X
ovi : IsOpen vi
j : ι
hi : ¬j ∈ v.carrier
I : s ∩ ⋂ (j_1 : ι) (_ : j_1 ≠ j), (toFun v j_1)ᶜ ⊆ toFun v j
C : IsClosed (s ∩ ⋂ (j_1 : ι) (_ : j_1 ≠ j), (toFun v j_1)ᶜ)
hvi : s ∩ ⋂ (j_1 : ι) (_ : j_1 ≠ j), (toFun v j_1)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v j
⊢ IsOpen (update v.toFun j vi j)
[PROOFSTEP]
simp [*, v.isOpen]
[GOAL]
case intro.intro.intro.refine'_1.inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
hne : j ≠ i
⊢ IsOpen (update v.toFun i vi j)
[PROOFSTEP]
simp [*, v.isOpen]
[GOAL]
case intro.intro.intro.refine'_2
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ s ⊆ ⋃ (i_1 : ι), update v.toFun i vi i_1
[PROOFSTEP]
refine' fun x hx => mem_iUnion.2 _
[GOAL]
case intro.intro.intro.refine'_2
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
⊢ ∃ i_1, x ∈ update v.toFun i vi i_1
[PROOFSTEP]
rcases em (∃ (j : _) (_ : j ≠ i), x ∈ v j) with (⟨j, hji, hj⟩ | h)
[GOAL]
case intro.intro.intro.refine'_2.inl.intro.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
j : ι
hji : j ≠ i
hj : x ∈ toFun v j
⊢ ∃ i_1, x ∈ update v.toFun i vi i_1
[PROOFSTEP]
use j
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
j : ι
hji : j ≠ i
hj : x ∈ toFun v j
⊢ x ∈ update v.toFun i vi j
[PROOFSTEP]
rwa [update_noteq hji]
[GOAL]
case intro.intro.intro.refine'_2.inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
h : ¬∃ j x_1, x ∈ toFun v j
⊢ ∃ i_1, x ∈ update v.toFun i vi i_1
[PROOFSTEP]
push_neg at h
[GOAL]
case intro.intro.intro.refine'_2.inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
h : ∀ (j : ι), j ≠ i → ¬x ∈ toFun v j
⊢ ∃ i_1, x ∈ update v.toFun i vi i_1
[PROOFSTEP]
use i
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
h : ∀ (j : ι), j ≠ i → ¬x ∈ toFun v j
⊢ x ∈ update v.toFun i vi i
[PROOFSTEP]
rw [update_same]
[GOAL]
case h
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
x : X
hx : x ∈ s
h : ∀ (j : ι), j ≠ i → ¬x ∈ toFun v j
⊢ x ∈ vi
[PROOFSTEP]
exact hvi ⟨hx, mem_biInter h⟩
[GOAL]
case intro.intro.intro.refine'_3
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ ∀ {i_1 : ι}, i_1 ∈ insert i v.carrier → closure (update v.toFun i vi i_1) ⊆ u i_1
[PROOFSTEP]
rintro j (rfl | hj)
[GOAL]
case intro.intro.intro.refine'_3.inl
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
vi : Set X
ovi : IsOpen vi
j : ι
hi : ¬j ∈ v.carrier
I : s ∩ ⋂ (j_1 : ι) (_ : j_1 ≠ j), (toFun v j_1)ᶜ ⊆ toFun v j
C : IsClosed (s ∩ ⋂ (j_1 : ι) (_ : j_1 ≠ j), (toFun v j_1)ᶜ)
hvi : s ∩ ⋂ (j_1 : ι) (_ : j_1 ≠ j), (toFun v j_1)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v j
⊢ closure (update v.toFun j vi j) ⊆ u j
[PROOFSTEP]
rwa [update_same, ← v.apply_eq hi]
[GOAL]
case intro.intro.intro.refine'_3.inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
hj : j ∈ v.carrier
⊢ closure (update v.toFun i vi j) ⊆ u j
[PROOFSTEP]
rw [update_noteq (ne_of_mem_of_not_mem hj hi)]
[GOAL]
case intro.intro.intro.refine'_3.inr
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
hj : j ∈ v.carrier
⊢ closure (toFun v j) ⊆ u j
[PROOFSTEP]
exact v.closure_subset hj
[GOAL]
case intro.intro.intro.refine'_4
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ ∀ {i_1 : ι}, ¬i_1 ∈ insert i v.carrier → update v.toFun i vi i_1 = u i_1
[PROOFSTEP]
intro j hj
[GOAL]
case intro.intro.intro.refine'_4
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
hj : ¬j ∈ insert i v.carrier
⊢ update v.toFun i vi j = u j
[PROOFSTEP]
rw [mem_insert_iff, not_or] at hj
[GOAL]
case intro.intro.intro.refine'_4
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
hj : ¬j = i ∧ ¬j ∈ v.carrier
⊢ update v.toFun i vi j = u j
[PROOFSTEP]
rw [update_noteq hj.1, v.apply_eq hj.2]
[GOAL]
case intro.intro.intro.refine'_5
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ v.carrier ⊆
{ toFun := update v.toFun i vi, carrier := insert i v.carrier,
isOpen := (_ : ∀ (j : ι), IsOpen (update v.toFun i vi j)),
subset_iUnion := (_ : ∀ (x : X), x ∈ s → x ∈ ⋃ (i_1 : ι), update v.toFun i vi i_1),
closure_subset := (_ : ∀ {j : ι}, j ∈ insert i v.carrier → closure (update v.toFun i vi j) ⊆ u j),
apply_eq := (_ : ∀ {j : ι}, ¬j ∈ insert i v.carrier → update v.toFun i vi j = u j) }.carrier ∧
∀ (i_1 : ι),
i_1 ∈ v.carrier →
toFun v i_1 =
toFun
{ toFun := update v.toFun i vi, carrier := insert i v.carrier,
isOpen := (_ : ∀ (j : ι), IsOpen (update v.toFun i vi j)),
subset_iUnion := (_ : ∀ (x : X), x ∈ s → x ∈ ⋃ (i_2 : ι), update v.toFun i vi i_2),
closure_subset := (_ : ∀ {j : ι}, j ∈ insert i v.carrier → closure (update v.toFun i vi j) ⊆ u j),
apply_eq := (_ : ∀ {j : ι}, ¬j ∈ insert i v.carrier → update v.toFun i vi j = u j) }
i_1
[PROOFSTEP]
refine' ⟨subset_insert _ _, fun j hj => _⟩
[GOAL]
case intro.intro.intro.refine'_5
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
j : ι
hj : j ∈ v.carrier
⊢ toFun v j =
toFun
{ toFun := update v.toFun i vi, carrier := insert i v.carrier,
isOpen := (_ : ∀ (j : ι), IsOpen (update v.toFun i vi j)),
subset_iUnion := (_ : ∀ (x : X), x ∈ s → x ∈ ⋃ (i_1 : ι), update v.toFun i vi i_1),
closure_subset := (_ : ∀ {j : ι}, j ∈ insert i v.carrier → closure (update v.toFun i vi j) ⊆ u j),
apply_eq := (_ : ∀ {j : ι}, ¬j ∈ insert i v.carrier → update v.toFun i vi j = u j) }
j
[PROOFSTEP]
exact (update_noteq (ne_of_mem_of_not_mem hj hi) _ _).symm
[GOAL]
case intro.intro.intro.refine'_6
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
v : PartialRefinement u s
hs : IsClosed s
i : ι
hi : ¬i ∈ v.carrier
I : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ toFun v i
C : IsClosed (s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ)
vi : Set X
ovi : IsOpen vi
hvi : s ∩ ⋂ (j : ι) (_ : j ≠ i), (toFun v j)ᶜ ⊆ vi
cvi : closure vi ⊆ toFun v i
⊢ ¬({ toFun := update v.toFun i vi, carrier := insert i v.carrier,
isOpen := (_ : ∀ (j : ι), IsOpen (update v.toFun i vi j)),
subset_iUnion := (_ : ∀ (x : X), x ∈ s → x ∈ ⋃ (i_1 : ι), update v.toFun i vi i_1),
closure_subset := (_ : ∀ {j : ι}, j ∈ insert i v.carrier → closure (update v.toFun i vi j) ⊆ u j),
apply_eq := (_ : ∀ {j : ι}, ¬j ∈ insert i v.carrier → update v.toFun i vi j = u j) }.carrier ⊆
v.carrier ∧
∀ (i_1 : ι),
i_1 ∈
{ toFun := update v.toFun i vi, carrier := insert i v.carrier,
isOpen := (_ : ∀ (j : ι), IsOpen (update v.toFun i vi j)),
subset_iUnion := (_ : ∀ (x : X), x ∈ s → x ∈ ⋃ (i_2 : ι), update v.toFun i vi i_2),
closure_subset := (_ : ∀ {j : ι}, j ∈ insert i v.carrier → closure (update v.toFun i vi j) ⊆ u j),
apply_eq := (_ : ∀ {j : ι}, ¬j ∈ insert i v.carrier → update v.toFun i vi j = u j) }.carrier →
toFun
{ toFun := update v.toFun i vi, carrier := insert i v.carrier,
isOpen := (_ : ∀ (j : ι), IsOpen (update v.toFun i vi j)),
subset_iUnion := (_ : ∀ (x : X), x ∈ s → x ∈ ⋃ (i_2 : ι), update v.toFun i vi i_2),
closure_subset := (_ : ∀ {j : ι}, j ∈ insert i v.carrier → closure (update v.toFun i vi j) ⊆ u j),
apply_eq := (_ : ∀ {j : ι}, ¬j ∈ insert i v.carrier → update v.toFun i vi j = u j) }
i_1 =
toFun v i_1)
[PROOFSTEP]
exact fun hle => hi (hle.1 <| mem_insert _ _)
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
⊢ ∃ v, s ⊆ iUnion v ∧ (∀ (i : ι), IsOpen (v i)) ∧ ∀ (i : ι), closure (v i) ⊆ u i
[PROOFSTEP]
haveI : Nonempty (PartialRefinement u s) := ⟨⟨u, ∅, uo, us, False.elim, fun _ => rfl⟩⟩
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this : Nonempty (PartialRefinement u s)
⊢ ∃ v, s ⊆ iUnion v ∧ (∀ (i : ι), IsOpen (v i)) ∧ ∀ (i : ι), closure (v i) ⊆ u i
[PROOFSTEP]
have : ∀ c : Set (PartialRefinement u s), IsChain (· ≤ ·) c → c.Nonempty → ∃ ub, ∀ v ∈ c, v ≤ ub := fun c hc ne =>
⟨.chainSup c hc ne uf us, fun v hv => PartialRefinement.le_chainSup _ _ _ _ hv⟩
[GOAL]
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
⊢ ∃ v, s ⊆ iUnion v ∧ (∀ (i : ι), IsOpen (v i)) ∧ ∀ (i : ι), closure (v i) ⊆ u i
[PROOFSTEP]
rcases zorn_nonempty_partialOrder this with ⟨v, hv⟩
[GOAL]
case intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
hv : ∀ (a : PartialRefinement u s), v ≤ a → a = v
⊢ ∃ v, s ⊆ iUnion v ∧ (∀ (i : ι), IsOpen (v i)) ∧ ∀ (i : ι), closure (v i) ⊆ u i
[PROOFSTEP]
suffices : ∀ i, i ∈ v.carrier
[GOAL]
case intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝¹ : Nonempty (PartialRefinement u s)
this✝ :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
hv : ∀ (a : PartialRefinement u s), v ≤ a → a = v
this : ∀ (i : ι), i ∈ v.carrier
⊢ ∃ v, s ⊆ iUnion v ∧ (∀ (i : ι), IsOpen (v i)) ∧ ∀ (i : ι), closure (v i) ⊆ u i
case this
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
hv : ∀ (a : PartialRefinement u s), v ≤ a → a = v
⊢ ∀ (i : ι), i ∈ v.carrier
[PROOFSTEP]
exact ⟨v, v.subset_iUnion, fun i => v.isOpen _, fun i => v.closure_subset (this i)⟩
[GOAL]
case this
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
hv : ∀ (a : PartialRefinement u s), v ≤ a → a = v
⊢ ∀ (i : ι), i ∈ v.carrier
[PROOFSTEP]
contrapose! hv
[GOAL]
case this
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
hv : ∃ i, ¬i ∈ v.carrier
⊢ ∃ a, v ≤ a ∧ a ≠ v
[PROOFSTEP]
rcases hv with ⟨i, hi⟩
[GOAL]
case this.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
i : ι
hi : ¬i ∈ v.carrier
⊢ ∃ a, v ≤ a ∧ a ≠ v
[PROOFSTEP]
rcases v.exists_gt hs i hi with ⟨v', hlt⟩
[GOAL]
case this.intro.intro
ι : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
u : ι → Set X
s : Set X
hs : IsClosed s
uo : ∀ (i : ι), IsOpen (u i)
uf : ∀ (x : X), x ∈ s → Set.Finite {i | x ∈ u i}
us : s ⊆ ⋃ (i : ι), u i
this✝ : Nonempty (PartialRefinement u s)
this :
∀ (c : Set (PartialRefinement u s)),
IsChain (fun x x_1 => x ≤ x_1) c → Set.Nonempty c → ∃ ub, ∀ (v : PartialRefinement u s), v ∈ c → v ≤ ub
v : PartialRefinement u s
i : ι
hi : ¬i ∈ v.carrier
v' : PartialRefinement u s
hlt : v < v'
⊢ ∃ a, v ≤ a ∧ a ≠ v
[PROOFSTEP]
exact ⟨v', hlt.le, hlt.ne'⟩
| {"mathlib_filename": "Mathlib.Topology.ShrinkingLemma", "llama_tokens": 17167} |
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
A : GL n R
⊢ Matrix.det ↑A * Matrix.det ↑A⁻¹ = 1
[PROOFSTEP]
rw [← det_mul, A.mul_inv, det_one]
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
A : GL n R
⊢ Matrix.det ↑A⁻¹ * Matrix.det ↑A = 1
[PROOFSTEP]
rw [← det_mul, A.inv_mul, det_one]
[GOAL]
n : Type u
R : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrderedCommRing R
inst✝ : Fact (Even (Fintype.card n))
g : { x // x ∈ GLPos n R }
⊢ -↑g ∈ GLPos n R
[PROOFSTEP]
rw [mem_glpos, GeneralLinearGroup.det_apply_val, Units.val_neg, det_neg,
(Fact.out (p := Even <| Fintype.card n)).neg_one_pow, one_mul]
[GOAL]
n : Type u
R : Type v
inst✝³ : DecidableEq n
inst✝² : Fintype n
inst✝¹ : LinearOrderedCommRing R
inst✝ : Fact (Even (Fintype.card n))
g : { x // x ∈ GLPos n R }
⊢ 0 < det ↑↑g
[PROOFSTEP]
exact g.prop
[GOAL]
R : Type ?u.1604470
inst✝ : Field R
a b : R
hab : a ^ 2 + b ^ 2 ≠ 0
⊢ det (↑of ![![a, -b], ![b, a]]) ≠ 0
[PROOFSTEP]
simpa [det_fin_two, sq] using hab
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.GeneralLinearGroup", "llama_tokens": 557} |
[GOAL]
E : Type u_1
X : Type u_2
inst✝² : TopologicalSpace E
inst✝¹ : TopologicalSpace X
f : E → X
s : Set X
x : E
I : Type u_3
inst✝ : TopologicalSpace I
h✝ : IsEvenlyCovered f (f x) I
e : Trivialization I f := Classical.choose (_ : ∃ t, f x ∈ t.baseSet)
h : f x ∈ (Classical.choose (_ : ∃ t, f x ∈ t.baseSet)).baseSet := Classical.choose_spec h✝.right
he : (f x, (↑e x).snd) = ↑e x := Trivialization.mk_proj_snd' e h
⊢ (f x, (↑e x).snd) ∈ e.target
[PROOFSTEP]
rwa [he, e.mem_target, e.coe_fst (e.mem_source.mpr h)]
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
hf : IsCoveringMapOn f s
⊢ IsLocallyHomeomorphOn f (f ⁻¹' s)
[PROOFSTEP]
refine' IsLocallyHomeomorphOn.mk f (f ⁻¹' s) fun x hx => _
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
hf : IsCoveringMapOn f s
x : E
hx : x ∈ f ⁻¹' s
⊢ ∃ e, x ∈ e.source ∧ ∀ (y : E), y ∈ e.source → f y = ↑e y
[PROOFSTEP]
let e := (hf (f x) hx).toTrivialization
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
hf : IsCoveringMapOn f s
x : E
hx : x ∈ f ⁻¹' s
e : Trivialization (↑(f ⁻¹' {f x})) f := IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))
⊢ ∃ e, x ∈ e.source ∧ ∀ (y : E), y ∈ e.source → f y = ↑e y
[PROOFSTEP]
have h := (hf (f x) hx).mem_toTrivialization_baseSet
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
hf : IsCoveringMapOn f s
x : E
hx : x ∈ f ⁻¹' s
e : Trivialization (↑(f ⁻¹' {f x})) f := IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))
h : f x ∈ (IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))).baseSet
⊢ ∃ e, x ∈ e.source ∧ ∀ (y : E), y ∈ e.source → f y = ↑e y
[PROOFSTEP]
let he := e.mem_source.2 h
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
hf : IsCoveringMapOn f s
x : E
hx : x ∈ f ⁻¹' s
e : Trivialization (↑(f ⁻¹' {f x})) f := IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))
h : f x ∈ (IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))).baseSet
he : x ∈ e.source := Iff.mpr (Trivialization.mem_source e) h
⊢ ∃ e, x ∈ e.source ∧ ∀ (y : E), y ∈ e.source → f y = ↑e y
[PROOFSTEP]
refine'
⟨e.toLocalHomeomorph.trans
{ toFun := fun p => p.1
invFun := fun p => ⟨p, x, rfl⟩
source := e.baseSet ×ˢ ({⟨x, rfl⟩} : Set (f ⁻¹' {f x}))
target := e.baseSet
open_source := e.open_baseSet.prod (singletons_open_iff_discrete.2 (hf (f x) hx).1 ⟨x, rfl⟩)
open_target := e.open_baseSet
map_source' := fun p => And.left
map_target' := fun p hp => ⟨hp, rfl⟩
left_inv' := fun p hp => Prod.ext rfl hp.2.symm
right_inv' := fun p _ => rfl
continuous_toFun := continuous_fst.continuousOn
continuous_invFun := (continuous_id'.prod_mk continuous_const).continuousOn },
⟨he, by rwa [e.toLocalHomeomorph.symm_symm, e.proj_toFun x he], (hf (f x) hx).toTrivialization_apply⟩, fun p h =>
(e.proj_toFun p h.1).symm⟩
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
hf : IsCoveringMapOn f s
x : E
hx : x ∈ f ⁻¹' s
e : Trivialization (↑(f ⁻¹' {f x})) f := IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))
h : f x ∈ (IsEvenlyCovered.toTrivialization (_ : IsEvenlyCovered f (f x) ↑(f ⁻¹' {f x}))).baseSet
he : x ∈ e.source := Iff.mpr (Trivialization.mem_source e) h
⊢ (↑(LocalHomeomorph.symm (LocalHomeomorph.symm e.toLocalHomeomorph)) x).fst ∈ e.baseSet
[PROOFSTEP]
rwa [e.toLocalHomeomorph.symm_symm, e.proj_toFun x he]
[GOAL]
E : Type u_1
X : Type u_2
inst✝¹ : TopologicalSpace E
inst✝ : TopologicalSpace X
f : E → X
s : Set X
⊢ IsCoveringMap f ↔ IsCoveringMapOn f Set.univ
[PROOFSTEP]
simp only [IsCoveringMap, IsCoveringMapOn, Set.mem_univ, forall_true_left]
| {"mathlib_filename": "Mathlib.Topology.Covering", "llama_tokens": 1915} |
[GOAL]
ι : Type u
X : Type v
inst✝⁴ : TopologicalSpace X
E : Type u_1
inst✝³ : AddCommMonoid E
inst✝² : SMulWithZero ℝ E
inst✝¹ : TopologicalSpace E
inst✝ : ContinuousSMul ℝ E
s : Set X
f✝ f g : PartitionOfUnity ι X s
h : f.toFun = g.toFun
⊢ f = g
[PROOFSTEP]
cases f
[GOAL]
case mk
ι : Type u
X : Type v
inst✝⁴ : TopologicalSpace X
E : Type u_1
inst✝³ : AddCommMonoid E
inst✝² : SMulWithZero ℝ E
inst✝¹ : TopologicalSpace E
inst✝ : ContinuousSMul ℝ E
s : Set X
f g : PartitionOfUnity ι X s
toFun✝ : ι → C(X, ℝ)
locallyFinite'✝ : LocallyFinite fun i => support ↑(toFun✝ i)
nonneg'✝ : 0 ≤ toFun✝
sum_eq_one'✝ : ∀ (x : X), x ∈ s → ∑ᶠ (i : ι), ↑(toFun✝ i) x = 1
sum_le_one'✝ : ∀ (x : X), ∑ᶠ (i : ι), ↑(toFun✝ i) x ≤ 1
h : (mk s toFun✝ locallyFinite'✝ nonneg'✝ sum_eq_one'✝ sum_le_one'✝).toFun = g.toFun
⊢ mk s toFun✝ locallyFinite'✝ nonneg'✝ sum_eq_one'✝ sum_le_one'✝ = g
[PROOFSTEP]
cases g
[GOAL]
case mk.mk
ι : Type u
X : Type v
inst✝⁴ : TopologicalSpace X
E : Type u_1
inst✝³ : AddCommMonoid E
inst✝² : SMulWithZero ℝ E
inst✝¹ : TopologicalSpace E
inst✝ : ContinuousSMul ℝ E
s : Set X
f : PartitionOfUnity ι X s
toFun✝¹ : ι → C(X, ℝ)
locallyFinite'✝¹ : LocallyFinite fun i => support ↑(toFun✝¹ i)
nonneg'✝¹ : 0 ≤ toFun✝¹
sum_eq_one'✝¹ : ∀ (x : X), x ∈ s → ∑ᶠ (i : ι), ↑(toFun✝¹ i) x = 1
sum_le_one'✝¹ : ∀ (x : X), ∑ᶠ (i : ι), ↑(toFun✝¹ i) x ≤ 1
toFun✝ : ι → C(X, ℝ)
locallyFinite'✝ : LocallyFinite fun i => support ↑(toFun✝ i)
nonneg'✝ : 0 ≤ toFun✝
sum_eq_one'✝ : ∀ (x : X), x ∈ s → ∑ᶠ (i : ι), ↑(toFun✝ i) x = 1
sum_le_one'✝ : ∀ (x : X), ∑ᶠ (i : ι), ↑(toFun✝ i) x ≤ 1
h :
(mk s toFun✝¹ locallyFinite'✝¹ nonneg'✝¹ sum_eq_one'✝¹ sum_le_one'✝¹).toFun =
(mk s toFun✝ locallyFinite'✝ nonneg'✝ sum_eq_one'✝ sum_le_one'✝).toFun
⊢ mk s toFun✝¹ locallyFinite'✝¹ nonneg'✝¹ sum_eq_one'✝¹ sum_le_one'✝¹ =
mk s toFun✝ locallyFinite'✝ nonneg'✝ sum_eq_one'✝ sum_le_one'✝
[PROOFSTEP]
congr
[GOAL]
ι : Type u
X : Type v
inst✝⁴ : TopologicalSpace X
E : Type u_1
inst✝³ : AddCommMonoid E
inst✝² : SMulWithZero ℝ E
inst✝¹ : TopologicalSpace E
inst✝ : ContinuousSMul ℝ E
s : Set X
f : PartitionOfUnity ι X s
x : X
hx : x ∈ s
⊢ ∃ i, 0 < ↑(↑f i) x
[PROOFSTEP]
have H := f.sum_eq_one hx
[GOAL]
ι : Type u
X : Type v
inst✝⁴ : TopologicalSpace X
E : Type u_1
inst✝³ : AddCommMonoid E
inst✝² : SMulWithZero ℝ E
inst✝¹ : TopologicalSpace E
inst✝ : ContinuousSMul ℝ E
s : Set X
f : PartitionOfUnity ι X s
x : X
hx : x ∈ s
H : ∑ᶠ (i : ι), ↑(↑f i) x = 1
⊢ ∃ i, 0 < ↑(↑f i) x
[PROOFSTEP]
contrapose! H
[GOAL]
ι : Type u
X : Type v
inst✝⁴ : TopologicalSpace X
E : Type u_1
inst✝³ : AddCommMonoid E
inst✝² : SMulWithZero ℝ E
inst✝¹ : TopologicalSpace E
inst✝ : ContinuousSMul ℝ E
s : Set X
f : PartitionOfUnity ι X s
x : X
hx : x ∈ s
H : ∀ (i : ι), ↑(↑f i) x ≤ 0
⊢ ∑ᶠ (i : ι), ↑(↑f i) x ≠ 1
[PROOFSTEP]
simpa only [fun i => (H i).antisymm (f.nonneg i x), finsum_zero] using zero_ne_one
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f✝ f g : BumpCovering ι X s
h : f.toFun = g.toFun
⊢ f = g
[PROOFSTEP]
cases f
[GOAL]
case mk
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f g : BumpCovering ι X s
toFun✝ : ι → C(X, ℝ)
locallyFinite'✝ : LocallyFinite fun i => support ↑(toFun✝ i)
nonneg'✝ : 0 ≤ toFun✝
le_one'✝ : toFun✝ ≤ 1
eventuallyEq_one'✝ : ∀ (x : X), x ∈ s → ∃ i, ↑(toFun✝ i) =ᶠ[𝓝 x] 1
h : (mk s toFun✝ locallyFinite'✝ nonneg'✝ le_one'✝ eventuallyEq_one'✝).toFun = g.toFun
⊢ mk s toFun✝ locallyFinite'✝ nonneg'✝ le_one'✝ eventuallyEq_one'✝ = g
[PROOFSTEP]
cases g
[GOAL]
case mk.mk
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
toFun✝¹ : ι → C(X, ℝ)
locallyFinite'✝¹ : LocallyFinite fun i => support ↑(toFun✝¹ i)
nonneg'✝¹ : 0 ≤ toFun✝¹
le_one'✝¹ : toFun✝¹ ≤ 1
eventuallyEq_one'✝¹ : ∀ (x : X), x ∈ s → ∃ i, ↑(toFun✝¹ i) =ᶠ[𝓝 x] 1
toFun✝ : ι → C(X, ℝ)
locallyFinite'✝ : LocallyFinite fun i => support ↑(toFun✝ i)
nonneg'✝ : 0 ≤ toFun✝
le_one'✝ : toFun✝ ≤ 1
eventuallyEq_one'✝ : ∀ (x : X), x ∈ s → ∃ i, ↑(toFun✝ i) =ᶠ[𝓝 x] 1
h :
(mk s toFun✝¹ locallyFinite'✝¹ nonneg'✝¹ le_one'✝¹ eventuallyEq_one'✝¹).toFun =
(mk s toFun✝ locallyFinite'✝ nonneg'✝ le_one'✝ eventuallyEq_one'✝).toFun
⊢ mk s toFun✝¹ locallyFinite'✝¹ nonneg'✝¹ le_one'✝¹ eventuallyEq_one'✝¹ =
mk s toFun✝ locallyFinite'✝ nonneg'✝ le_one'✝ eventuallyEq_one'✝
[PROOFSTEP]
congr
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
i : ι
s : Set X
x : X
⊢ ∃ t, t ∈ 𝓝 x ∧ Set.Finite {i_1 | Set.Nonempty ((fun i_2 => support ↑(Pi.single i 1 i_2)) i_1 ∩ t)}
[PROOFSTEP]
refine' ⟨univ, univ_mem, (finite_singleton i).subset _⟩
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
i : ι
s : Set X
x : X
⊢ {i_1 | Set.Nonempty ((fun i_2 => support ↑(Pi.single i 1 i_2)) i_1 ∩ univ)} ⊆ {i}
[PROOFSTEP]
rintro j ⟨x, hx, -⟩
[GOAL]
case intro.intro
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
i : ι
s : Set X
x✝ : X
j : ι
x : X
hx : x ∈ (fun i_1 => support ↑(Pi.single i 1 i_1)) j
⊢ j ∈ {i}
[PROOFSTEP]
contrapose! hx
[GOAL]
case intro.intro
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
i : ι
s : Set X
x✝ : X
j : ι
x : X
hx : ¬j ∈ {i}
⊢ ¬x ∈ support ↑(Pi.single i 1 j)
[PROOFSTEP]
rw [mem_singleton_iff] at hx
[GOAL]
case intro.intro
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
i : ι
s : Set X
x✝ : X
j : ι
x : X
hx : ¬j = i
⊢ ¬x ∈ support ↑(Pi.single i 1 j)
[PROOFSTEP]
simp [hx]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
i : ι
s : Set X
x : X
x✝ : x ∈ s
⊢ ↑(Pi.single i 1 i) =ᶠ[𝓝 x] 1
[PROOFSTEP]
rw [Pi.single_eq_same, ContinuousMap.coe_one]
[GOAL]
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
rcases exists_subset_iUnion_closure_subset hs ho (fun x _ => hf.point_finite x) hU with ⟨V, hsV, hVo, hVU⟩
[GOAL]
case intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
have hVU' : ∀ i, V i ⊆ U i := fun i => Subset.trans subset_closure (hVU i)
[GOAL]
case intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
hVU' : ∀ (i : ι), V i ⊆ U i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
rcases exists_subset_iUnion_closure_subset hs hVo (fun x _ => (hf.subset hVU').point_finite x) hsV with
⟨W, hsW, hWo, hWV⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
hVU' : ∀ (i : ι), V i ⊆ U i
W : ι → Set X
hsW : s ⊆ iUnion W
hWo : ∀ (i : ι), IsOpen (W i)
hWV : ∀ (i : ι), closure (W i) ⊆ V i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
choose f hfp hf0 hf1 hf01 using fun i =>
h01 _ _ (isClosed_compl_iff.2 <| hVo i) isClosed_closure (disjoint_right.2 fun x hx => Classical.not_not.2 (hWV i hx))
[GOAL]
case intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f✝ : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
hVU' : ∀ (i : ι), V i ⊆ U i
W : ι → Set X
hsW : s ⊆ iUnion W
hWo : ∀ (i : ι), IsOpen (W i)
hWV : ∀ (i : ι), closure (W i) ⊆ V i
f : ι → C(X, ℝ)
hfp : ∀ (i : ι), p ↑(f i)
hf0 : ∀ (i : ι), EqOn (↑(f i)) 0 (V i)ᶜ
hf1 : ∀ (i : ι), EqOn (↑(f i)) 1 (closure (W i))
hf01 : ∀ (i : ι) (x : X), ↑(f i) x ∈ Icc 0 1
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
have hsupp : ∀ i, support (f i) ⊆ V i := fun i => support_subset_iff'.2 (hf0 i)
[GOAL]
case intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f✝ : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
hVU' : ∀ (i : ι), V i ⊆ U i
W : ι → Set X
hsW : s ⊆ iUnion W
hWo : ∀ (i : ι), IsOpen (W i)
hWV : ∀ (i : ι), closure (W i) ⊆ V i
f : ι → C(X, ℝ)
hfp : ∀ (i : ι), p ↑(f i)
hf0 : ∀ (i : ι), EqOn (↑(f i)) 0 (V i)ᶜ
hf1 : ∀ (i : ι), EqOn (↑(f i)) 1 (closure (W i))
hf01 : ∀ (i : ι) (x : X), ↑(f i) x ∈ Icc 0 1
hsupp : ∀ (i : ι), support ↑(f i) ⊆ V i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
refine'
⟨⟨f, hf.subset fun i => Subset.trans (hsupp i) (hVU' i), fun i x => (hf01 i x).1, fun i x => (hf01 i x).2, fun x hx =>
_⟩,
hfp, fun i => Subset.trans (closure_mono (hsupp i)) (hVU i)⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f✝ : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
hVU' : ∀ (i : ι), V i ⊆ U i
W : ι → Set X
hsW : s ⊆ iUnion W
hWo : ∀ (i : ι), IsOpen (W i)
hWV : ∀ (i : ι), closure (W i) ⊆ V i
f : ι → C(X, ℝ)
hfp : ∀ (i : ι), p ↑(f i)
hf0 : ∀ (i : ι), EqOn (↑(f i)) 0 (V i)ᶜ
hf1 : ∀ (i : ι), EqOn (↑(f i)) 1 (closure (W i))
hf01 : ∀ (i : ι) (x : X), ↑(f i) x ∈ Icc 0 1
hsupp : ∀ (i : ι), support ↑(f i) ⊆ V i
x : X
hx : x ∈ s
⊢ ∃ i, ↑(f i) =ᶠ[𝓝 x] 1
[PROOFSTEP]
rcases mem_iUnion.1 (hsW hx) with ⟨i, hi⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝¹ : TopologicalSpace X
s : Set X
f✝ : BumpCovering ι X s
inst✝ : NormalSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hf : LocallyFinite U
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hsV : s ⊆ iUnion V
hVo : ∀ (i : ι), IsOpen (V i)
hVU : ∀ (i : ι), closure (V i) ⊆ U i
hVU' : ∀ (i : ι), V i ⊆ U i
W : ι → Set X
hsW : s ⊆ iUnion W
hWo : ∀ (i : ι), IsOpen (W i)
hWV : ∀ (i : ι), closure (W i) ⊆ V i
f : ι → C(X, ℝ)
hfp : ∀ (i : ι), p ↑(f i)
hf0 : ∀ (i : ι), EqOn (↑(f i)) 0 (V i)ᶜ
hf1 : ∀ (i : ι), EqOn (↑(f i)) 1 (closure (W i))
hf01 : ∀ (i : ι) (x : X), ↑(f i) x ∈ Icc 0 1
hsupp : ∀ (i : ι), support ↑(f i) ⊆ V i
x : X
hx : x ∈ s
i : ι
hi : x ∈ W i
⊢ ∃ i, ↑(f i) =ᶠ[𝓝 x] 1
[PROOFSTEP]
exact ⟨i, ((hf1 i).mono subset_closure).eventuallyEq_of_mem ((hWo i).mem_nhds hi)⟩
[GOAL]
ι : Type u
X : Type v
inst✝² : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝¹ : NormalSpace X
inst✝ : ParacompactSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hU : s ⊆ ⋃ (i : ι), U i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
rcases precise_refinement_set hs _ ho hU with ⟨V, hVo, hsV, hVf, hVU⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
inst✝² : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝¹ : NormalSpace X
inst✝ : ParacompactSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hVo : ∀ (i : ι), IsOpen (V i)
hsV : s ⊆ ⋃ (i : ι), V i
hVf : LocallyFinite V
hVU : ∀ (i : ι), V i ⊆ U i
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
rcases exists_isSubordinate_of_locallyFinite_of_prop p h01 hs V hVo hVf hsV with ⟨f, hfp, hf⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝² : TopologicalSpace X
s : Set X
f✝ : BumpCovering ι X s
inst✝¹ : NormalSpace X
inst✝ : ParacompactSpace X
p : (X → ℝ) → Prop
h01 :
∀ (s t : Set X),
IsClosed s → IsClosed t → Disjoint s t → ∃ f, p ↑f ∧ EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hVo : ∀ (i : ι), IsOpen (V i)
hsV : s ⊆ ⋃ (i : ι), V i
hVf : LocallyFinite V
hVU : ∀ (i : ι), V i ⊆ U i
f : BumpCovering ι X s
hfp : ∀ (i : ι), p ↑(↑f i)
hf : IsSubordinate f V
⊢ ∃ f, (∀ (i : ι), p ↑(↑f i)) ∧ IsSubordinate f U
[PROOFSTEP]
exact ⟨f, hfp, hf.mono hVU⟩
[GOAL]
ι : Type u
X : Type v
inst✝² : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝¹ : NormalSpace X
inst✝ : ParacompactSpace X
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hU : s ⊆ ⋃ (i : ι), U i
⊢ ∃ f, IsSubordinate f U
[PROOFSTEP]
rcases precise_refinement_set hs _ ho hU with ⟨V, hVo, hsV, hVf, hVU⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
inst✝² : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
inst✝¹ : NormalSpace X
inst✝ : ParacompactSpace X
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hVo : ∀ (i : ι), IsOpen (V i)
hsV : s ⊆ ⋃ (i : ι), V i
hVf : LocallyFinite V
hVU : ∀ (i : ι), V i ⊆ U i
⊢ ∃ f, IsSubordinate f U
[PROOFSTEP]
rcases exists_isSubordinate_of_locallyFinite hs V hVo hVf hsV with ⟨f, hf⟩
[GOAL]
case intro.intro.intro.intro.intro
ι : Type u
X : Type v
inst✝² : TopologicalSpace X
s : Set X
f✝ : BumpCovering ι X s
inst✝¹ : NormalSpace X
inst✝ : ParacompactSpace X
hs : IsClosed s
U : ι → Set X
ho : ∀ (i : ι), IsOpen (U i)
hU : s ⊆ ⋃ (i : ι), U i
V : ι → Set X
hVo : ∀ (i : ι), IsOpen (V i)
hsV : s ⊆ ⋃ (i : ι), V i
hVf : LocallyFinite V
hVU : ∀ (i : ι), V i ⊆ U i
f : BumpCovering ι X s
hf : IsSubordinate f V
⊢ ∃ f, IsSubordinate f U
[PROOFSTEP]
exact ⟨f, hf.mono hVU⟩
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
h : ↑(↑f i) x = 0
⊢ toPOUFun f i x = 0
[PROOFSTEP]
rw [toPOUFun, h, zero_mul]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
t : Finset ι
ht : ∀ (j : ι), WellOrderingRel j i → ↑(↑f j) x ≠ 0 → j ∈ t
⊢ toPOUFun f i x = ↑(↑f i) x * ∏ j in Finset.filter (fun j => WellOrderingRel j i) t, (1 - ↑(↑f j) x)
[PROOFSTEP]
refine' congr_arg _ (finprod_cond_eq_prod_of_cond_iff _ fun {j} hj => _)
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
t : Finset ι
ht : ∀ (j : ι), WellOrderingRel j i → ↑(↑f j) x ≠ 0 → j ∈ t
j : ι
hj : 1 - ↑(↑f j) x ≠ 1
⊢ WellOrderingRel j i ↔ j ∈ Finset.filter (fun j => WellOrderingRel j i) t
[PROOFSTEP]
rw [Ne.def, sub_eq_self] at hj
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
t : Finset ι
ht : ∀ (j : ι), WellOrderingRel j i → ↑(↑f j) x ≠ 0 → j ∈ t
j : ι
hj : ¬↑(↑f j) x = 0
⊢ WellOrderingRel j i ↔ j ∈ Finset.filter (fun j => WellOrderingRel j i) t
[PROOFSTEP]
rw [Finset.mem_filter, Iff.comm, and_iff_right_iff_imp]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
t : Finset ι
ht : ∀ (j : ι), WellOrderingRel j i → ↑(↑f j) x ≠ 0 → j ∈ t
j : ι
hj : ¬↑(↑f j) x = 0
⊢ WellOrderingRel j i → j ∈ t
[PROOFSTEP]
exact flip (ht j) hj
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
⊢ ∑ᶠ (i : ι), toPOUFun f i x = 1 - ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
set s := (f.point_finite x).toFinset
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
⊢ ∑ᶠ (i : ι), toPOUFun f i x = 1 - ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
have hs : (s : Set ι) = {i | f i x ≠ 0} := Finite.coe_toFinset _
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
⊢ ∑ᶠ (i : ι), toPOUFun f i x = 1 - ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
have A : (support fun i => toPOUFun f i x) ⊆ s := by
rw [hs]
exact fun i hi => f.support_toPOUFun_subset i hi
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
⊢ (support fun i => toPOUFun f i x) ⊆ ↑s
[PROOFSTEP]
rw [hs]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
⊢ (support fun i => toPOUFun f i x) ⊆ {i | ↑(↑f i) x ≠ 0}
[PROOFSTEP]
exact fun i hi => f.support_toPOUFun_subset i hi
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
⊢ ∑ᶠ (i : ι), toPOUFun f i x = 1 - ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
have B : (mulSupport fun i => 1 - f i x) ⊆ s :=
by
rw [hs, mulSupport_one_sub]
exact fun i => id
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
⊢ (mulSupport fun i => 1 - ↑(↑f i) x) ⊆ ↑s
[PROOFSTEP]
rw [hs, mulSupport_one_sub]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
⊢ (support fun i => ↑(↑f i) x) ⊆ {i | ↑(↑f i) x ≠ 0}
[PROOFSTEP]
exact fun i => id
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
B : (mulSupport fun i => 1 - ↑(↑f i) x) ⊆ ↑s
⊢ ∑ᶠ (i : ι), toPOUFun f i x = 1 - ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
letI : LinearOrder ι := linearOrderOfSTO WellOrderingRel
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
B : (mulSupport fun i => 1 - ↑(↑f i) x) ⊆ ↑s
this : LinearOrder ι := linearOrderOfSTO WellOrderingRel
⊢ ∑ᶠ (i : ι), toPOUFun f i x = 1 - ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
rw [finsum_eq_sum_of_support_subset _ A, finprod_eq_prod_of_mulSupport_subset _ B, Finset.prod_one_sub_ordered,
sub_sub_cancel]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
B : (mulSupport fun i => 1 - ↑(↑f i) x) ⊆ ↑s
this : LinearOrder ι := linearOrderOfSTO WellOrderingRel
⊢ ∑ i in s, toPOUFun f i x = ∑ i in s, ↑(↑f i) x * ∏ j in Finset.filter (fun x => x < i) s, (1 - ↑(↑f j) x)
[PROOFSTEP]
refine' Finset.sum_congr rfl fun i _ => _
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
B : (mulSupport fun i => 1 - ↑(↑f i) x) ⊆ ↑s
this : LinearOrder ι := linearOrderOfSTO WellOrderingRel
i : ι
x✝ : i ∈ s
⊢ toPOUFun f i x = ↑(↑f i) x * ∏ j in Finset.filter (fun x => x < i) s, (1 - ↑(↑f j) x)
[PROOFSTEP]
convert f.toPOUFun_eq_mul_prod _ _ _ fun j _ hj => _
[GOAL]
case convert_4
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s✝ : Set X
f : BumpCovering ι X s✝
x : X
s : Finset ι := Finite.toFinset (_ : Set.Finite {i | ↑(↑f i) x ≠ 0})
hs : ↑s = {i | ↑(↑f i) x ≠ 0}
A : (support fun i => toPOUFun f i x) ⊆ ↑s
B : (mulSupport fun i => 1 - ↑(↑f i) x) ⊆ ↑s
this : LinearOrder ι := linearOrderOfSTO WellOrderingRel
i : ι
x✝¹ : i ∈ s
j : ι
x✝ : WellOrderingRel j i
hj : ↑(↑f j) x ≠ 0
⊢ j ∈ s
[PROOFSTEP]
rwa [Finite.mem_toFinset]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
⊢ ∃ t, toPOUFun f i =ᶠ[𝓝 x] ↑(↑f i) * ↑(∏ j in Finset.filter (fun j => WellOrderingRel j i) t, (1 - ↑f j))
[PROOFSTEP]
rcases f.locallyFinite x with ⟨U, hU, hf⟩
[GOAL]
case intro.intro
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
U : Set X
hU : U ∈ 𝓝 x
hf : Set.Finite {i | Set.Nonempty ((fun i => support ↑(↑f i)) i ∩ U)}
⊢ ∃ t, toPOUFun f i =ᶠ[𝓝 x] ↑(↑f i) * ↑(∏ j in Finset.filter (fun j => WellOrderingRel j i) t, (1 - ↑f j))
[PROOFSTEP]
use hf.toFinset
[GOAL]
case h
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
U : Set X
hU : U ∈ 𝓝 x
hf : Set.Finite {i | Set.Nonempty ((fun i => support ↑(↑f i)) i ∩ U)}
⊢ toPOUFun f i =ᶠ[𝓝 x] ↑(↑f i) * ↑(∏ j in Finset.filter (fun j => WellOrderingRel j i) (Finite.toFinset hf), (1 - ↑f j))
[PROOFSTEP]
filter_upwards [hU] with y hyU
[GOAL]
case h
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
U : Set X
hU : U ∈ 𝓝 x
hf : Set.Finite {i | Set.Nonempty ((fun i => support ↑(↑f i)) i ∩ U)}
y : X
hyU : y ∈ U
⊢ toPOUFun f i y = (↑(↑f i) * ↑(∏ j in Finset.filter (fun j => WellOrderingRel j i) (Finite.toFinset hf), (1 - ↑f j))) y
[PROOFSTEP]
simp only [ContinuousMap.coe_prod, Pi.mul_apply, Finset.prod_apply]
[GOAL]
case h
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
U : Set X
hU : U ∈ 𝓝 x
hf : Set.Finite {i | Set.Nonempty ((fun i => support ↑(↑f i)) i ∩ U)}
y : X
hyU : y ∈ U
⊢ toPOUFun f i y = ↑(↑f i) y * ∏ c in Finset.filter (fun j => WellOrderingRel j i) (Finite.toFinset hf), ↑(1 - ↑f c) y
[PROOFSTEP]
apply toPOUFun_eq_mul_prod
[GOAL]
case h.ht
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
U : Set X
hU : U ∈ 𝓝 x
hf : Set.Finite {i | Set.Nonempty ((fun i => support ↑(↑f i)) i ∩ U)}
y : X
hyU : y ∈ U
⊢ ∀ (j : ι), WellOrderingRel j i → ↑(↑f j) y ≠ 0 → j ∈ Finite.toFinset hf
[PROOFSTEP]
intro j _ hj
[GOAL]
case h.ht
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
x : X
U : Set X
hU : U ∈ 𝓝 x
hf : Set.Finite {i | Set.Nonempty ((fun i => support ↑(↑f i)) i ∩ U)}
y : X
hyU : y ∈ U
j : ι
a✝ : WellOrderingRel j i
hj : ↑(↑f j) y ≠ 0
⊢ j ∈ Finite.toFinset hf
[PROOFSTEP]
exact hf.mem_toFinset.2 ⟨y, ⟨hj, hyU⟩⟩
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
⊢ Continuous (toPOUFun f i)
[PROOFSTEP]
refine' (f i).continuous.mul <| continuous_finprod_cond (fun j _ => continuous_const.sub (f j).continuous) _
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
⊢ LocallyFinite fun i => mulSupport fun x => 1 - ↑(↑f i) x
[PROOFSTEP]
simp only [mulSupport_one_sub]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
i : ι
⊢ LocallyFinite fun i => support fun x => ↑(↑f i) x
[PROOFSTEP]
exact f.locallyFinite
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
hx : x ∈ s
⊢ ∑ᶠ (i : ι), ↑((fun i => ContinuousMap.mk (toPOUFun f i)) i) x = 1
[PROOFSTEP]
simp only [ContinuousMap.coe_mk, sum_toPOUFun_eq, sub_eq_self]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
hx : x ∈ s
⊢ ∏ᶠ (i : ι), (1 - ↑(↑f i) x) = 0
[PROOFSTEP]
apply finprod_eq_zero (fun i => 1 - f i x) (f.ind x hx)
[GOAL]
case hx
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
hx : x ∈ s
⊢ 1 - ↑(↑f (ind f x hx)) x = 0
[PROOFSTEP]
simp only [f.ind_apply x hx, sub_self]
[GOAL]
case hf
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
hx : x ∈ s
⊢ Set.Finite (mulSupport fun i => 1 - ↑(↑f i) x)
[PROOFSTEP]
rw [mulSupport_one_sub]
[GOAL]
case hf
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
hx : x ∈ s
⊢ Set.Finite (support fun i => ↑(↑f i) x)
[PROOFSTEP]
exact f.point_finite x
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
⊢ ∑ᶠ (i : ι), ↑((fun i => ContinuousMap.mk (toPOUFun f i)) i) x ≤ 1
[PROOFSTEP]
simp only [ContinuousMap.coe_mk, sum_toPOUFun_eq, sub_le_self_iff]
[GOAL]
ι : Type u
X : Type v
inst✝ : TopologicalSpace X
s : Set X
f : BumpCovering ι X s
x : X
⊢ 0 ≤ ∏ᶠ (i : ι), (1 - ↑(↑f i) x)
[PROOFSTEP]
exact finprod_nonneg fun i => sub_nonneg.2 <| f.le_one i x
| {"mathlib_filename": "Mathlib.Topology.PartitionOfUnity", "llama_tokens": 14672} |
[GOAL]
t : ℝ
⊢ t ∈ I ↔ 1 - t ∈ I
[PROOFSTEP]
rw [mem_Icc, mem_Icc]
[GOAL]
t : ℝ
⊢ 0 ≤ t ∧ t ≤ 1 ↔ 0 ≤ 1 - t ∧ 1 - t ≤ 1
[PROOFSTEP]
constructor
[GOAL]
case mp
t : ℝ
⊢ 0 ≤ t ∧ t ≤ 1 → 0 ≤ 1 - t ∧ 1 - t ≤ 1
[PROOFSTEP]
intro
[GOAL]
case mpr
t : ℝ
⊢ 0 ≤ 1 - t ∧ 1 - t ≤ 1 → 0 ≤ t ∧ t ≤ 1
[PROOFSTEP]
intro
[GOAL]
case mp
t : ℝ
a✝ : 0 ≤ t ∧ t ≤ 1
⊢ 0 ≤ 1 - t ∧ 1 - t ≤ 1
[PROOFSTEP]
constructor
[GOAL]
case mpr
t : ℝ
a✝ : 0 ≤ 1 - t ∧ 1 - t ≤ 1
⊢ 0 ≤ t ∧ t ≤ 1
[PROOFSTEP]
constructor
[GOAL]
case mp.left
t : ℝ
a✝ : 0 ≤ t ∧ t ≤ 1
⊢ 0 ≤ 1 - t
[PROOFSTEP]
linarith
[GOAL]
case mp.right
t : ℝ
a✝ : 0 ≤ t ∧ t ≤ 1
⊢ 1 - t ≤ 1
[PROOFSTEP]
linarith
[GOAL]
case mpr.left
t : ℝ
a✝ : 0 ≤ 1 - t ∧ 1 - t ≤ 1
⊢ 0 ≤ t
[PROOFSTEP]
linarith
[GOAL]
case mpr.right
t : ℝ
a✝ : 0 ≤ 1 - t ∧ 1 - t ≤ 1
⊢ t ≤ 1
[PROOFSTEP]
linarith
[GOAL]
⊢ 1 ∈ I
[PROOFSTEP]
constructor
[GOAL]
case left
⊢ 0 ≤ 1
[PROOFSTEP]
norm_num
[GOAL]
case right
⊢ 1 ≤ 1
[PROOFSTEP]
norm_num
[GOAL]
⊢ ↑(σ 0) = ↑1
[PROOFSTEP]
simp [symm]
[GOAL]
⊢ ↑(σ 1) = ↑0
[PROOFSTEP]
simp [symm]
[GOAL]
x : ↑I
⊢ ↑(σ (σ x)) = ↑x
[PROOFSTEP]
simp [symm]
[GOAL]
⊢ CompactSpace ↑I
[PROOFSTEP]
infer_instance
[GOAL]
x : ↑I
⊢ 0 ≤ 1 - ↑x
[PROOFSTEP]
simpa using x.2.2
[GOAL]
x : ↑I
⊢ 1 - ↑x ≤ 1
[PROOFSTEP]
simpa using x.2.1
[GOAL]
a t : ℝ
ha : 0 < a
⊢ a * t ∈ I ↔ t ∈ Icc 0 (1 / a)
[PROOFSTEP]
constructor
[GOAL]
case mp
a t : ℝ
ha : 0 < a
⊢ a * t ∈ I → t ∈ Icc 0 (1 / a)
[PROOFSTEP]
rintro ⟨h₁, h₂⟩
[GOAL]
case mpr
a t : ℝ
ha : 0 < a
⊢ t ∈ Icc 0 (1 / a) → a * t ∈ I
[PROOFSTEP]
rintro ⟨h₁, h₂⟩
[GOAL]
case mp.intro
a t : ℝ
ha : 0 < a
h₁ : 0 ≤ a * t
h₂ : a * t ≤ 1
⊢ t ∈ Icc 0 (1 / a)
[PROOFSTEP]
constructor
[GOAL]
case mpr.intro
a t : ℝ
ha : 0 < a
h₁ : 0 ≤ t
h₂ : t ≤ 1 / a
⊢ a * t ∈ I
[PROOFSTEP]
constructor
[GOAL]
case mp.intro.left
a t : ℝ
ha : 0 < a
h₁ : 0 ≤ a * t
h₂ : a * t ≤ 1
⊢ 0 ≤ t
[PROOFSTEP]
exact nonneg_of_mul_nonneg_right h₁ ha
[GOAL]
case mp.intro.right
a t : ℝ
ha : 0 < a
h₁ : 0 ≤ a * t
h₂ : a * t ≤ 1
⊢ t ≤ 1 / a
[PROOFSTEP]
rwa [le_div_iff ha, mul_comm]
[GOAL]
case mpr.intro.left
a t : ℝ
ha : 0 < a
h₁ : 0 ≤ t
h₂ : t ≤ 1 / a
⊢ 0 ≤ a * t
[PROOFSTEP]
exact mul_nonneg ha.le h₁
[GOAL]
case mpr.intro.right
a t : ℝ
ha : 0 < a
h₁ : 0 ≤ t
h₂ : t ≤ 1 / a
⊢ a * t ≤ 1
[PROOFSTEP]
rwa [le_div_iff ha, mul_comm] at h₂
[GOAL]
t : ℝ
⊢ 2 * t - 1 ∈ I ↔ t ∈ Icc (1 / 2) 1
[PROOFSTEP]
constructor
[GOAL]
case mp
t : ℝ
⊢ 2 * t - 1 ∈ I → t ∈ Icc (1 / 2) 1
[PROOFSTEP]
rintro ⟨h₁, h₂⟩
[GOAL]
case mpr
t : ℝ
⊢ t ∈ Icc (1 / 2) 1 → 2 * t - 1 ∈ I
[PROOFSTEP]
rintro ⟨h₁, h₂⟩
[GOAL]
case mp.intro
t : ℝ
h₁ : 0 ≤ 2 * t - 1
h₂ : 2 * t - 1 ≤ 1
⊢ t ∈ Icc (1 / 2) 1
[PROOFSTEP]
constructor
[GOAL]
case mpr.intro
t : ℝ
h₁ : 1 / 2 ≤ t
h₂ : t ≤ 1
⊢ 2 * t - 1 ∈ I
[PROOFSTEP]
constructor
[GOAL]
case mp.intro.left
t : ℝ
h₁ : 0 ≤ 2 * t - 1
h₂ : 2 * t - 1 ≤ 1
⊢ 1 / 2 ≤ t
[PROOFSTEP]
linarith
[GOAL]
case mp.intro.right
t : ℝ
h₁ : 0 ≤ 2 * t - 1
h₂ : 2 * t - 1 ≤ 1
⊢ t ≤ 1
[PROOFSTEP]
linarith
[GOAL]
case mpr.intro.left
t : ℝ
h₁ : 1 / 2 ≤ t
h₂ : t ≤ 1
⊢ 0 ≤ 2 * t - 1
[PROOFSTEP]
linarith
[GOAL]
case mpr.intro.right
t : ℝ
h₁ : 1 / 2 ≤ t
h₂ : t ≤ 1
⊢ 2 * t - 1 ≤ 1
[PROOFSTEP]
linarith
[GOAL]
x : ↑unitInterval
⊢ 0 ≤ ↑x
[PROOFSTEP]
unit_interval
[GOAL]
𝕜 : Type u_1
inst✝² : LinearOrderedField 𝕜
inst✝¹ : TopologicalSpace 𝕜
inst✝ : TopologicalRing 𝕜
a b : 𝕜
h : 0 < a
⊢ ↑(affineHomeomorph a b (_ : a ≠ 0)) '' Icc 0 1 = Icc b (a + b)
[PROOFSTEP]
simp [h]
[GOAL]
𝕜 : Type u_1
inst✝² : LinearOrderedField 𝕜
inst✝¹ : TopologicalSpace 𝕜
inst✝ : TopologicalRing 𝕜
a b : 𝕜
h : a < b
⊢ ↑(Icc a b) ≃ₜ ↑(Icc 0 1)
[PROOFSTEP]
let e := Homeomorph.image (affineHomeomorph (b - a) a (sub_pos.mpr h).ne.symm) (Set.Icc 0 1)
[GOAL]
𝕜 : Type u_1
inst✝² : LinearOrderedField 𝕜
inst✝¹ : TopologicalSpace 𝕜
inst✝ : TopologicalRing 𝕜
a b : 𝕜
h : a < b
e : ↑(Icc 0 1) ≃ₜ ↑(↑(affineHomeomorph (b - a) a (_ : b - a ≠ 0)) '' Icc 0 1) :=
Homeomorph.image (affineHomeomorph (b - a) a (_ : b - a ≠ 0)) (Icc 0 1)
⊢ ↑(Icc a b) ≃ₜ ↑(Icc 0 1)
[PROOFSTEP]
refine' (e.trans _).symm
[GOAL]
𝕜 : Type u_1
inst✝² : LinearOrderedField 𝕜
inst✝¹ : TopologicalSpace 𝕜
inst✝ : TopologicalRing 𝕜
a b : 𝕜
h : a < b
e : ↑(Icc 0 1) ≃ₜ ↑(↑(affineHomeomorph (b - a) a (_ : b - a ≠ 0)) '' Icc 0 1) :=
Homeomorph.image (affineHomeomorph (b - a) a (_ : b - a ≠ 0)) (Icc 0 1)
⊢ ↑(↑(affineHomeomorph (b - a) a (_ : b - a ≠ 0)) '' Icc 0 1) ≃ₜ ↑(Icc a b)
[PROOFSTEP]
apply Homeomorph.setCongr
[GOAL]
case h
𝕜 : Type u_1
inst✝² : LinearOrderedField 𝕜
inst✝¹ : TopologicalSpace 𝕜
inst✝ : TopologicalRing 𝕜
a b : 𝕜
h : a < b
e : ↑(Icc 0 1) ≃ₜ ↑(↑(affineHomeomorph (b - a) a (_ : b - a ≠ 0)) '' Icc 0 1) :=
Homeomorph.image (affineHomeomorph (b - a) a (_ : b - a ≠ 0)) (Icc 0 1)
⊢ ↑(affineHomeomorph (b - a) a (_ : b - a ≠ 0)) '' Icc 0 1 = Icc a b
[PROOFSTEP]
rw [affineHomeomorph_image_I _ _ (sub_pos.2 h)]
[GOAL]
case h
𝕜 : Type u_1
inst✝² : LinearOrderedField 𝕜
inst✝¹ : TopologicalSpace 𝕜
inst✝ : TopologicalRing 𝕜
a b : 𝕜
h : a < b
e : ↑(Icc 0 1) ≃ₜ ↑(↑(affineHomeomorph (b - a) a (_ : b - a ≠ 0)) '' Icc 0 1) :=
Homeomorph.image (affineHomeomorph (b - a) a (_ : b - a ≠ 0)) (Icc 0 1)
⊢ Icc a (b - a + a) = Icc a b
[PROOFSTEP]
simp
| {"mathlib_filename": "Mathlib.Topology.UnitInterval", "llama_tokens": 3057} |
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
f : α✝ → β
α : Type u_3
inst✝ : TopologicalSpace α
⊢ IsQuasiSeparated Set.univ ↔ QuasiSeparatedSpace α
[PROOFSTEP]
rw [QuasiSeparatedSpace_iff]
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
f : α✝ → β
α : Type u_3
inst✝ : TopologicalSpace α
⊢ IsQuasiSeparated Set.univ ↔ ∀ (U V : Set α), IsOpen U → IsCompact U → IsOpen V → IsCompact V → IsCompact (U ∩ V)
[PROOFSTEP]
simp [IsQuasiSeparated]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
⊢ IsQuasiSeparated (f '' s)
[PROOFSTEP]
intro U V hU hU' hU'' hV hV' hV''
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (U ∩ V)
[PROOFSTEP]
convert (H (f ⁻¹' U) (f ⁻¹' V) ?_ (h.continuous.1 _ hU') ?_ ?_ (h.continuous.1 _ hV') ?_).image h.continuous
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ U ∩ V = f '' (f ⁻¹' U ∩ f ⁻¹' V)
[PROOFSTEP]
symm
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ f '' (f ⁻¹' U ∩ f ⁻¹' V) = U ∩ V
[PROOFSTEP]
rw [← Set.preimage_inter, Set.image_preimage_eq_inter_range, Set.inter_eq_left_iff_subset]
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ U ∩ V ⊆ Set.range f
[PROOFSTEP]
exact (Set.inter_subset_left _ _).trans (hU.trans (Set.image_subset_range _ _))
[GOAL]
case convert_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ f ⁻¹' U ⊆ s
[PROOFSTEP]
intro x hx
[GOAL]
case convert_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
x : α
hx : x ∈ f ⁻¹' U
⊢ x ∈ s
[PROOFSTEP]
rw [← (h.inj.injOn _).mem_image_iff (Set.subset_univ _) trivial]
[GOAL]
case convert_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
x : α
hx : x ∈ f ⁻¹' U
⊢ f x ∈ f '' s
[PROOFSTEP]
exact hU hx
[GOAL]
case convert_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (f ⁻¹' U)
[PROOFSTEP]
rw [h.isCompact_iff_isCompact_image]
[GOAL]
case convert_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (f '' (f ⁻¹' U))
[PROOFSTEP]
convert hU''
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ f '' (f ⁻¹' U) = U
[PROOFSTEP]
rw [Set.image_preimage_eq_inter_range, Set.inter_eq_left_iff_subset]
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ U ⊆ Set.range f
[PROOFSTEP]
exact hU.trans (Set.image_subset_range _ _)
[GOAL]
case convert_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ f ⁻¹' V ⊆ s
[PROOFSTEP]
intro x hx
[GOAL]
case convert_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
x : α
hx : x ∈ f ⁻¹' V
⊢ x ∈ s
[PROOFSTEP]
rw [← (h.inj.injOn _).mem_image_iff (Set.subset_univ _) trivial]
[GOAL]
case convert_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
x : α
hx : x ∈ f ⁻¹' V
⊢ f x ∈ f '' s
[PROOFSTEP]
exact hV hx
[GOAL]
case convert_4
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (f ⁻¹' V)
[PROOFSTEP]
rw [h.isCompact_iff_isCompact_image]
[GOAL]
case convert_4
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (f '' (f ⁻¹' V))
[PROOFSTEP]
convert hV''
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ f '' (f ⁻¹' V) = V
[PROOFSTEP]
rw [Set.image_preimage_eq_inter_range, Set.inter_eq_left_iff_subset]
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
H : IsQuasiSeparated s
h : Embedding f
U V : Set β
hU : U ⊆ f '' s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ f '' s
hV' : IsOpen V
hV'' : IsCompact V
⊢ V ⊆ Set.range f
[PROOFSTEP]
exact hV.trans (Set.image_subset_range _ _)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
h : OpenEmbedding f
s : Set α
⊢ IsQuasiSeparated s ↔ IsQuasiSeparated (f '' s)
[PROOFSTEP]
refine' ⟨fun hs => hs.image_of_embedding h.toEmbedding, _⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
h : OpenEmbedding f
s : Set α
⊢ IsQuasiSeparated (f '' s) → IsQuasiSeparated s
[PROOFSTEP]
intro H U V hU hU' hU'' hV hV' hV''
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
h : OpenEmbedding f
s : Set α
H : IsQuasiSeparated (f '' s)
U V : Set α
hU : U ⊆ s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (U ∩ V)
[PROOFSTEP]
rw [h.toEmbedding.isCompact_iff_isCompact_image, Set.image_inter h.inj]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
h : OpenEmbedding f
s : Set α
H : IsQuasiSeparated (f '' s)
U V : Set α
hU : U ⊆ s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (f '' U ∩ f '' V)
[PROOFSTEP]
exact
H (f '' U) (f '' V) (Set.image_subset _ hU) (h.isOpenMap _ hU') (hU''.image h.continuous) (Set.image_subset _ hV)
(h.isOpenMap _ hV') (hV''.image h.continuous)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
hs : IsOpen s
⊢ IsQuasiSeparated s ↔ QuasiSeparatedSpace ↑s
[PROOFSTEP]
rw [← isQuasiSeparated_univ_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
hs : IsOpen s
⊢ IsQuasiSeparated s ↔ IsQuasiSeparated Set.univ
[PROOFSTEP]
convert (hs.openEmbedding_subtype_val.isQuasiSeparated_iff (s := Set.univ)).symm
[GOAL]
case h.e'_1.h.e'_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
hs : IsOpen s
⊢ s = Subtype.val '' Set.univ
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s t : Set α
ht : IsQuasiSeparated t
h : s ⊆ t
⊢ IsQuasiSeparated s
[PROOFSTEP]
intro U V hU hU' hU'' hV hV' hV''
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s t : Set α
ht : IsQuasiSeparated t
h : s ⊆ t
U V : Set α
hU : U ⊆ s
hU' : IsOpen U
hU'' : IsCompact U
hV : V ⊆ s
hV' : IsOpen V
hV'' : IsCompact V
⊢ IsCompact (U ∩ V)
[PROOFSTEP]
exact ht U V (hU.trans h) hU' hU'' (hV.trans h) hV' hV''
| {"mathlib_filename": "Mathlib.Topology.QuasiSeparated", "llama_tokens": 4834} |
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
s : Set α
⊢ IsOpen {l | s ∈ l}
[PROOFSTEP]
simpa only [Iic_principal] using isOpen_Iic_principal
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
⊢ ∀ (t₁ : Set (Filter α)),
t₁ ∈ range (Iic ∘ 𝓟) →
∀ (t₂ : Set (Filter α)),
t₂ ∈ range (Iic ∘ 𝓟) → ∀ (x : Filter α), x ∈ t₁ ∩ t₂ → ∃ t₃, t₃ ∈ range (Iic ∘ 𝓟) ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
rintro _ ⟨s, rfl⟩ _ ⟨t, rfl⟩ l hl
[GOAL]
case intro.intro
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
s t : Set α
l : Filter α
hl : l ∈ (Iic ∘ 𝓟) s ∩ (Iic ∘ 𝓟) t
⊢ ∃ t₃, t₃ ∈ range (Iic ∘ 𝓟) ∧ l ∈ t₃ ∧ t₃ ⊆ (Iic ∘ 𝓟) s ∩ (Iic ∘ 𝓟) t
[PROOFSTEP]
exact ⟨Iic (𝓟 s) ∩ Iic (𝓟 t), ⟨s ∩ t, by simp⟩, hl, Subset.rfl⟩
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
s t : Set α
l : Filter α
hl : l ∈ (Iic ∘ 𝓟) s ∩ (Iic ∘ 𝓟) t
⊢ (Iic ∘ 𝓟) (s ∩ t) = Iic (𝓟 s) ∩ Iic (𝓟 t)
[PROOFSTEP]
simp
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
s : Set (Filter α)
⊢ (∃ S, S ⊆ range (Iic ∘ 𝓟) ∧ s = ⋃₀ S) ↔ ∃ T, s = ⋃ (t : Set α) (_ : t ∈ T), Iic (𝓟 t)
[PROOFSTEP]
simp only [exists_subset_range_and_iff, sUnion_image, (· ∘ ·)]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
⊢ ⨅ (s : Set (Filter α)) (_ : s ∈ {s | l ∈ s ∧ s ∈ range (Iic ∘ 𝓟)}), 𝓟 s = Filter.lift' l (Iic ∘ 𝓟)
[PROOFSTEP]
simp only [mem_setOf_eq, @and_comm (l ∈ _), iInf_and, iInf_range, Filter.lift', Filter.lift, (· ∘ ·), mem_Iic,
le_principal_iff]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
⊢ 𝓝 l = Filter.lift' l fun s => {l' | s ∈ l'}
[PROOFSTEP]
simpa only [(· ∘ ·), Iic_principal] using nhds_eq l
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
la : Filter α
lb : Filter β
f : α → Filter β
⊢ Tendsto f la (𝓝 lb) ↔ ∀ (s : Set β), s ∈ lb → ∀ᶠ (a : α) in la, s ∈ f a
[PROOFSTEP]
simp only [nhds_eq', tendsto_lift', mem_setOf_eq]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
p : ι → Prop
s : ι → Set α
h : HasBasis l p s
⊢ HasBasis (𝓝 l) p fun i => Iic (𝓟 (s i))
[PROOFSTEP]
rw [nhds_eq]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
p : ι → Prop
s : ι → Set α
h : HasBasis l p s
⊢ HasBasis (Filter.lift' l (Iic ∘ 𝓟)) p fun i => Iic (𝓟 (s i))
[PROOFSTEP]
exact h.lift' monotone_principal.Iic
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter X
⊢ Tendsto pure l (𝓝 l)
[PROOFSTEP]
rw [Filter.tendsto_nhds]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter X
⊢ ∀ (s : Set X), s ∈ l → ∀ᶠ (a : X) in l, s ∈ pure a
[PROOFSTEP]
refine fun s hs ↦ Eventually.mono hs fun x ↦ id
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
p : ι → Prop
s : ι → Set α
h : HasBasis l p s
⊢ HasBasis (𝓝 l) p fun i => {l' | s i ∈ l'}
[PROOFSTEP]
simpa only [Iic_principal] using h.nhds
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
⊢ 𝓝 ⊥ = pure ⊥
[PROOFSTEP]
simp [nhds_eq, (· ∘ ·), lift'_bot monotone_principal.Iic]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
⊢ 𝓝 ⊤ = ⊤
[PROOFSTEP]
simp [nhds_eq]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
x : α
⊢ 𝓝 (pure x) = 𝓟 {⊥, pure x}
[PROOFSTEP]
rw [← principal_singleton, nhds_principal, principal_singleton, Iic_pure]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
f : ι → Filter α
⊢ 𝓝 (⨅ (i : ι), f i) = ⨅ (i : ι), 𝓝 (f i)
[PROOFSTEP]
simp only [nhds_eq]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
f : ι → Filter α
⊢ Filter.lift' (⨅ (i : ι), f i) (Iic ∘ 𝓟) = ⨅ (i : ι), Filter.lift' (f i) (Iic ∘ 𝓟)
[PROOFSTEP]
apply lift'_iInf_of_map_univ
[GOAL]
case hg
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
f : ι → Filter α
⊢ ∀ {s t : Set α}, (Iic ∘ 𝓟) (s ∩ t) = (Iic ∘ 𝓟) s ∩ (Iic ∘ 𝓟) t
[PROOFSTEP]
simp
[GOAL]
case hg'
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
f : ι → Filter α
⊢ (Iic ∘ 𝓟) univ = univ
[PROOFSTEP]
simp
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l₁ l₂ : Filter α
⊢ 𝓝 (l₁ ⊓ l₂) = 𝓝 l₁ ⊓ 𝓝 l₂
[PROOFSTEP]
simpa only [iInf_bool_eq] using nhds_iInf fun b => cond b l₁ l₂
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
⊢ ⋂₀ {s | s ∈ 𝓝 l} = Iic l
[PROOFSTEP]
simp_rw [nhds_eq, (· ∘ ·), sInter_lift'_sets monotone_principal.Iic, Iic, le_principal_iff, ← setOf_forall, ←
Filter.le_def]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l₁ l₂ : Filter α
⊢ 𝓝 l₁ ≤ 𝓝 l₂ ↔ l₁ ≤ l₂
[PROOFSTEP]
refine' ⟨fun h => _, fun h => monotone_nhds h⟩
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l₁ l₂ : Filter α
h : 𝓝 l₁ ≤ 𝓝 l₂
⊢ l₁ ≤ l₂
[PROOFSTEP]
rw [← Iic_subset_Iic, ← sInter_nhds, ← sInter_nhds]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l₁ l₂ : Filter α
h : 𝓝 l₁ ≤ 𝓝 l₂
⊢ ⋂₀ {s | s ∈ 𝓝 l₁} ⊆ ⋂₀ {s | s ∈ 𝓝 l₂}
[PROOFSTEP]
exact sInter_subset_sInter h
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
s : Set (Filter α)
l : Filter α
⊢ l ∈ interior s ↔ ∃ t, t ∈ l ∧ Iic (𝓟 t) ⊆ s
[PROOFSTEP]
rw [mem_interior_iff_mem_nhds, mem_nhds_iff]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
s : Set (Filter α)
l : Filter α
⊢ l ∈ closure s ↔ ∀ (t : Set α), t ∈ l → ∃ l', l' ∈ s ∧ t ∈ l'
[PROOFSTEP]
simp only [closure_eq_compl_interior_compl, Filter.mem_interior, mem_compl_iff, not_exists, not_forall,
Classical.not_not, exists_prop, not_and, and_comm, subset_def, mem_Iic, le_principal_iff]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l : Filter α
⊢ closure {l} = Ici l
[PROOFSTEP]
ext l'
[GOAL]
case h
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l l' : Filter α
⊢ l' ∈ closure {l} ↔ l' ∈ Ici l
[PROOFSTEP]
simp [Filter.mem_closure, Filter.le_def]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
l₁ l₂ : Filter α
⊢ l₁ ⤳ l₂ ↔ l₁ ≤ l₂
[PROOFSTEP]
simp only [specializes_iff_closure_subset, Filter.closure_singleton, Ici_subset_Ici]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
inst✝ : Preorder α
⊢ 𝓝 atTop = ⨅ (x : α), 𝓟 (Iic (𝓟 (Ici x)))
[PROOFSTEP]
simp only [atTop, nhds_iInf, nhds_principal]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
inst✝ : Preorder β
l : Filter α
f : α → Filter β
⊢ Tendsto f l (𝓝 atTop) ↔ ∀ (y : β), ∀ᶠ (a : α) in l, Ici y ∈ f a
[PROOFSTEP]
simp only [nhds_atTop, tendsto_iInf, tendsto_principal, mem_Iic, le_principal_iff]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
inst✝ : TopologicalSpace X
x : X
⊢ 𝓝 (𝓝 x) = ⨅ (s : Set X) (_ : IsOpen s) (_ : x ∈ s), 𝓟 (Iic (𝓟 s))
[PROOFSTEP]
simp only [(nhds_basis_opens x).nhds.eq_biInf, iInf_and, @iInf_comm _ (_ ∈ _)]
[GOAL]
ι : Sort u_1
α : Type u_2
β : Type u_3
X : Type u_4
Y : Type u_5
inst✝ : TopologicalSpace X
x : X
⊢ ⨅ (s : Set X) (_ : IsOpen s) (_ : x ∈ s), 𝓟 s = comap 𝓝 (𝓝 (𝓝 x))
[PROOFSTEP]
simp (config := { contextual := true }) only [nhds_nhds, comap_iInf, comap_principal, Iic_principal, preimage_setOf_eq,
← mem_interior_iff_mem_nhds, setOf_mem_eq, IsOpen.interior_eq]
| {"mathlib_filename": "Mathlib.Topology.Filter", "llama_tokens": 4075} |
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a : (⨂[R]^i) M
b : (⨂[R]^j) M
⊢ ↑toTensorAlgebra (GradedMonoid.GMul.mul a b) = ↑toTensorAlgebra a * ↑toTensorAlgebra b
[PROOFSTEP]
rw [TensorPower.gMul_eq_coe_linearMap, ← LinearMap.compr₂_apply, ← @LinearMap.mul_apply' R, ← LinearMap.compl₂_apply, ←
LinearMap.comp_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a : (⨂[R]^i) M
b : (⨂[R]^j) M
⊢ ↑(↑(LinearMap.compr₂ (LinearMap.compr₂ (TensorProduct.mk R ((⨂[R]^i) M) ((⨂[R]^j) M)) ↑mulEquiv) toTensorAlgebra) a)
b =
↑(↑(LinearMap.comp (LinearMap.compl₂ (LinearMap.mul R ((fun x => TensorAlgebra R M) a)) toTensorAlgebra)
toTensorAlgebra)
a)
b
[PROOFSTEP]
refine' LinearMap.congr_fun (LinearMap.congr_fun _ a) b
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a : (⨂[R]^i) M
b : (⨂[R]^j) M
⊢ LinearMap.compr₂ (LinearMap.compr₂ (TensorProduct.mk R ((⨂[R]^i) M) ((⨂[R]^j) M)) ↑mulEquiv) toTensorAlgebra =
LinearMap.comp (LinearMap.compl₂ (LinearMap.mul R ((fun x => TensorAlgebra R M) a)) toTensorAlgebra) toTensorAlgebra
[PROOFSTEP]
clear! a b
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a : (⨂[R]^i) M
⊢ LinearMap.compr₂ (LinearMap.compr₂ (TensorProduct.mk R ((⨂[R]^i) M) ((⨂[R]^j) M)) ↑mulEquiv) toTensorAlgebra =
LinearMap.comp (LinearMap.compl₂ (LinearMap.mul R ((fun x => TensorAlgebra R M) a)) toTensorAlgebra) toTensorAlgebra
[PROOFSTEP]
ext
(a b)
-- Porting note: pulled the next two lines out of the long `simp only` below.
[GOAL]
case H.H.H.H
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a✝ : (⨂[R]^i) M
a : Fin i → M
b : Fin j → M
⊢ ↑(LinearMap.compMultilinearMap
(↑(LinearMap.compMultilinearMap
(LinearMap.compr₂ (LinearMap.compr₂ (TensorProduct.mk R ((⨂[R]^i) M) ((⨂[R]^j) M)) ↑mulEquiv)
toTensorAlgebra)
(PiTensorProduct.tprod R))
a)
(PiTensorProduct.tprod R))
b =
↑(LinearMap.compMultilinearMap
(↑(LinearMap.compMultilinearMap
(LinearMap.comp (LinearMap.compl₂ (LinearMap.mul R ((fun x => TensorAlgebra R M) a✝)) toTensorAlgebra)
toTensorAlgebra)
(PiTensorProduct.tprod R))
a)
(PiTensorProduct.tprod R))
b
[PROOFSTEP]
simp only [LinearMap.compMultilinearMap_apply]
[GOAL]
case H.H.H.H
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a✝ : (⨂[R]^i) M
a : Fin i → M
b : Fin j → M
⊢ ↑(↑(LinearMap.compr₂ (LinearMap.compr₂ (TensorProduct.mk R ((⨂[R]^i) M) ((⨂[R]^j) M)) ↑mulEquiv) toTensorAlgebra)
(↑(PiTensorProduct.tprod R) a))
(↑(PiTensorProduct.tprod R) b) =
↑(↑(LinearMap.comp (LinearMap.compl₂ (LinearMap.mul R ((fun x => TensorAlgebra R M) a✝)) toTensorAlgebra)
toTensorAlgebra)
(↑(PiTensorProduct.tprod R) a))
(↑(PiTensorProduct.tprod R) b)
[PROOFSTEP]
rw [LinearMap.compr₂_apply, ← gMul_eq_coe_linearMap]
[GOAL]
case H.H.H.H
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a✝ : (⨂[R]^i) M
a : Fin i → M
b : Fin j → M
⊢ ↑toTensorAlgebra (GradedMonoid.GMul.mul (↑(PiTensorProduct.tprod R) a) (↑(PiTensorProduct.tprod R) b)) =
↑(↑(LinearMap.comp (LinearMap.compl₂ (LinearMap.mul R ((fun x => TensorAlgebra R M) a✝)) toTensorAlgebra)
toTensorAlgebra)
(↑(PiTensorProduct.tprod R) a))
(↑(PiTensorProduct.tprod R) b)
[PROOFSTEP]
simp only [LinearMap.compr₂_apply, LinearMap.mul_apply', LinearMap.compl₂_apply, LinearMap.comp_apply,
LinearMap.compMultilinearMap_apply, PiTensorProduct.lift.tprod, TensorPower.tprod_mul_tprod,
TensorPower.toTensorAlgebra_tprod, TensorAlgebra.tprod_apply, ← gMul_eq_coe_linearMap]
[GOAL]
case H.H.H.H
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a✝ : (⨂[R]^i) M
a : Fin i → M
b : Fin j → M
⊢ List.prod (List.ofFn fun i_1 => ↑(TensorAlgebra.ι R) (Fin.append a b i_1)) =
List.prod (List.ofFn fun i => ↑(TensorAlgebra.ι R) (a i)) *
List.prod (List.ofFn fun i => ↑(TensorAlgebra.ι R) (b i))
[PROOFSTEP]
refine' Eq.trans _ List.prod_append
[GOAL]
case H.H.H.H
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a✝ : (⨂[R]^i) M
a : Fin i → M
b : Fin j → M
⊢ List.prod (List.ofFn fun i_1 => ↑(TensorAlgebra.ι R) (Fin.append a b i_1)) =
List.prod ((List.ofFn fun i => ↑(TensorAlgebra.ι R) (a i)) ++ List.ofFn fun i => ↑(TensorAlgebra.ι R) (b i))
[PROOFSTEP]
apply congr_arg
[GOAL]
case H.H.H.H.h
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i j : ℕ
a✝ : (⨂[R]^i) M
a : Fin i → M
b : Fin j → M
⊢ (List.ofFn fun i_1 => ↑(TensorAlgebra.ι R) (Fin.append a b i_1)) =
(List.ofFn fun i => ↑(TensorAlgebra.ι R) (a i)) ++ List.ofFn fun i => ↑(TensorAlgebra.ι R) (b i)
[PROOFSTEP]
erw [← List.map_ofFn _ (TensorAlgebra.ι R), ← List.map_ofFn _ (TensorAlgebra.ι R), ←
List.map_ofFn _ (TensorAlgebra.ι R), ← List.map_append, List.ofFn_fin_append]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
r : R
⊢ ↑toTensorAlgebra (↑DirectSum.GAlgebra.toFun r) = ↑(algebraMap R (TensorAlgebra R M)) r
[PROOFSTEP]
rw [TensorPower.galgebra_toFun_def, TensorPower.algebraMap₀_eq_smul_one, LinearMap.map_smul,
TensorPower.toTensorAlgebra_gOne, Algebra.algebraMap_eq_smul_one]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ AlgHom.comp ofDirectSum toDirectSum = AlgHom.id R (TensorAlgebra R M)
[PROOFSTEP]
ext
[GOAL]
case w.h
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x✝ : M
⊢ ↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.comp ofDirectSum toDirectSum)) (ι R)) x✝ =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (TensorAlgebra R M))) (ι R)) x✝
[PROOFSTEP]
simp [DirectSum.lof_eq_of, tprod_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n m : ℕ
h : n = m
x : (⨂[R]^n) M
⊢ GradedMonoid.mk m (↑(PiTensorProduct.reindex R M (Fin.castIso h).toEquiv) x) = GradedMonoid.mk n x
[PROOFSTEP]
rw [Fin.castIso_to_equiv, mk_reindex_cast h]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
refine' Fin.consInduction _ _ x
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x : Fin 1), Fin.elim0 a)) (List.finRange 0)) =
GradedMonoid.mk 0 (↑(PiTensorProduct.tprod R) Fin.elim0)
[PROOFSTEP]
clear x
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ ∀ {n : ℕ} (x₀ : M) (x : Fin n → M),
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x) →
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), Fin.cons x₀ x a)) (List.finRange (n + 1))) =
GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))
[PROOFSTEP]
clear x
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
⊢ List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x : Fin 1), Fin.elim0 a)) (List.finRange 0)) =
GradedMonoid.mk 0 (↑(PiTensorProduct.tprod R) Fin.elim0)
[PROOFSTEP]
rw [List.finRange_zero, List.map_nil, List.prod_nil]
[GOAL]
case refine'_1
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
⊢ 1 = GradedMonoid.mk 0 (↑(PiTensorProduct.tprod R) Fin.elim0)
[PROOFSTEP]
rfl
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
⊢ ∀ {n : ℕ} (x₀ : M) (x : Fin n → M),
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x) →
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), Fin.cons x₀ x a)) (List.finRange (n + 1))) =
GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))
[PROOFSTEP]
intro n x₀ x ih
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), Fin.cons x₀ x a)) (List.finRange (n + 1))) =
GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))
[PROOFSTEP]
rw [List.finRange_succ_eq_map, List.map_cons, List.prod_cons, List.map_map]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), Fin.cons x₀ x 0) *
List.prod
(List.map ((fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), Fin.cons x₀ x a)) ∘ Fin.succ) (List.finRange n)) =
GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))
[PROOFSTEP]
simp_rw [Function.comp, Fin.cons_zero, Fin.cons_succ]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ GradedMonoid.mk 1 (⨂ₜ[R] (x : Fin 1), x₀) *
List.prod (List.map (fun x_1 => GradedMonoid.mk 1 (⨂ₜ[R] (x_2 : Fin 1), x x_1)) (List.finRange n)) =
GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))
[PROOFSTEP]
rw [ih, GradedMonoid.mk_mul_mk, TensorPower.tprod_mul_tprod]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ GradedMonoid.mk (1 + n) (↑(PiTensorProduct.tprod R) (Fin.append (fun x => x₀) x)) =
GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))
[PROOFSTEP]
refine' TensorPower.gradedMonoid_eq_of_cast (add_comm _ _) _
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ ↑(TensorPower.cast R M (_ : 1 + n = n + 1))
(GradedMonoid.mk (1 + n) (↑(PiTensorProduct.tprod R) (Fin.append (fun x => x₀) x))).snd =
(GradedMonoid.mk (n + 1) (↑(PiTensorProduct.tprod R) (Fin.cons x₀ x))).snd
[PROOFSTEP]
dsimp only [GradedMonoid.mk]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ ↑(TensorPower.cast R M (_ : 1 + n = n + 1)) (↑(PiTensorProduct.tprod R) (Fin.append (fun x => x₀) x)) =
↑(PiTensorProduct.tprod R) (Fin.cons x₀ x)
[PROOFSTEP]
rw [TensorPower.cast_tprod]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ ↑(PiTensorProduct.tprod R) (Fin.append (fun x => x₀) x ∘ ↑(Fin.castIso (_ : n + 1 = 1 + n))) =
↑(PiTensorProduct.tprod R) (Fin.cons x₀ x)
[PROOFSTEP]
simp_rw [Fin.append_left_eq_cons, Function.comp]
[GOAL]
case refine'_2
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n✝ n : ℕ
x₀ : M
x : Fin n → M
ih :
List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
⊢ (⨂ₜ[R] (x_1 : Fin (n + 1)),
Fin.cons x₀ x (↑(Fin.castIso (_ : 1 + n = n + 1)) (↑(Fin.castIso (_ : n + 1 = 1 + n)) x_1))) =
↑(PiTensorProduct.tprod R) (Fin.cons x₀ x)
[PROOFSTEP]
congr 1 with i
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ ↑toDirectSum (↑(tprod R M n) x) = ↑(DirectSum.of (fun i => (⨂[R]^i) M) n) (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
rw [tprod_apply, AlgHom.map_list_prod, List.map_ofFn]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ List.prod (List.ofFn (↑toDirectSum ∘ fun i => ↑(ι R) (x i))) =
↑(DirectSum.of (fun i => (⨂[R]^i) M) n) (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
simp_rw [Function.comp, toDirectSum_ι]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ List.prod (List.ofFn fun x_1 => ↑(DirectSum.of (fun n => (⨂[R]^n) M) 1) (⨂ₜ[R] (x_2 : Fin 1), x x_1)) =
↑(DirectSum.of (fun i => (⨂[R]^i) M) n) (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
rw [DirectSum.list_prod_ofFn_of_eq_dProd]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ ↑(DirectSum.of (fun n => (⨂[R]^n) M) (List.dProdIndex (List.finRange n) fun x => 1))
(List.dProd (List.finRange n) (fun x => 1) fun x_1 => ⨂ₜ[R] (x_2 : Fin 1), x x_1) =
↑(DirectSum.of (fun i => (⨂[R]^i) M) n) (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
apply DirectSum.of_eq_of_gradedMonoid_eq
[GOAL]
case h
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ GradedMonoid.mk (List.dProdIndex (List.finRange n) fun x => 1)
(List.dProd (List.finRange n) (fun x => 1) fun x_1 => ⨂ₜ[R] (x_2 : Fin 1), x x_1) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
rw [GradedMonoid.mk_list_dProd]
[GOAL]
case h
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
n : ℕ
x : Fin n → M
⊢ List.prod (List.map (fun a => GradedMonoid.mk 1 (⨂ₜ[R] (x_1 : Fin 1), x a)) (List.finRange n)) =
GradedMonoid.mk n (↑(PiTensorProduct.tprod R) x)
[PROOFSTEP]
rw [TensorPower.list_prod_gradedMonoid_mk_single]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ AlgHom.comp toDirectSum ofDirectSum = AlgHom.id R (⨁ (n : ℕ), (⨂[R]^n) M)
[PROOFSTEP]
ext
[GOAL]
case h.H.H
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ : Fin i✝ → M
⊢ ↑(LinearMap.compMultilinearMap
(LinearMap.comp (AlgHom.toLinearMap (AlgHom.comp toDirectSum ofDirectSum))
(DirectSum.lof R ℕ (fun i => (⨂[R]^i) M) i✝))
(PiTensorProduct.tprod R))
x✝ =
↑(LinearMap.compMultilinearMap
(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (⨁ (n : ℕ), (⨂[R]^n) M)))
(DirectSum.lof R ℕ (fun i => (⨂[R]^i) M) i✝))
(PiTensorProduct.tprod R))
x✝
[PROOFSTEP]
simp [DirectSum.lof_eq_of, -tprod_apply, toDirectSum_tensorPower_tprod]
| {"mathlib_filename": "Mathlib.LinearAlgebra.TensorAlgebra.ToTensorPower", "llama_tokens": 8041} |
[GOAL]
R : Type u_1
S : Type u_2
A : Type u_3
B : Type u_4
inst✝⁸ : CommSemiring R
inst✝⁷ : CommSemiring S
inst✝⁶ : Semiring A
inst✝⁵ : Semiring B
inst✝⁴ : Algebra R S
inst✝³ : Algebra R A
inst✝² : Algebra R B
inst✝¹ : Algebra S A
inst✝ : IsScalarTower R S A
e₁ : Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ ≃ₗ[S] (A ⊗[R] B)ᵐᵒᵖ :=
LinearEquiv.trans
(TensorProduct.AlgebraTensorModule.congr (LinearEquiv.symm (opLinearEquiv S)) (LinearEquiv.symm (opLinearEquiv R)))
(opLinearEquiv S)
e₂ : A ⊗[R] B ≃ₗ[S] (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ :=
LinearEquiv.trans (TensorProduct.AlgebraTensorModule.congr (opLinearEquiv S) (opLinearEquiv R)) (opLinearEquiv S)
⊢ ↑AlgHom.op.symm
(AlgHom.comp
(algHomOfLinearMapTensorProduct ↑e₁
(_ :
∀ (a₁ a₂ : Aᵐᵒᵖ) (b₁ b₂ : Bᵐᵒᵖ), ↑↑e₁ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₁ (a₁ ⊗ₜ[R] b₁) * ↑↑e₁ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₁ (↑(algebraMap S Aᵐᵒᵖ) r ⊗ₜ[R] 1) = ↑(algebraMap S (A ⊗[R] B)ᵐᵒᵖ) r))
(↑AlgHom.opComm
(algHomOfLinearMapTensorProduct ↑e₂
(_ : ∀ (a₁ a₂ : A) (b₁ b₂ : B), ↑↑e₂ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₂ (a₁ ⊗ₜ[R] b₁) * ↑↑e₂ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₂ (↑(algebraMap S A) r ⊗ₜ[R] 1) = ↑(algebraMap S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ) r)))) =
↑AlgHom.op.symm (AlgHom.id S (A ⊗[R] B)ᵐᵒᵖ)
[PROOFSTEP]
ext
[GOAL]
case ha.H
R : Type u_1
S : Type u_2
A : Type u_3
B : Type u_4
inst✝⁸ : CommSemiring R
inst✝⁷ : CommSemiring S
inst✝⁶ : Semiring A
inst✝⁵ : Semiring B
inst✝⁴ : Algebra R S
inst✝³ : Algebra R A
inst✝² : Algebra R B
inst✝¹ : Algebra S A
inst✝ : IsScalarTower R S A
e₁ : Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ ≃ₗ[S] (A ⊗[R] B)ᵐᵒᵖ :=
LinearEquiv.trans
(TensorProduct.AlgebraTensorModule.congr (LinearEquiv.symm (opLinearEquiv S)) (LinearEquiv.symm (opLinearEquiv R)))
(opLinearEquiv S)
e₂ : A ⊗[R] B ≃ₗ[S] (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ :=
LinearEquiv.trans (TensorProduct.AlgebraTensorModule.congr (opLinearEquiv S) (opLinearEquiv R)) (opLinearEquiv S)
x✝ : A
⊢ ↑(AlgHom.comp
(↑AlgHom.op.symm
(AlgHom.comp
(algHomOfLinearMapTensorProduct ↑e₁
(_ :
∀ (a₁ a₂ : Aᵐᵒᵖ) (b₁ b₂ : Bᵐᵒᵖ),
↑↑e₁ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₁ (a₁ ⊗ₜ[R] b₁) * ↑↑e₁ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₁ (↑(algebraMap S Aᵐᵒᵖ) r ⊗ₜ[R] 1) = ↑(algebraMap S (A ⊗[R] B)ᵐᵒᵖ) r))
(↑AlgHom.opComm
(algHomOfLinearMapTensorProduct ↑e₂
(_ :
∀ (a₁ a₂ : A) (b₁ b₂ : B),
↑↑e₂ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₂ (a₁ ⊗ₜ[R] b₁) * ↑↑e₂ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₂ (↑(algebraMap S A) r ⊗ₜ[R] 1) = ↑(algebraMap S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ) r)))))
includeLeft)
x✝ =
↑(AlgHom.comp (↑AlgHom.op.symm (AlgHom.id S (A ⊗[R] B)ᵐᵒᵖ)) includeLeft) x✝
[PROOFSTEP]
rfl
[GOAL]
case hb.H
R : Type u_1
S : Type u_2
A : Type u_3
B : Type u_4
inst✝⁸ : CommSemiring R
inst✝⁷ : CommSemiring S
inst✝⁶ : Semiring A
inst✝⁵ : Semiring B
inst✝⁴ : Algebra R S
inst✝³ : Algebra R A
inst✝² : Algebra R B
inst✝¹ : Algebra S A
inst✝ : IsScalarTower R S A
e₁ : Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ ≃ₗ[S] (A ⊗[R] B)ᵐᵒᵖ :=
LinearEquiv.trans
(TensorProduct.AlgebraTensorModule.congr (LinearEquiv.symm (opLinearEquiv S)) (LinearEquiv.symm (opLinearEquiv R)))
(opLinearEquiv S)
e₂ : A ⊗[R] B ≃ₗ[S] (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ :=
LinearEquiv.trans (TensorProduct.AlgebraTensorModule.congr (opLinearEquiv S) (opLinearEquiv R)) (opLinearEquiv S)
x✝ : B
⊢ ↑(AlgHom.comp
(AlgHom.restrictScalars R
(↑AlgHom.op.symm
(AlgHom.comp
(algHomOfLinearMapTensorProduct ↑e₁
(_ :
∀ (a₁ a₂ : Aᵐᵒᵖ) (b₁ b₂ : Bᵐᵒᵖ),
↑↑e₁ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₁ (a₁ ⊗ₜ[R] b₁) * ↑↑e₁ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₁ (↑(algebraMap S Aᵐᵒᵖ) r ⊗ₜ[R] 1) = ↑(algebraMap S (A ⊗[R] B)ᵐᵒᵖ) r))
(↑AlgHom.opComm
(algHomOfLinearMapTensorProduct ↑e₂
(_ :
∀ (a₁ a₂ : A) (b₁ b₂ : B),
↑↑e₂ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₂ (a₁ ⊗ₜ[R] b₁) * ↑↑e₂ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₂ (↑(algebraMap S A) r ⊗ₜ[R] 1) = ↑(algebraMap S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ) r))))))
includeRight)
x✝ =
↑(AlgHom.comp (AlgHom.restrictScalars R (↑AlgHom.op.symm (AlgHom.id S (A ⊗[R] B)ᵐᵒᵖ))) includeRight) x✝
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
S : Type u_2
A : Type u_3
B : Type u_4
inst✝⁸ : CommSemiring R
inst✝⁷ : CommSemiring S
inst✝⁶ : Semiring A
inst✝⁵ : Semiring B
inst✝⁴ : Algebra R S
inst✝³ : Algebra R A
inst✝² : Algebra R B
inst✝¹ : Algebra S A
inst✝ : IsScalarTower R S A
e₁ : Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ ≃ₗ[S] (A ⊗[R] B)ᵐᵒᵖ :=
LinearEquiv.trans
(TensorProduct.AlgebraTensorModule.congr (LinearEquiv.symm (opLinearEquiv S)) (LinearEquiv.symm (opLinearEquiv R)))
(opLinearEquiv S)
e₂ : A ⊗[R] B ≃ₗ[S] (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ :=
LinearEquiv.trans (TensorProduct.AlgebraTensorModule.congr (opLinearEquiv S) (opLinearEquiv R)) (opLinearEquiv S)
⊢ AlgHom.comp
(↑AlgHom.opComm
(algHomOfLinearMapTensorProduct ↑e₂
(_ : ∀ (a₁ a₂ : A) (b₁ b₂ : B), ↑↑e₂ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₂ (a₁ ⊗ₜ[R] b₁) * ↑↑e₂ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₂ (↑(algebraMap S A) r ⊗ₜ[R] 1) = ↑(algebraMap S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ) r)))
(algHomOfLinearMapTensorProduct ↑e₁
(_ :
∀ (a₁ a₂ : Aᵐᵒᵖ) (b₁ b₂ : Bᵐᵒᵖ), ↑↑e₁ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₁ (a₁ ⊗ₜ[R] b₁) * ↑↑e₁ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₁ (↑(algebraMap S Aᵐᵒᵖ) r ⊗ₜ[R] 1) = ↑(algebraMap S (A ⊗[R] B)ᵐᵒᵖ) r)) =
AlgHom.id S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)
[PROOFSTEP]
ext
[GOAL]
case ha.H
R : Type u_1
S : Type u_2
A : Type u_3
B : Type u_4
inst✝⁸ : CommSemiring R
inst✝⁷ : CommSemiring S
inst✝⁶ : Semiring A
inst✝⁵ : Semiring B
inst✝⁴ : Algebra R S
inst✝³ : Algebra R A
inst✝² : Algebra R B
inst✝¹ : Algebra S A
inst✝ : IsScalarTower R S A
e₁ : Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ ≃ₗ[S] (A ⊗[R] B)ᵐᵒᵖ :=
LinearEquiv.trans
(TensorProduct.AlgebraTensorModule.congr (LinearEquiv.symm (opLinearEquiv S)) (LinearEquiv.symm (opLinearEquiv R)))
(opLinearEquiv S)
e₂ : A ⊗[R] B ≃ₗ[S] (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ :=
LinearEquiv.trans (TensorProduct.AlgebraTensorModule.congr (opLinearEquiv S) (opLinearEquiv R)) (opLinearEquiv S)
x✝ : Aᵐᵒᵖ
⊢ ↑(AlgHom.comp
(AlgHom.comp
(↑AlgHom.opComm
(algHomOfLinearMapTensorProduct ↑e₂
(_ :
∀ (a₁ a₂ : A) (b₁ b₂ : B), ↑↑e₂ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₂ (a₁ ⊗ₜ[R] b₁) * ↑↑e₂ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₂ (↑(algebraMap S A) r ⊗ₜ[R] 1) = ↑(algebraMap S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ) r)))
(algHomOfLinearMapTensorProduct ↑e₁
(_ :
∀ (a₁ a₂ : Aᵐᵒᵖ) (b₁ b₂ : Bᵐᵒᵖ),
↑↑e₁ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₁ (a₁ ⊗ₜ[R] b₁) * ↑↑e₁ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₁ (↑(algebraMap S Aᵐᵒᵖ) r ⊗ₜ[R] 1) = ↑(algebraMap S (A ⊗[R] B)ᵐᵒᵖ) r)))
includeLeft)
x✝ =
↑(AlgHom.comp (AlgHom.id S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)) includeLeft) x✝
[PROOFSTEP]
rfl
[GOAL]
case hb.H
R : Type u_1
S : Type u_2
A : Type u_3
B : Type u_4
inst✝⁸ : CommSemiring R
inst✝⁷ : CommSemiring S
inst✝⁶ : Semiring A
inst✝⁵ : Semiring B
inst✝⁴ : Algebra R S
inst✝³ : Algebra R A
inst✝² : Algebra R B
inst✝¹ : Algebra S A
inst✝ : IsScalarTower R S A
e₁ : Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ ≃ₗ[S] (A ⊗[R] B)ᵐᵒᵖ :=
LinearEquiv.trans
(TensorProduct.AlgebraTensorModule.congr (LinearEquiv.symm (opLinearEquiv S)) (LinearEquiv.symm (opLinearEquiv R)))
(opLinearEquiv S)
e₂ : A ⊗[R] B ≃ₗ[S] (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ :=
LinearEquiv.trans (TensorProduct.AlgebraTensorModule.congr (opLinearEquiv S) (opLinearEquiv R)) (opLinearEquiv S)
x✝ : Bᵐᵒᵖ
⊢ ↑(AlgHom.comp
(AlgHom.restrictScalars R
(AlgHom.comp
(↑AlgHom.opComm
(algHomOfLinearMapTensorProduct ↑e₂
(_ :
∀ (a₁ a₂ : A) (b₁ b₂ : B),
↑↑e₂ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₂ (a₁ ⊗ₜ[R] b₁) * ↑↑e₂ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₂ (↑(algebraMap S A) r ⊗ₜ[R] 1) = ↑(algebraMap S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ)ᵐᵒᵖ) r)))
(algHomOfLinearMapTensorProduct ↑e₁
(_ :
∀ (a₁ a₂ : Aᵐᵒᵖ) (b₁ b₂ : Bᵐᵒᵖ),
↑↑e₁ ((a₁ * a₂) ⊗ₜ[R] (b₁ * b₂)) = ↑↑e₁ (a₁ ⊗ₜ[R] b₁) * ↑↑e₁ (a₂ ⊗ₜ[R] b₂))
(_ : ∀ (r : S), ↑↑e₁ (↑(algebraMap S Aᵐᵒᵖ) r ⊗ₜ[R] 1) = ↑(algebraMap S (A ⊗[R] B)ᵐᵒᵖ) r))))
includeRight)
x✝ =
↑(AlgHom.comp (AlgHom.restrictScalars R (AlgHom.id S (Aᵐᵒᵖ ⊗[R] Bᵐᵒᵖ))) includeRight) x✝
[PROOFSTEP]
rfl
| {"mathlib_filename": "Mathlib.LinearAlgebra.TensorProduct.Opposite", "llama_tokens": 5017} |
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
n : ℕ
x : X
hx : x ∈ c.C
⊢ approx n c x = 0
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : x ∈ c✝.C
c : CU X
hx : x ∈ c.C
⊢ approx Nat.zero c x = 0
[PROOFSTEP]
exact indicator_of_not_mem (fun (hU : x ∈ c.Uᶜ) => hU <| c.subset hx) _
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : x ∈ c✝.C
n : ℕ
ihn : ∀ (c : CU X), x ∈ c.C → approx n c x = 0
c : CU X
hx : x ∈ c.C
⊢ approx (Nat.succ n) c x = 0
[PROOFSTEP]
simp only [approx]
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : x ∈ c✝.C
n : ℕ
ihn : ∀ (c : CU X), x ∈ c.C → approx n c x = 0
c : CU X
hx : x ∈ c.C
⊢ midpoint ℝ (approx n (left c) x) (approx n (right c) x) = 0
[PROOFSTEP]
rw [ihn, ihn, midpoint_self]
[GOAL]
case succ.hx
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : x ∈ c✝.C
n : ℕ
ihn : ∀ (c : CU X), x ∈ c.C → approx n c x = 0
c : CU X
hx : x ∈ c.C
⊢ x ∈ (right c).C
case succ.hx
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : x ∈ c✝.C
n : ℕ
ihn : ∀ (c : CU X), x ∈ c.C → approx n c x = 0
c : CU X
hx : x ∈ c.C
⊢ x ∈ (left c).C
[PROOFSTEP]
exacts [c.subset_right_C hx, hx]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
n : ℕ
x : X
hx : ¬x ∈ c.U
⊢ approx n c x = 1
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : ¬x ∈ c✝.U
c : CU X
hx : ¬x ∈ c.U
⊢ approx Nat.zero c x = 1
[PROOFSTEP]
rw [← mem_compl_iff] at hx
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : ¬x ∈ c✝.U
c : CU X
hx : x ∈ c.Uᶜ
⊢ approx Nat.zero c x = 1
[PROOFSTEP]
exact indicator_of_mem hx _
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : ¬x ∈ c✝.U
n : ℕ
ihn : ∀ (c : CU X), ¬x ∈ c.U → approx n c x = 1
c : CU X
hx : ¬x ∈ c.U
⊢ approx (Nat.succ n) c x = 1
[PROOFSTEP]
simp only [approx]
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : ¬x ∈ c✝.U
n : ℕ
ihn : ∀ (c : CU X), ¬x ∈ c.U → approx n c x = 1
c : CU X
hx : ¬x ∈ c.U
⊢ midpoint ℝ (approx n (left c) x) (approx n (right c) x) = 1
[PROOFSTEP]
rw [ihn, ihn, midpoint_self]
[GOAL]
case succ.hx
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : ¬x ∈ c✝.U
n : ℕ
ihn : ∀ (c : CU X), ¬x ∈ c.U → approx n c x = 1
c : CU X
hx : ¬x ∈ c.U
⊢ ¬x ∈ (right c).U
case succ.hx
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
hx✝ : ¬x ∈ c✝.U
n : ℕ
ihn : ∀ (c : CU X), ¬x ∈ c.U → approx n c x = 1
c : CU X
hx : ¬x ∈ c.U
⊢ ¬x ∈ (left c).U
[PROOFSTEP]
exacts [hx, fun hU => hx <| c.left_U_subset hU]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
n : ℕ
x : X
⊢ 0 ≤ approx n c x
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
c : CU X
⊢ 0 ≤ approx Nat.zero c x
[PROOFSTEP]
exact indicator_nonneg (fun _ _ => zero_le_one) _
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), 0 ≤ approx n c x
c : CU X
⊢ 0 ≤ approx (Nat.succ n) c x
[PROOFSTEP]
simp only [approx, midpoint_eq_smul_add, invOf_eq_inv]
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), 0 ≤ approx n c x
c : CU X
⊢ 0 ≤ 2⁻¹ • (approx n (left c) x + approx n (right c) x)
[PROOFSTEP]
refine' mul_nonneg (inv_nonneg.2 zero_le_two) (add_nonneg _ _)
[GOAL]
case succ.refine'_1
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), 0 ≤ approx n c x
c : CU X
⊢ 0 ≤ approx n (left c) x
[PROOFSTEP]
apply ihn
[GOAL]
case succ.refine'_2
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), 0 ≤ approx n c x
c : CU X
⊢ 0 ≤ approx n (right c) x
[PROOFSTEP]
apply ihn
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
n : ℕ
x : X
⊢ approx n c x ≤ 1
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
c : CU X
⊢ approx Nat.zero c x ≤ 1
[PROOFSTEP]
exact indicator_apply_le' (fun _ => le_rfl) fun _ => zero_le_one
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ≤ 1
c : CU X
⊢ approx (Nat.succ n) c x ≤ 1
[PROOFSTEP]
simp only [approx, midpoint_eq_smul_add, invOf_eq_inv, smul_eq_mul, ← div_eq_inv_mul]
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ≤ 1
c : CU X
⊢ (approx n (left c) x + approx n (right c) x) / 2 ≤ 1
[PROOFSTEP]
have := add_le_add (ihn (left c)) (ihn (right c))
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ≤ 1
c : CU X
this : approx n (left c) x + approx n (right c) x ≤ 1 + 1
⊢ (approx n (left c) x + approx n (right c) x) / 2 ≤ 1
[PROOFSTEP]
norm_num at this
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ≤ 1
c : CU X
this : approx n (left c) x + approx n (right c) x ≤ 2
⊢ (approx n (left c) x + approx n (right c) x) / 2 ≤ 1
[PROOFSTEP]
exact Iff.mpr (div_le_one zero_lt_two) this
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c₁ c₂ : CU X
h : c₁.U ⊆ c₂.C
n₁ n₂ : ℕ
x : X
⊢ approx n₂ c₂ x ≤ approx n₁ c₁ x
[PROOFSTEP]
by_cases hx : x ∈ c₁.U
[GOAL]
case pos
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c₁ c₂ : CU X
h : c₁.U ⊆ c₂.C
n₁ n₂ : ℕ
x : X
hx : x ∈ c₁.U
⊢ approx n₂ c₂ x ≤ approx n₁ c₁ x
[PROOFSTEP]
calc
approx n₂ c₂ x = 0 := approx_of_mem_C _ _ (h hx)
_ ≤ approx n₁ c₁ x := approx_nonneg _ _ _
[GOAL]
case neg
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c₁ c₂ : CU X
h : c₁.U ⊆ c₂.C
n₁ n₂ : ℕ
x : X
hx : ¬x ∈ c₁.U
⊢ approx n₂ c₂ x ≤ approx n₁ c₁ x
[PROOFSTEP]
calc
approx n₂ c₂ x ≤ 1 := approx_le_one _ _ _
_ = approx n₁ c₁ x := (approx_of_nmem_U _ _ hx).symm
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
n : ℕ
x : X
⊢ approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
c : CU X
⊢ approx Nat.zero c x ∈ Icc (approx Nat.zero (right c) x) (approx Nat.zero (left c) x)
[PROOFSTEP]
exact ⟨le_rfl, indicator_le_indicator_of_subset (compl_subset_compl.2 c.left_U_subset) (fun _ => zero_le_one) _⟩
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
c : CU X
⊢ approx (Nat.succ n) c x ∈ Icc (approx (Nat.succ n) (right c) x) (approx (Nat.succ n) (left c) x)
[PROOFSTEP]
simp only [approx, mem_Icc]
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
c : CU X
⊢ midpoint ℝ (approx n (left (right c)) x) (approx n (right (right c)) x) ≤
midpoint ℝ (approx n (left c) x) (approx n (right c) x) ∧
midpoint ℝ (approx n (left c) x) (approx n (right c) x) ≤
midpoint ℝ (approx n (left (left c)) x) (approx n (right (left c)) x)
[PROOFSTEP]
refine' ⟨midpoint_le_midpoint _ (ihn _).1, midpoint_le_midpoint (ihn _).2 _⟩
[GOAL]
case succ.refine'_1
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
c : CU X
⊢ approx n (left (right c)) x ≤ approx n (left c) x
[PROOFSTEP]
apply approx_le_approx_of_U_sub_C
[GOAL]
case succ.refine'_2
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
c : CU X
⊢ approx n (right c) x ≤ approx n (right (left c)) x
[PROOFSTEP]
apply approx_le_approx_of_U_sub_C
[GOAL]
case succ.refine'_1.h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
c : CU X
⊢ (left c).U ⊆ (left (right c)).C
case succ.refine'_2.h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ∈ Icc (approx n (right c) x) (approx n (left c) x)
c : CU X
⊢ (right (left c)).U ⊆ (right c).C
[PROOFSTEP]
exacts [subset_closure, subset_closure]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
n : ℕ
x : X
⊢ approx n c x ≤ approx (n + 1) c x
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
c : CU X
⊢ approx Nat.zero c x ≤ approx (Nat.zero + 1) c x
[PROOFSTEP]
simp only [approx, right_U, right_le_midpoint]
[GOAL]
case zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
c : CU X
⊢ indicator c.Uᶜ 1 x ≤ indicator (left c).Uᶜ 1 x
[PROOFSTEP]
exact (approx_mem_Icc_right_left c 0 x).2
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ≤ approx (n + 1) c x
c : CU X
⊢ approx (Nat.succ n) c x ≤ approx (Nat.succ n + 1) c x
[PROOFSTEP]
rw [approx, approx]
[GOAL]
case succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
x : X
n : ℕ
ihn : ∀ (c : CU X), approx n c x ≤ approx (n + 1) c x
c : CU X
⊢ midpoint ℝ (approx n (left c) x) (approx n (right c) x) ≤
midpoint ℝ (approx (n + 1) (left c) x) (approx (n + 1) (right c) x)
[PROOFSTEP]
exact midpoint_le_midpoint (ihn _) (ihn _)
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
x : X
h : x ∈ c.C
⊢ CU.lim c x = 0
[PROOFSTEP]
simp only [CU.lim, approx_of_mem_C, h, ciSup_const]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
x : X
h : ¬x ∈ c.U
⊢ CU.lim c x = 1
[PROOFSTEP]
simp only [CU.lim, approx_of_nmem_U c _ h, ciSup_const]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
x : X
⊢ CU.lim c x = midpoint ℝ (CU.lim (left c) x) (CU.lim (right c) x)
[PROOFSTEP]
refine' tendsto_nhds_unique (c.tendsto_approx_atTop x) ((tendsto_add_atTop_iff_nat 1).1 _)
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
x : X
⊢ Tendsto (fun n => approx (n + 1) c x) atTop (𝓝 (midpoint ℝ (CU.lim (left c) x) (CU.lim (right c) x)))
[PROOFSTEP]
simp only [approx]
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
x : X
⊢ Tendsto (fun n => midpoint ℝ (approx (Nat.add n 0) (left c) x) (approx (Nat.add n 0) (right c) x)) atTop
(𝓝 (midpoint ℝ (CU.lim (left c) x) (CU.lim (right c) x)))
[PROOFSTEP]
exact (c.left.tendsto_approx_atTop x).midpoint (c.right.tendsto_approx_atTop x)
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
⊢ Continuous (CU.lim c)
[PROOFSTEP]
obtain ⟨h0, h1234, h1⟩ : 0 < (2⁻¹ : ℝ) ∧ (2⁻¹ : ℝ) < 3 / 4 ∧ (3 / 4 : ℝ) < 1 := by norm_num
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
⊢ 0 < 2⁻¹ ∧ 2⁻¹ < 3 / 4 ∧ 3 / 4 < 1
[PROOFSTEP]
norm_num
[GOAL]
case intro.intro
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
⊢ Continuous (CU.lim c)
[PROOFSTEP]
refine'
continuous_iff_continuousAt.2 fun x =>
(Metric.nhds_basis_closedBall_pow (h0.trans h1234) h1).tendsto_right_iff.2 fun n _ => _
[GOAL]
case intro.intro
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
n : ℕ
x✝ : True
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, CU.lim c x_1 ∈ Metric.closedBall (CU.lim c x) ((3 / 4) ^ n)
[PROOFSTEP]
simp only [Metric.mem_closedBall]
[GOAL]
case intro.intro
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
n : ℕ
x✝ : True
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
[PROOFSTEP]
induction' n with n ihn generalizing c
[GOAL]
case intro.intro.zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
c : CU X
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ Nat.zero
[PROOFSTEP]
refine' eventually_of_forall fun y => _
[GOAL]
case intro.intro.zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
c : CU X
y : X
⊢ dist (CU.lim c y) (CU.lim c x) ≤ (3 / 4) ^ Nat.zero
[PROOFSTEP]
rw [pow_zero]
[GOAL]
case intro.intro.zero
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
c : CU X
y : X
⊢ dist (CU.lim c y) (CU.lim c x) ≤ 1
[PROOFSTEP]
exact Real.dist_le_of_mem_Icc_01 (c.lim_mem_Icc _) (c.lim_mem_Icc _)
[GOAL]
case intro.intro.succ
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
by_cases hxl : x ∈ c.left.U
[GOAL]
case pos
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (left c).U
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
filter_upwards [IsOpen.mem_nhds c.left.open_U hxl, ihn c.left] with _ hyl hyd
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (left c).U
a✝ : X
hyl : a✝ ∈ (left c).U
hyd : dist (CU.lim (left c) a✝) (CU.lim (left c) x) ≤ (3 / 4) ^ n
⊢ dist (CU.lim c a✝) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
rw [pow_succ, c.lim_eq_midpoint, c.lim_eq_midpoint, c.right.lim_of_mem_C _ (c.left_U_subset_right_C hyl),
c.right.lim_of_mem_C _ (c.left_U_subset_right_C hxl)]
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (left c).U
a✝ : X
hyl : a✝ ∈ (left c).U
hyd : dist (CU.lim (left c) a✝) (CU.lim (left c) x) ≤ (3 / 4) ^ n
⊢ dist (midpoint ℝ (CU.lim (left c) a✝) 0) (midpoint ℝ (CU.lim (left c) x) 0) ≤ 3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
refine' (dist_midpoint_midpoint_le _ _ _ _).trans _
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (left c).U
a✝ : X
hyl : a✝ ∈ (left c).U
hyd : dist (CU.lim (left c) a✝) (CU.lim (left c) x) ≤ (3 / 4) ^ n
⊢ (dist (CU.lim (left c) a✝) (CU.lim (left c) x) + dist 0 0) / 2 ≤ 3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
rw [dist_self, add_zero, div_eq_inv_mul]
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (left c).U
a✝ : X
hyl : a✝ ∈ (left c).U
hyd : dist (CU.lim (left c) a✝) (CU.lim (left c) x) ≤ (3 / 4) ^ n
⊢ 2⁻¹ * dist (CU.lim (left c) a✝) (CU.lim (left c) x) ≤ 3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
gcongr
[GOAL]
case neg
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : ¬x ∈ (left c).U
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
replace hxl : x ∈ c.left.right.Cᶜ
[GOAL]
case hxl
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : ¬x ∈ (left c).U
⊢ x ∈ (right (left c)).Cᶜ
case neg
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (right (left c)).Cᶜ
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
exact compl_subset_compl.2 c.left.right.subset hxl
[GOAL]
case neg
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (right (left c)).Cᶜ
⊢ ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
filter_upwards [IsOpen.mem_nhds (isOpen_compl_iff.2 c.left.right.closed_C) hxl, ihn c.left.right, ihn c.right] with y
hyl hydl hydr
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (right (left c)).Cᶜ
y : X
hyl : y ∈ (right (left c)).Cᶜ
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
⊢ dist (CU.lim c y) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
replace hxl : x ∉ c.left.left.U
[GOAL]
case hxl
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
hxl : x ∈ (right (left c)).Cᶜ
y : X
hyl : y ∈ (right (left c)).Cᶜ
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
⊢ ¬x ∈ (left (left c)).U
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hyl : y ∈ (right (left c)).Cᶜ
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
⊢ dist (CU.lim c y) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
exact compl_subset_compl.2 c.left.left_U_subset_right_C hxl
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hyl : y ∈ (right (left c)).Cᶜ
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
⊢ dist (CU.lim c y) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
replace hyl : y ∉ c.left.left.U
[GOAL]
case hyl
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hyl : y ∈ (right (left c)).Cᶜ
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
⊢ ¬y ∈ (left (left c)).U
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
⊢ dist (CU.lim c y) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
exact compl_subset_compl.2 c.left.left_U_subset_right_C hyl
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
⊢ dist (CU.lim c y) (CU.lim c x) ≤ (3 / 4) ^ Nat.succ n
[PROOFSTEP]
simp only [pow_succ, c.lim_eq_midpoint, c.left.lim_eq_midpoint, c.left.left.lim_of_nmem_U _ hxl,
c.left.left.lim_of_nmem_U _ hyl]
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
⊢ dist (midpoint ℝ (midpoint ℝ 1 (CU.lim (right (left c)) y)) (CU.lim (right c) y))
(midpoint ℝ (midpoint ℝ 1 (CU.lim (right (left c)) x)) (CU.lim (right c) x)) ≤
3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
refine' (dist_midpoint_midpoint_le _ _ _ _).trans _
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
⊢ (dist (midpoint ℝ 1 (CU.lim (right (left c)) y)) (midpoint ℝ 1 (CU.lim (right (left c)) x)) +
dist (CU.lim (right c) y) (CU.lim (right c) x)) /
2 ≤
3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
refine' (div_le_div_of_le_of_nonneg (add_le_add_right (dist_midpoint_midpoint_le _ _ _ _) _) zero_le_two).trans _
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
⊢ ((dist 1 1 + dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x)) / 2 +
dist (CU.lim (right c) y) (CU.lim (right c) x)) /
2 ≤
3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
rw [dist_self, zero_add]
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ (3 / 4) ^ n
c : CU X
y : X
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ (3 / 4) ^ n
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ (3 / 4) ^ n
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
⊢ (dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) / 2 + dist (CU.lim (right c) y) (CU.lim (right c) x)) /
2 ≤
3 / 4 * (3 / 4) ^ n
[PROOFSTEP]
set r := (3 / 4 : ℝ) ^ n
[GOAL]
case h
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
c : CU X
y : X
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
r : ℝ := (3 / 4) ^ n
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ r
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ r
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ r
⊢ (dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) / 2 + dist (CU.lim (right c) y) (CU.lim (right c) x)) /
2 ≤
3 / 4 * r
[PROOFSTEP]
calc
_ ≤ (r / 2 + r) / 2 := by gcongr
_ = _ := by field_simp; ring
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
c : CU X
y : X
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
r : ℝ := (3 / 4) ^ n
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ r
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ r
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ r
⊢ (dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) / 2 + dist (CU.lim (right c) y) (CU.lim (right c) x)) /
2 ≤
(r / 2 + r) / 2
[PROOFSTEP]
gcongr
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
c : CU X
y : X
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
r : ℝ := (3 / 4) ^ n
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ r
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ r
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ r
⊢ (r / 2 + r) / 2 = 3 / 4 * r
[PROOFSTEP]
field_simp
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
c✝ : CU X
h0 : 0 < 2⁻¹
h1234 : 2⁻¹ < 3 / 4
h1 : 3 / 4 < 1
x : X
x✝ : True
n : ℕ
c : CU X
y : X
hxl : ¬x ∈ (left (left c)).U
hyl : ¬y ∈ (left (left c)).U
r : ℝ := (3 / 4) ^ n
ihn : ∀ (c : CU X), ∀ᶠ (x_1 : X) in 𝓝 x, dist (CU.lim c x_1) (CU.lim c x) ≤ r
hydl : dist (CU.lim (right (left c)) y) (CU.lim (right (left c)) x) ≤ r
hydr : dist (CU.lim (right c) y) (CU.lim (right c) x) ≤ r
⊢ (3 ^ n * 4 ^ n + 3 ^ n * (4 ^ n * 2)) * (4 * 4 ^ n) = 3 * 3 ^ n * (4 ^ n * 2 * 4 ^ n * 2)
[PROOFSTEP]
ring
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
⊢ ∃ f, EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
[PROOFSTEP]
set c : Urysohns.CU X := ⟨s, tᶜ, hs, ht.isOpen_compl, disjoint_left.1 hd⟩
[GOAL]
X : Type u_1
inst✝¹ : TopologicalSpace X
inst✝ : NormalSpace X
s t : Set X
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
c : Urysohns.CU X :=
{ C := s, U := tᶜ, closed_C := hs, open_U := (_ : IsOpen tᶜ), subset := (_ : ∀ ⦃a : X⦄, a ∈ s → ¬a ∈ t) }
⊢ ∃ f, EqOn (↑f) 0 s ∧ EqOn (↑f) 1 t ∧ ∀ (x : X), ↑f x ∈ Icc 0 1
[PROOFSTEP]
exact ⟨⟨c.lim, c.continuous_lim⟩, c.lim_of_mem_C, fun x hx => c.lim_of_nmem_U _ fun h => h hx, c.lim_mem_Icc⟩
| {"mathlib_filename": "Mathlib.Topology.UrysohnsLemma", "llama_tokens": 15770} |
[GOAL]
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
i : ι
m : M
k : κ
n : N
⊢ ↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i m ⊗ₜ[R] Finsupp.single k n) = Finsupp.single (i, k) (m ⊗ₜ[R] n)
[PROOFSTEP]
classical simp [finsuppTensorFinsupp]
[GOAL]
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
i : ι
m : M
k : κ
n : N
⊢ ↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i m ⊗ₜ[R] Finsupp.single k n) = Finsupp.single (i, k) (m ⊗ₜ[R] n)
[PROOFSTEP]
simp [finsuppTensorFinsupp]
[GOAL]
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) (f ⊗ₜ[R] g)) (i, k) = ↑f i ⊗ₜ[R] ↑g k
[PROOFSTEP]
apply Finsupp.induction_linear f
[GOAL]
case h0
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) (0 ⊗ₜ[R] g)) (i, k) = ↑0 i ⊗ₜ[R] ↑g k
[PROOFSTEP]
simp
[GOAL]
case hadd
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
⊢ ∀ (f g_1 : ι →₀ M),
↑(↑(finsuppTensorFinsupp R M N ι κ) (f ⊗ₜ[R] g)) (i, k) = ↑f i ⊗ₜ[R] ↑g k →
↑(↑(finsuppTensorFinsupp R M N ι κ) (g_1 ⊗ₜ[R] g)) (i, k) = ↑g_1 i ⊗ₜ[R] ↑g k →
↑(↑(finsuppTensorFinsupp R M N ι κ) ((f + g_1) ⊗ₜ[R] g)) (i, k) = ↑(f + g_1) i ⊗ₜ[R] ↑g k
[PROOFSTEP]
intro f₁ f₂ hf₁ hf₂
[GOAL]
case hadd
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
f₁ f₂ : ι →₀ M
hf₁ : ↑(↑(finsuppTensorFinsupp R M N ι κ) (f₁ ⊗ₜ[R] g)) (i, k) = ↑f₁ i ⊗ₜ[R] ↑g k
hf₂ : ↑(↑(finsuppTensorFinsupp R M N ι κ) (f₂ ⊗ₜ[R] g)) (i, k) = ↑f₂ i ⊗ₜ[R] ↑g k
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) ((f₁ + f₂) ⊗ₜ[R] g)) (i, k) = ↑(f₁ + f₂) i ⊗ₜ[R] ↑g k
[PROOFSTEP]
simp [add_tmul, hf₁, hf₂]
[GOAL]
case hsingle
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
⊢ ∀ (a : ι) (b : M),
↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single a b ⊗ₜ[R] g)) (i, k) = ↑(Finsupp.single a b) i ⊗ₜ[R] ↑g k
[PROOFSTEP]
intro i' m
[GOAL]
case hsingle
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] g)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑g k
[PROOFSTEP]
apply Finsupp.induction_linear g
[GOAL]
case hsingle.h0
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] 0)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑0 k
[PROOFSTEP]
simp
[GOAL]
case hsingle.hadd
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
⊢ ∀ (f g : κ →₀ N),
↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] f)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑f k →
↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] g)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑g k →
↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] (f + g))) (i, k) =
↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(f + g) k
[PROOFSTEP]
intro g₁ g₂ hg₁ hg₂
[GOAL]
case hsingle.hadd
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
g₁ g₂ : κ →₀ N
hg₁ : ↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] g₁)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑g₁ k
hg₂ : ↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] g₂)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑g₂ k
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] (g₁ + g₂))) (i, k) =
↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(g₁ + g₂) k
[PROOFSTEP]
simp [tmul_add, hg₁, hg₂]
[GOAL]
case hsingle.hsingle
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
⊢ ∀ (a : κ) (b : N),
↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] Finsupp.single a b)) (i, k) =
↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single a b) k
[PROOFSTEP]
intro k' n
[GOAL]
case hsingle.hsingle
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
⊢ ↑(↑(finsuppTensorFinsupp R M N ι κ) (Finsupp.single i' m ⊗ₜ[R] Finsupp.single k' n)) (i, k) =
↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
simp only [finsuppTensorFinsupp_single]
-- split_ifs; finish can close the goal from here
[GOAL]
case hsingle.hsingle
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
by_cases h1 : (i', k') = (i, k)
[GOAL]
case pos
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
h1 : (i', k') = (i, k)
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
simp only [Prod.mk.inj_iff] at h1
[GOAL]
case pos
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
h1 : i' = i ∧ k' = k
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
simp [h1]
[GOAL]
case neg
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
h1 : ¬(i', k') = (i, k)
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
simp only [Prod.mk.inj_iff, not_and_or] at h1
[GOAL]
case neg
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
h1 : ¬i' = i ∨ ¬k' = k
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
cases' h1 with h1 h1
[GOAL]
case neg.inl
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
h1 : ¬i' = i
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
simp [h1]
[GOAL]
case neg.inr
R✝ : Type u
M✝ : Type v
N✝ : Type w
inst✝⁹ : Ring R✝
inst✝⁸ : AddCommGroup M✝
inst✝⁷ : Module R✝ M✝
inst✝⁶ : AddCommGroup N✝
inst✝⁵ : Module R✝ N✝
R : Type u_1
M : Type u_2
N : Type u_3
ι : Type u_4
κ : Type u_5
inst✝⁴ : CommRing R
inst✝³ : AddCommGroup M
inst✝² : Module R M
inst✝¹ : AddCommGroup N
inst✝ : Module R N
f : ι →₀ M
g : κ →₀ N
i : ι
k : κ
i' : ι
m : M
k' : κ
n : N
h1 : ¬k' = k
⊢ ↑(Finsupp.single (i', k') (m ⊗ₜ[R] n)) (i, k) = ↑(Finsupp.single i' m) i ⊗ₜ[R] ↑(Finsupp.single k' n) k
[PROOFSTEP]
simp [h1]
[GOAL]
R : Type u
M : Type v
N : Type w
inst✝⁵ : Ring R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : AddCommGroup N
inst✝¹ : Module R N
S : Type u_1
inst✝ : CommRing S
α : Type u_2
β : Type u_3
f : α →₀ S
g : β →₀ S
a : α
b : β
⊢ ↑(↑(finsuppTensorFinsupp' S α β) (f ⊗ₜ[S] g)) (a, b) = ↑f a * ↑g b
[PROOFSTEP]
simp [finsuppTensorFinsupp']
[GOAL]
R : Type u
M : Type v
N : Type w
inst✝⁵ : Ring R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : AddCommGroup N
inst✝¹ : Module R N
S : Type u_1
inst✝ : CommRing S
α : Type u_2
β : Type u_3
a : α
b : β
r₁ r₂ : S
⊢ ↑(finsuppTensorFinsupp' S α β) (Finsupp.single a r₁ ⊗ₜ[S] Finsupp.single b r₂) = Finsupp.single (a, b) (r₁ * r₂)
[PROOFSTEP]
ext ⟨a', b'⟩
[GOAL]
case h.mk
R : Type u
M : Type v
N : Type w
inst✝⁵ : Ring R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : AddCommGroup N
inst✝¹ : Module R N
S : Type u_1
inst✝ : CommRing S
α : Type u_2
β : Type u_3
a : α
b : β
r₁ r₂ : S
a' : α
b' : β
⊢ ↑(↑(finsuppTensorFinsupp' S α β) (Finsupp.single a r₁ ⊗ₜ[S] Finsupp.single b r₂)) (a', b') =
↑(Finsupp.single (a, b) (r₁ * r₂)) (a', b')
[PROOFSTEP]
classical aesop (add norm [Finsupp.single_apply])
[GOAL]
case h.mk
R : Type u
M : Type v
N : Type w
inst✝⁵ : Ring R
inst✝⁴ : AddCommGroup M
inst✝³ : Module R M
inst✝² : AddCommGroup N
inst✝¹ : Module R N
S : Type u_1
inst✝ : CommRing S
α : Type u_2
β : Type u_3
a : α
b : β
r₁ r₂ : S
a' : α
b' : β
⊢ ↑(↑(finsuppTensorFinsupp' S α β) (Finsupp.single a r₁ ⊗ₜ[S] Finsupp.single b r₂)) (a', b') =
↑(Finsupp.single (a, b) (r₁ * r₂)) (a', b')
[PROOFSTEP]
aesop (add norm [Finsupp.single_apply])
| {"mathlib_filename": "Mathlib.LinearAlgebra.DirectSum.Finsupp", "llama_tokens": 7921} |
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x y : M
⊢ (fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y
[PROOFSTEP]
rw [← AlgHom.map_add]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x y : M
⊢ (fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R x + FreeAlgebra.ι R y)
[PROOFSTEP]
exact RingQuot.mkAlgHom_rel R Rel.add
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
r : R
x : M
⊢ AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
x
[PROOFSTEP]
rw [← AlgHom.map_smul]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
r : R
x : M
⊢ AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
(r • x) =
↑(RingQuot.mkAlgHom R (Rel R M)) (↑(RingHom.id R) r • FreeAlgebra.ι R x)
[PROOFSTEP]
exact RingQuot.mkAlgHom_rel R Rel.smul
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m) = ↑(ι R) m
[PROOFSTEP]
rw [ι]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m) =
↑{
toAddHom :=
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) },
map_smul' :=
(_ :
∀ (r : R) (x : M),
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
x) }
m
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x y : FreeAlgebra R M
h : Rel R M x y
⊢ ↑(↑(FreeAlgebra.lift R) ↑f) x = ↑(↑(FreeAlgebra.lift R) ↑f) y
[PROOFSTEP]
induction h
[GOAL]
case add
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x y : FreeAlgebra R M
a✝ b✝ : M
⊢ ↑(↑(FreeAlgebra.lift R) ↑f) (FreeAlgebra.ι R (a✝ + b✝)) =
↑(↑(FreeAlgebra.lift R) ↑f) (FreeAlgebra.ι R a✝ + FreeAlgebra.ι R b✝)
[PROOFSTEP]
simp only [Algebra.smul_def, FreeAlgebra.lift_ι_apply, LinearMap.map_smulₛₗ, RingHom.id_apply, map_mul, AlgHom.commutes,
map_add]
[GOAL]
case smul
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x y : FreeAlgebra R M
r✝ : R
a✝ : M
⊢ ↑(↑(FreeAlgebra.lift R) ↑f) (FreeAlgebra.ι R (r✝ • a✝)) =
↑(↑(FreeAlgebra.lift R) ↑f) (↑(algebraMap R (FreeAlgebra R M)) r✝ * FreeAlgebra.ι R a✝)
[PROOFSTEP]
simp only [Algebra.smul_def, FreeAlgebra.lift_ι_apply, LinearMap.map_smulₛₗ, RingHom.id_apply, map_mul, AlgHom.commutes,
map_add]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
⊢ (fun F => LinearMap.comp (AlgHom.toLinearMap F) (ι R))
((↑(RingQuot.liftAlgHom R) ∘ fun f =>
{ val := ↑(FreeAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : FreeAlgebra R M),
Rel R M x y → ↑(↑(FreeAlgebra.lift R) ↑f) x = ↑(↑(FreeAlgebra.lift R) ↑f) y) })
f) =
f
[PROOFSTEP]
rw [ι]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
⊢ (fun F =>
LinearMap.comp (AlgHom.toLinearMap F)
{
toAddHom :=
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) },
map_smul' :=
(_ :
∀ (r : R) (x : M),
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
x) })
((↑(RingQuot.liftAlgHom R) ∘ fun f =>
{ val := ↑(FreeAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : FreeAlgebra R M),
Rel R M x y → ↑(↑(FreeAlgebra.lift R) ↑f) x = ↑(↑(FreeAlgebra.lift R) ↑f) y) })
f) =
f
[PROOFSTEP]
ext1 x
[GOAL]
case h
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x : M
⊢ ↑((fun F =>
LinearMap.comp (AlgHom.toLinearMap F)
{
toAddHom :=
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) },
map_smul' :=
(_ :
∀ (r : R) (x : M),
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
x) })
((↑(RingQuot.liftAlgHom R) ∘ fun f =>
{ val := ↑(FreeAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : FreeAlgebra R M),
Rel R M x y → ↑(↑(FreeAlgebra.lift R) ↑f) x = ↑(↑(FreeAlgebra.lift R) ↑f) y) })
f))
x =
↑f x
[PROOFSTEP]
exact (RingQuot.liftAlgHom_mkAlgHom_apply _ _ _ _).trans (FreeAlgebra.lift_ι_apply f x)
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
F : TensorAlgebra R M →ₐ[R] A
x : M
⊢ (↑(AlgHom.comp
((↑(RingQuot.liftAlgHom R) ∘ fun f =>
{ val := ↑(FreeAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : FreeAlgebra R M),
Rel R M x y → ↑(↑(FreeAlgebra.lift R) ↑f) x = ↑(↑(FreeAlgebra.lift R) ↑f) y) })
((fun F => LinearMap.comp (AlgHom.toLinearMap F) (ι R)) F))
(RingQuot.mkAlgHom R (Rel R M))) ∘
FreeAlgebra.ι R)
x =
(↑(AlgHom.comp F (RingQuot.mkAlgHom R (Rel R M))) ∘ FreeAlgebra.ι R) x
[PROOFSTEP]
rw [ι]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
F : TensorAlgebra R M →ₐ[R] A
x : M
⊢ (↑(AlgHom.comp
((↑(RingQuot.liftAlgHom R) ∘ fun f =>
{ val := ↑(FreeAlgebra.lift R) ↑f,
property :=
(_ :
∀ (x y : FreeAlgebra R M),
Rel R M x y → ↑(↑(FreeAlgebra.lift R) ↑f) x = ↑(↑(FreeAlgebra.lift R) ↑f) y) })
((fun F =>
LinearMap.comp (AlgHom.toLinearMap F)
{
toAddHom :=
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) },
map_smul' :=
(_ :
∀ (r : R) (x : M),
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
(r • x) =
↑(RingHom.id R) r •
AddHom.toFun
{ toFun := fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m),
map_add' :=
(_ :
∀ (x y : M),
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) (x + y) =
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) x +
(fun m => ↑(RingQuot.mkAlgHom R (Rel R M)) (FreeAlgebra.ι R m)) y) }
x) })
F))
(RingQuot.mkAlgHom R (Rel R M))) ∘
FreeAlgebra.ι R)
x =
(↑(AlgHom.comp F (RingQuot.mkAlgHom R (Rel R M))) ∘ FreeAlgebra.ι R) x
[PROOFSTEP]
exact (RingQuot.liftAlgHom_mkAlgHom_apply _ _ _ _).trans (FreeAlgebra.lift_ι_apply _ _)
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
⊢ LinearMap.comp (AlgHom.toLinearMap (↑(lift R) f)) (ι R) = f
[PROOFSTEP]
convert (lift R).symm_apply_apply f
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x : M
⊢ ↑(↑(lift R) f) (↑(ι R) x) = ↑f x
[PROOFSTEP]
conv_rhs => rw [← ι_comp_lift f]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x : M
| ↑f x
[PROOFSTEP]
rw [← ι_comp_lift f]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x : M
| ↑f x
[PROOFSTEP]
rw [← ι_comp_lift f]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
x : M
| ↑f x
[PROOFSTEP]
rw [← ι_comp_lift f]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
g : TensorAlgebra R M →ₐ[R] A
⊢ LinearMap.comp (AlgHom.toLinearMap g) (ι R) = f ↔ g = ↑(lift R) f
[PROOFSTEP]
rw [← (lift R).symm_apply_eq]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f : M →ₗ[R] A
g : TensorAlgebra R M →ₐ[R] A
⊢ LinearMap.comp (AlgHom.toLinearMap g) (ι R) = f ↔ ↑(lift R).symm g = f
[PROOFSTEP]
simp only [lift, Equiv.coe_fn_symm_mk]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
g : TensorAlgebra R M →ₐ[R] A
⊢ ↑(lift R) (LinearMap.comp (AlgHom.toLinearMap g) (ι R)) = g
[PROOFSTEP]
rw [← lift_symm_apply]
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
g : TensorAlgebra R M →ₐ[R] A
⊢ ↑(lift R) (↑(lift R).symm g) = g
[PROOFSTEP]
exact (lift R).apply_symm_apply g
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f g : TensorAlgebra R M →ₐ[R] A
w : LinearMap.comp (AlgHom.toLinearMap f) (ι R) = LinearMap.comp (AlgHom.toLinearMap g) (ι R)
⊢ f = g
[PROOFSTEP]
rw [← lift_symm_apply, ← lift_symm_apply] at w
[GOAL]
R : Type u_1
inst✝⁴ : CommSemiring R
M : Type u_2
inst✝³ : AddCommMonoid M
inst✝² : Module R M
A : Type u_3
inst✝¹ : Semiring A
inst✝ : Algebra R A
f g : TensorAlgebra R M →ₐ[R] A
w : ↑(lift R).symm f = ↑(lift R).symm g
⊢ f = g
[PROOFSTEP]
exact (lift R).symm.injective w
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
⊢ C a
[PROOFSTEP]
let s : Subalgebra R (TensorAlgebra R M) :=
{ carrier := C
mul_mem' := @h_mul
add_mem' := @h_add
algebraMap_mem' := h_grade0 }
-- porting note: Added `h`. `h` is needed for `of`.
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
⊢ C a
[PROOFSTEP]
let h : AddCommMonoid s := inferInstanceAs (AddCommMonoid (Subalgebra.toSubmodule s))
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
⊢ C a
[PROOFSTEP]
let of : M →ₗ[R] s := (ι R).codRestrict (Subalgebra.toSubmodule s) h_grade1
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : M →ₗ[R] { x // x ∈ s } := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1
⊢ C a
[PROOFSTEP]
have of_id : AlgHom.id R (TensorAlgebra R M) = s.val.comp (lift R of) :=
by
ext
simp
erw [LinearMap.codRestrict_apply]
-- finding a proof is finding an element of the subalgebra
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : M →ₗ[R] { x // x ∈ s } := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1
⊢ AlgHom.id R (TensorAlgebra R M) = AlgHom.comp (Subalgebra.val s) (↑(lift R) of)
[PROOFSTEP]
ext
[GOAL]
case w.h
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : M →ₗ[R] { x // x ∈ s } := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1
x✝ : M
⊢ ↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (TensorAlgebra R M))) (ι R)) x✝ =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.comp (Subalgebra.val s) (↑(lift R) of))) (ι R)) x✝
[PROOFSTEP]
simp
[GOAL]
case w.h
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : M →ₗ[R] { x // x ∈ s } := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1
x✝ : M
⊢ ↑(ι R) x✝ = ↑(↑(LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1) x✝)
[PROOFSTEP]
erw [LinearMap.codRestrict_apply]
-- finding a proof is finding an element of the subalgebra
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : M →ₗ[R] { x // x ∈ s } := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1
of_id : AlgHom.id R (TensorAlgebra R M) = AlgHom.comp (Subalgebra.val s) (↑(lift R) of)
⊢ C a
[PROOFSTEP]
rw [← AlgHom.id_apply (R := R) a, of_id]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
C : TensorAlgebra R M → Prop
h_grade0 : ∀ (r : R), C (↑(algebraMap R (TensorAlgebra R M)) r)
h_grade1 : ∀ (x : M), C (↑(ι R) x)
h_mul : ∀ (a b : TensorAlgebra R M), C a → C b → C (a * b)
h_add : ∀ (a b : TensorAlgebra R M), C a → C b → C (a + b)
a : TensorAlgebra R M
s : Subalgebra R (TensorAlgebra R M) :=
{
toSubsemiring :=
{ toSubmonoid := { toSubsemigroup := { carrier := C, mul_mem' := h_mul }, one_mem' := (_ : 1 ∈ C) },
add_mem' := h_add, zero_mem' := (_ : 0 ∈ C) },
algebraMap_mem' := h_grade0 }
h : AddCommMonoid { x // x ∈ s } := inferInstanceAs (AddCommMonoid { x // x ∈ ↑Subalgebra.toSubmodule s })
of : M →ₗ[R] { x // x ∈ s } := LinearMap.codRestrict (↑Subalgebra.toSubmodule s) (ι R) h_grade1
of_id : AlgHom.id R (TensorAlgebra R M) = AlgHom.comp (Subalgebra.val s) (↑(lift R) of)
⊢ C (↑(AlgHom.comp (Subalgebra.val s) (↑(lift R) of)) a)
[PROOFSTEP]
exact Subtype.prop (lift R of a)
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : R
⊢ ↑algebraMapInv (↑(algebraMap R (TensorAlgebra R M)) x) = x
[PROOFSTEP]
simp [algebraMapInv]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ TensorAlgebra R M →ₗ[R] M
[PROOFSTEP]
letI : Module Rᵐᵒᵖ M := Module.compHom _ ((RingHom.id R).fromOpposite mul_comm)
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
this : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
⊢ TensorAlgebra R M →ₗ[R] M
[PROOFSTEP]
haveI : IsCentralScalar R M := ⟨fun r m => rfl⟩
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
this✝ : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
this : IsCentralScalar R M
⊢ TensorAlgebra R M →ₗ[R] M
[PROOFSTEP]
exact (TrivSqZeroExt.sndHom R M).comp toTrivSqZeroExt.toLinearMap
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
⊢ ↑ιInv (↑(ι R) x) = x
[PROOFSTEP]
simp [ιInv, (AlgHom.toLinearMap_apply), toTrivSqZeroExt_ι _]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
⊢ ↑(ι R) x = 0 ↔ x = 0
[PROOFSTEP]
rw [← ι_inj R x 0, LinearMap.map_zero]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
⊢ ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r ↔ x = 0 ∧ r = 0
[PROOFSTEP]
refine' ⟨fun h => _, _⟩
[GOAL]
case refine'_1
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
h : ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
⊢ x = 0 ∧ r = 0
[PROOFSTEP]
letI : Module Rᵐᵒᵖ M := Module.compHom _ ((RingHom.id R).fromOpposite mul_comm)
[GOAL]
case refine'_1
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
h : ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
this : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
⊢ x = 0 ∧ r = 0
[PROOFSTEP]
haveI : IsCentralScalar R M := ⟨fun r m => rfl⟩
[GOAL]
case refine'_1
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
h : ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
this✝ : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
this : IsCentralScalar R M
⊢ x = 0 ∧ r = 0
[PROOFSTEP]
have hf0 : toTrivSqZeroExt (ι R x) = (0, x) := lift_ι_apply _ _
[GOAL]
case refine'_1
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
h : ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
this✝ : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
this : IsCentralScalar R M
hf0 : ↑toTrivSqZeroExt (↑(ι R) x) = (0, x)
⊢ x = 0 ∧ r = 0
[PROOFSTEP]
rw [h, AlgHom.commutes] at hf0
[GOAL]
case refine'_1
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
h : ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
this✝ : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
this : IsCentralScalar R M
hf0 : ↑(algebraMap R (TrivSqZeroExt R M)) r = (0, x)
⊢ x = 0 ∧ r = 0
[PROOFSTEP]
have : r = 0 ∧ 0 = x := Prod.ext_iff.1 hf0
[GOAL]
case refine'_1
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
h : ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
this✝¹ : Module Rᵐᵒᵖ M := Module.compHom M (RingHom.fromOpposite (RingHom.id R) (_ : ∀ (a b : R), a * b = b * a))
this✝ : IsCentralScalar R M
hf0 : ↑(algebraMap R (TrivSqZeroExt R M)) r = (0, x)
this : r = 0 ∧ 0 = x
⊢ x = 0 ∧ r = 0
[PROOFSTEP]
exact this.symm.imp_left Eq.symm
[GOAL]
case refine'_2
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
⊢ x = 0 ∧ r = 0 → ↑(ι R) x = ↑(algebraMap R (TensorAlgebra R M)) r
[PROOFSTEP]
rintro ⟨rfl, rfl⟩
[GOAL]
case refine'_2.intro
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ ↑(ι R) 0 = ↑(algebraMap R (TensorAlgebra R M)) 0
[PROOFSTEP]
rw [LinearMap.map_zero, RingHom.map_zero]
[GOAL]
R : Type u_1
inst✝³ : CommSemiring R
M : Type u_2
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : Nontrivial R
x : M
⊢ ↑(ι R) x ≠ 1
[PROOFSTEP]
rw [← (algebraMap R (TensorAlgebra R M)).map_one, Ne.def, ι_eq_algebraMap_iff]
[GOAL]
R : Type u_1
inst✝³ : CommSemiring R
M : Type u_2
inst✝² : AddCommMonoid M
inst✝¹ : Module R M
inst✝ : Nontrivial R
x : M
⊢ ¬(x = 0 ∧ 1 = 0)
[PROOFSTEP]
exact one_ne_zero ∘ And.right
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ Disjoint (LinearMap.range (ι R)) 1
[PROOFSTEP]
rw [Submodule.disjoint_def]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ ∀ (x : TensorAlgebra R M), x ∈ LinearMap.range (ι R) → x ∈ 1 → x = 0
[PROOFSTEP]
rintro _ ⟨x, hx⟩ ⟨r, rfl⟩
[GOAL]
case intro.intro
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
hx : ↑(ι R) x = ↑(Algebra.linearMap R (TensorAlgebra R M)) r
⊢ ↑(Algebra.linearMap R (TensorAlgebra R M)) r = 0
[PROOFSTEP]
rw [Algebra.linearMap_apply, ι_eq_algebraMap_iff] at hx
[GOAL]
case intro.intro
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x : M
r : R
hx : x = 0 ∧ r = 0
⊢ ↑(Algebra.linearMap R (TensorAlgebra R M)) r = 0
[PROOFSTEP]
rw [hx.2, map_zero]
[GOAL]
R : Type u_1
inst✝² : CommSemiring R
M : Type u_2
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑toTensor (ι R m) = ↑(TensorAlgebra.ι R) m
[PROOFSTEP]
simp [toTensor]
| {"mathlib_filename": "Mathlib.LinearAlgebra.TensorAlgebra.Basic", "llama_tokens": 14221} |
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : ι' → ι
hf : LocallyFinite f
hg : InjOn g {i | Set.Nonempty (f (g i))}
x : X
⊢ ∃ t, t ∈ 𝓝 x ∧ Set.Finite {i | Set.Nonempty ((f ∘ g) i ∩ t)}
[PROOFSTEP]
let ⟨t, htx, htf⟩ := hf x
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : ι' → ι
hf : LocallyFinite f
hg : InjOn g {i | Set.Nonempty (f (g i))}
x : X
t : Set X
htx : t ∈ 𝓝 x
htf : Set.Finite {i | Set.Nonempty (f i ∩ t)}
⊢ ∃ t, t ∈ 𝓝 x ∧ Set.Finite {i | Set.Nonempty ((f ∘ g) i ∩ t)}
[PROOFSTEP]
refine ⟨t, htx, htf.preimage <| ?_⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : ι' → ι
hf : LocallyFinite f
hg : InjOn g {i | Set.Nonempty (f (g i))}
x : X
t : Set X
htx : t ∈ 𝓝 x
htf : Set.Finite {i | Set.Nonempty (f i ∩ t)}
⊢ InjOn (fun i => g i) ((fun i => g i) ⁻¹' {i | Set.Nonempty (f i ∩ t)})
[PROOFSTEP]
exact hg.mono fun i (hi : Set.Nonempty _) => hi.left
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
a : X
⊢ 𝓝[⋃ (i : ι), f i] a = ⨆ (i : ι), 𝓝[f i] a
[PROOFSTEP]
rcases hf a with ⟨U, haU, hfin⟩
[GOAL]
case intro.intro
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
a : X
U : Set X
haU : U ∈ 𝓝 a
hfin : Set.Finite {i | Set.Nonempty (f i ∩ U)}
⊢ 𝓝[⋃ (i : ι), f i] a = ⨆ (i : ι), 𝓝[f i] a
[PROOFSTEP]
refine le_antisymm ?_ (Monotone.le_map_iSup fun _ _ ↦ nhdsWithin_mono _)
[GOAL]
case intro.intro
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
a : X
U : Set X
haU : U ∈ 𝓝 a
hfin : Set.Finite {i | Set.Nonempty (f i ∩ U)}
⊢ 𝓝[⋃ (i : ι), f i] a ≤ ⨆ (i : ι), 𝓝[f i] a
[PROOFSTEP]
calc
𝓝[⋃ i, f i] a = 𝓝[⋃ i, f i ∩ U] a := by rw [← iUnion_inter, ← nhdsWithin_inter_of_mem' (nhdsWithin_le_nhds haU)]
_ = 𝓝[⋃ i ∈ {j | (f j ∩ U).Nonempty}, (f i ∩ U)] a := by simp only [mem_setOf_eq, iUnion_nonempty_self]
_ = ⨆ i ∈ {j | (f j ∩ U).Nonempty}, 𝓝[f i ∩ U] a := (nhdsWithin_biUnion hfin _ _)
_ ≤ ⨆ i, 𝓝[f i ∩ U] a := (iSup₂_le_iSup _ _)
_ ≤ ⨆ i, 𝓝[f i] a := iSup_mono fun i ↦ nhdsWithin_mono _ <| inter_subset_left _ _
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
a : X
U : Set X
haU : U ∈ 𝓝 a
hfin : Set.Finite {i | Set.Nonempty (f i ∩ U)}
⊢ 𝓝[⋃ (i : ι), f i] a = 𝓝[⋃ (i : ι), f i ∩ U] a
[PROOFSTEP]
rw [← iUnion_inter, ← nhdsWithin_inter_of_mem' (nhdsWithin_le_nhds haU)]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
a : X
U : Set X
haU : U ∈ 𝓝 a
hfin : Set.Finite {i | Set.Nonempty (f i ∩ U)}
⊢ 𝓝[⋃ (i : ι), f i ∩ U] a = 𝓝[⋃ (i : ι) (_ : i ∈ {j | Set.Nonempty (f j ∩ U)}), f i ∩ U] a
[PROOFSTEP]
simp only [mem_setOf_eq, iUnion_nonempty_self]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
⊢ ContinuousOn g (⋃ (i : ι), f i)
[PROOFSTEP]
rintro x -
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
⊢ ContinuousWithinAt g (⋃ (i : ι), f i) x
[PROOFSTEP]
rw [ContinuousWithinAt, hf.nhdsWithin_iUnion, tendsto_iSup]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
⊢ ∀ (i : ι), Tendsto g (𝓝[f i] x) (𝓝 (g x))
[PROOFSTEP]
intro i
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
i : ι
⊢ Tendsto g (𝓝[f i] x) (𝓝 (g x))
[PROOFSTEP]
by_cases hx : x ∈ closure (f i)
[GOAL]
case pos
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
i : ι
hx : x ∈ closure (f i)
⊢ Tendsto g (𝓝[f i] x) (𝓝 (g x))
[PROOFSTEP]
exact hc i _ hx
[GOAL]
case neg
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
i : ι
hx : ¬x ∈ closure (f i)
⊢ Tendsto g (𝓝[f i] x) (𝓝 (g x))
[PROOFSTEP]
rw [mem_closure_iff_nhdsWithin_neBot, not_neBot] at hx
[GOAL]
case neg
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
i : ι
hx : 𝓝[f i] x = ⊥
⊢ Tendsto g (𝓝[f i] x) (𝓝 (g x))
[PROOFSTEP]
rw [hx]
[GOAL]
case neg
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g✝ : ι → Set X
g : X → Y
hf : LocallyFinite f
hc : ∀ (i : ι) (x : X), x ∈ closure (f i) → ContinuousWithinAt g (f i) x
x : X
i : ι
hx : 𝓝[f i] x = ⊥
⊢ Tendsto g ⊥ (𝓝 (g x))
[PROOFSTEP]
exact tendsto_bot
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
⊢ LocallyFinite fun i => closure (f i)
[PROOFSTEP]
intro x
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
x : X
⊢ ∃ t, t ∈ 𝓝 x ∧ Set.Finite {i | Set.Nonempty ((fun i => closure (f i)) i ∩ t)}
[PROOFSTEP]
rcases hf x with ⟨s, hsx, hsf⟩
[GOAL]
case intro.intro
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
x : X
s : Set X
hsx : s ∈ 𝓝 x
hsf : Set.Finite {i | Set.Nonempty (f i ∩ s)}
⊢ ∃ t, t ∈ 𝓝 x ∧ Set.Finite {i | Set.Nonempty ((fun i => closure (f i)) i ∩ t)}
[PROOFSTEP]
refine' ⟨interior s, interior_mem_nhds.2 hsx, hsf.subset fun i hi => _⟩
[GOAL]
case intro.intro
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
x : X
s : Set X
hsx : s ∈ 𝓝 x
hsf : Set.Finite {i | Set.Nonempty (f i ∩ s)}
i : ι
hi : i ∈ {i | Set.Nonempty ((fun i => closure (f i)) i ∩ interior s)}
⊢ i ∈ {i | Set.Nonempty (f i ∩ s)}
[PROOFSTEP]
exact (hi.mono isOpen_interior.closure_inter).of_closure.mono (inter_subset_inter_right _ interior_subset)
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
h : LocallyFinite f
⊢ closure (⋃ (i : ι), f i) = ⋃ (i : ι), closure (f i)
[PROOFSTEP]
ext x
[GOAL]
case h
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
h : LocallyFinite f
x : X
⊢ x ∈ closure (⋃ (i : ι), f i) ↔ x ∈ ⋃ (i : ι), closure (f i)
[PROOFSTEP]
simp only [mem_closure_iff_nhdsWithin_neBot, h.nhdsWithin_iUnion, iSup_neBot, mem_iUnion]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
hc : ∀ (i : ι), IsClosed (f i)
⊢ IsClosed (⋃ (i : ι), f i)
[PROOFSTEP]
simp only [← closure_eq_iff_isClosed, hf.closure_iUnion, (hc _).closure_eq]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
hc : ∀ (i : ι), IsClosed (f i)
x : X
⊢ ⋂ (i : ι) (_ : ¬x ∈ f i), (f i)ᶜ ∈ 𝓝 x
[PROOFSTEP]
refine' IsOpen.mem_nhds _ (mem_iInter₂.2 fun i => id)
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
hc : ∀ (i : ι), IsClosed (f i)
x : X
⊢ IsOpen (⋂ (i : ι) (_ : ¬x ∈ f i), (f i)ᶜ)
[PROOFSTEP]
suffices IsClosed (⋃ i : { i // x ∉ f i }, f i) by rwa [← isOpen_compl_iff, compl_iUnion, iInter_subtype] at this
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
hc : ∀ (i : ι), IsClosed (f i)
x : X
this : IsClosed (⋃ (i : { i // ¬x ∈ f i }), f ↑i)
⊢ IsOpen (⋂ (i : ι) (_ : ¬x ∈ f i), (f i)ᶜ)
[PROOFSTEP]
rwa [← isOpen_compl_iff, compl_iUnion, iInter_subtype] at this
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
hf : LocallyFinite f
hc : ∀ (i : ι), IsClosed (f i)
x : X
⊢ IsClosed (⋃ (i : { i // ¬x ∈ f i }), f ↑i)
[PROOFSTEP]
exact (hf.comp_injective Subtype.val_injective).isClosed_iUnion fun i => hc _
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
hf : LocallyFinite fun n => {x | f (n + 1) x ≠ f n x}
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
choose U hUx hU using hf
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
choose N hN using fun x => (hU x).bddAbove
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X), N x ∈ upperBounds {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
replace hN : ∀ (x), ∀ n > N x, ∀ y ∈ U x, f (n + 1) y = f n y
[GOAL]
case hN
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X), N x ∈ upperBounds {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
⊢ ∀ (x : X) (n : ℕ), n > N x → ∀ (y : X), y ∈ U x → f (n + 1) y = f n y
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n > N x → ∀ (y : X), y ∈ U x → f (n + 1) y = f n y
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
exact fun x n hn y hy => by_contra fun hne => hn.lt.not_le <| hN x ⟨y, hne, hy⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n > N x → ∀ (y : X), y ∈ U x → f (n + 1) y = f n y
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
replace hN : ∀ (x), ∀ n ≥ N x + 1, ∀ y ∈ U x, f n y = f (N x + 1) y
[GOAL]
case hN
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n > N x → ∀ (y : X), y ∈ U x → f (n + 1) y = f n y
⊢ ∀ (x : X) (n : ℕ), n ≥ N x + 1 → ∀ (y : X), y ∈ U x → f n y = f (N x + 1) y
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n ≥ N x + 1 → ∀ (y : X), y ∈ U x → f n y = f (N x + 1) y
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
exact fun x n hn y hy => Nat.le_induction rfl (fun k hle => (hN x _ hle _ hy).trans) n hn
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n ≥ N x + 1 → ∀ (y : X), y ∈ U x → f n y = f (N x + 1) y
⊢ ∃ F, ∀ (x : X), ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = F p.snd
[PROOFSTEP]
refine ⟨fun x => f (N x + 1) x, fun x => ?_⟩
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n ≥ N x + 1 → ∀ (y : X), y ∈ U x → f n y = f (N x + 1) y
x : X
⊢ ∀ᶠ (p : ℕ × X) in atTop ×ˢ 𝓝 x, f p.fst p.snd = (fun x => f (N x + 1) x) p.snd
[PROOFSTEP]
filter_upwards [Filter.prod_mem_prod (eventually_gt_atTop (N x)) (hUx x)]
[GOAL]
case h
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n ≥ N x + 1 → ∀ (y : X), y ∈ U x → f n y = f (N x + 1) y
x : X
⊢ ∀ (a : ℕ × X), a ∈ {x_1 | N x < x_1} ×ˢ U x → f a.fst a.snd = f (N a.snd + 1) a.snd
[PROOFSTEP]
rintro ⟨n, y⟩ ⟨hn : N x < n, hy : y ∈ U x⟩
[GOAL]
case h.mk.intro
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
π : X → Sort u_6
f : ℕ → (x : X) → π x
U : X → Set X
hUx : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty ((fun n => {x | f (n + 1) x ≠ f n x}) i ∩ U x)}
N : X → ℕ
hN : ∀ (x : X) (n : ℕ), n ≥ N x + 1 → ∀ (y : X), y ∈ U x → f n y = f (N x + 1) y
x : X
n : ℕ
y : X
hn : N x < n
hy : y ∈ U x
⊢ f (n, y).fst (n, y).snd = f (N (n, y).snd + 1) (n, y).snd
[PROOFSTEP]
calc
f n y = f (N x + 1) y := hN _ _ hn _ hy
_ = f (max (N x + 1) (N y + 1)) y := (hN _ _ (le_max_left _ _) _ hy).symm
_ = f (N y + 1) y := hN _ _ (le_max_right _ _) _ (mem_of_mem_nhds <| hUx y)
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f g : ι → Set X
e : ι' ≃ ι
h : LocallyFinite (f ∘ ↑e)
⊢ LocallyFinite f
[PROOFSTEP]
simpa only [(· ∘ ·), e.apply_symm_apply] using h.comp_injective e.symm.injective
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
f : ι ⊕ ι' → Set X
⊢ LocallyFinite f ↔ LocallyFinite (f ∘ Sum.inl) ∧ LocallyFinite (f ∘ Sum.inr)
[PROOFSTEP]
simp only [locallyFinite_iff_smallSets, ← forall_and, ← finite_preimage_inl_and_inr, preimage_setOf_eq, (· ∘ ·),
eventually_and]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
f : Option ι → Set X
⊢ LocallyFinite f ↔ LocallyFinite (f ∘ some)
[PROOFSTEP]
rw [← (Equiv.optionEquivSumPUnit.{_, 0} ι).symm.locallyFinite_comp_iff, locallyFinite_sum]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
f : Option ι → Set X
⊢ LocallyFinite ((f ∘ ↑(Equiv.optionEquivSumPUnit ι).symm) ∘ Sum.inl) ∧
LocallyFinite ((f ∘ ↑(Equiv.optionEquivSumPUnit ι).symm) ∘ Sum.inr) ↔
LocallyFinite (f ∘ some)
[PROOFSTEP]
simp only [locallyFinite_of_finite, and_true]
[GOAL]
ι : Type u_1
ι' : Type u_2
α : Type u_3
X : Type u_4
Y : Type u_5
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f✝ g : ι → Set X
f : Option ι → Set X
⊢ LocallyFinite ((f ∘ ↑(Equiv.optionEquivSumPUnit ι).symm) ∘ Sum.inl) ↔ LocallyFinite (f ∘ some)
[PROOFSTEP]
rfl
| {"mathlib_filename": "Mathlib.Topology.LocallyFinite", "llama_tokens": 9642} |
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
⊢ IsLocallyHomeomorphOn f s
[PROOFSTEP]
intro x hx
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx : x ∈ s
⊢ ∃ e, x ∈ e.source ∧ f = ↑e
[PROOFSTEP]
obtain ⟨e, hx, he⟩ := h x hx
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx✝ : x ∈ s
e : LocalHomeomorph X Y
hx : x ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
⊢ ∃ e, x ∈ e.source ∧ f = ↑e
[PROOFSTEP]
exact
⟨{ e with
toFun := f
map_source' := fun x hx => by rw [he x hx]; exact e.map_source' hx
left_inv' := fun x hx => by rw [he x hx]; exact e.left_inv' hx
right_inv' := fun y hy => by rw [he _ (e.map_target' hy)]; exact e.right_inv' hy
continuous_toFun := (continuousOn_congr he).mpr e.continuous_toFun },
hx, rfl⟩
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x✝ : X
hx✝¹ : x✝ ∈ s
e : LocalHomeomorph X Y
hx✝ : x✝ ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx : x ∈ e.source
⊢ f x ∈ e.target
[PROOFSTEP]
rw [he x hx]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x✝ : X
hx✝¹ : x✝ ∈ s
e : LocalHomeomorph X Y
hx✝ : x✝ ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx : x ∈ e.source
⊢ ↑e x ∈ e.target
[PROOFSTEP]
exact e.map_source' hx
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x✝ : X
hx✝¹ : x✝ ∈ s
e : LocalHomeomorph X Y
hx✝ : x✝ ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx : x ∈ e.source
⊢ LocalEquiv.invFun e.toLocalEquiv (f x) = x
[PROOFSTEP]
rw [he x hx]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x✝ : X
hx✝¹ : x✝ ∈ s
e : LocalHomeomorph X Y
hx✝ : x✝ ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx : x ∈ e.source
⊢ LocalEquiv.invFun e.toLocalEquiv (↑e x) = x
[PROOFSTEP]
exact e.left_inv' hx
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx✝ : x ∈ s
e : LocalHomeomorph X Y
hx : x ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
y : Y
hy : y ∈ e.target
⊢ f (LocalEquiv.invFun e.toLocalEquiv y) = y
[PROOFSTEP]
rw [he _ (e.map_target' hy)]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
h : ∀ (x : X), x ∈ s → ∃ e, x ∈ e.source ∧ ∀ (y : X), y ∈ e.source → f y = ↑e y
x : X
hx✝ : x ∈ s
e : LocalHomeomorph X Y
hx : x ∈ e.source
he : ∀ (y : X), y ∈ e.source → f y = ↑e y
y : Y
hy : y ∈ e.target
⊢ ↑e (LocalEquiv.invFun e.toLocalEquiv y) = y
[PROOFSTEP]
exact e.right_inv' hy
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
hg : IsLocallyHomeomorphOn g t
hf : IsLocallyHomeomorphOn f s
h : Set.MapsTo f s t
⊢ IsLocallyHomeomorphOn (g ∘ f) s
[PROOFSTEP]
intro x hx
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
hg : IsLocallyHomeomorphOn g t
hf : IsLocallyHomeomorphOn f s
h : Set.MapsTo f s t
x : X
hx : x ∈ s
⊢ ∃ e, x ∈ e.source ∧ g ∘ f = ↑e
[PROOFSTEP]
obtain ⟨eg, hxg, rfl⟩ := hg (f x) (h hx)
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
f : X → Y
s : Set X
t : Set Y
hf : IsLocallyHomeomorphOn f s
h : Set.MapsTo f s t
x : X
hx : x ∈ s
eg : LocalHomeomorph Y Z
hxg : f x ∈ eg.source
hg : IsLocallyHomeomorphOn (↑eg) t
⊢ ∃ e, x ∈ e.source ∧ ↑eg ∘ f = ↑e
[PROOFSTEP]
obtain ⟨ef, hxf, rfl⟩ := hf x hx
[GOAL]
case intro.intro.intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
s : Set X
t : Set Y
x : X
hx : x ∈ s
eg : LocalHomeomorph Y Z
hg : IsLocallyHomeomorphOn (↑eg) t
ef : LocalHomeomorph X Y
hxf : x ∈ ef.source
hf : IsLocallyHomeomorphOn (↑ef) s
h : Set.MapsTo (↑ef) s t
hxg : ↑ef x ∈ eg.source
⊢ ∃ e, x ∈ e.source ∧ ↑eg ∘ ↑ef = ↑e
[PROOFSTEP]
exact ⟨ef.trans eg, ⟨hxf, hxg⟩, rfl⟩
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
g : Y → Z
f : X → Y
s : Set X
t : Set Y
⊢ IsLocallyHomeomorph f ↔ IsLocallyHomeomorphOn f Set.univ
[PROOFSTEP]
simp only [IsLocallyHomeomorph, IsLocallyHomeomorphOn, Set.mem_univ, forall_true_left]
| {"mathlib_filename": "Mathlib.Topology.IsLocallyHomeomorph", "llama_tokens": 3034} |
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ Tendsto f cofinite (cocompact Y) ↔ ∀ (K : Set Y), IsCompact K → Set.Finite (f ⁻¹' K)
[PROOFSTEP]
rw [hasBasis_cocompact.tendsto_right_iff]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ (∀ (i : Set Y), IsCompact i → ∀ᶠ (x : X) in cofinite, f x ∈ iᶜ) ↔ ∀ (K : Set Y), IsCompact K → Set.Finite (f ⁻¹' K)
[PROOFSTEP]
refine' forall₂_congr (fun K _ ↦ _)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
K : Set Y
x✝ : IsCompact K
⊢ (∀ᶠ (x : X) in cofinite, f x ∈ Kᶜ) ↔ Set.Finite (f ⁻¹' K)
[PROOFSTEP]
simp only [mem_compl_iff, eventually_cofinite, not_not, preimage]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
f : X → Y
inst✝¹ : T1Space X
inst✝ : LocallyCompactSpace Y
hf' : Continuous f
hf : Tendsto f cofinite (cocompact Y)
⊢ DiscreteTopology X
[PROOFSTEP]
refine' singletons_open_iff_discrete.mp (fun x ↦ _)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
f : X → Y
inst✝¹ : T1Space X
inst✝ : LocallyCompactSpace Y
hf' : Continuous f
hf : Tendsto f cofinite (cocompact Y)
x : X
⊢ IsOpen {x}
[PROOFSTEP]
obtain ⟨K : Set Y, hK : IsCompact K, hK' : K ∈ 𝓝 (f x)⟩ := exists_compact_mem_nhds (f x)
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
f : X → Y
inst✝¹ : T1Space X
inst✝ : LocallyCompactSpace Y
hf' : Continuous f
hf : Tendsto f cofinite (cocompact Y)
x : X
K : Set Y
hK : IsCompact K
hK' : K ∈ 𝓝 (f x)
⊢ IsOpen {x}
[PROOFSTEP]
obtain ⟨U : Set Y, hU₁ : U ⊆ K, hU₂ : IsOpen U, hU₃ : f x ∈ U⟩ := mem_nhds_iff.mp hK'
[GOAL]
case intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
f : X → Y
inst✝¹ : T1Space X
inst✝ : LocallyCompactSpace Y
hf' : Continuous f
hf : Tendsto f cofinite (cocompact Y)
x : X
K : Set Y
hK : IsCompact K
hK' : K ∈ 𝓝 (f x)
U : Set Y
hU₁ : U ⊆ K
hU₂ : IsOpen U
hU₃ : f x ∈ U
⊢ IsOpen {x}
[PROOFSTEP]
have hU₄ : Set.Finite (f ⁻¹' U) := Finite.subset (tendsto_cofinite_cocompact_iff.mp hf K hK) (preimage_mono hU₁)
[GOAL]
case intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
f : X → Y
inst✝¹ : T1Space X
inst✝ : LocallyCompactSpace Y
hf' : Continuous f
hf : Tendsto f cofinite (cocompact Y)
x : X
K : Set Y
hK : IsCompact K
hK' : K ∈ 𝓝 (f x)
U : Set Y
hU₁ : U ⊆ K
hU₂ : IsOpen U
hU₃ : f x ∈ U
hU₄ : Set.Finite (f ⁻¹' U)
⊢ IsOpen {x}
[PROOFSTEP]
exact isOpen_singleton_of_finite_mem_nhds _ ((hU₂.preimage hf').mem_nhds hU₃) hU₄
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
f : X → Y
inst✝ : DiscreteTopology X
hf : Tendsto f (cocompact X) (cocompact Y)
⊢ Tendsto f cofinite (cocompact Y)
[PROOFSTEP]
convert hf
[GOAL]
case h.e'_4
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
f : X → Y
inst✝ : DiscreteTopology X
hf : Tendsto f (cocompact X) (cocompact Y)
⊢ cofinite = cocompact X
[PROOFSTEP]
rw [cocompact_eq_cofinite X]
| {"mathlib_filename": "Mathlib.Topology.DiscreteSubset", "llama_tokens": 1588} |
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have h3 : (0 : ℝ) < 3 := by norm_num1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
⊢ 0 < 3
[PROOFSTEP]
norm_num1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have h23 : 0 < (2 / 3 : ℝ) := by
norm_num1
-- In the trivial case `f = 0`, we take `g = 0`
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
⊢ 0 < 2 / 3
[PROOFSTEP]
norm_num1
-- In the trivial case `f = 0`, we take `g = 0`
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
rcases eq_or_ne f 0 with (rfl | hf)
[GOAL]
case inl
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
⊢ ∃ g, ‖g‖ ≤ ‖0‖ / 3 ∧ dist (compContinuous g e) 0 ≤ 2 / 3 * ‖0‖
[PROOFSTEP]
use 0
[GOAL]
case h
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
⊢ ‖0‖ ≤ ‖0‖ / 3 ∧ dist (compContinuous 0 e) 0 ≤ 2 / 3 * ‖0‖
[PROOFSTEP]
simp
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : f ≠ 0
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
replace hf : 0 < ‖f‖ := norm_pos_iff.2 hf
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have hf3 : -‖f‖ / 3 < ‖f‖ / 3 := (div_lt_div_right h3).2 (Left.neg_lt_self hf)
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have hc₁ : IsClosed (e '' (f ⁻¹' Iic (-‖f‖ / 3))) := he.isClosedMap _ (isClosed_Iic.preimage f.continuous)
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have hc₂ : IsClosed (e '' (f ⁻¹' Ici (‖f‖ / 3))) := he.isClosedMap _ (isClosed_Ici.preimage f.continuous)
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have hd : Disjoint (e '' (f ⁻¹' Iic (-‖f‖ / 3))) (e '' (f ⁻¹' Ici (‖f‖ / 3))) :=
by
refine' disjoint_image_of_injective he.inj (Disjoint.preimage _ _)
rwa [Iic_disjoint_Ici, not_le]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
⊢ Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
[PROOFSTEP]
refine' disjoint_image_of_injective he.inj (Disjoint.preimage _ _)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
⊢ Disjoint (Iic (-‖f‖ / 3)) (Ici (‖f‖ / 3))
[PROOFSTEP]
rwa [Iic_disjoint_Ici, not_le]
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
rcases exists_bounded_mem_Icc_of_closed_of_le hc₁ hc₂ hd hf3.le with ⟨g, hg₁, hg₂, hgf⟩
[GOAL]
case inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
⊢ ∃ g, ‖g‖ ≤ ‖f‖ / 3 ∧ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
refine' ⟨g, _, _⟩
[GOAL]
case inr.intro.intro.intro.refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
⊢ ‖g‖ ≤ ‖f‖ / 3
[PROOFSTEP]
refine' (norm_le <| div_nonneg hf.le h3.le).mpr fun y => _
[GOAL]
case inr.intro.intro.intro.refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
y : Y
⊢ ‖↑g y‖ ≤ ‖f‖ / 3
[PROOFSTEP]
simpa [abs_le, neg_div] using hgf y
[GOAL]
case inr.intro.intro.intro.refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
⊢ dist (compContinuous g e) f ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
refine' (dist_le <| mul_nonneg h23.le hf.le).mpr fun x => _
[GOAL]
case inr.intro.intro.intro.refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
have hfx : -‖f‖ ≤ f x ∧ f x ≤ ‖f‖ := by simpa only [Real.norm_eq_abs, abs_le] using f.norm_coe_le_norm x
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
⊢ -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
[PROOFSTEP]
simpa only [Real.norm_eq_abs, abs_le] using f.norm_coe_le_norm x
[GOAL]
case inr.intro.intro.intro.refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
cases' le_total (f x) (-‖f‖ / 3) with hle₁ hle₁
[GOAL]
case inr.intro.intro.intro.refine'_2.inl
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : ↑f x ≤ -‖f‖ / 3
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
calc
|g (e x) - f x| = -‖f‖ / 3 - f x := by
rw [hg₁ (mem_image_of_mem _ hle₁), Function.const_apply, abs_of_nonneg (sub_nonneg.2 hle₁)]
_ ≤ 2 / 3 * ‖f‖ := by linarith
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : ↑f x ≤ -‖f‖ / 3
⊢ |↑g (↑e x) - ↑f x| = -‖f‖ / 3 - ↑f x
[PROOFSTEP]
rw [hg₁ (mem_image_of_mem _ hle₁), Function.const_apply, abs_of_nonneg (sub_nonneg.2 hle₁)]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : ↑f x ≤ -‖f‖ / 3
⊢ -‖f‖ / 3 - ↑f x ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
linarith
[GOAL]
case inr.intro.intro.intro.refine'_2.inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : -‖f‖ / 3 ≤ ↑f x
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
cases' le_total (f x) (‖f‖ / 3) with hle₂ hle₂
[GOAL]
case inr.intro.intro.intro.refine'_2.inr.inl
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : -‖f‖ / 3 ≤ ↑f x
hle₂ : ↑f x ≤ ‖f‖ / 3
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
simp only [neg_div] at *
[GOAL]
case inr.intro.intro.intro.refine'_2.inr.inl
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
g : Y →ᵇ ℝ
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₂ : ↑f x ≤ ‖f‖ / 3
hf3 : -(‖f‖ / 3) < ‖f‖ / 3
hc₁ : IsClosed ((fun a => ↑e a) '' (↑f ⁻¹' Iic (-(‖f‖ / 3))))
hc₂ : IsClosed ((fun a => ↑e a) '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint ((fun a => ↑e a) '' (↑f ⁻¹' Iic (-(‖f‖ / 3)))) ((fun a => ↑e a) '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hg₁ : EqOn (↑g) (Function.const Y (-(‖f‖ / 3))) ((fun a => ↑e a) '' (↑f ⁻¹' Iic (-(‖f‖ / 3))))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) ((fun a => ↑e a) '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-(‖f‖ / 3)) (‖f‖ / 3)
hle₁ : -(‖f‖ / 3) ≤ ↑f x
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
calc
dist (g (e x)) (f x) ≤ |g (e x)| + |f x| := dist_le_norm_add_norm _ _
_ ≤ ‖f‖ / 3 + ‖f‖ / 3 := (add_le_add (abs_le.2 <| hgf _) (abs_le.2 ⟨hle₁, hle₂⟩))
_ = 2 / 3 * ‖f‖ := by linarith
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
g : Y →ᵇ ℝ
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₂ : ↑f x ≤ ‖f‖ / 3
hf3 : -(‖f‖ / 3) < ‖f‖ / 3
hc₁ : IsClosed ((fun a => ↑e a) '' (↑f ⁻¹' Iic (-(‖f‖ / 3))))
hc₂ : IsClosed ((fun a => ↑e a) '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint ((fun a => ↑e a) '' (↑f ⁻¹' Iic (-(‖f‖ / 3)))) ((fun a => ↑e a) '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hg₁ : EqOn (↑g) (Function.const Y (-(‖f‖ / 3))) ((fun a => ↑e a) '' (↑f ⁻¹' Iic (-(‖f‖ / 3))))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) ((fun a => ↑e a) '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-(‖f‖ / 3)) (‖f‖ / 3)
hle₁ : -(‖f‖ / 3) ≤ ↑f x
⊢ ‖f‖ / 3 + ‖f‖ / 3 = 2 / 3 * ‖f‖
[PROOFSTEP]
linarith
[GOAL]
case inr.intro.intro.intro.refine'_2.inr.inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : -‖f‖ / 3 ≤ ↑f x
hle₂ : ‖f‖ / 3 ≤ ↑f x
⊢ dist (↑(compContinuous g e) x) (↑f x) ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
calc
|g (e x) - f x| = f x - ‖f‖ / 3 := by
rw [hg₂ (mem_image_of_mem _ hle₂), abs_sub_comm, Function.const_apply, abs_of_nonneg (sub_nonneg.2 hle₂)]
_ ≤ 2 / 3 * ‖f‖ := by linarith
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : -‖f‖ / 3 ≤ ↑f x
hle₂ : ‖f‖ / 3 ≤ ↑f x
⊢ |↑g (↑e x) - ↑f x| = ↑f x - ‖f‖ / 3
[PROOFSTEP]
rw [hg₂ (mem_image_of_mem _ hle₂), abs_sub_comm, Function.const_apply, abs_of_nonneg (sub_nonneg.2 hle₂)]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
h3 : 0 < 3
h23 : 0 < 2 / 3
hf : 0 < ‖f‖
hf3 : -‖f‖ / 3 < ‖f‖ / 3
hc₁ : IsClosed (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hc₂ : IsClosed (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hd : Disjoint (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3))) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
g : Y →ᵇ ℝ
hg₁ : EqOn (↑g) (Function.const Y (-‖f‖ / 3)) (↑e '' (↑f ⁻¹' Iic (-‖f‖ / 3)))
hg₂ : EqOn (↑g) (Function.const Y (‖f‖ / 3)) (↑e '' (↑f ⁻¹' Ici (‖f‖ / 3)))
hgf : ∀ (x : Y), ↑g x ∈ Icc (-‖f‖ / 3) (‖f‖ / 3)
x : X
hfx : -‖f‖ ≤ ↑f x ∧ ↑f x ≤ ‖f‖
hle₁ : -‖f‖ / 3 ≤ ↑f x
hle₂ : ‖f‖ / 3 ≤ ↑f x
⊢ ↑f x - ‖f‖ / 3 ≤ 2 / 3 * ‖f‖
[PROOFSTEP]
linarith
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
choose F hF_norm hF_dist using fun f : X →ᵇ ℝ => tietze_extension_step f e he
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
set g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - g.compContinuous e))^[n] 0
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have g0 : g 0 = 0 := rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have g_succ : ∀ n, g (n + 1) = g n + F (f - (g n).compContinuous e) := fun n => Function.iterate_succ_apply' _ _ _
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have hgf : ∀ n, dist ((g n).compContinuous e) f ≤ (2 / 3) ^ n * ‖f‖ :=
by
intro n
induction' n with n ihn
· simp [g0]
· rw [g_succ n, add_compContinuous, ← dist_sub_right, add_sub_cancel', pow_succ, mul_assoc]
refine' (hF_dist _).trans (mul_le_mul_of_nonneg_left _ (by norm_num1))
rwa [← dist_eq_norm']
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
⊢ ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
[PROOFSTEP]
intro n
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
n : ℕ
⊢ dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
[PROOFSTEP]
induction' n with n ihn
[GOAL]
case zero
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
⊢ dist (compContinuous (g Nat.zero) e) f ≤ (2 / 3) ^ Nat.zero * ‖f‖
[PROOFSTEP]
simp [g0]
[GOAL]
case succ
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
n : ℕ
ihn : dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
⊢ dist (compContinuous (g (Nat.succ n)) e) f ≤ (2 / 3) ^ Nat.succ n * ‖f‖
[PROOFSTEP]
rw [g_succ n, add_compContinuous, ← dist_sub_right, add_sub_cancel', pow_succ, mul_assoc]
[GOAL]
case succ
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
n : ℕ
ihn : dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
⊢ dist (compContinuous (F (f - compContinuous (g n) e)) e) (f - compContinuous (g n) e) ≤ 2 / 3 * ((2 / 3) ^ n * ‖f‖)
[PROOFSTEP]
refine' (hF_dist _).trans (mul_le_mul_of_nonneg_left _ (by norm_num1))
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
n : ℕ
ihn : dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
⊢ 0 ≤ 2 / 3
[PROOFSTEP]
norm_num1
[GOAL]
case succ
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
n : ℕ
ihn : dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
⊢ ‖f - compContinuous (g n) e‖ ≤ (2 / 3) ^ n * ‖f‖
[PROOFSTEP]
rwa [← dist_eq_norm']
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have hg_dist : ∀ n, dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n :=
by
intro n
calc
dist (g n) (g (n + 1)) = ‖F (f - (g n).compContinuous e)‖ := by rw [g_succ, dist_eq_norm', add_sub_cancel']
_ ≤ ‖f - (g n).compContinuous e‖ / 3 := (hF_norm _)
_ = 1 / 3 * dist ((g n).compContinuous e) f := by rw [dist_eq_norm', one_div, div_eq_inv_mul]
_ ≤ 1 / 3 * ((2 / 3) ^ n * ‖f‖) := (mul_le_mul_of_nonneg_left (hgf n) (by norm_num1))
_ = 1 / 3 * ‖f‖ * (2 / 3) ^ n := by ac_rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
⊢ ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
[PROOFSTEP]
intro n
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
n : ℕ
⊢ dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
[PROOFSTEP]
calc
dist (g n) (g (n + 1)) = ‖F (f - (g n).compContinuous e)‖ := by rw [g_succ, dist_eq_norm', add_sub_cancel']
_ ≤ ‖f - (g n).compContinuous e‖ / 3 := (hF_norm _)
_ = 1 / 3 * dist ((g n).compContinuous e) f := by rw [dist_eq_norm', one_div, div_eq_inv_mul]
_ ≤ 1 / 3 * ((2 / 3) ^ n * ‖f‖) := (mul_le_mul_of_nonneg_left (hgf n) (by norm_num1))
_ = 1 / 3 * ‖f‖ * (2 / 3) ^ n := by ac_rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
n : ℕ
⊢ dist (g n) (g (n + 1)) = ‖F (f - compContinuous (g n) e)‖
[PROOFSTEP]
rw [g_succ, dist_eq_norm', add_sub_cancel']
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
n : ℕ
⊢ ‖f - compContinuous (g n) e‖ / 3 = 1 / 3 * dist (compContinuous (g n) e) f
[PROOFSTEP]
rw [dist_eq_norm', one_div, div_eq_inv_mul]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
n : ℕ
⊢ 0 ≤ 1 / 3
[PROOFSTEP]
norm_num1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
n : ℕ
⊢ 1 / 3 * ((2 / 3) ^ n * ‖f‖) = 1 / 3 * ‖f‖ * (2 / 3) ^ n
[PROOFSTEP]
ac_rfl
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have hg_cau : CauchySeq g := cauchySeq_of_le_geometric _ _ (by norm_num1) hg_dist
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
⊢ 2 / 3 < 1
[PROOFSTEP]
norm_num1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have : Tendsto (fun n => (g n).compContinuous e) atTop (𝓝 <| (limUnder atTop g).compContinuous e) :=
((continuous_compContinuous e).tendsto _).comp hg_cau.tendsto_limUnder
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
have hge : (limUnder atTop g).compContinuous e = f :=
by
refine' tendsto_nhds_unique this (tendsto_iff_dist_tendsto_zero.2 _)
refine' squeeze_zero (fun _ => dist_nonneg) hgf _
rw [← zero_mul ‖f‖]
refine' (tendsto_pow_atTop_nhds_0_of_lt_1 _ _).mul tendsto_const_nhds <;> norm_num1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ compContinuous (limUnder atTop g) e = f
[PROOFSTEP]
refine' tendsto_nhds_unique this (tendsto_iff_dist_tendsto_zero.2 _)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ Tendsto (fun b => dist (compContinuous (g b) e) f) atTop (𝓝 0)
[PROOFSTEP]
refine' squeeze_zero (fun _ => dist_nonneg) hgf _
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ Tendsto (fun t => (2 / 3) ^ t * ‖f‖) atTop (𝓝 0)
[PROOFSTEP]
rw [← zero_mul ‖f‖]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ Tendsto (fun t => (2 / 3) ^ t * ‖f‖) atTop (𝓝 (0 * ‖f‖))
[PROOFSTEP]
refine' (tendsto_pow_atTop_nhds_0_of_lt_1 _ _).mul tendsto_const_nhds
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ 0 ≤ 2 / 3
[PROOFSTEP]
norm_num1
[GOAL]
case refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
⊢ 2 / 3 < 1
[PROOFSTEP]
norm_num1
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ compContinuous g e = f
[PROOFSTEP]
refine' ⟨limUnder atTop g, le_antisymm _ _, hge⟩
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ ‖limUnder atTop g‖ ≤ ‖f‖
[PROOFSTEP]
rw [← dist_zero_left, ← g0]
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ dist (g 0) (limUnder atTop g) ≤ ‖f‖
[PROOFSTEP]
refine' (dist_le_of_le_geometric_of_tendsto₀ _ _ (by norm_num1) hg_dist hg_cau.tendsto_limUnder).trans_eq _
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ 2 / 3 < 1
[PROOFSTEP]
norm_num1
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ 1 / 3 * ‖f‖ / (1 - 2 / 3) = ‖f‖
[PROOFSTEP]
field_simp [show (3 - 2 : ℝ) = 1 by norm_num1]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ 3 - 2 = 1
[PROOFSTEP]
norm_num1
[GOAL]
case refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ ‖f‖ ≤ ‖limUnder atTop g‖
[PROOFSTEP]
rw [← hge]
[GOAL]
case refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : C(X, Y)
he : ClosedEmbedding ↑e
F : (X →ᵇ ℝ) → Y →ᵇ ℝ
hF_norm : ∀ (f : X →ᵇ ℝ), ‖F f‖ ≤ ‖f‖ / 3
hF_dist : ∀ (f : X →ᵇ ℝ), dist (compContinuous (F f) e) f ≤ 2 / 3 * ‖f‖
g : ℕ → Y →ᵇ ℝ := fun n => (fun g => g + F (f - compContinuous g e))^[n] 0
g0 : g 0 = 0
g_succ : ∀ (n : ℕ), g (n + 1) = g n + F (f - compContinuous (g n) e)
hgf : ∀ (n : ℕ), dist (compContinuous (g n) e) f ≤ (2 / 3) ^ n * ‖f‖
hg_dist : ∀ (n : ℕ), dist (g n) (g (n + 1)) ≤ 1 / 3 * ‖f‖ * (2 / 3) ^ n
hg_cau : CauchySeq g
this : Tendsto (fun n => compContinuous (g n) e) atTop (𝓝 (compContinuous (limUnder atTop g) e))
hge : compContinuous (limUnder atTop g) e = f
⊢ ‖compContinuous (limUnder atTop g) e‖ ≤ ‖limUnder atTop g‖
[PROOFSTEP]
exact norm_compContinuous_le _ _
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
⊢ ∃ g, ‖g‖ = ‖f‖ ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases exists_extension_norm_eq_of_closedEmbedding' f ⟨e, he.continuous⟩ he with ⟨g, hg, rfl⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
e : X → Y
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hg : ‖g‖ = ‖compContinuous g (ContinuousMap.mk e)‖
⊢ ∃ g_1, ‖g_1‖ = ‖compContinuous g (ContinuousMap.mk e)‖ ∧ ↑g_1 ∘ e = ↑(compContinuous g (ContinuousMap.mk e))
[PROOFSTEP]
exact ⟨g, hg, rfl⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ Icc a b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases exists_extension_norm_eq_of_closedEmbedding (f - const X ((a + b) / 2)) he with ⟨g, hgf, hge⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ Icc a b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
refine' ⟨const Y ((a + b) / 2) + g, fun y => _, _⟩
[GOAL]
case intro.intro.refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
y : Y
⊢ ↑(const Y ((a + b) / 2) + g) y ∈ Icc a b
[PROOFSTEP]
suffices ‖f - const X ((a + b) / 2)‖ ≤ (b - a) / 2 by
simpa [Real.Icc_eq_closedBall, add_mem_closedBall_iff_norm] using (norm_coe_le_norm g y).trans (hgf.trans_le this)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
y : Y
this : ‖f - const X ((a + b) / 2)‖ ≤ (b - a) / 2
⊢ ↑(const Y ((a + b) / 2) + g) y ∈ Icc a b
[PROOFSTEP]
simpa [Real.Icc_eq_closedBall, add_mem_closedBall_iff_norm] using (norm_coe_le_norm g y).trans (hgf.trans_le this)
[GOAL]
case intro.intro.refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
y : Y
⊢ ‖f - const X ((a + b) / 2)‖ ≤ (b - a) / 2
[PROOFSTEP]
refine' (norm_le <| div_nonneg (sub_nonneg.2 hle) zero_le_two).2 fun x => _
[GOAL]
case intro.intro.refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
y : Y
x : X
⊢ ‖↑(f - const X ((a + b) / 2)) x‖ ≤ (b - a) / 2
[PROOFSTEP]
simpa only [Real.Icc_eq_closedBall] using hf x
[GOAL]
case intro.intro.refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
⊢ ↑(const Y ((a + b) / 2) + g) ∘ e = ↑f
[PROOFSTEP]
ext x
[GOAL]
case intro.intro.refine'_2.h
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
x : X
⊢ (↑(const Y ((a + b) / 2) + g) ∘ e) x = ↑f x
[PROOFSTEP]
have : g (e x) = f x - (a + b) / 2 := congr_fun hge x
[GOAL]
case intro.intro.refine'_2.h
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
a b : ℝ
e : X → Y
hf : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
he : ClosedEmbedding e
g : Y →ᵇ ℝ
hgf : ‖g‖ = ‖f - const X ((a + b) / 2)‖
hge : ↑g ∘ e = ↑(f - const X ((a + b) / 2))
x : X
this : ↑g (e x) = ↑f x - (a + b) / 2
⊢ (↑(const Y ((a + b) / 2) + g) ∘ e) x = ↑f x
[PROOFSTEP]
simp [this]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
inhabit X
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
obtain ⟨a, ha⟩ : ∃ a, IsGLB (range f) a
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
⊢ ∃ a, IsGLB (range ↑f) a
case intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
exact ⟨_, isGLB_ciInf (Real.bounded_iff_bddBelow_bddAbove.1 f.bounded_range).1⟩
[GOAL]
case intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
obtain ⟨b, hb⟩ : ∃ b, IsLUB (range f) b
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
⊢ ∃ b, IsLUB (range ↑f) b
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
exact
⟨_, isLUB_ciSup (Real.bounded_iff_bddBelow_bddAbove.1 f.bounded_range).2⟩
-- Then `f x ∈ [a, b]` for all `x`
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hmem : ∀ x, f x ∈ Icc a b := fun x =>
⟨ha.1 ⟨x, rfl⟩, hb.1 ⟨x, rfl⟩⟩
-- Rule out the trivial case `a = b`
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hle : a ≤ b := (hmem default).1.trans (hmem default).2
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases hle.eq_or_lt with (rfl | hlt)
[GOAL]
case intro.intro.inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
hb : IsLUB (range ↑f) a
hmem : ∀ (x : X), ↑f x ∈ Icc a a
hle : a ≤ a
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have : ∀ x, f x = a := by simpa using hmem
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
hb : IsLUB (range ↑f) a
hmem : ∀ (x : X), ↑f x ∈ Icc a a
hle : a ≤ a
⊢ ∀ (x : X), ↑f x = a
[PROOFSTEP]
simpa using hmem
[GOAL]
case intro.intro.inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
hb : IsLUB (range ↑f) a
hmem : ∀ (x : X), ↑f x ∈ Icc a a
hle : a ≤ a
this : ∀ (x : X), ↑f x = a
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
use const Y a
[GOAL]
case h
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
hb : IsLUB (range ↑f) a
hmem : ∀ (x : X), ↑f x ∈ Icc a a
hle : a ≤ a
this : ∀ (x : X), ↑f x = a
⊢ (∀ (y : Y), ∃ x₁ x₂, ↑(const Y a) y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑(const Y a) ∘ e = ↑f
[PROOFSTEP]
simp [this, Function.funext_iff]
-- Put `c = (a + b) / 2`. Then `a < c < b` and `c - a = b - c`.
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
set c := (a + b) / 2
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hac : a < c := left_lt_add_div_two.2 hlt
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hcb : c < b := add_div_two_lt_right.2 hlt
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hsub : c - a = b - c := by
field_simp
ring
/- Due to `exists_extension_forall_mem_Icc_of_closedEmbedding`, there exists an extension `g`
such that `g y ∈ [a, b]` for all `y`. However, if `a` and/or `b` do not belong to the range of
`f`, then we need to ensure that these points do not belong to the range of `g`. This is done
in two almost identical steps. First we deal with the case `∀ x, f x ≠ a`. -/
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
⊢ c - a = b - c
[PROOFSTEP]
field_simp
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
⊢ a + b - 2 * a = b * 2 - (a + b)
[PROOFSTEP]
ring
/- Due to `exists_extension_forall_mem_Icc_of_closedEmbedding`, there exists an extension `g`
such that `g y ∈ [a, b]` for all `y`. However, if `a` and/or `b` do not belong to the range of
`f`, then we need to ensure that these points do not belong to the range of `g`. This is done
in two almost identical steps. First we deal with the case `∀ x, f x ≠ a`. -/
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
obtain ⟨g, hg_mem, hgf⟩ : ∃ g : Y →ᵇ ℝ, (∀ y, ∃ x, g y ∈ Icc (f x) b) ∧ g ∘ e = f :=
by
rcases exists_extension_forall_mem_Icc_of_closedEmbedding f hmem hle he with
⟨g, hg_mem, hgf⟩
-- If `a ∈ range f`, then we are done.
rcases em (∃ x, f x = a) with (⟨x, rfl⟩ | ha')
·
exact
⟨g, fun y => ⟨x, hg_mem _⟩, hgf⟩
/- Otherwise, `g ⁻¹' {a}` is disjoint with `range e ∪ g ⁻¹' (Ici c)`, hence there exists a
function `dg : Y → ℝ` such that `dg ∘ e = 0`, `dg y = 0` whenever `c ≤ g y`, `dg y = c - a`
whenever `g y = a`, and `0 ≤ dg y ≤ c - a` for all `y`. -/
have hd : Disjoint (range e ∪ g ⁻¹' Ici c) (g ⁻¹' { a }) :=
by
refine' disjoint_union_left.2 ⟨_, Disjoint.preimage _ _⟩
· rw [Set.disjoint_left]
rintro _ ⟨x, rfl⟩ (rfl : g (e x) = a)
exact ha' ⟨x, (congr_fun hgf x).symm⟩
· exact Set.disjoint_singleton_right.2 hac.not_le
rcases exists_bounded_mem_Icc_of_closed_of_le (he.closed_range.union <| isClosed_Ici.preimage g.continuous)
(isClosed_singleton.preimage g.continuous) hd (sub_nonneg.2 hac.le) with
⟨dg, dg0, dga, dgmem⟩
replace hgf : ∀ x, (g + dg) (e x) = f x
· intro x
simp [dg0 (Or.inl <| mem_range_self _), ← hgf]
refine' ⟨g + dg, fun y => _, funext hgf⟩
· have hay : a < (g + dg) y := by
rcases(hg_mem y).1.eq_or_lt with (rfl | hlt)
· refine' (lt_add_iff_pos_right _).2 _
calc
0 < c - g y := sub_pos.2 hac
_ = dg y := (dga rfl).symm
· exact hlt.trans_le ((le_add_iff_nonneg_right _).2 <| (dgmem y).1)
rcases ha.exists_between hay with ⟨_, ⟨x, rfl⟩, _, hxy⟩
refine' ⟨x, hxy.le, _⟩
cases' le_total c (g y) with hc hc
· simp [dg0 (Or.inr hc), (hg_mem y).2]
·
calc
g y + dg y ≤ c + (c - a) := add_le_add hc (dgmem _).2
_ = b := by
rw [hsub, add_sub_cancel'_right]
/- Now we deal with the case `∀ x, f x ≠ b`. The proof is the same as in the first case, with
minor modifications that make it hard to deduplicate code. -/
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases exists_extension_forall_mem_Icc_of_closedEmbedding f hmem hle he with
⟨g, hg_mem, hgf⟩
-- If `a ∈ range f`, then we are done.
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases em (∃ x, f x = a) with (⟨x, rfl⟩ | ha')
[GOAL]
case intro.intro.inl.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
x : X
ha : IsGLB (range ↑f) (↑f x)
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc (↑f x) b
hle : ↑f x ≤ b
hlt : ↑f x < b
c : ℝ := (↑f x + b) / 2
hac : ↑f x < c
hcb : c < b
hsub : c - ↑f x = b - c
hg_mem : ∀ (y : Y), ↑g y ∈ Icc (↑f x) b
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
exact
⟨g, fun y => ⟨x, hg_mem _⟩, hgf⟩
/- Otherwise, `g ⁻¹' {a}` is disjoint with `range e ∪ g ⁻¹' (Ici c)`, hence there exists a
function `dg : Y → ℝ` such that `dg ∘ e = 0`, `dg y = 0` whenever `c ≤ g y`, `dg y = c - a`
whenever `g y = a`, and `0 ≤ dg y ≤ c - a` for all `y`. -/
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hd : Disjoint (range e ∪ g ⁻¹' Ici c) (g ⁻¹' { a }) :=
by
refine' disjoint_union_left.2 ⟨_, Disjoint.preimage _ _⟩
· rw [Set.disjoint_left]
rintro _ ⟨x, rfl⟩ (rfl : g (e x) = a)
exact ha' ⟨x, (congr_fun hgf x).symm⟩
· exact Set.disjoint_singleton_right.2 hac.not_le
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
⊢ Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
[PROOFSTEP]
refine' disjoint_union_left.2 ⟨_, Disjoint.preimage _ _⟩
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
⊢ Disjoint (range e) (↑g ⁻¹' {a})
[PROOFSTEP]
rw [Set.disjoint_left]
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
⊢ ∀ ⦃a_1 : Y⦄, a_1 ∈ range e → ¬a_1 ∈ ↑g ⁻¹' {a}
[PROOFSTEP]
rintro _ ⟨x, rfl⟩ (rfl : g (e x) = a)
[GOAL]
case refine'_1.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
x : X
ha : IsGLB (range ↑f) (↑g (e x))
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc (↑g (e x)) b
hle : ↑g (e x) ≤ b
hlt : ↑g (e x) < b
c : ℝ := (↑g (e x) + b) / 2
hac : ↑g (e x) < c
hcb : c < b
hsub : c - ↑g (e x) = b - c
hg_mem : ∀ (y : Y), ↑g y ∈ Icc (↑g (e x)) b
ha' : ¬∃ x_1, ↑f x_1 = ↑g (e x)
⊢ False
[PROOFSTEP]
exact ha' ⟨x, (congr_fun hgf x).symm⟩
[GOAL]
case refine'_2
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
⊢ Disjoint (Ici c) {a}
[PROOFSTEP]
exact Set.disjoint_singleton_right.2 hac.not_le
[GOAL]
case intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases exists_bounded_mem_Icc_of_closed_of_le (he.closed_range.union <| isClosed_Ici.preimage g.continuous)
(isClosed_singleton.preimage g.continuous) hd (sub_nonneg.2 hac.le) with
⟨dg, dg0, dga, dgmem⟩
[GOAL]
case intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
replace hgf : ∀ x, (g + dg) (e x) = f x
[GOAL]
case hgf
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
⊢ ∀ (x : X), ↑(g + dg) (e x) = ↑f x
[PROOFSTEP]
intro x
[GOAL]
case hgf
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
hgf : ↑g ∘ e = ↑f
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
x : X
⊢ ↑(g + dg) (e x) = ↑f x
[PROOFSTEP]
simp [dg0 (Or.inl <| mem_range_self _), ← hgf]
[GOAL]
case intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
⊢ ∃ g, (∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
refine' ⟨g + dg, fun y => _, funext hgf⟩
[GOAL]
case intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
⊢ ∃ x, ↑(g + dg) y ∈ Icc (↑f x) b
[PROOFSTEP]
have hay : a < (g + dg) y := by
rcases(hg_mem y).1.eq_or_lt with (rfl | hlt)
· refine' (lt_add_iff_pos_right _).2 _
calc
0 < c - g y := sub_pos.2 hac
_ = dg y := (dga rfl).symm
· exact hlt.trans_le ((le_add_iff_nonneg_right _).2 <| (dgmem y).1)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
⊢ a < ↑(g + dg) y
[PROOFSTEP]
rcases(hg_mem y).1.eq_or_lt with (rfl | hlt)
[GOAL]
case inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
ha : IsGLB (range ↑f) (↑g y)
hmem : ∀ (x : X), ↑f x ∈ Icc (↑g y) b
hle : ↑g y ≤ b
hlt : ↑g y < b
c : ℝ := (↑g y + b) / 2
hac : ↑g y < c
hcb : c < b
hsub : c - ↑g y = b - c
hg_mem : ∀ (y_1 : Y), ↑g y_1 ∈ Icc (↑g y) b
ha' : ¬∃ x, ↑f x = ↑g y
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {↑g y})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - ↑g y)) (↑g ⁻¹' {↑g y})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - ↑g y)
⊢ ↑g y < ↑(g + dg) y
[PROOFSTEP]
refine' (lt_add_iff_pos_right _).2 _
[GOAL]
case inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
ha : IsGLB (range ↑f) (↑g y)
hmem : ∀ (x : X), ↑f x ∈ Icc (↑g y) b
hle : ↑g y ≤ b
hlt : ↑g y < b
c : ℝ := (↑g y + b) / 2
hac : ↑g y < c
hcb : c < b
hsub : c - ↑g y = b - c
hg_mem : ∀ (y_1 : Y), ↑g y_1 ∈ Icc (↑g y) b
ha' : ¬∃ x, ↑f x = ↑g y
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {↑g y})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - ↑g y)) (↑g ⁻¹' {↑g y})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - ↑g y)
⊢ 0 < ↑dg.toContinuousMap y
[PROOFSTEP]
calc
0 < c - g y := sub_pos.2 hac
_ = dg y := (dga rfl).symm
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt✝ : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hlt : a < ↑g y
⊢ a < ↑(g + dg) y
[PROOFSTEP]
exact hlt.trans_le ((le_add_iff_nonneg_right _).2 <| (dgmem y).1)
[GOAL]
case intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hay : a < ↑(g + dg) y
⊢ ∃ x, ↑(g + dg) y ∈ Icc (↑f x) b
[PROOFSTEP]
rcases ha.exists_between hay with ⟨_, ⟨x, rfl⟩, _, hxy⟩
[GOAL]
case intro.intro.inr.intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hay : a < ↑(g + dg) y
x : X
left✝ : a ≤ ↑f x
hxy : ↑f x < ↑(g + dg) y
⊢ ∃ x, ↑(g + dg) y ∈ Icc (↑f x) b
[PROOFSTEP]
refine' ⟨x, hxy.le, _⟩
[GOAL]
case intro.intro.inr.intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hay : a < ↑(g + dg) y
x : X
left✝ : a ≤ ↑f x
hxy : ↑f x < ↑(g + dg) y
⊢ ↑(g + dg) y ≤ b
[PROOFSTEP]
cases' le_total c (g y) with hc hc
[GOAL]
case intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hay : a < ↑(g + dg) y
x : X
left✝ : a ≤ ↑f x
hxy : ↑f x < ↑(g + dg) y
hc : c ≤ ↑g y
⊢ ↑(g + dg) y ≤ b
[PROOFSTEP]
simp [dg0 (Or.inr hc), (hg_mem y).2]
[GOAL]
case intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hay : a < ↑(g + dg) y
x : X
left✝ : a ≤ ↑f x
hxy : ↑f x < ↑(g + dg) y
hc : ↑g y ≤ c
⊢ ↑(g + dg) y ≤ b
[PROOFSTEP]
calc
g y + dg y ≤ c + (c - a) := add_le_add hc (dgmem _).2
_ = b := by
rw [hsub, add_sub_cancel'_right]
/- Now we deal with the case `∀ x, f x ≠ b`. The proof is the same as in the first case, with
minor modifications that make it hard to deduplicate code. -/
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ↑g y ∈ Icc a b
ha' : ¬∃ x, ↑f x = a
hd : Disjoint (range e ∪ ↑g ⁻¹' Ici c) (↑g ⁻¹' {a})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Ici c)
dga : EqOn (↑dg) (Function.const Y (c - a)) (↑g ⁻¹' {a})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (c - a)
hgf : ∀ (x : X), ↑(g + dg) (e x) = ↑f x
y : Y
hay : a < ↑(g + dg) y
x : X
left✝ : a ≤ ↑f x
hxy : ↑f x < ↑(g + dg) y
hc : ↑g y ≤ c
⊢ c + (c - a) = b
[PROOFSTEP]
rw [hsub, add_sub_cancel'_right]
/- Now we deal with the case `∀ x, f x ≠ b`. The proof is the same as in the first case, with
minor modifications that make it hard to deduplicate code. -/
[GOAL]
case intro.intro.inr.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hg_mem : ∀ (y : Y), ∃ x, ↑g y ∈ Icc (↑f x) b
hgf : ↑g ∘ e = ↑f
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
choose xl hxl hgb using hg_mem
[GOAL]
case intro.intro.inr.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases em (∃ x, f x = b) with (⟨x, rfl⟩ | hb')
[GOAL]
case intro.intro.inr.intro.intro.inl.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
x : X
hb : IsLUB (range ↑f) (↑f x)
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc a (↑f x)
hle : a ≤ ↑f x
hlt : a < ↑f x
c : ℝ := (a + ↑f x) / 2
hac : a < c
hcb : c < ↑f x
hsub : c - a = ↑f x - c
hgb : ∀ (y : Y), ↑g y ≤ ↑f x
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
exact ⟨g, fun y => ⟨xl y, x, hxl y, hgb y⟩, hgf⟩
[GOAL]
case intro.intro.inr.intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hd : Disjoint (range e ∪ g ⁻¹' Iic c) (g ⁻¹' { b }) :=
by
refine' disjoint_union_left.2 ⟨_, Disjoint.preimage _ _⟩
· rw [Set.disjoint_left]
rintro _ ⟨x, rfl⟩ (rfl : g (e x) = b)
exact hb' ⟨x, (congr_fun hgf x).symm⟩
· exact Set.disjoint_singleton_right.2 hcb.not_le
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
⊢ Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
[PROOFSTEP]
refine' disjoint_union_left.2 ⟨_, Disjoint.preimage _ _⟩
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
⊢ Disjoint (range e) (↑g ⁻¹' {b})
[PROOFSTEP]
rw [Set.disjoint_left]
[GOAL]
case refine'_1
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
⊢ ∀ ⦃a : Y⦄, a ∈ range e → ¬a ∈ ↑g ⁻¹' {b}
[PROOFSTEP]
rintro _ ⟨x, rfl⟩ (rfl : g (e x) = b)
[GOAL]
case refine'_1.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
x : X
hb : IsLUB (range ↑f) (↑g (e x))
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc a (↑g (e x))
hle : a ≤ ↑g (e x)
hlt : a < ↑g (e x)
c : ℝ := (a + ↑g (e x)) / 2
hac : a < c
hcb : c < ↑g (e x)
hsub : c - a = ↑g (e x) - c
hgb : ∀ (y : Y), ↑g y ≤ ↑g (e x)
hb' : ¬∃ x_1, ↑f x_1 = ↑g (e x)
⊢ False
[PROOFSTEP]
exact hb' ⟨x, (congr_fun hgf x).symm⟩
[GOAL]
case refine'_2
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
⊢ Disjoint (Iic c) {b}
[PROOFSTEP]
exact Set.disjoint_singleton_right.2 hcb.not_le
[GOAL]
case intro.intro.inr.intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases exists_bounded_mem_Icc_of_closed_of_le (he.closed_range.union <| isClosed_Iic.preimage g.continuous)
(isClosed_singleton.preimage g.continuous) hd (sub_nonneg.2 hcb.le) with
⟨dg, dg0, dgb, dgmem⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
replace hgf : ∀ x, (g - dg) (e x) = f x
[GOAL]
case hgf
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
⊢ ∀ (x : X), ↑(g - dg) (e x) = ↑f x
[PROOFSTEP]
intro x
[GOAL]
case hgf
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
hgf : ↑g ∘ e = ↑f
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
x : X
⊢ ↑(g - dg) (e x) = ↑f x
[PROOFSTEP]
simp [dg0 (Or.inl <| mem_range_self _), ← hgf]
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
⊢ ∃ g, (∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
refine' ⟨g - dg, fun y => _, funext hgf⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
have hyb : (g - dg) y < b := by
rcases(hgb y).eq_or_lt with (rfl | hlt)
· refine' (sub_lt_self_iff _).2 _
calc
0 < g y - c := sub_pos.2 hcb
_ = dg y := (dgb rfl).symm
· exact ((sub_le_self_iff _).2 (dgmem _).1).trans_lt hlt
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
⊢ ↑(g - dg) y < b
[PROOFSTEP]
rcases(hgb y).eq_or_lt with (rfl | hlt)
[GOAL]
case inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hb : IsLUB (range ↑f) (↑g y)
hmem : ∀ (x : X), ↑f x ∈ Icc a (↑g y)
hle : a ≤ ↑g y
hlt : a < ↑g y
c : ℝ := (a + ↑g y) / 2
hac : a < c
hcb : c < ↑g y
hsub : c - a = ↑g y - c
hgb : ∀ (y_1 : Y), ↑g y_1 ≤ ↑g y
hb' : ¬∃ x, ↑f x = ↑g y
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {↑g y})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (↑g y - c)) (↑g ⁻¹' {↑g y})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (↑g y - c)
⊢ ↑(g - dg) y < ↑g y
[PROOFSTEP]
refine' (sub_lt_self_iff _).2 _
[GOAL]
case inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hb : IsLUB (range ↑f) (↑g y)
hmem : ∀ (x : X), ↑f x ∈ Icc a (↑g y)
hle : a ≤ ↑g y
hlt : a < ↑g y
c : ℝ := (a + ↑g y) / 2
hac : a < c
hcb : c < ↑g y
hsub : c - a = ↑g y - c
hgb : ∀ (y_1 : Y), ↑g y_1 ≤ ↑g y
hb' : ¬∃ x, ↑f x = ↑g y
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {↑g y})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (↑g y - c)) (↑g ⁻¹' {↑g y})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (↑g y - c)
⊢ 0 < ↑dg y
[PROOFSTEP]
calc
0 < g y - c := sub_pos.2 hcb
_ = dg y := (dgb rfl).symm
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt✝ : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hlt : ↑g y < b
⊢ ↑(g - dg) y < b
[PROOFSTEP]
exact ((sub_le_self_iff _).2 (dgmem _).1).trans_lt hlt
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
rcases hb.exists_between hyb with ⟨_, ⟨xu, rfl⟩, hyxu, _⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
cases' lt_or_le c (g y) with hc hc
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : c < ↑g y
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
rcases em (a ∈ range f) with (⟨x, rfl⟩ | _)
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl.inl.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
x : X
ha : IsGLB (range ↑f) (↑f x)
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc (↑f x) b
hle : ↑f x ≤ b
hlt : ↑f x < b
c : ℝ := (↑f x + b) / 2
hac : ↑f x < c
hcb : c < b
hsub : c - ↑f x = b - c
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hc : c < ↑g y
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
refine' ⟨x, xu, _, hyxu.le⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl.inl.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
x : X
ha : IsGLB (range ↑f) (↑f x)
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc (↑f x) b
hle : ↑f x ≤ b
hlt : ↑f x < b
c : ℝ := (↑f x + b) / 2
hac : ↑f x < c
hcb : c < b
hsub : c - ↑f x = b - c
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hc : c < ↑g y
⊢ ↑f x ≤ ↑(g - dg) y
[PROOFSTEP]
calc
f x = c - (b - c) := by rw [← hsub, sub_sub_cancel]
_ ≤ g y - dg y := sub_le_sub hc.le (dgmem _).2
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
b : ℝ
hb : IsLUB (range ↑f) b
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
dg : Y →ᵇ ℝ
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
x : X
ha : IsGLB (range ↑f) (↑f x)
hmem : ∀ (x_1 : X), ↑f x_1 ∈ Icc (↑f x) b
hle : ↑f x ≤ b
hlt : ↑f x < b
c : ℝ := (↑f x + b) / 2
hac : ↑f x < c
hcb : c < b
hsub : c - ↑f x = b - c
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hc : c < ↑g y
⊢ ↑f x = c - (b - c)
[PROOFSTEP]
rw [← hsub, sub_sub_cancel]
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : c < ↑g y
h✝ : ¬a ∈ range ↑f
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
have hay : a < (g - dg) y := by
calc
a = c - (b - c) := by rw [← hsub, sub_sub_cancel]
_ < g y - (b - c) := (sub_lt_sub_right hc _)
_ ≤ g y - dg y := sub_le_sub_left (dgmem _).2 _
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : c < ↑g y
h✝ : ¬a ∈ range ↑f
⊢ a < ↑(g - dg) y
[PROOFSTEP]
calc
a = c - (b - c) := by rw [← hsub, sub_sub_cancel]
_ < g y - (b - c) := (sub_lt_sub_right hc _)
_ ≤ g y - dg y := sub_le_sub_left (dgmem _).2 _
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : c < ↑g y
h✝ : ¬a ∈ range ↑f
⊢ a = c - (b - c)
[PROOFSTEP]
rw [← hsub, sub_sub_cancel]
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : c < ↑g y
h✝ : ¬a ∈ range ↑f
hay : a < ↑(g - dg) y
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
rcases ha.exists_between hay with ⟨_, ⟨x, rfl⟩, _, hxy⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inl.inr.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : c < ↑g y
h✝ : ¬a ∈ range ↑f
hay : a < ↑(g - dg) y
x : X
left✝ : a ≤ ↑f x
hxy : ↑f x < ↑(g - dg) y
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
exact ⟨x, xu, hxy.le, hyxu.le⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : ↑g y ≤ c
⊢ ∃ x₁ x₂, ↑(g - dg) y ∈ Icc (↑f x₁) (↑f x₂)
[PROOFSTEP]
refine' ⟨xl y, xu, _, hyxu.le⟩
[GOAL]
case intro.intro.inr.intro.intro.inr.intro.intro.intro.intro.intro.intro.intro.inr
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
inst✝ : Nonempty X
f : X →ᵇ ℝ
e : X → Y
he : ClosedEmbedding e
inhabited_h : Inhabited X
a : ℝ
ha : IsGLB (range ↑f) a
b : ℝ
hb : IsLUB (range ↑f) b
hmem : ∀ (x : X), ↑f x ∈ Icc a b
hle : a ≤ b
hlt : a < b
c : ℝ := (a + b) / 2
hac : a < c
hcb : c < b
hsub : c - a = b - c
g : Y →ᵇ ℝ
xl : Y → X
hxl : ∀ (y : Y), ↑f (xl y) ≤ ↑g y
hgb : ∀ (y : Y), ↑g y ≤ b
hb' : ¬∃ x, ↑f x = b
hd : Disjoint (range e ∪ ↑g ⁻¹' Iic c) (↑g ⁻¹' {b})
dg : Y →ᵇ ℝ
dg0 : EqOn (↑dg) (Function.const Y 0) (range e ∪ ↑g ⁻¹' Iic c)
dgb : EqOn (↑dg) (Function.const Y (b - c)) (↑g ⁻¹' {b})
dgmem : ∀ (x : Y), ↑dg x ∈ Icc 0 (b - c)
hgf : ∀ (x : X), ↑(g - dg) (e x) = ↑f x
y : Y
hyb : ↑(g - dg) y < b
xu : X
hyxu : ↑(g - dg) y < ↑f xu
right✝ : ↑f xu ≤ b
hc : ↑g y ≤ c
⊢ ↑f (xl y) ≤ ↑(g - dg) y
[PROOFSTEP]
simp [dg0 (Or.inr hc), hxl]
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
cases isEmpty_or_nonempty X
[GOAL]
case inl
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h✝ : IsEmpty X
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases hne with ⟨c, hc⟩
[GOAL]
case inl.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
he : ClosedEmbedding e
h✝ : IsEmpty X
c : ℝ
hc : c ∈ t
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
refine' ⟨const Y c, fun _ => hc, funext fun x => isEmptyElim x⟩
[GOAL]
case inr
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h✝ : Nonempty X
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases exists_extension_forall_exists_le_ge_of_closedEmbedding f he with ⟨g, hg, hgf⟩
[GOAL]
case inr.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h✝ : Nonempty X
g : Y →ᵇ ℝ
hg : ∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)
hgf : ↑g ∘ e = ↑f
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
refine' ⟨g, fun y => _, hgf⟩
[GOAL]
case inr.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h✝ : Nonempty X
g : Y →ᵇ ℝ
hg : ∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)
hgf : ↑g ∘ e = ↑f
y : Y
⊢ ↑g y ∈ t
[PROOFSTEP]
rcases hg y with ⟨xl, xu, h⟩
[GOAL]
case inr.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : X →ᵇ ℝ
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h✝ : Nonempty X
g : Y →ᵇ ℝ
hg : ∀ (y : Y), ∃ x₁ x₂, ↑g y ∈ Icc (↑f x₁) (↑f x₂)
hgf : ↑g ∘ e = ↑f
y : Y
xl xu : X
h : ↑g y ∈ Icc (↑f xl) (↑f xu)
⊢ ↑g y ∈ t
[PROOFSTEP]
exact hs.out (hf _) (hf _) h
[GOAL]
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
s : Set Y
f : ↑s →ᵇ ℝ
hs : IsClosed s
t : Set ℝ
inst✝ : OrdConnected t
hf : ∀ (x : ↑s), ↑f x ∈ t
hne : Set.Nonempty t
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ restrict g s = f
[PROOFSTEP]
rcases exists_extension_forall_mem_of_closedEmbedding f hf hne (closedEmbedding_subtype_val hs) with ⟨g, hg, hgf⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : NormalSpace Y
s : Set Y
f : ↑s →ᵇ ℝ
hs : IsClosed s
t : Set ℝ
inst✝ : OrdConnected t
hf : ∀ (x : ↑s), ↑f x ∈ t
hne : Set.Nonempty t
g : Y →ᵇ ℝ
hg : ∀ (y : Y), ↑g y ∈ t
hgf : ↑g ∘ Subtype.val = ↑f
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ restrict g s = f
[PROOFSTEP]
exact ⟨g, hg, FunLike.coe_injective hgf⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have h : ℝ ≃o Ioo (-1 : ℝ) 1 := orderIsoIooNegOneOne ℝ
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
let F : X →ᵇ ℝ :=
{ toFun := (↑) ∘ h ∘ f
continuous_toFun := continuous_subtype_val.comp (h.continuous.comp f.continuous)
map_bounded' := bounded_range_iff.1 ((bounded_Ioo (-1 : ℝ) 1).mono <| forall_range_iff.2 fun x => (h (f x)).2) }
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
let t' : Set ℝ := (↑) ∘ h '' t
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have ht_sub : t' ⊆ Ioo (-1 : ℝ) 1 := image_subset_iff.2 fun x _ => (h x).2
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have : OrdConnected t' := by
constructor
rintro _ ⟨x, hx, rfl⟩ _ ⟨y, hy, rfl⟩ z hz
lift z to Ioo (-1 : ℝ) 1 using Icc_subset_Ioo (h x).2.1 (h y).2.2 hz
change z ∈ Icc (h x) (h y) at hz
rw [← h.image_Icc] at hz
rcases hz with ⟨z, hz, rfl⟩
exact ⟨z, hs.out hx hy hz, rfl⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
⊢ OrdConnected t'
[PROOFSTEP]
constructor
[GOAL]
case out'
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
⊢ ∀ ⦃x : ℝ⦄, x ∈ t' → ∀ ⦃y : ℝ⦄, y ∈ t' → Icc x y ⊆ t'
[PROOFSTEP]
rintro _ ⟨x, hx, rfl⟩ _ ⟨y, hy, rfl⟩ z hz
[GOAL]
case out'.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
x : ℝ
hx : x ∈ t
y : ℝ
hy : y ∈ t
z : ℝ
hz : z ∈ Icc ((Subtype.val ∘ ↑h) x) ((Subtype.val ∘ ↑h) y)
⊢ z ∈ t'
[PROOFSTEP]
lift z to Ioo (-1 : ℝ) 1 using Icc_subset_Ioo (h x).2.1 (h y).2.2 hz
[GOAL]
case out'.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
x : ℝ
hx : x ∈ t
y : ℝ
hy : y ∈ t
z : { x // x ∈ Ioo (-1) 1 }
hz : ↑z ∈ Icc ((Subtype.val ∘ ↑h) x) ((Subtype.val ∘ ↑h) y)
⊢ ↑z ∈ t'
[PROOFSTEP]
change z ∈ Icc (h x) (h y) at hz
[GOAL]
case out'.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
x : ℝ
hx : x ∈ t
y : ℝ
hy : y ∈ t
z : { x // x ∈ Ioo (-1) 1 }
hz : z ∈ Icc (↑h x) (↑h y)
⊢ ↑z ∈ t'
[PROOFSTEP]
rw [← h.image_Icc] at hz
[GOAL]
case out'.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
x : ℝ
hx : x ∈ t
y : ℝ
hy : y ∈ t
z : { x // x ∈ Ioo (-1) 1 }
hz : z ∈ ↑h '' Icc x y
⊢ ↑z ∈ t'
[PROOFSTEP]
rcases hz with ⟨z, hz, rfl⟩
[GOAL]
case out'.intro.intro.intro.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
x : ℝ
hx : x ∈ t
y : ℝ
hy : y ∈ t
z : ℝ
hz : z ∈ Icc x y
⊢ ↑(↑h z) ∈ t'
[PROOFSTEP]
exact ⟨z, hs.out hx hy hz, rfl⟩
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hFt : ∀ x, F x ∈ t' := fun x => mem_image_of_mem _ (hf x)
[GOAL]
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
rcases F.exists_extension_forall_mem_of_closedEmbedding hFt (hne.image _) he with ⟨G, hG, hGF⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
let g : C(Y, ℝ) :=
⟨h.symm ∘ codRestrict G _ fun y => ht_sub (hG y), h.symm.continuous.comp <| G.continuous.subtype_mk _⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
have hgG : ∀ {y a}, g y = a ↔ G y = h a := @fun y a => h.toEquiv.symm_apply_eq.trans Subtype.ext_iff
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
hgG : ∀ {y : Y} {a : (fun x => ℝ) y}, ↑g y = a ↔ ↑G y = ↑(↑h a)
⊢ ∃ g, (∀ (y : Y), ↑g y ∈ t) ∧ ↑g ∘ e = ↑f
[PROOFSTEP]
refine' ⟨g, fun y => _, _⟩
[GOAL]
case intro.intro.refine'_1
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
hgG : ∀ {y : Y} {a : (fun x => ℝ) y}, ↑g y = a ↔ ↑G y = ↑(↑h a)
y : Y
⊢ ↑g y ∈ t
[PROOFSTEP]
rcases hG y with ⟨a, ha, hay⟩
[GOAL]
case intro.intro.refine'_1.intro.intro
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
hgG : ∀ {y : Y} {a : (fun x => ℝ) y}, ↑g y = a ↔ ↑G y = ↑(↑h a)
y : Y
a : ℝ
ha : a ∈ t
hay : (Subtype.val ∘ ↑h) a = ↑G y
⊢ ↑g y ∈ t
[PROOFSTEP]
convert ha
[GOAL]
case h.e'_4
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
hgG : ∀ {y : Y} {a : (fun x => ℝ) y}, ↑g y = a ↔ ↑G y = ↑(↑h a)
y : Y
a : ℝ
ha : a ∈ t
hay : (Subtype.val ∘ ↑h) a = ↑G y
⊢ ↑g y = a
[PROOFSTEP]
exact hgG.2 hay.symm
[GOAL]
case intro.intro.refine'_2
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
hgG : ∀ {y : Y} {a : (fun x => ℝ) y}, ↑g y = a ↔ ↑G y = ↑(↑h a)
⊢ ↑g ∘ e = ↑f
[PROOFSTEP]
ext x
[GOAL]
case intro.intro.refine'_2.h
X : Type u_1
Y : Type u_2
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : NormalSpace Y
f : C(X, ℝ)
t : Set ℝ
e : X → Y
hs : OrdConnected t
hf : ∀ (x : X), ↑f x ∈ t
hne : Set.Nonempty t
he : ClosedEmbedding e
h : ℝ ≃o ↑(Ioo (-1) 1)
F : X →ᵇ ℝ :=
{ toContinuousMap := mk (Subtype.val ∘ ↑h ∘ ↑f),
map_bounded' :=
(_ :
∃ C,
∀ (x y : X),
dist (ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) x)
(ContinuousMap.toFun (mk (Subtype.val ∘ ↑h ∘ ↑f)) y) ≤
C) }
t' : Set ℝ := Subtype.val ∘ ↑h '' t
ht_sub : t' ⊆ Ioo (-1) 1
this : OrdConnected t'
hFt : ∀ (x : X), ↑F x ∈ t'
G : Y →ᵇ ℝ
hG : ∀ (y : Y), ↑G y ∈ t'
hGF : ↑G ∘ e = ↑F
g : C(Y, ℝ) := mk (↑(OrderIso.symm h) ∘ Set.codRestrict (↑G) (Ioo (-1) 1) (_ : ∀ (y : Y), ↑G y ∈ Ioo (-1) 1))
hgG : ∀ {y : Y} {a : (fun x => ℝ) y}, ↑g y = a ↔ ↑G y = ↑(↑h a)
x : X
⊢ (↑g ∘ e) x = ↑f x
[PROOFSTEP]
exact hgG.2 (congr_fun hGF _)
| {"mathlib_filename": "Mathlib.Topology.TietzeExtension", "llama_tokens": 74789} |
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.666
W : Type ?u.669
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
e : X ≃ₜ Y
⊢ IsProperMap ↑e
[PROOFSTEP]
rw [isProperMap_iff_clusterPt]
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.666
W : Type ?u.669
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
e : X ≃ₜ Y
⊢ Continuous ↑e ∧ ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ ↑e → ∃ x, ↑e x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
refine ⟨e.continuous, fun ℱ y ↦ ?_⟩
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.666
W : Type ?u.669
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
e : X ≃ₜ Y
ℱ : Filter X
y : Y
⊢ MapClusterPt y ℱ ↑e → ∃ x, ↑e x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
simp_rw [MapClusterPt, ClusterPt, ← Filter.push_pull', map_neBot_iff, e.comap_nhds_eq, ← e.coe_toEquiv, ←
e.eq_symm_apply, exists_eq_left]
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.666
W : Type ?u.669
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
e : X ≃ₜ Y
ℱ : Filter X
y : Y
⊢ NeBot (𝓝 (↑(Homeomorph.symm e) y) ⊓ ℱ) → NeBot (𝓝 (↑e.symm y) ⊓ ℱ)
[PROOFSTEP]
exact id
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.2964
W : Type ?u.2967
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
⊢ IsClosedMap f
[PROOFSTEP]
rw [isClosedMap_iff_clusterPt]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.2964
W : Type ?u.2967
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
⊢ ∀ (s : Set X) (y : Y), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
[PROOFSTEP]
exact fun s y ↦ h.clusterPt_of_mapClusterPt (ℱ := 𝓟 s) (y := y)
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
⊢ IsProperMap f ↔ Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rw [isProperMap_iff_clusterPt]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
⊢ (Continuous f ∧ ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ) ↔
Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine and_congr_right (fun _ ↦ ?_)
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
⊢ (∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ) ↔
∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
constructor
[GOAL]
case mp
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
⊢ (∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ) →
∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
intro H
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
⊢ (∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x) →
∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
intro H
[GOAL]
case mp
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ
⊢ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
intro 𝒰 y (hY : (Ultrafilter.map f 𝒰 : Filter Y) ≤ _)
[GOAL]
case mp
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ
𝒰 : Ultrafilter X
y : Y
hY : ↑(Ultrafilter.map f 𝒰) ≤ 𝓝 y
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
simp_rw [← Ultrafilter.clusterPt_iff] at hY ⊢
[GOAL]
case mp
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ
𝒰 : Ultrafilter X
y : Y
hY : ClusterPt y ↑(Ultrafilter.map f 𝒰)
⊢ ∃ x, f x = y ∧ ClusterPt x ↑𝒰
[PROOFSTEP]
exact H hY
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
simp_rw [MapClusterPt, ClusterPt, ← Filter.push_pull', map_neBot_iff, ← exists_ultrafilter_iff, forall_exists_index]
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄ (x : Ultrafilter X), ↑x ≤ comap f (𝓝 y) ⊓ ℱ → ∃ x, f x = y ∧ ∃ u, ↑u ≤ 𝓝 x ⊓ ℱ
[PROOFSTEP]
intro ℱ y 𝒰 hy
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
ℱ : Filter X
y : Y
𝒰 : Ultrafilter X
hy : ↑𝒰 ≤ comap f (𝓝 y) ⊓ ℱ
⊢ ∃ x, f x = y ∧ ∃ u, ↑u ≤ 𝓝 x ⊓ ℱ
[PROOFSTEP]
rcases H (tendsto_iff_comap.mpr <| hy.trans inf_le_left) with ⟨x, hxy, hx⟩
[GOAL]
case mpr.intro.intro
X : Type u_1
Y : Type u_2
Z : Type ?u.3327
W : Type ?u.3330
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
x✝ : Continuous f
H : ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
ℱ : Filter X
y : Y
𝒰 : Ultrafilter X
hy : ↑𝒰 ≤ comap f (𝓝 y) ⊓ ℱ
x : X
hxy : f x = y
hx : ↑𝒰 ≤ 𝓝 x
⊢ ∃ x, f x = y ∧ ∃ u, ↑u ≤ 𝓝 x ⊓ ℱ
[PROOFSTEP]
exact ⟨x, hxy, 𝒰, le_inf hx (hy.trans inf_le_right)⟩
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : IsProperMap f
hg : IsProperMap g
⊢ IsProperMap (Prod.map f g)
[PROOFSTEP]
simp_rw [isProperMap_iff_ultrafilter] at hf hg ⊢
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ Continuous (Prod.map f g) ∧
∀ ⦃𝒰 : Ultrafilter (X × Z)⦄ ⦃y : Y × W⦄, Tendsto (Prod.map f g) (↑𝒰) (𝓝 y) → ∃ x, Prod.map f g x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
constructor
-- Continuity is clear.
[GOAL]
case left
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ Continuous (Prod.map f g)
[PROOFSTEP]
exact
hf.1.prod_map
hg.1
-- Let `𝒰 : Ultrafilter (X × Z)`, and assume that `f × g` tends to some `(y, w) : Y × W`
-- along `𝒰`.
[GOAL]
case right
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ ∀ ⦃𝒰 : Ultrafilter (X × Z)⦄ ⦃y : Y × W⦄, Tendsto (Prod.map f g) (↑𝒰) (𝓝 y) → ∃ x, Prod.map f g x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
intro 𝒰 ⟨y, w⟩ hyw
[GOAL]
case right
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (Prod.map f g) (↑𝒰) (𝓝 (y, w))
⊢ ∃ x, Prod.map f g x = (y, w) ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
simp_rw [nhds_prod_eq, tendsto_prod_iff'] at hyw
[GOAL]
case right
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
⊢ ∃ x, Prod.map f g x = (y, w) ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rcases hf.2 (show Tendsto f (Ultrafilter.map fst 𝒰) (𝓝 y) by simpa using hyw.1) with ⟨x, hxy, hx⟩
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
⊢ Tendsto f (↑(Ultrafilter.map fst 𝒰)) (𝓝 y)
[PROOFSTEP]
simpa using hyw.1
[GOAL]
case right.intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
x : X
hxy : f x = y
hx : ↑(Ultrafilter.map fst 𝒰) ≤ 𝓝 x
⊢ ∃ x, Prod.map f g x = (y, w) ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rcases hg.2 (show Tendsto g (Ultrafilter.map snd 𝒰) (𝓝 w) by simpa using hyw.2) with
⟨z, hzw, hz⟩
-- By the properties of the product topology, that means that `𝒰` tends to `(x, z)`,
-- which completes the proof since `(f × g)(x, z) = (y, w)`.
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
x : X
hxy : f x = y
hx : ↑(Ultrafilter.map fst 𝒰) ≤ 𝓝 x
⊢ Tendsto g (↑(Ultrafilter.map snd 𝒰)) (𝓝 w)
[PROOFSTEP]
simpa using hyw.2
[GOAL]
case right.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
x : X
hxy : f x = y
hx : ↑(Ultrafilter.map fst 𝒰) ≤ 𝓝 x
z : Z
hzw : g z = w
hz : ↑(Ultrafilter.map snd 𝒰) ≤ 𝓝 z
⊢ ∃ x, Prod.map f g x = (y, w) ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine ⟨⟨x, z⟩, Prod.ext hxy hzw, ?_⟩
[GOAL]
case right.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
x : X
hxy : f x = y
hx : ↑(Ultrafilter.map fst 𝒰) ≤ 𝓝 x
z : Z
hzw : g z = w
hz : ↑(Ultrafilter.map snd 𝒰) ≤ 𝓝 z
⊢ ↑𝒰 ≤ 𝓝 (x, z)
[PROOFSTEP]
rw [nhds_prod_eq, le_prod]
[GOAL]
case right.intro.intro.intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
W : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
g : Z → W
hf : Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
hg : Continuous g ∧ ∀ ⦃𝒰 : Ultrafilter Z⦄ ⦃y : W⦄, Tendsto g (↑𝒰) (𝓝 y) → ∃ x, g x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter (X × Z)
y : Y
w : W
hyw : Tendsto (fun n => (Prod.map f g n).fst) (↑𝒰) (𝓝 y) ∧ Tendsto (fun n => (Prod.map f g n).snd) (↑𝒰) (𝓝 w)
x : X
hxy : f x = y
hx : ↑(Ultrafilter.map fst 𝒰) ≤ 𝓝 x
z : Z
hzw : g z = w
hz : ↑(Ultrafilter.map snd 𝒰) ≤ 𝓝 z
⊢ Tendsto fst (↑𝒰) (𝓝 x) ∧ Tendsto snd (↑𝒰) (𝓝 z)
[PROOFSTEP]
exact ⟨hx, hz⟩
[GOAL]
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h : ∀ (i : ι), IsProperMap (f i)
⊢ IsProperMap fun x i => f i (x i)
[PROOFSTEP]
simp_rw [isProperMap_iff_ultrafilter] at h ⊢
[GOAL]
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ (Continuous fun x i => f i (x i)) ∧
∀ ⦃𝒰 : Ultrafilter ((i : ι) → X i)⦄ ⦃y : (i : ι) → Y i⦄,
Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y) → ∃ x, (fun i => f i (x i)) = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
constructor
-- Continuity is clear.
[GOAL]
case left
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ Continuous fun x i => f i (x i)
[PROOFSTEP]
exact
continuous_pi fun i ↦
(h i).1.comp
(continuous_apply i)
-- Let `𝒰 : Ultrafilter (Π i, X i)`, and assume that `Π i, f i` tends to some `y : Π i, Y i`
-- along `𝒰`.
[GOAL]
case right
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
⊢ ∀ ⦃𝒰 : Ultrafilter ((i : ι) → X i)⦄ ⦃y : (i : ι) → Y i⦄,
Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y) → ∃ x, (fun i => f i (x i)) = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
intro 𝒰 y hy
[GOAL]
case right
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter ((i : ι) → X i)
y : (i : ι) → Y i
hy : Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y)
⊢ ∃ x, (fun i => f i (x i)) = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
have : ∀ i, Tendsto (f i) (Ultrafilter.map (eval i) 𝒰) (𝓝 (y i)) := by simpa [tendsto_pi_nhds] using hy
[GOAL]
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter ((i : ι) → X i)
y : (i : ι) → Y i
hy : Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y)
⊢ ∀ (i : ι), Tendsto (f i) (↑(Ultrafilter.map (eval i) 𝒰)) (𝓝 (y i))
[PROOFSTEP]
simpa [tendsto_pi_nhds] using hy
[GOAL]
case right
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter ((i : ι) → X i)
y : (i : ι) → Y i
hy : Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y)
this : ∀ (i : ι), Tendsto (f i) (↑(Ultrafilter.map (eval i) 𝒰)) (𝓝 (y i))
⊢ ∃ x, (fun i => f i (x i)) = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
choose x hxy hx using fun i ↦
(h i).2
(this i)
-- By the properties of the product topology, that means that `𝒰` tends to `x`,
-- which completes the proof since `(Π i, f i) x = y`.
[GOAL]
case right
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter ((i : ι) → X i)
y : (i : ι) → Y i
hy : Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y)
this : ∀ (i : ι), Tendsto (f i) (↑(Ultrafilter.map (eval i) 𝒰)) (𝓝 (y i))
x : (i : ι) → X i
hxy : ∀ (i : ι), f i (x i) = y i
hx : ∀ (i : ι), ↑(Ultrafilter.map (eval i) 𝒰) ≤ 𝓝 (x i)
⊢ ∃ x, (fun i => f i (x i)) = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine ⟨x, funext hxy, ?_⟩
[GOAL]
case right
X✝ : Type ?u.30436
Y✝ : Type ?u.30439
Z : Type ?u.30442
W : Type ?u.30445
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
ι : Type u_3
X : ι → Type u_1
Y : ι → Type u_2
inst✝¹ : (i : ι) → TopologicalSpace (X i)
inst✝ : (i : ι) → TopologicalSpace (Y i)
f : (i : ι) → X i → Y i
h :
∀ (i : ι),
Continuous (f i) ∧ ∀ ⦃𝒰 : Ultrafilter (X i)⦄ ⦃y : Y i⦄, Tendsto (f i) (↑𝒰) (𝓝 y) → ∃ x, f i x = y ∧ ↑𝒰 ≤ 𝓝 x
𝒰 : Ultrafilter ((i : ι) → X i)
y : (i : ι) → Y i
hy : Tendsto (fun x i => f i (x i)) (↑𝒰) (𝓝 y)
this : ∀ (i : ι), Tendsto (f i) (↑(Ultrafilter.map (eval i) 𝒰)) (𝓝 (y i))
x : (i : ι) → X i
hxy : ∀ (i : ι), f i (x i) = y i
hx : ∀ (i : ι), ↑(Ultrafilter.map (eval i) 𝒰) ≤ 𝓝 (x i)
⊢ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rwa [nhds_pi, le_pi]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.36187
W : Type ?u.36190
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
K : Set Y
hK : IsCompact K
⊢ IsCompact (f ⁻¹' K)
[PROOFSTEP]
rw [isCompact_iff_ultrafilter_le_nhds]
-- Let `𝒰 ≤ 𝓟 (f ⁻¹' K)` an ultrafilter.
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.36187
W : Type ?u.36190
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
K : Set Y
hK : IsCompact K
⊢ ∀ (f_1 : Ultrafilter X), ↑f_1 ≤ 𝓟 (f ⁻¹' K) → ∃ a, a ∈ f ⁻¹' K ∧ ↑f_1 ≤ 𝓝 a
[PROOFSTEP]
intro 𝒰 h𝒰
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.36187
W : Type ?u.36190
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
K : Set Y
hK : IsCompact K
𝒰 : Ultrafilter X
h𝒰 : ↑𝒰 ≤ 𝓟 (f ⁻¹' K)
⊢ ∃ a, a ∈ f ⁻¹' K ∧ ↑𝒰 ≤ 𝓝 a
[PROOFSTEP]
rw [← comap_principal, ← map_le_iff_le_comap, ← Ultrafilter.coe_map] at h𝒰
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.36187
W : Type ?u.36190
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
K : Set Y
hK : IsCompact K
𝒰 : Ultrafilter X
h𝒰 : ↑(Ultrafilter.map f 𝒰) ≤ 𝓟 K
⊢ ∃ a, a ∈ f ⁻¹' K ∧ ↑𝒰 ≤ 𝓝 a
[PROOFSTEP]
rcases hK.ultrafilter_le_nhds _ h𝒰 with
⟨y, hyK, hy⟩
-- Then, by properness of `f`, that means that `𝒰` tends to some `x ∈ f ⁻¹' {y} ⊆ f ⁻¹' K`,
-- which completes the proof.
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
Z : Type ?u.36187
W : Type ?u.36190
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
K : Set Y
hK : IsCompact K
𝒰 : Ultrafilter X
h𝒰 : ↑(Ultrafilter.map f 𝒰) ≤ 𝓟 K
y : Y
hyK : y ∈ K
hy : ↑(Ultrafilter.map f 𝒰) ≤ 𝓝 y
⊢ ∃ a, a ∈ f ⁻¹' K ∧ ↑𝒰 ≤ 𝓝 a
[PROOFSTEP]
rcases h.ultrafilter_le_nhds_of_tendsto hy with ⟨x, rfl, hx⟩
[GOAL]
case intro.intro.intro.intro
X : Type u_1
Y : Type u_2
Z : Type ?u.36187
W : Type ?u.36190
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
h : IsProperMap f
K : Set Y
hK : IsCompact K
𝒰 : Ultrafilter X
h𝒰 : ↑(Ultrafilter.map f 𝒰) ≤ 𝓟 K
x : X
hx : ↑𝒰 ≤ 𝓝 x
hyK : f x ∈ K
hy : ↑(Ultrafilter.map f 𝒰) ≤ 𝓝 (f x)
⊢ ∃ a, a ∈ f ⁻¹' K ∧ ↑𝒰 ≤ 𝓝 a
[PROOFSTEP]
exact ⟨x, hyK, hx⟩
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
⊢ IsProperMap f ↔ Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
[PROOFSTEP]
constructor
[GOAL]
case mp
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
⊢ IsProperMap f → Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
[PROOFSTEP]
intro H
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
⊢ (Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})) → IsProperMap f
[PROOFSTEP]
intro H
[GOAL]
case mp
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : IsProperMap f
⊢ Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
[PROOFSTEP]
exact ⟨H.continuous, H.isClosedMap, fun y ↦ H.isCompact_preimage isCompact_singleton⟩
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
⊢ IsProperMap f
[PROOFSTEP]
rw [isProperMap_iff_clusterPt]
-- Let `ℱ : Filter X` and `y` some cluster point of `map f ℱ`.
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
⊢ Continuous f ∧ ∀ ⦃ℱ : Filter X⦄ ⦃y : Y⦄, MapClusterPt y ℱ f → ∃ x, f x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
refine
⟨H.1, fun ℱ y hy ↦ ?_⟩
-- That means that the singleton `pure y` meets the "closure" of `map f ℱ`, by which we mean
-- `Filter.lift' (map f ℱ) closure`. But `f` is closed, so
-- `closure (map f ℱ) = map f (closure ℱ)` (see `IsClosedMap.lift'_closure_map_eq`).
-- Thus `map f (closure ℱ ⊓ 𝓟 (f ⁻¹' {y})) = map f (closure ℱ) ⊓ 𝓟 {y} ≠ ⊥`, hence
-- `closure ℱ ⊓ 𝓟 (f ⁻¹' {y}) ≠ ⊥`.
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
ℱ : Filter X
y : Y
hy : MapClusterPt y ℱ f
⊢ ∃ x, f x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
rw [H.2.1.mapClusterPt_iff_lift'_closure H.1] at hy
[GOAL]
case mpr
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
ℱ : Filter X
y : Y
hy : NeBot (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
⊢ ∃ x, f x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
rcases H.2.2 y (f := Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' { y })) inf_le_right with ⟨x, hxy, hx⟩
[GOAL]
case mpr.intro.intro
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
ℱ : Filter X
y : Y
hy : NeBot (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
x : X
hxy : x ∈ f ⁻¹' {y}
hx : ClusterPt x (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
⊢ ∃ x, f x = y ∧ ClusterPt x ℱ
[PROOFSTEP]
refine
⟨x, hxy, ?_⟩
-- In particular `x` is a cluster point of `closure ℱ`. Since cluster points of `closure ℱ`
-- are exactly cluster points of `ℱ` (see `clusterPt_lift'_closure_iff`), this completes
-- the proof.
[GOAL]
case mpr.intro.intro
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
ℱ : Filter X
y : Y
hy : NeBot (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
x : X
hxy : x ∈ f ⁻¹' {y}
hx : ClusterPt x (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
⊢ ClusterPt x ℱ
[PROOFSTEP]
rw [← clusterPt_lift'_closure_iff]
[GOAL]
case mpr.intro.intro
X : Type u_1
Y : Type u_2
Z : Type ?u.36806
W : Type ?u.36809
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : TopologicalSpace W
f : X → Y
H : Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})
ℱ : Filter X
y : Y
hy : NeBot (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
x : X
hxy : x ∈ f ⁻¹' {y}
hx : ClusterPt x (Filter.lift' ℱ closure ⊓ 𝓟 (f ⁻¹' {y}))
⊢ ClusterPt x (Filter.lift' ℱ closure)
[PROOFSTEP]
exact hx.mono inf_le_left
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.37764
W : Type ?u.37767
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
inst✝¹ : TopologicalSpace W
f : X → Y
inst✝ : T1Space Y
⊢ IsProperMap f ↔ Continuous f ∧ IsClosedMap f ∧ Tendsto f (cocompact X) cofinite
[PROOFSTEP]
simp_rw [isProperMap_iff_isClosedMap_and_compact_fibers, Tendsto, le_cofinite_iff_compl_singleton_mem, mem_map,
preimage_compl]
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.37764
W : Type ?u.37767
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
inst✝¹ : TopologicalSpace W
f : X → Y
inst✝ : T1Space Y
⊢ (Continuous f ∧ IsClosedMap f ∧ ∀ (y : Y), IsCompact (f ⁻¹' {y})) ↔
Continuous f ∧ IsClosedMap f ∧ ∀ (x : Y), (f ⁻¹' {x})ᶜ ∈ cocompact X
[PROOFSTEP]
refine and_congr_right fun f_cont ↦ and_congr_right fun _ ↦ ⟨fun H y ↦ (H y).compl_mem_cocompact, fun H y ↦ ?_⟩
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.37764
W : Type ?u.37767
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
inst✝¹ : TopologicalSpace W
f : X → Y
inst✝ : T1Space Y
f_cont : Continuous f
x✝ : IsClosedMap f
H : ∀ (x : Y), (f ⁻¹' {x})ᶜ ∈ cocompact X
y : Y
⊢ IsCompact (f ⁻¹' {y})
[PROOFSTEP]
rcases mem_cocompact.mp (H y) with ⟨K, hK, hKy⟩
[GOAL]
case intro.intro
X : Type u_2
Y : Type u_1
Z : Type ?u.37764
W : Type ?u.37767
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
inst✝¹ : TopologicalSpace W
f : X → Y
inst✝ : T1Space Y
f_cont : Continuous f
x✝ : IsClosedMap f
H : ∀ (x : Y), (f ⁻¹' {x})ᶜ ∈ cocompact X
y : Y
K : Set X
hK : IsCompact K
hKy : Kᶜ ⊆ (f ⁻¹' {y})ᶜ
⊢ IsCompact (f ⁻¹' {y})
[PROOFSTEP]
exact isCompact_of_isClosed_subset hK (isClosed_singleton.preimage f_cont) (compl_le_compl_iff_le.mp hKy)
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
⊢ IsProperMap f ↔ Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
[PROOFSTEP]
constructor
[GOAL]
case mp
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
⊢ IsProperMap f → Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
[PROOFSTEP]
intro H
[GOAL]
case mpr
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
⊢ (Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)) → IsProperMap f
[PROOFSTEP]
intro H
[GOAL]
case mp
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : IsProperMap f
⊢ Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
[PROOFSTEP]
exact ⟨H.continuous, fun K hK ↦ H.isCompact_preimage hK⟩
[GOAL]
case mpr
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
⊢ IsProperMap f
[PROOFSTEP]
rw [isProperMap_iff_ultrafilter]
-- Let `𝒰 : Ultrafilter X`, and assume that `f` tends to some `y` along `𝒰`.
[GOAL]
case mpr
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
⊢ Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine
⟨H.1, fun 𝒰 y hy ↦ ?_⟩
-- Pick `K` some compact neighborhood of `y`, which exists by local compactness.
[GOAL]
case mpr
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rcases exists_compact_mem_nhds y with
⟨K, hK, hKy⟩
-- Then `map f 𝒰 ≤ 𝓝 y ≤ 𝓟 K`, hence `𝒰 ≤ 𝓟 (f ⁻¹' K)`
[GOAL]
case mpr.intro.intro
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
K : Set Y
hK : IsCompact K
hKy : K ∈ 𝓝 y
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
have : 𝒰 ≤ 𝓟 (f ⁻¹' K) := by
simpa only [← comap_principal, ← tendsto_iff_comap] using
hy.mono_right
(le_principal_iff.mpr hKy)
-- By compactness of `f ⁻¹' K`, `𝒰` converges to some `x ∈ f ⁻¹' K`.
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
K : Set Y
hK : IsCompact K
hKy : K ∈ 𝓝 y
⊢ ↑𝒰 ≤ 𝓟 (f ⁻¹' K)
[PROOFSTEP]
simpa only [← comap_principal, ← tendsto_iff_comap] using
hy.mono_right
(le_principal_iff.mpr hKy)
-- By compactness of `f ⁻¹' K`, `𝒰` converges to some `x ∈ f ⁻¹' K`.
[GOAL]
case mpr.intro.intro
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
K : Set Y
hK : IsCompact K
hKy : K ∈ 𝓝 y
this : ↑𝒰 ≤ 𝓟 (f ⁻¹' K)
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rcases(H.2 hK).ultrafilter_le_nhds _ this with
⟨x, -, hx⟩
-- Finally, `f` tends to `f x` along `𝒰` by continuity, thus `f x = y`.
[GOAL]
case mpr.intro.intro.intro.intro
X : Type u_2
Y : Type u_1
Z : Type ?u.39226
W : Type ?u.39229
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
H : Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
K : Set Y
hK : IsCompact K
hKy : K ∈ 𝓝 y
this : ↑𝒰 ≤ 𝓟 (f ⁻¹' K)
x : X
hx : ↑𝒰 ≤ 𝓝 x
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine ⟨x, tendsto_nhds_unique ((H.1.tendsto _).comp hx) hy, hx⟩
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.49990
W : Type ?u.49993
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
⊢ IsProperMap f ↔ Continuous f ∧ Tendsto f (cocompact X) (cocompact Y)
[PROOFSTEP]
simp_rw [isProperMap_iff_isCompact_preimage, hasBasis_cocompact.tendsto_right_iff, ← mem_preimage, eventually_mem_set,
preimage_compl]
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.49990
W : Type ?u.49993
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
⊢ (Continuous f ∧ ∀ ⦃K : Set Y⦄, IsCompact K → IsCompact (f ⁻¹' K)) ↔
Continuous f ∧ ∀ (i : Set Y), IsCompact i → (f ⁻¹' i)ᶜ ∈ cocompact X
[PROOFSTEP]
refine and_congr_right fun f_cont ↦ ⟨fun H K hK ↦ (H hK).compl_mem_cocompact, fun H K hK ↦ ?_⟩
[GOAL]
X : Type u_2
Y : Type u_1
Z : Type ?u.49990
W : Type ?u.49993
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
f_cont : Continuous f
H : ∀ (i : Set Y), IsCompact i → (f ⁻¹' i)ᶜ ∈ cocompact X
K : Set Y
hK : IsCompact K
⊢ IsCompact (f ⁻¹' K)
[PROOFSTEP]
rcases mem_cocompact.mp (H K hK) with ⟨K', hK', hK'y⟩
[GOAL]
case intro.intro
X : Type u_2
Y : Type u_1
Z : Type ?u.49990
W : Type ?u.49993
inst✝⁵ : TopologicalSpace X
inst✝⁴ : TopologicalSpace Y
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f : X → Y
inst✝¹ : T2Space Y
inst✝ : LocallyCompactSpace Y
f_cont : Continuous f
H : ∀ (i : Set Y), IsCompact i → (f ⁻¹' i)ᶜ ∈ cocompact X
K : Set Y
hK : IsCompact K
K' : Set X
hK' : IsCompact K'
hK'y : K'ᶜ ⊆ (f ⁻¹' K)ᶜ
⊢ IsCompact (f ⁻¹' K)
[PROOFSTEP]
exact isCompact_of_isClosed_subset hK' (hK.isClosed.preimage f_cont) (compl_le_compl_iff_le.mp hK'y)
[GOAL]
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ IsProperMap f ↔ Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
constructor
[GOAL]
case mp
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ IsProperMap f → Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
intro H
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ Continuous f ∧ IsClosedMap (Prod.map f id) → IsProperMap f
[PROOFSTEP]
intro H
[GOAL]
case mp
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : IsProperMap f
⊢ Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
exact ⟨H.continuous, H.universally_closed _⟩
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
⊢ IsProperMap f
[PROOFSTEP]
rw [isProperMap_iff_ultrafilter]
-- Let `𝒰 : Ultrafilter X`, and assume that `f` tends to some `y` along `𝒰`.
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
⊢ Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine
⟨H.1, fun 𝒰 y hy ↦ ?_⟩
-- In `X × Filter X`, consider the closed set `F := closure {(x, ℱ) | ℱ = pure x}`
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
let F : Set (X × Filter X) :=
closure
{xℱ | xℱ.2 = pure xℱ.1}
-- Since `f × id` is closed, the set `(f × id) '' F` is also closed.
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
have := H.2 F isClosed_closure
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
have : (y, ↑𝒰) ∈ Prod.map f id '' F :=
-- Note that, by the properties of the topology on `Filter X`, the function `pure : X → Filter X`
-- tends to the point `𝒰` of `Filter X` along the filter `𝒰` on `X`. Since `f` tends to `y` along
-- `𝒰`, we get that the function `(f, pure) : X → (Y, Filter X)` tends to `(y, 𝒰)` along
-- `𝒰`. Furthermore, each `(f, pure)(x) = (f × id)(x, pure x)` is clearly an element of
-- the closed set `(f × id) '' F`, thus the limit `(y, 𝒰)` also belongs to that set.this.mem_of_tendsto
(hy.prod_mk_nhds (Filter.tendsto_pure_self (𝒰 : Filter X)))
(eventually_of_forall fun x ↦ ⟨⟨x, pure x⟩, subset_closure rfl, rfl⟩)
-- The above shows that `(y, 𝒰) = (f x, 𝒰)`, for some `x : X` such that `(x, 𝒰) ∈ F`.
[GOAL]
case mpr
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this✝ : IsClosed (Prod.map f id '' F)
this : (y, ↑𝒰) ∈ Prod.map f id '' F
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rcases this with
⟨⟨x, _⟩, hx, ⟨_, _⟩⟩
-- We already know that `f x = y`, so to finish the proof we just have to check that `𝒰` tends
-- to `x`. So, for `U ∈ 𝓝 x` arbitrary, let's show that `U ∈ 𝒰`. Since `𝒰` is a ultrafilter,
-- it is enough to show that `Uᶜ` is not in `𝒰`.
[GOAL]
case mpr.intro.mk.intro.refl
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
hy : Tendsto f (↑𝒰) (𝓝 (f x))
hx : (x, 𝒰.1) ∈ F
⊢ ∃ x_1, f x_1 = f x ∧ ↑𝒰 ≤ 𝓝 x_1
[PROOFSTEP]
refine ⟨x, rfl, fun U hU ↦ Ultrafilter.compl_not_mem_iff.mp fun hUc ↦ ?_⟩
[GOAL]
case mpr.intro.mk.intro.refl
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
hy : Tendsto f (↑𝒰) (𝓝 (f x))
hx : (x, 𝒰.1) ∈ F
U : Set X
hU : U ∈ 𝓝 x
hUc : Uᶜ ∈ 𝒰
⊢ False
[PROOFSTEP]
rw [mem_closure_iff_nhds] at hx
[GOAL]
case mpr.intro.mk.intro.refl
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
hy : Tendsto f (↑𝒰) (𝓝 (f x))
hx : ∀ (t : Set (X × Filter X)), t ∈ 𝓝 (x, 𝒰.1) → Set.Nonempty (t ∩ {xℱ | xℱ.snd = pure xℱ.fst})
U : Set X
hU : U ∈ 𝓝 x
hUc : Uᶜ ∈ 𝒰
⊢ False
[PROOFSTEP]
rcases hx (U ×ˢ {𝒢 | Uᶜ ∈ 𝒢}) (prod_mem_nhds hU (isOpen_setOf_mem.mem_nhds hUc)) with
⟨⟨z, 𝒢⟩, ⟨⟨hz : z ∈ U, hz' : Uᶜ ∈ 𝒢⟩, rfl : 𝒢 = pure z⟩⟩
[GOAL]
case mpr.intro.mk.intro.refl.intro.mk.intro.intro
X✝ : Type ?u.52247
Y✝ : Type ?u.52250
Z : Type ?u.52253
W : Type ?u.52256
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
F : Set (X × Filter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
hy : Tendsto f (↑𝒰) (𝓝 (f x))
hx : ∀ (t : Set (X × Filter X)), t ∈ 𝓝 (x, 𝒰.1) → Set.Nonempty (t ∩ {xℱ | xℱ.snd = pure xℱ.fst})
U : Set X
hU : U ∈ 𝓝 x
hUc : Uᶜ ∈ 𝒰
z : X
hz : z ∈ U
hz' : Uᶜ ∈ pure z
⊢ False
[PROOFSTEP]
exact hz' hz
[GOAL]
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ IsProperMap f ↔ Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
constructor
[GOAL]
case mp
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ IsProperMap f → Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
intro H
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ Continuous f ∧ IsClosedMap (Prod.map f id) → IsProperMap f
[PROOFSTEP]
intro H
[GOAL]
case mp
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : IsProperMap f
⊢ Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
exact ⟨H.continuous, H.universally_closed _⟩
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
⊢ IsProperMap f
[PROOFSTEP]
rw [isProperMap_iff_ultrafilter]
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
⊢ Continuous f ∧ ∀ ⦃𝒰 : Ultrafilter X⦄ ⦃y : Y⦄, Tendsto f (↑𝒰) (𝓝 y) → ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
refine ⟨H.1, fun 𝒰 y hy ↦ ?_⟩
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
let F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.2 = pure xℱ.1}
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
have := H.2 F isClosed_closure
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
have : (y, 𝒰) ∈ Prod.map f id '' F :=
this.mem_of_tendsto (hy.prod_mk_nhds (Ultrafilter.tendsto_pure_self 𝒰))
(eventually_of_forall fun x ↦ ⟨⟨x, pure x⟩, subset_closure rfl, rfl⟩)
[GOAL]
case mpr
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
𝒰 : Ultrafilter X
y : Y
hy : Tendsto f (↑𝒰) (𝓝 y)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this✝ : IsClosed (Prod.map f id '' F)
this : (y, 𝒰) ∈ Prod.map f id '' F
⊢ ∃ x, f x = y ∧ ↑𝒰 ≤ 𝓝 x
[PROOFSTEP]
rcases this with ⟨⟨x, _⟩, hx, ⟨_, _⟩⟩
[GOAL]
case mpr.intro.mk.intro.refl
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
snd✝ : Ultrafilter X
hx : (x, snd✝) ∈ F
hy : Tendsto f (↑(id snd✝)) (𝓝 (f x))
⊢ ∃ x_1, f x_1 = f x ∧ ↑(id snd✝) ≤ 𝓝 x_1
[PROOFSTEP]
refine ⟨x, rfl, fun U hU ↦ Ultrafilter.compl_not_mem_iff.mp fun hUc ↦ ?_⟩
[GOAL]
case mpr.intro.mk.intro.refl
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
snd✝ : Ultrafilter X
hx : (x, snd✝) ∈ F
hy : Tendsto f (↑(id snd✝)) (𝓝 (f x))
U : Set X
hU : U ∈ 𝓝 x
hUc : Uᶜ ∈ id snd✝
⊢ False
[PROOFSTEP]
rw [mem_closure_iff_nhds] at hx
[GOAL]
case mpr.intro.mk.intro.refl
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
snd✝ : Ultrafilter X
hx : ∀ (t : Set (X × Ultrafilter X)), t ∈ 𝓝 (x, snd✝) → Set.Nonempty (t ∩ {xℱ | xℱ.snd = pure xℱ.fst})
hy : Tendsto f (↑(id snd✝)) (𝓝 (f x))
U : Set X
hU : U ∈ 𝓝 x
hUc : Uᶜ ∈ id snd✝
⊢ False
[PROOFSTEP]
rcases hx (U ×ˢ {𝒢 | Uᶜ ∈ 𝒢}) (prod_mem_nhds hU ((ultrafilter_isOpen_basic _).mem_nhds hUc)) with
⟨⟨y, 𝒢⟩, ⟨⟨hy : y ∈ U, hy' : Uᶜ ∈ 𝒢⟩, rfl : 𝒢 = pure y⟩⟩
[GOAL]
case mpr.intro.mk.intro.refl.intro.mk.intro.intro
X✝ : Type ?u.54240
Y✝ : Type ?u.54243
Z : Type ?u.54246
W : Type ?u.54249
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ IsClosedMap (Prod.map f id)
F : Set (X × Ultrafilter X) := closure {xℱ | xℱ.snd = pure xℱ.fst}
this : IsClosed (Prod.map f id '' F)
x : X
snd✝ : Ultrafilter X
hx : ∀ (t : Set (X × Ultrafilter X)), t ∈ 𝓝 (x, snd✝) → Set.Nonempty (t ∩ {xℱ | xℱ.snd = pure xℱ.fst})
hy✝ : Tendsto f (↑(id snd✝)) (𝓝 (f x))
U : Set X
hU : U ∈ 𝓝 x
hUc : Uᶜ ∈ id snd✝
y : X
hy : y ∈ U
hy' : Uᶜ ∈ pure y
⊢ False
[PROOFSTEP]
exact hy' hy
[GOAL]
X✝ : Type ?u.56079
Y✝ : Type ?u.56082
Z : Type ?u.56085
W : Type ?u.56088
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ IsProperMap f ↔ Continuous f ∧ ∀ (Z : Type u) [inst : TopologicalSpace Z], IsClosedMap (Prod.map f id)
[PROOFSTEP]
constructor
[GOAL]
case mp
X✝ : Type ?u.56079
Y✝ : Type ?u.56082
Z : Type ?u.56085
W : Type ?u.56088
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ IsProperMap f → Continuous f ∧ ∀ (Z : Type u) [inst : TopologicalSpace Z], IsClosedMap (Prod.map f id)
[PROOFSTEP]
intro H
[GOAL]
case mpr
X✝ : Type ?u.56079
Y✝ : Type ?u.56082
Z : Type ?u.56085
W : Type ?u.56088
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
⊢ (Continuous f ∧ ∀ (Z : Type u) [inst : TopologicalSpace Z], IsClosedMap (Prod.map f id)) → IsProperMap f
[PROOFSTEP]
intro H
[GOAL]
case mp
X✝ : Type ?u.56079
Y✝ : Type ?u.56082
Z : Type ?u.56085
W : Type ?u.56088
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : IsProperMap f
⊢ Continuous f ∧ ∀ (Z : Type u) [inst : TopologicalSpace Z], IsClosedMap (Prod.map f id)
[PROOFSTEP]
exact ⟨H.continuous, fun Z ↦ H.universally_closed _⟩
[GOAL]
case mpr
X✝ : Type ?u.56079
Y✝ : Type ?u.56082
Z : Type ?u.56085
W : Type ?u.56088
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ ∀ (Z : Type u) [inst : TopologicalSpace Z], IsClosedMap (Prod.map f id)
⊢ IsProperMap f
[PROOFSTEP]
rw [isProperMap_iff_isClosedMap_ultrafilter]
[GOAL]
case mpr
X✝ : Type ?u.56079
Y✝ : Type ?u.56082
Z : Type ?u.56085
W : Type ?u.56088
inst✝⁵ : TopologicalSpace X✝
inst✝⁴ : TopologicalSpace Y✝
inst✝³ : TopologicalSpace Z
inst✝² : TopologicalSpace W
f✝ : X✝ → Y✝
X : Type u
Y : Type v
inst✝¹ : TopologicalSpace X
inst✝ : TopologicalSpace Y
f : X → Y
H : Continuous f ∧ ∀ (Z : Type u) [inst : TopologicalSpace Z], IsClosedMap (Prod.map f id)
⊢ Continuous f ∧ IsClosedMap (Prod.map f id)
[PROOFSTEP]
exact ⟨H.1, H.2 _⟩
| {"mathlib_filename": "Mathlib.Topology.ProperMap", "llama_tokens": 32009} |
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
A : SpecialLinearGroup n R
⊢ det (adjugate ↑A) = 1
[PROOFSTEP]
rw [det_adjugate, A.prop, one_pow]
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
A B : SpecialLinearGroup n R
⊢ det (↑A * ↑B) = 1
[PROOFSTEP]
rw [det_mul, A.prop, B.prop, one_mul]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
A B : SpecialLinearGroup n R
inst✝ : Nontrivial R
g : SpecialLinearGroup n R
⊢ det ↑g ≠ 0
[PROOFSTEP]
rw [g.det_coe]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
A B : SpecialLinearGroup n R
inst✝ : Nontrivial R
g : SpecialLinearGroup n R
⊢ 1 ≠ 0
[PROOFSTEP]
norm_num
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
A B : SpecialLinearGroup n R
inst✝ : Nontrivial R
g : SpecialLinearGroup n R
i : n
h : ↑g i = 0
⊢ ∀ (j : n), ↑g i j = 0
[PROOFSTEP]
simp [h]
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
src✝¹ : Monoid (SpecialLinearGroup n R) := monoid
src✝ : Inv (SpecialLinearGroup n R) := hasInv
A : SpecialLinearGroup n R
⊢ A⁻¹ * A = 1
[PROOFSTEP]
ext1
[GOAL]
case a
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
src✝¹ : Monoid (SpecialLinearGroup n R) := monoid
src✝ : Inv (SpecialLinearGroup n R) := hasInv
A : SpecialLinearGroup n R
i✝ j✝ : n
⊢ ↑(A⁻¹ * A) i✝ j✝ = ↑1 i✝ j✝
[PROOFSTEP]
simp [adjugate_mul]
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
A : SpecialLinearGroup n R
⊢ comp (↑Matrix.toLin' ↑A) (↑Matrix.toLin' ↑A⁻¹) = LinearMap.id
[PROOFSTEP]
rw [← toLin'_mul, ← coe_mul, mul_right_inv, coe_one, toLin'_one]
[GOAL]
n : Type u
inst✝² : DecidableEq n
inst✝¹ : Fintype n
R : Type v
inst✝ : CommRing R
A : SpecialLinearGroup n R
⊢ comp (↑Matrix.toLin' ↑A⁻¹) (↑Matrix.toLin' ↑A) = LinearMap.id
[PROOFSTEP]
rw [← toLin'_mul, ← coe_mul, mul_left_inv, coe_one, toLin'_one]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
f : R →+* S
g : SpecialLinearGroup n R
⊢ det (↑(RingHom.mapMatrix f) ↑g) = 1
[PROOFSTEP]
rw [← f.map_det]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
f : R →+* S
g : SpecialLinearGroup n R
⊢ ↑f (det ↑g) = 1
[PROOFSTEP]
simp [g.prop]
[GOAL]
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R : Type v
inst✝² : CommRing R
S : Type u_1
inst✝¹ : CommRing S
inst✝ : Fact (Even (Fintype.card n))
g : SpecialLinearGroup n R
⊢ det (-↑g) = 1
[PROOFSTEP]
simpa [(@Fact.out <| Even <| Fintype.card n).neg_one_pow, g.det_coe] using det_smul (↑ₘg) (-1)
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
⊢ det ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]] = 1
[PROOFSTEP]
rw [Matrix.det_fin_two, mul_comm]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
⊢ vecCons ![↑A 1 1, -↑A 0 1] ![![-↑A 1 0, ↑A 0 0]] 1 1 * vecCons ![↑A 1 1, -↑A 0 1] ![![-↑A 1 0, ↑A 0 0]] 0 0 -
vecCons ![↑A 1 1, -↑A 0 1] ![![-↑A 1 0, ↑A 0 0]] 0 1 * vecCons ![↑A 1 1, -↑A 0 1] ![![-↑A 1 0, ↑A 0 0]] 1 0 =
1
[PROOFSTEP]
simp only [cons_val_zero, cons_val_one, head_cons, mul_neg, neg_mul, neg_neg]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
⊢ ↑A 0 0 * ↑A 1 1 - ↑A 0 1 * ↑A 1 0 = 1
[PROOFSTEP]
have := A.2
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
this : det ↑A = 1
⊢ ↑A 0 0 * ↑A 1 1 - ↑A 0 1 * ↑A 1 0 = 1
[PROOFSTEP]
rw [Matrix.det_fin_two] at this
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
this : ↑A 0 0 * ↑A 1 1 - ↑A 0 1 * ↑A 1 0 = 1
⊢ ↑A 0 0 * ↑A 1 1 - ↑A 0 1 * ↑A 1 0 = 1
[PROOFSTEP]
convert this
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
⊢ A⁻¹ =
{ val := ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]],
property := (_ : det ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]] = 1) }
[PROOFSTEP]
ext
[GOAL]
case a
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
i✝ j✝ : Fin 2
⊢ ↑A⁻¹ i✝ j✝ =
↑{ val := ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]],
property := (_ : det ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]] = 1) }
i✝ j✝
[PROOFSTEP]
have := Matrix.adjugate_fin_two A.1
[GOAL]
case a
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
i✝ j✝ : Fin 2
this : adjugate ↑A = ↑of ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]]
⊢ ↑A⁻¹ i✝ j✝ =
↑{ val := ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]],
property := (_ : det ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]] = 1) }
i✝ j✝
[PROOFSTEP]
rw [coe_inv, this]
[GOAL]
case a
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
A : SL(2, R)
i✝ j✝ : Fin 2
this : adjugate ↑A = ↑of ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]]
⊢ ↑of ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]] i✝ j✝ =
↑{ val := ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]],
property := (_ : det ![![↑A 1 1, -↑A 0 1], ![-↑A 1 0, ↑A 0 0]] = 1) }
i✝ j✝
[PROOFSTEP]
rfl
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
a b c d : R
hdet : a * d - b * c = 1
⊢ det (↑of ![![a, b], ![c, d]]) = 1
[PROOFSTEP]
rwa [det_fin_two_of]
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
g : SL(2, R)
⊢ P g
[PROOFSTEP]
obtain ⟨m, hm⟩ := g
[GOAL]
case mk
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ P { val := m, property := hm }
[PROOFSTEP]
convert h (m 0 0) (m 0 1) (m 1 0) (m 1 1) (by rwa [det_fin_two] at hm )
[GOAL]
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ m 0 0 * m 1 1 - m 0 1 * m 1 0 = 1
[PROOFSTEP]
rwa [det_fin_two] at hm
[GOAL]
case h.e'_1.h.e'_3
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ m = ↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]]
[PROOFSTEP]
ext i j
[GOAL]
case h.e'_1.h.e'_3.a.h
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
i j : Fin 2
⊢ m i j = ↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] i j
[PROOFSTEP]
fin_cases i
[GOAL]
case h.e'_1.h.e'_3.a.h.head
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
j : Fin 2
⊢ m { val := 0, isLt := (_ : 0 < 2) } j = ↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] { val := 0, isLt := (_ : 0 < 2) } j
[PROOFSTEP]
fin_cases j
[GOAL]
case h.e'_1.h.e'_3.a.h.tail.head
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
j : Fin 2
⊢ m { val := 1, isLt := (_ : (fun a => a < 2) 1) } j =
↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] { val := 1, isLt := (_ : (fun a => a < 2) 1) } j
[PROOFSTEP]
fin_cases j
[GOAL]
case h.e'_1.h.e'_3.a.h.head.head
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ m { val := 0, isLt := (_ : 0 < 2) } { val := 0, isLt := (_ : 0 < 2) } =
↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] { val := 0, isLt := (_ : 0 < 2) } { val := 0, isLt := (_ : 0 < 2) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_1.h.e'_3.a.h.head.tail.head
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ m { val := 0, isLt := (_ : 0 < 2) } { val := 1, isLt := (_ : (fun a => a < 2) 1) } =
↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] { val := 0, isLt := (_ : 0 < 2) }
{ val := 1, isLt := (_ : (fun a => a < 2) 1) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_1.h.e'_3.a.h.tail.head.head
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ m { val := 1, isLt := (_ : (fun a => a < 2) 1) } { val := 0, isLt := (_ : 0 < 2) } =
↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] { val := 1, isLt := (_ : (fun a => a < 2) 1) }
{ val := 0, isLt := (_ : 0 < 2) }
[PROOFSTEP]
rfl
[GOAL]
case h.e'_1.h.e'_3.a.h.tail.head.tail.head
n : Type u
inst✝³ : DecidableEq n
inst✝² : Fintype n
R : Type v
inst✝¹ : CommRing R
S : Type u_1
inst✝ : CommRing S
P : SL(2, R) → Prop
h :
∀ (a b c d : R) (hdet : a * d - b * c = 1),
P { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) }
m : Matrix (Fin 2) (Fin 2) R
hm : det m = 1
⊢ m { val := 1, isLt := (_ : (fun a => a < 2) 1) } { val := 1, isLt := (_ : (fun a => a < 2) 1) } =
↑of ![![m 0 0, m 0 1], ![m 1 0, m 1 1]] { val := 1, isLt := (_ : (fun a => a < 2) 1) }
{ val := 1, isLt := (_ : (fun a => a < 2) 1) }
[PROOFSTEP]
rfl
[GOAL]
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg : ↑g 1 0 = 0
a b : R
h : a ≠ 0
⊢ det (↑of ![![a, b], ![0, a⁻¹]]) = 1
[PROOFSTEP]
simp [h]
[GOAL]
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg : ↑g 1 0 = 0
⊢ ∃ a b h, g = { val := ↑of ![![a, b], ![0, a⁻¹]], property := (_ : det (↑of ![![a, b], ![0, a⁻¹]]) = 1) }
[PROOFSTEP]
induction' g using Matrix.SpecialLinearGroup.fin_two_induction with a b c d h_det
[GOAL]
case h
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg✝ : ↑g 1 0 = 0
a b c d : R
h_det : a * d - b * c = 1
hg : ↑{ val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) } 1 0 = 0
⊢ ∃ a_1 b_1 h,
{ val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) } =
{ val := ↑of ![![a_1, b_1], ![0, a_1⁻¹]], property := (_ : det (↑of ![![a_1, b_1], ![0, a_1⁻¹]]) = 1) }
[PROOFSTEP]
replace hg : c = 0 := by simpa using hg
[GOAL]
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg✝ : ↑g 1 0 = 0
a b c d : R
h_det : a * d - b * c = 1
hg : ↑{ val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) } 1 0 = 0
⊢ c = 0
[PROOFSTEP]
simpa using hg
[GOAL]
case h
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg✝ : ↑g 1 0 = 0
a b c d : R
h_det : a * d - b * c = 1
hg : c = 0
⊢ ∃ a_1 b_1 h,
{ val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) } =
{ val := ↑of ![![a_1, b_1], ![0, a_1⁻¹]], property := (_ : det (↑of ![![a_1, b_1], ![0, a_1⁻¹]]) = 1) }
[PROOFSTEP]
have had : a * d = 1 := by rwa [hg, mul_zero, sub_zero] at h_det
[GOAL]
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg✝ : ↑g 1 0 = 0
a b c d : R
h_det : a * d - b * c = 1
hg : c = 0
⊢ a * d = 1
[PROOFSTEP]
rwa [hg, mul_zero, sub_zero] at h_det
[GOAL]
case h
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg✝ : ↑g 1 0 = 0
a b c d : R
h_det : a * d - b * c = 1
hg : c = 0
had : a * d = 1
⊢ ∃ a_1 b_1 h,
{ val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) } =
{ val := ↑of ![![a_1, b_1], ![0, a_1⁻¹]], property := (_ : det (↑of ![![a_1, b_1], ![0, a_1⁻¹]]) = 1) }
[PROOFSTEP]
refine' ⟨a, b, left_ne_zero_of_mul_eq_one had, _⟩
[GOAL]
case h
n : Type u
inst✝⁴ : DecidableEq n
inst✝³ : Fintype n
R✝ : Type v
inst✝² : CommRing R✝
S : Type u_1
inst✝¹ : CommRing S
R : Type u_2
inst✝ : Field R
g : SL(2, R)
hg✝ : ↑g 1 0 = 0
a b c d : R
h_det : a * d - b * c = 1
hg : c = 0
had : a * d = 1
⊢ { val := ↑of ![![a, b], ![c, d]], property := (_ : det (↑of ![![a, b], ![c, d]]) = 1) } =
{ val := ↑of ![![a, b], ![0, a⁻¹]], property := (_ : det (↑of ![![a, b], ![0, a⁻¹]]) = 1) }
[PROOFSTEP]
simp_rw [eq_inv_of_mul_eq_one_right had, hg]
[GOAL]
⊢ det (↑of ![![0, -1], ![1, 0]]) = 1
[PROOFSTEP]
norm_num [Matrix.det_fin_two_of]
[GOAL]
⊢ det (↑of ![![1, 1], ![0, 1]]) = 1
[PROOFSTEP]
norm_num [Matrix.det_fin_two_of]
[GOAL]
⊢ ↑T⁻¹ = ↑of ![![1, -1], ![0, 1]]
[PROOFSTEP]
simp [coe_inv, coe_T, adjugate_fin_two]
[GOAL]
n : ℤ
⊢ ↑(T ^ n) = ↑of ![![1, n], ![0, 1]]
[PROOFSTEP]
induction' n using Int.induction_on with n h n h
[GOAL]
case hz
⊢ ↑(T ^ 0) = ↑of ![![1, 0], ![0, 1]]
[PROOFSTEP]
rw [zpow_zero, coe_one, Matrix.one_fin_two]
[GOAL]
case hp
n : ℕ
h : ↑(T ^ ↑n) = ↑of ![![1, ↑n], ![0, 1]]
⊢ ↑(T ^ (↑n + 1)) = ↑of ![![1, ↑n + 1], ![0, 1]]
[PROOFSTEP]
simp_rw [zpow_add, zpow_one, coe_mul, h, coe_T, Matrix.mul_fin_two]
-- Porting note: was congrm !![_, _; _, _]
[GOAL]
case hp
n : ℕ
h : ↑(T ^ ↑n) = ↑of ![![1, ↑n], ![0, 1]]
⊢ ↑of ![![1 * 1 + ↑n * 0, 1 * 1 + ↑n * 1], ![0 * 1 + 1 * 0, 0 * 1 + 1 * 1]] = ↑of ![![1, ↑n + 1], ![0, 1]]
[PROOFSTEP]
ring_nf
[GOAL]
case hn
n : ℕ
h : ↑(T ^ (-↑n)) = ↑of ![![1, -↑n], ![0, 1]]
⊢ ↑(T ^ (-↑n - 1)) = ↑of ![![1, -↑n - 1], ![0, 1]]
[PROOFSTEP]
simp_rw [zpow_sub, zpow_one, coe_mul, h, coe_T_inv, Matrix.mul_fin_two]
-- Porting note: was congrm !![_, _; _, _]
[GOAL]
case hn
n : ℕ
h : ↑(T ^ (-↑n)) = ↑of ![![1, -↑n], ![0, 1]]
⊢ ↑of ![![1 * 1 + -↑n * 0, 1 * -1 + -↑n * 1], ![0 * 1 + 1 * 0, 0 * -1 + 1 * 1]] = ↑of ![![1, -↑n - 1], ![0, 1]]
[PROOFSTEP]
ring_nf
[GOAL]
n : ℤ
g : SL(2, ℤ)
⊢ ↑(T ^ n * g) 1 = ↑g 1
[PROOFSTEP]
ext j
[GOAL]
case h
n : ℤ
g : SL(2, ℤ)
j : Fin 2
⊢ ↑(T ^ n * g) 1 j = ↑g 1 j
[PROOFSTEP]
simp [coe_T_zpow, Matrix.vecMul, Matrix.dotProduct, Fin.sum_univ_succ, vecTail]
[GOAL]
g : SL(2, ℤ)
⊢ ↑(T * g) 1 = ↑g 1
[PROOFSTEP]
simpa using T_pow_mul_apply_one 1 g
[GOAL]
g : SL(2, ℤ)
⊢ ↑(T⁻¹ * g) 1 = ↑g 1
[PROOFSTEP]
simpa using T_pow_mul_apply_one (-1) g
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.SpecialLinearGroup", "llama_tokens": 9583} |
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f g : α → β
x : α
s t : Set α
y z : β
⊢ LowerSemicontinuousWithinAt f univ x ↔ LowerSemicontinuousAt f x
[PROOFSTEP]
simp [LowerSemicontinuousWithinAt, LowerSemicontinuousAt, nhdsWithin_univ]
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f g : α → β
x : α
s t : Set α
y z : β
⊢ LowerSemicontinuousOn f univ ↔ LowerSemicontinuous f
[PROOFSTEP]
simp [LowerSemicontinuousOn, LowerSemicontinuous, lowerSemicontinuousWithinAt_univ_iff]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x : α
s t : Set α
y z : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
⊢ LowerSemicontinuous (indicator s fun _x => y)
[PROOFSTEP]
intro x z hz
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
hz : z < indicator s (fun _x => y) x
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
by_cases h : x ∈ s
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
hz : z < indicator s (fun _x => y) x
h : x ∈ s
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h] at hz
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
hz : z < indicator s (fun _x => y) x
h : ¬x ∈ s
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h] at hz
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
h : x ∈ s
hz : z < y
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
filter_upwards [hs.mem_nhds h]
[GOAL]
case h
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
h : x ∈ s
hz : z < y
⊢ ∀ (a : α), a ∈ s → z < indicator s (fun _x => y) a
[PROOFSTEP]
simp (config := { contextual := true }) [hz]
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
h : ¬x ∈ s
hz : z < 0
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
refine Filter.eventually_of_forall fun x' => ?_
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
h : ¬x ∈ s
hz : z < 0
x' : α
⊢ z < indicator s (fun _x => y) x'
[PROOFSTEP]
by_cases h' : x' ∈ s
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
h : ¬x ∈ s
hz : z < 0
x' : α
h' : x' ∈ s
⊢ z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h', hz.trans_le hy, hz]
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsOpen s
hy : 0 ≤ y
x : α
z : β
h : ¬x ∈ s
hz : z < 0
x' : α
h' : ¬x' ∈ s
⊢ z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h', hz.trans_le hy, hz]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x : α
s t : Set α
y z : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
⊢ LowerSemicontinuous (indicator s fun _x => y)
[PROOFSTEP]
intro x z hz
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
hz : z < indicator s (fun _x => y) x
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
by_cases h : x ∈ s
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
hz : z < indicator s (fun _x => y) x
h : x ∈ s
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h] at hz
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
hz : z < indicator s (fun _x => y) x
h : ¬x ∈ s
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h] at hz
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
h : x ∈ s
hz : z < y
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
refine Filter.eventually_of_forall fun x' => ?_
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
h : x ∈ s
hz : z < y
x' : α
⊢ z < indicator s (fun _x => y) x'
[PROOFSTEP]
by_cases h' : x' ∈ s
[GOAL]
case pos
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
h : x ∈ s
hz : z < y
x' : α
h' : x' ∈ s
⊢ z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h', hz, hz.trans_le hy]
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
h : x ∈ s
hz : z < y
x' : α
h' : ¬x' ∈ s
⊢ z < indicator s (fun _x => y) x'
[PROOFSTEP]
simp [h', hz, hz.trans_le hy]
[GOAL]
case neg
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
h : ¬x ∈ s
hz : z < 0
⊢ ∀ᶠ (x' : α) in 𝓝 x, z < indicator s (fun _x => y) x'
[PROOFSTEP]
filter_upwards [hs.isOpen_compl.mem_nhds h]
[GOAL]
case h
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f g : α → β
x✝ : α
s t : Set α
y z✝ : β
inst✝ : Zero β
hs : IsClosed s
hy : y ≤ 0
x : α
z : β
h : ¬x ∈ s
hz : z < 0
⊢ ∀ (a : α), a ∈ sᶜ → z < indicator s (fun _x => y) a
[PROOFSTEP]
simp (config := { contextual := true }) [hz]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝ : LinearOrder γ
f : α → γ
⊢ LowerSemicontinuous f ↔ ∀ (y : γ), IsClosed (f ⁻¹' Iic y)
[PROOFSTEP]
rw [lowerSemicontinuous_iff_isOpen_preimage]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝ : LinearOrder γ
f : α → γ
⊢ (∀ (y : γ), IsOpen (f ⁻¹' Ioi y)) ↔ ∀ (y : γ), IsClosed (f ⁻¹' Iic y)
[PROOFSTEP]
simp only [← isOpen_compl_iff, ← preimage_compl, compl_Iic]
[GOAL]
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
⊢ LowerSemicontinuousWithinAt (g ∘ f) s x
[PROOFSTEP]
intro y hy
[GOAL]
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (g ∘ f) x'
[PROOFSTEP]
by_cases h : ∃ l, l < f x
[GOAL]
case pos
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
h : ∃ l, l < f x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (g ∘ f) x'
[PROOFSTEP]
obtain ⟨z, zlt, hz⟩ : ∃ z < f x, Ioc z (f x) ⊆ g ⁻¹' Ioi y := exists_Ioc_subset_of_mem_nhds (hg (Ioi_mem_nhds hy)) h
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
h : ∃ l, l < f x
z : γ
zlt : z < f x
hz : Ioc z (f x) ⊆ g ⁻¹' Ioi y
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (g ∘ f) x'
[PROOFSTEP]
filter_upwards [hf z zlt] with a ha
[GOAL]
case h
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
h : ∃ l, l < f x
z : γ
zlt : z < f x
hz : Ioc z (f x) ⊆ g ⁻¹' Ioi y
a : α
ha : z < f a
⊢ y < (g ∘ f) a
[PROOFSTEP]
calc
y < g (min (f x) (f a)) := hz (by simp [zlt, ha, le_refl])
_ ≤ g (f a) := gmon (min_le_right _ _)
[GOAL]
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
h : ∃ l, l < f x
z : γ
zlt : z < f x
hz : Ioc z (f x) ⊆ g ⁻¹' Ioi y
a : α
ha : z < f a
⊢ min (f x) (f a) ∈ Ioc z (f x)
[PROOFSTEP]
simp [zlt, ha, le_refl]
[GOAL]
case neg
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
h : ¬∃ l, l < f x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (g ∘ f) x'
[PROOFSTEP]
simp only [not_exists, not_lt] at h
[GOAL]
case neg
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousWithinAt f s x
gmon : Monotone g
y : δ
hy : y < (g ∘ f) x
h : ∀ (x_1 : γ), f x ≤ x_1
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (g ∘ f) x'
[PROOFSTEP]
exact Filter.eventually_of_forall fun a => hy.trans_le (gmon (h (f a)))
[GOAL]
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
hf : LowerSemicontinuousAt f x
gmon : Monotone g
⊢ LowerSemicontinuousAt (g ∘ f) x
[PROOFSTEP]
simp only [← lowerSemicontinuousWithinAt_univ_iff] at hf ⊢
[GOAL]
α : Type u_1
inst✝⁷ : TopologicalSpace α
β : Type u_2
inst✝⁶ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝⁵ : LinearOrder γ
inst✝⁴ : TopologicalSpace γ
inst✝³ : OrderTopology γ
δ : Type u_4
inst✝² : LinearOrder δ
inst✝¹ : TopologicalSpace δ
inst✝ : OrderTopology δ
g : γ → δ
f : α → γ
hg : ContinuousAt g (f x)
gmon : Monotone g
hf : LowerSemicontinuousWithinAt f univ x
⊢ LowerSemicontinuousWithinAt (g ∘ f) univ x
[PROOFSTEP]
exact hg.comp_lowerSemicontinuousWithinAt hf gmon
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
⊢ LowerSemicontinuousWithinAt (fun z => f z + g z) s x
[PROOFSTEP]
intro y hy
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
obtain ⟨u, v, u_open, xu, v_open, xv, h⟩ :
∃ u v : Set γ, IsOpen u ∧ f x ∈ u ∧ IsOpen v ∧ g x ∈ v ∧ u ×ˢ v ⊆ {p : γ × γ | y < p.fst + p.snd} :=
mem_nhds_prod_iff'.1 (hcont (isOpen_Ioi.mem_nhds hy))
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
by_cases hx₁ : ∃ l, l < f x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
obtain ⟨z₁, z₁lt, h₁⟩ : ∃ z₁ < f x, Ioc z₁ (f x) ⊆ u := exists_Ioc_subset_of_mem_nhds (u_open.mem_nhds xu) hx₁
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
by_cases hx₂ : ∃ l, l < g x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
obtain ⟨z₂, z₂lt, h₂⟩ : ∃ z₂ < g x, Ioc z₂ (g x) ⊆ v := exists_Ioc_subset_of_mem_nhds (v_open.mem_nhds xv) hx₂
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
filter_upwards [hf z₁ z₁lt, hg z₂ z₂lt] with z h₁z h₂z
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
⊢ y < f z + g z
[PROOFSTEP]
have A1 : min (f z) (f x) ∈ u := by
by_cases H : f z ≤ f x
· simp [H]
exact h₁ ⟨h₁z, H⟩
· simp [le_of_not_le H]
exact h₁ ⟨z₁lt, le_rfl⟩
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
⊢ min (f z) (f x) ∈ u
[PROOFSTEP]
by_cases H : f z ≤ f x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
H : f z ≤ f x
⊢ min (f z) (f x) ∈ u
[PROOFSTEP]
simp [H]
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
H : f z ≤ f x
⊢ f z ∈ u
[PROOFSTEP]
exact h₁ ⟨h₁z, H⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
H : ¬f z ≤ f x
⊢ min (f z) (f x) ∈ u
[PROOFSTEP]
simp [le_of_not_le H]
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
H : ¬f z ≤ f x
⊢ f x ∈ u
[PROOFSTEP]
exact h₁ ⟨z₁lt, le_rfl⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
⊢ y < f z + g z
[PROOFSTEP]
have A2 : min (g z) (g x) ∈ v := by
by_cases H : g z ≤ g x
· simp [H]
exact h₂ ⟨h₂z, H⟩
· simp [le_of_not_le H]
exact h₂ ⟨z₂lt, le_rfl⟩
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
⊢ min (g z) (g x) ∈ v
[PROOFSTEP]
by_cases H : g z ≤ g x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
H : g z ≤ g x
⊢ min (g z) (g x) ∈ v
[PROOFSTEP]
simp [H]
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
H : g z ≤ g x
⊢ g z ∈ v
[PROOFSTEP]
exact h₂ ⟨h₂z, H⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
H : ¬g z ≤ g x
⊢ min (g z) (g x) ∈ v
[PROOFSTEP]
simp [le_of_not_le H]
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
H : ¬g z ≤ g x
⊢ g x ∈ v
[PROOFSTEP]
exact h₂ ⟨z₂lt, le_rfl⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
A2 : min (g z) (g x) ∈ v
⊢ y < f z + g z
[PROOFSTEP]
have : (min (f z) (f x), min (g z) (g x)) ∈ u ×ˢ v := ⟨A1, A2⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₁z : z₁ < f z
h₂z : z₂ < g z
A1 : min (f z) (f x) ∈ u
A2 : min (g z) (g x) ∈ v
this : (min (f z) (f x), min (g z) (g x)) ∈ u ×ˢ v
⊢ y < f z + g z
[PROOFSTEP]
calc
y < min (f z) (f x) + min (g z) (g x) := h this
_ ≤ f z + g z := add_le_add (min_le_left _ _) (min_le_left _ _)
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ¬∃ l, l < g x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
simp only [not_exists, not_lt] at hx₂
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
filter_upwards [hf z₁ z₁lt] with z h₁z
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
⊢ y < f z + g z
[PROOFSTEP]
have A1 : min (f z) (f x) ∈ u := by
by_cases H : f z ≤ f x
· simp [H]
exact h₁ ⟨h₁z, H⟩
· simp [le_of_not_le H]
exact h₁ ⟨z₁lt, le_rfl⟩
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
⊢ min (f z) (f x) ∈ u
[PROOFSTEP]
by_cases H : f z ≤ f x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
H : f z ≤ f x
⊢ min (f z) (f x) ∈ u
[PROOFSTEP]
simp [H]
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
H : f z ≤ f x
⊢ f z ∈ u
[PROOFSTEP]
exact h₁ ⟨h₁z, H⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
H : ¬f z ≤ f x
⊢ min (f z) (f x) ∈ u
[PROOFSTEP]
simp [le_of_not_le H]
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
H : ¬f z ≤ f x
⊢ f x ∈ u
[PROOFSTEP]
exact h₁ ⟨z₁lt, le_rfl⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
A1 : min (f z) (f x) ∈ u
⊢ y < f z + g z
[PROOFSTEP]
have : (min (f z) (f x), g x) ∈ u ×ˢ v := ⟨A1, xv⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∃ l, l < f x
z₁ : γ
z₁lt : z₁ < f x
h₁ : Ioc z₁ (f x) ⊆ u
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
h₁z : z₁ < f z
A1 : min (f z) (f x) ∈ u
this : (min (f z) (f x), g x) ∈ u ×ˢ v
⊢ y < f z + g z
[PROOFSTEP]
calc
y < min (f z) (f x) + g x := h this
_ ≤ f z + g z := add_le_add (min_le_left _ _) (hx₂ (g z))
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ¬∃ l, l < f x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
simp only [not_exists, not_lt] at hx₁
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
by_cases hx₂ : ∃ l, l < g x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
obtain ⟨z₂, z₂lt, h₂⟩ : ∃ z₂ < g x, Ioc z₂ (g x) ⊆ v := exists_Ioc_subset_of_mem_nhds (v_open.mem_nhds xv) hx₂
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
filter_upwards [hg z₂ z₂lt] with z h₂z
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
⊢ y < f z + g z
[PROOFSTEP]
have A2 : min (g z) (g x) ∈ v := by
by_cases H : g z ≤ g x
· simp [H]
exact h₂ ⟨h₂z, H⟩
· simp [le_of_not_le H]
exact h₂ ⟨z₂lt, le_rfl⟩
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
⊢ min (g z) (g x) ∈ v
[PROOFSTEP]
by_cases H : g z ≤ g x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
H : g z ≤ g x
⊢ min (g z) (g x) ∈ v
[PROOFSTEP]
simp [H]
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
H : g z ≤ g x
⊢ g z ∈ v
[PROOFSTEP]
exact h₂ ⟨h₂z, H⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
H : ¬g z ≤ g x
⊢ min (g z) (g x) ∈ v
[PROOFSTEP]
simp [le_of_not_le H]
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
H : ¬g z ≤ g x
⊢ g x ∈ v
[PROOFSTEP]
exact h₂ ⟨z₂lt, le_rfl⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
A2 : min (g z) (g x) ∈ v
⊢ y < f z + g z
[PROOFSTEP]
have : (f x, min (g z) (g x)) ∈ u ×ˢ v := ⟨xu, A2⟩
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∃ l, l < g x
z₂ : γ
z₂lt : z₂ < g x
h₂ : Ioc z₂ (g x) ⊆ v
z : α
h₂z : z₂ < g z
A2 : min (g z) (g x) ∈ v
this : (f x, min (g z) (g x)) ∈ u ×ˢ v
⊢ y < f z + g z
[PROOFSTEP]
calc
y < f x + min (g z) (g x) := h this
_ ≤ f z + g z := add_le_add (hx₁ (f z)) (min_le_left _ _)
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ¬∃ l, l < g x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
simp only [not_exists, not_lt] at hx₁ hx₂
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun z => f z + g z) x'
[PROOFSTEP]
apply Filter.eventually_of_forall
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
⊢ ∀ (x : α), y < (fun z => f z + g z) x
[PROOFSTEP]
intro z
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
⊢ y < (fun z => f z + g z) z
[PROOFSTEP]
have : (f x, g x) ∈ u ×ˢ v := ⟨xu, xv⟩
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y✝ z✝ : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousWithinAt f s x
hg : LowerSemicontinuousWithinAt g s x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
y : γ
hy : y < (fun z => f z + g z) x
u v : Set γ
u_open : IsOpen u
xu : f x ∈ u
v_open : IsOpen v
xv : g x ∈ v
h : u ×ˢ v ⊆ {p | y < p.fst + p.snd}
hx₁ : ∀ (x_1 : γ), f x ≤ x_1
hx₂ : ∀ (x_1 : γ), g x ≤ x_1
z : α
this : (f x, g x) ∈ u ×ˢ v
⊢ y < (fun z => f z + g z) z
[PROOFSTEP]
calc
y < f x + g x := h this
_ ≤ f z + g z := add_le_add (hx₁ (f z)) (hx₂ (g z))
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : LowerSemicontinuousAt f x
hg : LowerSemicontinuousAt g x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
⊢ LowerSemicontinuousAt (fun z => f z + g z) x
[PROOFSTEP]
simp_rw [← lowerSemicontinuousWithinAt_univ_iff] at *
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
hf : LowerSemicontinuousWithinAt f univ x
hg : LowerSemicontinuousWithinAt g univ x
⊢ LowerSemicontinuousWithinAt (fun z => f z + g z) univ x
[PROOFSTEP]
exact hf.add' hg hcont
[GOAL]
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha : ∀ (i : ι), i ∈ a → LowerSemicontinuousWithinAt (f i) s x
⊢ LowerSemicontinuousWithinAt (fun z => ∑ i in a, f i z) s x
[PROOFSTEP]
classical
induction' a using Finset.induction_on with i a ia IH
· exact lowerSemicontinuousWithinAt_const
· simp only [ia, Finset.sum_insert, not_false_iff]
exact
LowerSemicontinuousWithinAt.add (ha _ (Finset.mem_insert_self i a))
(IH fun j ja => ha j (Finset.mem_insert_of_mem ja))
[GOAL]
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha : ∀ (i : ι), i ∈ a → LowerSemicontinuousWithinAt (f i) s x
⊢ LowerSemicontinuousWithinAt (fun z => ∑ i in a, f i z) s x
[PROOFSTEP]
induction' a using Finset.induction_on with i a ia IH
[GOAL]
case empty
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha✝ : ∀ (i : ι), i ∈ a → LowerSemicontinuousWithinAt (f i) s x
ha : ∀ (i : ι), i ∈ ∅ → LowerSemicontinuousWithinAt (f i) s x
⊢ LowerSemicontinuousWithinAt (fun z => ∑ i in ∅, f i z) s x
[PROOFSTEP]
exact lowerSemicontinuousWithinAt_const
[GOAL]
case insert
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a✝ : Finset ι
ha✝ : ∀ (i : ι), i ∈ a✝ → LowerSemicontinuousWithinAt (f i) s x
i : ι
a : Finset ι
ia : ¬i ∈ a
IH :
(∀ (i : ι), i ∈ a → LowerSemicontinuousWithinAt (f i) s x) →
LowerSemicontinuousWithinAt (fun z => ∑ i in a, f i z) s x
ha : ∀ (i_1 : ι), i_1 ∈ insert i a → LowerSemicontinuousWithinAt (f i_1) s x
⊢ LowerSemicontinuousWithinAt (fun z => ∑ i in insert i a, f i z) s x
[PROOFSTEP]
simp only [ia, Finset.sum_insert, not_false_iff]
[GOAL]
case insert
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a✝ : Finset ι
ha✝ : ∀ (i : ι), i ∈ a✝ → LowerSemicontinuousWithinAt (f i) s x
i : ι
a : Finset ι
ia : ¬i ∈ a
IH :
(∀ (i : ι), i ∈ a → LowerSemicontinuousWithinAt (f i) s x) →
LowerSemicontinuousWithinAt (fun z => ∑ i in a, f i z) s x
ha : ∀ (i_1 : ι), i_1 ∈ insert i a → LowerSemicontinuousWithinAt (f i_1) s x
⊢ LowerSemicontinuousWithinAt (fun z => f i z + ∑ i in a, f i z) s x
[PROOFSTEP]
exact
LowerSemicontinuousWithinAt.add (ha _ (Finset.mem_insert_self i a))
(IH fun j ja => ha j (Finset.mem_insert_of_mem ja))
[GOAL]
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha : ∀ (i : ι), i ∈ a → LowerSemicontinuousAt (f i) x
⊢ LowerSemicontinuousAt (fun z => ∑ i in a, f i z) x
[PROOFSTEP]
simp_rw [← lowerSemicontinuousWithinAt_univ_iff] at *
[GOAL]
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha : ∀ (i : ι), i ∈ a → LowerSemicontinuousWithinAt (f i) univ x
⊢ LowerSemicontinuousWithinAt (fun z => ∑ i in a, f i z) univ x
[PROOFSTEP]
exact lowerSemicontinuousWithinAt_sum ha
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝[s] x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
⊢ LowerSemicontinuousWithinAt (fun x' => ⨆ (i : ι), f i x') s x
[PROOFSTEP]
cases isEmpty_or_nonempty ι
[GOAL]
case inl
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝[s] x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
h✝ : IsEmpty ι
⊢ LowerSemicontinuousWithinAt (fun x' => ⨆ (i : ι), f i x') s x
[PROOFSTEP]
simpa only [iSup_of_empty'] using lowerSemicontinuousWithinAt_const
[GOAL]
case inr
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝[s] x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
h✝ : Nonempty ι
⊢ LowerSemicontinuousWithinAt (fun x' => ⨆ (i : ι), f i x') s x
[PROOFSTEP]
intro y hy
[GOAL]
case inr
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y✝ z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝[s] x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
h✝ : Nonempty ι
y : δ'
hy : y < (fun x' => ⨆ (i : ι), f i x') x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun x' => ⨆ (i : ι), f i x') x'
[PROOFSTEP]
rcases exists_lt_of_lt_ciSup hy with ⟨i, hi⟩
[GOAL]
case inr.intro
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y✝ z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝[s] x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
h✝ : Nonempty ι
y : δ'
hy : y < (fun x' => ⨆ (i : ι), f i x') x
i : ι
hi : y < f i x
⊢ ∀ᶠ (x' : α) in 𝓝[s] x, y < (fun x' => ⨆ (i : ι), f i x') x'
[PROOFSTEP]
filter_upwards [h i y hi, bdd] with y hy hy' using hy.trans_le (le_ciSup hy' i)
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
⊢ ∀ᶠ (y : α) in 𝓝[s] x, BddAbove (range fun i => f i y)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝 x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousAt (f i) x
⊢ LowerSemicontinuousAt (fun x' => ⨆ (i : ι), f i x') x
[PROOFSTEP]
simp_rw [← lowerSemicontinuousWithinAt_univ_iff] at *
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝 x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) univ x
⊢ LowerSemicontinuousWithinAt (fun x' => ⨆ (i : ι), f i x') univ x
[PROOFSTEP]
rw [← nhdsWithin_univ] at bdd
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ'
bdd : ∀ᶠ (y : α) in 𝓝[univ] x, BddAbove (range fun i => f i y)
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) univ x
⊢ LowerSemicontinuousWithinAt (fun x' => ⨆ (i : ι), f i x') univ x
[PROOFSTEP]
exact lowerSemicontinuousWithinAt_ciSup bdd h
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ
h : ∀ (i : ι), LowerSemicontinuousAt (f i) x
⊢ ∀ᶠ (y : α) in 𝓝 x, BddAbove (range fun i => f i y)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ
h : ∀ (i : ι), LowerSemicontinuousOn (f i) s
⊢ ∀ (x : α), x ∈ s → BddAbove (range fun i => f i x)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
inst✝³ : TopologicalSpace α
β : Type u_2
inst✝² : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Sort u_3
δ : Type u_4
δ' : Type u_5
inst✝¹ : CompleteLinearOrder δ
inst✝ : ConditionallyCompleteLinearOrder δ'
f : ι → α → δ
h : ∀ (i : ι), LowerSemicontinuous (f i)
⊢ ∀ (x : α), BddAbove (range fun i => f i x)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
f : ι → α → ℝ≥0∞
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
⊢ LowerSemicontinuousWithinAt (fun x' => ∑' (i : ι), f i x') s x
[PROOFSTEP]
simp_rw [ENNReal.tsum_eq_iSup_sum]
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
f : ι → α → ℝ≥0∞
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
⊢ LowerSemicontinuousWithinAt (fun x' => ⨆ (s : Finset ι), ∑ i in s, f i x') s x
[PROOFSTEP]
refine lowerSemicontinuousWithinAt_iSup fun b => ?_
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
f : ι → α → ℝ≥0∞
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) s x
b : Finset ι
⊢ LowerSemicontinuousWithinAt (fun x' => ∑ i in b, f i x') s x
[PROOFSTEP]
exact lowerSemicontinuousWithinAt_sum fun i _hi => h i
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
f : ι → α → ℝ≥0∞
h : ∀ (i : ι), LowerSemicontinuousAt (f i) x
⊢ LowerSemicontinuousAt (fun x' => ∑' (i : ι), f i x') x
[PROOFSTEP]
simp_rw [← lowerSemicontinuousWithinAt_univ_iff] at *
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
f : ι → α → ℝ≥0∞
h : ∀ (i : ι), LowerSemicontinuousWithinAt (f i) univ x
⊢ LowerSemicontinuousWithinAt (fun x' => ∑' (i : ι), f i x') univ x
[PROOFSTEP]
exact lowerSemicontinuousWithinAt_tsum h
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f g : α → β
x : α
s t : Set α
y z : β
⊢ UpperSemicontinuousWithinAt f univ x ↔ UpperSemicontinuousAt f x
[PROOFSTEP]
simp [UpperSemicontinuousWithinAt, UpperSemicontinuousAt, nhdsWithin_univ]
[GOAL]
α : Type u_1
inst✝¹ : TopologicalSpace α
β : Type u_2
inst✝ : Preorder β
f g : α → β
x : α
s t : Set α
y z : β
⊢ UpperSemicontinuousOn f univ ↔ UpperSemicontinuous f
[PROOFSTEP]
simp [UpperSemicontinuousOn, UpperSemicontinuous, upperSemicontinuousWithinAt_univ_iff]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝ : LinearOrder γ
f : α → γ
⊢ UpperSemicontinuous f ↔ ∀ (y : γ), IsClosed (f ⁻¹' Ici y)
[PROOFSTEP]
rw [upperSemicontinuous_iff_isOpen_preimage]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
β : Type u_2
inst✝¹ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝ : LinearOrder γ
f : α → γ
⊢ (∀ (y : γ), IsOpen (f ⁻¹' Iio y)) ↔ ∀ (y : γ), IsClosed (f ⁻¹' Ici y)
[PROOFSTEP]
simp only [← isOpen_compl_iff, ← preimage_compl, compl_Ici]
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hf : UpperSemicontinuousAt f x
hg : UpperSemicontinuousAt g x
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
⊢ UpperSemicontinuousAt (fun z => f z + g z) x
[PROOFSTEP]
simp_rw [← upperSemicontinuousWithinAt_univ_iff] at *
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g✝ : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝² : LinearOrderedAddCommMonoid γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f g : α → γ
hcont : ContinuousAt (fun p => p.fst + p.snd) (f x, g x)
hf : UpperSemicontinuousWithinAt f univ x
hg : UpperSemicontinuousWithinAt g univ x
⊢ UpperSemicontinuousWithinAt (fun z => f z + g z) univ x
[PROOFSTEP]
exact hf.add' hg hcont
[GOAL]
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha : ∀ (i : ι), i ∈ a → UpperSemicontinuousAt (f i) x
⊢ UpperSemicontinuousAt (fun z => ∑ i in a, f i z) x
[PROOFSTEP]
simp_rw [← upperSemicontinuousWithinAt_univ_iff] at *
[GOAL]
α : Type u_1
inst✝⁵ : TopologicalSpace α
β : Type u_2
inst✝⁴ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
ι : Type u_3
γ : Type u_4
inst✝³ : LinearOrderedAddCommMonoid γ
inst✝² : TopologicalSpace γ
inst✝¹ : OrderTopology γ
inst✝ : ContinuousAdd γ
f : ι → α → γ
a : Finset ι
ha : ∀ (i : ι), i ∈ a → UpperSemicontinuousWithinAt (f i) univ x
⊢ UpperSemicontinuousWithinAt (fun z => ∑ i in a, f i z) univ x
[PROOFSTEP]
exact upperSemicontinuousWithinAt_sum ha
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
⊢ ContinuousWithinAt f s x ↔ LowerSemicontinuousWithinAt f s x ∧ UpperSemicontinuousWithinAt f s x
[PROOFSTEP]
refine' ⟨fun h => ⟨h.lowerSemicontinuousWithinAt, h.upperSemicontinuousWithinAt⟩, _⟩
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
⊢ LowerSemicontinuousWithinAt f s x ∧ UpperSemicontinuousWithinAt f s x → ContinuousWithinAt f s x
[PROOFSTEP]
rintro ⟨h₁, h₂⟩
[GOAL]
case intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
intro v hv
[GOAL]
case intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
⊢ v ∈ map f (𝓝[s] x)
[PROOFSTEP]
simp only [Filter.mem_map]
[GOAL]
case intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
by_cases Hl : ∃ l, l < f x
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
rcases exists_Ioc_subset_of_mem_nhds hv Hl with ⟨l, lfx, hl⟩
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
by_cases Hu : ∃ u, f x < u
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ∃ u, f x < u
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
rcases exists_Ico_subset_of_mem_nhds hv Hu with ⟨u, fxu, hu⟩
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
filter_upwards [h₁ l lfx, h₂ u fxu] with a lfa fau
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
a : α
lfa : l < f a
fau : f a < u
⊢ a ∈ f ⁻¹' v
[PROOFSTEP]
cases' le_or_gt (f a) (f x) with h h
[GOAL]
case h.inl
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
a : α
lfa : l < f a
fau : f a < u
h : f a ≤ f x
⊢ a ∈ f ⁻¹' v
[PROOFSTEP]
exact hl ⟨lfa, h⟩
[GOAL]
case h.inr
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
a : α
lfa : l < f a
fau : f a < u
h : f a > f x
⊢ a ∈ f ⁻¹' v
[PROOFSTEP]
exact hu ⟨le_of_lt h, fau⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ¬∃ u, f x < u
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
simp only [not_exists, not_lt] at Hu
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∃ l, l < f x
l : γ
lfx : l < f x
hl : Ioc l (f x) ⊆ v
Hu : ∀ (x_1 : γ), x_1 ≤ f x
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
filter_upwards [h₁ l lfx] with a lfa using hl ⟨lfa, Hu (f a)⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ¬∃ l, l < f x
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
simp only [not_exists, not_lt] at Hl
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
by_cases Hu : ∃ u, f x < u
[GOAL]
case pos
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∃ u, f x < u
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
rcases exists_Ico_subset_of_mem_nhds hv Hu with ⟨u, fxu, hu⟩
[GOAL]
case pos.intro.intro
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
filter_upwards [h₂ u fxu] with a lfa
[GOAL]
case h
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
a : α
lfa : f a < u
⊢ a ∈ f ⁻¹' v
[PROOFSTEP]
apply hu
[GOAL]
case h.a
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∃ u, f x < u
u : γ
fxu : f x < u
hu : Ico (f x) u ⊆ v
a : α
lfa : f a < u
⊢ f a ∈ Ico (f x) u
[PROOFSTEP]
exact ⟨Hl (f a), lfa⟩
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ¬∃ u, f x < u
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
simp only [not_exists, not_lt] at Hu
[GOAL]
case neg
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∀ (x_1 : γ), x_1 ≤ f x
⊢ f ⁻¹' v ∈ 𝓝[s] x
[PROOFSTEP]
apply Filter.eventually_of_forall
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∀ (x_1 : γ), x_1 ≤ f x
⊢ ∀ (x : α), f x ∈ v
[PROOFSTEP]
intro a
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∀ (x_1 : γ), x_1 ≤ f x
a : α
⊢ f a ∈ v
[PROOFSTEP]
have : f a = f x := le_antisymm (Hu _) (Hl _)
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∀ (x_1 : γ), x_1 ≤ f x
a : α
this : f a = f x
⊢ f a ∈ v
[PROOFSTEP]
rw [this]
[GOAL]
case neg.hp
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
h₁ : LowerSemicontinuousWithinAt f s x
h₂ : UpperSemicontinuousWithinAt f s x
v : Set γ
hv : v ∈ 𝓝 (f x)
Hl : ∀ (x_1 : γ), f x ≤ x_1
Hu : ∀ (x_1 : γ), x_1 ≤ f x
a : α
this : f a = f x
⊢ f x ∈ v
[PROOFSTEP]
exact mem_of_mem_nhds hv
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
⊢ ContinuousAt f x ↔ LowerSemicontinuousAt f x ∧ UpperSemicontinuousAt f x
[PROOFSTEP]
simp_rw [← continuousWithinAt_univ, ← lowerSemicontinuousWithinAt_univ_iff, ← upperSemicontinuousWithinAt_univ_iff,
continuousWithinAt_iff_lower_upperSemicontinuousWithinAt]
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
⊢ ContinuousOn f s ↔ LowerSemicontinuousOn f s ∧ UpperSemicontinuousOn f s
[PROOFSTEP]
simp only [ContinuousOn, continuousWithinAt_iff_lower_upperSemicontinuousWithinAt]
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
⊢ (∀ (x : α), x ∈ s → LowerSemicontinuousWithinAt f s x ∧ UpperSemicontinuousWithinAt f s x) ↔
LowerSemicontinuousOn f s ∧ UpperSemicontinuousOn f s
[PROOFSTEP]
exact ⟨fun H => ⟨fun x hx => (H x hx).1, fun x hx => (H x hx).2⟩, fun H x hx => ⟨H.1 x hx, H.2 x hx⟩⟩
[GOAL]
α : Type u_1
inst✝⁴ : TopologicalSpace α
β : Type u_2
inst✝³ : Preorder β
f✝ g : α → β
x : α
s t : Set α
y z : β
γ : Type u_3
inst✝² : LinearOrder γ
inst✝¹ : TopologicalSpace γ
inst✝ : OrderTopology γ
f : α → γ
⊢ Continuous f ↔ LowerSemicontinuous f ∧ UpperSemicontinuous f
[PROOFSTEP]
simp_rw [continuous_iff_continuousOn_univ, continuousOn_iff_lower_upperSemicontinuousOn, lowerSemicontinuousOn_univ_iff,
upperSemicontinuousOn_univ_iff]
| {"mathlib_filename": "Mathlib.Topology.Semicontinuous", "llama_tokens": 42428} |
[GOAL]
X : Type ?u.7
inst✝² : TopologicalSpace X
s : Set X
inst✝¹ : T0Space ↑s
inst✝ : SecondCountableTopology ↑s
⊢ HasCountableSeparatingOn X IsOpen s
[PROOFSTEP]
suffices HasCountableSeparatingOn s IsOpen univ from .of_subtype fun _ ↦ isOpen_induced_iff.1
[GOAL]
X : Type ?u.7
inst✝² : TopologicalSpace X
s : Set X
inst✝¹ : T0Space ↑s
inst✝ : SecondCountableTopology ↑s
⊢ HasCountableSeparatingOn (↑s) IsOpen univ
[PROOFSTEP]
refine ⟨⟨countableBasis s, countable_countableBasis _, fun _ ↦ isOpen_of_mem_countableBasis, fun x _ y _ h ↦ ?_⟩⟩
[GOAL]
X : Type ?u.7
inst✝² : TopologicalSpace X
s : Set X
inst✝¹ : T0Space ↑s
inst✝ : SecondCountableTopology ↑s
x : ↑s
x✝¹ : x ∈ univ
y : ↑s
x✝ : y ∈ univ
h : ∀ (s_1 : Set ↑s), s_1 ∈ countableBasis ↑s → (x ∈ s_1 ↔ y ∈ s_1)
⊢ x = y
[PROOFSTEP]
exact ((isBasis_countableBasis _).inseparable_iff.2 h).eq
| {"mathlib_filename": "Mathlib.Topology.CountableSeparatingOn", "llama_tokens": 416} |
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
z : α
s : Set α
p : α → Prop
⊢ (∃ᶠ (x : α) in 𝓝[s] z, p x) ↔ ∃ᶠ (x : α) in 𝓝 z, p x ∧ x ∈ s
[PROOFSTEP]
simp only [Filter.Frequently, eventually_nhdsWithin_iff, not_and']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
z : α
s : Set α
⊢ z ∈ closure (s \ {z}) ↔ ∃ᶠ (x : α) in 𝓝[{z}ᶜ] z, x ∈ s
[PROOFSTEP]
simp [mem_closure_iff_frequently, frequently_nhdsWithin_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
p : α → Prop
⊢ (∀ᶠ (y : α) in 𝓝[s] a, ∀ᶠ (x : α) in 𝓝[s] y, p x) ↔ ∀ᶠ (x : α) in 𝓝[s] a, p x
[PROOFSTEP]
refine' ⟨fun h => _, fun h => (eventually_nhds_nhdsWithin.2 h).filter_mono inf_le_left⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
p : α → Prop
h : ∀ᶠ (y : α) in 𝓝[s] a, ∀ᶠ (x : α) in 𝓝[s] y, p x
⊢ ∀ᶠ (x : α) in 𝓝[s] a, p x
[PROOFSTEP]
simp only [eventually_nhdsWithin_iff] at h ⊢
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
p : α → Prop
h : ∀ᶠ (x : α) in 𝓝 a, x ∈ s → ∀ᶠ (x : α) in 𝓝 x, x ∈ s → p x
⊢ ∀ᶠ (x : α) in 𝓝 a, x ∈ s → p x
[PROOFSTEP]
exact h.mono fun x hx hxs => (hx hxs).self_of_nhds hxs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
⊢ 𝓝[univ] a = 𝓝 a
[PROOFSTEP]
rw [nhdsWithin, principal_univ, inf_top_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
t : Set α
a : α
s : Set α
⊢ t ∈ 𝓝[s] a ↔ ∃ u, IsOpen u ∧ a ∈ u ∧ u ∩ s ⊆ t
[PROOFSTEP]
simpa only [and_assoc, and_left_comm] using (nhdsWithin_basis_open a s).mem_iff
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
x : α
s t : Set α
hs : s ∈ 𝓝[t] x
t' : Set α
⊢ s \ t' ∈ 𝓝[t \ t'] x
[PROOFSTEP]
rw [nhdsWithin, diff_eq, diff_eq, ← inf_principal, ← inf_assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
x : α
s t : Set α
hs : s ∈ 𝓝[t] x
t' : Set α
⊢ s ∩ t'ᶜ ∈ 𝓝 x ⊓ 𝓟 t ⊓ 𝓟 t'ᶜ
[PROOFSTEP]
exact inter_mem_inf hs (mem_principal_self _)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
a : α
h1 : s ∈ 𝓝 a
h2 : t ∈ 𝓝[s] a
⊢ t ∈ 𝓝 a
[PROOFSTEP]
rcases mem_nhdsWithin_iff_exists_mem_nhds_inter.mp h2 with ⟨_, Hw, hw⟩
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
a : α
h1 : s ∈ 𝓝 a
h2 : t ∈ 𝓝[s] a
w✝ : Set α
Hw : w✝ ∈ 𝓝 a
hw : w✝ ∩ s ⊆ t
⊢ t ∈ 𝓝 a
[PROOFSTEP]
exact (nhds a).sets_of_superset ((nhds a).inter_sets Hw h1) hw
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
x : α
⊢ t ∈ 𝓝[s] x ↔ s =ᶠ[𝓝 x] s ∩ t
[PROOFSTEP]
simp_rw [mem_nhdsWithin_iff_eventually, eventuallyEq_set, mem_inter_iff, iff_self_and]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
π : α → β
s : Set β
t : Set α
a : α
h : a ∈ t
hs : s ∈ 𝓝 (π a)
⊢ π ⁻¹' s ∈ 𝓝[t] a
[PROOFSTEP]
lift a to t using h
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
π : α → β
s : Set β
t : Set α
a : { x // x ∈ t }
hs : s ∈ 𝓝 (π ↑a)
⊢ π ⁻¹' s ∈ 𝓝[t] ↑a
[PROOFSTEP]
replace hs : (fun x : t => π x) ⁻¹' s ∈ 𝓝 a := preimage_nhds_coinduced hs
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
π : α → β
s : Set β
t : Set α
a : { x // x ∈ t }
hs : (fun x => π ↑x) ⁻¹' s ∈ 𝓝 a
⊢ π ⁻¹' s ∈ 𝓝[t] ↑a
[PROOFSTEP]
rwa [← map_nhds_subtype_val, mem_map]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
⊢ 𝓝[s] a ≤ 𝓝 a
[PROOFSTEP]
rw [← nhdsWithin_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
⊢ 𝓝[s] a ≤ 𝓝[univ] a
[PROOFSTEP]
apply nhdsWithin_le_of_mem
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
⊢ univ ∈ 𝓝[s] a
[PROOFSTEP]
exact univ_mem
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t u : Set α
hs : s ∈ 𝓝 a
h₂ : t ∩ s = u ∩ s
⊢ 𝓝[t] a = 𝓝[u] a
[PROOFSTEP]
rw [nhdsWithin_restrict' t hs, nhdsWithin_restrict' u hs, h₂]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t u : Set α
h₀ : a ∈ s
h₁ : IsOpen s
h₂ : t ∩ s = u ∩ s
⊢ 𝓝[t] a = 𝓝[u] a
[PROOFSTEP]
rw [nhdsWithin_restrict t h₀ h₁, nhdsWithin_restrict u h₀ h₁, h₂]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
π : α → β
s : Set β
t : Set α
a : α
h : a ∈ t
ht : IsOpen t
hs : s ∈ 𝓝 (π a)
⊢ π ⁻¹' s ∈ 𝓝 a
[PROOFSTEP]
rw [← ht.nhdsWithin_eq h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
π : α → β
s : Set β
t : Set α
a : α
h : a ∈ t
ht : IsOpen t
hs : s ∈ 𝓝 (π a)
⊢ π ⁻¹' s ∈ 𝓝[t] a
[PROOFSTEP]
exact preimage_nhdsWithin_coinduced' h hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
⊢ 𝓝[∅] a = ⊥
[PROOFSTEP]
rw [nhdsWithin, principal_empty, inf_bot_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ 𝓝[s ∪ t] a = 𝓝[s] a ⊔ 𝓝[t] a
[PROOFSTEP]
delta nhdsWithin
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ 𝓝 a ⊓ 𝓟 (s ∪ t) = 𝓝 a ⊓ 𝓟 s ⊔ 𝓝 a ⊓ 𝓟 t
[PROOFSTEP]
rw [← inf_sup_left, sup_principal]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
ι : Type u_5
I : Set ι
hI : Set.Finite I
s : ι → Set α
a : α
⊢ 𝓝[⋃ (i : ι) (_ : i ∈ ∅), s i] a = ⨆ (i : ι) (_ : i ∈ ∅), 𝓝[s i] a
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
ι : Type u_5
I : Set ι
hI : Set.Finite I
s : ι → Set α
a : α
a✝ : ι
s✝ : Set ι
x✝¹ : ¬a✝ ∈ s✝
x✝ : Set.Finite s✝
hT : 𝓝[⋃ (i : ι) (_ : i ∈ s✝), s i] a = ⨆ (i : ι) (_ : i ∈ s✝), 𝓝[s i] a
⊢ 𝓝[⋃ (i : ι) (_ : i ∈ insert a✝ s✝), s i] a = ⨆ (i : ι) (_ : i ∈ insert a✝ s✝), 𝓝[s i] a
[PROOFSTEP]
simp only [hT, nhdsWithin_union, iSup_insert, biUnion_insert]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
S : Set (Set α)
hS : Set.Finite S
a : α
⊢ 𝓝[⋃₀ S] a = ⨆ (s : Set α) (_ : s ∈ S), 𝓝[s] a
[PROOFSTEP]
rw [sUnion_eq_biUnion, nhdsWithin_biUnion hS]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
ι : Sort u_5
inst✝ : Finite ι
s : ι → Set α
a : α
⊢ 𝓝[⋃ (i : ι), s i] a = ⨆ (i : ι), 𝓝[s i] a
[PROOFSTEP]
rw [← sUnion_range, nhdsWithin_sUnion (finite_range s), iSup_range]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ 𝓝[s ∩ t] a = 𝓝[s] a ⊓ 𝓝[t] a
[PROOFSTEP]
delta nhdsWithin
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ 𝓝 a ⊓ 𝓟 (s ∩ t) = 𝓝 a ⊓ 𝓟 s ⊓ (𝓝 a ⊓ 𝓟 t)
[PROOFSTEP]
rw [inf_left_comm, inf_assoc, inf_principal, ← inf_assoc, inf_idem]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ 𝓝[s ∩ t] a = 𝓝[s] a ⊓ 𝓟 t
[PROOFSTEP]
delta nhdsWithin
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ 𝓝 a ⊓ 𝓟 (s ∩ t) = 𝓝 a ⊓ 𝓟 s ⊓ 𝓟 t
[PROOFSTEP]
rw [← inf_principal, inf_assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
h : s ∈ 𝓝[t] a
⊢ 𝓝[s ∩ t] a = 𝓝[t] a
[PROOFSTEP]
rw [nhdsWithin_inter, inf_eq_right]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
h : s ∈ 𝓝[t] a
⊢ 𝓝[t] a ≤ 𝓝[s] a
[PROOFSTEP]
exact nhdsWithin_le_of_mem h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
h : t ∈ 𝓝[s] a
⊢ 𝓝[s ∩ t] a = 𝓝[s] a
[PROOFSTEP]
rw [inter_comm, nhdsWithin_inter_of_mem h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
⊢ 𝓝[{a}] a = pure a
[PROOFSTEP]
rw [nhdsWithin, principal_singleton, inf_eq_right.2 (pure_le_nhds a)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
⊢ 𝓝[insert a s] a = pure a ⊔ 𝓝[s] a
[PROOFSTEP]
rw [← singleton_union, nhdsWithin_union, nhdsWithin_singleton]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
⊢ t ∈ 𝓝[insert a s] a ↔ a ∈ t ∧ t ∈ 𝓝[s] a
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s t : Set α
h : t ∈ 𝓝[s] a
⊢ insert a t ∈ 𝓝[insert a s] a
[PROOFSTEP]
simp [mem_of_superset h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
s : Set α
⊢ insert a s ∈ 𝓝 a ↔ s ∈ 𝓝[{a}ᶜ] a
[PROOFSTEP]
simp only [nhdsWithin, mem_inf_principal, mem_compl_iff, mem_singleton_iff, or_iff_not_imp_left, insert_def]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
a : α
⊢ 𝓝[{a}ᶜ] a ⊔ pure a = 𝓝 a
[PROOFSTEP]
rw [← nhdsWithin_singleton, ← nhdsWithin_union, compl_union_self, nhdsWithin_univ]
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α✝
α : Type u_5
inst✝¹ : TopologicalSpace α
β : Type u_6
inst✝ : TopologicalSpace β
s u : Set α
t v : Set β
a : α
b : β
hu : u ∈ 𝓝[s] a
hv : v ∈ 𝓝[t] b
⊢ u ×ˢ v ∈ 𝓝[s ×ˢ t] (a, b)
[PROOFSTEP]
rw [nhdsWithin_prod_eq]
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α✝
α : Type u_5
inst✝¹ : TopologicalSpace α
β : Type u_6
inst✝ : TopologicalSpace β
s u : Set α
t v : Set β
a : α
b : β
hu : u ∈ 𝓝[s] a
hv : v ∈ 𝓝[t] b
⊢ u ×ˢ v ∈ 𝓝[s] a ×ˢ 𝓝[t] b
[PROOFSTEP]
exact prod_mem_prod hu hv
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ 𝓝[Set.pi I s] x = ⨅ (i : ι), comap (fun x => x i) (𝓝 (x i) ⊓ ⨅ (_ : i ∈ I), 𝓟 (s i))
[PROOFSTEP]
simp only [nhdsWithin, nhds_pi, Filter.pi, comap_inf, comap_iInf, pi_def, comap_principal, ← iInf_principal_finite hI, ←
iInf_inf_eq]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ 𝓝[Set.pi I s] x =
(⨅ (i : ι) (_ : i ∈ I), comap (fun x => x i) (𝓝[s i] x i)) ⊓ ⨅ (i : ι) (_ : ¬i ∈ I), comap (fun x => x i) (𝓝 (x i))
[PROOFSTEP]
simp only [nhdsWithin, nhds_pi, Filter.pi, pi_def, ← iInf_principal_finite hI, comap_inf, comap_principal, eval]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ (⨅ (i : ι), comap (fun f => f i) (𝓝 (x i))) ⊓ ⨅ (i : ι) (_ : i ∈ I), 𝓟 ((fun f => f i) ⁻¹' s i) =
(⨅ (i : ι) (_ : i ∈ I), comap (fun x => x i) (𝓝 (x i)) ⊓ 𝓟 ((fun x => x i) ⁻¹' s i)) ⊓
⨅ (i : ι) (_ : ¬i ∈ I), comap (fun x => x i) (𝓝 (x i))
[PROOFSTEP]
rw [iInf_split _ fun i => i ∈ I, inf_right_comm]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ ((⨅ (i : ι) (_ : i ∈ I), comap (fun f => f i) (𝓝 (x i))) ⊓ ⨅ (i : ι) (_ : i ∈ I), 𝓟 ((fun f => f i) ⁻¹' s i)) ⊓
⨅ (i : ι) (_ : ¬i ∈ I), comap (fun f => f i) (𝓝 (x i)) =
(⨅ (i : ι) (_ : i ∈ I), comap (fun x => x i) (𝓝 (x i)) ⊓ 𝓟 ((fun x => x i) ⁻¹' s i)) ⊓
⨅ (i : ι) (_ : ¬i ∈ I), comap (fun x => x i) (𝓝 (x i))
[PROOFSTEP]
simp only [iInf_inf_eq]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝¹ : Finite ι
inst✝ : (i : ι) → TopologicalSpace (α i)
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ 𝓝[Set.pi univ s] x = ⨅ (i : ι), comap (fun x => x i) (𝓝[s i] x i)
[PROOFSTEP]
simpa [nhdsWithin] using nhdsWithin_pi_eq finite_univ s x
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ 𝓝[Set.pi I s] x = ⊥ ↔ ∃ i, i ∈ I ∧ 𝓝[s i] x i = ⊥
[PROOFSTEP]
simp only [nhdsWithin, nhds_pi, pi_inf_principal_pi_eq_bot]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ NeBot (𝓝[Set.pi I s] x) ↔ ∀ (i : ι), i ∈ I → NeBot (𝓝[s i] x i)
[PROOFSTEP]
simp [neBot_iff, nhdsWithin_pi_eq_bot]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
f g : α → β
t : Set α
inst✝ : (x : α) → Decidable (x ∈ t)
a : α
s : Set α
l : Filter β
h₀ : Tendsto f (𝓝[s ∩ t] a) l
h₁ : Tendsto g (𝓝[s ∩ tᶜ] a) l
⊢ Tendsto (piecewise t f g) (𝓝[s] a) l
[PROOFSTEP]
apply Tendsto.piecewise
[GOAL]
case h₀
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
f g : α → β
t : Set α
inst✝ : (x : α) → Decidable (x ∈ t)
a : α
s : Set α
l : Filter β
h₀ : Tendsto f (𝓝[s ∩ t] a) l
h₁ : Tendsto g (𝓝[s ∩ tᶜ] a) l
⊢ Tendsto f (𝓝[s] a ⊓ 𝓟 t) l
[PROOFSTEP]
rwa [← nhdsWithin_inter']
[GOAL]
case h₁
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
f g : α → β
t : Set α
inst✝ : (x : α) → Decidable (x ∈ t)
a : α
s : Set α
l : Filter β
h₀ : Tendsto f (𝓝[s ∩ t] a) l
h₁ : Tendsto g (𝓝[s ∩ tᶜ] a) l
⊢ Tendsto g (𝓝[s] a ⊓ 𝓟 tᶜ) l
[PROOFSTEP]
rwa [← nhdsWithin_inter']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
f : β → α
a : α
s : Set α
l : Filter β
h : Tendsto f l (𝓝[s] a)
⊢ ∀ᶠ (i : β) in l, f i ∈ s
[PROOFSTEP]
simp_rw [nhdsWithin_eq, tendsto_iInf, mem_setOf_eq, tendsto_principal, mem_inter_iff, eventually_and] at h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
f : β → α
a : α
s : Set α
l : Filter β
h : ∀ (i : Set α), a ∈ i ∧ IsOpen i → (∀ᶠ (x : β) in l, f x ∈ i) ∧ ∀ᶠ (x : β) in l, f x ∈ s
⊢ ∀ᶠ (i : β) in l, f i ∈ s
[PROOFSTEP]
exact (h univ ⟨mem_univ a, isOpen_univ⟩).2
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α✝
α : Type u_5
s : Set α
t : Set ↑s
⊢ 𝓟 t = comap Subtype.val (𝓟 (Subtype.val '' t))
[PROOFSTEP]
rw [comap_principal, preimage_image_eq _ Subtype.coe_injective]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
I : Set ι
s : (i : ι) → Set (α i)
x : (i : ι) → α i
⊢ x ∈ closure (Set.pi I s) ↔ ∀ (i : ι), i ∈ I → x i ∈ closure (s i)
[PROOFSTEP]
simp only [mem_closure_iff_nhdsWithin_neBot, nhdsWithin_pi_neBot]
[GOAL]
α✝ : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α✝
ι : Type u_5
α : ι → Type u_6
inst✝ : (i : ι) → TopologicalSpace (α i)
s : (i : ι) → Set (α i)
I : Set ι
hs : ∀ (i : ι), i ∈ I → Dense (s i)
⊢ Dense (Set.pi I s)
[PROOFSTEP]
simp only [dense_iff_closure_eq, closure_pi_set, pi_congr rfl fun i hi => (hs i hi).closure_eq, pi_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s : Set α
a : { x // x ∈ s }
t u : Set { x // x ∈ s }
⊢ t ∈ 𝓝[u] a ↔ t ∈ comap Subtype.val (𝓝[Subtype.val '' u] ↑a)
[PROOFSTEP]
rw [nhdsWithin, nhds_subtype, principal_subtype, ← comap_inf, ← nhdsWithin]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s : Set α
a : ↑s
t : Set ↑s
⊢ t ∈ 𝓝 a ↔ Subtype.val '' t ∈ 𝓝[s] ↑a
[PROOFSTEP]
rw [← map_nhds_subtype_val, image_mem_map_iff Subtype.val_injective]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
a : ↑s
⊢ Subtype.val ⁻¹' t ∈ 𝓝 a ↔ t ∈ 𝓝[s] ↑a
[PROOFSTEP]
rw [← map_nhds_subtype_val, mem_map]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s : Set α
a : α
h : a ∈ s
f : α → β
l : Filter β
⊢ Tendsto f (𝓝[s] a) l ↔ Tendsto (restrict s f) (𝓝 { val := a, property := h }) l
[PROOFSTEP]
rw [nhdsWithin_eq_map_subtype_coe h, tendsto_map'_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝ : TopologicalSpace α
s : Set α
a : α
h : a ∈ s
f : α → β
l : Filter β
⊢ Tendsto (f ∘ Subtype.val) (𝓝 { val := a, property := h }) l ↔ Tendsto (restrict s f) (𝓝 { val := a, property := h }) l
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
x : α
⊢ ContinuousWithinAt f univ x ↔ ContinuousAt f x
[PROOFSTEP]
rw [ContinuousAt, ContinuousWithinAt, nhdsWithin_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → γ
g : β → δ
s : Set α
t : Set β
x : α
y : β
hf : ContinuousWithinAt f s x
hg : ContinuousWithinAt g t y
⊢ ContinuousWithinAt (Prod.map f g) (s ×ˢ t) (x, y)
[PROOFSTEP]
unfold ContinuousWithinAt at *
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → γ
g : β → δ
s : Set α
t : Set β
x : α
y : β
hf : Tendsto f (𝓝[s] x) (𝓝 (f x))
hg : Tendsto g (𝓝[t] y) (𝓝 (g y))
⊢ Tendsto (Prod.map f g) (𝓝[s ×ˢ t] (x, y)) (𝓝 (Prod.map f g (x, y)))
[PROOFSTEP]
rw [nhdsWithin_prod_eq, Prod.map, nhds_prod_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → γ
g : β → δ
s : Set α
t : Set β
x : α
y : β
hf : Tendsto f (𝓝[s] x) (𝓝 (f x))
hg : Tendsto g (𝓝[t] y) (𝓝 (g y))
⊢ Tendsto (Prod.map f g) (𝓝[s] x ×ˢ 𝓝[t] y) (𝓝 (f x) ×ˢ 𝓝 (g y))
[PROOFSTEP]
exact hf.prod_map hg
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ ContinuousOn f s ↔ ∀ (x : α), x ∈ s → ∀ (t : Set β), IsOpen t → f x ∈ t → ∃ u, IsOpen u ∧ x ∈ u ∧ u ∩ s ⊆ f ⁻¹' t
[PROOFSTEP]
simp only [ContinuousOn, ContinuousWithinAt, tendsto_nhds, mem_nhdsWithin]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ ContinuousOn f s ↔ Continuous (restrict s f)
[PROOFSTEP]
rw [ContinuousOn, continuous_iff_continuousAt]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ (∀ (x : α), x ∈ s → ContinuousWithinAt f s x) ↔ ∀ (x : ↑s), ContinuousAt (restrict s f) x
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ (∀ (x : α), x ∈ s → ContinuousWithinAt f s x) → ∀ (x : ↑s), ContinuousAt (restrict s f) x
[PROOFSTEP]
rintro h ⟨x, xs⟩
[GOAL]
case mp.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ∀ (x : α), x ∈ s → ContinuousWithinAt f s x
x : α
xs : x ∈ s
⊢ ContinuousAt (restrict s f) { val := x, property := xs }
[PROOFSTEP]
exact (continuousWithinAt_iff_continuousAt_restrict f xs).mp (h x xs)
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ (∀ (x : ↑s), ContinuousAt (restrict s f) x) → ∀ (x : α), x ∈ s → ContinuousWithinAt f s x
[PROOFSTEP]
intro h x xs
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ∀ (x : ↑s), ContinuousAt (restrict s f) x
x : α
xs : x ∈ s
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
exact (continuousWithinAt_iff_continuousAt_restrict f xs).mpr (h ⟨x, xs⟩)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ ContinuousOn f s ↔ ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
have : ∀ t, IsOpen (s.restrict f ⁻¹' t) ↔ ∃ u : Set α, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s :=
by
intro t
rw [isOpen_induced_iff, Set.restrict_eq, Set.preimage_comp]
simp only [Subtype.preimage_coe_eq_preimage_coe_iff]
constructor <;>
· rintro ⟨u, ou, useq⟩
exact ⟨u, ou, useq.symm⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ ∀ (t : Set β), IsOpen (restrict s f ⁻¹' t) ↔ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
intro t
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ IsOpen (restrict s f ⁻¹' t) ↔ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
rw [isOpen_induced_iff, Set.restrict_eq, Set.preimage_comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ (∃ t_1, IsOpen t_1 ∧ Subtype.val ⁻¹' t_1 = Subtype.val ⁻¹' (f ⁻¹' t)) ↔ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
simp only [Subtype.preimage_coe_eq_preimage_coe_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ (∃ t_1, IsOpen t_1 ∧ t_1 ∩ s = f ⁻¹' t ∩ s) ↔ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ (∃ t_1, IsOpen t_1 ∧ t_1 ∩ s = f ⁻¹' t ∩ s) → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
rintro ⟨u, ou, useq⟩
[GOAL]
case mp.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
u : Set α
ou : IsOpen u
useq : u ∩ s = f ⁻¹' t ∩ s
⊢ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
exact ⟨u, ou, useq.symm⟩
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ (∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) → ∃ t_1, IsOpen t_1 ∧ t_1 ∩ s = f ⁻¹' t ∩ s
[PROOFSTEP]
rintro ⟨u, ou, useq⟩
[GOAL]
case mpr.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
u : Set α
ou : IsOpen u
useq : f ⁻¹' t ∩ s = u ∩ s
⊢ ∃ t_1, IsOpen t_1 ∧ t_1 ∩ s = f ⁻¹' t ∩ s
[PROOFSTEP]
exact ⟨u, ou, useq.symm⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
this : ∀ (t : Set β), IsOpen (restrict s f ⁻¹' t) ↔ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
⊢ ContinuousOn f s ↔ ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
rw [continuousOn_iff_continuous_restrict, continuous_def]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
this : ∀ (t : Set β), IsOpen (restrict s f ⁻¹' t) ↔ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
⊢ (∀ (s_1 : Set β), IsOpen s_1 → IsOpen (restrict s f ⁻¹' s_1)) ↔
∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
simp only [this]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ ContinuousOn f s ↔ ∀ (t : Set β), IsClosed t → ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
have : ∀ t, IsClosed (s.restrict f ⁻¹' t) ↔ ∃ u : Set α, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s :=
by
intro t
rw [isClosed_induced_iff, Set.restrict_eq, Set.preimage_comp]
simp only [Subtype.preimage_coe_eq_preimage_coe_iff, eq_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
⊢ ∀ (t : Set β), IsClosed (restrict s f ⁻¹' t) ↔ ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
intro t
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ IsClosed (restrict s f ⁻¹' t) ↔ ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
rw [isClosed_induced_iff, Set.restrict_eq, Set.preimage_comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
⊢ (∃ t_1, IsClosed t_1 ∧ Subtype.val ⁻¹' t_1 = Subtype.val ⁻¹' (f ⁻¹' t)) ↔ ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
simp only [Subtype.preimage_coe_eq_preimage_coe_iff, eq_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
this : ∀ (t : Set β), IsClosed (restrict s f ⁻¹' t) ↔ ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
⊢ ContinuousOn f s ↔ ∀ (t : Set β), IsClosed t → ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
rw [continuousOn_iff_continuous_restrict, continuous_iff_isClosed]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
this : ∀ (t : Set β), IsClosed (restrict s f ⁻¹' t) ↔ ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
⊢ (∀ (s_1 : Set β), IsClosed s_1 → IsClosed (restrict s f ⁻¹' s_1)) ↔
∀ (t : Set β), IsClosed t → ∃ u, IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
simp only [this]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
ι : Sort u_5
f : α → β
s : ι → Set α
hs : ∀ (x : α), ∃ i, s i ∈ 𝓝 x
hf : ∀ (i : ι), ContinuousOn f (s i)
x : α
i : ι
hi : s i ∈ 𝓝 x
⊢ ContinuousAt f x
[PROOFSTEP]
rw [ContinuousAt, ← nhdsWithin_eq_nhds.2 hi]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
ι : Sort u_5
f : α → β
s : ι → Set α
hs : ∀ (x : α), ∃ i, s i ∈ 𝓝 x
hf : ∀ (i : ι), ContinuousOn f (s i)
x : α
i : ι
hi : s i ∈ 𝓝 x
⊢ Tendsto f (𝓝[s i] x) (𝓝 (f x))
[PROOFSTEP]
exact hf _ _ (mem_of_mem_nhds hi)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
a : α
⊢ ContinuousWithinAt f {a} a
[PROOFSTEP]
simpa only [ContinuousWithinAt, nhdsWithin_singleton, tendsto_pure_left] using fun s => mem_of_mem_nhds
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
⊢ Continuous f ↔ ContinuousOn f univ
[PROOFSTEP]
simp [continuous_iff_continuousAt, ContinuousOn, ContinuousAt, ContinuousWithinAt, nhdsWithin_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
x : α
s t : Set α
f : α → β
h : 𝓝[s] x = 𝓝[t] x
⊢ ContinuousWithinAt f s x ↔ ContinuousWithinAt f t x
[PROOFSTEP]
simp only [ContinuousWithinAt, h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s t : Set α
x : α
h : t ∈ 𝓝[s] x
⊢ ContinuousWithinAt f (s ∩ t) x ↔ ContinuousWithinAt f s x
[PROOFSTEP]
simp [ContinuousWithinAt, nhdsWithin_restrict'' s h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s t : Set α
x : α
h : t ∈ 𝓝 x
⊢ ContinuousWithinAt f (s ∩ t) x ↔ ContinuousWithinAt f s x
[PROOFSTEP]
simp [ContinuousWithinAt, nhdsWithin_restrict' s h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s t : Set α
x : α
⊢ ContinuousWithinAt f (s ∪ t) x ↔ ContinuousWithinAt f s x ∧ ContinuousWithinAt f t x
[PROOFSTEP]
simp only [ContinuousWithinAt, nhdsWithin_union, tendsto_sup]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
x : α
⊢ ContinuousWithinAt f {x} x
[PROOFSTEP]
simp only [ContinuousWithinAt, nhdsWithin_singleton, tendsto_pure_nhds]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
x : α
s : Set α
⊢ ContinuousWithinAt f (insert x s) x ↔ ContinuousWithinAt f s x
[PROOFSTEP]
simp only [← singleton_union, continuousWithinAt_union, continuousWithinAt_singleton, true_and_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s t : Set α
x : α
ht : ContinuousWithinAt f t x
h : ContinuousWithinAt f (s \ t) x
⊢ s ⊆ s \ t ∪ t
[PROOFSTEP]
simp only [diff_union_self, subset_union_left]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
a : α
⊢ ContinuousWithinAt f {a}ᶜ a ↔ ContinuousAt f a
[PROOFSTEP]
rw [compl_eq_univ_diff, continuousWithinAt_diff_self, continuousWithinAt_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
inst✝ : DecidableEq α
f : α → β
s : Set α
x : α
y : β
⊢ ContinuousWithinAt (update f x y) s x ↔ Tendsto (update f x y) (𝓝[s \ {x}] x) (𝓝 y)
[PROOFSTEP]
{rw [← continuousWithinAt_diff_self, ContinuousWithinAt, update_same]
}
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
inst✝ : DecidableEq α
f : α → β
s : Set α
x : α
y : β
⊢ ContinuousWithinAt (update f x y) s x ↔ Tendsto (update f x y) (𝓝[s \ {x}] x) (𝓝 y)
[PROOFSTEP]
rw [← continuousWithinAt_diff_self, ContinuousWithinAt, update_same]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
inst✝ : DecidableEq α
f : α → β
x : α
y : β
⊢ ContinuousAt (update f x y) x ↔ Tendsto f (𝓝[{x}ᶜ] x) (𝓝 y)
[PROOFSTEP]
rw [← continuousWithinAt_univ, continuousWithinAt_update_same, compl_eq_univ_diff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : IsOpenMap (Set.restrict s f)
finv : β → α
hleft : LeftInvOn finv f s
⊢ ContinuousOn finv (f '' s)
[PROOFSTEP]
refine' continuousOn_iff'.2 fun t ht => ⟨f '' (t ∩ s), _, _⟩
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : IsOpenMap (Set.restrict s f)
finv : β → α
hleft : LeftInvOn finv f s
t : Set α
ht : IsOpen t
⊢ IsOpen (f '' (t ∩ s))
[PROOFSTEP]
rw [← image_restrict]
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : IsOpenMap (Set.restrict s f)
finv : β → α
hleft : LeftInvOn finv f s
t : Set α
ht : IsOpen t
⊢ IsOpen (Set.restrict s f '' (Subtype.val ⁻¹' t))
[PROOFSTEP]
exact h _ (ht.preimage continuous_subtype_val)
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : IsOpenMap (Set.restrict s f)
finv : β → α
hleft : LeftInvOn finv f s
t : Set α
ht : IsOpen t
⊢ finv ⁻¹' t ∩ f '' s = f '' (t ∩ s) ∩ f '' s
[PROOFSTEP]
rw [inter_eq_self_of_subset_left (image_subset f (inter_subset_right t s)), hleft.image_inter']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : IsOpenMap f
finv : β → α
hleft : LeftInverse finv f
⊢ ContinuousOn finv (range f)
[PROOFSTEP]
rw [← image_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : IsOpenMap f
finv : β → α
hleft : LeftInverse finv f
⊢ ContinuousOn finv (f '' univ)
[PROOFSTEP]
exact (hf.restrict isOpen_univ).continuousOn_image_of_leftInvOn fun x _ => hleft x
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s s₁ : Set α
h : ContinuousOn f s
h' : EqOn g f s₁
h₁ : s₁ ⊆ s
⊢ ContinuousOn g s₁
[PROOFSTEP]
intro x hx
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s s₁ : Set α
h : ContinuousOn f s
h' : EqOn g f s₁
h₁ : s₁ ⊆ s
x : α
hx : x ∈ s₁
⊢ ContinuousWithinAt g s₁ x
[PROOFSTEP]
unfold ContinuousWithinAt
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s s₁ : Set α
h : ContinuousOn f s
h' : EqOn g f s₁
h₁ : s₁ ⊆ s
x : α
hx : x ∈ s₁
⊢ Tendsto g (𝓝[s₁] x) (𝓝 (g x))
[PROOFSTEP]
have A := (h x (h₁ hx)).mono h₁
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s s₁ : Set α
h : ContinuousOn f s
h' : EqOn g f s₁
h₁ : s₁ ⊆ s
x : α
hx : x ∈ s₁
A : ContinuousWithinAt f s₁ x
⊢ Tendsto g (𝓝[s₁] x) (𝓝 (g x))
[PROOFSTEP]
unfold ContinuousWithinAt at A
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s s₁ : Set α
h : ContinuousOn f s
h' : EqOn g f s₁
h₁ : s₁ ⊆ s
x : α
hx : x ∈ s₁
A : Tendsto f (𝓝[s₁] x) (𝓝 (f x))
⊢ Tendsto g (𝓝[s₁] x) (𝓝 (g x))
[PROOFSTEP]
rw [← h' hx] at A
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s s₁ : Set α
h : ContinuousOn f s
h' : EqOn g f s₁
h₁ : s₁ ⊆ s
x : α
hx : x ∈ s₁
A : Tendsto f (𝓝[s₁] x) (𝓝 (g x))
⊢ Tendsto g (𝓝[s₁] x) (𝓝 (g x))
[PROOFSTEP]
exact A.congr' h'.eventuallyEq_nhdsWithin.symm
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
x : α
h : s ∈ 𝓝 x
⊢ ContinuousWithinAt f s x ↔ ContinuousAt f x
[PROOFSTEP]
rw [← univ_inter s, continuousWithinAt_inter h, continuousWithinAt_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : Continuous f
⊢ ContinuousOn f s
[PROOFSTEP]
rw [continuous_iff_continuousOn_univ] at h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ContinuousOn f univ
⊢ ContinuousOn f s
[PROOFSTEP]
exact h.mono (subset_univ _)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
s : Set β
hg : ContinuousOn g s
hf : Continuous f
hs : ∀ (x : α), f x ∈ s
⊢ Continuous (g ∘ f)
[PROOFSTEP]
rw [continuous_iff_continuousOn_univ] at *
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
s : Set β
hg : ContinuousOn g s
hf : ContinuousOn f univ
hs : ∀ (x : α), f x ∈ s
⊢ ContinuousOn (g ∘ f) univ
[PROOFSTEP]
exact hg.comp hf fun x _ => hs x
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
s : Set β
h : LeftInvOn f g s
hx : f (g x) = x
hf : ContinuousWithinAt f (g '' s) (g x)
hg : ContinuousWithinAt g s x
⊢ map g (𝓝[s] x) = 𝓝[g '' s] g x
[PROOFSTEP]
apply le_antisymm
[GOAL]
case a
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
s : Set β
h : LeftInvOn f g s
hx : f (g x) = x
hf : ContinuousWithinAt f (g '' s) (g x)
hg : ContinuousWithinAt g s x
⊢ map g (𝓝[s] x) ≤ 𝓝[g '' s] g x
[PROOFSTEP]
exact hg.tendsto_nhdsWithin (mapsTo_image _ _)
[GOAL]
case a
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
s : Set β
h : LeftInvOn f g s
hx : f (g x) = x
hf : ContinuousWithinAt f (g '' s) (g x)
hg : ContinuousWithinAt g s x
⊢ 𝓝[g '' s] g x ≤ map g (𝓝[s] x)
[PROOFSTEP]
have A : g ∘ f =ᶠ[𝓝[g '' s] g x] id := h.rightInvOn_image.eqOn.eventuallyEq_of_mem self_mem_nhdsWithin
[GOAL]
case a
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
s : Set β
h : LeftInvOn f g s
hx : f (g x) = x
hf : ContinuousWithinAt f (g '' s) (g x)
hg : ContinuousWithinAt g s x
A : g ∘ f =ᶠ[𝓝[g '' s] g x] id
⊢ 𝓝[g '' s] g x ≤ map g (𝓝[s] x)
[PROOFSTEP]
refine' le_map_of_right_inverse A _
[GOAL]
case a
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
s : Set β
h : LeftInvOn f g s
hx : f (g x) = x
hf : ContinuousWithinAt f (g '' s) (g x)
hg : ContinuousWithinAt g s x
A : g ∘ f =ᶠ[𝓝[g '' s] g x] id
⊢ Tendsto f (𝓝[g '' s] g x) (𝓝[s] x)
[PROOFSTEP]
simpa only [hx] using hf.tendsto_nhdsWithin (h.mapsTo (surjOn_image _ _))
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
h : LeftInverse f g
hf : ContinuousWithinAt f (range g) (g x)
hg : ContinuousAt g x
⊢ map g (𝓝 x) = 𝓝[range g] g x
[PROOFSTEP]
simpa only [nhdsWithin_univ, image_univ] using
(h.leftInvOn univ).map_nhdsWithin_eq (h x) (by rwa [image_univ]) hg.continuousWithinAt
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → α
x : β
h : LeftInverse f g
hf : ContinuousWithinAt f (range g) (g x)
hg : ContinuousAt g x
⊢ ContinuousWithinAt f (g '' univ) (g x)
[PROOFSTEP]
rwa [image_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f g : α → β
s : Set α
x : α
h : f =ᶠ[𝓝[s] x] g
hx : f x = g x
⊢ ContinuousWithinAt f s x ↔ ContinuousWithinAt g s x
[PROOFSTEP]
rw [ContinuousWithinAt, hx, tendsto_congr' h, ContinuousWithinAt]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
⊢ ContinuousOn f s ↔ ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)
[PROOFSTEP]
rw [continuousOn_iff']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
⊢ (∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) ↔ ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
⊢ (∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) → ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)
[PROOFSTEP]
intro h t ht
[GOAL]
case mp
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
h : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
t : Set β
ht : IsOpen t
⊢ IsOpen (s ∩ f ⁻¹' t)
[PROOFSTEP]
rcases h t ht with ⟨u, u_open, hu⟩
[GOAL]
case mp.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
h : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
t : Set β
ht : IsOpen t
u : Set α
u_open : IsOpen u
hu : f ⁻¹' t ∩ s = u ∩ s
⊢ IsOpen (s ∩ f ⁻¹' t)
[PROOFSTEP]
rw [inter_comm, hu]
[GOAL]
case mp.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
h : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
t : Set β
ht : IsOpen t
u : Set α
u_open : IsOpen u
hu : f ⁻¹' t ∩ s = u ∩ s
⊢ IsOpen (u ∩ s)
[PROOFSTEP]
apply IsOpen.inter u_open hs
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
⊢ (∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)) → ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
intro h t ht
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
h : ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)
t : Set β
ht : IsOpen t
⊢ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s
[PROOFSTEP]
refine' ⟨s ∩ f ⁻¹' t, h t ht, _⟩
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
hs : IsOpen s
h : ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)
t : Set β
ht : IsOpen t
⊢ f ⁻¹' t ∩ s = s ∩ f ⁻¹' t ∩ s
[PROOFSTEP]
rw [@inter_comm _ s (f ⁻¹' t), inter_assoc, inter_self]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
h : ContinuousOn f s
hs : IsOpen s
hp : f ⁻¹' t ⊆ s
ht : IsOpen t
⊢ IsOpen (f ⁻¹' t)
[PROOFSTEP]
convert (continuousOn_open_iff hs).mp h t ht
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
h : ContinuousOn f s
hs : IsOpen s
hp : f ⁻¹' t ⊆ s
ht : IsOpen t
⊢ f ⁻¹' t = s ∩ f ⁻¹' t
[PROOFSTEP]
rw [inter_comm, inter_eq_self_of_subset_left hp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
hf : ContinuousOn f s
hs : IsClosed s
ht : IsClosed t
⊢ IsClosed (s ∩ f ⁻¹' t)
[PROOFSTEP]
rcases continuousOn_iff_isClosed.1 hf t ht with ⟨u, hu⟩
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
hf : ContinuousOn f s
hs : IsClosed s
ht : IsClosed t
u : Set α
hu : IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
⊢ IsClosed (s ∩ f ⁻¹' t)
[PROOFSTEP]
rw [inter_comm, hu.2]
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
hf : ContinuousOn f s
hs : IsClosed s
ht : IsClosed t
u : Set α
hu : IsClosed u ∧ f ⁻¹' t ∩ s = u ∩ s
⊢ IsClosed (u ∩ s)
[PROOFSTEP]
apply IsClosed.inter hu.1 hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
t : Set β
hf : ContinuousOn f s
hs : IsOpen s
⊢ interior (s ∩ f ⁻¹' t) = s ∩ interior (f ⁻¹' t)
[PROOFSTEP]
rw [interior_inter, hs.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ∀ (x : α), x ∈ s → ∃ t, IsOpen t ∧ x ∈ t ∧ ContinuousOn f (s ∩ t)
⊢ ContinuousOn f s
[PROOFSTEP]
intro x xs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ∀ (x : α), x ∈ s → ∃ t, IsOpen t ∧ x ∈ t ∧ ContinuousOn f (s ∩ t)
x : α
xs : x ∈ s
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
rcases h x xs with ⟨t, open_t, xt, ct⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ∀ (x : α), x ∈ s → ∃ t, IsOpen t ∧ x ∈ t ∧ ContinuousOn f (s ∩ t)
x : α
xs : x ∈ s
t : Set α
open_t : IsOpen t
xt : x ∈ t
ct : ContinuousOn f (s ∩ t)
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
have := ct x ⟨xs, xt⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
h : ∀ (x : α), x ∈ s → ∃ t, IsOpen t ∧ x ∈ t ∧ ContinuousOn f (s ∩ t)
x : α
xs : x ∈ s
t : Set α
open_t : IsOpen t
xt : x ∈ t
ct : ContinuousOn f (s ∩ t)
this : ContinuousWithinAt f (s ∩ t) x
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
rwa [ContinuousWithinAt, ← nhdsWithin_restrict _ xt open_t] at this
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set α
T : Set (Set β)
f : α → β
x : α
x✝ : x ∈ s
⊢ ContinuousWithinAt f s x ↔ ∀ (t : Set β), t ∈ T → f x ∈ t → f ⁻¹' t ∈ 𝓝[s] x
[PROOFSTEP]
delta ContinuousWithinAt
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set α
T : Set (Set β)
f : α → β
x : α
x✝ : x ∈ s
⊢ Tendsto f (𝓝[s] x) (𝓝 (f x)) ↔ ∀ (t : Set β), t ∈ T → f x ∈ t → f ⁻¹' t ∈ 𝓝[s] x
[PROOFSTEP]
simp only [TopologicalSpace.nhds_generateFrom, tendsto_iInf, tendsto_principal, mem_setOf_eq, and_imp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set α
T : Set (Set β)
f : α → β
x : α
x✝ : x ∈ s
⊢ (∀ (i : Set β), f x ∈ i → i ∈ T → ∀ᶠ (a : α) in 𝓝[s] x, f a ∈ i) ↔ ∀ (t : Set β), t ∈ T → f x ∈ t → f ⁻¹' t ∈ 𝓝[s] x
[PROOFSTEP]
exact forall_congr' fun t => forall_swap
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
s : Set α
x : α
⊢ ContinuousWithinAt f s x ↔ ContinuousWithinAt (g ∘ f) s x
[PROOFSTEP]
simp_rw [ContinuousWithinAt, Inducing.tendsto_nhds_iff hg]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
s : Set α
x : α
⊢ Tendsto (g ∘ f) (𝓝[s] x) (𝓝 (g (f x))) ↔ Tendsto (g ∘ f) (𝓝[s] x) (𝓝 ((g ∘ f) x))
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
s : Set α
⊢ ContinuousOn f s ↔ ContinuousOn (g ∘ f) s
[PROOFSTEP]
simp_rw [ContinuousOn, hg.continuousWithinAt_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : _root_.Embedding f
s : Set α
x : α
⊢ map f (𝓝[s] x) = 𝓝[f '' s] f x
[PROOFSTEP]
rw [nhdsWithin, Filter.map_inf hf.inj, hf.map_nhds_eq, map_principal, ← nhdsWithin_inter',
inter_eq_self_of_subset_right (image_subset_range _ _)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : OpenEmbedding f
s : Set β
x : α
⊢ map f (𝓝[f ⁻¹' s] x) = 𝓝[s] f x
[PROOFSTEP]
rw [hf.toEmbedding.map_nhdsWithin_eq, image_preimage_eq_inter_range]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : OpenEmbedding f
s : Set β
x : α
⊢ 𝓝[s ∩ range f] f x = 𝓝[s] f x
[PROOFSTEP]
apply nhdsWithin_eq_nhdsWithin (mem_range_self _) hf.open_range
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : OpenEmbedding f
s : Set β
x : α
⊢ s ∩ range f ∩ range f = s ∩ range f
[PROOFSTEP]
rw [inter_assoc, inter_self]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
x : α
⊢ ¬x ∈ closure s → ContinuousWithinAt f s x
[PROOFSTEP]
intro hx
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
x : α
hx : ¬x ∈ closure s
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
rw [mem_closure_iff_nhdsWithin_neBot, neBot_iff, not_not] at hx
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
x : α
hx : 𝓝[s] x = ⊥
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
rw [ContinuousWithinAt, hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
s : Set α
x : α
hx : 𝓝[s] x = ⊥
⊢ Tendsto f ⊥ (𝓝 (f x))
[PROOFSTEP]
exact tendsto_bot
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
⊢ ContinuousOn (fun a => if p a then f a else g a) s
[PROOFSTEP]
intro x hx
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx : x ∈ s
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) s x
[PROOFSTEP]
by_cases hx' : x ∈ frontier {a | p a}
[GOAL]
case pos
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx : x ∈ s
hx' : x ∈ frontier {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) s x
[PROOFSTEP]
exact (hpf x ⟨hx, hx'⟩).piecewise_nhdsWithin (hpg x ⟨hx, hx'⟩)
[GOAL]
case neg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx : x ∈ s
hx' : ¬x ∈ frontier {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) s x
[PROOFSTEP]
rw [← inter_univ s, ← union_compl_self {a | p a}, inter_union_distrib_left] at hx ⊢
[GOAL]
case neg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx : x ∈ s ∩ {a | p a} ∪ s ∩ {a | p a}ᶜ
hx' : ¬x ∈ frontier {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a} ∪ s ∩ {a | p a}ᶜ) x
[PROOFSTEP]
cases' hx with hx hx
[GOAL]
case neg.inl
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a} ∪ s ∩ {a | p a}ᶜ) x
[PROOFSTEP]
apply ContinuousWithinAt.union
[GOAL]
case neg.inl.hs
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a}) x
[PROOFSTEP]
exact (hf x hx).congr (fun y hy => if_pos hy.2) (if_pos hx.2)
[GOAL]
case neg.inl.ht
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a}ᶜ) x
[PROOFSTEP]
have : x ∉ closure {a | p a}ᶜ := fun h => hx' ⟨subset_closure hx.2, by rwa [closure_compl] at h ⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}
h : x ∈ closure {a | p a}ᶜ
⊢ ¬x ∈ interior {a | p a}
[PROOFSTEP]
rwa [closure_compl] at h
[GOAL]
case neg.inl.ht
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}
this : ¬x ∈ closure {a | p a}ᶜ
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a}ᶜ) x
[PROOFSTEP]
exact continuousWithinAt_of_not_mem_closure fun h => this (closure_inter_subset_inter_closure _ _ h).2
[GOAL]
case neg.inr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}ᶜ
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a} ∪ s ∩ {a | p a}ᶜ) x
[PROOFSTEP]
apply ContinuousWithinAt.union
[GOAL]
case neg.inr.hs
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}ᶜ
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a}) x
[PROOFSTEP]
have : x ∉ closure {a | p a} := fun h => hx' ⟨h, fun h' : x ∈ interior {a | p a} => hx.2 (interior_subset h')⟩
[GOAL]
case neg.inr.hs
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}ᶜ
this : ¬x ∈ closure {a | p a}
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a}) x
[PROOFSTEP]
exact continuousWithinAt_of_not_mem_closure fun h => this (closure_inter_subset_inter_closure _ _ h).2
[GOAL]
case neg.inr.ht
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Set α
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto f (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto g (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f (s ∩ {a | p a})
hg : ContinuousOn g (s ∩ {a | ¬p a})
x : α
hx' : ¬x ∈ frontier {a | p a}
hx : x ∈ s ∩ {a | p a}ᶜ
⊢ ContinuousWithinAt (fun a => if p a then f a else g a) (s ∩ {a | p a}ᶜ) x
[PROOFSTEP]
exact (hg x hx).congr (fun y hy => if_neg hy.2) (if_neg hx.2)
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
⊢ ContinuousOn (fun a => if p a then f a else g a) s
[PROOFSTEP]
apply ContinuousOn.if'
[GOAL]
case hpf
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
⊢ ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto (fun a => f a) (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
rintro a ha
[GOAL]
case hpf
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
ha : a ∈ s ∩ frontier {a | p a}
⊢ Tendsto (fun a => f a) (𝓝[s ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
simp only [← hp a ha, ite_self]
[GOAL]
case hpf
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
ha : a ∈ s ∩ frontier {a | p a}
⊢ Tendsto (fun a => f a) (𝓝[s ∩ {a | p a}] a) (𝓝 (f a))
[PROOFSTEP]
apply tendsto_nhdsWithin_mono_left (inter_subset_inter_right s subset_closure)
[GOAL]
case hpf
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
ha : a ∈ s ∩ frontier {a | p a}
⊢ Tendsto (fun a => f a) (𝓝[s ∩ closure {a | p a}] a) (𝓝 (f a))
[PROOFSTEP]
exact hf a ⟨ha.1, ha.2.1⟩
[GOAL]
case hpg
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
⊢ ∀ (a : α), a ∈ s ∩ frontier {a | p a} → Tendsto (fun a => g a) (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
rintro a ha
[GOAL]
case hpg
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
ha : a ∈ s ∩ frontier {a | p a}
⊢ Tendsto (fun a => g a) (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
simp only [hp a ha, ite_self]
[GOAL]
case hpg
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
ha : a ∈ s ∩ frontier {a | p a}
⊢ Tendsto (fun a => g a) (𝓝[s ∩ {a | ¬p a}] a) (𝓝 (g a))
[PROOFSTEP]
apply tendsto_nhdsWithin_mono_left (inter_subset_inter_right s subset_closure)
[GOAL]
case hpg
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
ha : a ∈ s ∩ frontier {a | p a}
⊢ Tendsto (fun a => g a) (𝓝[s ∩ closure {a | ¬p a}] a) (𝓝 (g a))
[PROOFSTEP]
rcases ha with ⟨has, ⟨_, ha⟩⟩
[GOAL]
case hpg.intro.intro
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
has : a ∈ s
left✝ : a ∈ closure {a | p a}
ha : ¬a ∈ interior {a | p a}
⊢ Tendsto (fun a => g a) (𝓝[s ∩ closure {a | ¬p a}] a) (𝓝 (g a))
[PROOFSTEP]
rw [← mem_compl_iff, ← closure_compl] at ha
[GOAL]
case hpg.intro.intro
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
a : α
has : a ∈ s
left✝ : a ∈ closure {a | p a}
ha : a ∈ closure {a | p a}ᶜ
⊢ Tendsto (fun a => g a) (𝓝[s ∩ closure {a | ¬p a}] a) (𝓝 (g a))
[PROOFSTEP]
apply hg a ⟨has, ha⟩
[GOAL]
case hf
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
⊢ ContinuousOn (fun a => f a) (s ∩ {a | p a})
[PROOFSTEP]
exact hf.mono (inter_subset_inter_right s subset_closure)
[GOAL]
case hg
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α✝
inst✝⁵ : TopologicalSpace β✝
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
α : Type u_5
β : Type u_6
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
p : α → Prop
inst✝ : (a : α) → Decidable (p a)
s : Set α
f g : α → β
hp : ∀ (a : α), a ∈ s ∩ frontier {a | p a} → f a = g a
hf : ContinuousOn f (s ∩ closure {a | p a})
hg : ContinuousOn g (s ∩ closure {a | ¬p a})
⊢ ContinuousOn (fun a => g a) (s ∩ {a | ¬p a})
[PROOFSTEP]
exact hg.mono (inter_subset_inter_right s subset_closure)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ Continuous fun a => if p a then f a else g a
[PROOFSTEP]
rw [continuous_iff_continuousOn_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ContinuousOn (fun a => if p a then f a else g a) univ
[PROOFSTEP]
apply ContinuousOn.if'
[GOAL]
case hpf
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ∀ (a : α),
a ∈ univ ∩ frontier {a | p a} → Tendsto (fun a => f a) (𝓝[univ ∩ {a | p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
simp [*]
[GOAL]
case hpg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ∀ (a : α),
a ∈ univ ∩ frontier {a | p a} → Tendsto (fun a => g a) (𝓝[univ ∩ {a | ¬p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
simp [*]
[GOAL]
case hf
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ContinuousOn (fun a => f a) (univ ∩ {a | p a})
[PROOFSTEP]
simp [*]
[GOAL]
case hg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ContinuousOn (fun a => g a) (univ ∩ {a | ¬p a})
[PROOFSTEP]
simp [*]
[GOAL]
case hpf
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ∀ (a : α), a ∈ frontier {a | p a} → Tendsto (fun a => f a) (𝓝[{a | p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
assumption
[GOAL]
case hpg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hpf : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto f (𝓝[{x | p x}] a) (𝓝 (if p a then f a else g a))
hpg : ∀ (a : α), a ∈ frontier {x | p x} → Tendsto g (𝓝[{x | ¬p x}] a) (𝓝 (if p a then f a else g a))
hf : ContinuousOn f {x | p x}
hg : ContinuousOn g {x | ¬p x}
⊢ ∀ (a : α), a ∈ frontier {a | p a} → Tendsto (fun a => g a) (𝓝[{a | ¬p a}] a) (𝓝 (if p a then f a else g a))
[PROOFSTEP]
assumption
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ Continuous fun a => if p a then f a else g a
[PROOFSTEP]
rw [continuous_iff_continuousOn_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ContinuousOn (fun a => if p a then f a else g a) univ
[PROOFSTEP]
apply ContinuousOn.if
[GOAL]
case hp
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ∀ (a : α), a ∈ univ ∩ frontier {a | p a} → f a = g a
[PROOFSTEP]
simp
[GOAL]
case hf
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ContinuousOn (fun a => f a) (univ ∩ closure {a | p a})
[PROOFSTEP]
simp
[GOAL]
case hg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ContinuousOn (fun a => g a) (univ ∩ closure {a | ¬p a})
[PROOFSTEP]
simp
[GOAL]
case hp
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ∀ (a : α), a ∈ frontier {a | p a} → f a = g a
[PROOFSTEP]
assumption
[GOAL]
case hf
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ContinuousOn (fun a => f a) (closure {a | p a})
[PROOFSTEP]
assumption
[GOAL]
case hg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : α → Prop
f g : α → β
inst✝ : (a : α) → Decidable (p a)
hp : ∀ (a : α), a ∈ frontier {x | p x} → f a = g a
hf : ContinuousOn f (closure {x | p x})
hg : ContinuousOn g (closure {x | ¬p x})
⊢ ContinuousOn (fun a => g a) (closure {a | ¬p a})
[PROOFSTEP]
assumption
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : Prop
f g : α → β
inst✝ : Decidable p
hf : p → Continuous f
hg : ¬p → Continuous g
⊢ Continuous fun a => if p then f a else g a
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : Prop
f g : α → β
inst✝ : Decidable p
hf : p → Continuous f
hg : ¬p → Continuous g
h : p
⊢ Continuous fun a => f a
case neg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
p : Prop
f g : α → β
inst✝ : Decidable p
hf : p → Continuous f
hg : ¬p → Continuous g
h : ¬p
⊢ Continuous fun a => g a
[PROOFSTEP]
exacts [hf h, hg h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
hs : IsOpen s
hs' : IsOpen s'
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
⊢ IsOpen (Set.ite t s s')
[PROOFSTEP]
classical
simp only [isOpen_iff_continuous_mem, Set.ite] at *
convert continuous_piecewise (fun x hx => propext (ht x hx)) hs.continuousOn hs'.continuousOn
rename_i x
by_cases hx : x ∈ t <;> simp [hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
hs : IsOpen s
hs' : IsOpen s'
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
⊢ IsOpen (Set.ite t s s')
[PROOFSTEP]
simp only [isOpen_iff_continuous_mem, Set.ite] at *
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
hs : Continuous fun x => x ∈ s
hs' : Continuous fun x => x ∈ s'
⊢ Continuous fun x => x ∈ s ∩ t ∪ s' \ t
[PROOFSTEP]
convert continuous_piecewise (fun x hx => propext (ht x hx)) hs.continuousOn hs'.continuousOn
[GOAL]
case h.e'_5.h.a
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
hs : Continuous fun x => x ∈ s
hs' : Continuous fun x => x ∈ s'
x✝ : α
⊢ x✝ ∈ s ∩ t ∪ s' \ t ↔ piecewise t (fun x => x ∈ s) (fun x => x ∈ s') x✝
[PROOFSTEP]
rename_i x
[GOAL]
case h.e'_5.h.a
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
hs : Continuous fun x => x ∈ s
hs' : Continuous fun x => x ∈ s'
x : α
⊢ x ∈ s ∩ t ∪ s' \ t ↔ piecewise t (fun x => x ∈ s) (fun x => x ∈ s') x
[PROOFSTEP]
by_cases hx : x ∈ t
[GOAL]
case pos
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
hs : Continuous fun x => x ∈ s
hs' : Continuous fun x => x ∈ s'
x : α
hx : x ∈ t
⊢ x ∈ s ∩ t ∪ s' \ t ↔ piecewise t (fun x => x ∈ s) (fun x => x ∈ s') x
[PROOFSTEP]
simp [hx]
[GOAL]
case neg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : ∀ (x : α), x ∈ frontier t → (x ∈ s ↔ x ∈ s')
hs : Continuous fun x => x ∈ s
hs' : Continuous fun x => x ∈ s'
x : α
hx : ¬x ∈ t
⊢ x ∈ s ∩ t ∪ s' \ t ↔ piecewise t (fun x => x ∈ s) (fun x => x ∈ s') x
[PROOFSTEP]
simp [hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
hs : IsOpen s
hs' : IsOpen s'
ht : s ∩ frontier t = s' ∩ frontier t
x : α
hx : x ∈ frontier t
⊢ x ∈ s ↔ x ∈ s'
[PROOFSTEP]
simpa [hx] using ext_iff.1 ht x
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : s ∩ frontier t = s' ∩ frontier t
⊢ Set.ite t s s' ∩ closure t = s ∩ closure t
[PROOFSTEP]
rw [closure_eq_self_union_frontier, inter_union_distrib_left, inter_union_distrib_left, ite_inter_self,
ite_inter_of_inter_eq _ ht]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : s ∩ frontier t = s' ∩ frontier t
⊢ Set.ite t s s' ∩ closure tᶜ = s' ∩ closure tᶜ
[PROOFSTEP]
rw [← ite_compl, ite_inter_closure_eq_of_inter_frontier_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s s' t : Set α
ht : s ∩ frontier t = s' ∩ frontier t
⊢ s' ∩ frontier tᶜ = s ∩ frontier tᶜ
[PROOFSTEP]
rwa [frontier_compl, eq_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s s' t : Set α
f f' : α → β
inst✝ : (x : α) → Decidable (x ∈ t)
h : ContinuousOn f (s ∩ closure t)
h' : ContinuousOn f' (s' ∩ closure tᶜ)
H : s ∩ frontier t = s' ∩ frontier t
Heq : EqOn f f' (s ∩ frontier t)
⊢ ContinuousOn (piecewise t f f') (Set.ite t s s')
[PROOFSTEP]
apply ContinuousOn.piecewise
[GOAL]
case ht
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s s' t : Set α
f f' : α → β
inst✝ : (x : α) → Decidable (x ∈ t)
h : ContinuousOn f (s ∩ closure t)
h' : ContinuousOn f' (s' ∩ closure tᶜ)
H : s ∩ frontier t = s' ∩ frontier t
Heq : EqOn f f' (s ∩ frontier t)
⊢ ∀ (a : α), a ∈ Set.ite t s s' ∩ frontier t → f a = f' a
[PROOFSTEP]
rwa [ite_inter_of_inter_eq _ H]
[GOAL]
case hf
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s s' t : Set α
f f' : α → β
inst✝ : (x : α) → Decidable (x ∈ t)
h : ContinuousOn f (s ∩ closure t)
h' : ContinuousOn f' (s' ∩ closure tᶜ)
H : s ∩ frontier t = s' ∩ frontier t
Heq : EqOn f f' (s ∩ frontier t)
⊢ ContinuousOn f (Set.ite t s s' ∩ closure t)
[PROOFSTEP]
rwa [ite_inter_closure_eq_of_inter_frontier_eq H]
[GOAL]
case hg
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s s' t : Set α
f f' : α → β
inst✝ : (x : α) → Decidable (x ∈ t)
h : ContinuousOn f (s ∩ closure t)
h' : ContinuousOn f' (s' ∩ closure tᶜ)
H : s ∩ frontier t = s' ∩ frontier t
Heq : EqOn f f' (s ∩ frontier t)
⊢ ContinuousOn f' (Set.ite t s s' ∩ closure tᶜ)
[PROOFSTEP]
rwa [ite_inter_closure_compl_eq_of_inter_frontier_eq H]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s t : Set α
ht : IsOpen t
⊢ frontier (s ∩ t) ∩ t = frontier s ∩ t
[PROOFSTEP]
simp only [← Subtype.preimage_coe_eq_preimage_coe_iff,
ht.isOpenMap_subtype_val.preimage_frontier_eq_frontier_preimage continuous_subtype_val,
Subtype.preimage_coe_inter_self]
| {"mathlib_filename": "Mathlib.Topology.ContinuousOn", "llama_tokens": 45071} |
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
s : Set α
a : α
di : DenseInducing i
hs : s ∈ 𝓝 a
⊢ closure (i '' s) ∈ 𝓝 (i a)
[PROOFSTEP]
rw [di.nhds_eq_comap a, ((nhds_basis_opens _).comap _).mem_iff] at hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
s : Set α
a : α
di : DenseInducing i
hs : ∃ i_1, (i a ∈ i_1 ∧ IsOpen i_1) ∧ i ⁻¹' i_1 ⊆ s
⊢ closure (i '' s) ∈ 𝓝 (i a)
[PROOFSTEP]
rcases hs with ⟨U, ⟨haU, hUo⟩, sub : i ⁻¹' U ⊆ s⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
s : Set α
a : α
di : DenseInducing i
U : Set β
sub : i ⁻¹' U ⊆ s
haU : i a ∈ U
hUo : IsOpen U
⊢ closure (i '' s) ∈ 𝓝 (i a)
[PROOFSTEP]
refine' mem_of_superset (hUo.mem_nhds haU) _
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
s : Set α
a : α
di : DenseInducing i
U : Set β
sub : i ⁻¹' U ⊆ s
haU : i a ∈ U
hUo : IsOpen U
⊢ U ⊆ closure (i '' s)
[PROOFSTEP]
calc
U ⊆ closure (i '' (i ⁻¹' U)) := di.dense.subset_closure_image_preimage_of_isOpen hUo
_ ⊆ closure (i '' s) := closure_mono (image_subset i sub)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ di : DenseInducing i
s : Set α
⊢ Dense (i '' s) ↔ Dense s
[PROOFSTEP]
refine' ⟨fun H x => _, di.dense.dense_image di.continuous⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ di : DenseInducing i
s : Set α
H : Dense (i '' s)
x : α
⊢ x ∈ closure s
[PROOFSTEP]
rw [di.toInducing.closure_eq_preimage_closure_image, H.closure_eq, preimage_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
i : α → β
di✝ di : DenseInducing i
s : Set α
H : Dense (i '' s)
x : α
⊢ x ∈ univ
[PROOFSTEP]
trivial
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : T2Space β
di : DenseInducing i
hd : Dense (range i)ᶜ
s : Set α
hs : IsCompact s
⊢ interior s = ∅
[PROOFSTEP]
refine' eq_empty_iff_forall_not_mem.2 fun x hx => _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : T2Space β
di : DenseInducing i
hd : Dense (range i)ᶜ
s : Set α
hs : IsCompact s
x : α
hx : x ∈ interior s
⊢ False
[PROOFSTEP]
rw [mem_interior_iff_mem_nhds] at hx
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : T2Space β
di : DenseInducing i
hd : Dense (range i)ᶜ
s : Set α
hs : IsCompact s
x : α
hx : s ∈ 𝓝 x
⊢ False
[PROOFSTEP]
have := di.closure_image_mem_nhds hx
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : T2Space β
di : DenseInducing i
hd : Dense (range i)ᶜ
s : Set α
hs : IsCompact s
x : α
hx : s ∈ 𝓝 x
this : closure (i '' s) ∈ 𝓝 (i x)
⊢ False
[PROOFSTEP]
rw [(hs.image di.continuous).isClosed.closure_eq] at this
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : T2Space β
di : DenseInducing i
hd : Dense (range i)ᶜ
s : Set α
hs : IsCompact s
x : α
hx : s ∈ 𝓝 x
this : i '' s ∈ 𝓝 (i x)
⊢ False
[PROOFSTEP]
rcases hd.inter_nhds_nonempty this with ⟨y, hyi, hys⟩
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : T2Space β
di : DenseInducing i
hd : Dense (range i)ᶜ
s : Set α
hs : IsCompact s
x : α
hx : s ∈ 𝓝 x
this : i '' s ∈ 𝓝 (i x)
y : β
hyi : y ∈ (range i)ᶜ
hys : y ∈ i '' s
⊢ False
[PROOFSTEP]
exact hyi (image_subset_range _ _ hys)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
d : δ
a : α
di : DenseInducing i
H : Tendsto h (𝓝 d) (𝓝 (i a))
comm : h ∘ g = i ∘ f
⊢ Tendsto f (comap g (𝓝 d)) (𝓝 a)
[PROOFSTEP]
have lim1 : map g (comap g (𝓝 d)) ≤ 𝓝 d := map_comap_le
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
d : δ
a : α
di : DenseInducing i
H : Tendsto h (𝓝 d) (𝓝 (i a))
comm : h ∘ g = i ∘ f
lim1 : map g (comap g (𝓝 d)) ≤ 𝓝 d
⊢ Tendsto f (comap g (𝓝 d)) (𝓝 a)
[PROOFSTEP]
replace lim1 : map h (map g (comap g (𝓝 d))) ≤ map h (𝓝 d) := map_mono lim1
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
d : δ
a : α
di : DenseInducing i
H : Tendsto h (𝓝 d) (𝓝 (i a))
comm : h ∘ g = i ∘ f
lim1 : map h (map g (comap g (𝓝 d))) ≤ map h (𝓝 d)
⊢ Tendsto f (comap g (𝓝 d)) (𝓝 a)
[PROOFSTEP]
rw [Filter.map_map, comm, ← Filter.map_map, map_le_iff_le_comap] at lim1
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
d : δ
a : α
di : DenseInducing i
H : Tendsto h (𝓝 d) (𝓝 (i a))
comm : h ∘ g = i ∘ f
lim1 : map f (comap g (𝓝 d)) ≤ comap i (map h (𝓝 d))
⊢ Tendsto f (comap g (𝓝 d)) (𝓝 a)
[PROOFSTEP]
have lim2 : comap i (map h (𝓝 d)) ≤ comap i (𝓝 (i a)) := comap_mono H
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
d : δ
a : α
di : DenseInducing i
H : Tendsto h (𝓝 d) (𝓝 (i a))
comm : h ∘ g = i ∘ f
lim1 : map f (comap g (𝓝 d)) ≤ comap i (map h (𝓝 d))
lim2 : comap i (map h (𝓝 d)) ≤ comap i (𝓝 (i a))
⊢ Tendsto f (comap g (𝓝 d)) (𝓝 a)
[PROOFSTEP]
rw [← di.nhds_eq_comap] at lim2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
d : δ
a : α
di : DenseInducing i
H : Tendsto h (𝓝 d) (𝓝 (i a))
comm : h ∘ g = i ∘ f
lim1 : map f (comap g (𝓝 d)) ≤ comap i (map h (𝓝 d))
lim2 : comap i (map h (𝓝 d)) ≤ 𝓝 a
⊢ Tendsto f (comap g (𝓝 d)) (𝓝 a)
[PROOFSTEP]
exact le_trans lim1 lim2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
di : DenseInducing i
b : β
s : Set β
hs : s ∈ 𝓝 b
⊢ ∃ a, i a ∈ s
[PROOFSTEP]
rcases mem_closure_iff_nhds.1 (di.dense b) s hs with ⟨_, ⟨ha, a, rfl⟩⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
di : DenseInducing i
b : β
s : Set β
hs : s ∈ 𝓝 b
a : α
ha : i a ∈ s
⊢ ∃ a, i a ∈ s
[PROOFSTEP]
exact ⟨a, ha⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
f : α → γ
di : DenseInducing i
hf : ∀ (b : β), ∃ c, Tendsto f (comap i (𝓝 b)) (𝓝 c)
a : α
⊢ extend di f (i a) = f a
[PROOFSTEP]
rcases hf (i a) with ⟨b, hb⟩
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
f : α → γ
di : DenseInducing i
hf : ∀ (b : β), ∃ c, Tendsto f (comap i (𝓝 b)) (𝓝 c)
a : α
b : γ
hb : Tendsto f (comap i (𝓝 (i a))) (𝓝 b)
⊢ extend di f (i a) = f a
[PROOFSTEP]
refine' di.extend_eq_at' b _
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
f : α → γ
di : DenseInducing i
hf : ∀ (b : β), ∃ c, Tendsto f (comap i (𝓝 b)) (𝓝 c)
a : α
b : γ
hb : Tendsto f (comap i (𝓝 (i a))) (𝓝 b)
⊢ Tendsto f (𝓝 a) (𝓝 b)
[PROOFSTEP]
rwa [← di.toInducing.nhds_eq_comap] at hb
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
f : α → γ
g : β → γ
di : DenseInducing i
hf : ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) = f x
hg : ContinuousAt g b
⊢ extend di f b = g b
[PROOFSTEP]
refine' di.extend_eq_of_tendsto fun s hs => mem_map.2 _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
f : α → γ
g : β → γ
di : DenseInducing i
hf : ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) = f x
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
⊢ f ⁻¹' s ∈ comap i (𝓝 b)
[PROOFSTEP]
suffices : ∀ᶠ x : α in comap i (𝓝 b), g (i x) ∈ s
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
f : α → γ
g : β → γ
di : DenseInducing i
hf : ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) = f x
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
this : ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) ∈ s
⊢ f ⁻¹' s ∈ comap i (𝓝 b)
case this
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
f : α → γ
g : β → γ
di : DenseInducing i
hf : ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) = f x
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
⊢ ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) ∈ s
[PROOFSTEP]
exact hf.mp (this.mono fun x hgx hfx => hfx ▸ hgx)
[GOAL]
case this
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
f : α → γ
g : β → γ
di : DenseInducing i
hf : ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) = f x
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
⊢ ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) ∈ s
[PROOFSTEP]
clear hf f
[GOAL]
case this
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
g : β → γ
di : DenseInducing i
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
⊢ ∀ᶠ (x : α) in comap i (𝓝 b), g (i x) ∈ s
[PROOFSTEP]
refine' eventually_comap.2 ((hg.eventually hs).mono _)
[GOAL]
case this
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
g : β → γ
di : DenseInducing i
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
⊢ ∀ (x : β), s (g x) → ∀ (a : α), i a = x → g (i a) ∈ s
[PROOFSTEP]
rintro _ hxs x rfl
[GOAL]
case this
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f : γ → α
g✝ : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
b : β
g : β → γ
di : DenseInducing i
hg : ContinuousAt g b
s : Set γ
hs : s ∈ 𝓝 (g b)
x : α
hxs : s (g (i x))
⊢ g (i x) ∈ s
[PROOFSTEP]
exact hxs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
⊢ ContinuousAt (extend di f) b
[PROOFSTEP]
set φ := di.extend f
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
⊢ ContinuousAt φ b
[PROOFSTEP]
haveI := di.comap_nhds_neBot
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
⊢ ContinuousAt φ b
[PROOFSTEP]
suffices ∀ V' ∈ 𝓝 (φ b), IsClosed V' → φ ⁻¹' V' ∈ 𝓝 b by
simpa [ContinuousAt, (closed_nhds_basis (φ b)).tendsto_right_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this✝ : ∀ (b : β), NeBot (comap i (𝓝 b))
this : ∀ (V' : Set γ), V' ∈ 𝓝 (φ b) → IsClosed V' → φ ⁻¹' V' ∈ 𝓝 b
⊢ ContinuousAt φ b
[PROOFSTEP]
simpa [ContinuousAt, (closed_nhds_basis (φ b)).tendsto_right_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
⊢ ∀ (V' : Set γ), V' ∈ 𝓝 (φ b) → IsClosed V' → φ ⁻¹' V' ∈ 𝓝 b
[PROOFSTEP]
intro V' V'_in V'_closed
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
⊢ φ ⁻¹' V' ∈ 𝓝 b
[PROOFSTEP]
set V₁ := {x | Tendsto f (comap i <| 𝓝 x) (𝓝 <| φ x)}
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
⊢ φ ⁻¹' V' ∈ 𝓝 b
[PROOFSTEP]
have V₁_in : V₁ ∈ 𝓝 b := by
filter_upwards [hf]
rintro x ⟨c, hc⟩
rwa [di.extend_eq_of_tendsto hc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
⊢ V₁ ∈ 𝓝 b
[PROOFSTEP]
filter_upwards [hf]
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
⊢ ∀ (a : β), (∃ c, Tendsto f (comap i (𝓝 a)) (𝓝 c)) → Tendsto f (comap i (𝓝 a)) (𝓝 (extend di f a))
[PROOFSTEP]
rintro x ⟨c, hc⟩
[GOAL]
case h.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
x : β
c : γ
hc : Tendsto f (comap i (𝓝 x)) (𝓝 c)
⊢ Tendsto f (comap i (𝓝 x)) (𝓝 (extend di f x))
[PROOFSTEP]
rwa [di.extend_eq_of_tendsto hc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
⊢ φ ⁻¹' V' ∈ 𝓝 b
[PROOFSTEP]
obtain ⟨V₂, V₂_in, V₂_op, hV₂⟩ : ∃ V₂ ∈ 𝓝 b, IsOpen V₂ ∧ ∀ x ∈ i ⁻¹' V₂, f x ∈ V' := by
simpa [and_assoc] using ((nhds_basis_opens' b).comap i).tendsto_left_iff.mp (mem_of_mem_nhds V₁_in : b ∈ V₁) V' V'_in
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
⊢ ∃ V₂, V₂ ∈ 𝓝 b ∧ IsOpen V₂ ∧ ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
[PROOFSTEP]
simpa [and_assoc] using ((nhds_basis_opens' b).comap i).tendsto_left_iff.mp (mem_of_mem_nhds V₁_in : b ∈ V₁) V' V'_in
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
⊢ φ ⁻¹' V' ∈ 𝓝 b
[PROOFSTEP]
suffices ∀ x ∈ V₁ ∩ V₂, φ x ∈ V' by filter_upwards [inter_mem V₁_in V₂_in] using this
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this✝ : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
this : ∀ (x : β), x ∈ V₁ ∩ V₂ → φ x ∈ V'
⊢ φ ⁻¹' V' ∈ 𝓝 b
[PROOFSTEP]
filter_upwards [inter_mem V₁_in V₂_in] using this
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
⊢ ∀ (x : β), x ∈ V₁ ∩ V₂ → φ x ∈ V'
[PROOFSTEP]
rintro x ⟨x_in₁, x_in₂⟩
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
x : β
x_in₁ : x ∈ V₁
x_in₂ : x ∈ V₂
⊢ φ x ∈ V'
[PROOFSTEP]
have hV₂x : V₂ ∈ 𝓝 x := IsOpen.mem_nhds V₂_op x_in₂
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
x : β
x_in₁ : x ∈ V₁
x_in₂ : x ∈ V₂
hV₂x : V₂ ∈ 𝓝 x
⊢ φ x ∈ V'
[PROOFSTEP]
apply V'_closed.mem_of_tendsto x_in₁
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
x : β
x_in₁ : x ∈ V₁
x_in₂ : x ∈ V₂
hV₂x : V₂ ∈ 𝓝 x
⊢ ∀ᶠ (x : α) in comap i (𝓝 x), f x ∈ V'
[PROOFSTEP]
use V₂
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
i : α → β
di✝ : DenseInducing i
inst✝² : TopologicalSpace δ
f✝ : γ → α
g : γ → δ
h : δ → β
inst✝¹ : TopologicalSpace γ
inst✝ : T3Space γ
b : β
f : α → γ
di : DenseInducing i
hf : ∀ᶠ (x : β) in 𝓝 b, ∃ c, Tendsto f (comap i (𝓝 x)) (𝓝 c)
φ : β → γ := extend di f
this : ∀ (b : β), NeBot (comap i (𝓝 b))
V' : Set γ
V'_in : V' ∈ 𝓝 (φ b)
V'_closed : IsClosed V'
V₁ : Set β := {x | Tendsto f (comap i (𝓝 x)) (𝓝 (φ x))}
V₁_in : V₁ ∈ 𝓝 b
V₂ : Set β
V₂_in : V₂ ∈ 𝓝 b
V₂_op : IsOpen V₂
hV₂ : ∀ (x : α), x ∈ i ⁻¹' V₂ → f x ∈ V'
x : β
x_in₁ : x ∈ V₁
x_in₂ : x ∈ V₂
hV₂x : V₂ ∈ 𝓝 x
⊢ V₂ ∈ 𝓝 x ∧ i ⁻¹' V₂ ⊆ {x | (fun x => f x ∈ V') x}
[PROOFSTEP]
tauto
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
i✝ : α → β
di : DenseInducing i✝
inst✝¹ : TopologicalSpace δ
f : γ → α
g : γ → δ
h : δ → β
inst✝ : TopologicalSpace γ
i : α → β
c : Continuous i
dense : ∀ (x : β), x ∈ closure (range i)
H : ∀ (a : α) (s : Set α), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 (i a) ∧ ∀ (b : α), i b ∈ t → b ∈ s
a : α
⊢ comap i (𝓝 (i a)) ≤ 𝓝 a
[PROOFSTEP]
simpa [Filter.le_def] using H a
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α → β
de : DenseEmbedding e
p : α → Prop
x✝ : { x // p x }
x : α
hx : p x
⊢ 𝓝 { val := x, property := hx } = comap (subtypeEmb p e) (𝓝 (subtypeEmb p e { val := x, property := hx }))
[PROOFSTEP]
simp [subtypeEmb, nhds_subtype_eq_comap, de.toInducing.nhds_eq_comap, comap_comap, (· ∘ ·)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α → β
de : DenseEmbedding e
p : α → Prop
⊢ closure (range (subtypeEmb p e)) = univ
[PROOFSTEP]
ext ⟨x, hx⟩
[GOAL]
case h.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α → β
de : DenseEmbedding e
p : α → Prop
x : β
hx : x ∈ closure (e '' {x | p x})
⊢ { val := x, property := hx } ∈ closure (range (subtypeEmb p e)) ↔ { val := x, property := hx } ∈ univ
[PROOFSTEP]
rw [image_eq_range] at hx
[GOAL]
case h.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α → β
de : DenseEmbedding e
p : α → Prop
x : β
hx✝ : x ∈ closure (e '' {x | p x})
hx : x ∈ closure (range fun x => e ↑x)
⊢ { val := x, property := hx✝ } ∈ closure (range (subtypeEmb p e)) ↔ { val := x, property := hx✝ } ∈ univ
[PROOFSTEP]
simpa [closure_subtype, ← range_comp, (· ∘ ·)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : HasBasis (𝓝 x) p s
f : α → β
hf : DenseInducing f
⊢ HasBasis (𝓝 (f x)) p fun i => closure (f '' s i)
[PROOFSTEP]
rw [Filter.hasBasis_iff] at h ⊢
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
⊢ ∀ (t : Set β), t ∈ 𝓝 (f x) ↔ ∃ i, p i ∧ closure (f '' s i) ⊆ t
[PROOFSTEP]
intro T
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
⊢ T ∈ 𝓝 (f x) ↔ ∃ i, p i ∧ closure (f '' s i) ⊆ T
[PROOFSTEP]
refine' ⟨fun hT => _, fun hT => _⟩
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : T ∈ 𝓝 (f x)
⊢ ∃ i, p i ∧ closure (f '' s i) ⊆ T
[PROOFSTEP]
obtain ⟨T', hT₁, hT₂, hT₃⟩ := exists_mem_nhds_isClosed_subset hT
[GOAL]
case refine'_1.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : T ∈ 𝓝 (f x)
T' : Set β
hT₁ : T' ∈ 𝓝 (f x)
hT₂ : IsClosed T'
hT₃ : T' ⊆ T
⊢ ∃ i, p i ∧ closure (f '' s i) ⊆ T
[PROOFSTEP]
have hT₄ : f ⁻¹' T' ∈ 𝓝 x := by
rw [hf.toInducing.nhds_eq_comap x]
exact ⟨T', hT₁, Subset.rfl⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : T ∈ 𝓝 (f x)
T' : Set β
hT₁ : T' ∈ 𝓝 (f x)
hT₂ : IsClosed T'
hT₃ : T' ⊆ T
⊢ f ⁻¹' T' ∈ 𝓝 x
[PROOFSTEP]
rw [hf.toInducing.nhds_eq_comap x]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : T ∈ 𝓝 (f x)
T' : Set β
hT₁ : T' ∈ 𝓝 (f x)
hT₂ : IsClosed T'
hT₃ : T' ⊆ T
⊢ f ⁻¹' T' ∈ Filter.comap f (𝓝 (f x))
[PROOFSTEP]
exact ⟨T', hT₁, Subset.rfl⟩
[GOAL]
case refine'_1.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : T ∈ 𝓝 (f x)
T' : Set β
hT₁ : T' ∈ 𝓝 (f x)
hT₂ : IsClosed T'
hT₃ : T' ⊆ T
hT₄ : f ⁻¹' T' ∈ 𝓝 x
⊢ ∃ i, p i ∧ closure (f '' s i) ⊆ T
[PROOFSTEP]
obtain ⟨i, hi, hi'⟩ := (h _).mp hT₄
[GOAL]
case refine'_1.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : T ∈ 𝓝 (f x)
T' : Set β
hT₁ : T' ∈ 𝓝 (f x)
hT₂ : IsClosed T'
hT₃ : T' ⊆ T
hT₄ : f ⁻¹' T' ∈ 𝓝 x
i : ι
hi : p i
hi' : s i ⊆ f ⁻¹' T'
⊢ ∃ i, p i ∧ closure (f '' s i) ⊆ T
[PROOFSTEP]
exact
⟨i, hi,
(closure_mono (image_subset f hi')).trans (Subset.trans (closure_minimal (image_preimage_subset _ _) hT₂) hT₃)⟩
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
hT : ∃ i, p i ∧ closure (f '' s i) ⊆ T
⊢ T ∈ 𝓝 (f x)
[PROOFSTEP]
obtain ⟨i, hi, hi'⟩ := hT
[GOAL]
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
i : ι
hi : p i
hi' : closure (f '' s i) ⊆ T
⊢ T ∈ 𝓝 (f x)
[PROOFSTEP]
suffices closure (f '' s i) ∈ 𝓝 (f x) by filter_upwards [this] using hi'
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
i : ι
hi : p i
hi' : closure (f '' s i) ⊆ T
this : closure (f '' s i) ∈ 𝓝 (f x)
⊢ T ∈ 𝓝 (f x)
[PROOFSTEP]
filter_upwards [this] using hi'
[GOAL]
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
h : ∀ (t : Set α), t ∈ 𝓝 x ↔ ∃ i, p i ∧ s i ⊆ t
f : α → β
hf : DenseInducing f
T : Set β
i : ι
hi : p i
hi' : closure (f '' s i) ⊆ T
⊢ closure (f '' s i) ∈ 𝓝 (f x)
[PROOFSTEP]
replace h := (h (s i)).mpr ⟨i, hi, Subset.rfl⟩
[GOAL]
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T3Space β
ι : Type u_5
s : ι → Set α
p : ι → Prop
x : α
f : α → β
hf : DenseInducing f
T : Set β
i : ι
hi : p i
hi' : closure (f '' s i) ⊆ T
h : s i ∈ 𝓝 x
⊢ closure (f '' s i) ∈ 𝓝 (f x)
[PROOFSTEP]
exact hf.closure_image_mem_nhds h
| {"mathlib_filename": "Mathlib.Topology.DenseEmbedding", "llama_tokens": 18186} |
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
⊢ Homeomorph.trans h (Homeomorph.symm h) = Homeomorph.refl α
[PROOFSTEP]
ext
[GOAL]
case H
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
x✝ : α
⊢ ↑(Homeomorph.trans h (Homeomorph.symm h)) x✝ = ↑(Homeomorph.refl α) x✝
[PROOFSTEP]
apply symm_apply_apply
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
⊢ Homeomorph.trans (Homeomorph.symm h) h = Homeomorph.refl β
[PROOFSTEP]
ext
[GOAL]
case H
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
x✝ : β
⊢ ↑(Homeomorph.trans (Homeomorph.symm h) h) x✝ = ↑(Homeomorph.refl β) x✝
[PROOFSTEP]
apply apply_symm_apply
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α ≃ₜ β
g : β → α
hg : Function.RightInverse g ↑f
this : g = ↑(Homeomorph.symm f)
⊢ Function.LeftInverse g ↑f
[PROOFSTEP]
convert f.left_inv
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α ≃ₜ β
g : β → α
hg : Function.RightInverse g ↑f
this : g = ↑(Homeomorph.symm f)
⊢ Function.RightInverse g ↑f
[PROOFSTEP]
convert f.right_inv using 1
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α ≃ₜ β
g : β → α
hg : Function.RightInverse g ↑f
this : g = ↑(Homeomorph.symm f)
⊢ Continuous
{ toFun := ↑f, invFun := g, left_inv := (_ : Function.LeftInverse g ↑f),
right_inv := (_ : Function.RightInverse g ↑f) }.invFun
[PROOFSTEP]
convert f.symm.continuous
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
⊢ Inducing (↑(Homeomorph.symm h) ∘ ↑h)
[PROOFSTEP]
simp only [symm_comp_self, inducing_id]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
⊢ QuotientMap (↑h ∘ ↑(Homeomorph.symm h))
[PROOFSTEP]
simp only [self_comp_symm, QuotientMap.id]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Embedding f
⊢ Continuous (f ∘ (Equiv.ofInjective f (_ : Function.Injective f)).invFun)
[PROOFSTEP]
simp [continuous_subtype_val]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set β
h : α ≃ₜ β
⊢ IsCompact (↑h ⁻¹' s) ↔ IsCompact s
[PROOFSTEP]
rw [← image_symm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set β
h : α ≃ₜ β
⊢ IsCompact (↑(Homeomorph.symm h) '' s) ↔ IsCompact s
[PROOFSTEP]
exact h.symm.isCompact_image
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set α
h : α ≃ₜ β
hs : IsPreconnected (↑h '' s)
⊢ IsPreconnected s
[PROOFSTEP]
simpa only [image_symm, preimage_image] using hs.image _ h.symm.continuous.continuousOn
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set β
h : α ≃ₜ β
⊢ IsPreconnected (↑h ⁻¹' s) ↔ IsPreconnected s
[PROOFSTEP]
rw [← image_symm, isPreconnected_image]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set β
h : α ≃ₜ β
⊢ IsConnected (↑h ⁻¹' s) ↔ IsConnected s
[PROOFSTEP]
rw [← image_symm, isConnected_image]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
⊢ map (↑h) (cocompact α) = cocompact β
[PROOFSTEP]
rw [← h.comap_cocompact, map_comap_of_surjective h.surjective]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
s : Set α
⊢ IsOpen (↑h '' s) ↔ IsOpen s
[PROOFSTEP]
rw [← preimage_symm, isOpen_preimage]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
s : Set β
⊢ IsClosed (↑h ⁻¹' s) ↔ IsClosed s
[PROOFSTEP]
simp only [← isOpen_compl_iff, ← preimage_compl, isOpen_preimage]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
s : Set α
⊢ IsClosed (↑h '' s) ↔ IsClosed s
[PROOFSTEP]
rw [← preimage_symm, isClosed_preimage]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
s : Set α
⊢ ↑h '' closure s = closure (↑h '' s)
[PROOFSTEP]
rw [← preimage_symm, preimage_closure]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
s : Set α
⊢ ↑h '' interior s = interior (↑h '' s)
[PROOFSTEP]
rw [← preimage_symm, preimage_interior]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
s : Set α
⊢ ↑h '' frontier s = frontier (↑h '' s)
[PROOFSTEP]
rw [← preimage_symm, preimage_frontier]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
x : α
⊢ range ↑h ∈ 𝓝 (↑h x)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
x : α
⊢ map (↑(Homeomorph.symm h)) (𝓝 (↑h x)) = 𝓝 x
[PROOFSTEP]
rw [h.symm.map_nhds_eq, h.symm_apply_apply]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
y : β
⊢ comap (↑h) (𝓝 y) = 𝓝 (↑(Homeomorph.symm h) y)
[PROOFSTEP]
rw [h.nhds_eq_comap, h.apply_symm_apply]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
i : LocallyConnectedSpace β
h : α ≃ₜ β
⊢ LocallyConnectedSpace α
[PROOFSTEP]
have : ∀ x, (𝓝 x).HasBasis (fun s ↦ IsOpen s ∧ h x ∈ s ∧ IsConnected s) (h.symm '' ·) := fun x ↦
by
rw [← h.symm_map_nhds_eq]
exact (i.1 _).map _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
i : LocallyConnectedSpace β
h : α ≃ₜ β
x : α
⊢ HasBasis (𝓝 x) (fun s => IsOpen s ∧ ↑h x ∈ s ∧ IsConnected s) fun x => ↑(Homeomorph.symm h) '' x
[PROOFSTEP]
rw [← h.symm_map_nhds_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
i : LocallyConnectedSpace β
h : α ≃ₜ β
x : α
⊢ HasBasis (map (↑(Homeomorph.symm h)) (𝓝 (↑h x))) (fun s => IsOpen s ∧ ↑h x ∈ s ∧ IsConnected s) fun x =>
↑(Homeomorph.symm h) '' x
[PROOFSTEP]
exact (i.1 _).map _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
i : LocallyConnectedSpace β
h : α ≃ₜ β
this : ∀ (x : α), HasBasis (𝓝 x) (fun s => IsOpen s ∧ ↑h x ∈ s ∧ IsConnected s) fun x => ↑(Homeomorph.symm h) '' x
⊢ LocallyConnectedSpace α
[PROOFSTEP]
refine locallyConnectedSpace_of_connected_bases _ _ this fun _ _ hs ↦ ?_
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
i : LocallyConnectedSpace β
h : α ≃ₜ β
this : ∀ (x : α), HasBasis (𝓝 x) (fun s => IsOpen s ∧ ↑h x ∈ s ∧ IsConnected s) fun x => ↑(Homeomorph.symm h) '' x
x✝¹ : α
x✝ : Set β
hs : IsOpen x✝ ∧ ↑h x✝¹ ∈ x✝ ∧ IsConnected x✝
⊢ IsPreconnected (↑(Homeomorph.symm h) '' x✝)
[PROOFSTEP]
exact hs.2.2.2.image _ h.symm.continuous.continuousOn
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α ≃ β
h₁ : Continuous ↑e
h₂ : IsOpenMap ↑e
⊢ Continuous e.invFun
[PROOFSTEP]
rw [continuous_def]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α ≃ β
h₁ : Continuous ↑e
h₂ : IsOpenMap ↑e
⊢ ∀ (s : Set α), IsOpen s → IsOpen (e.invFun ⁻¹' s)
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α ≃ β
h₁ : Continuous ↑e
h₂ : IsOpenMap ↑e
s : Set α
hs : IsOpen s
⊢ IsOpen (e.invFun ⁻¹' s)
[PROOFSTEP]
convert ← h₂ s hs using 1
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : α ≃ β
h₁ : Continuous ↑e
h₂ : IsOpenMap ↑e
s : Set α
hs : IsOpen s
⊢ ↑e '' s = e.invFun ⁻¹' s
[PROOFSTEP]
apply e.image_eq_preimage
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : β → γ
x : α
⊢ range ↑h ∈ 𝓝 (↑h x)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : γ → α
⊢ IsOpenMap (↑h ∘ f) ↔ IsOpenMap f
[PROOFSTEP]
refine' ⟨_, fun hf => h.isOpenMap.comp hf⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : γ → α
⊢ IsOpenMap (↑h ∘ f) → IsOpenMap f
[PROOFSTEP]
intro hf
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : γ → α
hf : IsOpenMap (↑h ∘ f)
⊢ IsOpenMap f
[PROOFSTEP]
rw [← Function.comp.left_id f, ← h.symm_comp_self, Function.comp.assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : γ → α
hf : IsOpenMap (↑h ∘ f)
⊢ IsOpenMap (↑(Homeomorph.symm h) ∘ ↑h ∘ f)
[PROOFSTEP]
exact h.symm.isOpenMap.comp hf
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : β → γ
⊢ IsOpenMap (f ∘ ↑h) ↔ IsOpenMap f
[PROOFSTEP]
refine' ⟨_, fun hf => hf.comp h.isOpenMap⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : β → γ
⊢ IsOpenMap (f ∘ ↑h) → IsOpenMap f
[PROOFSTEP]
intro hf
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : β → γ
hf : IsOpenMap (f ∘ ↑h)
⊢ IsOpenMap f
[PROOFSTEP]
rw [← Function.comp.right_id f, ← h.self_comp_symm, ← Function.comp.assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
h : α ≃ₜ β
f : β → γ
hf : IsOpenMap (f ∘ ↑h)
⊢ IsOpenMap ((f ∘ ↑h) ∘ ↑(Homeomorph.symm h))
[PROOFSTEP]
exact hf.comp h.symm.isOpenMap
[GOAL]
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
⊢ Continuous (Equiv.piEquivPiSubtypeProd p β).toFun
[PROOFSTEP]
apply Continuous.prod_mk
[GOAL]
case hf
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
⊢ Continuous fun x x_1 => x ↑x_1
[PROOFSTEP]
exact continuous_pi fun j => continuous_apply j.1
[GOAL]
case hg
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
⊢ Continuous fun x x_1 => x ↑x_1
[PROOFSTEP]
exact continuous_pi fun j => continuous_apply j.1
[GOAL]
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
j : ι
⊢ Continuous fun a => Equiv.invFun (Equiv.piEquivPiSubtypeProd p β) a j
[PROOFSTEP]
dsimp only [Equiv.piEquivPiSubtypeProd]
[GOAL]
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
j : ι
⊢ Continuous fun a => if h : p j then Prod.fst a { val := j, property := h } else Prod.snd a { val := j, property := h }
[PROOFSTEP]
split_ifs
[GOAL]
case pos
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
j : ι
h✝ : p j
⊢ Continuous fun a => Prod.fst a { val := j, property := h✝ }
case neg
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
p : ι → Prop
β : ι → Type u_6
inst✝¹ : (i : ι) → TopologicalSpace (β i)
inst✝ : DecidablePred p
j : ι
h✝ : ¬p j
⊢ Continuous fun a => Prod.snd a { val := j, property := h✝ }
[PROOFSTEP]
exacts [(continuous_apply _).comp continuous_fst, (continuous_apply _).comp continuous_snd]
[GOAL]
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
inst✝¹ : DecidableEq ι
i : ι
β : ι → Type u_6
inst✝ : (j : ι) → TopologicalSpace (β j)
j : ι
⊢ Continuous fun a => Equiv.invFun (Equiv.piSplitAt i β) a j
[PROOFSTEP]
dsimp only [Equiv.piSplitAt]
[GOAL]
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
inst✝¹ : DecidableEq ι
i : ι
β : ι → Type u_6
inst✝ : (j : ι) → TopologicalSpace (β j)
j : ι
⊢ Continuous fun a => if h : j = i then (_ : i = j) ▸ a.fst else Prod.snd a { val := j, property := h }
[PROOFSTEP]
split_ifs with h
[GOAL]
case pos
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
inst✝¹ : DecidableEq ι
i : ι
β : ι → Type u_6
inst✝ : (j : ι) → TopologicalSpace (β j)
j : ι
h : j = i
⊢ Continuous fun a => (_ : i = j) ▸ a.fst
case neg
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
inst✝¹ : DecidableEq ι
i : ι
β : ι → Type u_6
inst✝ : (j : ι) → TopologicalSpace (β j)
j : ι
h : ¬j = i
⊢ Continuous fun a => Prod.snd a { val := j, property := h }
[PROOFSTEP]
subst h
[GOAL]
case pos
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
inst✝¹ : DecidableEq ι
β : ι → Type u_6
inst✝ : (j : ι) → TopologicalSpace (β j)
j : ι
⊢ Continuous fun a => (_ : j = j) ▸ a.fst
case neg
α : Type u_1
β✝ : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
ι : Type u_5
inst✝¹ : DecidableEq ι
i : ι
β : ι → Type u_6
inst✝ : (j : ι) → TopologicalSpace (β j)
j : ι
h : ¬j = i
⊢ Continuous fun a => Prod.snd a { val := j, property := h }
[PROOFSTEP]
exacts [continuous_fst, (continuous_apply _).comp continuous_snd]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α ≃ β
hf : Inducing ↑f
⊢ Continuous
(↑f ∘
{ toFun := f.toFun, invFun := f.invFun, left_inv := (_ : Function.LeftInverse f.invFun f.toFun),
right_inv := (_ : Function.RightInverse f.invFun f.toFun) }.invFun)
[PROOFSTEP]
simpa using continuous_id
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : CompactSpace α
inst✝ : T2Space β
f : α ≃ β
hf : Continuous ↑f
⊢ Continuous ↑f.symm
[PROOFSTEP]
rw [continuous_iff_isClosed]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : CompactSpace α
inst✝ : T2Space β
f : α ≃ β
hf : Continuous ↑f
⊢ ∀ (s : Set α), IsClosed s → IsClosed (↑f.symm ⁻¹' s)
[PROOFSTEP]
intro C hC
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : CompactSpace α
inst✝ : T2Space β
f : α ≃ β
hf : Continuous ↑f
C : Set α
hC : IsClosed C
⊢ IsClosed (↑f.symm ⁻¹' C)
[PROOFSTEP]
have hC' : IsClosed (f '' C) := (hC.isCompact.image hf).isClosed
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : CompactSpace α
inst✝ : T2Space β
f : α ≃ β
hf : Continuous ↑f
C : Set α
hC : IsClosed C
hC' : IsClosed (↑f '' C)
⊢ IsClosed (↑f.symm ⁻¹' C)
[PROOFSTEP]
rwa [Equiv.image_eq_preimage] at hC'
| {"mathlib_filename": "Mathlib.Topology.Homeomorph", "llama_tokens": 9687} |
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : α ≃ₜ β
s : Set α
hs : IsOpen s
t : Set β
h : ↑e '' s = t
⊢ IsOpen (Equiv.toLocalEquivOfImageEq e.toEquiv s t h).target
[PROOFSTEP]
simpa [← h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : α ≃ₜ β
⊢ ↑e '' univ = univ
[PROOFSTEP]
rw [image_univ, e.surjective.range_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e : LocalHomeomorph α β
e' : LocalEquiv α β
h : e.toLocalEquiv = e'
⊢ replaceEquiv e e' h = e
[PROOFSTEP]
cases e
[GOAL]
case mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e' toLocalEquiv✝ : LocalEquiv α β
open_source✝ : IsOpen toLocalEquiv✝.source
open_target✝ : IsOpen toLocalEquiv✝.target
continuous_toFun✝ : ContinuousOn (↑toLocalEquiv✝) toLocalEquiv✝.source
continuous_invFun✝ : ContinuousOn toLocalEquiv✝.invFun toLocalEquiv✝.target
h :
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }.toLocalEquiv =
e'
⊢ replaceEquiv
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }
e' h =
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }
[PROOFSTEP]
subst e'
[GOAL]
case mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
toLocalEquiv✝ : LocalEquiv α β
open_source✝ : IsOpen toLocalEquiv✝.source
open_target✝ : IsOpen toLocalEquiv✝.target
continuous_toFun✝ : ContinuousOn (↑toLocalEquiv✝) toLocalEquiv✝.source
continuous_invFun✝ : ContinuousOn toLocalEquiv✝.invFun toLocalEquiv✝.target
⊢ replaceEquiv
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }.toLocalEquiv
(_ :
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }.toLocalEquiv =
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }.toLocalEquiv) =
{ toLocalEquiv := toLocalEquiv✝, open_source := open_source✝, open_target := open_target✝,
continuous_toFun := continuous_toFun✝, continuous_invFun := continuous_invFun✝ }
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
hx : x ∈ e.source
x' : α
hx' : ↑(LocalHomeomorph.symm e) (↑e x') = x'
h : ↑e x' = ↑e x
⊢ x' ∈ {x}
[PROOFSTEP]
rw [mem_singleton_iff, ← e.left_inv hx, ← h, hx']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
⊢ e = e' →
(∀ (x : α), ↑e x = ↑e' x) ∧
(∀ (x : β), ↑(LocalHomeomorph.symm e) x = ↑(LocalHomeomorph.symm e') x) ∧ e.source = e'.source
[PROOFSTEP]
rintro rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
⊢ (∀ (x : α), ↑e x = ↑e x) ∧
(∀ (x : β), ↑(LocalHomeomorph.symm e) x = ↑(LocalHomeomorph.symm e) x) ∧ e.source = e.source
[PROOFSTEP]
exact ⟨fun x => rfl, fun x => rfl, rfl⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
x : α
hx : x ∈ e.source
⊢ Tendsto (↑(LocalHomeomorph.symm e)) (𝓝 (↑e x)) (𝓝 x)
[PROOFSTEP]
simpa only [ContinuousAt, e.left_inv hx] using e.continuousAt_symm (e.map_source hx)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
x : α
hx : x ∈ e.source
⊢ 𝓝 (↑(LocalHomeomorph.symm e) (↑e x)) = 𝓝 x
[PROOFSTEP]
rw [e.left_inv hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
hx : x ∈ e.source
s : Set β
⊢ map (↑e) (𝓝[↑e ⁻¹' s] x) = 𝓝[s] ↑e x
[PROOFSTEP]
rw [e.map_nhdsWithin_eq hx, e.image_source_inter_eq', e.target_inter_inv_preimage_preimage,
e.nhdsWithin_target_inter (e.map_source hx)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : β → Prop
hx : x ∈ e.source
⊢ (∀ᶠ (y : β) in 𝓝 (↑e x), p y) ↔ ∀ᶠ (b : β) in map (fun x => ↑e x) (𝓝 x), p b
[PROOFSTEP]
rw [e.map_nhds_eq hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : α → Prop
hx : x ∈ e.source
⊢ (∀ᶠ (y : β) in 𝓝 (↑e x), p (↑(LocalHomeomorph.symm e) y)) ↔ ∀ᶠ (x : α) in 𝓝 x, p x
[PROOFSTEP]
rw [e.eventually_nhds _ hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : α → Prop
hx : x ∈ e.source
⊢ (∀ᶠ (x : α) in 𝓝 x, p (↑(LocalHomeomorph.symm e) (↑e x))) ↔ ∀ᶠ (x : α) in 𝓝 x, p x
[PROOFSTEP]
refine' eventually_congr ((e.eventually_left_inverse hx).mono fun y hy => _)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : α → Prop
hx : x ∈ e.source
y : α
hy : ↑(LocalHomeomorph.symm e) (↑e y) = y
⊢ p (↑(LocalHomeomorph.symm e) (↑e y)) ↔ p y
[PROOFSTEP]
rw [hy]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : β → Prop
s : Set α
hx : x ∈ e.source
⊢ (∀ᶠ (y : β) in 𝓝[↑(LocalHomeomorph.symm e) ⁻¹' s] ↑e x, p y) ↔ ∀ᶠ (x : α) in 𝓝[s] x, p (↑e x)
[PROOFSTEP]
refine' Iff.trans _ eventually_map
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : β → Prop
s : Set α
hx : x ∈ e.source
⊢ (∀ᶠ (y : β) in 𝓝[↑(LocalHomeomorph.symm e) ⁻¹' s] ↑e x, p y) ↔ ∀ᶠ (b : β) in map (fun x => ↑e x) (𝓝[s] x), p b
[PROOFSTEP]
rw [e.map_nhdsWithin_eq hx, e.image_source_inter_eq', e.nhdsWithin_target_inter (e.mapsTo hx)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : α → Prop
s : Set α
hx : x ∈ e.source
⊢ (∀ᶠ (y : β) in 𝓝[↑(LocalHomeomorph.symm e) ⁻¹' s] ↑e x, p (↑(LocalHomeomorph.symm e) y)) ↔ ∀ᶠ (x : α) in 𝓝[s] x, p x
[PROOFSTEP]
rw [e.eventually_nhdsWithin _ hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : α → Prop
s : Set α
hx : x ∈ e.source
⊢ (∀ᶠ (x : α) in 𝓝[s] x, p (↑(LocalHomeomorph.symm e) (↑e x))) ↔ ∀ᶠ (x : α) in 𝓝[s] x, p x
[PROOFSTEP]
refine
eventually_congr <| (eventually_nhdsWithin_of_eventually_nhds <| e.eventually_left_inverse hx).mono fun y hy => ?_
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
x : α
p : α → Prop
s : Set α
hx : x ∈ e.source
y : α
hy : ↑(LocalHomeomorph.symm e) (↑e y) = y
⊢ p (↑(LocalHomeomorph.symm e) (↑e y)) ↔ p y
[PROOFSTEP]
rw [hy]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
s : Set α
t : Set γ
x : α
f : α → γ
hf : ContinuousWithinAt f s x
hxe : x ∈ e.source
ht : t ∈ 𝓝 (f x)
⊢ ↑(LocalHomeomorph.symm e) ⁻¹' s =ᶠ[𝓝 (↑e x)] e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (s ∩ f ⁻¹' t)
[PROOFSTEP]
rw [eventuallyEq_set, e.eventually_nhds _ hxe]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
s : Set α
t : Set γ
x : α
f : α → γ
hf : ContinuousWithinAt f s x
hxe : x ∈ e.source
ht : t ∈ 𝓝 (f x)
⊢ ∀ᶠ (x : α) in 𝓝 x,
↑e x ∈ ↑(LocalHomeomorph.symm e) ⁻¹' s ↔ ↑e x ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (s ∩ f ⁻¹' t)
[PROOFSTEP]
filter_upwards [e.open_source.mem_nhds hxe, mem_nhdsWithin_iff_eventually.mp (hf.preimage_mem_nhdsWithin ht)]
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
s : Set α
t : Set γ
x : α
f : α → γ
hf : ContinuousWithinAt f s x
hxe : x ∈ e.source
ht : t ∈ 𝓝 (f x)
⊢ ∀ (a : α),
a ∈ e.source →
(a ∈ s → a ∈ f ⁻¹' t) →
(↑e a ∈ ↑(LocalHomeomorph.symm e) ⁻¹' s ↔ ↑e a ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (s ∩ f ⁻¹' t))
[PROOFSTEP]
intro y hy hyu
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalHomeomorph α β
s : Set α
t : Set γ
x : α
f : α → γ
hf : ContinuousWithinAt f s x
hxe : x ∈ e.source
ht : t ∈ 𝓝 (f x)
y : α
hy : y ∈ e.source
hyu : y ∈ s → y ∈ f ⁻¹' t
⊢ ↑e y ∈ ↑(LocalHomeomorph.symm e) ⁻¹' s ↔ ↑e y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (s ∩ f ⁻¹' t)
[PROOFSTEP]
simp_rw [mem_inter_iff, mem_preimage, mem_inter_iff, e.mapsTo hy, true_and_iff, iff_self_and, e.left_inv hy,
iff_true_intro hyu]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
t : Set β
x : α
y : β
⊢ IsImage e s t ↔ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (e.source ∩ s) = e.target ∩ t
[PROOFSTEP]
rw [iff_symm_preimage_eq, ← image_source_inter_eq, ← image_source_inter_eq']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
t : Set β
x : α
y : β
h : IsImage e s t
hx : x ∈ e.source
⊢ map (↑e) (𝓝[s] x) = 𝓝[t] ↑e x
[PROOFSTEP]
rw [e.map_nhdsWithin_eq hx, h.image_eq, e.nhdsWithin_target_inter (e.map_source hx)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
t : Set β
x✝ : α
y : β
h : IsImage e s t
x : α
hx : x ∈ e.source
⊢ ↑e x ∈ closure t ↔ x ∈ closure s
[PROOFSTEP]
simp only [mem_closure_iff_nhdsWithin_neBot, ← h.map_nhdsWithin_eq hx, map_neBot_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
t : Set β
x : α
y : β
h : IsImage e s t
⊢ IsImage e (interior s) (interior t)
[PROOFSTEP]
simpa only [closure_compl, compl_compl] using h.compl.closure.compl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
h : s ⊆ e.source
⊢ IsOpen (↑e '' s)
[PROOFSTEP]
have : e '' s = e.target ∩ e.symm ⁻¹' s := e.toLocalEquiv.image_eq_target_inter_inv_preimage h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
h : s ⊆ e.source
this : ↑e '' s = e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' s
⊢ IsOpen (↑e '' s)
[PROOFSTEP]
rw [this]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
h : s ⊆ e.source
this : ↑e '' s = e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' s
⊢ IsOpen (e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' s)
[PROOFSTEP]
exact e.continuousOn_symm.preimage_open_of_open e.open_target hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e : LocalEquiv α β
hc : ContinuousOn (↑e) e.source
ho : IsOpenMap (restrict e.source ↑e)
hs : IsOpen e.source
⊢ IsOpen e.target
[PROOFSTEP]
simpa only [range_restrict, e.image_source_eq_target] using ho.isOpen_range
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
⊢ (LocalHomeomorph.restr e s).toLocalEquiv.source = e.source ∩ s
[PROOFSTEP]
rw [e.restr_source, hs.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
⊢ (LocalHomeomorph.restr e s).toLocalEquiv = LocalEquiv.restr e.toLocalEquiv s
[PROOFSTEP]
rw [e.restr_toLocalEquiv, hs.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
⊢ LocalHomeomorph.restr e (e.source ∩ s) = LocalHomeomorph.restr e s
[PROOFSTEP]
refine' LocalHomeomorph.ext _ _ (fun x => rfl) (fun x => rfl) _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
⊢ (LocalHomeomorph.restr e (e.source ∩ s)).toLocalEquiv.source = (LocalHomeomorph.restr e s).toLocalEquiv.source
[PROOFSTEP]
simp [e.open_source.interior_eq, ← inter_assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
⊢ ofSet univ (_ : IsOpen univ) = LocalHomeomorph.refl α
[PROOFSTEP]
ext
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
x✝ : α
⊢ ↑(ofSet univ (_ : IsOpen univ)) x✝ = ↑(LocalHomeomorph.refl α) x✝
[PROOFSTEP]
simp
[GOAL]
case hinv
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
x✝ : α
⊢ ↑(LocalHomeomorph.symm (ofSet univ (_ : IsOpen univ))) x✝ = ↑(LocalHomeomorph.symm (LocalHomeomorph.refl α)) x✝
[PROOFSTEP]
simp
[GOAL]
case hs.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
x✝ : α
⊢ x✝ ∈ (ofSet univ (_ : IsOpen univ)).toLocalEquiv.source ↔ x✝ ∈ (LocalHomeomorph.refl α).toLocalEquiv.source
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
⊢ (LocalHomeomorph.symm
(LocalHomeomorph.restrOpen (LocalHomeomorph.symm e) e'.source (_ : IsOpen e'.source))).toLocalEquiv.target =
(LocalHomeomorph.restrOpen e' e.target (_ : IsOpen e.target)).toLocalEquiv.source
[PROOFSTEP]
simp [inter_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set β
hs : IsOpen s
⊢ (LocalHomeomorph.trans e (ofSet s hs)).toLocalEquiv.source = (LocalHomeomorph.restr e (↑e ⁻¹' s)).toLocalEquiv.source
[PROOFSTEP]
rw [trans_source, restr_source, ofSet_source, ← preimage_interior, hs.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set β
hs : IsOpen s
⊢ LocalHomeomorph.trans e (ofSet s hs) = LocalHomeomorph.restr e (e.source ∩ ↑e ⁻¹' s)
[PROOFSTEP]
rw [trans_ofSet, restr_source_inter]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
⊢ (LocalHomeomorph.trans (ofSet s hs) e).toLocalEquiv.source = (LocalHomeomorph.restr e s).toLocalEquiv.source
[PROOFSTEP]
simp [hs.interior_eq, inter_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
⊢ LocalHomeomorph.trans (ofSet s hs) e = LocalHomeomorph.restr e (e.source ∩ s)
[PROOFSTEP]
rw [ofSet_trans, restr_source_inter]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
s' : Set α
hs' : IsOpen s'
⊢ LocalHomeomorph.trans (ofSet s hs) (ofSet s' hs') = ofSet (s ∩ s') (_ : IsOpen (s ∩ s'))
[PROOFSTEP]
rw [(ofSet s hs).trans_ofSet hs']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
s' : Set α
hs' : IsOpen s'
⊢ LocalHomeomorph.restr (ofSet s hs) (↑(ofSet s hs) ⁻¹' s') = ofSet (s ∩ s') (_ : IsOpen (s ∩ s'))
[PROOFSTEP]
ext
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
s' : Set α
hs' : IsOpen s'
x✝ : α
⊢ ↑(LocalHomeomorph.restr (ofSet s hs) (↑(ofSet s hs) ⁻¹' s')) x✝ = ↑(ofSet (s ∩ s') (_ : IsOpen (s ∩ s'))) x✝
[PROOFSTEP]
simp [hs'.interior_eq]
[GOAL]
case hinv
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
s' : Set α
hs' : IsOpen s'
x✝ : α
⊢ ↑(LocalHomeomorph.symm (LocalHomeomorph.restr (ofSet s hs) (↑(ofSet s hs) ⁻¹' s'))) x✝ =
↑(LocalHomeomorph.symm (ofSet (s ∩ s') (_ : IsOpen (s ∩ s')))) x✝
[PROOFSTEP]
simp [hs'.interior_eq]
[GOAL]
case hs.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
s : Set α
hs : IsOpen s
s' : Set α
hs' : IsOpen s'
x✝ : α
⊢ x✝ ∈ (LocalHomeomorph.restr (ofSet s hs) (↑(ofSet s hs) ⁻¹' s')).toLocalEquiv.source ↔
x✝ ∈ (ofSet (s ∩ s') (_ : IsOpen (s ∩ s'))).toLocalEquiv.source
[PROOFSTEP]
simp [hs'.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ LocalHomeomorph.restr e e'.source ≈ LocalHomeomorph.restr e' e.source
[PROOFSTEP]
constructor
[GOAL]
case left
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ (LocalHomeomorph.restr e e'.source).toLocalEquiv.source = (LocalHomeomorph.restr e' e.source).toLocalEquiv.source
[PROOFSTEP]
rw [e'.restr_source' _ e.open_source]
[GOAL]
case left
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ (LocalHomeomorph.restr e e'.source).toLocalEquiv.source = e'.source ∩ e.source
[PROOFSTEP]
rw [e.restr_source' _ e'.open_source]
[GOAL]
case left
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ e.source ∩ e'.source = e'.source ∩ e.source
[PROOFSTEP]
exact Set.inter_comm _ _
[GOAL]
case right
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ EqOn (↑(LocalHomeomorph.restr e e'.source)) (↑(LocalHomeomorph.restr e' e.source))
(LocalHomeomorph.restr e e'.source).toLocalEquiv.source
[PROOFSTEP]
rw [e.restr_source' _ e'.open_source]
[GOAL]
case right
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ EqOn (↑(LocalHomeomorph.restr e e'.source)) (↑(LocalHomeomorph.restr e' e.source)) (e.source ∩ e'.source)
[PROOFSTEP]
refine' (EqOn.trans _ h).trans _
[GOAL]
case right.refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ EqOn (↑(LocalHomeomorph.restr e e'.source)) (↑e) (e.source ∩ e'.source)
[PROOFSTEP]
simp only [mfld_simps, eqOn_refl]
[GOAL]
case right.refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
h : EqOn (↑e) (↑e') (e.source ∩ e'.source)
⊢ EqOn (↑e') (↑(LocalHomeomorph.restr e' e.source)) (e.source ∩ e'.source)
[PROOFSTEP]
simp only [mfld_simps, eqOn_refl]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁ e₂).toLocalEquiv.source
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
obtain ⟨⟨x, y⟩, -⟩ := id h
[GOAL]
case intro.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁ e₂).toLocalEquiv.source
x : α
y : γ
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
haveI : Nonempty α := ⟨x⟩
[GOAL]
case intro.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁ e₂).toLocalEquiv.source
x : α
y : γ
this : Nonempty α
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
haveI : Nonempty β := ⟨e₁ x⟩
[GOAL]
case intro.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁ e₂).toLocalEquiv.source
x : α
y : γ
this✝ : Nonempty α
this : Nonempty β
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
haveI : Nonempty γ := ⟨y⟩
[GOAL]
case intro.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁ e₂).toLocalEquiv.source
x : α
y : γ
this✝¹ : Nonempty α
this✝ : Nonempty β
this : Nonempty γ
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
haveI : Nonempty δ := ⟨e₂ y⟩
[GOAL]
case intro.mk
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁ e₂).toLocalEquiv.source
x : α
y : γ
this✝² : Nonempty α
this✝¹ : Nonempty β
this✝ : Nonempty γ
this : Nonempty δ
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
simp_rw [LocalHomeomorph.ext_iff, prod_apply, prod_symm_apply, prod_source, Prod.ext_iff,
Set.prod_eq_prod_iff_of_nonempty h, forall_and, Prod.forall, forall_const, and_assoc, and_left_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
e₁ e₁' : LocalHomeomorph α β
e₂ e₂' : LocalHomeomorph γ δ
h : Set.Nonempty (prod e₁' e₂').toLocalEquiv.source
⊢ prod e₁ e₂ = prod e₁' e₂' ↔ e₁ = e₁' ∧ e₂ = e₂'
[PROOFSTEP]
rw [eq_comm, prod_eq_prod_of_nonempty h, eq_comm, @eq_comm _ e₂']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
inst✝¹ : (x : α) → Decidable (x ∈ e.source)
inst✝ : (y : β) → Decidable (y ∈ e.target)
Hs : Disjoint e.source e'.source
Ht : Disjoint e.target e'.target
⊢ e.source ∩ frontier e.source = e'.source ∩ frontier e.source
[PROOFSTEP]
rw [e.open_source.inter_frontier_eq, (Hs.symm.frontier_right e'.open_source).inter_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
inst✝¹ : (x : α) → Decidable (x ∈ e.source)
inst✝ : (y : β) → Decidable (y ∈ e.target)
Hs : Disjoint e.source e'.source
Ht : Disjoint e.target e'.target
⊢ EqOn (↑e) (↑e') (e.source ∩ frontier e.source)
[PROOFSTEP]
rw [e.open_source.inter_frontier_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
e✝ : LocalHomeomorph α β
e'✝ : LocalHomeomorph β γ
e e' : LocalHomeomorph α β
inst✝¹ : (x : α) → Decidable (x ∈ e.source)
inst✝ : (y : β) → Decidable (y ∈ e.target)
Hs : Disjoint e.source e'.source
Ht : Disjoint e.target e'.target
⊢ EqOn ↑e ↑e' ∅
[PROOFSTEP]
exact eqOn_empty _ _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : β → γ
s : Set β
x : β
h : x ∈ e.target
⊢ ContinuousWithinAt f s x ↔ ContinuousWithinAt (f ∘ ↑e) (↑e ⁻¹' s) (↑(LocalHomeomorph.symm e) x)
[PROOFSTEP]
simp_rw [ContinuousWithinAt, ← @tendsto_map'_iff _ _ _ _ e, e.map_nhdsWithin_preimage_eq (e.map_target h), (· ∘ ·),
e.right_inv h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : β → γ
x : β
h : x ∈ e.target
⊢ ContinuousAt f x ↔ ContinuousAt (f ∘ ↑e) (↑(LocalHomeomorph.symm e) x)
[PROOFSTEP]
rw [← continuousWithinAt_univ, e.continuousWithinAt_iff_continuousWithinAt_comp_right h, preimage_univ,
continuousWithinAt_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : β → γ
s : Set β
h : s ⊆ e.target
⊢ ContinuousOn f s ↔ ContinuousOn (f ∘ ↑e) (e.source ∩ ↑e ⁻¹' s)
[PROOFSTEP]
simp only [← e.symm_image_eq_source_inter_preimage h, ContinuousOn, ball_image_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : β → γ
s : Set β
h : s ⊆ e.target
⊢ (∀ (x : β), x ∈ s → ContinuousWithinAt f s x) ↔
∀ (x : β), x ∈ s → ContinuousWithinAt (f ∘ ↑e) (↑(LocalHomeomorph.symm e) '' s) (↑(LocalHomeomorph.symm e) x)
[PROOFSTEP]
refine' forall₂_congr fun x hx => _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : β → γ
s : Set β
h : s ⊆ e.target
x : β
hx : x ∈ s
⊢ ContinuousWithinAt f s x ↔ ContinuousWithinAt (f ∘ ↑e) (↑(LocalHomeomorph.symm e) '' s) (↑(LocalHomeomorph.symm e) x)
[PROOFSTEP]
rw [e.continuousWithinAt_iff_continuousWithinAt_comp_right (h hx), e.symm_image_eq_source_inter_preimage h, inter_comm,
continuousWithinAt_inter]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : β → γ
s : Set β
h : s ⊆ e.target
x : β
hx : x ∈ s
⊢ e.source ∈ 𝓝 (↑(LocalHomeomorph.symm e) x)
[PROOFSTEP]
exact IsOpen.mem_nhds e.open_source (e.map_target (h hx))
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
s : Set γ
x : γ
hx : f x ∈ e.source
h : f ⁻¹' e.source ∈ 𝓝[s] x
⊢ ContinuousWithinAt f s x ↔ ContinuousWithinAt (↑e ∘ f) s x
[PROOFSTEP]
refine' ⟨(e.continuousAt hx).comp_continuousWithinAt, fun fe_cont => _⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
s : Set γ
x : γ
hx : f x ∈ e.source
h : f ⁻¹' e.source ∈ 𝓝[s] x
fe_cont : ContinuousWithinAt (↑e ∘ f) s x
⊢ ContinuousWithinAt f s x
[PROOFSTEP]
rw [← continuousWithinAt_inter' h] at fe_cont ⊢
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
s : Set γ
x : γ
hx : f x ∈ e.source
h : f ⁻¹' e.source ∈ 𝓝[s] x
fe_cont : ContinuousWithinAt (↑e ∘ f) (s ∩ f ⁻¹' e.source) x
⊢ ContinuousWithinAt f (s ∩ f ⁻¹' e.source) x
[PROOFSTEP]
have : ContinuousWithinAt (e.symm ∘ e ∘ f) (s ∩ f ⁻¹' e.source) x :=
haveI : ContinuousWithinAt e.symm univ (e (f x)) := (e.continuousAt_symm (e.map_source hx)).continuousWithinAt
ContinuousWithinAt.comp this fe_cont (subset_univ _)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
s : Set γ
x : γ
hx : f x ∈ e.source
h : f ⁻¹' e.source ∈ 𝓝[s] x
fe_cont : ContinuousWithinAt (↑e ∘ f) (s ∩ f ⁻¹' e.source) x
this : ContinuousWithinAt (↑(LocalHomeomorph.symm e) ∘ ↑e ∘ f) (s ∩ f ⁻¹' e.source) x
⊢ ContinuousWithinAt f (s ∩ f ⁻¹' e.source) x
[PROOFSTEP]
exact this.congr (fun y hy => by simp [e.left_inv hy.2]) (by simp [e.left_inv hx])
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
s : Set γ
x : γ
hx : f x ∈ e.source
h : f ⁻¹' e.source ∈ 𝓝[s] x
fe_cont : ContinuousWithinAt (↑e ∘ f) (s ∩ f ⁻¹' e.source) x
this : ContinuousWithinAt (↑(LocalHomeomorph.symm e) ∘ ↑e ∘ f) (s ∩ f ⁻¹' e.source) x
y : γ
hy : y ∈ s ∩ f ⁻¹' e.source
⊢ f y = (↑(LocalHomeomorph.symm e) ∘ ↑e ∘ f) y
[PROOFSTEP]
simp [e.left_inv hy.2]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
s : Set γ
x : γ
hx : f x ∈ e.source
h : f ⁻¹' e.source ∈ 𝓝[s] x
fe_cont : ContinuousWithinAt (↑e ∘ f) (s ∩ f ⁻¹' e.source) x
this : ContinuousWithinAt (↑(LocalHomeomorph.symm e) ∘ ↑e ∘ f) (s ∩ f ⁻¹' e.source) x
⊢ f x = (↑(LocalHomeomorph.symm e) ∘ ↑e ∘ f) x
[PROOFSTEP]
simp [e.left_inv hx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
x : γ
h : f ⁻¹' e.source ∈ 𝓝 x
⊢ ContinuousAt f x ↔ ContinuousAt (↑e ∘ f) x
[PROOFSTEP]
have hx : f x ∈ e.source := (mem_of_mem_nhds h : _)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
x : γ
h : f ⁻¹' e.source ∈ 𝓝 x
hx : f x ∈ e.source
⊢ ContinuousAt f x ↔ ContinuousAt (↑e ∘ f) x
[PROOFSTEP]
have h' : f ⁻¹' e.source ∈ 𝓝[univ] x := by rwa [nhdsWithin_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
x : γ
h : f ⁻¹' e.source ∈ 𝓝 x
hx : f x ∈ e.source
⊢ f ⁻¹' e.source ∈ 𝓝[univ] x
[PROOFSTEP]
rwa [nhdsWithin_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
x : γ
h : f ⁻¹' e.source ∈ 𝓝 x
hx : f x ∈ e.source
h' : f ⁻¹' e.source ∈ 𝓝[univ] x
⊢ ContinuousAt f x ↔ ContinuousAt (↑e ∘ f) x
[PROOFSTEP]
rw [← continuousWithinAt_univ, ← continuousWithinAt_univ, e.continuousWithinAt_iff_continuousWithinAt_comp_left hx h']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
h : f ⁻¹' e.source = univ
⊢ Continuous f ↔ Continuous (↑e ∘ f)
[PROOFSTEP]
simp only [continuous_iff_continuousOn_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
f : γ → α
h : f ⁻¹' e.source = univ
⊢ ContinuousOn f univ ↔ ContinuousOn (↑e ∘ f) univ
[PROOFSTEP]
exact e.continuousOn_iff_continuousOn_comp_left (Eq.symm h).subset
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
x : α
hx : x ∈ e.source
⊢ 𝓝 x = comap (↑e) (𝓝 (↑e x)) ⊓ 𝓟 e.source
[PROOFSTEP]
lift x to e.source using hx
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
x : { x // x ∈ e.source }
⊢ 𝓝 ↑x = comap (↑e) (𝓝 (↑e ↑x)) ⊓ 𝓟 e.source
[PROOFSTEP]
rw [← e.open_source.nhdsWithin_eq x.2, ← map_nhds_subtype_val, ← map_comap_setCoe_val,
e.toHomeomorphSourceTarget.nhds_eq_comap, nhds_subtype_eq_comap]
[GOAL]
case intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
x : { x // x ∈ e.source }
⊢ map Subtype.val (comap (↑(toHomeomorphSourceTarget e)) (comap Subtype.val (𝓝 ↑(↑(toHomeomorphSourceTarget e) x)))) =
map Subtype.val (comap Subtype.val (comap (↑e) (𝓝 (↑e ↑x))))
[PROOFSTEP]
simp only [(· ∘ ·), toHomeomorphSourceTarget_apply_coe, comap_comap]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
h' : e.target = univ
x : α
⊢ x ∈ e.source
[PROOFSTEP]
rw [h]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
h' : e.target = univ
x : α
⊢ x ∈ univ
[PROOFSTEP]
exact mem_univ _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
h' : e.target = univ
x : β
⊢ x ∈ e.target
[PROOFSTEP]
rw [h']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
h' : e.target = univ
x : β
⊢ x ∈ univ
[PROOFSTEP]
exact mem_univ _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
h' : e.target = univ
⊢ Continuous
{ toFun := ↑e, invFun := ↑(LocalHomeomorph.symm e),
left_inv := (_ : ∀ (x : α), ↑(LocalHomeomorph.symm e) (↑e x) = x),
right_inv := (_ : ∀ (x : β), ↑e (↑(LocalHomeomorph.symm e) x) = x) }.toFun
[PROOFSTEP]
simpa only [continuous_iff_continuousOn_univ, h] using e.continuousOn
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
h' : e.target = univ
⊢ Continuous
{ toFun := ↑e, invFun := ↑(LocalHomeomorph.symm e),
left_inv := (_ : ∀ (x : α), ↑(LocalHomeomorph.symm e) (↑e x) = x),
right_inv := (_ : ∀ (x : β), ↑e (↑(LocalHomeomorph.symm e) x) = x) }.invFun
[PROOFSTEP]
simpa only [continuous_iff_continuousOn_univ, h'] using e.continuousOn_symm
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ OpenEmbedding ↑e
[PROOFSTEP]
apply openEmbedding_of_continuous_injective_open
[GOAL]
case h₁
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ Continuous ↑e
[PROOFSTEP]
apply continuous_iff_continuousOn_univ.mpr
[GOAL]
case h₁
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ ContinuousOn (↑e) univ
[PROOFSTEP]
rw [← h]
[GOAL]
case h₁
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ ContinuousOn (↑e) e.source
[PROOFSTEP]
exact e.continuousOn
[GOAL]
case h₂
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ Injective ↑e
[PROOFSTEP]
apply Set.injective_iff_injOn_univ.mpr
[GOAL]
case h₂
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ InjOn (↑e) univ
[PROOFSTEP]
rw [← h]
[GOAL]
case h₂
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ InjOn (↑e) e.source
[PROOFSTEP]
exact e.injOn
[GOAL]
case h₃
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
⊢ IsOpenMap ↑e
[PROOFSTEP]
intro U hU
[GOAL]
case h₃
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
e : LocalHomeomorph α β
e' : LocalHomeomorph β γ
h : e.source = univ
U : Set α
hU : IsOpen U
⊢ IsOpen (↑e '' U)
[PROOFSTEP]
simpa only [h, subset_univ, mfld_simps] using e.image_open_of_open hU
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
⊢ (localHomeomorphSubtypeCoe s).toLocalEquiv.target = ↑s
[PROOFSTEP]
simp only [localHomeomorphSubtypeCoe, Subtype.range_coe_subtype, mfld_simps]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
⊢ {x | x ∈ s.carrier} = ↑s
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
⊢ (subtypeRestr e s).toLocalEquiv.source = Subtype.val ⁻¹' e.source
[PROOFSTEP]
simp only [subtypeRestr_def, mfld_simps]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
x : { x // x ∈ s }
hxe : ↑x ∈ e.source
⊢ ↑e ↑x ∈ (subtypeRestr e s).toLocalEquiv.target
[PROOFSTEP]
refine' ⟨e.map_source hxe, _⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
x : { x // x ∈ s }
hxe : ↑x ∈ e.source
⊢ ↑e ↑x ∈ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe s).toLocalEquiv.target
[PROOFSTEP]
rw [s.localHomeomorphSubtypeCoe_target, mem_preimage, e.leftInvOn hxe]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
x : { x // x ∈ s }
hxe : ↑x ∈ e.source
⊢ ↑x ∈ ↑s
[PROOFSTEP]
exact x.prop
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
⊢ LocalHomeomorph.trans (LocalHomeomorph.symm (subtypeRestr f s)) (subtypeRestr f' s) ≈
LocalHomeomorph.restr (LocalHomeomorph.trans (LocalHomeomorph.symm f) f')
(f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
[PROOFSTEP]
simp only [subtypeRestr_def, trans_symm_eq_symm_trans_symm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
⊢ LocalHomeomorph.trans
(LocalHomeomorph.trans (LocalHomeomorph.symm f) (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)))
(LocalHomeomorph.trans (Opens.localHomeomorphSubtypeCoe s) f') ≈
LocalHomeomorph.restr (LocalHomeomorph.trans (LocalHomeomorph.symm f) f')
(f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
[PROOFSTEP]
have openness₁ : IsOpen (f.target ∩ f.symm ⁻¹' s) := f.preimage_open_of_open_symm s.2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
⊢ LocalHomeomorph.trans
(LocalHomeomorph.trans (LocalHomeomorph.symm f) (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)))
(LocalHomeomorph.trans (Opens.localHomeomorphSubtypeCoe s) f') ≈
LocalHomeomorph.restr (LocalHomeomorph.trans (LocalHomeomorph.symm f) f')
(f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
[PROOFSTEP]
rw [← ofSet_trans _ openness₁, ← trans_assoc, ← trans_assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
⊢ LocalHomeomorph.trans
(LocalHomeomorph.trans
(LocalHomeomorph.trans (LocalHomeomorph.symm f) (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)))
(Opens.localHomeomorphSubtypeCoe s))
f' ≈
LocalHomeomorph.trans
(LocalHomeomorph.trans (ofSet (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) openness₁) (LocalHomeomorph.symm f))
f'
[PROOFSTEP]
refine'
EqOnSource.trans' _
(eqOnSource_refl _)
-- f' has been eliminated !!!
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
⊢ LocalHomeomorph.trans
(LocalHomeomorph.trans (LocalHomeomorph.symm f) (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)))
(Opens.localHomeomorphSubtypeCoe s) ≈
LocalHomeomorph.trans (ofSet (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) openness₁) (LocalHomeomorph.symm f)
[PROOFSTEP]
have sets_identity : f.symm.source ∩ (f.target ∩ f.symm ⁻¹' s) = f.symm.source ∩ f.symm ⁻¹' s := by mfld_set_tac
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
⊢ (LocalHomeomorph.symm f).toLocalEquiv.source ∩ (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) =
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s
[PROOFSTEP]
mfld_set_tac
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
sets_identity :
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) =
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s
⊢ LocalHomeomorph.trans
(LocalHomeomorph.trans (LocalHomeomorph.symm f) (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)))
(Opens.localHomeomorphSubtypeCoe s) ≈
LocalHomeomorph.trans (ofSet (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) openness₁) (LocalHomeomorph.symm f)
[PROOFSTEP]
have openness₂ : IsOpen (s : Set α) := s.2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
sets_identity :
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) =
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s
openness₂ : IsOpen ↑s
⊢ LocalHomeomorph.trans
(LocalHomeomorph.trans (LocalHomeomorph.symm f) (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)))
(Opens.localHomeomorphSubtypeCoe s) ≈
LocalHomeomorph.trans (ofSet (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) openness₁) (LocalHomeomorph.symm f)
[PROOFSTEP]
rw [ofSet_trans', sets_identity, ← trans_of_set' _ openness₂, trans_assoc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
sets_identity :
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) =
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s
openness₂ : IsOpen ↑s
⊢ LocalHomeomorph.trans (LocalHomeomorph.symm f)
(LocalHomeomorph.trans (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s))
(Opens.localHomeomorphSubtypeCoe s)) ≈
LocalHomeomorph.trans (LocalHomeomorph.symm f) (ofSet (↑s) openness₂)
[PROOFSTEP]
refine'
EqOnSource.trans' (eqOnSource_refl _)
_
-- f has been eliminated !!!
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
sets_identity :
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) =
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s
openness₂ : IsOpen ↑s
⊢ LocalHomeomorph.trans (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe s)) (Opens.localHomeomorphSubtypeCoe s) ≈
ofSet (↑s) openness₂
[PROOFSTEP]
refine' Setoid.trans (trans_symm_self s.localHomeomorphSubtypeCoe) _
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝ : Nonempty { x // x ∈ s }
f f' : LocalHomeomorph α β
openness₁ : IsOpen (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s)
sets_identity :
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ (f.target ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s) =
(LocalHomeomorph.symm f).toLocalEquiv.source ∩ ↑(LocalHomeomorph.symm f) ⁻¹' ↑s
openness₂ : IsOpen ↑s
⊢ ofSet (Opens.localHomeomorphSubtypeCoe s).toLocalEquiv.target
(_ : IsOpen (Opens.localHomeomorphSubtypeCoe s).toLocalEquiv.target) ≈
ofSet (↑s) openness₂
[PROOFSTEP]
simp only [mfld_simps, Setoid.refl]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
⊢ EqOn (↑(LocalHomeomorph.symm (subtypeRestr e V))) (inclusion hUV ∘ ↑(LocalHomeomorph.symm (subtypeRestr e U)))
(subtypeRestr e U).toLocalEquiv.target
[PROOFSTEP]
set i := Set.inclusion hUV
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
⊢ EqOn (↑(LocalHomeomorph.symm (subtypeRestr e V))) (i ∘ ↑(LocalHomeomorph.symm (subtypeRestr e U)))
(subtypeRestr e U).toLocalEquiv.target
[PROOFSTEP]
intro y hy
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ (subtypeRestr e U).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm (subtypeRestr e V)) y = (i ∘ ↑(LocalHomeomorph.symm (subtypeRestr e U))) y
[PROOFSTEP]
dsimp [LocalHomeomorph.subtypeRestr_def] at hy ⊢
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)) (↑(LocalHomeomorph.symm e) y) =
inclusion hUV (↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe U)) (↑(LocalHomeomorph.symm e) y))
[PROOFSTEP]
have hyV : e.symm y ∈ V.localHomeomorphSubtypeCoe.target :=
by
rw [Opens.localHomeomorphSubtypeCoe_target] at hy ⊢
exact hUV hy.2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
[PROOFSTEP]
rw [Opens.localHomeomorphSubtypeCoe_target] at hy ⊢
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' ↑U
⊢ ↑(LocalHomeomorph.symm e) y ∈ ↑V
[PROOFSTEP]
exact hUV hy.2
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)) (↑(LocalHomeomorph.symm e) y) =
inclusion hUV (↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe U)) (↑(LocalHomeomorph.symm e) y))
[PROOFSTEP]
refine' V.localHomeomorphSubtypeCoe.injOn _ trivial _
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)) (↑(LocalHomeomorph.symm e) y) ∈
(Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.source
[PROOFSTEP]
rw [← LocalHomeomorph.symm_target]
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)) (↑(LocalHomeomorph.symm e) y) ∈
(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)).toLocalEquiv.target
[PROOFSTEP]
apply LocalHomeomorph.map_source
[GOAL]
case refine'_1.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm e) y ∈ (LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)).toLocalEquiv.source
[PROOFSTEP]
rw [LocalHomeomorph.symm_source]
[GOAL]
case refine'_1.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
[PROOFSTEP]
exact hyV
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(Opens.localHomeomorphSubtypeCoe V)
(↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe V)) (↑(LocalHomeomorph.symm e) y)) =
↑(Opens.localHomeomorphSubtypeCoe V)
(inclusion hUV (↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe U)) (↑(LocalHomeomorph.symm e) y)))
[PROOFSTEP]
rw [V.localHomeomorphSubtypeCoe.right_inv hyV]
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm e) y =
↑(Opens.localHomeomorphSubtypeCoe V)
(inclusion hUV (↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe U)) (↑(LocalHomeomorph.symm e) y)))
[PROOFSTEP]
show _ = U.localHomeomorphSubtypeCoe _
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
e : LocalHomeomorph α β
s : Opens α
inst✝² : Nonempty { x // x ∈ s }
U V : Opens α
inst✝¹ : Nonempty { x // x ∈ U }
inst✝ : Nonempty { x // x ∈ V }
hUV : U ≤ V
i : ↑↑U → ↑↑V := inclusion hUV
y : β
hy : y ∈ e.target ∩ ↑(LocalHomeomorph.symm e) ⁻¹' (Opens.localHomeomorphSubtypeCoe U).toLocalEquiv.target
hyV : ↑(LocalHomeomorph.symm e) y ∈ (Opens.localHomeomorphSubtypeCoe V).toLocalEquiv.target
⊢ ↑(LocalHomeomorph.symm e) y =
↑(Opens.localHomeomorphSubtypeCoe U)
(↑(LocalHomeomorph.symm (Opens.localHomeomorphSubtypeCoe U)) (↑(LocalHomeomorph.symm e) y))
[PROOFSTEP]
rw [U.localHomeomorphSubtypeCoe.right_inv hy.2]
| {"mathlib_filename": "Mathlib.Topology.LocalHomeomorph", "llama_tokens": 30769} |
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) ≃ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
refine LinearEquiv.ofLinear (R := R) (R₂ := R) ?toFun ?invFun ?left ?right
[GOAL]
case toFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
refine lift ?_
[GOAL]
case toFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ (⨁ (i₁ : ι₁), M₁ i₁) →ₗ[R] (⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
refine DirectSum.toModule R _ _ fun i₁ => ?_
[GOAL]
case toFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
⊢ M₁ i₁ →ₗ[R] (⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
refine @LinearMap.flip R _ R _ R _ R _ _ _ _ _ _ _ _ _ _ _ _ _ _ ?_
[GOAL]
case toFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
⊢ (⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
refine DirectSum.toModule R _ _ fun i₂ => LinearMap.flip <| ?_
[GOAL]
case toFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
i₂ : ι₂
⊢ M₁ i₁ →ₗ[R] M₂ i₂ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
refine curry ?_
[GOAL]
case toFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
i₂ : ι₂
⊢ M₁ i₁ ⊗[R] M₂ i₂ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd
[PROOFSTEP]
exact DirectSum.lof R (ι₁ × ι₂) (fun i => M₁ i.1 ⊗[R] M₂ i.2) (i₁, i₂)
[GOAL]
case invFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ (⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) →ₗ[R] (⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂
[PROOFSTEP]
refine DirectSum.toModule R _ _ fun i => ?_
[GOAL]
case invFun
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁ × ι₂
⊢ M₁ i.fst ⊗[R] M₂ i.snd →ₗ[R] (⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂
[PROOFSTEP]
exact map (DirectSum.lof R _ M₁ i.1) (DirectSum.lof R _ M₂ i.2)
[GOAL]
case left
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ comp
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd)) =
LinearMap.id
[PROOFSTEP]
refine DirectSum.linearMap_ext R fun ⟨i₁, i₂⟩ => ?_
[GOAL]
case left
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x✝ : ι₁ × ι₂
i₁ : ι₁
i₂ : ι₂
⊢ comp
(comp
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd)))
(lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂)) =
comp LinearMap.id (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))
[PROOFSTEP]
refine TensorProduct.ext ?_
[GOAL]
case left
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x✝ : ι₁ × ι₂
i₁ : ι₁
i₂ : ι₂
⊢ compr₂ (mk R (M₁ (i₁, i₂).fst) (M₂ (i₁, i₂).snd))
(comp
(comp
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd)))
(lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))) =
compr₂ (mk R (M₁ (i₁, i₂).fst) (M₂ (i₁, i₂).snd))
(comp LinearMap.id (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂)))
[PROOFSTEP]
refine
LinearMap.ext₂ fun m₁ m₂ =>
?_
-- porting note: seems much nicer than the `repeat` lean 3 proof.
[GOAL]
case left
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x✝ : ι₁ × ι₂
i₁ : ι₁
i₂ : ι₂
m₁ : M₁ (i₁, i₂).fst
m₂ : M₂ (i₁, i₂).snd
⊢ ↑(↑(compr₂ (mk R (M₁ (i₁, i₂).fst) (M₂ (i₁, i₂).snd))
(comp
(comp
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd)))
(lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))
m₁)
m₂ =
↑(↑(compr₂ (mk R (M₁ (i₁, i₂).fst) (M₂ (i₁, i₂).snd))
(comp LinearMap.id (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))
m₁)
m₂
[PROOFSTEP]
simp only [compr₂_apply, comp_apply, id_apply, mk_apply, DirectSum.toModule_lof, map_tmul, lift.tmul, flip_apply,
curry_apply]
[GOAL]
case right
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ comp
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd))
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂)))))) =
LinearMap.id
[PROOFSTEP]
refine TensorProduct.ext ?_
[GOAL]
case right
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
⊢ compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂))
(comp
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd))
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))) =
compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂)) LinearMap.id
[PROOFSTEP]
refine @DirectSum.linearMap_ext R _ _ _ _ _ _ _ _ (_) _ _ fun i₁ => ?_
[GOAL]
case right
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
⊢ comp
(compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂))
(comp
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd))
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))))
(lof R ι₁ (fun i => M₁ i) i₁) =
comp (compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂)) LinearMap.id) (lof R ι₁ (fun i => M₁ i) i₁)
[PROOFSTEP]
refine @LinearMap.ext _ _ _ _ _ _ _ _ (_) (_) _ _ _ fun x₁ => ?_
[GOAL]
case right
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
x₁ : M₁ i₁
⊢ ↑(comp
(compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂))
(comp
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd))
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))))
(lof R ι₁ (fun i => M₁ i) i₁))
x₁ =
↑(comp (compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂)) LinearMap.id) (lof R ι₁ (fun i => M₁ i) i₁)) x₁
[PROOFSTEP]
refine @DirectSum.linearMap_ext R _ _ _ _ _ _ _ _ (_) _ _ fun i₂ => ?_
[GOAL]
case right
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
x₁ : M₁ i₁
i₂ : ι₂
⊢ comp
(↑(comp
(compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂))
(comp
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd))
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))))
(lof R ι₁ (fun i => M₁ i) i₁))
x₁)
(lof R ι₂ (fun i => M₂ i) i₂) =
comp
(↑(comp (compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂)) LinearMap.id) (lof R ι₁ (fun i => M₁ i) i₁)) x₁)
(lof R ι₂ (fun i => M₂ i) i₂)
[PROOFSTEP]
refine
LinearMap.ext fun x₂ =>
?_
-- porting note: seems much nicer than the `repeat` lean 3 proof.
[GOAL]
case right
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
x₁ : M₁ i₁
i₂ : ι₂
x₂ : M₂ i₂
⊢ ↑(comp
(↑(comp
(compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂))
(comp
(toModule R (ι₁ × ι₂) ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] ⨁ (i₂ : ι₂), M₂ i₂) fun i =>
map (lof R ι₁ M₁ i.fst) (lof R ι₂ M₂ i.snd))
(lift
(toModule R ι₁ ((⨁ (i₂ : ι₂), M₂ i₂) →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₁ =>
LinearMap.flip
(toModule R ι₂ (M₁ i₁ →ₗ[R] ⨁ (i : ι₁ × ι₂), M₁ i.fst ⊗[R] M₂ i.snd) fun i₂ =>
LinearMap.flip (curry (lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂))))))))
(lof R ι₁ (fun i => M₁ i) i₁))
x₁)
(lof R ι₂ (fun i => M₂ i) i₂))
x₂ =
↑(comp
(↑(comp (compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) (⨁ (i₂ : ι₂), M₂ i₂)) LinearMap.id) (lof R ι₁ (fun i => M₁ i) i₁))
x₁)
(lof R ι₂ (fun i => M₂ i) i₂))
x₂
[PROOFSTEP]
simp only [compr₂_apply, comp_apply, id_apply, mk_apply, DirectSum.toModule_lof, map_tmul, lift.tmul, flip_apply,
curry_apply]
/- was:
refine'
LinearEquiv.ofLinear
(lift <|
DirectSum.toModule R _ _ fun i₁ => LinearMap.flip <| DirectSum.toModule R _ _ fun i₂ =>
LinearMap.flip <| curry <|
DirectSum.lof R (ι₁ × ι₂) (fun i => M₁ i.1 ⊗[R] M₂ i.2) (i₁, i₂))
(DirectSum.toModule R _ _ fun i => map (DirectSum.lof R _ _ _) (DirectSum.lof R _ _ _)) _
_ <;>
[ext ⟨i₁, i₂⟩ x₁ x₂ : 4, ext i₁ i₂ x₁ x₂ : 5]
repeat'
first
|rw [compr₂_apply]|rw [comp_apply]|rw [id_apply]|rw [mk_apply]|rw [DirectSum.toModule_lof]
|rw [map_tmul]|rw [lift.tmul]|rw [flip_apply]|rw [curry_apply]
-/
/- alternative with explicit types:
refine'
LinearEquiv.ofLinear
(lift <|
DirectSum.toModule
(R := R) (M := M₁) (N := (⨁ i₂, M₂ i₂) →ₗ[R] ⨁ i : ι₁ × ι₂, M₁ i.1 ⊗[R] M₂ i.2)
(φ := fun i₁ => LinearMap.flip <|
DirectSum.toModule (R := R) (M := M₂) (N := ⨁ i : ι₁ × ι₂, M₁ i.1 ⊗[R] M₂ i.2)
(φ := fun i₂ => LinearMap.flip <| curry <|
DirectSum.lof R (ι₁ × ι₂) (fun i => M₁ i.1 ⊗[R] M₂ i.2) (i₁, i₂))))
(DirectSum.toModule
(R := R)
(M := fun i : ι₁ × ι₂ => M₁ i.1 ⊗[R] M₂ i.2)
(N := (⨁ i₁, M₁ i₁) ⊗[R] ⨁ i₂, M₂ i₂)
(φ := fun i : ι₁ × ι₂ => map (DirectSum.lof R _ M₁ i.1) (DirectSum.lof R _ M₂ i.2))) _
_ <;>
[ext ⟨i₁, i₂⟩ x₁ x₂ : 4, ext i₁ i₂ x₁ x₂ : 5]
repeat'
first
|rw [compr₂_apply]|rw [comp_apply]|rw [id_apply]|rw [mk_apply]|rw [DirectSum.toModule_lof]
|rw [map_tmul]|rw [lift.tmul]|rw [flip_apply]|rw [curry_apply]
-/
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
m₁ : M₁ i
m₂ : M₂'
⊢ ↑(↑(compr₂ (mk R (M₁ i) M₂')
(comp
(comp
(lift
(toModule R ι₁ (M₂' →ₗ[R] ⨁ (i : ι₁), M₁ i ⊗[R] M₂') fun i =>
compr₂ (mk R (M₁ i) M₂') (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i)))
(toModule R ι₁ ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] M₂') fun i => rTensor M₂' (lof R ι₁ M₁ i)))
(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i)))
m₁)
m₂ =
↑(↑(compr₂ (mk R (M₁ i) M₂') (comp LinearMap.id (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i))) m₁) m₂
[PROOFSTEP]
dsimp only [comp_apply, compr₂_apply, id_apply, mk_apply]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
m₁ : M₁ i
m₂ : M₂'
⊢ ↑(lift
(toModule R ι₁ (M₂' →ₗ[R] ⨁ (i : ι₁), M₁ i ⊗[R] M₂') fun i =>
compr₂ (mk R (M₁ i) M₂') (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i)))
(↑(toModule R ι₁ ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] M₂') fun i => rTensor M₂' (lof R ι₁ M₁ i))
(↑(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i) (m₁ ⊗ₜ[R] m₂))) =
↑(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i) (m₁ ⊗ₜ[R] m₂)
[PROOFSTEP]
simp_rw [DirectSum.toModule_lof, rTensor_tmul, lift.tmul, DirectSum.toModule_lof, compr₂_apply, mk_apply]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
m₁ : M₁ i
m₂ : M₂'
⊢ ↑(↑(comp
(compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) M₂')
(comp (toModule R ι₁ ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] M₂') fun i => rTensor M₂' (lof R ι₁ M₁ i))
(lift
(toModule R ι₁ (M₂' →ₗ[R] ⨁ (i : ι₁), M₁ i ⊗[R] M₂') fun i =>
compr₂ (mk R (M₁ i) M₂') (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i)))))
(lof R ι₁ (fun i => M₁ i) i))
m₁)
m₂ =
↑(↑(comp (compr₂ (mk R (⨁ (i₁ : ι₁), M₁ i₁) M₂') LinearMap.id) (lof R ι₁ (fun i => M₁ i) i)) m₁) m₂
[PROOFSTEP]
dsimp only [comp_apply, compr₂_apply, id_apply, mk_apply]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
m₁ : M₁ i
m₂ : M₂'
⊢ ↑(toModule R ι₁ ((⨁ (i₁ : ι₁), M₁ i₁) ⊗[R] M₂') fun i => rTensor M₂' (lof R ι₁ M₁ i))
(↑(lift
(toModule R ι₁ (M₂' →ₗ[R] ⨁ (i : ι₁), M₁ i ⊗[R] M₂') fun i =>
compr₂ (mk R (M₁ i) M₂') (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i)))
(↑(lof R ι₁ (fun i => M₁ i) i) m₁ ⊗ₜ[R] m₂)) =
↑(lof R ι₁ (fun i => M₁ i) i) m₁ ⊗ₜ[R] m₂
[PROOFSTEP]
simp_rw [lift.tmul, DirectSum.toModule_lof, compr₂_apply, mk_apply, DirectSum.toModule_lof, rTensor_tmul]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i₁ : ι₁
m₁ : M₁ i₁
i₂ : ι₂
m₂ : M₂ i₂
⊢ ↑(TensorProduct.directSum R M₁ M₂) (↑(lof R ι₁ M₁ i₁) m₁ ⊗ₜ[R] ↑(lof R ι₂ M₂ i₂) m₂) =
↑(lof R (ι₁ × ι₂) (fun i => M₁ i.fst ⊗[R] M₂ i.snd) (i₁, i₂)) (m₁ ⊗ₜ[R] m₂)
[PROOFSTEP]
simp [TensorProduct.directSum]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
x : M₁ i
y : M₂'
⊢ ↑(directSumLeft R M₁ M₂') (↑(lof R ι₁ M₁ i) x ⊗ₜ[R] y) = ↑(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i) (x ⊗ₜ[R] y)
[PROOFSTEP]
dsimp only [directSumLeft, LinearEquiv.ofLinear_apply, lift.tmul]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
x : M₁ i
y : M₂'
⊢ ↑(↑(toModule R ι₁ (M₂' →ₗ[R] ⨁ (i : ι₁), M₁ i ⊗[R] M₂') fun i =>
compr₂ (mk R (M₁ i) M₂') (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i))
(↑(lof R ι₁ M₁ i) x))
y =
↑(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i) (x ⊗ₜ[R] y)
[PROOFSTEP]
rw [DirectSum.toModule_lof R i]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
x : M₁ i
y : M₂'
⊢ ↑(↑(compr₂ (mk R (M₁ i) M₂') (lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i)) x) y =
↑(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i) (x ⊗ₜ[R] y)
[PROOFSTEP]
rfl
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
i : ι₁
x : M₁ i
y : M₂'
⊢ ↑(LinearEquiv.symm (directSumLeft R M₁ M₂')) (↑(lof R ι₁ (fun i => M₁ i ⊗[R] M₂') i) (x ⊗ₜ[R] y)) =
↑(lof R ι₁ M₁ i) x ⊗ₜ[R] y
[PROOFSTEP]
rw [LinearEquiv.symm_apply_eq, directSumLeft_tmul_lof]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x : M₁'
i : ι₂
y : M₂ i
⊢ ↑(directSumRight R M₁' M₂) (x ⊗ₜ[R] ↑(lof R ι₂ M₂ i) y) = ↑(lof R ι₂ (fun i => M₁' ⊗[R] M₂ i) i) (x ⊗ₜ[R] y)
[PROOFSTEP]
dsimp only [directSumRight, LinearEquiv.trans_apply, TensorProduct.comm_tmul]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x : M₁'
i : ι₂
y : M₂ i
⊢ ↑(DFinsupp.mapRange.linearEquiv fun x => TensorProduct.comm R (M₂ x) M₁')
(↑(directSumLeft R M₂ M₁') (↑(lof R ι₂ M₂ i) y ⊗ₜ[R] x)) =
↑(lof R ι₂ (fun i => M₁' ⊗[R] M₂ i) i) (x ⊗ₜ[R] y)
[PROOFSTEP]
rw [directSumLeft_tmul_lof]
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x : M₁'
i : ι₂
y : M₂ i
⊢ ↑(DFinsupp.mapRange.linearEquiv fun x => TensorProduct.comm R (M₂ x) M₁')
(↑(lof R ι₂ (fun i => M₂ i ⊗[R] M₁') i) (y ⊗ₜ[R] x)) =
↑(lof R ι₂ (fun i => M₁' ⊗[R] M₂ i) i) (x ⊗ₜ[R] y)
[PROOFSTEP]
exact DFinsupp.mapRange_single (hf := fun _ => rfl)
[GOAL]
R : Type u
inst✝¹⁰ : CommRing R
ι₁ : Type v₁
ι₂ : Type v₂
inst✝⁹ : DecidableEq ι₁
inst✝⁸ : DecidableEq ι₂
M₁ : ι₁ → Type w₁
M₁' : Type w₁'
M₂ : ι₂ → Type w₂
M₂' : Type w₂'
inst✝⁷ : (i₁ : ι₁) → AddCommGroup (M₁ i₁)
inst✝⁶ : AddCommGroup M₁'
inst✝⁵ : (i₂ : ι₂) → AddCommGroup (M₂ i₂)
inst✝⁴ : AddCommGroup M₂'
inst✝³ : (i₁ : ι₁) → Module R (M₁ i₁)
inst✝² : Module R M₁'
inst✝¹ : (i₂ : ι₂) → Module R (M₂ i₂)
inst✝ : Module R M₂'
x : M₁'
i : ι₂
y : M₂ i
⊢ ↑(LinearEquiv.symm (directSumRight R M₁' M₂)) (↑(lof R ι₂ (fun i => M₁' ⊗[R] M₂ i) i) (x ⊗ₜ[R] y)) =
x ⊗ₜ[R] ↑(lof R ι₂ M₂ i) y
[PROOFSTEP]
rw [LinearEquiv.symm_apply_eq, directSumRight_tmul_lof]
| {"mathlib_filename": "Mathlib.LinearAlgebra.DirectSum.TensorProduct", "llama_tokens": 16937} |
{"mathlib_filename": "Mathlib.Topology.LocalExtr", "llama_tokens": 0} |
|
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
x✝ : Set C(α, β)
⊢ x✝ ∈ {m | ∃ s x u x, m = CompactOpen.gen s u} ↔ x✝ ∈ image2 CompactOpen.gen {s | IsCompact s} {t | IsOpen t}
[PROOFSTEP]
simp [eq_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
⊢ CompactOpen.gen s u ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
dsimp [mem_setOf_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
⊢ ∃ s_1 x u_1 x, CompactOpen.gen s u = CompactOpen.gen s_1 u_1
[PROOFSTEP]
tauto
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
s : Set α
u : Set γ
⊢ comp g ⁻¹' CompactOpen.gen s u = CompactOpen.gen s (↑g ⁻¹' u)
[PROOFSTEP]
ext ⟨f, _⟩
[GOAL]
case h.mk
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
s : Set α
u : Set γ
f : α → β
continuous_toFun✝ : Continuous f
⊢ mk f ∈ comp g ⁻¹' CompactOpen.gen s u ↔ mk f ∈ CompactOpen.gen s (↑g ⁻¹' u)
[PROOFSTEP]
change g ∘ f '' s ⊆ u ↔ f '' s ⊆ g ⁻¹' u
[GOAL]
case h.mk
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
s : Set α
u : Set γ
f : α → β
continuous_toFun✝ : Continuous f
⊢ ↑g ∘ f '' s ⊆ u ↔ f '' s ⊆ ↑g ⁻¹' u
[PROOFSTEP]
rw [image_comp, image_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
m : Set C(α, γ)
x✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}
s : Set α
hs : IsCompact s
u : Set γ
hu : IsOpen u
hm : m = CompactOpen.gen s u
⊢ IsOpen (comp g ⁻¹' m)
[PROOFSTEP]
rw [hm, preimage_gen g]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
m : Set C(α, γ)
x✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}
s : Set α
hs : IsCompact s
u : Set γ
hu : IsOpen u
hm : m = CompactOpen.gen s u
⊢ IsOpen (CompactOpen.gen s (↑g ⁻¹' u))
[PROOFSTEP]
exact ContinuousMap.isOpen_gen hs (hu.preimage g.2)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
hg : Inducing ↑g
⊢ compactOpen = TopologicalSpace.induced (comp g) compactOpen
[PROOFSTEP]
simp only [compactOpen_eq, induced_generateFrom_eq, image_image2, preimage_gen, hg.setOf_isOpen, image2_image_right]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
s : Set α
x✝¹ : IsCompact s
u : Set γ
x✝ : IsOpen u
⊢ (fun g => comp g f) ⁻¹' CompactOpen.gen s u = CompactOpen.gen (↑f '' s) u
[PROOFSTEP]
ext ⟨g, _⟩
[GOAL]
case h.mk
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g✝ : C(β, γ)
f : C(α, β)
s : Set α
x✝¹ : IsCompact s
u : Set γ
x✝ : IsOpen u
g : β → γ
continuous_toFun✝ : Continuous g
⊢ mk g ∈ (fun g => comp g f) ⁻¹' CompactOpen.gen s u ↔ mk g ∈ CompactOpen.gen (↑f '' s) u
[PROOFSTEP]
change g ∘ f '' s ⊆ u ↔ g '' (f '' s) ⊆ u
[GOAL]
case h.mk
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g✝ : C(β, γ)
f : C(α, β)
s : Set α
x✝¹ : IsCompact s
u : Set γ
x✝ : IsOpen u
g : β → γ
continuous_toFun✝ : Continuous g
⊢ g ∘ ↑f '' s ⊆ u ↔ g '' (↑f '' s) ⊆ u
[PROOFSTEP]
rw [Set.image_comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
m : Set C(α, γ)
x✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}
s : Set α
hs : IsCompact s
u : Set γ
hu : IsOpen u
hm : m = CompactOpen.gen s u
⊢ IsOpen ((fun g => comp g f) ⁻¹' m)
[PROOFSTEP]
rw [hm, image_gen f hs hu]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
m : Set C(α, γ)
x✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}
s : Set α
hs : IsCompact s
u : Set γ
hu : IsOpen u
hm : m = CompactOpen.gen s u
⊢ IsOpen (CompactOpen.gen (↑f '' s) u)
[PROOFSTEP]
exact ContinuousMap.isOpen_gen (hs.image f.2) hu
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
⊢ ∀ (s : Set C(α, γ)), s ∈ {m | ∃ s x u x, m = CompactOpen.gen s u} → IsOpen ((fun x => comp x.snd x.fst) ⁻¹' s)
[PROOFSTEP]
rintro M ⟨K, hK, U, hU, rfl⟩
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
⊢ IsOpen ((fun x => comp x.snd x.fst) ⁻¹' CompactOpen.gen K U)
[PROOFSTEP]
conv =>
congr
rw [CompactOpen.gen, preimage_setOf_eq]
--congr
ext; dsimp [setOf]
rw [image_comp, image_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
| IsOpen ((fun x => comp x.snd x.fst) ⁻¹' CompactOpen.gen K U)
[PROOFSTEP]
congr
rw [CompactOpen.gen, preimage_setOf_eq]
--congr
ext; dsimp [setOf]
rw [image_comp, image_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
| IsOpen ((fun x => comp x.snd x.fst) ⁻¹' CompactOpen.gen K U)
[PROOFSTEP]
congr
rw [CompactOpen.gen, preimage_setOf_eq]
--congr
ext; dsimp [setOf]
rw [image_comp, image_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
| IsOpen ((fun x => comp x.snd x.fst) ⁻¹' CompactOpen.gen K U)
[PROOFSTEP]
congr
[GOAL]
case a
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
| (fun x => comp x.snd x.fst) ⁻¹' CompactOpen.gen K U
[PROOFSTEP]
rw [CompactOpen.gen, preimage_setOf_eq]
--congr
[GOAL]
case a
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
| {a | ↑(comp a.snd a.fst) '' K ⊆ U}
[PROOFSTEP]
ext
[GOAL]
case a.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
x✝ : C(α, β) × C(β, γ)
| setOf (fun a => ↑(comp a.snd a.fst) '' K ⊆ U) x✝
[PROOFSTEP]
dsimp [setOf]
[GOAL]
case a.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
x✝ : C(α, β) × C(β, γ)
| ↑x✝.snd ∘ ↑x✝.fst '' K ⊆ U
[PROOFSTEP]
rw [image_comp, image_subset_iff]
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
⊢ IsOpen fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U
[PROOFSTEP]
rw [isOpen_iff_forall_mem_open]
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
⊢ ∀ (x : C(α, β) × C(β, γ)),
(x ∈ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U) → ∃ t, (t ⊆ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U) ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
rintro ⟨φ₀, ψ₀⟩ H
[GOAL]
case intro.intro.intro.intro.mk
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
φ₀ : C(α, β)
ψ₀ : C(β, γ)
H : (φ₀, ψ₀) ∈ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U
⊢ ∃ t, (t ⊆ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U) ∧ IsOpen t ∧ (φ₀, ψ₀) ∈ t
[PROOFSTEP]
obtain ⟨L, hL, hKL, hLU⟩ := exists_compact_between (hK.image φ₀.2) (hU.preimage ψ₀.2) H
[GOAL]
case intro.intro.intro.intro.mk.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
φ₀ : C(α, β)
ψ₀ : C(β, γ)
H : (φ₀, ψ₀) ∈ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U
L : Set β
hL : IsCompact L
hKL : φ₀.toFun '' K ⊆ interior L
hLU : L ⊆ ψ₀.toFun ⁻¹' U
⊢ ∃ t, (t ⊆ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U) ∧ IsOpen t ∧ (φ₀, ψ₀) ∈ t
[PROOFSTEP]
use{φ : C(α, β) | φ '' K ⊆ interior L} ×ˢ
{ψ : C(β, γ) | ψ '' L ⊆ U}
-- porting note: typing hint `: φ '' K ⊆ interior L` wasn't previously required
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
φ₀ : C(α, β)
ψ₀ : C(β, γ)
H : (φ₀, ψ₀) ∈ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U
L : Set β
hL : IsCompact L
hKL : φ₀.toFun '' K ⊆ interior L
hLU : L ⊆ ψ₀.toFun ⁻¹' U
⊢ ({φ | ↑φ '' K ⊆ interior L} ×ˢ {ψ | ↑ψ '' L ⊆ U} ⊆ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U) ∧
IsOpen ({φ | ↑φ '' K ⊆ interior L} ×ˢ {ψ | ↑ψ '' L ⊆ U}) ∧
(φ₀, ψ₀) ∈ {φ | ↑φ '' K ⊆ interior L} ×ˢ {ψ | ↑ψ '' L ⊆ U}
[PROOFSTEP]
use fun ⟨φ, ψ⟩ ⟨(hφ : φ '' K ⊆ interior L), hψ⟩ => subset_trans hφ (interior_subset.trans <| image_subset_iff.mp hψ)
[GOAL]
case right
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
φ₀ : C(α, β)
ψ₀ : C(β, γ)
H : (φ₀, ψ₀) ∈ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U
L : Set β
hL : IsCompact L
hKL : φ₀.toFun '' K ⊆ interior L
hLU : L ⊆ ψ₀.toFun ⁻¹' U
⊢ IsOpen ({φ | ↑φ '' K ⊆ interior L} ×ˢ {ψ | ↑ψ '' L ⊆ U}) ∧ (φ₀, ψ₀) ∈ {φ | ↑φ '' K ⊆ interior L} ×ˢ {ψ | ↑ψ '' L ⊆ U}
[PROOFSTEP]
use(ContinuousMap.isOpen_gen hK isOpen_interior).prod (ContinuousMap.isOpen_gen hL hU)
[GOAL]
case right
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
g : C(β, γ)
f : C(α, β)
inst✝ : LocallyCompactSpace β
K : Set α
hK : IsCompact K
U : Set γ
hU : IsOpen U
φ₀ : C(α, β)
ψ₀ : C(β, γ)
H : (φ₀, ψ₀) ∈ fun x => ↑x.fst '' K ⊆ ↑x.snd ⁻¹' U
L : Set β
hL : IsCompact L
hKL : φ₀.toFun '' K ⊆ interior L
hLU : L ⊆ ψ₀.toFun ⁻¹' U
⊢ (φ₀, ψ₀) ∈ {φ | ↑φ '' K ⊆ interior L} ×ˢ {ψ | ↑ψ '' L ⊆ U}
[PROOFSTEP]
exact mem_prod.mpr ⟨hKL, image_subset_iff.mpr hLU⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace α
x✝ : C(α, β) × α
n : Set β
f : C(α, β)
x : α
hn : n ∈ 𝓝 (↑(f, x).fst (f, x).snd)
v : Set β
vn : v ⊆ n
vo : IsOpen v
fxv : ↑(f, x).fst (f, x).snd ∈ v
this✝² : v ∈ 𝓝 (↑f x)
s : Set α
hs : s ∈ 𝓝 x
sv : s ⊆ ↑f ⁻¹' v
sc : IsCompact s
u : Set α
us : u ⊆ s
uo : IsOpen u
xu : x ∈ u
w : Set (C(α, β) × α) := CompactOpen.gen s v ×ˢ u
this✝¹ : w ⊆ (fun p => ↑p.fst p.snd) ⁻¹' n
this✝ : IsOpen w
this : (f, x) ∈ w
⊢ w ⊆ (fun p => ↑p.fst p.snd) ⁻¹' n
[PROOFSTEP]
assumption
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace α
x✝ : C(α, β) × α
n : Set β
f : C(α, β)
x : α
hn : n ∈ 𝓝 (↑(f, x).fst (f, x).snd)
v : Set β
vn : v ⊆ n
vo : IsOpen v
fxv : ↑(f, x).fst (f, x).snd ∈ v
this✝² : v ∈ 𝓝 (↑f x)
s : Set α
hs : s ∈ 𝓝 x
sv : s ⊆ ↑f ⁻¹' v
sc : IsCompact s
u : Set α
us : u ⊆ s
uo : IsOpen u
xu : x ∈ u
w : Set (C(α, β) × α) := CompactOpen.gen s v ×ˢ u
this✝¹ : w ⊆ (fun p => ↑p.fst p.snd) ⁻¹' n
this✝ : IsOpen w
this : (f, x) ∈ w
⊢ IsOpen w
[PROOFSTEP]
assumption
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace α
x✝ : C(α, β) × α
n : Set β
f : C(α, β)
x : α
hn : n ∈ 𝓝 (↑(f, x).fst (f, x).snd)
v : Set β
vn : v ⊆ n
vo : IsOpen v
fxv : ↑(f, x).fst (f, x).snd ∈ v
this✝² : v ∈ 𝓝 (↑f x)
s : Set α
hs : s ∈ 𝓝 x
sv : s ⊆ ↑f ⁻¹' v
sc : IsCompact s
u : Set α
us : u ⊆ s
uo : IsOpen u
xu : x ∈ u
w : Set (C(α, β) × α) := CompactOpen.gen s v ×ˢ u
this✝¹ : w ⊆ (fun p => ↑p.fst p.snd) ⁻¹' n
this✝ : IsOpen w
this : (f, x) ∈ w
⊢ (f, x) ∈ w
[PROOFSTEP]
assumption
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
a : α
⊢ Continuous fun f => ↑f a
[PROOFSTEP]
refine continuous_def.2 fun U hU ↦ ?_
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
a : α
U : Set ((fun x => β) a)
hU : IsOpen U
⊢ IsOpen ((fun f => ↑f a) ⁻¹' U)
[PROOFSTEP]
convert ContinuousMap.isOpen_gen (isCompact_singleton (a := a)) hU using 1
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
a : α
U : Set ((fun x => β) a)
hU : IsOpen U
⊢ (fun f => ↑f a) ⁻¹' U = CompactOpen.gen {a} U
[PROOFSTEP]
ext
[GOAL]
case h.e'_3.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
a : α
U : Set ((fun x => β) a)
hU : IsOpen U
x✝ : C(α, β)
⊢ x✝ ∈ (fun f => ↑f a) ⁻¹' U ↔ x✝ ∈ CompactOpen.gen {a} U
[PROOFSTEP]
simp [CompactOpen.gen]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
⊢ compactOpen ≤ TopologicalSpace.induced (restrict s) compactOpen
[PROOFSTEP]
simp only [induced_generateFrom_eq, ContinuousMap.compactOpen]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
⊢ TopologicalSpace.generateFrom {m | ∃ s x u x, m = CompactOpen.gen s u} ≤
TopologicalSpace.generateFrom (preimage (restrict s) '' {m | ∃ s_1 x u x, m = CompactOpen.gen s_1 u})
[PROOFSTEP]
apply TopologicalSpace.generateFrom_anti
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
⊢ preimage (restrict s) '' {m | ∃ s_1 x u x, m = CompactOpen.gen s_1 u} ⊆ {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
rintro b ⟨a, ⟨c, hc, u, hu, rfl⟩, rfl⟩
[GOAL]
case h.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
c : Set ↑s
hc : IsCompact c
u : Set β
hu : IsOpen u
⊢ restrict s ⁻¹' CompactOpen.gen c u ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
refine' ⟨(↑) '' c, hc.image continuous_subtype_val, u, hu, _⟩
[GOAL]
case h.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
c : Set ↑s
hc : IsCompact c
u : Set β
hu : IsOpen u
⊢ restrict s ⁻¹' CompactOpen.gen c u = CompactOpen.gen (Subtype.val '' c) u
[PROOFSTEP]
ext f
[GOAL]
case h.intro.intro.intro.intro.intro.intro.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
c : Set ↑s
hc : IsCompact c
u : Set β
hu : IsOpen u
f : C(α, β)
⊢ f ∈ restrict s ⁻¹' CompactOpen.gen c u ↔ f ∈ CompactOpen.gen (Subtype.val '' c) u
[PROOFSTEP]
simp only [CompactOpen.gen, mem_setOf_eq, mem_preimage, ContinuousMap.coe_restrict]
[GOAL]
case h.intro.intro.intro.intro.intro.intro.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
c : Set ↑s
hc : IsCompact c
u : Set β
hu : IsOpen u
f : C(α, β)
⊢ (fun a => (↑f ∘ Subtype.val) a) '' c ⊆ u ↔ (fun a => ↑f a) '' (Subtype.val '' c) ⊆ u
[PROOFSTEP]
rw [image_comp f ((↑) : s → α)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ compactOpen = ⨅ (s : Set α) (_ : IsCompact s), TopologicalSpace.induced (restrict s) compactOpen
[PROOFSTEP]
refine' le_antisymm _ _
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ compactOpen ≤ ⨅ (s : Set α) (_ : IsCompact s), TopologicalSpace.induced (restrict s) compactOpen
[PROOFSTEP]
refine' le_iInf₂ _
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ ∀ (i : Set α), IsCompact i → compactOpen ≤ TopologicalSpace.induced (restrict i) compactOpen
[PROOFSTEP]
exact fun s _ => compactOpen_le_induced s
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ ⨅ (s : Set α) (_ : IsCompact s), TopologicalSpace.induced (restrict s) compactOpen ≤ compactOpen
[PROOFSTEP]
simp only [← generateFrom_iUnion, induced_generateFrom_eq, ContinuousMap.compactOpen]
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ TopologicalSpace.generateFrom
(⋃ (i : Set α) (_ : IsCompact i), preimage (restrict i) '' {m | ∃ s x u x, m = CompactOpen.gen s u}) ≤
TopologicalSpace.generateFrom {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
apply TopologicalSpace.generateFrom_anti
[GOAL]
case refine'_2.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ {m | ∃ s x u x, m = CompactOpen.gen s u} ⊆
⋃ (i : Set α) (_ : IsCompact i), preimage (restrict i) '' {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
rintro _ ⟨s, hs, u, hu, rfl⟩
[GOAL]
case refine'_2.h.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
⊢ CompactOpen.gen s u ∈
⋃ (i : Set α) (_ : IsCompact i), preimage (restrict i) '' {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
rw [mem_iUnion₂]
[GOAL]
case refine'_2.h.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
⊢ ∃ i j, CompactOpen.gen s u ∈ preimage (restrict i) '' {m | ∃ s x u x, m = CompactOpen.gen s u}
[PROOFSTEP]
refine' ⟨s, hs, _, ⟨univ, isCompact_iff_isCompact_univ.mp hs, u, hu, rfl⟩, _⟩
[GOAL]
case refine'_2.h.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
⊢ restrict s ⁻¹' CompactOpen.gen univ u = CompactOpen.gen s u
[PROOFSTEP]
ext f
[GOAL]
case refine'_2.h.intro.intro.intro.intro.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
f : C(α, β)
⊢ f ∈ restrict s ⁻¹' CompactOpen.gen univ u ↔ f ∈ CompactOpen.gen s u
[PROOFSTEP]
simp only [CompactOpen.gen, mem_setOf_eq, mem_preimage, ContinuousMap.coe_restrict]
[GOAL]
case refine'_2.h.intro.intro.intro.intro.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
f : C(α, β)
⊢ (fun a => (↑f ∘ Subtype.val) a) '' univ ⊆ u ↔ (fun a => ↑f a) '' s ⊆ u
[PROOFSTEP]
rw [image_comp f ((↑) : s → α)]
[GOAL]
case refine'_2.h.intro.intro.intro.intro.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsCompact s
u : Set β
hu : IsOpen u
f : C(α, β)
⊢ ↑f '' (Subtype.val '' univ) ⊆ u ↔ (fun a => ↑f a) '' s ⊆ u
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
⊢ Continuous fun F => restrict s F
[PROOFSTEP]
rw [continuous_iff_le_induced]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
⊢ compactOpen ≤ TopologicalSpace.induced (fun F => restrict s F) compactOpen
[PROOFSTEP]
exact compactOpen_le_induced s
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : C(α, β)
⊢ 𝓝 f = ⨅ (s : Set α) (_ : IsCompact s), Filter.comap (restrict s) (𝓝 (restrict s f))
[PROOFSTEP]
rw [compactOpen_eq_sInf_induced]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : C(α, β)
⊢ 𝓝 f = ⨅ (s : Set α) (_ : IsCompact s), Filter.comap (restrict s) (𝓝 (restrict s f))
[PROOFSTEP]
simp [nhds_iInf, nhds_induced]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
ι : Type u_4
l : Filter ι
F : ι → C(α, β)
f : C(α, β)
⊢ Filter.Tendsto F l (𝓝 f) ↔
∀ (s : Set α), IsCompact s → Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (restrict s f))
[PROOFSTEP]
rw [compactOpen_eq_sInf_induced]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
ι : Type u_4
l : Filter ι
F : ι → C(α, β)
f : C(α, β)
⊢ Filter.Tendsto F l (𝓝 f) ↔
∀ (s : Set α), IsCompact s → Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (restrict s f))
[PROOFSTEP]
simp [nhds_iInf, nhds_induced, Filter.tendsto_comap_iff, Function.comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
⊢ (∃ f, Filter.Tendsto F l (𝓝 f)) ↔ ∀ (s : Set α), IsCompact s → ∃ f, Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 f)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
⊢ (∃ f, Filter.Tendsto F l (𝓝 f)) → ∀ (s : Set α), IsCompact s → ∃ f, Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 f)
[PROOFSTEP]
rintro ⟨f, hf⟩ s _
[GOAL]
case mp.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : C(α, β)
hf : Filter.Tendsto F l (𝓝 f)
s : Set α
hs✝ : IsCompact s
⊢ ∃ f, Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 f)
[PROOFSTEP]
exact ⟨f.restrict s, tendsto_compactOpen_restrict hf s⟩
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
⊢ (∀ (s : Set α), IsCompact s → ∃ f, Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 f)) → ∃ f, Filter.Tendsto F l (𝓝 f)
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
h : ∀ (s : Set α), IsCompact s → ∃ f, Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 f)
⊢ ∃ f, Filter.Tendsto F l (𝓝 f)
[PROOFSTEP]
choose f hf using h
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
⊢ ∃ f, Filter.Tendsto F l (𝓝 f)
[PROOFSTEP]
have h :
∀ (s₁) (hs₁ : IsCompact s₁) (s₂) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
f s₁ hs₁ ⟨x, hxs₁⟩ = f s₂ hs₂ ⟨x, hxs₂⟩ :=
by
rintro s₁ hs₁ s₂ hs₂ x hxs₁ hxs₂
haveI := isCompact_iff_compactSpace.mp hs₁
haveI := isCompact_iff_compactSpace.mp hs₂
have h₁ := (continuous_eval_const (⟨x, hxs₁⟩ : s₁)).continuousAt.tendsto.comp (hf s₁ hs₁)
have h₂ := (continuous_eval_const (⟨x, hxs₂⟩ : s₂)).continuousAt.tendsto.comp (hf s₂ hs₂)
exact tendsto_nhds_unique h₁ h₂
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
⊢ ∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
[PROOFSTEP]
rintro s₁ hs₁ s₂ hs₂ x hxs₁ hxs₂
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
s₁ : Set α
hs₁ : IsCompact s₁
s₂ : Set α
hs₂ : IsCompact s₂
x : α
hxs₁ : x ∈ s₁
hxs₂ : x ∈ s₂
⊢ ↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
[PROOFSTEP]
haveI := isCompact_iff_compactSpace.mp hs₁
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
s₁ : Set α
hs₁ : IsCompact s₁
s₂ : Set α
hs₂ : IsCompact s₂
x : α
hxs₁ : x ∈ s₁
hxs₂ : x ∈ s₂
this : CompactSpace ↑s₁
⊢ ↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
[PROOFSTEP]
haveI := isCompact_iff_compactSpace.mp hs₂
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
s₁ : Set α
hs₁ : IsCompact s₁
s₂ : Set α
hs₂ : IsCompact s₂
x : α
hxs₁ : x ∈ s₁
hxs₂ : x ∈ s₂
this✝ : CompactSpace ↑s₁
this : CompactSpace ↑s₂
⊢ ↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
[PROOFSTEP]
have h₁ := (continuous_eval_const (⟨x, hxs₁⟩ : s₁)).continuousAt.tendsto.comp (hf s₁ hs₁)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
s₁ : Set α
hs₁ : IsCompact s₁
s₂ : Set α
hs₂ : IsCompact s₂
x : α
hxs₁ : x ∈ s₁
hxs₂ : x ∈ s₂
this✝ : CompactSpace ↑s₁
this : CompactSpace ↑s₂
h₁ :
Filter.Tendsto ((fun f => ↑f { val := x, property := hxs₁ }) ∘ fun i => restrict s₁ (F i)) l
(𝓝 (↑(f s₁ hs₁) { val := x, property := hxs₁ }))
⊢ ↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
[PROOFSTEP]
have h₂ := (continuous_eval_const (⟨x, hxs₂⟩ : s₂)).continuousAt.tendsto.comp (hf s₂ hs₂)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
s₁ : Set α
hs₁ : IsCompact s₁
s₂ : Set α
hs₂ : IsCompact s₂
x : α
hxs₁ : x ∈ s₁
hxs₂ : x ∈ s₂
this✝ : CompactSpace ↑s₁
this : CompactSpace ↑s₂
h₁ :
Filter.Tendsto ((fun f => ↑f { val := x, property := hxs₁ }) ∘ fun i => restrict s₁ (F i)) l
(𝓝 (↑(f s₁ hs₁) { val := x, property := hxs₁ }))
h₂ :
Filter.Tendsto ((fun f => ↑f { val := x, property := hxs₂ }) ∘ fun i => restrict s₂ (F i)) l
(𝓝 (↑(f s₂ hs₂) { val := x, property := hxs₂ }))
⊢ ↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
[PROOFSTEP]
exact tendsto_nhds_unique h₁ h₂
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
⊢ ∃ f, Filter.Tendsto F l (𝓝 f)
[PROOFSTEP]
have hs : ∀ x : α, ∃ (s : _), IsCompact s ∧ s ∈ 𝓝 x := by
intro x
obtain ⟨s, hs, hs'⟩ := exists_compact_mem_nhds x
exact ⟨s, hs, hs'⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
⊢ ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
[PROOFSTEP]
intro x
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
x : α
⊢ ∃ s, IsCompact s ∧ s ∈ 𝓝 x
[PROOFSTEP]
obtain ⟨s, hs, hs'⟩ := exists_compact_mem_nhds x
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
x : α
s : Set α
hs : IsCompact s
hs' : s ∈ 𝓝 x
⊢ ∃ s, IsCompact s ∧ s ∈ 𝓝 x
[PROOFSTEP]
exact ⟨s, hs, hs'⟩
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
hs : ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
⊢ ∃ f, Filter.Tendsto F l (𝓝 f)
[PROOFSTEP]
refine ⟨liftCover' _ _ h hs, ?_⟩
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
hs : ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
⊢ Filter.Tendsto F l
(𝓝
(liftCover'
(fun s => ∀ ⦃f : Filter α⦄ [inst : Filter.NeBot f], f ≤ Filter.principal s → ∃ a, a ∈ s ∧ ClusterPt a f)
(fun s hs => f s hs) h hs))
[PROOFSTEP]
rw [tendsto_compactOpen_iff_forall]
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
hs : ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
⊢ ∀ (s : Set α),
IsCompact s →
Filter.Tendsto (fun i => restrict s (F i)) l
(𝓝
(restrict s
(liftCover'
(fun s => ∀ ⦃f : Filter α⦄ [inst : Filter.NeBot f], f ≤ Filter.principal s → ∃ a, a ∈ s ∧ ClusterPt a f)
(fun s hs => f s hs) h hs)))
[PROOFSTEP]
intro s hs
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
hs✝ : ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
s : Set α
hs : IsCompact s
⊢ Filter.Tendsto (fun i => restrict s (F i)) l
(𝓝
(restrict s
(liftCover'
(fun s => ∀ ⦃f : Filter α⦄ [inst : Filter.NeBot f], f ≤ Filter.principal s → ∃ a, a ∈ s ∧ ClusterPt a f)
(fun s hs => f s hs) h hs✝)))
[PROOFSTEP]
rw [liftCover_restrict']
[GOAL]
case mpr
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
hs✝ : ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
s : Set α
hs : IsCompact s
⊢ Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s ?m.52935))
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : LocallyCompactSpace α
inst✝¹ : T2Space β
ι : Type u_4
l : Filter ι
inst✝ : Filter.NeBot l
F : ι → C(α, β)
f : (s : Set α) → IsCompact s → C(↑s, β)
hf : ∀ (s : Set α) (hs : IsCompact s), Filter.Tendsto (fun i => restrict s (F i)) l (𝓝 (f s hs))
h :
∀ (s₁ : Set α) (hs₁ : IsCompact s₁) (s₂ : Set α) (hs₂ : IsCompact s₂) (x : α) (hxs₁ : x ∈ s₁) (hxs₂ : x ∈ s₂),
↑(f s₁ hs₁) { val := x, property := hxs₁ } = ↑(f s₂ hs₂) { val := x, property := hxs₂ }
hs✝ : ∀ (x : α), ∃ s, IsCompact s ∧ s ∈ 𝓝 x
s : Set α
hs : IsCompact s
⊢ s ∈ fun s => ∀ ⦃f : Filter α⦄ [inst : Filter.NeBot f], f ≤ Filter.principal s → ∃ a, a ∈ s ∧ ClusterPt a f
[PROOFSTEP]
exact hf s hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
y : β
s : Set α
⊢ ↑(coev α β y) '' s = {y} ×ˢ s
[PROOFSTEP]
aesop
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
⊢ ∀ (s : Set C(α, β × α)), s ∈ {m | ∃ s x u x, m = CompactOpen.gen s u} → IsOpen (coev α β ⁻¹' s)
[PROOFSTEP]
rintro _ ⟨s, sc, u, uo, rfl⟩
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
⊢ IsOpen (coev α β ⁻¹' CompactOpen.gen s u)
[PROOFSTEP]
rw [isOpen_iff_forall_mem_open]
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
⊢ ∀ (x : β), x ∈ coev α β ⁻¹' CompactOpen.gen s u → ∃ t, t ⊆ coev α β ⁻¹' CompactOpen.gen s u ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
intro y hy
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
⊢ ∃ t, t ⊆ coev α β ⁻¹' CompactOpen.gen s u ∧ IsOpen t ∧ y ∈ t
[PROOFSTEP]
have hy' : (↑(coev α β y) '' s ⊆ u) := hy
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy' : ↑(coev α β y) '' s ⊆ u
⊢ ∃ t, t ⊆ coev α β ⁻¹' CompactOpen.gen s u ∧ IsOpen t ∧ y ∈ t
[PROOFSTEP]
rw [image_coev s] at hy'
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy' : {y} ×ˢ s ⊆ u
⊢ ∃ t, t ⊆ coev α β ⁻¹' CompactOpen.gen s u ∧ IsOpen t ∧ y ∈ t
[PROOFSTEP]
rcases generalized_tube_lemma isCompact_singleton sc uo hy' with ⟨v, w, vo, _, yv, sw, vwu⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy' : {y} ×ˢ s ⊆ u
v : Set β
w : Set α
vo : IsOpen v
left✝ : IsOpen w
yv : {y} ⊆ v
sw : s ⊆ w
vwu : v ×ˢ w ⊆ u
⊢ ∃ t, t ⊆ coev α β ⁻¹' CompactOpen.gen s u ∧ IsOpen t ∧ y ∈ t
[PROOFSTEP]
refine' ⟨v, _, vo, singleton_subset_iff.mp yv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy' : {y} ×ˢ s ⊆ u
v : Set β
w : Set α
vo : IsOpen v
left✝ : IsOpen w
yv : {y} ⊆ v
sw : s ⊆ w
vwu : v ×ˢ w ⊆ u
⊢ v ⊆ coev α β ⁻¹' CompactOpen.gen s u
[PROOFSTEP]
intro y' hy'
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy'✝ : {y} ×ˢ s ⊆ u
v : Set β
w : Set α
vo : IsOpen v
left✝ : IsOpen w
yv : {y} ⊆ v
sw : s ⊆ w
vwu : v ×ˢ w ⊆ u
y' : β
hy' : y' ∈ v
⊢ y' ∈ coev α β ⁻¹' CompactOpen.gen s u
[PROOFSTEP]
change coev α β y' '' s ⊆ u
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy'✝ : {y} ×ˢ s ⊆ u
v : Set β
w : Set α
vo : IsOpen v
left✝ : IsOpen w
yv : {y} ⊆ v
sw : s ⊆ w
vwu : v ×ˢ w ⊆ u
y' : β
hy' : y' ∈ v
⊢ ↑(coev α β y') '' s ⊆ u
[PROOFSTEP]
rw [image_coev s]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
sc : IsCompact s
u : Set (β × α)
uo : IsOpen u
y : β
hy : y ∈ coev α β ⁻¹' CompactOpen.gen s u
hy'✝ : {y} ×ˢ s ⊆ u
v : Set β
w : Set α
vo : IsOpen v
left✝ : IsOpen w
yv : {y} ⊆ v
sw : s ⊆ w
vwu : v ×ˢ w ⊆ u
y' : β
hy' : y' ∈ v
⊢ {y'} ×ˢ s ⊆ u
[PROOFSTEP]
exact (prod_mono (singleton_subset_iff.mpr hy') sw).trans vwu
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : C(α × β, γ)
⊢ curry' f = comp f ∘ coev β α
[PROOFSTEP]
ext
[GOAL]
case h.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : C(α × β, γ)
x✝ : α
a✝ : β
⊢ ↑(curry' f x✝) a✝ = ↑((comp f ∘ coev β α) x✝) a✝
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace (α × β)
⊢ Continuous curry
[PROOFSTEP]
apply continuous_of_continuous_uncurry
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace (α × β)
⊢ Continuous (Function.uncurry fun x y => ↑(curry x) y)
[PROOFSTEP]
apply continuous_of_continuous_uncurry
[GOAL]
case h.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace (α × β)
⊢ Continuous (Function.uncurry fun x y => ↑(Function.uncurry (fun x y => ↑(curry x) y) x) y)
[PROOFSTEP]
rw [← (Homeomorph.prodAssoc _ _ _).symm.comp_continuous_iff']
[GOAL]
case h.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : LocallyCompactSpace (α × β)
⊢ Continuous
((Function.uncurry fun x y => ↑(Function.uncurry (fun x y => ↑(curry x) y) x) y) ∘
↑(Homeomorph.symm (Homeomorph.prodAssoc C(α × β, γ) α β)))
[PROOFSTEP]
exact continuous_eval'
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
⊢ Continuous uncurry
[PROOFSTEP]
apply continuous_of_continuous_uncurry
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
⊢ Continuous (Function.uncurry fun x y => ↑(uncurry x) y)
[PROOFSTEP]
rw [← (Homeomorph.prodAssoc _ _ _).comp_continuous_iff']
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
⊢ Continuous ((Function.uncurry fun x y => ↑(uncurry x) y) ∘ ↑(Homeomorph.prodAssoc C(α, C(β, γ)) α β))
[PROOFSTEP]
apply continuous_eval'.comp (continuous_eval'.prod_map continuous_id)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
⊢ Function.LeftInverse uncurry ContinuousMap.curry
[PROOFSTEP]
intro
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
x✝ : C(α × β, γ)
⊢ uncurry (ContinuousMap.curry x✝) = x✝
[PROOFSTEP]
ext
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
x✝ : C(α × β, γ)
a✝ : α × β
⊢ ↑(uncurry (ContinuousMap.curry x✝)) a✝ = ↑x✝ a✝
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
⊢ Function.RightInverse uncurry ContinuousMap.curry
[PROOFSTEP]
intro
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
x✝ : C(α, C(β, γ))
⊢ ContinuousMap.curry (uncurry x✝) = x✝
[PROOFSTEP]
ext
[GOAL]
case h.h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : LocallyCompactSpace β
x✝ : C(α, C(β, γ))
a✝¹ : α
a✝ : β
⊢ ↑(↑(ContinuousMap.curry (uncurry x✝)) a✝¹) a✝ = ↑(↑x✝ a✝¹) a✝
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : Unique α
f : C(α, β)
⊢ const α ((fun f => ↑f default) f) = f
[PROOFSTEP]
ext a
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : Unique α
f : C(α, β)
a : α
⊢ ↑(const α ((fun f => ↑f default) f)) a = ↑f a
[PROOFSTEP]
rw [Unique.eq_default a]
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : Unique α
f : C(α, β)
a : α
⊢ ↑(const α ((fun f => ↑f default) f)) default = ↑f default
[PROOFSTEP]
rfl
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
⊢ Continuous g
[PROOFSTEP]
let Gf : C(X₀, C(Y, Z)) := ContinuousMap.curry ⟨_, hg⟩
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
⊢ Continuous g
[PROOFSTEP]
have h : ∀ x : X, Continuous fun y => g (x, y) := by
intro x
obtain ⟨x₀, rfl⟩ := hf.surjective x
exact (Gf x₀).continuous
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
⊢ ∀ (x : X), Continuous fun y => g (x, y)
[PROOFSTEP]
intro x
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
x : X
⊢ Continuous fun y => g (x, y)
[PROOFSTEP]
obtain ⟨x₀, rfl⟩ := hf.surjective x
[GOAL]
case intro
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
x₀ : X₀
⊢ Continuous fun y => g (f x₀, y)
[PROOFSTEP]
exact (Gf x₀).continuous
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
h : ∀ (x : X), Continuous fun y => g (x, y)
⊢ Continuous g
[PROOFSTEP]
let G : X → C(Y, Z) := fun x => ⟨_, h x⟩
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
h : ∀ (x : X), Continuous fun y => g (x, y)
G : X → C(Y, Z) := fun x => mk fun y => g (x, y)
⊢ Continuous g
[PROOFSTEP]
have : Continuous G := by
rw [hf.continuous_iff]
exact Gf.continuous
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
h : ∀ (x : X), Continuous fun y => g (x, y)
G : X → C(Y, Z) := fun x => mk fun y => g (x, y)
⊢ Continuous G
[PROOFSTEP]
rw [hf.continuous_iff]
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
h : ∀ (x : X), Continuous fun y => g (x, y)
G : X → C(Y, Z) := fun x => mk fun y => g (x, y)
⊢ Continuous (G ∘ f)
[PROOFSTEP]
exact Gf.continuous
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : X × Y → Z
hg : Continuous fun p => g (f p.fst, p.snd)
Gf : C(X₀, C(Y, Z)) := curry (mk fun p => g (f p.fst, p.snd))
h : ∀ (x : X), Continuous fun y => g (x, y)
G : X → C(Y, Z) := fun x => mk fun y => g (x, y)
this : Continuous G
⊢ Continuous g
[PROOFSTEP]
exact ContinuousMap.continuous_uncurry_of_continuous ⟨G, this⟩
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : Y × X → Z
hg : Continuous fun p => g (p.fst, f p.snd)
⊢ Continuous g
[PROOFSTEP]
have : Continuous fun p : X₀ × Y => g ((Prod.swap p).1, f (Prod.swap p).2) := hg.comp continuous_swap
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : Y × X → Z
hg : Continuous fun p => g (p.fst, f p.snd)
this : Continuous fun p => g ((Prod.swap p).fst, f (Prod.swap p).snd)
⊢ Continuous g
[PROOFSTEP]
have : Continuous fun p : X₀ × Y => (g ∘ Prod.swap) (f p.1, p.2) := this
[GOAL]
X₀ : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X₀
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : LocallyCompactSpace Y
f : X₀ → X
hf : QuotientMap f
g : Y × X → Z
hg : Continuous fun p => g (p.fst, f p.snd)
this✝ : Continuous fun p => g ((Prod.swap p).fst, f (Prod.swap p).snd)
this : Continuous fun p => (g ∘ Prod.swap) (f p.fst, p.snd)
⊢ Continuous g
[PROOFSTEP]
exact (hf.continuous_lift_prod_left this).comp continuous_swap
| {"mathlib_filename": "Mathlib.Topology.CompactOpen", "llama_tokens": 27184} |
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
toSetoid✝¹ : Setoid X
isOpen_setOf_rel✝¹ : ∀ (x : X), IsOpen (setOf (Setoid.Rel toSetoid✝¹ x))
toSetoid✝ : Setoid X
isOpen_setOf_rel✝ : ∀ (x : X), IsOpen (setOf (Setoid.Rel toSetoid✝ x))
x✝ :
{ toSetoid := toSetoid✝¹, isOpen_setOf_rel := isOpen_setOf_rel✝¹ }.toSetoid =
{ toSetoid := toSetoid✝, isOpen_setOf_rel := isOpen_setOf_rel✝ }.toSetoid
⊢ { toSetoid := toSetoid✝¹, isOpen_setOf_rel := isOpen_setOf_rel✝¹ } =
{ toSetoid := toSetoid✝, isOpen_setOf_rel := isOpen_setOf_rel✝ }
[PROOFSTEP]
congr
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
A : Set X
h : IsClopen A
x : X
⊢ IsOpen (setOf (Setoid.Rel { r := fun x y => x ∈ A ↔ y ∈ A, iseqv := (_ : Equivalence fun x y => x ∈ A ↔ y ∈ A) } x))
[PROOFSTEP]
by_cases hx : x ∈ A
[GOAL]
case pos
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
A : Set X
h : IsClopen A
x : X
hx : x ∈ A
⊢ IsOpen (setOf (Setoid.Rel { r := fun x y => x ∈ A ↔ y ∈ A, iseqv := (_ : Equivalence fun x y => x ∈ A ↔ y ∈ A) } x))
[PROOFSTEP]
simp [Setoid.Rel, hx, h.1, h.2, ← compl_setOf]
[GOAL]
case neg
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
A : Set X
h : IsClopen A
x : X
hx : ¬x ∈ A
⊢ IsOpen (setOf (Setoid.Rel { r := fun x y => x ∈ A ↔ y ∈ A, iseqv := (_ : Equivalence fun x y => x ∈ A ↔ y ∈ A) } x))
[PROOFSTEP]
simp [Setoid.Rel, hx, h.1, h.2, ← compl_setOf]
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
x : X
⊢ IsOpen {proj S x}
[PROOFSTEP]
rw [← S.proj_quotientMap.isOpen_preimage, fiber_eq]
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
x : X
⊢ IsOpen (setOf (Setoid.Rel S.toSetoid x))
[PROOFSTEP]
exact S.isOpen_setOf_rel _
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
x : X
⊢ IsClopen (setOf (Setoid.Rel S.toSetoid x))
[PROOFSTEP]
rw [← fiber_eq]
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
x : X
⊢ IsClopen (proj S ⁻¹' {proj S x})
[PROOFSTEP]
apply isClopen_preimage
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S a : DiscreteQuotient X
⊢ a ≤ ⊤
[PROOFSTEP]
tauto
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
⊢ ∀ (a b : Quotient ⊤.toSetoid), a = b
[PROOFSTEP]
rintro ⟨_⟩ ⟨_⟩
[GOAL]
case mk.mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
a✝² : Quotient ⊤.toSetoid
a✝¹ : X
b✝ : Quotient ⊤.toSetoid
a✝ : X
⊢ Quot.mk Setoid.r a✝¹ = Quot.mk Setoid.r a✝
[PROOFSTEP]
exact Quotient.sound trivial
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
g : C(Y, Z)
f : C(X, Y)
A B : DiscreteQuotient Y
h : A ≤ B
⊢ comap f A ≤ comap f B
[PROOFSTEP]
tauto
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B C : DiscreteQuotient X
⊢ ofLE (_ : A ≤ A) = id
[PROOFSTEP]
ext ⟨⟩
[GOAL]
case h.mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B C : DiscreteQuotient X
x✝ : Quotient A.toSetoid
a✝ : X
⊢ ofLE (_ : A ≤ A) (Quot.mk Setoid.r a✝) = id (Quot.mk Setoid.r a✝)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B C : DiscreteQuotient X
a : Quotient A.toSetoid
⊢ ofLE (_ : A ≤ A) a = a
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B C : DiscreteQuotient X
h₁ : A ≤ B
h₂ : B ≤ C
x : Quotient A.toSetoid
⊢ ofLE h₂ (ofLE h₁ x) = ofLE (_ : A ≤ C) x
[PROOFSTEP]
rcases x with ⟨⟩
[GOAL]
case mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B C : DiscreteQuotient X
h₁ : A ≤ B
h₂ : B ≤ C
x : Quotient A.toSetoid
a✝ : X
⊢ ofLE h₂ (ofLE h₁ (Quot.mk Setoid.r a✝)) = ofLE (_ : A ≤ C) (Quot.mk Setoid.r a✝)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : LocallyConnectedSpace X
x : X
⊢ IsOpen (setOf (Setoid.Rel (connectedComponentSetoid X) x))
[PROOFSTEP]
convert isOpen_connectedComponent (x := x)
[GOAL]
case h.e'_3
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : LocallyConnectedSpace X
x : X
⊢ setOf (Setoid.Rel (connectedComponentSetoid X) x) = connectedComponent x
[PROOFSTEP]
ext y
[GOAL]
case h.e'_3.h
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : LocallyConnectedSpace X
x y : X
⊢ y ∈ setOf (Setoid.Rel (connectedComponentSetoid X) x) ↔ y ∈ connectedComponent x
[PROOFSTEP]
simpa only [connectedComponentSetoid, ← connectedComponent_eq_iff_mem] using eq_comm
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : DiscreteTopology X
x y : X
⊢ proj ⊥ x = proj ⊥ y ↔ x = y
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
⊢ LEComap g B C → LEComap f A B → LEComap (ContinuousMap.comp g f) A C
[PROOFSTEP]
tauto
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
⊢ map (ContinuousMap.id X) (_ : LEComap (ContinuousMap.id X) A A) = id
[PROOFSTEP]
ext ⟨⟩
[GOAL]
case h.mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
x✝ : Quotient A.toSetoid
a✝ : X
⊢ map (ContinuousMap.id X) (_ : LEComap (ContinuousMap.id X) A A) (Quot.mk Setoid.r a✝) = id (Quot.mk Setoid.r a✝)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
h1 : LEComap g B C
h2 : LEComap f A B
⊢ map (ContinuousMap.comp g f) (_ : LEComap (ContinuousMap.comp g f) A C) = map g h1 ∘ map f h2
[PROOFSTEP]
ext ⟨⟩
[GOAL]
case h.mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
h1 : LEComap g B C
h2 : LEComap f A B
x✝ : Quotient A.toSetoid
a✝ : X
⊢ map (ContinuousMap.comp g f) (_ : LEComap (ContinuousMap.comp g f) A C) (Quot.mk Setoid.r a✝) =
(map g h1 ∘ map f h2) (Quot.mk Setoid.r a✝)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
cond : LEComap f A B
h : B ≤ B'
a : Quotient A.toSetoid
⊢ ofLE h (map f cond a) = map f (_ : LEComap f A B') a
[PROOFSTEP]
rcases a with ⟨⟩
[GOAL]
case mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
cond : LEComap f A B
h : B ≤ B'
a : Quotient A.toSetoid
a✝ : X
⊢ ofLE h (map f cond (Quot.mk Setoid.r a✝)) = map f (_ : LEComap f A B') (Quot.mk Setoid.r a✝)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
cond : LEComap f A B
h : A' ≤ A
c : Quotient A'.toSetoid
⊢ map f cond (ofLE h c) = map f (_ : LEComap f A' B) c
[PROOFSTEP]
rcases c with ⟨⟩
[GOAL]
case mk
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S : DiscreteQuotient X
f : C(X, Y)
A A' : DiscreteQuotient X
B B' : DiscreteQuotient Y
g : C(Y, Z)
C : DiscreteQuotient Z
cond : LEComap f A B
h : A' ≤ A
c : Quotient A'.toSetoid
a✝ : X
⊢ map f cond (ofLE h (Quot.mk Setoid.r a✝)) = map f (_ : LEComap f A' B) (Quot.mk Setoid.r a✝)
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
S : DiscreteQuotient X
inst✝¹ : T2Space X
inst✝ : CompactSpace X
disc : TotallyDisconnectedSpace X
x y : X
h : ∀ (Q : DiscreteQuotient X), proj Q x = proj Q y
⊢ x = y
[PROOFSTEP]
rw [← mem_singleton_iff, ← connectedComponent_eq_singleton, connectedComponent_eq_iInter_clopen, mem_iInter]
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
S : DiscreteQuotient X
inst✝¹ : T2Space X
inst✝ : CompactSpace X
disc : TotallyDisconnectedSpace X
x y : X
h : ∀ (Q : DiscreteQuotient X), proj Q x = proj Q y
⊢ ∀ (i : { Z // IsClopen Z ∧ y ∈ Z }), x ∈ ↑i
[PROOFSTEP]
rintro ⟨U, hU1, hU2⟩
[GOAL]
case mk.intro
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : TopologicalSpace Z
S : DiscreteQuotient X
inst✝¹ : T2Space X
inst✝ : CompactSpace X
disc : TotallyDisconnectedSpace X
x y : X
h : ∀ (Q : DiscreteQuotient X), proj Q x = proj Q y
U : Set X
hU1 : IsClopen U
hU2 : y ∈ U
⊢ x ∈ ↑{ val := U, property := (_ : IsClopen U ∧ y ∈ U) }
[PROOFSTEP]
exact (Quotient.exact' (h (ofClopen hU1))).mpr hU2
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B : DiscreteQuotient X
h : A ≤ B
a : Quotient A.toSetoid
⊢ proj A ⁻¹' {a} ⊆ proj B ⁻¹' {ofLE h a}
[PROOFSTEP]
rcases A.proj_surjective a with ⟨a, rfl⟩
[GOAL]
case intro
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B : DiscreteQuotient X
h : A ≤ B
a : X
⊢ proj A ⁻¹' {proj A a} ⊆ proj B ⁻¹' {ofLE h (proj A a)}
[PROOFSTEP]
rw [fiber_eq, ofLE_proj, fiber_eq]
[GOAL]
case intro
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : TopologicalSpace Z
S A B : DiscreteQuotient X
h : A ≤ B
a : X
⊢ setOf (Setoid.Rel A.toSetoid a) ⊆ setOf (Setoid.Rel B.toSetoid a)
[PROOFSTEP]
exact fun _ h' => h h'
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
Qs : (Q : DiscreteQuotient X) → Quotient Q.toSetoid
compat : ∀ (A B : DiscreteQuotient X) (h : A ≤ B), ofLE h (Qs A) = Qs B
⊢ ∃ x, ∀ (Q : DiscreteQuotient X), proj Q x = Qs Q
[PROOFSTEP]
have H₁ : ∀ Q₁ Q₂, Q₁ ≤ Q₂ → proj Q₁ ⁻¹' {Qs Q₁} ⊆ proj Q₂ ⁻¹' {Qs Q₂} := fun _ _ h =>
by
rw [← compat _ _ h]
exact fiber_subset_ofLE _ _
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
Qs : (Q : DiscreteQuotient X) → Quotient Q.toSetoid
compat : ∀ (A B : DiscreteQuotient X) (h : A ≤ B), ofLE h (Qs A) = Qs B
x✝¹ x✝ : DiscreteQuotient X
h : x✝¹ ≤ x✝
⊢ proj x✝¹ ⁻¹' {Qs x✝¹} ⊆ proj x✝ ⁻¹' {Qs x✝}
[PROOFSTEP]
rw [← compat _ _ h]
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
Qs : (Q : DiscreteQuotient X) → Quotient Q.toSetoid
compat : ∀ (A B : DiscreteQuotient X) (h : A ≤ B), ofLE h (Qs A) = Qs B
x✝¹ x✝ : DiscreteQuotient X
h : x✝¹ ≤ x✝
⊢ proj x✝¹ ⁻¹' {Qs x✝¹} ⊆ proj x✝ ⁻¹' {ofLE h (Qs x✝¹)}
[PROOFSTEP]
exact fiber_subset_ofLE _ _
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
Qs : (Q : DiscreteQuotient X) → Quotient Q.toSetoid
compat : ∀ (A B : DiscreteQuotient X) (h : A ≤ B), ofLE h (Qs A) = Qs B
H₁ : ∀ (Q₁ Q₂ : DiscreteQuotient X), Q₁ ≤ Q₂ → proj Q₁ ⁻¹' {Qs Q₁} ⊆ proj Q₂ ⁻¹' {Qs Q₂}
⊢ ∃ x, ∀ (Q : DiscreteQuotient X), proj Q x = Qs Q
[PROOFSTEP]
obtain ⟨x, hx⟩ : Set.Nonempty (⋂ Q, proj Q ⁻¹' {Qs Q}) :=
IsCompact.nonempty_iInter_of_directed_nonempty_compact_closed (fun Q : DiscreteQuotient X => Q.proj ⁻¹' {Qs _})
(directed_of_inf H₁) (fun Q => (singleton_nonempty _).preimage Q.proj_surjective)
(fun Q => (Q.isClosed_preimage {Qs _}).isCompact) fun Q => Q.isClosed_preimage _
[GOAL]
case intro
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
Qs : (Q : DiscreteQuotient X) → Quotient Q.toSetoid
compat : ∀ (A B : DiscreteQuotient X) (h : A ≤ B), ofLE h (Qs A) = Qs B
H₁ : ∀ (Q₁ Q₂ : DiscreteQuotient X), Q₁ ≤ Q₂ → proj Q₁ ⁻¹' {Qs Q₁} ⊆ proj Q₂ ⁻¹' {Qs Q₂}
x : X
hx : x ∈ ⋂ (Q : DiscreteQuotient X), proj Q ⁻¹' {Qs Q}
⊢ ∃ x, ∀ (Q : DiscreteQuotient X), proj Q x = Qs Q
[PROOFSTEP]
exact ⟨x, mem_iInter.1 hx⟩
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
⊢ Finite (Quotient S.toSetoid)
[PROOFSTEP]
have : CompactSpace S := Quotient.compactSpace
[GOAL]
α : Type u_1
X : Type u_2
Y : Type u_3
Z : Type u_4
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
S : DiscreteQuotient X
inst✝ : CompactSpace X
this : CompactSpace (Quotient S.toSetoid)
⊢ Finite (Quotient S.toSetoid)
[PROOFSTEP]
rwa [← isCompact_univ_iff, isCompact_iff_finite, finite_univ_iff] at this
| {"mathlib_filename": "Mathlib.Topology.DiscreteQuotient", "llama_tokens": 7607} |
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑(TensorAlgebra.ι R) m ∈ LinearMap.range (TensorAlgebra.ι R) ^ 1
[PROOFSTEP]
simpa only [pow_one] using LinearMap.mem_range_self _ m
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑(TensorAlgebra.ι R) m ∈ LinearMap.range (TensorAlgebra.ι R) ^ 1
[PROOFSTEP]
simpa only [pow_one] using LinearMap.mem_range_self _ m
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ AlgHom.comp (DirectSum.coeAlgHom fun x => LinearMap.range (ι R) ^ x) (↑(lift R) (GradedAlgebra.ι R M)) =
AlgHom.id R (TensorAlgebra R M)
[PROOFSTEP]
ext m
[GOAL]
case w.h
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑(LinearMap.comp
(AlgHom.toLinearMap
(AlgHom.comp (DirectSum.coeAlgHom fun x => LinearMap.range (ι R) ^ x) (↑(lift R) (GradedAlgebra.ι R M))))
(ι R))
m =
↑(LinearMap.comp (AlgHom.toLinearMap (AlgHom.id R (TensorAlgebra R M))) (ι R)) m
[PROOFSTEP]
dsimp only [LinearMap.comp_apply, AlgHom.toLinearMap_apply, AlgHom.comp_apply, AlgHom.id_apply]
[GOAL]
case w.h
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
m : M
⊢ ↑(DirectSum.coeAlgHom fun x => LinearMap.range (ι R) ^ x) (↑(↑(lift R) (GradedAlgebra.ι R M)) (↑(ι R) m)) = ↑(ι R) m
[PROOFSTEP]
rw [lift_ι_apply, GradedAlgebra.ι_apply R M, DirectSum.coeAlgHom_of, Subtype.coe_mk]
[GOAL]
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : { x // x ∈ LinearMap.range (ι R) ^ i }
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) ↑x = ↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) x
[PROOFSTEP]
cases' x with x hx
[GOAL]
case mk
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) ↑{ val := x, property := hx } =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
[PROOFSTEP]
dsimp only [Subtype.coe_mk, DirectSum.lof_eq_of]
-- porting note: use new `induction using` support that failed in Lean 3
[GOAL]
case mk
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
[PROOFSTEP]
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy => rw [AlgHom.map_add, ihx, ihy, ← map_add]; rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply R M, DirectSum.of_mul_of]
exact DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext (add_comm _ _) rfl)
[GOAL]
case mk
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
[PROOFSTEP]
induction hx using Submodule.pow_induction_on_left' with
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
| hadd x y i hx hy ihx ihy => rw [AlgHom.map_add, ihx, ihy, ← map_add]; rfl
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply R M, DirectSum.of_mul_of]
exact DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext (add_comm _ _) rfl)
[GOAL]
case mk.hr
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : TensorAlgebra R M
r : R
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (↑(algebraMap R (TensorAlgebra R M)) r) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) 0)
{ val := ↑(algebraMap R (TensorAlgebra R M)) r, property := (_ : ↑(algebraMap R (TensorAlgebra R M)) r ∈ 1) }
[PROOFSTEP]
| hr r => rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl
[GOAL]
case mk.hr
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : TensorAlgebra R M
r : R
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (↑(algebraMap R (TensorAlgebra R M)) r) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) 0)
{ val := ↑(algebraMap R (TensorAlgebra R M)) r, property := (_ : ↑(algebraMap R (TensorAlgebra R M)) r ∈ 1) }
[PROOFSTEP]
rw [AlgHom.commutes, DirectSum.algebraMap_apply]
[GOAL]
case mk.hr
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i : ℕ
x : TensorAlgebra R M
r : R
⊢ ↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) 0) (↑DirectSum.GAlgebra.toFun r) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) 0)
{ val := ↑(algebraMap R (TensorAlgebra R M)) r, property := (_ : ↑(algebraMap R (TensorAlgebra R M)) r ∈ 1) }
[PROOFSTEP]
rfl
[GOAL]
case mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ x y : TensorAlgebra R M
i : ℕ
hx : x ∈ LinearMap.range (ι R) ^ i
hy : y ∈ LinearMap.range (ι R) ^ i
ihx :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
ihy :
↑(↑(lift R) (GradedAlgebra.ι R M)) y =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := y, property := hy }
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (x + y) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i)
{ val := x + y, property := (_ : x + y ∈ LinearMap.range (ι R) ^ i) }
[PROOFSTEP]
| hadd x y i hx hy ihx ihy => rw [AlgHom.map_add, ihx, ihy, ← map_add]; rfl
[GOAL]
case mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ x y : TensorAlgebra R M
i : ℕ
hx : x ∈ LinearMap.range (ι R) ^ i
hy : y ∈ LinearMap.range (ι R) ^ i
ihx :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
ihy :
↑(↑(lift R) (GradedAlgebra.ι R M)) y =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := y, property := hy }
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (x + y) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i)
{ val := x + y, property := (_ : x + y ∈ LinearMap.range (ι R) ^ i) }
[PROOFSTEP]
rw [AlgHom.map_add, ihx, ihy, ← map_add]
[GOAL]
case mk.hadd
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ x y : TensorAlgebra R M
i : ℕ
hx : x ∈ LinearMap.range (ι R) ^ i
hy : y ∈ LinearMap.range (ι R) ^ i
ihx :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
ihy :
↑(↑(lift R) (GradedAlgebra.ι R M)) y =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := y, property := hy }
⊢ ↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i)
({ val := x, property := hx } + { val := y, property := hy }) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i)
{ val := x + y, property := (_ : x + y ∈ LinearMap.range (ι R) ^ i) }
[PROOFSTEP]
rfl
[GOAL]
case mk.hmul
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ m : TensorAlgebra R M
hm : m ∈ LinearMap.range (ι R)
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
ih :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (m * x) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) (Nat.succ i))
{ val := m * x, property := (_ : m * x ∈ LinearMap.range (ι R) * npowRec i (LinearMap.range (ι R))) }
[PROOFSTEP]
| hmul m hm i x hx ih =>
obtain ⟨_, rfl⟩ := hm
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply R M, DirectSum.of_mul_of]
exact DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext (add_comm _ _) rfl)
[GOAL]
case mk.hmul
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ m : TensorAlgebra R M
hm : m ∈ LinearMap.range (ι R)
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
ih :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (m * x) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) (Nat.succ i))
{ val := m * x, property := (_ : m * x ∈ LinearMap.range (ι R) * npowRec i (LinearMap.range (ι R))) }
[PROOFSTEP]
obtain ⟨_, rfl⟩ := hm
[GOAL]
case mk.hmul.intro
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ : TensorAlgebra R M
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
ih :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
w✝ : M
⊢ ↑(↑(lift R) (GradedAlgebra.ι R M)) (↑(ι R) w✝ * x) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) (Nat.succ i))
{ val := ↑(ι R) w✝ * x,
property := (_ : ↑(ι R) w✝ * x ∈ LinearMap.range (ι R) * npowRec i (LinearMap.range (ι R))) }
[PROOFSTEP]
rw [AlgHom.map_mul, ih, lift_ι_apply, GradedAlgebra.ι_apply R M, DirectSum.of_mul_of]
[GOAL]
case mk.hmul.intro
R : Type u_1
M : Type u_2
inst✝² : CommSemiring R
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
i✝ : ℕ
x✝ : TensorAlgebra R M
i : ℕ
x : TensorAlgebra R M
hx : x ∈ LinearMap.range (ι R) ^ i
ih :
↑(↑(lift R) (GradedAlgebra.ι R M)) x =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) i) { val := x, property := hx }
w✝ : M
⊢ ↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) (1 + i))
(GradedMonoid.GMul.mul { val := ↑(ι R) w✝, property := (_ : ↑(ι R) w✝ ∈ LinearMap.range (ι R) ^ 1) }
{ val := x, property := hx }) =
↑(DirectSum.of (fun i => { x // x ∈ LinearMap.range (ι R) ^ i }) (Nat.succ i))
{ val := ↑(ι R) w✝ * x,
property := (_ : ↑(ι R) w✝ * x ∈ LinearMap.range (ι R) * npowRec i (LinearMap.range (ι R))) }
[PROOFSTEP]
exact DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext (add_comm _ _) rfl)
| {"mathlib_filename": "Mathlib.LinearAlgebra.TensorAlgebra.Grading", "llama_tokens": 5057} |
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁵ : Semiring R
inst✝¹⁴ : AddCommMonoid M✝
inst✝¹³ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹² : Ring R₁
inst✝¹¹ : AddCommGroup M₁
inst✝¹⁰ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝⁹ : CommSemiring R₂
inst✝⁸ : AddCommMonoid M₂
inst✝⁷ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁶ : CommRing R₃
inst✝⁵ : AddCommGroup M₃
inst✝⁴ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝ : Fintype n
M : Matrix n n R₂
x y z : n → R₂
⊢ (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) (x + y) z =
(fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x z + (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) y z
[PROOFSTEP]
simp only [Pi.add_apply, add_mul, sum_add_distrib]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁵ : Semiring R
inst✝¹⁴ : AddCommMonoid M✝
inst✝¹³ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹² : Ring R₁
inst✝¹¹ : AddCommGroup M₁
inst✝¹⁰ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝⁹ : CommSemiring R₂
inst✝⁸ : AddCommMonoid M₂
inst✝⁷ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁶ : CommRing R₃
inst✝⁵ : AddCommGroup M₃
inst✝⁴ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝ : Fintype n
M : Matrix n n R₂
a : R₂
x y : n → R₂
⊢ (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) (a • x) y = a * (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x y
[PROOFSTEP]
simp only [Pi.smul_apply, smul_eq_mul, mul_assoc, mul_sum]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁵ : Semiring R
inst✝¹⁴ : AddCommMonoid M✝
inst✝¹³ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹² : Ring R₁
inst✝¹¹ : AddCommGroup M₁
inst✝¹⁰ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝⁹ : CommSemiring R₂
inst✝⁸ : AddCommMonoid M₂
inst✝⁷ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁶ : CommRing R₃
inst✝⁵ : AddCommGroup M₃
inst✝⁴ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝ : Fintype n
M : Matrix n n R₂
x y z : n → R₂
⊢ (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x (y + z) =
(fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x y + (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x z
[PROOFSTEP]
simp only [Pi.add_apply, mul_add, sum_add_distrib]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁵ : Semiring R
inst✝¹⁴ : AddCommMonoid M✝
inst✝¹³ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹² : Ring R₁
inst✝¹¹ : AddCommGroup M₁
inst✝¹⁰ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝⁹ : CommSemiring R₂
inst✝⁸ : AddCommMonoid M₂
inst✝⁷ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁶ : CommRing R₃
inst✝⁵ : AddCommGroup M₃
inst✝⁴ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝³ : Field K
inst✝² : AddCommGroup V
inst✝¹ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝ : Fintype n
M : Matrix n n R₂
a : R₂
x y : n → R₂
⊢ (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x (a • y) = a * (fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j) x y
[PROOFSTEP]
simp only [Pi.smul_apply, smul_eq_mul, mul_assoc, mul_left_comm, mul_sum]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ bilin (toBilin'Aux M) (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) =
M i j
[PROOFSTEP]
rw [Matrix.toBilin'Aux]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ bilin
{ bilin := fun v w => ∑ i : n, ∑ j : n, v i * M i j * w j,
bilin_add_left :=
(_ :
∀ (x y z : n → R₂),
∑ i : n, ∑ j : n, (x + y) i * M i j * z j =
∑ x_1 : n, ∑ x_2 : n, x x_1 * M x_1 x_2 * z x_2 + ∑ x : n, ∑ x_1 : n, y x * M x x_1 * z x_1),
bilin_smul_left :=
(_ :
∀ (a : R₂) (x y : n → R₂),
∑ i : n, ∑ j : n, (a • x) i * M i j * y j = a * ∑ i : n, ∑ j : n, x i * M i j * y j),
bilin_add_right :=
(_ :
∀ (x y z : n → R₂),
∑ i : n, ∑ j : n, x i * M i j * (y + z) j =
∑ x_1 : n, ∑ x_2 : n, x x_1 * M x_1 x_2 * y x_2 + ∑ x_1 : n, ∑ x_2 : n, x x_1 * M x_1 x_2 * z x_2),
bilin_smul_right :=
(_ :
∀ (a : R₂) (x y : n → R₂),
∑ i : n, ∑ j : n, x i * M i j * (a • y) j = a * ∑ i : n, ∑ j : n, x i * M i j * y j) }
(↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) =
M i j
[PROOFSTEP]
dsimp only
-- Porting note: had to add `dsimp only` to get rid of the projections
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ ∑ i_1 : n,
∑ j_1 : n,
↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i_1 * M i_1 j_1 * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j_1 =
M i j
[PROOFSTEP]
rw [sum_eq_single i, sum_eq_single j]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j = M i j
[PROOFSTEP]
simp only [stdBasis_same, stdBasis_same, one_mul, mul_one]
[GOAL]
case h₀
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ ∀ (b : n),
b ∈ univ →
b ≠ j → ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i b * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 b = 0
[PROOFSTEP]
rintro j' - hj'
[GOAL]
case h₀
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j j' : n
hj' : j' ≠ j
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j' * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j' = 0
[PROOFSTEP]
apply mul_eq_zero_of_right
[GOAL]
case h₀.h
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j j' : n
hj' : j' ≠ j
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j' = 0
[PROOFSTEP]
exact stdBasis_ne R₂ (fun _ => R₂) _ _ hj' 1
[GOAL]
case h₁
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ ¬j ∈ univ → ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j = 0
[PROOFSTEP]
intros
[GOAL]
case h₁
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
a✝ : ¬j ∈ univ
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j = 0
[PROOFSTEP]
have := Finset.mem_univ j
[GOAL]
case h₁
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
a✝ : ¬j ∈ univ
this : j ∈ univ
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j = 0
[PROOFSTEP]
contradiction
[GOAL]
case h₀
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ ∀ (b : n),
b ∈ univ →
b ≠ i →
∑ j_1 : n,
↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 b * M b j_1 * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j_1 =
0
[PROOFSTEP]
rintro i' - hi'
[GOAL]
case h₀
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j i' : n
hi' : i' ≠ i
⊢ ∑ j_1 : n, ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i' * M i' j_1 * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j_1 =
0
[PROOFSTEP]
refine' Finset.sum_eq_zero fun j _ => _
[GOAL]
case h₀
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j✝ i' : n
hi' : i' ≠ i
j : n
x✝ : j ∈ univ
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i' * M i' j * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j✝) 1 j = 0
[PROOFSTEP]
apply mul_eq_zero_of_left
[GOAL]
case h₀.h
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j✝ i' : n
hi' : i' ≠ i
j : n
x✝ : j ∈ univ
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i' * M i' j = 0
[PROOFSTEP]
apply mul_eq_zero_of_left
[GOAL]
case h₀.h.h
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j✝ i' : n
hi' : i' ≠ i
j : n
x✝ : j ∈ univ
⊢ ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i' = 0
[PROOFSTEP]
exact stdBasis_ne R₂ (fun _ => R₂) _ _ hi' 1
[GOAL]
case h₁
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
⊢ ¬i ∈ univ →
∑ j_1 : n, ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j_1 * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j_1 =
0
[PROOFSTEP]
intros
[GOAL]
case h₁
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
a✝ : ¬i ∈ univ
⊢ ∑ j_1 : n, ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j_1 * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j_1 = 0
[PROOFSTEP]
have := Finset.mem_univ i
[GOAL]
case h₁
R : Type u_1
M✝ : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝¹ : Fintype n
inst✝ : DecidableEq n
M : Matrix n n R₂
i j : n
a✝ : ¬i ∈ univ
this : i ∈ univ
⊢ ∑ j_1 : n, ↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1 i * M i j_1 * ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1 j_1 = 0
[PROOFSTEP]
contradiction
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂✝ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
B₂ : BilinForm R₂ (n → R₂)
⊢ toBilin'Aux (↑(toMatrixAux fun j => ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) B₂) = B₂
[PROOFSTEP]
refine' ext_basis (Pi.basisFun R₂ n) fun i j => _
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂✝ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
B₂ : BilinForm R₂ (n → R₂)
i j : n
⊢ bilin (toBilin'Aux (↑(toMatrixAux fun j => ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) B₂)) (↑(Pi.basisFun R₂ n) i)
(↑(Pi.basisFun R₂ n) j) =
bilin B₂ (↑(Pi.basisFun R₂ n) i) (↑(Pi.basisFun R₂ n) j)
[PROOFSTEP]
rw [Pi.basisFun_apply, Pi.basisFun_apply, Matrix.toBilin'Aux_stdBasis, BilinForm.toMatrixAux_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
src✝ : BilinForm R₂ ((fun x => n → R₂) 1) →ₗ[R₂] Matrix n n R₂ :=
toMatrixAux fun j => ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1
B : BilinForm R₂ (n → R₂)
⊢ toBilin'Aux
(AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R₂) (x : BilinForm R₂ ((fun x => n → R₂) 1)),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R₂) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
B) =
B
[PROOFSTEP]
convert toBilin'Aux_toMatrixAux B
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
src✝ : BilinForm R₂ ((fun x => n → R₂) 1) →ₗ[R₂] Matrix n n R₂ :=
toMatrixAux fun j => ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1
M : Matrix n n R₂
⊢ AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R₂) (x : BilinForm R₂ ((fun x => n → R₂) 1)),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R₂) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
(toBilin'Aux M) =
M
[PROOFSTEP]
ext i j
[GOAL]
case a.h
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
src✝ : BilinForm R₂ ((fun x => n → R₂) 1) →ₗ[R₂] Matrix n n R₂ :=
toMatrixAux fun j => ↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1
M : Matrix n n R₂
i j : n
⊢ AddHom.toFun
{ toAddHom := src✝.toAddHom,
map_smul' :=
(_ :
∀ (r : R₂) (x : BilinForm R₂ ((fun x => n → R₂) 1)),
AddHom.toFun src✝.toAddHom (r • x) = ↑(RingHom.id R₂) r • AddHom.toFun src✝.toAddHom x) }.toAddHom
(toBilin'Aux M) i j =
M i j
[PROOFSTEP]
simp only [toFun_eq_coe, BilinForm.toMatrixAux_apply, Matrix.toBilin'Aux_stdBasis]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
M : Matrix n n R₂
v w : n → R₂
⊢ bilin (↑toBilin' M) v w = v ⬝ᵥ mulVec M w
[PROOFSTEP]
simp_rw [Matrix.toBilin'_apply, Matrix.dotProduct, Matrix.mulVec, Matrix.dotProduct]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
M : Matrix n n R₂
v w : n → R₂
⊢ ∑ i : n, ∑ j : n, v i * M i j * w j = ∑ x : n, v x * ∑ x_1 : n, M x x_1 * w x_1
[PROOFSTEP]
refine' Finset.sum_congr rfl fun _ _ => _
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
M : Matrix n n R₂
v w : n → R₂
x✝¹ : n
x✝ : x✝¹ ∈ univ
⊢ ∑ j : n, v x✝¹ * M x✝¹ j * w j = v x✝¹ * ∑ x : n, M x✝¹ x * w x
[PROOFSTEP]
rw [Finset.mul_sum]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
M : Matrix n n R₂
v w : n → R₂
x✝¹ : n
x✝ : x✝¹ ∈ univ
⊢ ∑ j : n, v x✝¹ * M x✝¹ j * w j = ∑ x : n, v x✝¹ * (M x✝¹ x * w x)
[PROOFSTEP]
refine' Finset.sum_congr rfl fun _ _ => _
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
M : Matrix n n R₂
v w : n → R₂
x✝³ : n
x✝² : x✝³ ∈ univ
x✝¹ : n
x✝ : x✝¹ ∈ univ
⊢ v x✝³ * M x✝³ x✝¹ * w x✝¹ = v x✝³ * (M x✝³ x✝¹ * w x✝¹)
[PROOFSTEP]
rw [← mul_assoc]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
⊢ ↑toMatrix' (comp B l r) = (↑LinearMap.toMatrix' l)ᵀ * ↑toMatrix' B * ↑LinearMap.toMatrix' r
[PROOFSTEP]
ext i j
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ ↑toMatrix' (comp B l r) i j = ((↑LinearMap.toMatrix' l)ᵀ * ↑toMatrix' B * ↑LinearMap.toMatrix' r) i j
[PROOFSTEP]
simp only [BilinForm.toMatrix'_apply, BilinForm.comp_apply, transpose_apply, Matrix.mul_apply, LinearMap.toMatrix',
LinearEquiv.coe_mk, sum_mul]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ bilin B (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1)) (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1)) =
∑ x : n,
∑ x_1 : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x_1 i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) x_1) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
rw [sum_comm]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ bilin B (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1)) (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1)) =
∑ y : n,
∑ x : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) y i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) y) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
conv_lhs => rw [← BilinForm.sum_repr_mul_repr_mul (Pi.basisFun R₂ n) (l _) (r _)]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
| bilin B (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1)) (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))
[PROOFSTEP]
rw [← BilinForm.sum_repr_mul_repr_mul (Pi.basisFun R₂ n) (l _) (r _)]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
| bilin B (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1)) (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))
[PROOFSTEP]
rw [← BilinForm.sum_repr_mul_repr_mul (Pi.basisFun R₂ n) (l _) (r _)]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
| bilin B (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1)) (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))
[PROOFSTEP]
rw [← BilinForm.sum_repr_mul_repr_mul (Pi.basisFun R₂ n) (l _) (r _)]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ (Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) fun i xi =>
Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) fun j yj =>
xi • yj • bilin B (↑(Pi.basisFun R₂ n) i) (↑(Pi.basisFun R₂ n) j)) =
∑ y : n,
∑ x : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) y i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) y) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
rw [Finsupp.sum_fintype]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ (∑ i_1 : n,
Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) fun j yj =>
↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i_1 •
yj • bilin B (↑(Pi.basisFun R₂ n) i_1) (↑(Pi.basisFun R₂ n) j)) =
∑ y : n,
∑ x : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) y i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) y) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
apply sum_congr rfl
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ ∀ (x : n),
x ∈ univ →
(Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) fun j yj =>
↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) x •
yj • bilin B (↑(Pi.basisFun R₂ n) x) (↑(Pi.basisFun R₂ n) j)) =
∑ x_1 : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x_1) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x_1 j
[PROOFSTEP]
rintro i' -
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i' : n
⊢ (Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) fun j yj =>
↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i' •
yj • bilin B (↑(Pi.basisFun R₂ n) i') (↑(Pi.basisFun R₂ n) j)) =
∑ x : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) i' i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) i') 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
rw [Finsupp.sum_fintype]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i' : n
⊢ ∑ i_1 : n,
↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i' •
↑(↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) i_1 •
bilin B (↑(Pi.basisFun R₂ n) i') (↑(Pi.basisFun R₂ n) i_1) =
∑ x : n,
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) i' i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) i') 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
apply sum_congr rfl
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i' : n
⊢ ∀ (x : n),
x ∈ univ →
↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i' •
↑(↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) x •
bilin B (↑(Pi.basisFun R₂ n) i') (↑(Pi.basisFun R₂ n) x) =
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) i' i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) i') 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) x) 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) x j
[PROOFSTEP]
rintro j' -
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i' j' : n
⊢ ↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i' •
↑(↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) j' •
bilin B (↑(Pi.basisFun R₂ n) i') (↑(Pi.basisFun R₂ n) j') =
↑of (fun i j => ↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) i' i *
bilin B (↑(LinearMap.stdBasis R₂ (fun x => R₂) i') 1) (↑(LinearMap.stdBasis R₂ (fun x => R₂) j') 1) *
↑of (fun i j => ↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1) i) j' j
[PROOFSTEP]
simp only [smul_eq_mul, Pi.basisFun_repr, mul_assoc, mul_comm, mul_left_comm, Pi.basisFun_apply, of_apply]
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i' : n
⊢ ∀ (i_1 : n),
↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i' •
0 • bilin B (↑(Pi.basisFun R₂ n) i') (↑(Pi.basisFun R₂ n) i_1) =
0
[PROOFSTEP]
intros
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i' i✝ : n
⊢ ↑(↑(Pi.basisFun R₂ n).repr (↑l (↑(LinearMap.stdBasis R₂ (fun x => R₂) i) 1))) i' •
0 • bilin B (↑(Pi.basisFun R₂ n) i') (↑(Pi.basisFun R₂ n) i✝) =
0
[PROOFSTEP]
simp only [zero_smul, smul_zero]
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
⊢ ∀ (i : n),
(Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) fun j yj =>
0 • yj • bilin B (↑(Pi.basisFun R₂ n) i) (↑(Pi.basisFun R₂ n) j)) =
0
[PROOFSTEP]
intros
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
l r : (o → R₂) →ₗ[R₂] n → R₂
i j : o
i✝ : n
⊢ (Finsupp.sum (↑(Pi.basisFun R₂ n).repr (↑r (↑(LinearMap.stdBasis R₂ (fun x => R₂) j) 1))) fun j yj =>
0 • yj • bilin B (↑(Pi.basisFun R₂ n) i✝) (↑(Pi.basisFun R₂ n) j)) =
0
[PROOFSTEP]
simp only [zero_smul, Finsupp.sum_zero]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
f : (n → R₂) →ₗ[R₂] n → R₂
⊢ ↑toMatrix' (compLeft B f) = (↑LinearMap.toMatrix' f)ᵀ * ↑toMatrix' B
[PROOFSTEP]
simp only [BilinForm.compLeft, BilinForm.toMatrix'_comp, toMatrix'_id, Matrix.mul_one]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M
inst✝¹⁶ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
f : (n → R₂) →ₗ[R₂] n → R₂
⊢ ↑toMatrix' (compRight B f) = ↑toMatrix' B * ↑LinearMap.toMatrix' f
[PROOFSTEP]
simp only [BilinForm.compRight, BilinForm.toMatrix'_comp, toMatrix'_id, transpose_one, Matrix.one_mul]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
M : Matrix o n R₂
N : Matrix n o R₂
⊢ M * ↑toMatrix' B * N = ↑toMatrix' (comp B (↑Matrix.toLin' Mᵀ) (↑Matrix.toLin' N))
[PROOFSTEP]
simp only [B.toMatrix'_comp, transpose_transpose, toMatrix'_toLin']
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
M : Matrix n n R₂
⊢ M * ↑toMatrix' B = ↑toMatrix' (compLeft B (↑Matrix.toLin' Mᵀ))
[PROOFSTEP]
simp only [toMatrix'_compLeft, transpose_transpose, toMatrix'_toLin']
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B✝ : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
B : BilinForm R₂ (n → R₂)
M : Matrix n n R₂
⊢ ↑toMatrix' B * M = ↑toMatrix' (compRight B (↑Matrix.toLin' M))
[PROOFSTEP]
simp only [toMatrix'_compRight, toMatrix'_toLin']
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁸ : Semiring R
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁵ : Ring R₁
inst✝¹⁴ : AddCommGroup M₁
inst✝¹³ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹² : CommSemiring R₂
inst✝¹¹ : AddCommMonoid M₂
inst✝¹⁰ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁹ : CommRing R₃
inst✝⁸ : AddCommGroup M₃
inst✝⁷ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁶ : Field K
inst✝⁵ : AddCommGroup V
inst✝⁴ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝³ : Fintype n
inst✝² : Fintype o
inst✝¹ : DecidableEq n
inst✝ : DecidableEq o
M : Matrix n n R₂
P Q : Matrix n o R₂
⊢ ↑BilinForm.toMatrix' (BilinForm.comp (↑toBilin' M) (↑toLin' P) (↑toLin' Q)) =
↑BilinForm.toMatrix' (↑toBilin' (Pᵀ * M * Q))
[PROOFSTEP]
simp only [BilinForm.toMatrix'_comp, BilinForm.toMatrix'_toBilin', toMatrix'_toLin']
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
B : BilinForm R₂ M₂
i j : n
⊢ ↑(toMatrix b) B i j = bilin B (↑b i) (↑b j)
[PROOFSTEP]
rw [BilinForm.toMatrix, LinearEquiv.trans_apply, BilinForm.toMatrix'_apply, congr_apply, b.equivFun_symm_stdBasis,
b.equivFun_symm_stdBasis]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
M : Matrix n n R₂
x y : M₂
⊢ bilin (↑(toBilin b) M) x y = ∑ i : n, ∑ j : n, ↑(↑b.repr x) i * M i j * ↑(↑b.repr y) j
[PROOFSTEP]
rw [Matrix.toBilin, BilinForm.toMatrix, LinearEquiv.symm_trans_apply, ← Matrix.toBilin']
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
M : Matrix n n R₂
x y : M₂
⊢ bilin (↑(LinearEquiv.symm (BilinForm.congr (Basis.equivFun b))) (↑toBilin' M)) x y =
∑ i : n, ∑ j : n, ↑(↑b.repr x) i * M i j * ↑(↑b.repr y) j
[PROOFSTEP]
simp only [congr_symm, congr_apply, LinearEquiv.symm_symm, Matrix.toBilin'_apply, Basis.equivFun_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
B : BilinForm R₂ M₂
i j : n
⊢ ↑(toMatrixAux ↑b) B i j = ↑(BilinForm.toMatrix b) B i j
[PROOFSTEP]
rw [BilinForm.toMatrix_apply, BilinForm.toMatrixAux_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
⊢ toBilin (Pi.basisFun R₂ n) = toBilin'
[PROOFSTEP]
ext M
[GOAL]
case h.H
R : Type u_1
M✝ : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
M : Matrix n n R₂
x✝ y✝ : n → R₂
⊢ bilin (↑(toBilin (Pi.basisFun R₂ n)) M) x✝ y✝ = bilin (↑toBilin' M) x✝ y✝
[PROOFSTEP]
simp only [Matrix.toBilin_apply, Matrix.toBilin'_apply, Pi.basisFun_repr]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
⊢ toMatrix (Pi.basisFun R₂ n) = toMatrix'
[PROOFSTEP]
ext B
[GOAL]
case h.a.h
R : Type u_1
M : Type u_2
inst✝¹⁷ : Semiring R
inst✝¹⁶ : AddCommMonoid M
inst✝¹⁵ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁴ : Ring R₁
inst✝¹³ : AddCommGroup M₁
inst✝¹² : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹¹ : CommSemiring R₂
inst✝¹⁰ : AddCommMonoid M₂
inst✝⁹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁸ : CommRing R₃
inst✝⁷ : AddCommGroup M₃
inst✝⁶ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁵ : Field K
inst✝⁴ : AddCommGroup V
inst✝³ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝² : Fintype n
inst✝¹ : Fintype o
inst✝ : DecidableEq n
b : Basis n R₂ M₂
B : BilinForm R₂ (n → R₂)
i✝ x✝ : n
⊢ ↑(toMatrix (Pi.basisFun R₂ n)) B i✝ x✝ = ↑toMatrix' B i✝ x✝
[PROOFSTEP]
rw [BilinForm.toMatrix_apply, BilinForm.toMatrix'_apply, Pi.basisFun_apply, Pi.basisFun_apply]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
⊢ ↑(toMatrix c) (comp B l r) = (↑(LinearMap.toMatrix c b) l)ᵀ * ↑(toMatrix b) B * ↑(LinearMap.toMatrix c b) r
[PROOFSTEP]
ext i j
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ ↑(toMatrix c) (comp B l r) i j = ((↑(LinearMap.toMatrix c b) l)ᵀ * ↑(toMatrix b) B * ↑(LinearMap.toMatrix c b) r) i j
[PROOFSTEP]
simp only [BilinForm.toMatrix_apply, BilinForm.comp_apply, transpose_apply, Matrix.mul_apply, LinearMap.toMatrix',
LinearEquiv.coe_mk, sum_mul]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ bilin B (↑l (↑c i)) (↑r (↑c j)) =
∑ x : n, ∑ x_1 : n, ↑(LinearMap.toMatrix c b) l x_1 i * bilin B (↑b x_1) (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
rw [sum_comm]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ bilin B (↑l (↑c i)) (↑r (↑c j)) =
∑ y : n, ∑ x : n, ↑(LinearMap.toMatrix c b) l y i * bilin B (↑b y) (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
conv_lhs => rw [← BilinForm.sum_repr_mul_repr_mul b]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
| bilin B (↑l (↑c i)) (↑r (↑c j))
[PROOFSTEP]
rw [← BilinForm.sum_repr_mul_repr_mul b]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
| bilin B (↑l (↑c i)) (↑r (↑c j))
[PROOFSTEP]
rw [← BilinForm.sum_repr_mul_repr_mul b]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
| bilin B (↑l (↑c i)) (↑r (↑c j))
[PROOFSTEP]
rw [← BilinForm.sum_repr_mul_repr_mul b]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ (Finsupp.sum (↑b.repr (↑l (↑c i))) fun i xi =>
Finsupp.sum (↑b.repr (↑r (↑c j))) fun j yj => xi • yj • bilin B (↑b i) (↑b j)) =
∑ y : n, ∑ x : n, ↑(LinearMap.toMatrix c b) l y i * bilin B (↑b y) (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
rw [Finsupp.sum_fintype]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ (∑ i_1 : n, Finsupp.sum (↑b.repr (↑r (↑c j))) fun j yj => ↑(↑b.repr (↑l (↑c i))) i_1 • yj • bilin B (↑b i_1) (↑b j)) =
∑ y : n, ∑ x : n, ↑(LinearMap.toMatrix c b) l y i * bilin B (↑b y) (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
apply sum_congr rfl
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ ∀ (x : n),
x ∈ univ →
(Finsupp.sum (↑b.repr (↑r (↑c j))) fun j yj => ↑(↑b.repr (↑l (↑c i))) x • yj • bilin B (↑b x) (↑b j)) =
∑ x_1 : n, ↑(LinearMap.toMatrix c b) l x i * bilin B (↑b x) (↑b x_1) * ↑(LinearMap.toMatrix c b) r x_1 j
[PROOFSTEP]
rintro i' -
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i' : n
⊢ (Finsupp.sum (↑b.repr (↑r (↑c j))) fun j yj => ↑(↑b.repr (↑l (↑c i))) i' • yj • bilin B (↑b i') (↑b j)) =
∑ x : n, ↑(LinearMap.toMatrix c b) l i' i * bilin B (↑b i') (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
rw [Finsupp.sum_fintype]
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i' : n
⊢ ∑ i_1 : n, ↑(↑b.repr (↑l (↑c i))) i' • ↑(↑b.repr (↑r (↑c j))) i_1 • bilin B (↑b i') (↑b i_1) =
∑ x : n, ↑(LinearMap.toMatrix c b) l i' i * bilin B (↑b i') (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
apply sum_congr rfl
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i' : n
⊢ ∀ (x : n),
x ∈ univ →
↑(↑b.repr (↑l (↑c i))) i' • ↑(↑b.repr (↑r (↑c j))) x • bilin B (↑b i') (↑b x) =
↑(LinearMap.toMatrix c b) l i' i * bilin B (↑b i') (↑b x) * ↑(LinearMap.toMatrix c b) r x j
[PROOFSTEP]
rintro j' -
[GOAL]
case a.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i' j' : n
⊢ ↑(↑b.repr (↑l (↑c i))) i' • ↑(↑b.repr (↑r (↑c j))) j' • bilin B (↑b i') (↑b j') =
↑(LinearMap.toMatrix c b) l i' i * bilin B (↑b i') (↑b j') * ↑(LinearMap.toMatrix c b) r j' j
[PROOFSTEP]
simp only [smul_eq_mul, LinearMap.toMatrix_apply, Basis.equivFun_apply, mul_assoc, mul_comm, mul_left_comm]
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i' : n
⊢ ∀ (i_1 : n), ↑(↑b.repr (↑l (↑c i))) i' • 0 • bilin B (↑b i') (↑b i_1) = 0
[PROOFSTEP]
intros
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i' i✝ : n
⊢ ↑(↑b.repr (↑l (↑c i))) i' • 0 • bilin B (↑b i') (↑b i✝) = 0
[PROOFSTEP]
simp only [zero_smul, smul_zero]
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
⊢ ∀ (i : n), (Finsupp.sum (↑b.repr (↑r (↑c j))) fun j yj => 0 • yj • bilin B (↑b i) (↑b j)) = 0
[PROOFSTEP]
intros
[GOAL]
case a.h.h
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
l r : M₂' →ₗ[R₂] M₂
i j : o
i✝ : n
⊢ (Finsupp.sum (↑b.repr (↑r (↑c j))) fun j yj => 0 • yj • bilin B (↑b i✝) (↑b j)) = 0
[PROOFSTEP]
simp only [zero_smul, Finsupp.sum_zero]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
f : M₂ →ₗ[R₂] M₂
⊢ ↑(toMatrix b) (compLeft B f) = (↑(LinearMap.toMatrix b b) f)ᵀ * ↑(toMatrix b) B
[PROOFSTEP]
simp only [compLeft, BilinForm.toMatrix_comp b b, toMatrix_id, Matrix.mul_one]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
f : M₂ →ₗ[R₂] M₂
⊢ ↑(toMatrix b) (compRight B f) = ↑(toMatrix b) B * ↑(LinearMap.toMatrix b b) f
[PROOFSTEP]
simp only [BilinForm.compRight, BilinForm.toMatrix_comp b b, toMatrix_id, transpose_one, Matrix.one_mul]
[GOAL]
R : Type u_1
M : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M
inst✝¹⁸ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c✝ : Basis o R₂ M₂'
inst✝ : DecidableEq o
c : Basis o R₂ M₂
B : BilinForm R₂ M₂
⊢ (Basis.toMatrix b ↑c)ᵀ * ↑(toMatrix b) B * Basis.toMatrix b ↑c = ↑(toMatrix c) B
[PROOFSTEP]
rw [← LinearMap.toMatrix_id_eq_basis_toMatrix, ← BilinForm.toMatrix_comp, BilinForm.comp_id_id]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M✝
inst✝¹⁸ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
M : Matrix o n R₂
N : Matrix n o R₂
⊢ M * ↑(toMatrix b) B * N = ↑(toMatrix c) (comp B (↑(Matrix.toLin c b) Mᵀ) (↑(Matrix.toLin c b) N))
[PROOFSTEP]
simp only [B.toMatrix_comp b c, toMatrix_toLin, transpose_transpose]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M✝
inst✝¹⁸ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
M : Matrix n n R₂
⊢ M * ↑(toMatrix b) B = ↑(toMatrix b) (compLeft B (↑(Matrix.toLin b b) Mᵀ))
[PROOFSTEP]
rw [B.toMatrix_compLeft b, toMatrix_toLin, transpose_transpose]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M✝
inst✝¹⁸ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B✝ : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
B : BilinForm R₂ M₂
M : Matrix n n R₂
⊢ ↑(toMatrix b) B * M = ↑(toMatrix b) (compRight B (↑(Matrix.toLin b b) M))
[PROOFSTEP]
rw [B.toMatrix_compRight b, toMatrix_toLin]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝²⁰ : Semiring R
inst✝¹⁹ : AddCommMonoid M✝
inst✝¹⁸ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁷ : Ring R₁
inst✝¹⁶ : AddCommGroup M₁
inst✝¹⁵ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁴ : CommSemiring R₂
inst✝¹³ : AddCommMonoid M₂
inst✝¹² : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹¹ : CommRing R₃
inst✝¹⁰ : AddCommGroup M₃
inst✝⁹ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁸ : Field K
inst✝⁷ : AddCommGroup V
inst✝⁶ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
o : Type u_12
inst✝⁵ : Fintype n
inst✝⁴ : Fintype o
inst✝³ : DecidableEq n
b : Basis n R₂ M₂
M₂' : Type u_13
inst✝² : AddCommMonoid M₂'
inst✝¹ : Module R₂ M₂'
c : Basis o R₂ M₂'
inst✝ : DecidableEq o
M : Matrix n n R₂
P Q : Matrix n o R₂
⊢ ↑(BilinForm.toMatrix c) (BilinForm.comp (↑(toBilin b) M) (↑(toLin c b) P) (↑(toLin c b) Q)) =
↑(BilinForm.toMatrix c) (↑(toBilin c) (Pᵀ * M * Q))
[PROOFSTEP]
simp only [BilinForm.toMatrix_comp b c, BilinForm.toMatrix_toBilin, toMatrix_toLin]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ BilinForm.IsAdjointPair (↑toBilin' J) (↑toBilin' J₃) (↑toLin' A) (↑toLin' A') ↔ IsAdjointPair J J₃ A A'
[PROOFSTEP]
rw [BilinForm.isAdjointPair_iff_compLeft_eq_compRight]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ BilinForm.compLeft (↑toBilin' J₃) (↑toLin' A) = BilinForm.compRight (↑toBilin' J) (↑toLin' A') ↔
IsAdjointPair J J₃ A A'
[PROOFSTEP]
have h : ∀ B B' : BilinForm R₃ (n → R₃), B = B' ↔ BilinForm.toMatrix' B = BilinForm.toMatrix' B' :=
by
intro B B'
constructor <;> intro h
· rw [h]
· exact BilinForm.toMatrix'.injective h
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ ∀ (B B' : BilinForm R₃ (n → R₃)), B = B' ↔ ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
[PROOFSTEP]
intro B B'
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ (n → R₃)
⊢ B = B' ↔ ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
[PROOFSTEP]
constructor
[GOAL]
case mp
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ (n → R₃)
⊢ B = B' → ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
[PROOFSTEP]
intro h
[GOAL]
case mpr
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ (n → R₃)
⊢ ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B' → B = B'
[PROOFSTEP]
intro h
[GOAL]
case mp
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ (n → R₃)
h : B = B'
⊢ ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
[PROOFSTEP]
rw [h]
[GOAL]
case mpr
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ (n → R₃)
h : ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
⊢ B = B'
[PROOFSTEP]
exact BilinForm.toMatrix'.injective h
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
h : ∀ (B B' : BilinForm R₃ (n → R₃)), B = B' ↔ ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
⊢ BilinForm.compLeft (↑toBilin' J₃) (↑toLin' A) = BilinForm.compRight (↑toBilin' J) (↑toLin' A') ↔
IsAdjointPair J J₃ A A'
[PROOFSTEP]
rw [h, BilinForm.toMatrix'_compLeft, BilinForm.toMatrix'_compRight, LinearMap.toMatrix'_toLin',
LinearMap.toMatrix'_toLin', BilinForm.toMatrix'_toBilin', BilinForm.toMatrix'_toBilin']
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
h : ∀ (B B' : BilinForm R₃ (n → R₃)), B = B' ↔ ↑BilinForm.toMatrix' B = ↑BilinForm.toMatrix' B'
⊢ Aᵀ * J₃ = J * A' ↔ IsAdjointPair J J₃ A A'
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ BilinForm.IsAdjointPair (↑(toBilin b) J) (↑(toBilin b) J₃) (↑(toLin b b) A) (↑(toLin b b) A') ↔
IsAdjointPair J J₃ A A'
[PROOFSTEP]
rw [BilinForm.isAdjointPair_iff_compLeft_eq_compRight]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ BilinForm.compLeft (↑(toBilin b) J₃) (↑(toLin b b) A) = BilinForm.compRight (↑(toBilin b) J) (↑(toLin b b) A') ↔
IsAdjointPair J J₃ A A'
[PROOFSTEP]
have h : ∀ B B' : BilinForm R₃ M₃, B = B' ↔ BilinForm.toMatrix b B = BilinForm.toMatrix b B' :=
by
intro B B'
constructor <;> intro h
· rw [h]
· exact (BilinForm.toMatrix b).injective h
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ ∀ (B B' : BilinForm R₃ M₃), B = B' ↔ ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
[PROOFSTEP]
intro B B'
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ M₃
⊢ B = B' ↔ ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
[PROOFSTEP]
constructor
[GOAL]
case mp
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ M₃
⊢ B = B' → ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
[PROOFSTEP]
intro h
[GOAL]
case mpr
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ M₃
⊢ ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B' → B = B'
[PROOFSTEP]
intro h
[GOAL]
case mp
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ M₃
h : B = B'
⊢ ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
[PROOFSTEP]
rw [h]
[GOAL]
case mpr
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
B B' : BilinForm R₃ M₃
h : ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
⊢ B = B'
[PROOFSTEP]
exact (BilinForm.toMatrix b).injective h
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
h : ∀ (B B' : BilinForm R₃ M₃), B = B' ↔ ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
⊢ BilinForm.compLeft (↑(toBilin b) J₃) (↑(toLin b b) A) = BilinForm.compRight (↑(toBilin b) J) (↑(toLin b b) A') ↔
IsAdjointPair J J₃ A A'
[PROOFSTEP]
rw [h, BilinForm.toMatrix_compLeft, BilinForm.toMatrix_compRight, LinearMap.toMatrix_toLin, LinearMap.toMatrix_toLin,
BilinForm.toMatrix_toBilin, BilinForm.toMatrix_toBilin]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
h : ∀ (B B' : BilinForm R₃ M₃), B = B' ↔ ↑(BilinForm.toMatrix b) B = ↑(BilinForm.toMatrix b) B'
⊢ Aᵀ * J₃ = J * A' ↔ IsAdjointPair J J₃ A A'
[PROOFSTEP]
rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
have h' : IsUnit P.det := P.isUnit_iff_isUnit_det.mp h
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
let u := P.nonsingInvUnit h'
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
have coe_u : (u : Matrix n n R₃) = P := rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
have coe_u_inv : (↑u⁻¹ : Matrix n n R₃) = P⁻¹ := rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
let v := Pᵀ.nonsingInvUnit (P.isUnit_det_transpose h')
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
have coe_v : (v : Matrix n n R₃) = Pᵀ := rfl
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
have coe_v_inv : (↑v⁻¹ : Matrix n n R₃) = P⁻¹ᵀ := P.transpose_nonsing_inv.symm
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
set x := Aᵀ * Pᵀ * J with x_def
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
set y := J * P * A' with y_def
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
y : Matrix n n R₃ := J * P * A'
y_def : y = J * P * A'
⊢ IsAdjointPair (Pᵀ * J * P) (Pᵀ * J * P) A A' ↔ IsAdjointPair J J (P * A * P⁻¹) (P * A' * P⁻¹)
[PROOFSTEP]
simp only [Matrix.IsAdjointPair]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
y : Matrix n n R₃ := J * P * A'
y_def : y = J * P * A'
⊢ Aᵀ * (Pᵀ * J * P) = Pᵀ * J * P * A' ↔ (P * A * P⁻¹)ᵀ * J = J * (P * A' * P⁻¹)
[PROOFSTEP]
calc
(Aᵀ * (Pᵀ * J * P) = Pᵀ * J * P * A') ↔ (x * ↑u = ↑v * y) := ?_
_ ↔ (↑v⁻¹ * x = y * ↑u⁻¹) := ?_
_ ↔ ((P * A * P⁻¹)ᵀ * J = J * (P * A' * P⁻¹)) := ?_
[GOAL]
case calc_1
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
y : Matrix n n R₃ := J * P * A'
y_def : y = J * P * A'
⊢ Aᵀ * (Pᵀ * J * P) = Pᵀ * J * P * A' ↔ x * ↑u = ↑v * y
[PROOFSTEP]
simp only [mul_assoc, x_def, y_def, coe_u, coe_v]
[GOAL]
case calc_2
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
y : Matrix n n R₃ := J * P * A'
y_def : y = J * P * A'
⊢ x * ↑u = ↑v * y ↔ ↑v⁻¹ * x = y * ↑u⁻¹
[PROOFSTEP]
rw [Units.eq_mul_inv_iff_mul_eq, mul_assoc (↑v⁻¹) x, Units.inv_mul_eq_iff_eq_mul]
[GOAL]
case calc_3
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
y : Matrix n n R₃ := J * P * A'
y_def : y = J * P * A'
⊢ ↑v⁻¹ * x = y * ↑u⁻¹ ↔ (P * A * P⁻¹)ᵀ * J = J * (P * A' * P⁻¹)
[PROOFSTEP]
rw [x_def, y_def, coe_u_inv, coe_v_inv]
[GOAL]
case calc_3
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
P : Matrix n n R₃
h : IsUnit P
h' : IsUnit (det P)
u : (Matrix n n R₃)ˣ := nonsingInvUnit P h'
coe_u : ↑u = P
coe_u_inv : ↑u⁻¹ = P⁻¹
v : (Matrix n n R₃)ˣ := nonsingInvUnit Pᵀ (_ : IsUnit (det Pᵀ))
coe_v : ↑v = Pᵀ
coe_v_inv : ↑v⁻¹ = P⁻¹ᵀ
x : Matrix n n R₃ := Aᵀ * Pᵀ * J
x_def : x = Aᵀ * Pᵀ * J
y : Matrix n n R₃ := J * P * A'
y_def : y = J * P * A'
⊢ P⁻¹ᵀ * (Aᵀ * Pᵀ * J) = J * P * A' * P⁻¹ ↔ (P * A * P⁻¹)ᵀ * J = J * (P * A' * P⁻¹)
[PROOFSTEP]
simp only [Matrix.mul_assoc, Matrix.transpose_mul]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ A ∈ pairSelfAdjointMatricesSubmodule J J₃ ↔ IsAdjointPair J J₃ A A
[PROOFSTEP]
simp only [mem_pairSelfAdjointMatricesSubmodule]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ A ∈ selfAdjointMatricesSubmodule J ↔ Matrix.IsSelfAdjoint J A
[PROOFSTEP]
simp only [mem_selfAdjointMatricesSubmodule]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁶ : Semiring R
inst✝¹⁵ : AddCommMonoid M
inst✝¹⁴ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹³ : Ring R₁
inst✝¹² : AddCommGroup M₁
inst✝¹¹ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹⁰ : CommSemiring R₂
inst✝⁹ : AddCommMonoid M₂
inst✝⁸ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝⁷ : CommRing R₃
inst✝⁶ : AddCommGroup M₃
inst✝⁵ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁴ : Field K
inst✝³ : AddCommGroup V
inst✝² : Module K V
B : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
n : Type u_11
inst✝¹ : Fintype n
b : Basis n R₃ M₃
J J₃ A A' : Matrix n n R₃
inst✝ : DecidableEq n
⊢ A ∈ skewAdjointMatricesSubmodule J ↔ IsSkewAdjoint J A
[PROOFSTEP]
simp only [mem_skewAdjointMatricesSubmodule]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁹ : Semiring R
inst✝¹⁸ : AddCommMonoid M✝
inst✝¹⁷ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁶ : Ring R₁
inst✝¹⁵ : AddCommGroup M₁
inst✝¹⁴ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹³ : CommSemiring R₂
inst✝¹² : AddCommMonoid M₂
inst✝¹¹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹⁰ : CommRing R₃
inst✝⁹ : AddCommGroup M₃
inst✝⁸ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁷ : Field K
inst✝⁶ : AddCommGroup V
inst✝⁵ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
A : Type u_11
inst✝⁴ : CommRing A
inst✝³ : IsDomain A
inst✝² : Module A M₃
B₃ : BilinForm A M₃
ι : Type u_12
inst✝¹ : DecidableEq ι
inst✝ : Fintype ι
M : Matrix ι ι R₃
h : Matrix.Nondegenerate M
x : ι → R₃
hx : ∀ (n : ι → R₃), bilin (↑Matrix.toBilin' M) x n = 0
y : ι → R₃
⊢ x ⬝ᵥ mulVec M y = 0
[PROOFSTEP]
simpa only [toBilin'_apply'] using hx y
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁹ : Semiring R
inst✝¹⁸ : AddCommMonoid M✝
inst✝¹⁷ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁶ : Ring R₁
inst✝¹⁵ : AddCommGroup M₁
inst✝¹⁴ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹³ : CommSemiring R₂
inst✝¹² : AddCommMonoid M₂
inst✝¹¹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹⁰ : CommRing R₃
inst✝⁹ : AddCommGroup M₃
inst✝⁸ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁷ : Field K
inst✝⁶ : AddCommGroup V
inst✝⁵ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
A : Type u_11
inst✝⁴ : CommRing A
inst✝³ : IsDomain A
inst✝² : Module A M₃
B₃ : BilinForm A M₃
ι : Type u_12
inst✝¹ : DecidableEq ι
inst✝ : Fintype ι
M : Matrix ι ι R₃
b : Basis ι R₃ M₃
⊢ Nondegenerate (↑(toBilin b) M) ↔ Matrix.Nondegenerate M
[PROOFSTEP]
rw [← Matrix.nondegenerate_toBilin'_iff_nondegenerate_toBilin, Matrix.nondegenerate_toBilin'_iff]
[GOAL]
R : Type u_1
M✝ : Type u_2
inst✝¹⁹ : Semiring R
inst✝¹⁸ : AddCommMonoid M✝
inst✝¹⁷ : Module R M✝
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁶ : Ring R₁
inst✝¹⁵ : AddCommGroup M₁
inst✝¹⁴ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹³ : CommSemiring R₂
inst✝¹² : AddCommMonoid M₂
inst✝¹¹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹⁰ : CommRing R₃
inst✝⁹ : AddCommGroup M₃
inst✝⁸ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁷ : Field K
inst✝⁶ : AddCommGroup V
inst✝⁵ : Module K V
B : BilinForm R M✝
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
A : Type u_11
inst✝⁴ : CommRing A
inst✝³ : IsDomain A
inst✝² : Module A M₃
B₃ : BilinForm A M₃
ι : Type u_12
inst✝¹ : DecidableEq ι
inst✝ : Fintype ι
M : Matrix ι ι A
⊢ Nondegenerate (↑toBilin' M) ↔ det M ≠ 0
[PROOFSTEP]
rw [Matrix.nondegenerate_toBilin'_iff, Matrix.nondegenerate_iff_det_ne_zero]
[GOAL]
R : Type u_1
M : Type u_2
inst✝¹⁹ : Semiring R
inst✝¹⁸ : AddCommMonoid M
inst✝¹⁷ : Module R M
R₁ : Type u_3
M₁ : Type u_4
inst✝¹⁶ : Ring R₁
inst✝¹⁵ : AddCommGroup M₁
inst✝¹⁴ : Module R₁ M₁
R₂ : Type u_5
M₂ : Type u_6
inst✝¹³ : CommSemiring R₂
inst✝¹² : AddCommMonoid M₂
inst✝¹¹ : Module R₂ M₂
R₃ : Type u_7
M₃ : Type u_8
inst✝¹⁰ : CommRing R₃
inst✝⁹ : AddCommGroup M₃
inst✝⁸ : Module R₃ M₃
V : Type u_9
K : Type u_10
inst✝⁷ : Field K
inst✝⁶ : AddCommGroup V
inst✝⁵ : Module K V
B✝ : BilinForm R M
B₁ : BilinForm R₁ M₁
B₂ : BilinForm R₂ M₂
A : Type u_11
inst✝⁴ : CommRing A
inst✝³ : IsDomain A
inst✝² : Module A M₃
B₃ : BilinForm A M₃
ι : Type u_12
inst✝¹ : DecidableEq ι
inst✝ : Fintype ι
B : BilinForm A M₃
b : Basis ι A M₃
⊢ Nondegenerate B ↔ det (↑(toMatrix b) B) ≠ 0
[PROOFSTEP]
rw [← Matrix.nondegenerate_iff_det_ne_zero, nondegenerate_toMatrix_iff]
| {"mathlib_filename": "Mathlib.LinearAlgebra.Matrix.BilinearForm", "llama_tokens": 66498} |
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
s t : Set α
⊢ SeparatedNhds s t ↔ Disjoint (𝓝ˢ s) (𝓝ˢ t)
[PROOFSTEP]
simp only [(hasBasis_nhdsSet s).disjoint_iff (hasBasis_nhdsSet t), SeparatedNhds, exists_prop, ← exists_and_left,
and_assoc, and_comm, and_left_comm]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
s s₁ s₂ t t₁ t₂ u : Set α
⊢ SeparatedNhds s u → SeparatedNhds t u → SeparatedNhds (s ∪ t) u
[PROOFSTEP]
simpa only [separatedNhds_iff_disjoint, nhdsSet_union, disjoint_sup_left] using And.intro
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
⊢ T0Space α ↔ ∀ (x y : α), x ≠ y → ¬Inseparable x y
[PROOFSTEP]
simp only [t0Space_iff_inseparable, Ne.def, not_imp_not]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
b : Set (Set α)
hb : IsTopologicalBasis b
x y : α
h : ∀ (s : Set α), s ∈ b → (x ∈ s ↔ y ∈ s)
⊢ HasBasis (𝓝 y) (fun t => t ∈ b ∧ x ∈ t) fun t => t
[PROOFSTEP]
convert hb.nhds_hasBasis using 2
[GOAL]
case h.e'_4.h.a
α : Type u
β : Type v
inst✝ : TopologicalSpace α
b : Set (Set α)
hb : IsTopologicalBasis b
x y : α
h : ∀ (s : Set α), s ∈ b → (x ∈ s ↔ y ∈ s)
x✝ : Set α
⊢ x✝ ∈ b ∧ x ∈ x✝ ↔ x✝ ∈ b ∧ y ∈ x✝
[PROOFSTEP]
exact and_congr_right (h _)
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
⊢ T0Space α ↔ ∀ (x y : α), x ≠ y → ∃ U, IsOpen U ∧ Xor' (x ∈ U) (y ∈ U)
[PROOFSTEP]
simp only [t0Space_iff_not_inseparable, xor_iff_not_iff, not_forall, exists_prop, inseparable_iff_forall_open]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
⊢ Set.Subsingleton s
[PROOFSTEP]
clear β
[GOAL]
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
⊢ Set.Subsingleton s
[PROOFSTEP]
refine' fun x hx y hy => of_not_not fun hxy => _
[GOAL]
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
⊢ False
[PROOFSTEP]
rcases exists_isOpen_xor'_mem hxy with ⟨U, hUo, hU⟩
[GOAL]
case intro.intro
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
⊢ False
[PROOFSTEP]
wlog h : x ∈ U ∧ y ∉ U
[GOAL]
case intro.intro.inr
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
this :
∀ {α : Type u} [inst : TopologicalSpace α] [inst_1 : T0Space α] {s : Set α},
IsClosed s →
(∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s) →
∀ (x : α),
x ∈ s → ∀ (y : α), y ∈ s → ¬x = y → ∀ (U : Set α), IsOpen U → Xor' (x ∈ U) (y ∈ U) → x ∈ U ∧ ¬y ∈ U → False
h : ¬(x ∈ U ∧ ¬y ∈ U)
⊢ False
[PROOFSTEP]
refine this hs hmin y hy x hx (Ne.symm hxy) U hUo hU.symm (hU.resolve_left h)
[GOAL]
α✝ : Type u
inst✝² : TopologicalSpace α✝
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
h : x ∈ U ∧ ¬y ∈ U
⊢ False
[PROOFSTEP]
cases' h with hxU hyU
[GOAL]
case intro
α✝ : Type u
inst✝² : TopologicalSpace α✝
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
hxU : x ∈ U
hyU : ¬y ∈ U
⊢ False
[PROOFSTEP]
have : s \ U = s := hmin (s \ U) (diff_subset _ _) ⟨y, hy, hyU⟩ (hs.sdiff hUo)
[GOAL]
case intro
α✝ : Type u
inst✝² : TopologicalSpace α✝
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsClosed s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsClosed t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
hxU : x ∈ U
hyU : ¬y ∈ U
this : s \ U = s
⊢ False
[PROOFSTEP]
exact (this.symm.subset hx).2 hxU
[GOAL]
α✝ : Type u
β : Type v
inst✝³ : TopologicalSpace α✝
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : T0Space α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
⊢ ∃ x, x ∈ S ∧ IsClosed {x}
[PROOFSTEP]
obtain ⟨V, Vsub, Vne, Vcls, hV⟩ := hS.exists_minimal_nonempty_closed_subset hne
[GOAL]
case intro.intro.intro.intro
α✝ : Type u
β : Type v
inst✝³ : TopologicalSpace α✝
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : T0Space α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
V : Set α
Vsub : V ⊆ S
Vne : Set.Nonempty V
Vcls : IsClosed V
hV : ∀ (V' : Set α), V' ⊆ V → Set.Nonempty V' → IsClosed V' → V' = V
⊢ ∃ x, x ∈ S ∧ IsClosed {x}
[PROOFSTEP]
rcases minimal_nonempty_closed_eq_singleton Vcls Vne hV with ⟨x, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro
α✝ : Type u
β : Type v
inst✝³ : TopologicalSpace α✝
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : T0Space α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
x : α
Vsub : {x} ⊆ S
Vne : Set.Nonempty {x}
Vcls : IsClosed {x}
hV : ∀ (V' : Set α), V' ⊆ {x} → Set.Nonempty V' → IsClosed V' → V' = {x}
⊢ ∃ x, x ∈ S ∧ IsClosed {x}
[PROOFSTEP]
exact ⟨x, Vsub (mem_singleton x), Vcls⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
⊢ Set.Subsingleton s
[PROOFSTEP]
clear β
[GOAL]
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
⊢ Set.Subsingleton s
[PROOFSTEP]
refine' fun x hx y hy => of_not_not fun hxy => _
[GOAL]
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
⊢ False
[PROOFSTEP]
rcases exists_isOpen_xor'_mem hxy with ⟨U, hUo, hU⟩
[GOAL]
case intro.intro
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
⊢ False
[PROOFSTEP]
wlog h : x ∈ U ∧ y ∉ U
[GOAL]
case intro.intro.inr
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
this :
∀ {α : Type u} [inst : TopologicalSpace α] [inst_1 : T0Space α] {s : Set α},
IsOpen s →
(∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s) →
∀ (x : α),
x ∈ s → ∀ (y : α), y ∈ s → ¬x = y → ∀ (U : Set α), IsOpen U → Xor' (x ∈ U) (y ∈ U) → x ∈ U ∧ ¬y ∈ U → False
h : ¬(x ∈ U ∧ ¬y ∈ U)
⊢ False
[PROOFSTEP]
exact this hs hmin y hy x hx (Ne.symm hxy) U hUo hU.symm (hU.resolve_left h)
[GOAL]
α✝ : Type u
inst✝² : TopologicalSpace α✝
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
h : x ∈ U ∧ ¬y ∈ U
⊢ False
[PROOFSTEP]
cases' h with hxU hyU
[GOAL]
case intro
α✝ : Type u
inst✝² : TopologicalSpace α✝
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
hxU : x ∈ U
hyU : ¬y ∈ U
⊢ False
[PROOFSTEP]
have : s ∩ U = s := hmin (s ∩ U) (inter_subset_left _ _) ⟨x, hx, hxU⟩ (hs.inter hUo)
[GOAL]
case intro
α✝ : Type u
inst✝² : TopologicalSpace α✝
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hs : IsOpen s
hmin : ∀ (t : Set α), t ⊆ s → Set.Nonempty t → IsOpen t → t = s
x : α
hx : x ∈ s
y : α
hy : y ∈ s
hxy : ¬x = y
U : Set α
hUo : IsOpen U
hU : Xor' (x ∈ U) (y ∈ U)
hxU : x ∈ U
hyU : ¬y ∈ U
this : s ∩ U = s
⊢ False
[PROOFSTEP]
exact hyU (this.symm.subset hy).2
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Set α
hfin : Set.Finite s
hne : Set.Nonempty s
ho : IsOpen s
⊢ ∃ x, x ∈ s ∧ IsOpen {x}
[PROOFSTEP]
lift s to Finset α using hfin
[GOAL]
case intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s : Finset α
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
⊢ ∃ x, x ∈ ↑s ∧ IsOpen {x}
[PROOFSTEP]
induction' s using Finset.strongInductionOn with s ihs
[GOAL]
case intro.a
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
⊢ ∃ x, x ∈ ↑s ∧ IsOpen {x}
[PROOFSTEP]
rcases em (∃ t, t ⊂ s ∧ t.Nonempty ∧ IsOpen (t : Set α)) with (⟨t, hts, htne, hto⟩ | ht)
[GOAL]
case intro.a.inl.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
t : Finset α
hts : t ⊂ s
htne : Finset.Nonempty t
hto : IsOpen ↑t
⊢ ∃ x, x ∈ ↑s ∧ IsOpen {x}
[PROOFSTEP]
rcases ihs t hts htne hto with ⟨x, hxt, hxo⟩
[GOAL]
case intro.a.inl.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
t : Finset α
hts : t ⊂ s
htne : Finset.Nonempty t
hto : IsOpen ↑t
x : α
hxt : x ∈ ↑t
hxo : IsOpen {x}
⊢ ∃ x, x ∈ ↑s ∧ IsOpen {x}
[PROOFSTEP]
exact ⟨x, hts.1 hxt, hxo⟩
[GOAL]
case intro.a.inr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
ht : ¬∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
⊢ ∃ x, x ∈ ↑s ∧ IsOpen {x}
[PROOFSTEP]
rsuffices ⟨x, hx⟩ : ∃ x, s.toSet = { x }
[GOAL]
case intro.a.inr.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
ht : ¬∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
x : α
hx : ↑s = {x}
⊢ ∃ x, x ∈ ↑s ∧ IsOpen {x}
[PROOFSTEP]
exact ⟨x, hx.symm ▸ rfl, hx ▸ ho⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
ht : ¬∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
⊢ ∃ x, ↑s = {x}
[PROOFSTEP]
refine minimal_nonempty_open_eq_singleton ho hne ?_
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
ht : ¬∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
⊢ ∀ (t : Set α), t ⊆ ↑s → Set.Nonempty t → IsOpen t → t = ↑s
[PROOFSTEP]
refine' fun t hts htne hto => of_not_not fun hts' => ht _
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
ht : ¬∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
t : Set α
hts : t ⊆ ↑s
htne : Set.Nonempty t
hto : IsOpen t
hts' : ¬t = ↑s
⊢ ∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
[PROOFSTEP]
lift t to Finset α using s.finite_toSet.subset hts
[GOAL]
case intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T0Space α
s✝ : Finset α
hne✝ : Set.Nonempty ↑s✝
ho✝ : IsOpen ↑s✝
s : Finset α
ihs : ∀ (t : Finset α), t ⊂ s → Set.Nonempty ↑t → IsOpen ↑t → ∃ x, x ∈ ↑t ∧ IsOpen {x}
hne : Set.Nonempty ↑s
ho : IsOpen ↑s
ht : ¬∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
t : Finset α
hts : ↑t ⊆ ↑s
htne : Set.Nonempty ↑t
hto : IsOpen ↑t
hts' : ¬↑t = ↑s
⊢ ∃ t, t ⊂ s ∧ Finset.Nonempty t ∧ IsOpen ↑t
[PROOFSTEP]
exact ⟨t, ssubset_iff_subset_ne.2 ⟨hts, mt Finset.coe_inj.2 hts'⟩, htne, hto⟩
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
⊢ T0Space α ↔ ∀ (a b : α), a ≠ b → ¬a ∈ closure {b} ∨ ¬b ∈ closure {a}
[PROOFSTEP]
simp only [t0Space_iff_not_inseparable, inseparable_iff_mem_closure, not_and_or]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
h : ∀ (x y : α), Inseparable x y → ∃ s, x ∈ s ∧ y ∈ s ∧ T0Space ↑s
⊢ T0Space α
[PROOFSTEP]
refine' ⟨fun x y hxy => _⟩
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
h : ∀ (x y : α), Inseparable x y → ∃ s, x ∈ s ∧ y ∈ s ∧ T0Space ↑s
x y : α
hxy : Inseparable x y
⊢ x = y
[PROOFSTEP]
rcases h x y hxy with ⟨s, hxs, hys, hs⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝ : TopologicalSpace α
h : ∀ (x y : α), Inseparable x y → ∃ s, x ∈ s ∧ y ∈ s ∧ T0Space ↑s
x y : α
hxy : Inseparable x y
s : Set α
hxs : x ∈ s
hys : y ∈ s
hs : T0Space ↑s
⊢ x = y
[PROOFSTEP]
lift x to s using hxs
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
inst✝ : TopologicalSpace α
h : ∀ (x y : α), Inseparable x y → ∃ s, x ∈ s ∧ y ∈ s ∧ T0Space ↑s
y : α
s : Set α
hys : y ∈ s
hs : T0Space ↑s
x : { x // x ∈ s }
hxy : Inseparable (↑x) y
⊢ ↑x = y
[PROOFSTEP]
lift y to s using hys
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝ : TopologicalSpace α
h : ∀ (x y : α), Inseparable x y → ∃ s, x ∈ s ∧ y ∈ s ∧ T0Space ↑s
s : Set α
hs : T0Space ↑s
x y : { x // x ∈ s }
hxy : Inseparable ↑x ↑y
⊢ ↑x = ↑y
[PROOFSTEP]
rw [← subtype_inseparable_iff] at hxy
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝ : TopologicalSpace α
h : ∀ (x y : α), Inseparable x y → ∃ s, x ∈ s ∧ y ∈ s ∧ T0Space ↑s
s : Set α
hs : T0Space ↑s
x y : { x // x ∈ s }
hxy : Inseparable x y
⊢ ↑x = ↑y
[PROOFSTEP]
exact congr_arg Subtype.val hxy.eq
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
h : x ≠ y
s : Set α
⊢ 𝓝[s \ {y}] x = 𝓝[s] x
[PROOFSTEP]
rw [diff_eq, inter_comm, nhdsWithin_inter_of_mem]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
h : x ≠ y
s : Set α
⊢ {y}ᶜ ∈ 𝓝[s] x
[PROOFSTEP]
exact mem_nhdsWithin_of_mem_nhds (isOpen_ne.mem_nhds h)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
p : α → Prop
⊢ IsOpen {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y}
[PROOFSTEP]
refine' isOpen_iff_mem_nhds.mpr fun a ha => _
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
p : α → Prop
a : α
ha : a ∈ {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y}
⊢ {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y} ∈ 𝓝 a
[PROOFSTEP]
filter_upwards [eventually_nhds_nhdsWithin.mpr ha] with b hb
[GOAL]
case h
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
p : α → Prop
a : α
ha : a ∈ {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y}
b : α
hb : ∀ᶠ (x : α) in 𝓝[{a}ᶜ] b, p x
⊢ ∀ᶠ (y : α) in 𝓝[{b}ᶜ] b, p y
[PROOFSTEP]
rcases eq_or_ne a b with rfl | h
[GOAL]
case h.inl
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
p : α → Prop
a : α
ha : a ∈ {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y}
hb : ∀ᶠ (x : α) in 𝓝[{a}ᶜ] a, p x
⊢ ∀ᶠ (y : α) in 𝓝[{a}ᶜ] a, p y
[PROOFSTEP]
exact hb
[GOAL]
case h.inr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
p : α → Prop
a : α
ha : a ∈ {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y}
b : α
hb : ∀ᶠ (x : α) in 𝓝[{a}ᶜ] b, p x
h : a ≠ b
⊢ ∀ᶠ (y : α) in 𝓝[{b}ᶜ] b, p y
[PROOFSTEP]
rw [h.symm.nhdsWithin_compl_singleton] at hb
[GOAL]
case h.inr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
p : α → Prop
a : α
ha : a ∈ {x | ∀ᶠ (y : α) in 𝓝[{x}ᶜ] x, p y}
b : α
hb : ∀ᶠ (x : α) in 𝓝 b, p x
h : a ≠ b
⊢ ∀ᶠ (y : α) in 𝓝[{b}ᶜ] b, p y
[PROOFSTEP]
exact hb.filter_mono nhdsWithin_le_nhds
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
hs : Set.Finite s
⊢ IsClosed s
[PROOFSTEP]
rw [← biUnion_of_singleton s]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
hs : Set.Finite s
⊢ IsClosed (⋃ (x : α) (_ : x ∈ s), {x})
[PROOFSTEP]
exact isClosed_biUnion hs fun i _ => isClosed_singleton
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
b : Set (Set α)
hb : IsTopologicalBasis b
x y : α
h : x ≠ y
⊢ ∃ a, a ∈ b ∧ x ∈ a ∧ ¬y ∈ a
[PROOFSTEP]
rcases hb.isOpen_iff.1 isOpen_ne x h with ⟨a, ab, xa, ha⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
b : Set (Set α)
hb : IsTopologicalBasis b
x y : α
h : x ≠ y
a : Set α
ab : a ∈ b
xa : x ∈ a
ha : a ⊆ {y_1 | y_1 ≠ y}
⊢ ∃ a, a ∈ b ∧ x ∈ a ∧ ¬y ∈ a
[PROOFSTEP]
exact ⟨a, ab, xa, fun h => ha h rfl⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
⊢ IsBounded s ↔ IsCompact (closure s)
[PROOFSTEP]
change sᶜ ∈ Filter.coclosedCompact α ↔ _
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
⊢ sᶜ ∈ coclosedCompact α ↔ IsCompact (closure s)
[PROOFSTEP]
rw [Filter.mem_coclosedCompact]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
⊢ (∃ t, IsClosed t ∧ IsCompact t ∧ tᶜ ⊆ sᶜ) ↔ IsCompact (closure s)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
⊢ (∃ t, IsClosed t ∧ IsCompact t ∧ tᶜ ⊆ sᶜ) → IsCompact (closure s)
[PROOFSTEP]
rintro ⟨t, ht₁, ht₂, hst⟩
[GOAL]
case mp.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
ht₁ : IsClosed t
ht₂ : IsCompact t
hst : tᶜ ⊆ sᶜ
⊢ IsCompact (closure s)
[PROOFSTEP]
rw [compl_subset_compl] at hst
[GOAL]
case mp.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
ht₁ : IsClosed t
ht₂ : IsCompact t
hst : s ⊆ t
⊢ IsCompact (closure s)
[PROOFSTEP]
exact isCompact_of_isClosed_subset ht₂ isClosed_closure (closure_minimal hst ht₁)
[GOAL]
case mpr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
⊢ IsCompact (closure s) → ∃ t, IsClosed t ∧ IsCompact t ∧ tᶜ ⊆ sᶜ
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
h : IsCompact (closure s)
⊢ ∃ t, IsClosed t ∧ IsCompact t ∧ tᶜ ⊆ sᶜ
[PROOFSTEP]
exact ⟨closure s, isClosed_closure, h, compl_subset_compl.mpr subset_closure⟩
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 1 ↔ 2
[GOAL]
case tfae_1_iff_2
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
⊢ T1Space α ↔ ∀ (x : α), IsClosed {x}
[PROOFSTEP]
exact ⟨fun h => h.1, fun h => ⟨h⟩⟩
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 2 ↔ 3
[GOAL]
case tfae_2_iff_3
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
⊢ (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
[PROOFSTEP]
simp only [isOpen_compl_iff]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 5 ↔ 3
[GOAL]
case tfae_5_iff_3
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
⊢ (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
[PROOFSTEP]
refine' forall_swap.trans _
[GOAL]
case tfae_5_iff_3
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
⊢ (∀ (y x : α), x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
[PROOFSTEP]
simp only [isOpen_iff_mem_nhds, mem_compl_iff, mem_singleton_iff]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 5 ↔ 6
[GOAL]
case tfae_5_iff_6
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
⊢ (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
[PROOFSTEP]
simp only [← subset_compl_singleton_iff, exists_mem_subset_iff]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 5 ↔ 7
[GOAL]
case tfae_5_iff_7
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
⊢ (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
[PROOFSTEP]
simp only [(nhds_basis_opens _).mem_iff, subset_compl_singleton_iff, exists_prop, and_assoc, and_left_comm]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 5 ↔ 8
[GOAL]
case tfae_5_iff_8
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
⊢ (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
[PROOFSTEP]
simp only [← principal_singleton, disjoint_principal_right]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 8 ↔ 9
[GOAL]
case tfae_8_iff_9
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
⊢ (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
[PROOFSTEP]
exact forall_swap.trans (by simp only [disjoint_comm, ne_comm])
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
⊢ (∀ (y x : α), x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
[PROOFSTEP]
simp only [disjoint_comm, ne_comm]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 1 → 4
[GOAL]
case tfae_1_to_4
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
⊢ T1Space α → Continuous ↑CofiniteTopology.of
[PROOFSTEP]
simp only [continuous_def, CofiniteTopology.isOpen_iff']
[GOAL]
case tfae_1_to_4
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
⊢ T1Space α → ∀ (s : Set (CofiniteTopology α)), s = ∅ ∨ Set.Finite sᶜ → IsOpen (↑CofiniteTopology.of ⁻¹' s)
[PROOFSTEP]
rintro H s (rfl | hs)
[GOAL]
case tfae_1_to_4.inl
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
H : T1Space α
⊢ IsOpen (↑CofiniteTopology.of ⁻¹' ∅)
case tfae_1_to_4.inr
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
H : T1Space α
s : Set (CofiniteTopology α)
hs : Set.Finite sᶜ
⊢ IsOpen (↑CofiniteTopology.of ⁻¹' s)
[PROOFSTEP]
exacts [isOpen_empty, compl_compl s ▸ (@Set.Finite.isClosed _ _ H _ hs).isOpen_compl]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
tfae_1_to_4 : T1Space α → Continuous ↑CofiniteTopology.of
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 4 → 2
[GOAL]
case tfae_4_to_2
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
tfae_1_to_4 : T1Space α → Continuous ↑CofiniteTopology.of
⊢ Continuous ↑CofiniteTopology.of → ∀ (x : α), IsClosed {x}
[PROOFSTEP]
exact fun h x => (CofiniteTopology.isClosed_iff.2 <| Or.inr (finite_singleton _)).preimage h
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
tfae_1_to_4 : T1Space α → Continuous ↑CofiniteTopology.of
tfae_4_to_2 : Continuous ↑CofiniteTopology.of → ∀ (x : α), IsClosed {x}
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_have 2 ↔ 10
[GOAL]
case tfae_2_iff_10
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
tfae_1_to_4 : T1Space α → Continuous ↑CofiniteTopology.of
tfae_4_to_2 : Continuous ↑CofiniteTopology.of → ∀ (x : α), IsClosed {x}
⊢ (∀ (x : α), IsClosed {x}) ↔ ∀ ⦃x y : α⦄, x ⤳ y → x = y
[PROOFSTEP]
simp only [← closure_subset_iff_isClosed, specializes_iff_mem_closure, subset_def, mem_singleton_iff, eq_comm]
[GOAL]
α✝ : Type u
β : Type v
inst✝¹ : TopologicalSpace α✝
α : Type u
inst✝ : TopologicalSpace α
tfae_1_iff_2 : T1Space α ↔ ∀ (x : α), IsClosed {x}
tfae_2_iff_3 : (∀ (x : α), IsClosed {x}) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_3 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ (x : α), IsOpen {x}ᶜ
tfae_5_iff_6 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s
tfae_5_iff_7 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U
tfae_5_iff_8 : (∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)
tfae_8_iff_9 : (∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y)) ↔ ∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y)
tfae_1_to_4 : T1Space α → Continuous ↑CofiniteTopology.of
tfae_4_to_2 : Continuous ↑CofiniteTopology.of → ∀ (x : α), IsClosed {x}
tfae_2_iff_10 : (∀ (x : α), IsClosed {x}) ↔ ∀ ⦃x y : α⦄, x ⤳ y → x = y
⊢ List.TFAE
[T1Space α, ∀ (x : α), IsClosed {x}, ∀ (x : α), IsOpen {x}ᶜ, Continuous ↑CofiniteTopology.of,
∀ ⦃x y : α⦄, x ≠ y → {y}ᶜ ∈ 𝓝 x, ∀ ⦃x y : α⦄, x ≠ y → ∃ s, s ∈ 𝓝 x ∧ ¬y ∈ s,
∀ ⦃x y : α⦄, x ≠ y → ∃ U, IsOpen U ∧ x ∈ U ∧ ¬y ∈ U, ∀ ⦃x y : α⦄, x ≠ y → Disjoint (𝓝 x) (pure y),
∀ ⦃x y : α⦄, x ≠ y → Disjoint (pure x) (𝓝 y), ∀ ⦃x y : α⦄, x ⤳ y → x = y]
[PROOFSTEP]
tfae_finish
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
x y : α
z : β
hne : y ≠ x
⊢ ContinuousAt (update f x z) y ↔ ContinuousAt f y
[PROOFSTEP]
simp only [← continuousWithinAt_univ, continuousWithinAt_update_of_ne hne]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
⊢ ContinuousOn (update f x y) s ↔ ContinuousOn f (s \ {x}) ∧ (x ∈ s → Tendsto f (𝓝[s \ {x}] x) (𝓝 y))
[PROOFSTEP]
rw [ContinuousOn, ← and_forall_ne x, and_comm]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
⊢ (∀ (b : α), b ≠ x → b ∈ s → ContinuousWithinAt (update f x y) s b) ∧ (x ∈ s → ContinuousWithinAt (update f x y) s x) ↔
ContinuousOn f (s \ {x}) ∧ (x ∈ s → Tendsto f (𝓝[s \ {x}] x) (𝓝 y))
[PROOFSTEP]
refine' and_congr ⟨fun H z hz => _, fun H z hzx hzs => _⟩ (forall_congr' fun _ => _)
[GOAL]
case refine'_1
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
H : ∀ (b : α), b ≠ x → b ∈ s → ContinuousWithinAt (update f x y) s b
z : α
hz : z ∈ s \ {x}
⊢ ContinuousWithinAt f (s \ {x}) z
[PROOFSTEP]
specialize H z hz.2 hz.1
[GOAL]
case refine'_1
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
z : α
hz : z ∈ s \ {x}
H : ContinuousWithinAt (update f x y) s z
⊢ ContinuousWithinAt f (s \ {x}) z
[PROOFSTEP]
rw [continuousWithinAt_update_of_ne hz.2] at H
[GOAL]
case refine'_1
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
z : α
hz : z ∈ s \ {x}
H : ContinuousWithinAt f s z
⊢ ContinuousWithinAt f (s \ {x}) z
[PROOFSTEP]
exact H.mono (diff_subset _ _)
[GOAL]
case refine'_2
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
H : ContinuousOn f (s \ {x})
z : α
hzx : z ≠ x
hzs : z ∈ s
⊢ ContinuousWithinAt (update f x y) s z
[PROOFSTEP]
rw [continuousWithinAt_update_of_ne hzx]
[GOAL]
case refine'_2
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
H : ContinuousOn f (s \ {x})
z : α
hzx : z ≠ x
hzs : z ∈ s
⊢ ContinuousWithinAt f s z
[PROOFSTEP]
refine' (H z ⟨hzs, hzx⟩).mono_of_mem (inter_mem_nhdsWithin _ _)
[GOAL]
case refine'_2
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
H : ContinuousOn f (s \ {x})
z : α
hzx : z ≠ x
hzs : z ∈ s
⊢ (fun a => a ∈ {x} → False) ∈ 𝓝 z
[PROOFSTEP]
exact isOpen_ne.mem_nhds hzx
[GOAL]
case refine'_3
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T1Space α
inst✝¹ : DecidableEq α
inst✝ : TopologicalSpace β
f : α → β
s : Set α
x : α
y : β
x✝ : x ∈ s
⊢ ContinuousWithinAt (update f x y) s x ↔ Tendsto f (𝓝[s \ {x}] x) (𝓝 y)
[PROOFSTEP]
exact continuousWithinAt_update_same
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
hs : Set.Subsingleton s
⊢ Set.Subsingleton (_root_.closure s)
[PROOFSTEP]
rcases hs.eq_empty_or_singleton with (rfl | ⟨x, rfl⟩)
[GOAL]
case inl
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
hs : Set.Subsingleton ∅
⊢ Set.Subsingleton (_root_.closure ∅)
[PROOFSTEP]
simp
[GOAL]
case inr.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
hs : Set.Subsingleton {x}
⊢ Set.Subsingleton (_root_.closure {x})
[PROOFSTEP]
simp
[GOAL]
α✝ : Type u
β✝ : Type v
inst✝³ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T1Space β
y : β
s : Set α
x✝ : IsClosed s
h2s : Set.Nonempty s
⊢ IsClosed (const α y '' s)
[PROOFSTEP]
simp_rw [const, h2s.image_const, isClosed_singleton]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s : Set α
hxy : x ≠ y
⊢ 𝓝[insert y s] x = 𝓝[s] x
[PROOFSTEP]
refine' le_antisymm (Filter.le_def.2 fun t ht => _) (nhdsWithin_mono x <| subset_insert y s)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s : Set α
hxy : x ≠ y
t : Set α
ht : t ∈ 𝓝[s] x
⊢ t ∈ 𝓝[insert y s] x
[PROOFSTEP]
obtain ⟨o, ho, hxo, host⟩ := mem_nhdsWithin.mp ht
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s : Set α
hxy : x ≠ y
t : Set α
ht : t ∈ 𝓝[s] x
o : Set α
ho : IsOpen o
hxo : x ∈ o
host : o ∩ s ⊆ t
⊢ t ∈ 𝓝[insert y s] x
[PROOFSTEP]
refine' mem_nhdsWithin.mpr ⟨o \ { y }, ho.sdiff isClosed_singleton, ⟨hxo, hxy⟩, _⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s : Set α
hxy : x ≠ y
t : Set α
ht : t ∈ 𝓝[s] x
o : Set α
ho : IsOpen o
hxo : x ∈ o
host : o ∩ s ⊆ t
⊢ o \ {y} ∩ insert y s ⊆ t
[PROOFSTEP]
rw [inter_insert_of_not_mem <| not_mem_diff_of_mem (mem_singleton y)]
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s : Set α
hxy : x ≠ y
t : Set α
ht : t ∈ 𝓝[s] x
o : Set α
ho : IsOpen o
hxo : x ∈ o
host : o ∩ s ⊆ t
⊢ o \ {y} ∩ s ⊆ t
[PROOFSTEP]
exact (inter_subset_inter (diff_subset _ _) Subset.rfl).trans host
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s t : Set α
hu : t ⊆ insert y s
⊢ insert x s ∈ 𝓝[t] x
[PROOFSTEP]
rcases eq_or_ne x y with (rfl | h)
[GOAL]
case inl
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s t : Set α
hu : t ⊆ insert x s
⊢ insert x s ∈ 𝓝[t] x
[PROOFSTEP]
exact mem_of_superset self_mem_nhdsWithin hu
[GOAL]
case inr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s t : Set α
hu : t ⊆ insert y s
h : x ≠ y
⊢ insert x s ∈ 𝓝[t] x
[PROOFSTEP]
refine' nhdsWithin_mono x hu _
[GOAL]
case inr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s t : Set α
hu : t ⊆ insert y s
h : x ≠ y
⊢ insert x s ∈ 𝓝[insert y s] x
[PROOFSTEP]
rw [nhdsWithin_insert_of_ne h]
[GOAL]
case inr
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x y : α
s t : Set α
hu : t ⊆ insert y s
h : x ≠ y
⊢ insert x s ∈ 𝓝[s] x
[PROOFSTEP]
exact mem_of_superset self_mem_nhdsWithin (subset_insert x s)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
⊢ ⋂₀ (𝓝 x).sets = {x}
[PROOFSTEP]
simp [sInter_nhds_sets_eq_specializes]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
ι : Sort u_1
p : ι → Prop
s : ι → Set α
x : α
h : HasBasis (𝓝 x) p s
⊢ ⋂ (i : ι) (_ : p i), s i = {x}
[PROOFSTEP]
rw [← h.sInter_sets, sInter_sets_nhds]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
⊢ {x}ᶜ ∈ 𝓝ˢ s ↔ ¬x ∈ s
[PROOFSTEP]
rw [isOpen_compl_singleton.mem_nhdsSet, subset_compl_singleton_iff]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
⊢ 𝓝ˢ s ≤ 𝓝ˢ t ↔ s ⊆ t
[PROOFSTEP]
refine' ⟨_, fun h => monotone_nhdsSet h⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
⊢ 𝓝ˢ s ≤ 𝓝ˢ t → s ⊆ t
[PROOFSTEP]
simp_rw [Filter.le_def]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
⊢ (∀ (x : Set α), x ∈ 𝓝ˢ t → x ∈ 𝓝ˢ s) → s ⊆ t
[PROOFSTEP]
intro h x hx
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
h : ∀ (x : Set α), x ∈ 𝓝ˢ t → x ∈ 𝓝ˢ s
x : α
hx : x ∈ s
⊢ x ∈ t
[PROOFSTEP]
specialize h { x }ᶜ
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
x : α
hx : x ∈ s
h : {x}ᶜ ∈ 𝓝ˢ t → {x}ᶜ ∈ 𝓝ˢ s
⊢ x ∈ t
[PROOFSTEP]
simp_rw [compl_singleton_mem_nhdsSet_iff] at h
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
x : α
hx : x ∈ s
h : ¬x ∈ t → ¬x ∈ s
⊢ x ∈ t
[PROOFSTEP]
by_contra hxt
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
x : α
hx : x ∈ s
h : ¬x ∈ t → ¬x ∈ s
hxt : ¬x ∈ t
⊢ False
[PROOFSTEP]
exact h hxt hx
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
⊢ 𝓝ˢ s = 𝓝ˢ t ↔ s = t
[PROOFSTEP]
simp_rw [le_antisymm_iff]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s t : Set α
⊢ 𝓝ˢ s ≤ 𝓝ˢ t ∧ 𝓝ˢ t ≤ 𝓝ˢ s ↔ s ≤ t ∧ t ≤ s
[PROOFSTEP]
exact and_congr nhdsSet_le_iff nhdsSet_le_iff
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
x : α
⊢ 𝓝 x ≤ 𝓝ˢ s ↔ x ∈ s
[PROOFSTEP]
rw [← nhdsSet_singleton, nhdsSet_le_iff, singleton_subset_iff]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
t : Finset α
⊢ Dense (s \ ↑t)
[PROOFSTEP]
induction t using Finset.induction_on with
| empty => simpa using hs
| insert _ ih =>
rw [Finset.coe_insert, ← union_singleton, ← diff_diff]
exact ih.diff_singleton _
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
t : Finset α
⊢ Dense (s \ ↑t)
[PROOFSTEP]
induction t using Finset.induction_on with
| empty => simpa using hs
| insert _ ih =>
rw [Finset.coe_insert, ← union_singleton, ← diff_diff]
exact ih.diff_singleton _
[GOAL]
case empty
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
⊢ Dense (s \ ↑∅)
[PROOFSTEP]
| empty => simpa using hs
[GOAL]
case empty
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
⊢ Dense (s \ ↑∅)
[PROOFSTEP]
simpa using hs
[GOAL]
case insert
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
a✝¹ : α
s✝ : Finset α
a✝ : ¬a✝¹ ∈ s✝
ih : Dense (s \ ↑s✝)
⊢ Dense (s \ ↑(insert a✝¹ s✝))
[PROOFSTEP]
| insert _ ih =>
rw [Finset.coe_insert, ← union_singleton, ← diff_diff]
exact ih.diff_singleton _
[GOAL]
case insert
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
a✝¹ : α
s✝ : Finset α
a✝ : ¬a✝¹ ∈ s✝
ih : Dense (s \ ↑s✝)
⊢ Dense (s \ ↑(insert a✝¹ s✝))
[PROOFSTEP]
rw [Finset.coe_insert, ← union_singleton, ← diff_diff]
[GOAL]
case insert
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
a✝¹ : α
s✝ : Finset α
a✝ : ¬a✝¹ ∈ s✝
ih : Dense (s \ ↑s✝)
⊢ Dense ((s \ ↑s✝) \ {a✝¹})
[PROOFSTEP]
exact ih.diff_singleton _
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
t : Set α
ht : Set.Finite t
⊢ Dense (s \ t)
[PROOFSTEP]
convert hs.diff_finset ht.toFinset
[GOAL]
case h.e'_3.h.e'_4
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
inst✝ : ∀ (x : α), NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : Dense s
t : Set α
ht : Set.Finite t
⊢ t = ↑(Finite.toFinset ht)
[PROOFSTEP]
exact (Finite.coe_toFinset _).symm
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T1Space β
f : α → β
a : α
b : β
h : Tendsto f (𝓝 a) (𝓝 b)
⊢ ContinuousAt f a
[PROOFSTEP]
rwa [ContinuousAt, eq_of_tendsto_nhds h]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T1Space α
l : Filter β
inst✝ : NeBot l
c d : α
⊢ Tendsto (fun x => c) l (𝓝 d) ↔ c = d
[PROOFSTEP]
simp_rw [Tendsto, Filter.map_const, pure_le_nhds_iff]
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
⊢ IsOpen {x}
[PROOFSTEP]
have A : { x } ⊆ s := by simp only [singleton_subset_iff, mem_of_mem_nhds hs]
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
⊢ {x} ⊆ s
[PROOFSTEP]
simp only [singleton_subset_iff, mem_of_mem_nhds hs]
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
A : {x} ⊆ s
⊢ IsOpen {x}
[PROOFSTEP]
have B : IsClosed (s \ { x }) := (hsf.subset (diff_subset _ _)).isClosed
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
A : {x} ⊆ s
B : IsClosed (s \ {x})
⊢ IsOpen {x}
[PROOFSTEP]
have C : (s \ { x })ᶜ ∈ 𝓝 x := B.isOpen_compl.mem_nhds fun h => h.2 rfl
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
A : {x} ⊆ s
B : IsClosed (s \ {x})
C : (s \ {x})ᶜ ∈ 𝓝 x
⊢ IsOpen {x}
[PROOFSTEP]
have D : { x } ∈ 𝓝 x := by simpa only [← diff_eq, diff_diff_cancel_left A] using inter_mem hs C
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
A : {x} ⊆ s
B : IsClosed (s \ {x})
C : (s \ {x})ᶜ ∈ 𝓝 x
⊢ {x} ∈ 𝓝 x
[PROOFSTEP]
simpa only [← diff_eq, diff_diff_cancel_left A] using inter_mem hs C
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
A : {x} ⊆ s
B : IsClosed (s \ {x})
C : (s \ {x})ᶜ ∈ 𝓝 x
D : {x} ∈ 𝓝 x
⊢ IsOpen {x}
[PROOFSTEP]
rwa [← mem_interior_iff_mem_nhds, ← singleton_subset_iff, subset_interior_iff_isOpen] at D
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
hx : NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : s ∈ 𝓝 x
⊢ Set.Infinite s
[PROOFSTEP]
refine' fun hsf => hx.1 _
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
hx : NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
⊢ 𝓝[{x}ᶜ] x = ⊥
[PROOFSTEP]
rw [← isOpen_singleton_iff_punctured_nhds]
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
α : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
x : α
hx : NeBot (𝓝[{x}ᶜ] x)
s : Set α
hs : s ∈ 𝓝 x
hsf : Set.Finite s
⊢ IsOpen {x}
[PROOFSTEP]
exact isOpen_singleton_of_finite_mem_nhds x hs hsf
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
X : Type u_1
inst✝² : TopologicalSpace X
inst✝¹ : T1Space X
inst✝ : Finite X
⊢ DiscreteTopology X
[PROOFSTEP]
apply singletons_open_iff_discrete.mp
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
X : Type u_1
inst✝² : TopologicalSpace X
inst✝¹ : T1Space X
inst✝ : Finite X
⊢ ∀ (a : X), IsOpen {a}
[PROOFSTEP]
intro x
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
X : Type u_1
inst✝² : TopologicalSpace X
inst✝¹ : T1Space X
inst✝ : Finite X
x : X
⊢ IsOpen {x}
[PROOFSTEP]
rw [← isClosed_compl_iff]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
X : Type u_1
inst✝² : TopologicalSpace X
inst✝¹ : T1Space X
inst✝ : Finite X
x : X
⊢ IsClosed {x}ᶜ
[PROOFSTEP]
exact (Set.toFinite _).isClosed
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : PreconnectedSpace α
inst✝ : DiscreteTopology α
⊢ Subsingleton α
[PROOFSTEP]
rw [← not_nontrivial_iff_subsingleton]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : PreconnectedSpace α
inst✝ : DiscreteTopology α
⊢ ¬Nontrivial α
[PROOFSTEP]
rintro ⟨x, y, hxy⟩
[GOAL]
case mk.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : PreconnectedSpace α
inst✝ : DiscreteTopology α
x y : α
hxy : x ≠ y
⊢ False
[PROOFSTEP]
rw [Ne.def, ← mem_singleton_iff, (isClopen_discrete _).eq_univ <| singleton_nonempty y] at hxy
[GOAL]
case mk.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : PreconnectedSpace α
inst✝ : DiscreteTopology α
x y : α
hxy : ¬x ∈ univ
⊢ False
[PROOFSTEP]
exact hxy (mem_univ x)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
h : IsPreconnected s
hs : Set.Nontrivial s
⊢ Set.Infinite s
[PROOFSTEP]
refine' mt (fun hf => (subsingleton_coe s).mp _) (not_subsingleton_iff.mpr hs)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
h : IsPreconnected s
hs : Set.Nontrivial s
hf : Set.Finite s
⊢ Subsingleton ↑s
[PROOFSTEP]
haveI := @discrete_of_t1_of_finite s _ _ hf.to_subtype
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
s : Set α
h : IsPreconnected s
hs : Set.Nontrivial s
hf : Set.Finite s
this : DiscreteTopology ↑s
⊢ Subsingleton ↑s
[PROOFSTEP]
exact @PreconnectedSpace.trivial_of_discrete _ _ (Subtype.preconnectedSpace h) _
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : ConnectedSpace α
inst✝¹ : Nontrivial α
inst✝ : T1Space α
x : α
⊢ NeBot (𝓝[{x}ᶜ] x)
[PROOFSTEP]
by_contra contra
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : ConnectedSpace α
inst✝¹ : Nontrivial α
inst✝ : T1Space α
x : α
contra : ¬NeBot (𝓝[{x}ᶜ] x)
⊢ False
[PROOFSTEP]
rw [not_neBot, ← isOpen_singleton_iff_punctured_nhds] at contra
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : ConnectedSpace α
inst✝¹ : Nontrivial α
inst✝ : T1Space α
x : α
contra : IsOpen {x}
⊢ False
[PROOFSTEP]
replace contra :=
nonempty_inter isOpen_compl_singleton contra (compl_union_self _) (Set.nonempty_compl_of_nontrivial _)
(singleton_nonempty _)
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : ConnectedSpace α
inst✝¹ : Nontrivial α
inst✝ : T1Space α
x : α
contra : Set.Nonempty ({x}ᶜ ∩ {x})
⊢ False
[PROOFSTEP]
simp [compl_inter_self { x }] at contra
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hx : x ∈ s
⊢ {x} ∈ 𝓝[s] x
[PROOFSTEP]
have : ({⟨x, hx⟩} : Set s) ∈ 𝓝 (⟨x, hx⟩ : s) := by simp [nhds_discrete]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hx : x ∈ s
⊢ {{ val := x, property := hx }} ∈ 𝓝 { val := x, property := hx }
[PROOFSTEP]
simp [nhds_discrete]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hx : x ∈ s
this : {{ val := x, property := hx }} ∈ 𝓝 { val := x, property := hx }
⊢ {x} ∈ 𝓝[s] x
[PROOFSTEP]
simpa only [nhdsWithin_eq_map_subtype_coe hx, image_singleton] using @image_mem_map _ _ _ ((↑) : s → α) _ this
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
ι : Type u_1
p : ι → Prop
t : ι → Set α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hb : HasBasis (𝓝 x) p t
hx : x ∈ s
⊢ ∃ i, p i ∧ t i ∩ s = {x}
[PROOFSTEP]
rcases(nhdsWithin_hasBasis hb s).mem_iff.1 (singleton_mem_nhdsWithin_of_mem_discrete hx) with ⟨i, hi, hix⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
ι : Type u_1
p : ι → Prop
t : ι → Set α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hb : HasBasis (𝓝 x) p t
hx : x ∈ s
i : ι
hi : p i
hix : t i ∩ s ⊆ {x}
⊢ ∃ i, p i ∧ t i ∩ s = {x}
[PROOFSTEP]
exact ⟨i, hi, hix.antisymm <| singleton_subset_iff.2 ⟨mem_of_mem_nhds <| hb.mem_of_mem hi, hx⟩⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hx : x ∈ s
⊢ ∃ U, U ∈ 𝓝 x ∧ U ∩ s = {x}
[PROOFSTEP]
simpa using (𝓝 x).basis_sets.exists_inter_eq_singleton_of_mem_discrete hx
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
s : Set α
inst✝ : DiscreteTopology ↑s
x : α
hx : x ∈ s
V : Set α
h : V ∈ 𝓝 x
h' : V ∩ s = {x}
⊢ {x}ᶜ ∩ V ∩ s = ∅
[PROOFSTEP]
rw [inter_assoc, h', compl_inter_self]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ T2Space α ↔ ∀ (x y : α), x ≠ y → Disjoint (𝓝 x) (𝓝 y)
[PROOFSTEP]
refine (t2Space_iff α).trans (forall₃_congr fun x y _ => ?_)
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
x y : α
x✝ : x ≠ y
⊢ (∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ Disjoint u v) ↔ Disjoint (𝓝 x) (𝓝 y)
[PROOFSTEP]
simp only [(nhds_basis_opens x).disjoint_iff (nhds_basis_opens y), exists_prop, ← exists_and_left, and_assoc, and_comm,
and_left_comm]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T2Space α
x y : α
hd : Disjoint (𝓝 x) (𝓝 y)
he : x = y
⊢ False
[PROOFSTEP]
simp [he, nhds_neBot.ne] at hd
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ IsOpen {p | Disjoint (𝓝 p.fst) (𝓝 p.snd)}
[PROOFSTEP]
simp only [isOpen_iff_mem_nhds, Prod.forall, mem_setOf_eq]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ ∀ (a b : α), Disjoint (𝓝 a) (𝓝 b) → {p | Disjoint (𝓝 p.fst) (𝓝 p.snd)} ∈ 𝓝 (a, b)
[PROOFSTEP]
intro x y h
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
x y : α
h : Disjoint (𝓝 x) (𝓝 y)
⊢ {p | Disjoint (𝓝 p.fst) (𝓝 p.snd)} ∈ 𝓝 (x, y)
[PROOFSTEP]
obtain ⟨U, hU, V, hV, hd⟩ := ((nhds_basis_opens x).disjoint_iff (nhds_basis_opens y)).mp h
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
inst✝ : TopologicalSpace α
x y : α
h : Disjoint (𝓝 x) (𝓝 y)
U : Set α
hU : x ∈ U ∧ IsOpen U
V : Set α
hV : y ∈ V ∧ IsOpen V
hd : Disjoint U V
⊢ {p | Disjoint (𝓝 p.fst) (𝓝 p.snd)} ∈ 𝓝 (x, y)
[PROOFSTEP]
exact
mem_nhds_prod_iff.mpr
⟨U, hU.2.mem_nhds hU.1, V, hV.2.mem_nhds hV.1, fun ⟨x', y'⟩ ⟨hx', hy'⟩ =>
disjoint_of_disjoint_of_mem hd (hU.2.mem_nhds hx') (hV.2.mem_nhds hy')⟩
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ T2Space α ↔ ∀ {x y : α}, NeBot (𝓝 x ⊓ 𝓝 y) → x = y
[PROOFSTEP]
simp only [t2Space_iff_disjoint_nhds, disjoint_iff, neBot_iff, Ne.def, not_imp_comm]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ T2Space α ↔ ∀ {x y : α}, x ≠ y → ∃ U, U ∈ 𝓝 x ∧ ∃ V, V ∈ 𝓝 y ∧ Disjoint U V
[PROOFSTEP]
simp only [t2Space_iff_disjoint_nhds, Filter.disjoint_iff]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
x y : α
h : x ≠ y
⊢ ∃ u v, u ∈ 𝓝 x ∧ v ∈ 𝓝 y ∧ IsCompact u ∧ IsCompact v ∧ Disjoint u v
[PROOFSTEP]
simpa only [exists_prop, ← exists_and_left, and_comm, and_assoc, and_left_comm] using
((compact_basis_nhds x).disjoint_iff (compact_basis_nhds y)).1 (disjoint_nhds_nhds.2 h)
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ (∀ {x y : α}, NeBot (𝓝 x ⊓ 𝓝 y) → x = y) ↔ ∀ {x y : α} (f : Ultrafilter α), ↑f ≤ 𝓝 x → ↑f ≤ 𝓝 y → x = y
[PROOFSTEP]
simp only [← exists_ultrafilter_iff, and_imp, le_inf_iff, exists_imp]
[GOAL]
α : Type u
β : Type v
inst✝ : TopologicalSpace α
⊢ T2Space α ↔ IsClosed (diagonal α)
[PROOFSTEP]
simp only [t2Space_iff_disjoint_nhds, ← isOpen_compl_iff, isOpen_iff_mem_nhds, Prod.forall, nhds_prod_eq,
compl_diagonal_mem_prod, mem_compl_iff, mem_diagonal_iff]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T25Space α
x y : α
h : Disjoint (Filter.lift' (𝓝 x) closure) (Filter.lift' (𝓝 y) closure)
hxy : x = y
⊢ False
[PROOFSTEP]
simp [hxy, nhds_neBot.ne] at h
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T25Space α
x y : α
h : x ≠ y
⊢ ∃ u, x ∈ u ∧ IsOpen u ∧ ∃ v, y ∈ v ∧ IsOpen v ∧ Disjoint (closure u) (closure v)
[PROOFSTEP]
simpa only [exists_prop, and_assoc] using
((nhds_basis_opens x).lift'_closure.disjoint_iff (nhds_basis_opens y).lift'_closure).1
(disjoint_lift'_closure_nhds.2 h)
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
f : Filter α
inst✝ : CompactSpace α
U : Set α
⊢ IsOpen U ↔ ∀ (F : Ultrafilter α), Ultrafilter.lim F ∈ U → U ∈ ↑F
[PROOFSTEP]
rw [isOpen_iff_ultrafilter]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
f : Filter α
inst✝ : CompactSpace α
U : Set α
⊢ (∀ (x : α), x ∈ U → ∀ (l : Ultrafilter α), ↑l ≤ 𝓝 x → U ∈ l) ↔ ∀ (F : Ultrafilter α), Ultrafilter.lim F ∈ U → U ∈ ↑F
[PROOFSTEP]
refine' ⟨fun h F hF => h F.lim hF F F.le_nhds_lim, _⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
f : Filter α
inst✝ : CompactSpace α
U : Set α
⊢ (∀ (F : Ultrafilter α), Ultrafilter.lim F ∈ U → U ∈ ↑F) → ∀ (x : α), x ∈ U → ∀ (l : Ultrafilter α), ↑l ≤ 𝓝 x → U ∈ l
[PROOFSTEP]
intro cond x hx f h
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
f✝ : Filter α
inst✝ : CompactSpace α
U : Set α
cond : ∀ (F : Ultrafilter α), Ultrafilter.lim F ∈ U → U ∈ ↑F
x : α
hx : x ∈ U
f : Ultrafilter α
h : ↑f ≤ 𝓝 x
⊢ U ∈ f
[PROOFSTEP]
rw [← Ultrafilter.lim_eq_iff_le_nhds.2 h] at hx
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
f✝ : Filter α
inst✝ : CompactSpace α
U : Set α
cond : ∀ (F : Ultrafilter α), Ultrafilter.lim F ∈ U → U ∈ ↑F
x : α
f : Ultrafilter α
hx : Ultrafilter.lim f ∈ U
h : ↑f ≤ 𝓝 x
⊢ U ∈ f
[PROOFSTEP]
exact cond _ hx
[GOAL]
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
⊢ T2Space (α ⊕ β)
[PROOFSTEP]
constructor
[GOAL]
case t2
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
⊢ ∀ (x y : α ⊕ β), x ≠ y → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ Disjoint u v
[PROOFSTEP]
rintro (x | x) (y | y) h
[GOAL]
case t2.inl.inl
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
x y : α
h : Sum.inl x ≠ Sum.inl y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ Sum.inl x ∈ u ∧ Sum.inl y ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact separated_by_openEmbedding openEmbedding_inl <| ne_of_apply_ne _ h
[GOAL]
case t2.inl.inr
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
x : α
y : β
h : Sum.inl x ≠ Sum.inr y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ Sum.inl x ∈ u ∧ Sum.inr y ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact separated_by_continuous continuous_isLeft <| by simp
[GOAL]
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
x : α
y : β
h : Sum.inl x ≠ Sum.inr y
⊢ Sum.isLeft (Sum.inl x) ≠ Sum.isLeft (Sum.inr y)
[PROOFSTEP]
simp
[GOAL]
case t2.inr.inl
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
x : β
y : α
h : Sum.inr x ≠ Sum.inl y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ Sum.inr x ∈ u ∧ Sum.inl y ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact separated_by_continuous continuous_isLeft <| by simp
[GOAL]
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
x : β
y : α
h : Sum.inr x ≠ Sum.inl y
⊢ Sum.isLeft (Sum.inr x) ≠ Sum.isLeft (Sum.inl y)
[PROOFSTEP]
simp
[GOAL]
case t2.inr.inr
α✝ : Type u
β✝ : Type v
inst✝⁴ : TopologicalSpace α✝
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : TopologicalSpace β
inst✝ : T2Space β
x y : β
h : Sum.inr x ≠ Sum.inr y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ Sum.inr x ∈ u ∧ Sum.inr y ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact separated_by_openEmbedding openEmbedding_inr <| ne_of_apply_ne _ h
[GOAL]
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
⊢ T2Space ((i : ι) × α i)
[PROOFSTEP]
constructor
[GOAL]
case t2
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
⊢ ∀ (x y : (i : ι) × α i), x ≠ y → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ Disjoint u v
[PROOFSTEP]
rintro ⟨i, x⟩ ⟨j, y⟩ neq
[GOAL]
case t2.mk.mk
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
i : ι
x : α i
j : ι
y : α j
neq : { fst := i, snd := x } ≠ { fst := j, snd := y }
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ { fst := i, snd := x } ∈ u ∧ { fst := j, snd := y } ∈ v ∧ Disjoint u v
[PROOFSTEP]
rcases eq_or_ne i j with (rfl | h)
[GOAL]
case t2.mk.mk.inl
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
i : ι
x y : α i
neq : { fst := i, snd := x } ≠ { fst := i, snd := y }
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ { fst := i, snd := x } ∈ u ∧ { fst := i, snd := y } ∈ v ∧ Disjoint u v
[PROOFSTEP]
replace neq : x ≠ y := ne_of_apply_ne _ neq
[GOAL]
case t2.mk.mk.inl
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
i : ι
x y : α i
neq : x ≠ y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ { fst := i, snd := x } ∈ u ∧ { fst := i, snd := y } ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact separated_by_openEmbedding openEmbedding_sigmaMk neq
[GOAL]
case t2.mk.mk.inr
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
i : ι
x : α i
j : ι
y : α j
neq : { fst := i, snd := x } ≠ { fst := j, snd := y }
h : i ≠ j
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ { fst := i, snd := x } ∈ u ∧ { fst := j, snd := y } ∈ v ∧ Disjoint u v
[PROOFSTEP]
let _ := (⊥ : TopologicalSpace ι)
[GOAL]
case t2.mk.mk.inr
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
i : ι
x : α i
j : ι
y : α j
neq : { fst := i, snd := x } ≠ { fst := j, snd := y }
h : i ≠ j
x✝ : TopologicalSpace ι := ⊥
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ { fst := i, snd := x } ∈ u ∧ { fst := j, snd := y } ∈ v ∧ Disjoint u v
[PROOFSTEP]
have : DiscreteTopology ι := ⟨rfl⟩
[GOAL]
case t2.mk.mk.inr
α✝ : Type u
β : Type v
inst✝² : TopologicalSpace α✝
ι : Type ?u.128612
α : ι → Type u_1
inst✝¹ : (i : ι) → TopologicalSpace (α i)
inst✝ : ∀ (a : ι), T2Space (α a)
i : ι
x : α i
j : ι
y : α j
neq : { fst := i, snd := x } ≠ { fst := j, snd := y }
h : i ≠ j
x✝ : TopologicalSpace ι := ⊥
this : DiscreteTopology ι
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ { fst := i, snd := x } ∈ u ∧ { fst := j, snd := y } ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact separated_by_continuous (continuous_def.2 fun u _ => isOpen_sigma_fst_preimage u) h
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s : Set β
t : Set γ
f g : β → γ → α
h : ∀ (x : β), x ∈ s → ∀ (y : γ), y ∈ t → f x y = g x y
hf₁ : ∀ (x : β), Continuous (f x)
hf₂ : ∀ (y : γ), Continuous fun x => f x y
hg₁ : ∀ (x : β), Continuous (g x)
hg₂ : ∀ (y : γ), Continuous fun x => g x y
this : closure s ⊆ ⋂ (y : γ) (_ : y ∈ closure t), {x | f x y = g x y}
⊢ ∀ (x : β), x ∈ closure s → ∀ (y : γ), y ∈ closure t → f x y = g x y
[PROOFSTEP]
simpa only [subset_def, mem_iInter]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s t : Set β
f g : β → α
h : EqOn f g s
hf : ContinuousOn f t
hg : ContinuousOn g t
hst : s ⊆ t
hts : t ⊆ closure s
⊢ EqOn f g t
[PROOFSTEP]
intro x hx
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s t : Set β
f g : β → α
h : EqOn f g s
hf : ContinuousOn f t
hg : ContinuousOn g t
hst : s ⊆ t
hts : t ⊆ closure s
x : β
hx : x ∈ t
⊢ f x = g x
[PROOFSTEP]
have : (𝓝[s] x).NeBot := mem_closure_iff_clusterPt.mp (hts hx)
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s t : Set β
f g : β → α
h : EqOn f g s
hf : ContinuousOn f t
hg : ContinuousOn g t
hst : s ⊆ t
hts : t ⊆ closure s
x : β
hx : x ∈ t
this : NeBot (𝓝[s] x)
⊢ f x = g x
[PROOFSTEP]
exact
tendsto_nhds_unique_of_eventuallyEq ((hf x hx).mono_left <| nhdsWithin_mono _ hst)
((hg x hx).mono_left <| nhdsWithin_mono _ hst) (h.eventuallyEq_of_mem self_mem_nhdsWithin)
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s t : Set α
hs : IsCompact s
ht : IsCompact t
hst : Disjoint s t
⊢ SeparatedNhds s t
[PROOFSTEP]
simp only [SeparatedNhds, prod_subset_compl_diagonal_iff_disjoint.symm] at hst ⊢
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s t : Set α
hs : IsCompact s
ht : IsCompact t
hst : s ×ˢ t ⊆ (diagonal α)ᶜ
⊢ ∃ U V, IsOpen U ∧ IsOpen V ∧ s ⊆ U ∧ t ⊆ V ∧ U ×ˢ V ⊆ (diagonal α)ᶜ
[PROOFSTEP]
exact generalized_tube_lemma hs ht isClosed_diagonal.isOpen_compl hst
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s t : Finset α
h : Disjoint s t
⊢ Disjoint ↑s ↑t
[PROOFSTEP]
exact_mod_cast h
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
x : α
s : Finset α
h : ¬x ∈ s
⊢ SeparatedNhds {x} ↑s
[PROOFSTEP]
exact_mod_cast finset_disjoint_finset_opens_of_t2 { x } s (Finset.disjoint_singleton_left.mpr h)
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s : Set α
hs : IsCompact s
x : α
hx : x ∈ sᶜ
u v : Set α
left✝ : IsOpen u
vo : IsOpen v
su : s ⊆ u
xv : {x} ⊆ v
uv : Disjoint u v
⊢ x ∈ v
[PROOFSTEP]
simpa using xv
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
⊢ coclosedCompact α = cocompact α
[PROOFSTEP]
simp only [coclosedCompact, cocompact, iInf_and', and_iff_right_of_imp (@IsCompact.isClosed α _ _ _)]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
K U V : Set α
hK : IsCompact K
hU : IsOpen U
hV : IsOpen V
h2K : K ⊆ U ∪ V
⊢ ∃ K₁ K₂, IsCompact K₁ ∧ IsCompact K₂ ∧ K₁ ⊆ U ∧ K₂ ⊆ V ∧ K = K₁ ∪ K₂
[PROOFSTEP]
obtain ⟨O₁, O₂, h1O₁, h1O₂, h2O₁, h2O₂, hO⟩ :=
isCompact_isCompact_separated (hK.diff hU) (hK.diff hV)
(by rwa [disjoint_iff_inter_eq_empty, diff_inter_diff, diff_eq_empty])
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
K U V : Set α
hK : IsCompact K
hU : IsOpen U
hV : IsOpen V
h2K : K ⊆ U ∪ V
⊢ Disjoint (K \ U) (K \ V)
[PROOFSTEP]
rwa [disjoint_iff_inter_eq_empty, diff_inter_diff, diff_eq_empty]
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
K U V : Set α
hK : IsCompact K
hU : IsOpen U
hV : IsOpen V
h2K : K ⊆ U ∪ V
O₁ O₂ : Set α
h1O₁ : IsOpen O₁
h1O₂ : IsOpen O₂
h2O₁ : K \ U ⊆ O₁
h2O₂ : K \ V ⊆ O₂
hO : Disjoint O₁ O₂
⊢ ∃ K₁ K₂, IsCompact K₁ ∧ IsCompact K₂ ∧ K₁ ⊆ U ∧ K₂ ⊆ V ∧ K = K₁ ∪ K₂
[PROOFSTEP]
exact
⟨_, _, hK.diff h1O₁, hK.diff h1O₂, by rwa [diff_subset_comm], by rwa [diff_subset_comm], by
rw [← diff_inter, hO.inter_eq, diff_empty]⟩
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
K U V : Set α
hK : IsCompact K
hU : IsOpen U
hV : IsOpen V
h2K : K ⊆ U ∪ V
O₁ O₂ : Set α
h1O₁ : IsOpen O₁
h1O₂ : IsOpen O₂
h2O₁ : K \ U ⊆ O₁
h2O₂ : K \ V ⊆ O₂
hO : Disjoint O₁ O₂
⊢ K \ O₁ ⊆ U
[PROOFSTEP]
rwa [diff_subset_comm]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
K U V : Set α
hK : IsCompact K
hU : IsOpen U
hV : IsOpen V
h2K : K ⊆ U ∪ V
O₁ O₂ : Set α
h1O₁ : IsOpen O₁
h1O₂ : IsOpen O₂
h2O₁ : K \ U ⊆ O₁
h2O₂ : K \ V ⊆ O₂
hO : Disjoint O₁ O₂
⊢ K \ O₂ ⊆ V
[PROOFSTEP]
rwa [diff_subset_comm]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
K U V : Set α
hK : IsCompact K
hU : IsOpen U
hV : IsOpen V
h2K : K ⊆ U ∪ V
O₁ O₂ : Set α
h1O₁ : IsOpen O₁
h1O₂ : IsOpen O₂
h2O₁ : K \ U ⊆ O₁
h2O₂ : K \ V ⊆ O₂
hO : Disjoint O₁ O₂
⊢ K = K \ O₁ ∪ K \ O₂
[PROOFSTEP]
rw [← diff_inter, hO.inter_eq, diff_empty]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s : Set α
hs : IsCompact s
ι : Type u_2
t : Finset ι
U : ι → Set α
hU : ∀ (i : ι), i ∈ t → IsOpen (U i)
hsC : s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
[PROOFSTEP]
induction' t using Finset.induction with x t hx ih generalizing U s
[GOAL]
case empty
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t), U✝ i
s : Set α
hs : IsCompact s
U : ι → Set α
hU : ∀ (i : ι), i ∈ ∅ → IsOpen (U i)
hsC : s ⊆ ⋃ (i : ι) (_ : i ∈ ∅), U i
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ ∅), K i
[PROOFSTEP]
refine' ⟨fun _ => ∅, fun _ => isCompact_empty, fun i => empty_subset _, _⟩
[GOAL]
case empty
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t), U✝ i
s : Set α
hs : IsCompact s
U : ι → Set α
hU : ∀ (i : ι), i ∈ ∅ → IsOpen (U i)
hsC : s ⊆ ⋃ (i : ι) (_ : i ∈ ∅), U i
⊢ s = ⋃ (i : ι) (_ : i ∈ ∅), (fun x => ∅) i
[PROOFSTEP]
simpa only [subset_empty_iff, Finset.not_mem_empty, iUnion_false, iUnion_empty] using hsC
[GOAL]
case insert
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hU : ∀ (i : ι), i ∈ insert x t → IsOpen (U i)
hsC : s ⊆ ⋃ (i : ι) (_ : i ∈ insert x t), U i
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ insert x t), K i
[PROOFSTEP]
simp only [Finset.set_biUnion_insert] at hsC
[GOAL]
case insert
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hU : ∀ (i : ι), i ∈ insert x t → IsOpen (U i)
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ insert x t), K i
[PROOFSTEP]
simp only [Finset.forall_mem_insert] at hU
[GOAL]
case insert
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ insert x t), K i
[PROOFSTEP]
have hU' : ∀ i ∈ t, IsOpen (U i) := fun i hi => hU.2 i hi
[GOAL]
case insert
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ insert x t), K i
[PROOFSTEP]
rcases hs.binary_compact_cover hU.1 (isOpen_biUnion hU') hsC with ⟨K₁, K₂, h1K₁, h1K₂, h2K₁, h2K₂, hK⟩
[GOAL]
case insert.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ insert x t), K i
[PROOFSTEP]
rcases ih h1K₂ U hU' h2K₂ with ⟨K, h1K, h2K, h3K⟩
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
⊢ ∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ insert x t), K i
[PROOFSTEP]
refine' ⟨update K x K₁, _, _, _⟩
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
⊢ ∀ (i : ι), IsCompact (update K x K₁ i)
[PROOFSTEP]
intro i
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
i : ι
⊢ IsCompact (update K x K₁ i)
[PROOFSTEP]
rcases eq_or_ne i x with rfl | hi
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1.inl
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
t : Finset ι
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
i : ι
hx : ¬i ∈ t
hsC : s ⊆ U i ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U i) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
h2K₁ : K₁ ⊆ U i
⊢ IsCompact (update K i K₁ i)
[PROOFSTEP]
simp only [update_same, h1K₁]
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1.inr
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
i : ι
hi : i ≠ x
⊢ IsCompact (update K x K₁ i)
[PROOFSTEP]
simp only [update_noteq hi, h1K]
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
⊢ ∀ (i : ι), update K x K₁ i ⊆ U i
[PROOFSTEP]
intro i
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
i : ι
⊢ update K x K₁ i ⊆ U i
[PROOFSTEP]
rcases eq_or_ne i x with rfl | hi
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2.inl
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
t : Finset ι
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
i : ι
hx : ¬i ∈ t
hsC : s ⊆ U i ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U i) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
h2K₁ : K₁ ⊆ U i
⊢ update K i K₁ i ⊆ U i
[PROOFSTEP]
simp only [update_same, h2K₁]
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2.inr
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
i : ι
hi : i ≠ x
⊢ update K x K₁ i ⊆ U i
[PROOFSTEP]
simp only [update_noteq hi, h2K]
[GOAL]
case insert.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_3
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
s✝ : Set α
hs✝ : IsCompact s✝
ι : Type u_2
t✝ : Finset ι
U✝ : ι → Set α
hU✝ : ∀ (i : ι), i ∈ t✝ → IsOpen (U✝ i)
hsC✝ : s✝ ⊆ ⋃ (i : ι) (_ : i ∈ t✝), U✝ i
x : ι
t : Finset ι
hx : ¬x ∈ t
ih :
∀ {s : Set α},
IsCompact s →
∀ (U : ι → Set α),
(∀ (i : ι), i ∈ t → IsOpen (U i)) →
s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i →
∃ K, (∀ (i : ι), IsCompact (K i)) ∧ (∀ (i : ι), K i ⊆ U i) ∧ s = ⋃ (i : ι) (_ : i ∈ t), K i
s : Set α
hs : IsCompact s
U : ι → Set α
hsC : s ⊆ U x ∪ ⋃ (x : ι) (_ : x ∈ t), U x
hU : IsOpen (U x) ∧ ∀ (x : ι), x ∈ t → IsOpen (U x)
hU' : ∀ (i : ι), i ∈ t → IsOpen (U i)
K₁ K₂ : Set α
h1K₁ : IsCompact K₁
h1K₂ : IsCompact K₂
h2K₁ : K₁ ⊆ U x
h2K₂ : K₂ ⊆ ⋃ (i : ι) (_ : i ∈ fun i => i ∈ t.val), U i
hK : s = K₁ ∪ K₂
K : ι → Set α
h1K : ∀ (i : ι), IsCompact (K i)
h2K : ∀ (i : ι), K i ⊆ U i
h3K : K₂ = ⋃ (i : ι) (_ : i ∈ t), K i
⊢ s = ⋃ (i : ι) (_ : i ∈ insert x t), update K x K₁ i
[PROOFSTEP]
simp only [set_biUnion_insert_update _ hx, hK, h3K]
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
x : α
⊢ ∃ U, IsOpen U ∧ x ∈ U ∧ IsCompact (closure U)
[PROOFSTEP]
rcases exists_compact_mem_nhds x with ⟨K, hKc, hxK⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
x : α
K : Set α
hKc : IsCompact K
hxK : K ∈ 𝓝 x
⊢ ∃ U, IsOpen U ∧ x ∈ U ∧ IsCompact (closure U)
[PROOFSTEP]
rcases mem_nhds_iff.1 hxK with ⟨t, h1t, h2t, h3t⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
x : α
K : Set α
hKc : IsCompact K
hxK : K ∈ 𝓝 x
t : Set α
h1t : t ⊆ K
h2t : IsOpen t
h3t : x ∈ t
⊢ ∃ U, IsOpen U ∧ x ∈ U ∧ IsCompact (closure U)
[PROOFSTEP]
exact ⟨t, h2t, h3t, isCompact_closure_of_subset_compact hKc h1t⟩
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
K : Set α
hK : IsCompact K
⊢ ∃ V, IsOpen V ∧ K ⊆ V ∧ IsCompact (closure V)
[PROOFSTEP]
rcases exists_compact_superset hK with ⟨K', hK', hKK'⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
K : Set α
hK : IsCompact K
K' : Set α
hK' : IsCompact K'
hKK' : K ⊆ interior K'
⊢ ∃ V, IsOpen V ∧ K ⊆ V ∧ IsCompact (closure V)
[PROOFSTEP]
refine' ⟨interior K', isOpen_interior, hKK', isCompact_closure_of_subset_compact hK' interior_subset⟩
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
K U : Set α
hK : IsCompact K
hU : IsOpen U
hKU : K ⊆ U
⊢ ∃ V, IsOpen V ∧ K ⊆ V ∧ closure V ⊆ U ∧ IsCompact (closure V)
[PROOFSTEP]
rcases exists_compact_between hK hU hKU with ⟨V, hV, hKV, hVU⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
γ : Type u_1
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
inst✝¹ : LocallyCompactSpace α
inst✝ : T2Space α
K U : Set α
hK : IsCompact K
hU : IsOpen U
hKU : K ⊆ U
V : Set α
hV : IsCompact V
hKV : K ⊆ interior V
hVU : V ⊆ U
⊢ ∃ V, IsOpen V ∧ K ⊆ V ∧ closure V ⊆ U ∧ IsCompact (closure V)
[PROOFSTEP]
exact
⟨interior V, isOpen_interior, hKV, (closure_minimal interior_subset hV.isClosed).trans hVU,
isCompact_closure_of_subset_compact hV interior_subset⟩
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
S : Set α
⊢ IsPreirreducible S ↔ Set.Subsingleton S
[PROOFSTEP]
refine' ⟨fun h x hx y hy => _, Set.Subsingleton.isPreirreducible⟩
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
S : Set α
h : IsPreirreducible S
x : α
hx : x ∈ S
y : α
hy : y ∈ S
⊢ x = y
[PROOFSTEP]
by_contra e
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
S : Set α
h : IsPreirreducible S
x : α
hx : x ∈ S
y : α
hy : y ∈ S
e : ¬x = y
⊢ False
[PROOFSTEP]
obtain ⟨U, V, hU, hV, hxU, hyV, h'⟩ := t2_separation e
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
S : Set α
h : IsPreirreducible S
x : α
hx : x ∈ S
y : α
hy : y ∈ S
e : ¬x = y
U V : Set α
hU : IsOpen U
hV : IsOpen V
hxU : x ∈ U
hyV : y ∈ V
h' : Disjoint U V
⊢ False
[PROOFSTEP]
exact ((h U V hU hV ⟨x, hx, hxU⟩ ⟨y, hy, hyV⟩).mono <| inter_subset_right _ _).not_disjoint h'
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
γ : Type u_1
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space α
S : Set α
⊢ IsIrreducible S ↔ ∃ x, S = {x}
[PROOFSTEP]
rw [IsIrreducible, isPreirreducible_iff_subsingleton, exists_eq_singleton_iff_nonempty_subsingleton]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_have 1 ↔ 5
[GOAL]
case tfae_1_iff_5
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
⊢ RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
[PROOFSTEP]
rw [regularSpace_iff, (@compl_surjective (Set X) _).forall, forall_swap]
[GOAL]
case tfae_1_iff_5
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
⊢ (∀ (y : X) (x : Set X), IsClosed xᶜ → ¬y ∈ xᶜ → Disjoint (𝓝ˢ xᶜ) (𝓝 y)) ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
[PROOFSTEP]
simp only [isClosed_compl_iff, mem_compl_iff, Classical.not_not, @and_comm (_ ∈ _),
(nhds_basis_opens _).lift'_closure.le_basis_iff (nhds_basis_opens _), and_imp,
(nhds_basis_opens _).disjoint_iff_right, exists_prop, ← subset_interior_iff_mem_nhdsSet, interior_compl,
compl_subset_compl]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_have 5 → 6
[GOAL]
case tfae_5_to_6
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
⊢ (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
[PROOFSTEP]
exact fun h a => (h a).antisymm (𝓝 _).le_lift'_closure
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_have 6 → 4
[GOAL]
case tfae_6_to_4
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
⊢ (∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
[PROOFSTEP]
intro H a s hs
[GOAL]
case tfae_6_to_4
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
H : ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
a : X
s : Set X
hs : s ∈ 𝓝 a
⊢ ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
[PROOFSTEP]
rw [← H] at hs
[GOAL]
case tfae_6_to_4
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
H : ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
a : X
s : Set X
hs : s ∈ Filter.lift' (𝓝 a) closure
⊢ ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
[PROOFSTEP]
rcases(𝓝 a).basis_sets.lift'_closure.mem_iff.mp hs with ⟨U, hU, hUs⟩
[GOAL]
case tfae_6_to_4.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
H : ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
a : X
s : Set X
hs : s ∈ Filter.lift' (𝓝 a) closure
U : Set X
hU : U ∈ 𝓝 a
hUs : closure (id U) ⊆ s
⊢ ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
[PROOFSTEP]
exact ⟨closure U, mem_of_superset hU subset_closure, isClosed_closure, hUs⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_have 4 → 2
[GOAL]
case tfae_4_to_2
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
⊢ (∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
[PROOFSTEP]
intro H s a ha
[GOAL]
case tfae_4_to_2
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
H : ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
s : Set X
a : X
ha : ¬a ∈ closure s
⊢ Disjoint (𝓝ˢ s) (𝓝 a)
[PROOFSTEP]
have ha' : sᶜ ∈ 𝓝 a := by rwa [← mem_interior_iff_mem_nhds, interior_compl]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
H : ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
s : Set X
a : X
ha : ¬a ∈ closure s
⊢ sᶜ ∈ 𝓝 a
[PROOFSTEP]
rwa [← mem_interior_iff_mem_nhds, interior_compl]
[GOAL]
case tfae_4_to_2
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
H : ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
s : Set X
a : X
ha : ¬a ∈ closure s
ha' : sᶜ ∈ 𝓝 a
⊢ Disjoint (𝓝ˢ s) (𝓝 a)
[PROOFSTEP]
rcases H _ _ ha' with ⟨U, hU, hUc, hUs⟩
[GOAL]
case tfae_4_to_2.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
H : ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
s : Set X
a : X
ha : ¬a ∈ closure s
ha' : sᶜ ∈ 𝓝 a
U : Set X
hU : U ∈ 𝓝 a
hUc : IsClosed U
hUs : U ⊆ sᶜ
⊢ Disjoint (𝓝ˢ s) (𝓝 a)
[PROOFSTEP]
refine' disjoint_of_disjoint_of_mem disjoint_compl_left _ hU
[GOAL]
case tfae_4_to_2.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
H : ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
s : Set X
a : X
ha : ¬a ∈ closure s
ha' : sᶜ ∈ 𝓝 a
U : Set X
hU : U ∈ 𝓝 a
hUc : IsClosed U
hUs : U ⊆ sᶜ
⊢ Uᶜ ∈ 𝓝ˢ s
[PROOFSTEP]
rwa [← subset_interior_iff_mem_nhdsSet, hUc.isOpen_compl.interior_eq, subset_compl_comm]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
tfae_4_to_2 :
(∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_have 2 → 3
[GOAL]
case tfae_2_to_3
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
tfae_4_to_2 :
(∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
⊢ (∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)) →
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
[PROOFSTEP]
refine' fun H a s => ⟨fun hd has => mem_closure_iff_nhds_neBot.mp has _, H s a⟩
[GOAL]
case tfae_2_to_3
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
tfae_4_to_2 :
(∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
H : ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
a : X
s : Set X
hd : Disjoint (𝓝ˢ s) (𝓝 a)
has : a ∈ closure s
⊢ 𝓝 a ⊓ 𝓟 s = ⊥
[PROOFSTEP]
exact (hd.symm.mono_right <| @principal_le_nhdsSet _ _ s).eq_bot
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
tfae_4_to_2 :
(∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
tfae_2_to_3 :
(∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)) →
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_have 3 → 1
[GOAL]
case tfae_3_to_1
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
tfae_4_to_2 :
(∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
tfae_2_to_3 :
(∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)) →
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
⊢ (∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s) → RegularSpace X
[PROOFSTEP]
exact fun H => ⟨fun hs ha => (H _ _).mpr <| hs.closure_eq.symm ▸ ha⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
X : Type u
inst✝ : TopologicalSpace X
tfae_1_iff_5 : RegularSpace X ↔ ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a
tfae_5_to_6 : (∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a) → ∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a
tfae_6_to_4 :
(∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a) → ∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
tfae_4_to_2 :
(∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s) →
∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)
tfae_2_to_3 :
(∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a)) →
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
tfae_3_to_1 : (∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s) → RegularSpace X
⊢ List.TFAE
[RegularSpace X, ∀ (s : Set X) (a : X), ¬a ∈ closure s → Disjoint (𝓝ˢ s) (𝓝 a),
∀ (a : X) (s : Set X), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s,
∀ (a : X) (s : Set X), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s, ∀ (a : X), Filter.lift' (𝓝 a) closure ≤ 𝓝 a,
∀ (a : X), Filter.lift' (𝓝 a) closure = 𝓝 a]
[PROOFSTEP]
tfae_finish
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
⊢ Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
[PROOFSTEP]
have h := (regularSpace_TFAE α).out 0 2
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
h : RegularSpace α ↔ ∀ (a : α) (s : Set α), Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
⊢ Disjoint (𝓝ˢ s) (𝓝 a) ↔ ¬a ∈ closure s
[PROOFSTEP]
exact h.mp ‹_› _ _
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s✝ : Set α
a : α
s : Set α
h : s ∈ 𝓝 a
⊢ ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
[PROOFSTEP]
have h' := (regularSpace_TFAE α).out 0 3
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s✝ : Set α
a : α
s : Set α
h : s ∈ 𝓝 a
h' : RegularSpace α ↔ ∀ (a : α) (s : Set α), s ∈ 𝓝 a → ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
⊢ ∃ t, t ∈ 𝓝 a ∧ IsClosed t ∧ t ⊆ s
[PROOFSTEP]
exact h'.mp ‹_› _ _ h
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s : Set α
B : Set (Set α)
hB : IsTopologicalBasis B
a : α
⊢ HasBasis (𝓝 a) (fun s => a ∈ s ∧ s ∈ B) closure
[PROOFSTEP]
simpa only [and_comm] using hB.nhds_hasBasis.nhds_closure
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s✝ : Set α
B : Set (Set α)
hB : IsTopologicalBasis B
a : α
s : Set α
h : s ∈ 𝓝 a
⊢ ∃ t, t ∈ B ∧ a ∈ t ∧ closure t ⊆ s
[PROOFSTEP]
simpa only [exists_prop, and_assoc] using hB.nhds_hasBasis.nhds_closure.mem_iff.mp h
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s : Set α
a b : α
⊢ Disjoint (𝓝 a) (𝓝 b) ↔ ¬a ⤳ b
[PROOFSTEP]
rw [← nhdsSet_singleton, disjoint_nhdsSet_nhds, specializes_iff_mem_closure]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s : Set α
a b : α
⊢ a ⤳ b ↔ b ⤳ a
[PROOFSTEP]
simp only [← (disjoint_nhds_nhds_iff_not_specializes (α := α)).not_left, disjoint_comm]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
⊢ IsClosed {p | p.fst ⤳ p.snd}
[PROOFSTEP]
simp only [← isOpen_compl_iff, compl_setOf, ← disjoint_nhds_nhds_iff_not_specializes, isOpen_setOf_disjoint_nhds_nhds]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
⊢ IsClosed {p | Inseparable p.fst p.snd}
[PROOFSTEP]
simp only [← specializes_iff_inseparable, isClosed_setOf_specializes]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : RegularSpace α
a : α
s : Set α
inst✝ : TopologicalSpace β
f : β → α
hf : Inducing f
b : β
⊢ HasBasis (𝓝 b) (?m.165807 hf b) (?m.165808 hf b)
[PROOFSTEP]
rw [hf.nhds_eq_comap b]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : RegularSpace α
a : α
s : Set α
inst✝ : TopologicalSpace β
f : β → α
hf : Inducing f
b : β
⊢ HasBasis (comap f (𝓝 (f b))) (?m.165807 hf b) (?m.165808 hf b)
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
⊢ [inst : TopologicalSpace β] → {f : β → α} → Inducing f → β → Sort ?u.165737
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
⊢ [inst : TopologicalSpace β] → {f : β → α} → (hf : Inducing f) → (a : β) → ?m.165806 hf a → Prop
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
⊢ [inst : TopologicalSpace β] → {f : β → α} → (hf : Inducing f) → (a : β) → ?m.165806 hf a → Set β
[PROOFSTEP]
exact (closed_nhds_basis _).comap _
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : RegularSpace α
a : α
s✝ : Set α
inst✝ : TopologicalSpace β
f : β → α
hf : Inducing f
b : β
s : Set α
hs : s ∈ 𝓝 (f b) ∧ IsClosed s
⊢ IsClosed (f ⁻¹' id s)
[PROOFSTEP]
exact hs.2.preimage hf.continuous
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
⊢ RegularSpace X
[PROOFSTEP]
let _ := sInf T
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
x✝ : TopologicalSpace X := sInf T
⊢ RegularSpace X
[PROOFSTEP]
have :
∀ a,
(𝓝 a).HasBasis
(fun If : Σ I : Set T, I → Set X => If.1.Finite ∧ ∀ i : If.1, If.2 i ∈ @nhds X i a ∧ @IsClosed X i (If.2 i))
fun If => ⋂ i : If.1, If.snd i :=
by
intro a
rw [nhds_sInf, ← iInf_subtype'']
exact hasBasis_iInf fun t : T => @closed_nhds_basis X t (h t t.2) a
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
x✝ : TopologicalSpace X := sInf T
⊢ ∀ (a : X),
HasBasis (𝓝 a) (fun If => Set.Finite If.fst ∧ ∀ (i : ↑If.fst), Sigma.snd If i ∈ 𝓝 a ∧ IsClosed (Sigma.snd If i))
fun If => ⋂ (i : ↑If.fst), Sigma.snd If i
[PROOFSTEP]
intro a
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
x✝ : TopologicalSpace X := sInf T
a : X
⊢ HasBasis (𝓝 a) (fun If => Set.Finite If.fst ∧ ∀ (i : ↑If.fst), Sigma.snd If i ∈ 𝓝 a ∧ IsClosed (Sigma.snd If i))
fun If => ⋂ (i : ↑If.fst), Sigma.snd If i
[PROOFSTEP]
rw [nhds_sInf, ← iInf_subtype'']
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
x✝ : TopologicalSpace X := sInf T
a : X
⊢ HasBasis (⨅ (i : ↑T), 𝓝 a)
(fun If => Set.Finite If.fst ∧ ∀ (i : ↑If.fst), Sigma.snd If i ∈ 𝓝 a ∧ IsClosed (Sigma.snd If i)) fun If =>
⋂ (i : ↑If.fst), Sigma.snd If i
[PROOFSTEP]
exact hasBasis_iInf fun t : T => @closed_nhds_basis X t (h t t.2) a
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
x✝ : TopologicalSpace X := sInf T
this :
∀ (a : X),
HasBasis (𝓝 a) (fun If => Set.Finite If.fst ∧ ∀ (i : ↑If.fst), Sigma.snd If i ∈ 𝓝 a ∧ IsClosed (Sigma.snd If i))
fun If => ⋂ (i : ↑If.fst), Sigma.snd If i
⊢ RegularSpace X
[PROOFSTEP]
refine' RegularSpace.ofBasis this fun a If hIf => isClosed_iInter fun i => _
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a✝ : α
s : Set α
X : Type u_1
T : Set (TopologicalSpace X)
h : ∀ (t : TopologicalSpace X), t ∈ T → RegularSpace X
x✝ : TopologicalSpace X := sInf T
this :
∀ (a : X),
HasBasis (𝓝 a) (fun If => Set.Finite If.fst ∧ ∀ (i : ↑If.fst), Sigma.snd If i ∈ 𝓝 a ∧ IsClosed (Sigma.snd If i))
fun If => ⋂ (i : ↑If.fst), Sigma.snd If i
a : X
If : (I : Set ↑T) × (↑I → Set X)
hIf : Set.Finite If.fst ∧ ∀ (i : ↑If.fst), Sigma.snd If i ∈ 𝓝 a ∧ IsClosed (Sigma.snd If i)
i : ↑If.fst
⊢ IsClosed (Sigma.snd If i)
[PROOFSTEP]
exact (hIf.2 i).2.mono (sInf_le (i : T).2)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
X : Type u_1
t₁ t₂ : TopologicalSpace X
h₁ : RegularSpace X
h₂ : RegularSpace X
⊢ RegularSpace X
[PROOFSTEP]
rw [inf_eq_iInf]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
a : α
s : Set α
X : Type u_1
t₁ t₂ : TopologicalSpace X
h₁ : RegularSpace X
h₂ : RegularSpace X
⊢ RegularSpace X
[PROOFSTEP]
exact regularSpace_iInf (Bool.forall_bool.2 ⟨h₂, h₁⟩)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
⊢ T25Space α
[PROOFSTEP]
refine' ⟨fun x y hne => _⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
hne : x ≠ y
⊢ Disjoint (Filter.lift' (𝓝 x) closure) (Filter.lift' (𝓝 y) closure)
[PROOFSTEP]
rw [lift'_nhds_closure, lift'_nhds_closure]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
hne : x ≠ y
⊢ Disjoint (𝓝 x) (𝓝 y)
[PROOFSTEP]
have : x ∉ closure { y } ∨ y ∉ closure { x } := (t0Space_iff_or_not_mem_closure α).mp inferInstance x y hne
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
hne : x ≠ y
this : ¬x ∈ closure {y} ∨ ¬y ∈ closure {x}
⊢ Disjoint (𝓝 x) (𝓝 y)
[PROOFSTEP]
simp only [← disjoint_nhds_nhdsSet, nhdsSet_singleton] at this
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
hne : x ≠ y
this : Disjoint (𝓝 x) (𝓝 y) ∨ Disjoint (𝓝 y) (𝓝 x)
⊢ Disjoint (𝓝 x) (𝓝 y)
[PROOFSTEP]
exact this.elim id fun h => h.symm
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
h : x ≠ y
⊢ ∃ U₁,
U₁ ∈ 𝓝 x ∧
∃ V₁,
V₁ ∈ 𝓝 x ∧
∃ U₂,
U₂ ∈ 𝓝 y ∧
∃ V₂, V₂ ∈ 𝓝 y ∧ IsClosed V₁ ∧ IsClosed V₂ ∧ IsOpen U₁ ∧ IsOpen U₂ ∧ V₁ ⊆ U₁ ∧ V₂ ⊆ U₂ ∧ Disjoint U₁ U₂
[PROOFSTEP]
rcases t2_separation h with ⟨U₁, U₂, U₁_op, U₂_op, x_in, y_in, H⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
h : x ≠ y
U₁ U₂ : Set α
U₁_op : IsOpen U₁
U₂_op : IsOpen U₂
x_in : x ∈ U₁
y_in : y ∈ U₂
H : Disjoint U₁ U₂
⊢ ∃ U₁,
U₁ ∈ 𝓝 x ∧
∃ V₁,
V₁ ∈ 𝓝 x ∧
∃ U₂,
U₂ ∈ 𝓝 y ∧
∃ V₂, V₂ ∈ 𝓝 y ∧ IsClosed V₁ ∧ IsClosed V₂ ∧ IsOpen U₁ ∧ IsOpen U₂ ∧ V₁ ⊆ U₁ ∧ V₂ ⊆ U₂ ∧ Disjoint U₁ U₂
[PROOFSTEP]
rcases exists_mem_nhds_isClosed_subset (U₁_op.mem_nhds x_in) with ⟨V₁, V₁_in, V₁_closed, h₁⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
h : x ≠ y
U₁ U₂ : Set α
U₁_op : IsOpen U₁
U₂_op : IsOpen U₂
x_in : x ∈ U₁
y_in : y ∈ U₂
H : Disjoint U₁ U₂
V₁ : Set α
V₁_in : V₁ ∈ 𝓝 x
V₁_closed : IsClosed V₁
h₁ : V₁ ⊆ U₁
⊢ ∃ U₁,
U₁ ∈ 𝓝 x ∧
∃ V₁,
V₁ ∈ 𝓝 x ∧
∃ U₂,
U₂ ∈ 𝓝 y ∧
∃ V₂, V₂ ∈ 𝓝 y ∧ IsClosed V₁ ∧ IsClosed V₂ ∧ IsOpen U₁ ∧ IsOpen U₂ ∧ V₁ ⊆ U₁ ∧ V₂ ⊆ U₂ ∧ Disjoint U₁ U₂
[PROOFSTEP]
rcases exists_mem_nhds_isClosed_subset (U₂_op.mem_nhds y_in) with ⟨V₂, V₂_in, V₂_closed, h₂⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T3Space α
x y : α
h : x ≠ y
U₁ U₂ : Set α
U₁_op : IsOpen U₁
U₂_op : IsOpen U₂
x_in : x ∈ U₁
y_in : y ∈ U₂
H : Disjoint U₁ U₂
V₁ : Set α
V₁_in : V₁ ∈ 𝓝 x
V₁_closed : IsClosed V₁
h₁ : V₁ ⊆ U₁
V₂ : Set α
V₂_in : V₂ ∈ 𝓝 y
V₂_closed : IsClosed V₂
h₂ : V₂ ⊆ U₂
⊢ ∃ U₁,
U₁ ∈ 𝓝 x ∧
∃ V₁,
V₁ ∈ 𝓝 x ∧
∃ U₂,
U₂ ∈ 𝓝 y ∧
∃ V₂, V₂ ∈ 𝓝 y ∧ IsClosed V₁ ∧ IsClosed V₂ ∧ IsOpen U₁ ∧ IsOpen U₂ ∧ V₁ ⊆ U₁ ∧ V₂ ⊆ U₂ ∧ Disjoint U₁ U₂
[PROOFSTEP]
exact
⟨U₁, mem_of_superset V₁_in h₁, V₁, V₁_in, U₂, mem_of_superset V₂_in h₂, V₂, V₂_in, V₁_closed, V₂_closed, U₁_op, U₂_op,
h₁, h₂, H⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
s : Set (SeparationQuotient α)
a : SeparationQuotient α
hs : IsClosed s
ha : ¬a ∈ s
⊢ Disjoint (𝓝ˢ s) (𝓝 a)
[PROOFSTEP]
rcases surjective_mk a with ⟨a, rfl⟩
[GOAL]
case intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
s : Set (SeparationQuotient α)
hs : IsClosed s
a : α
ha : ¬SeparationQuotient.mk a ∈ s
⊢ Disjoint (𝓝ˢ s) (𝓝 (SeparationQuotient.mk a))
[PROOFSTEP]
rw [← disjoint_comap_iff surjective_mk, comap_mk_nhds_mk, comap_mk_nhdsSet]
[GOAL]
case intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : RegularSpace α
s : Set (SeparationQuotient α)
hs : IsClosed s
a : α
ha : ¬SeparationQuotient.mk a ∈ s
⊢ Disjoint (𝓝ˢ (SeparationQuotient.mk ⁻¹' s)) (𝓝 a)
[PROOFSTEP]
exact RegularSpace.regular (hs.preimage continuous_mk) ha
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s t : Set α
hs : IsClosed s
ht : IsOpen t
hst : s ⊆ t
⊢ ∃ u, IsOpen u ∧ s ⊆ u ∧ closure u ⊆ t
[PROOFSTEP]
have : Disjoint s tᶜ := Set.disjoint_left.mpr fun x hxs hxt => hxt (hst hxs)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s t : Set α
hs : IsClosed s
ht : IsOpen t
hst : s ⊆ t
this : Disjoint s tᶜ
⊢ ∃ u, IsOpen u ∧ s ⊆ u ∧ closure u ⊆ t
[PROOFSTEP]
rcases normal_separation hs (isClosed_compl_iff.2 ht) this with ⟨s', t', hs', ht', hss', htt', hs't'⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s t : Set α
hs : IsClosed s
ht : IsOpen t
hst : s ⊆ t
this : Disjoint s tᶜ
s' t' : Set α
hs' : IsOpen s'
ht' : IsOpen t'
hss' : s ⊆ s'
htt' : tᶜ ⊆ t'
hs't' : Disjoint s' t'
⊢ ∃ u, IsOpen u ∧ s ⊆ u ∧ closure u ⊆ t
[PROOFSTEP]
refine ⟨s', hs', hss', Subset.trans (closure_minimal ?_ (isClosed_compl_iff.2 ht')) (compl_subset_comm.1 htt')⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s t : Set α
hs : IsClosed s
ht : IsOpen t
hst : s ⊆ t
this : Disjoint s tᶜ
s' t' : Set α
hs' : IsOpen s'
ht' : IsOpen t'
hss' : s ⊆ s'
htt' : tᶜ ⊆ t'
hs't' : Disjoint s' t'
⊢ s' ⊆ t'ᶜ
[PROOFSTEP]
exact fun x hxs hxt => hs't'.le_bot ⟨hxs, hxt⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s✝ : Set α
a✝ : α
hs : IsClosed s✝
hxs : ¬a✝ ∈ s✝
⊢ Disjoint (𝓝ˢ s✝) (𝓝 a✝)
[PROOFSTEP]
simpa only [nhdsSet_singleton] using
(normal_separation hs isClosed_singleton (disjoint_singleton_right.mpr hxs)).disjoint_nhdsSet
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NormalSpace β
f : α → β
hf : ClosedEmbedding f
s t : Set α
hs : IsClosed s
ht : IsClosed t
hst : Disjoint s t
⊢ SeparatedNhds s t
[PROOFSTEP]
have H : SeparatedNhds (f '' s) (f '' t) :=
NormalSpace.normal (f '' s) (f '' t) (hf.isClosedMap s hs) (hf.isClosedMap t ht)
(disjoint_image_of_injective hf.inj hst)
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NormalSpace β
f : α → β
hf : ClosedEmbedding f
s t : Set α
hs : IsClosed s
ht : IsClosed t
hst : Disjoint s t
H : SeparatedNhds (f '' s) (f '' t)
⊢ SeparatedNhds s t
[PROOFSTEP]
exact (H.preimage hf.continuous).mono (subset_preimage_image _ _) (subset_preimage_image _ _)
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s t : Set (SeparationQuotient α)
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
⊢ Disjoint (𝓝ˢ s) (𝓝ˢ t)
[PROOFSTEP]
rw [← disjoint_comap_iff surjective_mk, comap_mk_nhdsSet, comap_mk_nhdsSet]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : NormalSpace α
s t : Set (SeparationQuotient α)
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
⊢ Disjoint (𝓝ˢ (mk ⁻¹' s)) (𝓝ˢ (mk ⁻¹' t))
[PROOFSTEP]
exact (normal_separation (hs.preimage continuous_mk) (ht.preimage continuous_mk) (hd.preimage mk)).disjoint_nhdsSet
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
⊢ NormalSpace α
[PROOFSTEP]
have key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U : Set (countableBasis α),
(s ⊆ ⋃ u ∈ U, ↑u) ∧
(∀ u ∈ U, Disjoint (closure ↑u) t) ∧
∀ n : ℕ, IsClosed (⋃ (u ∈ U) (_ : Encodable.encode u ≤ n), closure (u : Set α)) :=
by
intro s t hc hd
rw [disjoint_left] at hd
have : ∀ x ∈ s, ∃ U ∈ countableBasis α, x ∈ U ∧ Disjoint (closure U) t :=
by
intro x hx
rcases(isBasis_countableBasis α).exists_closure_subset (hc.compl_mem_nhds (hd hx)) with ⟨u, hu, hxu, hut⟩
exact ⟨u, hu, hxu, disjoint_left.2 hut⟩
choose! U hu hxu hd using this
set V : s → countableBasis α := MapsTo.restrict _ _ _ hu
refine' ⟨range V, _, forall_range_iff.2 <| Subtype.forall.2 hd, fun n => _⟩
· rw [biUnion_range]
exact fun x hx => mem_iUnion.2 ⟨⟨x, hx⟩, hxu x hx⟩
· simp only [← iSup_eq_iUnion, iSup_and']
exact
isClosed_biUnion (((finite_le_nat n).preimage_embedding (Encodable.encode' _)).subset <| inter_subset_right _ _)
fun u _ => isClosed_closure
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
⊢ ∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
intro s t hc hd
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd : Disjoint s t
⊢ ∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
rw [disjoint_left] at hd
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
⊢ ∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
have : ∀ x ∈ s, ∃ U ∈ countableBasis α, x ∈ U ∧ Disjoint (closure U) t :=
by
intro x hx
rcases(isBasis_countableBasis α).exists_closure_subset (hc.compl_mem_nhds (hd hx)) with ⟨u, hu, hxu, hut⟩
exact ⟨u, hu, hxu, disjoint_left.2 hut⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
⊢ ∀ (x : α), x ∈ s → ∃ U, U ∈ countableBasis α ∧ x ∈ U ∧ Disjoint (closure U) t
[PROOFSTEP]
intro x hx
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
x : α
hx : x ∈ s
⊢ ∃ U, U ∈ countableBasis α ∧ x ∈ U ∧ Disjoint (closure U) t
[PROOFSTEP]
rcases(isBasis_countableBasis α).exists_closure_subset (hc.compl_mem_nhds (hd hx)) with ⟨u, hu, hxu, hut⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
x : α
hx : x ∈ s
u : Set α
hu : u ∈ countableBasis α
hxu : x ∈ u
hut : closure u ⊆ tᶜ
⊢ ∃ U, U ∈ countableBasis α ∧ x ∈ U ∧ Disjoint (closure U) t
[PROOFSTEP]
exact ⟨u, hu, hxu, disjoint_left.2 hut⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
this : ∀ (x : α), x ∈ s → ∃ U, U ∈ countableBasis α ∧ x ∈ U ∧ Disjoint (closure U) t
⊢ ∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
choose! U hu hxu hd using this
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd✝ : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
U : α → Set α
hu : ∀ (x : α), x ∈ s → U x ∈ countableBasis α
hxu : ∀ (x : α), x ∈ s → x ∈ U x
hd : ∀ (x : α), x ∈ s → Disjoint (closure (U x)) t
⊢ ∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
set V : s → countableBasis α := MapsTo.restrict _ _ _ hu
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd✝ : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
U : α → Set α
hu : ∀ (x : α), x ∈ s → U x ∈ countableBasis α
hxu : ∀ (x : α), x ∈ s → x ∈ U x
hd : ∀ (x : α), x ∈ s → Disjoint (closure (U x)) t
V : ↑s → ↑(countableBasis α) := MapsTo.restrict (fun x => U x) s (countableBasis α) hu
⊢ ∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
refine' ⟨range V, _, forall_range_iff.2 <| Subtype.forall.2 hd, fun n => _⟩
[GOAL]
case refine'_1
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd✝ : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
U : α → Set α
hu : ∀ (x : α), x ∈ s → U x ∈ countableBasis α
hxu : ∀ (x : α), x ∈ s → x ∈ U x
hd : ∀ (x : α), x ∈ s → Disjoint (closure (U x)) t
V : ↑s → ↑(countableBasis α) := MapsTo.restrict (fun x => U x) s (countableBasis α) hu
⊢ s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ range V), ↑u
[PROOFSTEP]
rw [biUnion_range]
[GOAL]
case refine'_1
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd✝ : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
U : α → Set α
hu : ∀ (x : α), x ∈ s → U x ∈ countableBasis α
hxu : ∀ (x : α), x ∈ s → x ∈ U x
hd : ∀ (x : α), x ∈ s → Disjoint (closure (U x)) t
V : ↑s → ↑(countableBasis α) := MapsTo.restrict (fun x => U x) s (countableBasis α) hu
⊢ s ⊆ ⋃ (y : ↑s), ↑(V y)
[PROOFSTEP]
exact fun x hx => mem_iUnion.2 ⟨⟨x, hx⟩, hxu x hx⟩
[GOAL]
case refine'_2
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd✝ : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
U : α → Set α
hu : ∀ (x : α), x ∈ s → U x ∈ countableBasis α
hxu : ∀ (x : α), x ∈ s → x ∈ U x
hd : ∀ (x : α), x ∈ s → Disjoint (closure (U x)) t
V : ↑s → ↑(countableBasis α) := MapsTo.restrict (fun x => U x) s (countableBasis α) hu
n : ℕ
⊢ IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ range V) (_ : Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
simp only [← iSup_eq_iUnion, iSup_and']
[GOAL]
case refine'_2
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
s t : Set α
hc : IsClosed t
hd✝ : ∀ ⦃a : α⦄, a ∈ s → ¬a ∈ t
U : α → Set α
hu : ∀ (x : α), x ∈ s → U x ∈ countableBasis α
hxu : ∀ (x : α), x ∈ s → x ∈ U x
hd : ∀ (x : α), x ∈ s → Disjoint (closure (U x)) t
V : ↑s → ↑(countableBasis α) := MapsTo.restrict (fun x => U x) s (countableBasis α) hu
n : ℕ
⊢ IsClosed
(⨆ (u : ↑(countableBasis α)) (_ :
u ∈ range (MapsTo.restrict (fun x => U x) s (countableBasis α) hu) ∧ Encodable.encode u ≤ n), closure ↑u)
[PROOFSTEP]
exact
isClosed_biUnion (((finite_le_nat n).preimage_embedding (Encodable.encode' _)).subset <| inter_subset_right _ _)
fun u _ => isClosed_closure
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
⊢ NormalSpace α
[PROOFSTEP]
refine' ⟨fun s t hs ht hd => _⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
⊢ SeparatedNhds s t
[PROOFSTEP]
rcases key ht hd with ⟨U, hsU, hUd, hUc⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
⊢ SeparatedNhds s t
[PROOFSTEP]
rcases key hs hd.symm with ⟨V, htV, hVd, hVc⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
⊢ SeparatedNhds s t
[PROOFSTEP]
refine
⟨⋃ u ∈ U, ↑u \ ⋃ (v ∈ V) (_ : Encodable.encode v ≤ Encodable.encode u), closure ↑v,
⋃ v ∈ V, ↑v \ ⋃ (u ∈ U) (_ : Encodable.encode u ≤ Encodable.encode v), closure ↑u,
isOpen_biUnion fun u _ => (isOpen_of_mem_countableBasis u.2).sdiff (hVc _),
isOpen_biUnion fun v _ => (isOpen_of_mem_countableBasis v.2).sdiff (hUc _), fun x hx => ?_, fun x hx => ?_, ?_⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_1
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ s
⊢ x ∈
⋃ (u : ↑(countableBasis α)) (_ : u ∈ U),
↑u \ ⋃ (v : ↑(countableBasis α)) (_ : v ∈ V) (_ : Encodable.encode v ≤ Encodable.encode u), closure ↑v
[PROOFSTEP]
rcases mem_iUnion₂.1 (hsU hx) with ⟨u, huU, hxu⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_1.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ s
u : ↑(countableBasis α)
huU : u ∈ U
hxu : x ∈ ↑u
⊢ x ∈
⋃ (u : ↑(countableBasis α)) (_ : u ∈ U),
↑u \ ⋃ (v : ↑(countableBasis α)) (_ : v ∈ V) (_ : Encodable.encode v ≤ Encodable.encode u), closure ↑v
[PROOFSTEP]
refine' mem_biUnion huU ⟨hxu, _⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_1.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ s
u : ↑(countableBasis α)
huU : u ∈ U
hxu : x ∈ ↑u
⊢ ¬x ∈ ⋃ (v : ↑(countableBasis α)) (_ : v ∈ V) (_ : Encodable.encode v ≤ Encodable.encode u), closure ↑v
[PROOFSTEP]
simp only [mem_iUnion]
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_1.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ s
u : ↑(countableBasis α)
huU : u ∈ U
hxu : x ∈ ↑u
⊢ ¬∃ i h i_1, x ∈ closure ↑i
[PROOFSTEP]
rintro ⟨v, hvV, -, hxv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_1.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ s
u : ↑(countableBasis α)
huU : u ∈ U
hxu : x ∈ ↑u
v : ↑(countableBasis α)
hvV : v ∈ V
hxv : x ∈ closure ↑v
⊢ False
[PROOFSTEP]
exact (hVd v hvV).le_bot ⟨hxv, hx⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_2
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ t
⊢ x ∈
⋃ (v : ↑(countableBasis α)) (_ : v ∈ V),
↑v \ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ Encodable.encode v), closure ↑u
[PROOFSTEP]
rcases mem_iUnion₂.1 (htV hx) with ⟨v, hvV, hxv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_2.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ t
v : ↑(countableBasis α)
hvV : v ∈ V
hxv : x ∈ ↑v
⊢ x ∈
⋃ (v : ↑(countableBasis α)) (_ : v ∈ V),
↑v \ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ Encodable.encode v), closure ↑u
[PROOFSTEP]
refine' mem_biUnion hvV ⟨hxv, _⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_2.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ t
v : ↑(countableBasis α)
hvV : v ∈ V
hxv : x ∈ ↑v
⊢ ¬x ∈ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ Encodable.encode v), closure ↑u
[PROOFSTEP]
simp only [mem_iUnion]
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_2.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ t
v : ↑(countableBasis α)
hvV : v ∈ V
hxv : x ∈ ↑v
⊢ ¬∃ i h i_1, x ∈ closure ↑i
[PROOFSTEP]
rintro ⟨u, huU, -, hxu⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_2.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
x : α
hx : x ∈ t
v : ↑(countableBasis α)
hvV : v ∈ V
hxv : x ∈ ↑v
u : ↑(countableBasis α)
huU : u ∈ U
hxu : x ∈ closure ↑u
⊢ False
[PROOFSTEP]
exact (hUd u huU).le_bot ⟨hxu, hx⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_3
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
⊢ Disjoint
(⋃ (u : ↑(countableBasis α)) (_ : u ∈ U),
↑u \ ⋃ (v : ↑(countableBasis α)) (_ : v ∈ V) (_ : Encodable.encode v ≤ Encodable.encode u), closure ↑v)
(⋃ (v : ↑(countableBasis α)) (_ : v ∈ V),
↑v \ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ Encodable.encode v), closure ↑u)
[PROOFSTEP]
simp only [disjoint_left, mem_iUnion, mem_diff, not_exists, not_and, not_forall, not_not]
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_3
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
⊢ ∀ ⦃a : α⦄,
(∃ i h, a ∈ ↑i ∧ ∀ (x : ↑(countableBasis α)), x ∈ V → Encodable.encode x ≤ Encodable.encode i → ¬a ∈ closure ↑x) →
∀ (x : ↑(countableBasis α)), x ∈ V → a ∈ ↑x → ∃ x_2 h h, a ∈ closure ↑x_2
[PROOFSTEP]
rintro a ⟨u, huU, hau, haV⟩ v hvV hav
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_3.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
a : α
u : ↑(countableBasis α)
huU : u ∈ U
hau : a ∈ ↑u
haV : ∀ (x : ↑(countableBasis α)), x ∈ V → Encodable.encode x ≤ Encodable.encode u → ¬a ∈ closure ↑x
v : ↑(countableBasis α)
hvV : v ∈ V
hav : a ∈ ↑v
⊢ ∃ x h h, a ∈ closure ↑x
[PROOFSTEP]
cases' le_total (Encodable.encode u) (Encodable.encode v) with hle hle
[GOAL]
case intro.intro.intro.intro.intro.intro.refine_3.intro.intro.intro.inl
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
a : α
u : ↑(countableBasis α)
huU : u ∈ U
hau : a ∈ ↑u
haV : ∀ (x : ↑(countableBasis α)), x ∈ V → Encodable.encode x ≤ Encodable.encode u → ¬a ∈ closure ↑x
v : ↑(countableBasis α)
hvV : v ∈ V
hav : a ∈ ↑v
hle : Encodable.encode u ≤ Encodable.encode v
⊢ ∃ x h h, a ∈ closure ↑x
case intro.intro.intro.intro.intro.intro.refine_3.intro.intro.intro.inr
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : SecondCountableTopology α
inst✝ : T3Space α
key :
∀ {s t : Set α},
IsClosed t →
Disjoint s t →
∃ U,
s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u ∧
(∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t) ∧
∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
U : Set ↑(countableBasis α)
hsU : s ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ U), ↑u
hUd : ∀ (u : ↑(countableBasis α)), u ∈ U → Disjoint (closure ↑u) t
hUc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ U) (_ : Encodable.encode u ≤ n), closure ↑u)
V : Set ↑(countableBasis α)
htV : t ⊆ ⋃ (u : ↑(countableBasis α)) (_ : u ∈ V), ↑u
hVd : ∀ (u : ↑(countableBasis α)), u ∈ V → Disjoint (closure ↑u) s
hVc : ∀ (n : ℕ), IsClosed (⋃ (u : ↑(countableBasis α)) (_ : u ∈ V) (_ : Encodable.encode u ≤ n), closure ↑u)
a : α
u : ↑(countableBasis α)
huU : u ∈ U
hau : a ∈ ↑u
haV : ∀ (x : ↑(countableBasis α)), x ∈ V → Encodable.encode x ≤ Encodable.encode u → ¬a ∈ closure ↑x
v : ↑(countableBasis α)
hvV : v ∈ V
hav : a ∈ ↑v
hle : Encodable.encode v ≤ Encodable.encode u
⊢ ∃ x h h, a ∈ closure ↑x
[PROOFSTEP]
exacts [⟨u, huU, hle, subset_closure hau⟩, (haV _ hvV hle <| subset_closure hav).elim]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T5Space β
e : α → β
he : _root_.Embedding e
⊢ T5Space α
[PROOFSTEP]
haveI := he.t1Space
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T5Space β
e : α → β
he : _root_.Embedding e
this : T1Space α
⊢ T5Space α
[PROOFSTEP]
refine' ⟨fun s t hd₁ hd₂ => _⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T5Space β
e : α → β
he : _root_.Embedding e
this : T1Space α
s t : Set α
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (𝓝ˢ s) (𝓝ˢ t)
[PROOFSTEP]
simp only [he.toInducing.nhdsSet_eq_comap]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T5Space β
e : α → β
he : _root_.Embedding e
this : T1Space α
s t : Set α
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (comap e (𝓝ˢ (e '' s))) (comap e (𝓝ˢ (e '' t)))
[PROOFSTEP]
refine disjoint_comap (completely_normal ?_ ?_)
[GOAL]
case refine_1
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T5Space β
e : α → β
he : _root_.Embedding e
this : T1Space α
s t : Set α
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (closure (e '' s)) (e '' t)
[PROOFSTEP]
rwa [← subset_compl_iff_disjoint_left, image_subset_iff, preimage_compl, ← he.closure_eq_preimage_closure_image,
subset_compl_iff_disjoint_left]
[GOAL]
case refine_2
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : T5Space β
e : α → β
he : _root_.Embedding e
this : T1Space α
s t : Set α
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (e '' s) (closure (e '' t))
[PROOFSTEP]
rwa [← subset_compl_iff_disjoint_right, image_subset_iff, preimage_compl, ← he.closure_eq_preimage_closure_image,
subset_compl_iff_disjoint_right]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
⊢ Disjoint (closure s) t
[PROOFSTEP]
rwa [hs.closure_eq]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set α
hs : IsClosed s
ht : IsClosed t
hd : Disjoint s t
⊢ Disjoint s (closure t)
[PROOFSTEP]
rwa [ht.closure_eq]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set (SeparationQuotient α)
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (𝓝ˢ s) (𝓝ˢ t)
[PROOFSTEP]
rw [← disjoint_comap_iff surjective_mk, comap_mk_nhdsSet, comap_mk_nhdsSet]
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set (SeparationQuotient α)
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (𝓝ˢ (SeparationQuotient.mk ⁻¹' s)) (𝓝ˢ (SeparationQuotient.mk ⁻¹' t))
[PROOFSTEP]
apply T5Space.completely_normal
[GOAL]
case a
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set (SeparationQuotient α)
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (closure (SeparationQuotient.mk ⁻¹' s)) (SeparationQuotient.mk ⁻¹' t)
[PROOFSTEP]
rw [← preimage_mk_closure]
[GOAL]
case a
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set (SeparationQuotient α)
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (SeparationQuotient.mk ⁻¹' s) (closure (SeparationQuotient.mk ⁻¹' t))
[PROOFSTEP]
rw [← preimage_mk_closure]
[GOAL]
case a
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set (SeparationQuotient α)
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (SeparationQuotient.mk ⁻¹' closure s) (SeparationQuotient.mk ⁻¹' t)
case a
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T5Space α
s t : Set (SeparationQuotient α)
hd₁ : Disjoint (closure s) t
hd₂ : Disjoint s (closure t)
⊢ Disjoint (SeparationQuotient.mk ⁻¹' s) (SeparationQuotient.mk ⁻¹' closure t)
[PROOFSTEP]
exacts [hd₁.preimage mk, hd₂.preimage mk]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
⊢ connectedComponent x = ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z
[PROOFSTEP]
apply Subset.antisymm connectedComponent_subset_iInter_clopen
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ connectedComponent x
[PROOFSTEP]
refine'
IsPreconnected.subset_connectedComponent _
(mem_iInter.2 fun Z => Z.2.2)
-- We do this by showing that any disjoint cover by two closed sets implies
-- that one of these closed sets must contain our whole thing.
-- To reduce to the case where the cover is disjoint on all of `α` we need that `s` is closed
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
⊢ IsPreconnected (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
[PROOFSTEP]
have hs : @IsClosed α _ (⋂ Z : { Z : Set α // IsClopen Z ∧ x ∈ Z }, Z) := isClosed_iInter fun Z => Z.2.1.2
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
⊢ IsPreconnected (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
[PROOFSTEP]
rw [isPreconnected_iff_subset_of_fully_disjoint_closed hs]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
⊢ ∀ (u v : Set α),
IsClosed u →
IsClosed v →
⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ u ∪ v →
Disjoint u v → ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ u ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ v
[PROOFSTEP]
intro a b ha hb hab ab_disj
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
haveI :=
@normalOfCompactT2 α _ _
_
-- Since our space is normal, we get two larger disjoint open sets containing the disjoint
-- closed sets. If we can show that our intersection is a subset of any of these we can then
-- "descend" this to show that it is a subset of either a or b.
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
rcases normal_separation ha hb ab_disj with ⟨u, v, hu, hv, hau, hbv, huv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
obtain ⟨Z, H⟩ : ∃ Z : Set α, IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
⊢ ∃ Z, IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
[PROOFSTEP]
have H1 :=
(hu.union hv).isClosed_compl.isCompact.inter_iInter_nonempty (fun Z : { Z : Set α // IsClopen Z ∧ x ∈ Z } => Z)
fun Z => Z.2.1.2
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
H1 :
(∀ (t : Finset { Z // IsClopen Z ∧ x ∈ Z }),
Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ t), (fun Z => ↑Z) i)) →
Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }), (fun Z => ↑Z) i)
⊢ ∃ Z, IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
[PROOFSTEP]
rw [← not_disjoint_iff_nonempty_inter, imp_not_comm, not_forall] at H1
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
H1 :
Disjoint (u ∪ v)ᶜ (⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }), (fun Z => ↑Z) i) →
∃ x_1, ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ x_1), (fun Z => ↑Z) i)
⊢ ∃ Z, IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
[PROOFSTEP]
cases' H1 (disjoint_compl_left_iff_subset.2 <| hab.trans <| union_subset_union hau hbv) with Zi H2
[GOAL]
case intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
H1 :
Disjoint (u ∪ v)ᶜ (⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }), (fun Z => ↑Z) i) →
∃ x_1, ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ x_1), (fun Z => ↑Z) i)
Zi : Finset { Z // IsClopen Z ∧ x ∈ Z }
H2 : ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ Zi), (fun Z => ↑Z) i)
⊢ ∃ Z, IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
[PROOFSTEP]
refine' ⟨⋂ U ∈ Zi, Subtype.val U, _, _, _⟩
[GOAL]
case intro.refine'_1
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
H1 :
Disjoint (u ∪ v)ᶜ (⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }), (fun Z => ↑Z) i) →
∃ x_1, ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ x_1), (fun Z => ↑Z) i)
Zi : Finset { Z // IsClopen Z ∧ x ∈ Z }
H2 : ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ Zi), (fun Z => ↑Z) i)
⊢ IsClopen (⋂ (U : { Z // IsClopen Z ∧ x ∈ Z }) (_ : U ∈ Zi), ↑U)
[PROOFSTEP]
exact isClopen_biInter_finset fun Z _ => Z.2.1
[GOAL]
case intro.refine'_2
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
H1 :
Disjoint (u ∪ v)ᶜ (⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }), (fun Z => ↑Z) i) →
∃ x_1, ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ x_1), (fun Z => ↑Z) i)
Zi : Finset { Z // IsClopen Z ∧ x ∈ Z }
H2 : ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ Zi), (fun Z => ↑Z) i)
⊢ x ∈ ⋂ (U : { Z // IsClopen Z ∧ x ∈ Z }) (_ : U ∈ Zi), ↑U
[PROOFSTEP]
exact mem_iInter₂.2 fun Z _ => Z.2.2
[GOAL]
case intro.refine'_3
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
H1 :
Disjoint (u ∪ v)ᶜ (⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }), (fun Z => ↑Z) i) →
∃ x_1, ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ x_1), (fun Z => ↑Z) i)
Zi : Finset { Z // IsClopen Z ∧ x ∈ Z }
H2 : ¬Set.Nonempty ((u ∪ v)ᶜ ∩ ⋂ (i : { Z // IsClopen Z ∧ x ∈ Z }) (_ : i ∈ Zi), (fun Z => ↑Z) i)
⊢ ⋂ (U : { Z // IsClopen Z ∧ x ∈ Z }) (_ : U ∈ Zi), ↑U ⊆ u ∪ v
[PROOFSTEP]
rwa [← disjoint_compl_left_iff_subset, disjoint_iff_inter_eq_empty, ← not_nonempty_iff_eq_empty]
-- So, we get a disjoint decomposition `Z = Z ∩ u ∪ Z ∩ v` of clopen sets. The intersection of all
-- clopen neighbourhoods will then lie in whichever of u or v x lies in and hence will be a subset
-- of either a or b.
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
have H1 := isClopen_inter_of_disjoint_cover_clopen H.1 H.2.2 hu hv huv
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ u ∪ v
H1 : IsClopen (Z ∩ u)
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
rw [union_comm] at H
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
have H2 := isClopen_inter_of_disjoint_cover_clopen H.1 H.2.2 hv hu huv.symm
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
by_cases hxu : x ∈ u <;> [left; right]
-- The x ∈ u case.
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
by_cases hxu : x ∈ u
[GOAL]
case pos
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : x ∈ u
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
left
[GOAL]
case neg
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : ¬x ∈ u
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∨ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
right
[GOAL]
case pos.h
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : x ∈ u
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a
[PROOFSTEP]
suffices ⋂ Z : { Z : Set α // IsClopen Z ∧ x ∈ Z }, ↑Z ⊆ u from Disjoint.left_le_of_le_sup_right hab (huv.mono this hbv)
[GOAL]
case pos.h
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : x ∈ u
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ u
[PROOFSTEP]
apply Subset.trans _ (inter_subset_right Z u)
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : x ∈ u
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ Z ∩ u
[PROOFSTEP]
exact
iInter_subset (fun Z : { Z : Set α // IsClopen Z ∧ x ∈ Z } => Z.1)
⟨Z ∩ u, H1, mem_inter H.2.1 hxu⟩
-- If x ∉ u, we get x ∈ v since x ∈ u ∪ v. The rest is then like the x ∈ u case.
[GOAL]
case neg.h
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : ¬x ∈ u
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
have h1 : x ∈ v := (hab.trans (union_subset_union hau hbv) (mem_iInter.2 fun i => i.2.2)).resolve_left hxu
[GOAL]
case neg.h
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : ¬x ∈ u
h1 : x ∈ v
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ b
[PROOFSTEP]
suffices ⋂ Z : { Z : Set α // IsClopen Z ∧ x ∈ Z }, ↑Z ⊆ v from (huv.symm.mono this hau).left_le_of_le_sup_left hab
[GOAL]
case neg.h
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : ¬x ∈ u
h1 : x ∈ v
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ v
[PROOFSTEP]
refine Subset.trans ?_ (inter_subset_right Z v)
[GOAL]
case neg.h
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
x : α
hs : IsClosed (⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z)
a b : Set α
ha : IsClosed a
hb : IsClosed b
hab : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ a ∪ b
ab_disj : Disjoint a b
this : NormalSpace α
u v : Set α
hu : IsOpen u
hv : IsOpen v
hau : a ⊆ u
hbv : b ⊆ v
huv : Disjoint u v
Z : Set α
H : IsClopen Z ∧ x ∈ Z ∧ Z ⊆ v ∪ u
H1 : IsClopen (Z ∩ u)
H2 : IsClopen (Z ∩ v)
hxu : ¬x ∈ u
h1 : x ∈ v
⊢ ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z ⊆ Z ∩ v
[PROOFSTEP]
exact iInter_subset (fun Z : { Z : Set α // IsClopen Z ∧ x ∈ Z } => Z.1) ⟨Z ∩ v, H2, mem_inter H.2.1 h1⟩
[GOAL]
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
h : IsTopologicalBasis {s | IsClopen s}
⊢ TotallySeparatedSpace α
[PROOFSTEP]
constructor
[GOAL]
case isTotallySeparated_univ
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
h : IsTopologicalBasis {s | IsClopen s}
⊢ IsTotallySeparated univ
[PROOFSTEP]
rintro x - y - hxy
[GOAL]
case isTotallySeparated_univ
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
h : IsTopologicalBasis {s | IsClopen s}
x y : α
hxy : x ≠ y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ univ ⊆ u ∪ v ∧ Disjoint u v
[PROOFSTEP]
rcases h.mem_nhds_iff.mp (isOpen_ne.mem_nhds hxy) with ⟨U, hU, hxU, hyU⟩
[GOAL]
case isTotallySeparated_univ.intro.intro.intro
α : Type u
β : Type v
inst✝¹ : TopologicalSpace α
inst✝ : T1Space α
h : IsTopologicalBasis {s | IsClopen s}
x y : α
hxy : x ≠ y
U : Set α
hU : U ∈ {s | IsClopen s}
hxU : x ∈ U
hyU : U ⊆ {y_1 | y_1 ≠ y}
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ univ ⊆ u ∪ v ∧ Disjoint u v
[PROOFSTEP]
exact ⟨U, Uᶜ, hU.isOpen, hU.compl.isOpen, hxU, fun h => hyU h rfl, (union_compl_self U).superset, disjoint_compl_right⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
⊢ TotallyDisconnectedSpace α ↔ TotallySeparatedSpace α
[PROOFSTEP]
refine ⟨fun h => ⟨fun x _ y _ => ?_⟩, @TotallySeparatedSpace.totallyDisconnectedSpace _ _⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
⊢ x ≠ y → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ univ ⊆ u ∪ v ∧ Disjoint u v
[PROOFSTEP]
contrapose!
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
⊢ (∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v) → x = y
[PROOFSTEP]
intro hyp
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
hyp : ∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v
⊢ x = y
[PROOFSTEP]
suffices x ∈ connectedComponent y by
simpa [totallyDisconnectedSpace_iff_connectedComponent_singleton.1 h y, mem_singleton_iff]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
hyp : ∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v
this : x ∈ connectedComponent y
⊢ x = y
[PROOFSTEP]
simpa [totallyDisconnectedSpace_iff_connectedComponent_singleton.1 h y, mem_singleton_iff]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
hyp : ∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v
⊢ x ∈ connectedComponent y
[PROOFSTEP]
rw [connectedComponent_eq_iInter_clopen, mem_iInter]
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
hyp : ∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v
⊢ ∀ (i : { Z // IsClopen Z ∧ y ∈ Z }), x ∈ ↑i
[PROOFSTEP]
rintro ⟨w : Set α, hw : IsClopen w, hy : y ∈ w⟩
[GOAL]
case mk.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
hyp : ∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v
w : Set α
hw : IsClopen w
hy : y ∈ w
⊢ x ∈ ↑{ val := w, property := (_ : IsClopen w ∧ y ∈ w) }
[PROOFSTEP]
by_contra hx
[GOAL]
case mk.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
h : TotallyDisconnectedSpace α
x : α
x✝¹ : x ∈ univ
y : α
x✝ : y ∈ univ
hyp : ∀ (u v : Set α), IsOpen u → IsOpen v → x ∈ u → y ∈ v → univ ⊆ u ∪ v → ¬Disjoint u v
w : Set α
hw : IsClopen w
hy : y ∈ w
hx : ¬x ∈ ↑{ val := w, property := (_ : IsClopen w ∧ y ∈ w) }
⊢ False
[PROOFSTEP]
exact hyp wᶜ w hw.2.isOpen_compl hw.1 hx hy (@isCompl_compl _ w _).symm.codisjoint.top_le disjoint_compl_left
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
⊢ U ∈ 𝓝 x ↔ ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
⊢ U ∈ 𝓝 x → ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
have hx : connectedComponent x = { x } := totallyDisconnectedSpace_iff_connectedComponent_singleton.mp ‹_› x
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : connectedComponent x = {x}
⊢ U ∈ 𝓝 x → ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
rw [connectedComponent_eq_iInter_clopen] at hx
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
⊢ U ∈ 𝓝 x → ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
intro hU
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
⊢ ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
let N := { Z // IsClopen Z ∧ x ∈ Z }
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
⊢ ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
suffices : ∃ Z : N, Z.val ⊆ U
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : ∃ Z, ↑Z ⊆ U
⊢ ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
rcases this with ⟨⟨s, hs, hs'⟩, hs''⟩
[GOAL]
case mp.intro.mk.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
s : Set α
hs : IsClopen s
hs' : x ∈ s
hs'' : ↑{ val := s, property := (_ : IsClopen s ∧ x ∈ s) } ⊆ U
⊢ ∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U
[PROOFSTEP]
exact ⟨s, ⟨hs', hs⟩, hs''⟩
[GOAL]
case this
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
⊢ ∃ Z, ↑Z ⊆ U
[PROOFSTEP]
haveI : Nonempty N := ⟨⟨univ, isClopen_univ, mem_univ x⟩⟩
[GOAL]
case this
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
⊢ ∃ Z, ↑Z ⊆ U
[PROOFSTEP]
have hNcl : ∀ Z : N, IsClosed Z.val := fun Z => Z.property.1.2
[GOAL]
case this
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
⊢ ∃ Z, ↑Z ⊆ U
[PROOFSTEP]
have hdir : Directed Superset fun Z : N => Z.val :=
by
rintro ⟨s, hs, hxs⟩ ⟨t, ht, hxt⟩
exact ⟨⟨s ∩ t, hs.inter ht, ⟨hxs, hxt⟩⟩, inter_subset_left s t, inter_subset_right s t⟩
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
⊢ Directed Superset fun Z => ↑Z
[PROOFSTEP]
rintro ⟨s, hs, hxs⟩ ⟨t, ht, hxt⟩
[GOAL]
case mk.intro.mk.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
s : Set α
hs : IsClopen s
hxs : x ∈ s
t : Set α
ht : IsClopen t
hxt : x ∈ t
⊢ ∃ z,
(fun Z => ↑Z) { val := s, property := (_ : IsClopen s ∧ x ∈ s) } ⊇ (fun Z => ↑Z) z ∧
(fun Z => ↑Z) { val := t, property := (_ : IsClopen t ∧ x ∈ t) } ⊇ (fun Z => ↑Z) z
[PROOFSTEP]
exact ⟨⟨s ∩ t, hs.inter ht, ⟨hxs, hxt⟩⟩, inter_subset_left s t, inter_subset_right s t⟩
[GOAL]
case this
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
hdir : Directed Superset fun Z => ↑Z
⊢ ∃ Z, ↑Z ⊆ U
[PROOFSTEP]
have h_nhd : ∀ y ∈ ⋂ Z : N, Z.val, U ∈ 𝓝 y := fun y y_in =>
by
erw [hx, mem_singleton_iff] at y_in
rwa [y_in]
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
hdir : Directed Superset fun Z => ↑Z
y : α
y_in : y ∈ ⋂ (Z : N), ↑Z
⊢ U ∈ 𝓝 y
[PROOFSTEP]
erw [hx, mem_singleton_iff] at y_in
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
hdir : Directed Superset fun Z => ↑Z
y : α
y_in : y = x
⊢ U ∈ 𝓝 y
[PROOFSTEP]
rwa [y_in]
[GOAL]
case this
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hx : ⋂ (Z : { Z // IsClopen Z ∧ x ∈ Z }), ↑Z = {x}
hU : U ∈ 𝓝 x
N : Type u := { Z // IsClopen Z ∧ x ∈ Z }
this : Nonempty N
hNcl : ∀ (Z : N), IsClosed ↑Z
hdir : Directed Superset fun Z => ↑Z
h_nhd : ∀ (y : α), y ∈ ⋂ (Z : N), ↑Z → U ∈ 𝓝 y
⊢ ∃ Z, ↑Z ⊆ U
[PROOFSTEP]
exact exists_subset_nhds_of_compactSpace hdir hNcl h_nhd
[GOAL]
case mpr
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
⊢ (∃ i, (x ∈ i ∧ IsClopen i) ∧ id i ⊆ U) → U ∈ 𝓝 x
[PROOFSTEP]
rintro ⟨V, ⟨hxV, V_op, -⟩, hUV : V ⊆ U⟩
[GOAL]
case mpr.intro.intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U V : Set α
hUV : V ⊆ U
hxV : x ∈ V
V_op : IsOpen V
⊢ U ∈ 𝓝 x
[PROOFSTEP]
rw [mem_nhds_iff]
[GOAL]
case mpr.intro.intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U V : Set α
hUV : V ⊆ U
hxV : x ∈ V
V_op : IsOpen V
⊢ ∃ t, t ⊆ U ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
exact ⟨V, hUV, V_op, hxV⟩
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
⊢ IsTopologicalBasis {s | IsClopen s}
[PROOFSTEP]
apply isTopologicalBasis_of_open_of_nhds fun U (hU : IsClopen U) => hU.1
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
⊢ ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, (v ∈ fun U => IsOpen U ∧ IsClosed U) ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
intro x U hxU U_op
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hxU : x ∈ U
U_op : IsOpen U
⊢ ∃ v, (v ∈ fun U => IsOpen U ∧ IsClosed U) ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
have : U ∈ 𝓝 x := IsOpen.mem_nhds U_op hxU
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hxU : x ∈ U
U_op : IsOpen U
this : U ∈ 𝓝 x
⊢ ∃ v, (v ∈ fun U => IsOpen U ∧ IsClosed U) ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
rcases(nhds_basis_clopen x).mem_iff.mp this with ⟨V, ⟨hxV, hV⟩, hVU : V ⊆ U⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hxU : x ∈ U
U_op : IsOpen U
this : U ∈ 𝓝 x
V : Set α
hVU : V ⊆ U
hxV : x ∈ V
hV : IsClopen V
⊢ ∃ v, (v ∈ fun U => IsOpen U ∧ IsClosed U) ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
use V
[GOAL]
case h
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
inst✝² : T2Space α
inst✝¹ : CompactSpace α
inst✝ : TotallyDisconnectedSpace α
x : α
U : Set α
hxU : x ∈ U
U_op : IsOpen U
this : U ∈ 𝓝 x
V : Set α
hVU : V ⊆ U
hxV : x ∈ V
hV : IsClopen V
⊢ (V ∈ fun U => IsOpen U ∧ IsClosed U) ∧ x ∈ V ∧ V ⊆ U
[PROOFSTEP]
tauto
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
⊢ IsTopologicalBasis {s | IsClopen s}
[PROOFSTEP]
refine isTopologicalBasis_of_open_of_nhds (fun u hu => hu.1) fun x U memU hU => ?_
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
x : H
U : Set H
memU : x ∈ U
hU : IsOpen U
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
obtain ⟨s, comp, xs, sU⟩ := exists_compact_subset hU memU
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
x : H
U : Set H
memU : x ∈ U
hU : IsOpen U
s : Set H
comp : IsCompact s
xs : x ∈ interior s
sU : s ⊆ U
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
let u : Set s := ((↑) : s → H) ⁻¹' interior s
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
x : H
U : Set H
memU : x ∈ U
hU : IsOpen U
s : Set H
comp : IsCompact s
xs : x ∈ interior s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
have u_open_in_s : IsOpen u := isOpen_interior.preimage continuous_subtype_val
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
x : H
U : Set H
memU : x ∈ U
hU : IsOpen U
s : Set H
comp : IsCompact s
xs : x ∈ interior s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ x ∈ v ∧ v ⊆ U
[PROOFSTEP]
lift x to s using interior_subset xs
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ ↑x ∈ v ∧ v ⊆ U
[PROOFSTEP]
haveI : CompactSpace s := isCompact_iff_compactSpace.1 comp
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ ↑x ∈ v ∧ v ⊆ U
[PROOFSTEP]
obtain ⟨V : Set s, clopen_in_s, Vx, V_sub⟩ := compact_exists_clopen_in_open u_open_in_s xs
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ ↑x ∈ v ∧ v ⊆ U
[PROOFSTEP]
have V_clopen : IsClopen (((↑) : s → H) '' V) :=
by
refine' ⟨_, comp.isClosed.closedEmbedding_subtype_val.closed_iff_image_closed.1 clopen_in_s.2⟩
let v : Set u := ((↑) : u → s) ⁻¹' V
have : ((↑) : u → H) = ((↑) : s → H) ∘ ((↑) : u → s) := rfl
have f0 : Embedding ((↑) : u → H) := embedding_subtype_val.comp embedding_subtype_val
have f1 : OpenEmbedding ((↑) : u → H) := by
refine' ⟨f0, _⟩
· have : Set.range ((↑) : u → H) = interior s :=
by
rw [this, Set.range_comp, Subtype.range_coe, Subtype.image_preimage_coe]
apply Set.inter_eq_self_of_subset_left interior_subset
rw [this]
apply isOpen_interior
have f2 : IsOpen v := clopen_in_s.1.preimage continuous_subtype_val
have f3 : ((↑) : s → H) '' V = ((↑) : u → H) '' v := by
rw [this, image_comp, Subtype.image_preimage_coe, inter_eq_self_of_subset_left V_sub]
rw [f3]
apply f1.isOpenMap v f2
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
⊢ IsClopen (Subtype.val '' V)
[PROOFSTEP]
refine' ⟨_, comp.isClosed.closedEmbedding_subtype_val.closed_iff_image_closed.1 clopen_in_s.2⟩
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
let v : Set u := ((↑) : u → s) ⁻¹' V
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
have : ((↑) : u → H) = ((↑) : s → H) ∘ ((↑) : u → s) := rfl
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
have f0 : Embedding ((↑) : u → H) := embedding_subtype_val.comp embedding_subtype_val
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
have f1 : OpenEmbedding ((↑) : u → H) := by
refine' ⟨f0, _⟩
· have : Set.range ((↑) : u → H) = interior s :=
by
rw [this, Set.range_comp, Subtype.range_coe, Subtype.image_preimage_coe]
apply Set.inter_eq_self_of_subset_left interior_subset
rw [this]
apply isOpen_interior
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
⊢ OpenEmbedding fun x => ↑↑x
[PROOFSTEP]
refine' ⟨f0, _⟩
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
⊢ IsOpen (range fun x => ↑↑x)
[PROOFSTEP]
have : Set.range ((↑) : u → H) = interior s :=
by
rw [this, Set.range_comp, Subtype.range_coe, Subtype.image_preimage_coe]
apply Set.inter_eq_self_of_subset_left interior_subset
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
⊢ (range fun x => ↑↑x) = interior s
[PROOFSTEP]
rw [this, Set.range_comp, Subtype.range_coe, Subtype.image_preimage_coe]
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
⊢ interior s ∩ s = interior s
[PROOFSTEP]
apply Set.inter_eq_self_of_subset_left interior_subset
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝¹ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this✝ : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
this : (range fun x => ↑↑x) = interior s
⊢ IsOpen (range fun x => ↑↑x)
[PROOFSTEP]
rw [this]
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝¹ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this✝ : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
this : (range fun x => ↑↑x) = interior s
⊢ IsOpen (interior s)
[PROOFSTEP]
apply isOpen_interior
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
f1 : OpenEmbedding fun x => ↑↑x
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
have f2 : IsOpen v := clopen_in_s.1.preimage continuous_subtype_val
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
f1 : OpenEmbedding fun x => ↑↑x
f2 : IsOpen v
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
have f3 : ((↑) : s → H) '' V = ((↑) : u → H) '' v := by
rw [this, image_comp, Subtype.image_preimage_coe, inter_eq_self_of_subset_left V_sub]
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
f1 : OpenEmbedding fun x => ↑↑x
f2 : IsOpen v
⊢ Subtype.val '' V = (fun x => ↑↑x) '' v
[PROOFSTEP]
rw [this, image_comp, Subtype.image_preimage_coe, inter_eq_self_of_subset_left V_sub]
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
f1 : OpenEmbedding fun x => ↑↑x
f2 : IsOpen v
f3 : Subtype.val '' V = (fun x => ↑↑x) '' v
⊢ IsOpen (Subtype.val '' V)
[PROOFSTEP]
rw [f3]
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this✝ : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
v : Set ↑u := Subtype.val ⁻¹' V
this : (fun x => ↑↑x) = Subtype.val ∘ Subtype.val
f0 : _root_.Embedding fun x => ↑↑x
f1 : OpenEmbedding fun x => ↑↑x
f2 : IsOpen v
f3 : Subtype.val '' V = (fun x => ↑↑x) '' v
⊢ IsOpen ((fun x => ↑↑x) '' v)
[PROOFSTEP]
apply f1.isOpenMap v f2
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
V_clopen : IsClopen (Subtype.val '' V)
⊢ ∃ v, v ∈ {s | IsClopen s} ∧ ↑x ∈ v ∧ v ⊆ U
[PROOFSTEP]
refine' ⟨(↑) '' V, V_clopen, by simp [Vx], Subset.trans _ sU⟩
[GOAL]
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
V_clopen : IsClopen (Subtype.val '' V)
⊢ ↑x ∈ Subtype.val '' V
[PROOFSTEP]
simp [Vx]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝⁴ : TopologicalSpace α
H : Type u_1
inst✝³ : TopologicalSpace H
inst✝² : LocallyCompactSpace H
inst✝¹ : T2Space H
inst✝ : TotallyDisconnectedSpace H
U : Set H
hU : IsOpen U
s : Set H
comp : IsCompact s
sU : s ⊆ U
u : Set ↑s := Subtype.val ⁻¹' interior s
u_open_in_s : IsOpen u
x : { x // x ∈ s }
memU : ↑x ∈ U
xs : ↑x ∈ interior s
this : CompactSpace ↑s
V : Set ↑s
clopen_in_s : IsClopen V
Vx : x ∈ V
V_sub : V ⊆ u
V_clopen : IsClopen (Subtype.val '' V)
⊢ Subtype.val '' V ⊆ s
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
H : Type u_1
inst✝² : TopologicalSpace H
inst✝¹ : LocallyCompactSpace H
inst✝ : T2Space H
⊢ TotallyDisconnectedSpace H ↔ TotallySeparatedSpace H
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
H : Type u_1
inst✝² : TopologicalSpace H
inst✝¹ : LocallyCompactSpace H
inst✝ : T2Space H
⊢ TotallyDisconnectedSpace H → TotallySeparatedSpace H
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
H : Type u_1
inst✝² : TopologicalSpace H
inst✝¹ : LocallyCompactSpace H
inst✝ : T2Space H
h : TotallyDisconnectedSpace H
⊢ TotallySeparatedSpace H
[PROOFSTEP]
exact totallySeparatedSpace_of_t1_of_basis_clopen loc_compact_Haus_tot_disc_of_zero_dim
[GOAL]
case mpr
α : Type u
β : Type v
inst✝³ : TopologicalSpace α
H : Type u_1
inst✝² : TopologicalSpace H
inst✝¹ : LocallyCompactSpace H
inst✝ : T2Space H
⊢ TotallySeparatedSpace H → TotallyDisconnectedSpace H
[PROOFSTEP]
apply TotallySeparatedSpace.totallyDisconnectedSpace
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
⊢ T2Space (ConnectedComponents α)
[PROOFSTEP]
refine ⟨ConnectedComponents.surjective_coe.forall₂.2 fun a b ne => ?_⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : mk a ≠ mk b
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ mk a ∈ u ∧ mk b ∈ v ∧ Disjoint u v
[PROOFSTEP]
rw [ConnectedComponents.coe_ne_coe] at ne
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ mk a ∈ u ∧ mk b ∈ v ∧ Disjoint u v
[PROOFSTEP]
have h := connectedComponent_disjoint ne
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : Disjoint (connectedComponent a) (connectedComponent b)
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ mk a ∈ u ∧ mk b ∈ v ∧ Disjoint u v
[PROOFSTEP]
rw [connectedComponent_eq_iInter_clopen b, disjoint_iff_inter_eq_empty] at h
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ mk a ∈ u ∧ mk b ∈ v ∧ Disjoint u v
[PROOFSTEP]
obtain ⟨U, V, hU, ha, hb, rfl⟩ :
∃ (U : Set α) (V : Set (ConnectedComponents α)),
IsClopen U ∧ connectedComponent a ∩ U = ∅ ∧ connectedComponent b ⊆ U ∧ (↑) ⁻¹' V = U :=
by
have h :=
(isClosed_connectedComponent (α := α)).isCompact.elim_finite_subfamily_closed _
(fun Z : { Z : Set α // IsClopen Z ∧ b ∈ Z } => Z.2.1.2) h
cases' h with fin_a ha
set U : Set α := ⋂ (i : { Z // IsClopen Z ∧ b ∈ Z }) (_ : i ∈ fin_a), i
have hU : IsClopen U := isClopen_biInter_finset fun i _ => i.2.1
exact
⟨U, (↑) '' U, hU, ha, subset_iInter₂ fun Z _ => Z.2.1.connectedComponent_subset Z.2.2,
(connectedComponents_preimage_image U).symm ▸ hU.biUnion_connectedComponent_eq⟩
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
⊢ ∃ U V, IsClopen U ∧ connectedComponent a ∩ U = ∅ ∧ connectedComponent b ⊆ U ∧ mk ⁻¹' V = U
[PROOFSTEP]
have h :=
(isClosed_connectedComponent (α := α)).isCompact.elim_finite_subfamily_closed _
(fun Z : { Z : Set α // IsClopen Z ∧ b ∈ Z } => Z.2.1.2) h
[GOAL]
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h✝ : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
h : ∃ t, connectedComponent a ∩ ⋂ (i : { Z // IsClopen Z ∧ b ∈ Z }) (_ : i ∈ t), ↑i = ∅
⊢ ∃ U V, IsClopen U ∧ connectedComponent a ∩ U = ∅ ∧ connectedComponent b ⊆ U ∧ mk ⁻¹' V = U
[PROOFSTEP]
cases' h with fin_a ha
[GOAL]
case intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
fin_a : Finset { Z // IsClopen Z ∧ b ∈ Z }
ha : connectedComponent a ∩ ⋂ (i : { Z // IsClopen Z ∧ b ∈ Z }) (_ : i ∈ fin_a), ↑i = ∅
⊢ ∃ U V, IsClopen U ∧ connectedComponent a ∩ U = ∅ ∧ connectedComponent b ⊆ U ∧ mk ⁻¹' V = U
[PROOFSTEP]
set U : Set α := ⋂ (i : { Z // IsClopen Z ∧ b ∈ Z }) (_ : i ∈ fin_a), i
[GOAL]
case intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
fin_a : Finset { Z // IsClopen Z ∧ b ∈ Z }
U : Set α := ⋂ (i : { Z // IsClopen Z ∧ b ∈ Z }) (_ : i ∈ fin_a), ↑i
ha : connectedComponent a ∩ U = ∅
⊢ ∃ U V, IsClopen U ∧ connectedComponent a ∩ U = ∅ ∧ connectedComponent b ⊆ U ∧ mk ⁻¹' V = U
[PROOFSTEP]
have hU : IsClopen U := isClopen_biInter_finset fun i _ => i.2.1
[GOAL]
case intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
fin_a : Finset { Z // IsClopen Z ∧ b ∈ Z }
U : Set α := ⋂ (i : { Z // IsClopen Z ∧ b ∈ Z }) (_ : i ∈ fin_a), ↑i
ha : connectedComponent a ∩ U = ∅
hU : IsClopen U
⊢ ∃ U V, IsClopen U ∧ connectedComponent a ∩ U = ∅ ∧ connectedComponent b ⊆ U ∧ mk ⁻¹' V = U
[PROOFSTEP]
exact
⟨U, (↑) '' U, hU, ha, subset_iInter₂ fun Z _ => Z.2.1.connectedComponent_subset Z.2.2,
(connectedComponents_preimage_image U).symm ▸ hU.biUnion_connectedComponent_eq⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
V : Set (ConnectedComponents α)
hU : IsClopen (mk ⁻¹' V)
ha : connectedComponent a ∩ mk ⁻¹' V = ∅
hb : connectedComponent b ⊆ mk ⁻¹' V
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ mk a ∈ u ∧ mk b ∈ v ∧ Disjoint u v
[PROOFSTEP]
rw [ConnectedComponents.quotientMap_coe.isClopen_preimage] at hU
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
V : Set (ConnectedComponents α)
hU : IsClopen V
ha : connectedComponent a ∩ mk ⁻¹' V = ∅
hb : connectedComponent b ⊆ mk ⁻¹' V
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ mk a ∈ u ∧ mk b ∈ v ∧ Disjoint u v
[PROOFSTEP]
refine' ⟨Vᶜ, V, hU.compl.isOpen, hU.isOpen, _, hb mem_connectedComponent, disjoint_compl_left⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
inst✝² : TopologicalSpace α
inst✝¹ : T2Space α
inst✝ : CompactSpace α
a b : α
ne : connectedComponent a ≠ connectedComponent b
h : connectedComponent a ∩ ⋂ (Z : { Z // IsClopen Z ∧ b ∈ Z }), ↑Z = ∅
V : Set (ConnectedComponents α)
hU : IsClopen V
ha : connectedComponent a ∩ mk ⁻¹' V = ∅
hb : connectedComponent b ⊆ mk ⁻¹' V
⊢ mk a ∈ Vᶜ
[PROOFSTEP]
exact fun h => flip Set.Nonempty.ne_empty ha ⟨a, mem_connectedComponent, h⟩
| {"mathlib_filename": "Mathlib.Topology.Separation", "llama_tokens": 115187} |
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
h : Inducing f
⊢ Inducing (restrictPreimage s f)
[PROOFSTEP]
simp_rw [inducing_subtype_val.inducing_iff, inducing_iff_nhds, restrictPreimage, MapsTo.coe_restrict, restrict_eq, ←
@Filter.comap_comap _ _ _ _ _ f, Function.comp_apply] at h ⊢
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
h : ∀ (a : α), 𝓝 a = comap f (𝓝 (f a))
⊢ ∀ (a : ↑(f ⁻¹' s)), 𝓝 a = comap Subtype.val (comap f (𝓝 (f ↑a)))
[PROOFSTEP]
intro a
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
h : ∀ (a : α), 𝓝 a = comap f (𝓝 (f a))
a : ↑(f ⁻¹' s)
⊢ 𝓝 a = comap Subtype.val (comap f (𝓝 (f ↑a)))
[PROOFSTEP]
rw [← h, ← inducing_subtype_val.nhds_eq_comap]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
⊢ IsClosedMap (restrictPreimage s f)
[PROOFSTEP]
rintro t ⟨u, hu, e⟩
[GOAL]
case mk.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
⊢ IsClosed (restrictPreimage s f '' t)
[PROOFSTEP]
refine' ⟨⟨_, (H _ (IsOpen.isClosed_compl hu)).1, _⟩⟩
[GOAL]
case mk.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
⊢ Subtype.val ⁻¹' (f '' uᶜ)ᶜ = (restrictPreimage s f '' t)ᶜ
[PROOFSTEP]
rw [← (congr_arg HasCompl.compl e).trans (compl_compl t)]
[GOAL]
case mk.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
⊢ Subtype.val ⁻¹' (f '' uᶜ)ᶜ = (restrictPreimage s f '' (Subtype.val ⁻¹' u)ᶜ)ᶜ
[PROOFSTEP]
simp only [Set.preimage_compl, compl_inj_iff]
[GOAL]
case mk.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
⊢ Subtype.val ⁻¹' (f '' uᶜ) = restrictPreimage s f '' (Subtype.val ⁻¹' u)ᶜ
[PROOFSTEP]
ext ⟨x, hx⟩
[GOAL]
case mk.intro.intro.h.mk
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
x : β
hx : x ∈ s
⊢ { val := x, property := hx } ∈ Subtype.val ⁻¹' (f '' uᶜ) ↔
{ val := x, property := hx } ∈ restrictPreimage s f '' (Subtype.val ⁻¹' u)ᶜ
[PROOFSTEP]
suffices (∃ y, y ∉ u ∧ f y = x) ↔ ∃ y, y ∉ u ∧ f y ∈ s ∧ f y = x by simpa [Set.restrictPreimage, ← Subtype.coe_inj]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
x : β
hx : x ∈ s
this : (∃ y, ¬y ∈ u ∧ f y = x) ↔ ∃ y, ¬y ∈ u ∧ f y ∈ s ∧ f y = x
⊢ { val := x, property := hx } ∈ Subtype.val ⁻¹' (f '' uᶜ) ↔
{ val := x, property := hx } ∈ restrictPreimage s f '' (Subtype.val ⁻¹' u)ᶜ
[PROOFSTEP]
simpa [Set.restrictPreimage, ← Subtype.coe_inj]
[GOAL]
case mk.intro.intro.h.mk
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : IsClosedMap f
t : Set ↑(f ⁻¹' s)
u : Set α
hu : IsOpen u
e : Subtype.val ⁻¹' u = tᶜ
x : β
hx : x ∈ s
⊢ (∃ y, ¬y ∈ u ∧ f y = x) ↔ ∃ y, ¬y ∈ u ∧ f y ∈ s ∧ f y = x
[PROOFSTEP]
exact ⟨fun ⟨a, b, c⟩ => ⟨a, b, c.symm ▸ hx, c⟩, fun ⟨a, b, _, c⟩ => ⟨a, b, c⟩⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
⊢ IsOpen s ↔ ∀ (i : ι), IsOpen (s ∩ ↑(U i))
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
⊢ IsOpen s → ∀ (i : ι), IsOpen (s ∩ ↑(U i))
[PROOFSTEP]
exact fun H i => H.inter (U i).2
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
⊢ (∀ (i : ι), IsOpen (s ∩ ↑(U i))) → IsOpen s
[PROOFSTEP]
intro H
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : ∀ (i : ι), IsOpen (s ∩ ↑(U i))
⊢ IsOpen s
[PROOFSTEP]
have : ⋃ i, (U i : Set β) = Set.univ := by
convert congr_arg (SetLike.coe) hU
simp
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : ∀ (i : ι), IsOpen (s ∩ ↑(U i))
⊢ ⋃ (i : ι), ↑(U i) = univ
[PROOFSTEP]
convert congr_arg (SetLike.coe) hU
[GOAL]
case h.e'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : ∀ (i : ι), IsOpen (s ∩ ↑(U i))
⊢ ⋃ (i : ι), ↑(U i) = ↑(iSup U)
[PROOFSTEP]
simp
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : ∀ (i : ι), IsOpen (s ∩ ↑(U i))
this : ⋃ (i : ι), ↑(U i) = univ
⊢ IsOpen s
[PROOFSTEP]
rw [← s.inter_univ, ← this, Set.inter_iUnion]
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
H : ∀ (i : ι), IsOpen (s ∩ ↑(U i))
this : ⋃ (i : ι), ↑(U i) = univ
⊢ IsOpen (⋃ (i : ι), s ∩ ↑(U i))
[PROOFSTEP]
exact isOpen_iUnion H
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
⊢ IsOpen s ↔ ∀ (i : ι), IsOpen (Subtype.val ⁻¹' s)
[PROOFSTEP]
rw [isOpen_iff_inter_of_iSup_eq_top hU s]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
⊢ (∀ (i : ι), IsOpen (s ∩ ↑(U i))) ↔ ∀ (i : ι), IsOpen (Subtype.val ⁻¹' s)
[PROOFSTEP]
refine forall_congr' fun i => ?_
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
i : ι
⊢ IsOpen (s ∩ ↑(U i)) ↔ IsOpen (Subtype.val ⁻¹' s)
[PROOFSTEP]
rw [(U _).2.openEmbedding_subtype_val.open_iff_image_open]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
i : ι
⊢ IsOpen (s ∩ ↑(U i)) ↔ IsOpen (Subtype.val '' (Subtype.val ⁻¹' s))
[PROOFSTEP]
erw [Set.image_preimage_eq_inter_range]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
i : ι
⊢ IsOpen (s ∩ ↑(U i)) ↔ IsOpen (s ∩ range Subtype.val)
[PROOFSTEP]
rw [Subtype.range_coe, Opens.carrier_eq_coe]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
s : Set β
⊢ IsClosed s ↔ ∀ (i : ι), IsClosed (Subtype.val ⁻¹' s)
[PROOFSTEP]
simpa using isOpen_iff_coe_preimage_of_iSup_eq_top hU sᶜ
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
⊢ IsClosedMap f ↔ ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
[PROOFSTEP]
refine' ⟨fun h i => Set.restrictPreimage_isClosedMap _ h, _⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
⊢ (∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)) → IsClosedMap f
[PROOFSTEP]
rintro H s hs
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
⊢ IsClosed (f '' s)
[PROOFSTEP]
rw [isClosed_iff_coe_preimage_of_iSup_eq_top hU]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
⊢ ∀ (i : ι), IsClosed (Subtype.val ⁻¹' (f '' s))
[PROOFSTEP]
intro i
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
i : ι
⊢ IsClosed (Subtype.val ⁻¹' (f '' s))
[PROOFSTEP]
convert H i _ ⟨⟨_, hs.1, eq_compl_comm.mpr rfl⟩⟩
[GOAL]
case h.e'_3.h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
i : ι
e_1✝ : { x // x ∈ U i } = ↑(U i).carrier
⊢ Subtype.val ⁻¹' (f '' s) = restrictPreimage (U i).carrier f '' (Subtype.val ⁻¹' sᶜ)ᶜ
[PROOFSTEP]
ext ⟨x, hx⟩
[GOAL]
case h.e'_3.h.h.mk
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
i : ι
e_1✝ : { x // x ∈ U i } = ↑(U i).carrier
x : β
hx : x ∈ U i
⊢ { val := x, property := hx } ∈ Subtype.val ⁻¹' (f '' s) ↔
{ val := x, property := hx } ∈ restrictPreimage (U i).carrier f '' (Subtype.val ⁻¹' sᶜ)ᶜ
[PROOFSTEP]
suffices (∃ y, y ∈ s ∧ f y = x) ↔ ∃ y, y ∈ s ∧ f y ∈ U i ∧ f y = x by simpa [Set.restrictPreimage, ← Subtype.coe_inj]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
i : ι
e_1✝ : { x // x ∈ U i } = ↑(U i).carrier
x : β
hx : x ∈ U i
this : (∃ y, y ∈ s ∧ f y = x) ↔ ∃ y, y ∈ s ∧ f y ∈ U i ∧ f y = x
⊢ { val := x, property := hx } ∈ Subtype.val ⁻¹' (f '' s) ↔
{ val := x, property := hx } ∈ restrictPreimage (U i).carrier f '' (Subtype.val ⁻¹' sᶜ)ᶜ
[PROOFSTEP]
simpa [Set.restrictPreimage, ← Subtype.coe_inj]
[GOAL]
case h.e'_3.h.h.mk
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s✝ : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
H : ∀ (i : ι), IsClosedMap (restrictPreimage (U i).carrier f)
s : Set α
hs : IsClosed s
i : ι
e_1✝ : { x // x ∈ U i } = ↑(U i).carrier
x : β
hx : x ∈ U i
⊢ (∃ y, y ∈ s ∧ f y = x) ↔ ∃ y, y ∈ s ∧ f y ∈ U i ∧ f y = x
[PROOFSTEP]
exact ⟨fun ⟨a, b, c⟩ => ⟨a, b, c.symm ▸ hx, c⟩, fun ⟨a, b, _, c⟩ => ⟨a, b, c⟩⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Inducing f ↔ ∀ (i : ι), Inducing (restrictPreimage (U i).carrier f)
[PROOFSTEP]
simp_rw [inducing_subtype_val.inducing_iff, inducing_iff_nhds, restrictPreimage, MapsTo.coe_restrict, restrict_eq, ←
@Filter.comap_comap _ _ _ _ _ f]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ (∀ (a : α), 𝓝 a = comap f (𝓝 (f a))) ↔
∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ (∀ (a : α), 𝓝 a = comap f (𝓝 (f a))) →
∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
[PROOFSTEP]
intro H i x
[GOAL]
case mp
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (a : α), 𝓝 a = comap f (𝓝 (f a))
i : ι
x : ↑(f ⁻¹' (U i).carrier)
⊢ 𝓝 x = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) x)))
[PROOFSTEP]
rw [Function.comp_apply, ← H, ← inducing_subtype_val.nhds_eq_comap]
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ (∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))) →
∀ (a : α), 𝓝 a = comap f (𝓝 (f a))
[PROOFSTEP]
intro H x
[GOAL]
case mpr
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
x : α
⊢ 𝓝 x = comap f (𝓝 (f x))
[PROOFSTEP]
obtain ⟨i, hi⟩ :=
Opens.mem_iSup.mp
(show f x ∈ iSup U by
rw [hU]
triv)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
x : α
⊢ f x ∈ iSup U
[PROOFSTEP]
rw [hU]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
x : α
⊢ f x ∈ ⊤
[PROOFSTEP]
triv
[GOAL]
case mpr.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
x : α
i : ι
hi : f x ∈ U i
⊢ 𝓝 x = comap f (𝓝 (f x))
[PROOFSTEP]
erw [← OpenEmbedding.map_nhds_eq (h.1 _ (U i).2).openEmbedding_subtype_val ⟨x, hi⟩]
[GOAL]
case mpr.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
x : α
i : ι
hi : f x ∈ U i
⊢ map Subtype.val (𝓝 { val := x, property := hi }) = comap f (𝓝 (f x))
[PROOFSTEP]
rw [(H i) ⟨x, hi⟩, Filter.subtype_coe_map_comap, Function.comp_apply, Subtype.coe_mk, inf_eq_left,
Filter.le_principal_iff]
[GOAL]
case mpr.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
H : ∀ (i : ι) (a : ↑(f ⁻¹' (U i).carrier)), 𝓝 a = comap Subtype.val (comap f (𝓝 ((f ∘ Subtype.val) a)))
x : α
i : ι
hi : f x ∈ U i
⊢ f ⁻¹' (U i).carrier ∈ comap f (𝓝 (f x))
[PROOFSTEP]
exact Filter.preimage_mem_comap ((U i).2.mem_nhds hi)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ↔ ∀ (i : ι), Embedding (restrictPreimage (U i).carrier f)
[PROOFSTEP]
simp_rw [embedding_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Inducing f ∧ Function.Injective f ↔
∀ (i : ι), Inducing (restrictPreimage (U i).carrier f) ∧ Function.Injective (restrictPreimage (U i).carrier f)
[PROOFSTEP]
rw [forall_and]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Inducing f ∧ Function.Injective f ↔
(∀ (x : ι), Inducing (restrictPreimage (U x).carrier f)) ∧
∀ (x : ι), Function.Injective (restrictPreimage (U x).carrier f)
[PROOFSTEP]
apply and_congr
[GOAL]
case h₁
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Inducing f ↔ ∀ (x : ι), Inducing (restrictPreimage (U x).carrier f)
[PROOFSTEP]
apply inducing_iff_inducing_of_iSup_eq_top
[GOAL]
case h₁.hU
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ ⨆ (i : ι), U i = ⊤
[PROOFSTEP]
assumption
[GOAL]
case h₁.h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Continuous f
[PROOFSTEP]
assumption
[GOAL]
case h₂
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Function.Injective f ↔ ∀ (x : ι), Function.Injective (restrictPreimage (U x).carrier f)
[PROOFSTEP]
apply Set.injective_iff_injective_of_iUnion_eq_univ
[GOAL]
case h₂.hU
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ ⋃ (i : ι), (U i).carrier = univ
[PROOFSTEP]
convert congr_arg SetLike.coe hU
[GOAL]
case h.e'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ ⋃ (i : ι), (U i).carrier = ↑(iSup U)
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ OpenEmbedding f ↔ ∀ (i : ι), OpenEmbedding (restrictPreimage (U i).carrier f)
[PROOFSTEP]
simp_rw [openEmbedding_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ∧ IsOpen (range f) ↔
∀ (i : ι), Embedding (restrictPreimage (U i).carrier f) ∧ IsOpen (range (restrictPreimage (U i).carrier f))
[PROOFSTEP]
rw [forall_and]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ∧ IsOpen (range f) ↔
(∀ (x : ι), Embedding (restrictPreimage (U x).carrier f)) ∧
∀ (x : ι), IsOpen (range (restrictPreimage (U x).carrier f))
[PROOFSTEP]
apply and_congr
[GOAL]
case h₁
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ↔ ∀ (x : ι), Embedding (restrictPreimage (U x).carrier f)
[PROOFSTEP]
apply embedding_iff_embedding_of_iSup_eq_top
[GOAL]
case h₁.hU
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ ⨆ (i : ι), U i = ⊤
[PROOFSTEP]
assumption
[GOAL]
case h₁.h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Continuous f
[PROOFSTEP]
assumption
[GOAL]
case h₂
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ IsOpen (range f) ↔ ∀ (x : ι), IsOpen (range (restrictPreimage (U x).carrier f))
[PROOFSTEP]
simp_rw [Set.range_restrictPreimage]
[GOAL]
case h₂
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ IsOpen (range f) ↔ ∀ (x : ι), IsOpen (Subtype.val ⁻¹' range f)
[PROOFSTEP]
apply isOpen_iff_coe_preimage_of_iSup_eq_top hU
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ ClosedEmbedding f ↔ ∀ (i : ι), ClosedEmbedding (restrictPreimage (U i).carrier f)
[PROOFSTEP]
simp_rw [closedEmbedding_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ∧ IsClosed (range f) ↔
∀ (i : ι), Embedding (restrictPreimage (U i).carrier f) ∧ IsClosed (range (restrictPreimage (U i).carrier f))
[PROOFSTEP]
rw [forall_and]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ∧ IsClosed (range f) ↔
(∀ (x : ι), Embedding (restrictPreimage (U x).carrier f)) ∧
∀ (x : ι), IsClosed (range (restrictPreimage (U x).carrier f))
[PROOFSTEP]
apply and_congr
[GOAL]
case h₁
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Embedding f ↔ ∀ (x : ι), Embedding (restrictPreimage (U x).carrier f)
[PROOFSTEP]
apply embedding_iff_embedding_of_iSup_eq_top
[GOAL]
case h₁.hU
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ ⨆ (i : ι), U i = ⊤
[PROOFSTEP]
assumption
[GOAL]
case h₁.h
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ Continuous f
[PROOFSTEP]
assumption
[GOAL]
case h₂
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ IsClosed (range f) ↔ ∀ (x : ι), IsClosed (range (restrictPreimage (U x).carrier f))
[PROOFSTEP]
simp_rw [Set.range_restrictPreimage]
[GOAL]
case h₂
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
s : Set β
ι : Type u_3
U : ι → Opens β
hU : iSup U = ⊤
h : Continuous f
⊢ IsClosed (range f) ↔ ∀ (x : ι), IsClosed (Subtype.val ⁻¹' range f)
[PROOFSTEP]
apply isClosed_iff_coe_preimage_of_iSup_eq_top hU
| {"mathlib_filename": "Mathlib.Topology.LocalAtTarget", "llama_tokens": 12327} |
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
hg : Inducing g
hf : Inducing f
⊢ inst✝³ = TopologicalSpace.induced (g ∘ f) inst✝¹
[PROOFSTEP]
rw [hf.induced, hg.induced, induced_compose]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hf : Continuous f
hg : Continuous g
hgf : Inducing (g ∘ f)
⊢ inst✝³ ≤ induced f inst✝²
[PROOFSTEP]
rwa [← continuous_iff_le_induced]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hf : Continuous f
hg : Continuous g
hgf : Inducing (g ∘ f)
⊢ induced f inst✝² ≤ inst✝³
[PROOFSTEP]
rw [hgf.induced, ← induced_compose]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hf : Continuous f
hg : Continuous g
hgf : Inducing (g ∘ f)
⊢ induced f inst✝² ≤ induced f (induced g inst✝¹)
[PROOFSTEP]
exact induced_mono hg.le_induced
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
⊢ 𝓝ˢ s = comap f (𝓝ˢ (f '' s))
[PROOFSTEP]
simp only [nhdsSet, sSup_image, comap_iSup, hf.nhds_eq_comap, iSup_image]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
a : α
l : Filter α
⊢ MapClusterPt (f a) l f ↔ ClusterPt a l
[PROOFSTEP]
delta MapClusterPt ClusterPt
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
a : α
l : Filter α
⊢ NeBot (𝓝 (f a) ⊓ map f l) ↔ NeBot (𝓝 a ⊓ l)
[PROOFSTEP]
rw [← Filter.push_pull', ← hf.nhds_eq_comap, map_neBot_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
ι : Type u_5
f : ι → β
g : β → γ
a : Filter ι
b : β
hg : Inducing g
⊢ Tendsto f a (𝓝 b) ↔ Tendsto (g ∘ f) a (𝓝 (g b))
[PROOFSTEP]
rw [hg.nhds_eq_comap, tendsto_comap_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
⊢ Continuous f ↔ Continuous (g ∘ f)
[PROOFSTEP]
simp_rw [continuous_iff_continuousAt, hg.continuousAt_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hf : Inducing f
x : α
h : range f ∈ 𝓝 (f x)
⊢ ContinuousAt (g ∘ f) x ↔ ContinuousAt g (f x)
[PROOFSTEP]
simp_rw [ContinuousAt, Filter.Tendsto, ← hf.map_nhds_of_mem _ h, Filter.map_map, comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
⊢ Inducing f ↔ Inducing (g ∘ f)
[PROOFSTEP]
refine' ⟨fun h => hg.comp h, fun hgf => inducing_of_inducing_compose _ hg.continuous hgf⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
hgf : Inducing (g ∘ f)
⊢ Continuous f
[PROOFSTEP]
rw [hg.continuous_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
g : β → γ
hg : Inducing g
hgf : Inducing (g ∘ f)
⊢ Continuous (g ∘ f)
[PROOFSTEP]
exact hgf.continuous
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
⊢ closure s = f ⁻¹' closure (f '' s)
[PROOFSTEP]
ext x
[GOAL]
case h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
x : α
⊢ x ∈ closure s ↔ x ∈ f ⁻¹' closure (f '' s)
[PROOFSTEP]
rw [Set.mem_preimage, ← closure_induced, hf.induced]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
⊢ IsClosed s ↔ ∃ t, IsClosed t ∧ f ⁻¹' t = s
[PROOFSTEP]
rw [hf.induced, isClosed_induced_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
⊢ IsClosed s ↔ ∀ (x : α), f x ∈ closure (f '' s) → x ∈ s
[PROOFSTEP]
rw [hf.induced, isClosed_induced_iff']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
⊢ IsOpen s ↔ ∃ t, IsOpen t ∧ f ⁻¹' t = s
[PROOFSTEP]
rw [hf.induced, isOpen_induced_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → β
hf : Inducing f
s : Set α
⊢ Dense s ↔ ∀ (x : α), f x ∈ closure (f '' s)
[PROOFSTEP]
simp only [Dense, hf.closure_eq_preimage_closure_image, mem_preimage]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
g : β → γ
hf : Continuous f
hg : Continuous g
hgf : _root_.Embedding (g ∘ f)
a₁ a₂ : α
h : f a₁ = f a₂
⊢ (g ∘ f) a₁ = (g ∘ f) a₂
[PROOFSTEP]
simp [h, (· ∘ ·)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
inst✝² : TopologicalSpace γ
X : Type u_5
Y : Type u_6
inst✝¹ : TopologicalSpace X
tY : TopologicalSpace Y
inst✝ : DiscreteTopology Y
f : X → Y
hf : _root_.Embedding f
x : X
⊢ 𝓝 x = pure x
[PROOFSTEP]
rw [hf.nhds_eq_comap, nhds_discrete, comap_pure, ← image_singleton, hf.inj.preimage_image, principal_singleton]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
⊢ (∀ (x : Set β), IsOpen xᶜ ↔ IsOpen (f ⁻¹' xᶜ)) ↔ ∀ (s : Set β), IsClosed s ↔ IsClosed (f ⁻¹' s)
[PROOFSTEP]
simp only [isOpen_compl_iff, preimage_compl]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
hg : QuotientMap g
hf : QuotientMap f
⊢ inst✝¹ = coinduced (g ∘ f) inst✝³
[PROOFSTEP]
rw [hg.right, hf.right, coinduced_compose]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
hf : Continuous f
hg : Continuous g
hgf : QuotientMap (g ∘ f)
⊢ inst✝¹ ≤ coinduced g inst✝²
[PROOFSTEP]
rw [hgf.right, ← coinduced_compose]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
hf : Continuous f
hg : Continuous g
hgf : QuotientMap (g ∘ f)
⊢ coinduced g (coinduced f inst✝³) ≤ coinduced g inst✝²
[PROOFSTEP]
exact coinduced_mono hf.coinduced_le
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
g : β → γ
f : α → β
hf : QuotientMap f
⊢ Continuous g ↔ Continuous (g ∘ f)
[PROOFSTEP]
rw [continuous_iff_coinduced_le, continuous_iff_coinduced_le, hf.right, coinduced_compose]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
s : Set α
hs : IsOpen s
⊢ IsOpen (id '' s)
[PROOFSTEP]
rwa [image_id]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f✝ : α → β
g : β → γ
f : α → β
hg : IsOpenMap g
hf : IsOpenMap f
s : Set α
hs : IsOpen s
⊢ IsOpen (g ∘ f '' s)
[PROOFSTEP]
rw [image_comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f✝ : α → β
g : β → γ
f : α → β
hg : IsOpenMap g
hf : IsOpenMap f
s : Set α
hs : IsOpen s
⊢ IsOpen (g '' (f '' s))
[PROOFSTEP]
exact hg _ (hf _ hs)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : IsOpenMap f
⊢ IsOpen (range f)
[PROOFSTEP]
rw [← image_univ]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : IsOpenMap f
⊢ IsOpen (f '' univ)
[PROOFSTEP]
exact hf _ isOpen_univ
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f✝ f : α → β
h : ∀ (x : α), ∃ g, ContinuousAt g (f x) ∧ g (f x) = x ∧ Function.RightInverse g f
x : α
g : β → α
hgc : ContinuousAt g (f x)
hgx : g (f x) = x
hgf : Function.RightInverse g f
⊢ 𝓝 (f x) = map f (map g (𝓝 (f x)))
[PROOFSTEP]
rw [map_map, hgf.comp_eq_id, map_id]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f✝ f : α → β
h : ∀ (x : α), ∃ g, ContinuousAt g (f x) ∧ g (f x) = x ∧ Function.RightInverse g f
x : α
g : β → α
hgc : ContinuousAt g (f x)
hgx : g (f x) = x
hgf : Function.RightInverse g f
⊢ map f (𝓝 (g (f x))) = map f (𝓝 x)
[PROOFSTEP]
rw [hgx]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : IsOpenMap f
s : Set β
⊢ f ⁻¹' closure s ⊆ closure (f ⁻¹' s)
[PROOFSTEP]
rw [← compl_subset_compl]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : IsOpenMap f
s : Set β
⊢ (closure (f ⁻¹' s))ᶜ ⊆ (f ⁻¹' closure s)ᶜ
[PROOFSTEP]
simp only [← interior_compl, ← preimage_compl, hf.interior_preimage_subset_preimage_interior]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : IsOpenMap f
s : Set β
⊢ f ⁻¹' frontier s ⊆ frontier (f ⁻¹' s)
[PROOFSTEP]
simpa only [frontier_eq_closure_inter_closure, preimage_inter] using
inter_subset_inter hf.preimage_closure_subset_closure_preimage hf.preimage_closure_subset_closure_preimage
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : IsOpenMap f
hfc : Continuous f
s : Set β
⊢ f ⁻¹' frontier s = frontier (f ⁻¹' s)
[PROOFSTEP]
simp only [frontier_eq_closure_inter_closure, preimage_inter, preimage_compl,
hf.preimage_closure_eq_closure_preimage hfc]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
hs : ∀ (s : Set α), f '' interior s ⊆ interior (f '' s)
u : Set α
hu : IsOpen u
⊢ f '' u = f '' interior u
[PROOFSTEP]
rw [hu.interior_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
hs : IsClosed s
⊢ IsClosed (id '' s)
[PROOFSTEP]
rwa [image_id]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : β → γ
f : α → β
hg : IsClosedMap g
hf : IsClosedMap f
⊢ IsClosedMap (g ∘ f)
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : β → γ
f : α → β
hg : IsClosedMap g
hf : IsClosedMap f
s : Set α
hs : IsClosed s
⊢ IsClosed (g ∘ f '' s)
[PROOFSTEP]
rw [image_comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : β → γ
f : α → β
hg : IsClosedMap g
hf : IsClosedMap f
s : Set α
hs : IsClosed s
⊢ IsClosed (g '' (f '' s))
[PROOFSTEP]
exact hg _ (hf _ hs)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
f' : β → α
h : Continuous f'
l_inv : LeftInverse f f'
r_inv : Function.RightInverse f f'
s : Set α
hs : IsClosed s
⊢ IsClosed (f '' s)
[PROOFSTEP]
rw [image_eq_preimage_of_inverse r_inv l_inv]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
f' : β → α
h : Continuous f'
l_inv : LeftInverse f f'
r_inv : Function.RightInverse f f'
s : Set α
hs : IsClosed s
⊢ IsClosed (f' ⁻¹' s)
[PROOFSTEP]
exact hs.preimage h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h : ∀ (s : Set α), IsClosed s → Set.Nonempty s → IsClosed (f '' s)
⊢ IsClosedMap f
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h : ∀ (s : Set α), IsClosed s → Set.Nonempty s → IsClosed (f '' s)
s : Set α
hs : IsClosed s
⊢ IsClosed (f '' s)
[PROOFSTEP]
cases' eq_empty_or_nonempty s with h2s h2s
[GOAL]
case inl
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h : ∀ (s : Set α), IsClosed s → Set.Nonempty s → IsClosed (f '' s)
s : Set α
hs : IsClosed s
h2s : s = ∅
⊢ IsClosed (f '' s)
[PROOFSTEP]
simp_rw [h2s, image_empty, isClosed_empty]
[GOAL]
case inr
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h : ∀ (s : Set α), IsClosed s → Set.Nonempty s → IsClosed (f '' s)
s : Set α
hs : IsClosed s
h2s : Set.Nonempty s
⊢ IsClosed (f '' s)
[PROOFSTEP]
exact h s hs h2s
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
hf : Inducing f
h : IsClosed (range f)
⊢ IsClosedMap f
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
hf : Inducing f
h : IsClosed (range f)
s : Set α
hs : IsClosed s
⊢ IsClosed (f '' s)
[PROOFSTEP]
rcases hf.isClosed_iff.1 hs with ⟨t, ht, rfl⟩
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
hf : Inducing f
h : IsClosed (range f)
t : Set β
ht : IsClosed t
hs : IsClosed (f ⁻¹' t)
⊢ IsClosed (f '' (f ⁻¹' t))
[PROOFSTEP]
rw [image_preimage_eq_inter_range]
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
hf : Inducing f
h : IsClosed (range f)
t : Set β
ht : IsClosed t
hs : IsClosed (f ⁻¹' t)
⊢ IsClosed (t ∩ range f)
[PROOFSTEP]
exact ht.inter h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
hs : ∀ (s : Set α), closure (f '' s) ⊆ f '' closure s
c : Set α
hc : IsClosed c
⊢ f '' closure c = f '' c
[PROOFSTEP]
rw [hc.closure_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
⊢ IsClosedMap f ↔ ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
[PROOFSTEP]
simp [MapClusterPt, isClosedMap_iff_closure_image, subset_def, mem_closure_iff_clusterPt, and_comm]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
f_closed : IsClosedMap f
f_cont : Continuous f
F : Filter α
⊢ Filter.lift' (map f F) closure = map f (Filter.lift' F closure)
[PROOFSTEP]
rw [map_lift'_eq2 (monotone_closure β), map_lift'_eq (monotone_closure α)]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
f_closed : IsClosedMap f
f_cont : Continuous f
F : Filter α
⊢ Filter.lift' F (closure ∘ image f) = Filter.lift' F (image f ∘ closure)
[PROOFSTEP]
congr
[GOAL]
case e_h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
f_closed : IsClosedMap f
f_cont : Continuous f
F : Filter α
⊢ closure ∘ image f = image f ∘ closure
[PROOFSTEP]
ext s : 1
[GOAL]
case e_h.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
f : α → β
f_closed : IsClosedMap f
f_cont : Continuous f
F : Filter α
s : Set α
⊢ (closure ∘ image f) s = (image f ∘ closure) s
[PROOFSTEP]
exact f_closed.closure_image_eq_of_continuous f_cont s
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
F : Filter α
f : α → β
f_closed : IsClosedMap f
f_cont : Continuous f
y : β
⊢ MapClusterPt y F f ↔ NeBot (Filter.lift' F closure ⊓ 𝓟 (f ⁻¹' {y}))
[PROOFSTEP]
rw [MapClusterPt, clusterPt_iff_lift'_closure', f_closed.lift'_closure_map_eq f_cont, ← comap_principal, ←
map_neBot_iff f, Filter.push_pull, principal_singleton]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : OpenEmbedding f
s : Set α
h : IsOpen (f '' s)
⊢ IsOpen s
[PROOFSTEP]
convert ← h.preimage hf.toEmbedding.continuous
[GOAL]
case h.e'_3
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : OpenEmbedding f
s : Set α
h : IsOpen (f '' s)
⊢ f ⁻¹' (f '' s) = s
[PROOFSTEP]
apply preimage_image_eq _ hf.inj
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : OpenEmbedding f
g : β → γ
l : Filter γ
a : α
⊢ Tendsto (g ∘ f) (𝓝 a) l ↔ Tendsto g (𝓝 (f a)) l
[PROOFSTEP]
rw [Tendsto, ← map_map, hf.map_nhds_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : OpenEmbedding f
g : β → γ
l : Filter γ
a : α
⊢ map g (𝓝 (f a)) ≤ l ↔ Tendsto g (𝓝 (f a)) l
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : OpenEmbedding f
s : Set β
hs : s ⊆ range f
⊢ IsOpen s ↔ IsOpen (f ⁻¹' s)
[PROOFSTEP]
rw [hf.open_iff_image_open, image_preimage_eq_inter_range, inter_eq_self_of_subset_left hs]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h₁ : Continuous f
h₂ : Injective f
h₃ : IsOpenMap f
⊢ OpenEmbedding f
[PROOFSTEP]
simp only [openEmbedding_iff_embedding_open, embedding_iff, inducing_iff_nhds, *, and_true_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h₁ : Continuous f
h₂ : Injective f
h₃ : IsOpenMap f
⊢ ∀ (a : α), 𝓝 a = comap f (𝓝 (f a))
[PROOFSTEP]
exact fun a => le_antisymm (h₁.tendsto _).le_comap (@comap_map _ _ (𝓝 a) _ h₂ ▸ comap_mono (h₃.nhds_le _))
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : β → γ
f : α → β
hg : OpenEmbedding g
⊢ IsOpenMap f ↔ IsOpenMap (g ∘ f)
[PROOFSTEP]
simp_rw [isOpenMap_iff_nhds_le, ← map_map, comp, ← hg.map_nhds_eq, Filter.map_le_map_iff hg.inj]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
g : β → γ
hg : OpenEmbedding g
⊢ OpenEmbedding (g ∘ f) ↔ OpenEmbedding f
[PROOFSTEP]
simp only [openEmbedding_iff_continuous_injective_open, ← hg.isOpenMap_iff, ← hg.1.continuous_iff, hg.inj.of_comp_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : ClosedEmbedding f
s : Set α
h : IsClosed (f '' s)
⊢ IsClosed s
[PROOFSTEP]
rw [← preimage_image_eq s hf.inj]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : ClosedEmbedding f
s : Set α
h : IsClosed (f '' s)
⊢ IsClosed (f ⁻¹' (f '' s))
[PROOFSTEP]
exact h.preimage hf.continuous
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : ClosedEmbedding f
s : Set β
hs : s ⊆ range f
⊢ IsClosed s ↔ IsClosed (f ⁻¹' s)
[PROOFSTEP]
rw [hf.closed_iff_image_closed, image_preimage_eq_of_subset hs]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h₁ : Continuous f
h₂ : Injective f
h₃ : IsClosedMap f
⊢ ClosedEmbedding f
[PROOFSTEP]
refine closedEmbedding_of_embedding_closed ⟨⟨?_⟩, h₂⟩ h₃
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h₁ : Continuous f
h₂ : Injective f
h₃ : IsClosedMap f
⊢ inst✝² = induced f inst✝¹
[PROOFSTEP]
refine h₁.le_induced.antisymm fun s hs => ?_
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h₁ : Continuous f
h₂ : Injective f
h₃ : IsClosedMap f
s : Set α
hs : IsOpen s
⊢ IsOpen s
[PROOFSTEP]
refine ⟨(f '' sᶜ)ᶜ, (h₃ _ hs.isClosed_compl).isOpen_compl, ?_⟩
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
h₁ : Continuous f
h₂ : Injective f
h₃ : IsClosedMap f
s : Set α
hs : IsOpen s
⊢ f ⁻¹' (f '' sᶜ)ᶜ = s
[PROOFSTEP]
rw [preimage_compl, preimage_image_eq _ h₂, compl_compl]
| {"mathlib_filename": "Mathlib.Topology.Maps", "llama_tokens": 11366} |
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
⊢ IsTotallySeparated univ
[PROOFSTEP]
intro x _ y _ hxy
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ univ ⊆ u ∪ v ∧ Disjoint u v
[PROOFSTEP]
obtain ⟨U, V, hUV⟩ := T2Space.t2 x y hxy
[GOAL]
case intro.intro
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ univ ⊆ u ∪ v ∧ Disjoint u v
[PROOFSTEP]
use closure U
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ∃ v, IsOpen (closure U) ∧ IsOpen v ∧ x ∈ closure U ∧ y ∈ v ∧ univ ⊆ closure U ∪ v ∧ Disjoint (closure U) v
[PROOFSTEP]
use(closure U)ᶜ
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ IsOpen (closure U) ∧
IsOpen (closure U)ᶜ ∧
x ∈ closure U ∧ y ∈ (closure U)ᶜ ∧ univ ⊆ closure U ∪ (closure U)ᶜ ∧ Disjoint (closure U) (closure U)ᶜ
[PROOFSTEP]
refine
⟨ExtremallyDisconnected.open_closure U hUV.1, by simp only [isOpen_compl_iff, isClosed_closure],
subset_closure hUV.2.2.1, ?_, by simp only [Set.union_compl_self, Set.subset_univ], disjoint_compl_right⟩
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ IsOpen (closure U)ᶜ
[PROOFSTEP]
simp only [isOpen_compl_iff, isClosed_closure]
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ univ ⊆ closure U ∪ (closure U)ᶜ
[PROOFSTEP]
simp only [Set.union_compl_self, Set.subset_univ]
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ y ∈ (closure U)ᶜ
[PROOFSTEP]
simp only [Set.mem_compl_iff]
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ¬y ∈ closure U
[PROOFSTEP]
rw [mem_closure_iff]
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ¬∀ (o : Set X), IsOpen o → y ∈ o → Set.Nonempty (o ∩ U)
[PROOFSTEP]
push_neg
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ∃ o, IsOpen o ∧ y ∈ o ∧ ¬Set.Nonempty (o ∩ U)
[PROOFSTEP]
refine' ⟨V, ⟨hUV.2.1, hUV.2.2.2.1, _⟩⟩
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ¬Set.Nonempty (V ∩ U)
[PROOFSTEP]
rw [Set.nonempty_iff_ne_empty]
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ ¬V ∩ U ≠ ∅
[PROOFSTEP]
simp only [not_not]
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ V ∩ U = ∅
[PROOFSTEP]
rw [← Set.disjoint_iff_inter_eq_empty, disjoint_comm]
[GOAL]
case h
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : ExtremallyDisconnected X
inst✝ : T2Space X
x : X
a✝¹ : x ∈ univ
y : X
a✝ : y ∈ univ
hxy : x ≠ y
U V : Set X
hUV : IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ Disjoint U V
⊢ Disjoint U V
[PROOFSTEP]
exact hUV.2.2.2.2
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
⊢ CompactT2.Projective (StoneCech X)
[PROOFSTEP]
intro Y Z _tsY _tsZ _csY _t2Y _csZ _csZ f g hf hg g_sur
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
let s : Z → Y := fun z => Classical.choose <| g_sur z
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
have hs : g ∘ s = id := funext fun z => Classical.choose_spec (g_sur z)
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
hs : g ∘ s = id
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
let t := s ∘ f ∘ stoneCechUnit
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
hs : g ∘ s = id
t : X → Y := s ∘ f ∘ stoneCechUnit
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
have ht : Continuous t := continuous_of_discreteTopology
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
hs : g ∘ s = id
t : X → Y := s ∘ f ∘ stoneCechUnit
ht : Continuous t
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
let h : StoneCech X → Y := stoneCechExtend ht
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
hs : g ∘ s = id
t : X → Y := s ∘ f ∘ stoneCechUnit
ht : Continuous t
h : StoneCech X → Y := stoneCechExtend ht
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
have hh : Continuous h := continuous_stoneCechExtend ht
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
hs : g ∘ s = id
t : X → Y := s ∘ f ∘ stoneCechUnit
ht : Continuous t
h : StoneCech X → Y := stoneCechExtend ht
hh : Continuous h
⊢ ∃ h, Continuous h ∧ g ∘ h = f
[PROOFSTEP]
refine' ⟨h, hh, denseRange_stoneCechUnit.equalizer (hg.comp hh) hf _⟩
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
inst✝ : DiscreteTopology X
Y Z : Type u
_tsY : TopologicalSpace Y
_tsZ : TopologicalSpace Z
_csY : CompactSpace Y
_t2Y : T2Space Y
_csZ✝ : CompactSpace Z
_csZ : T2Space Z
f : StoneCech X → Z
g : Y → Z
hf : Continuous f
hg : Continuous g
g_sur : Surjective g
s : Z → Y := fun z => choose (_ : ∃ a, g a = z)
hs : g ∘ s = id
t : X → Y := s ∘ f ∘ stoneCechUnit
ht : Continuous t
h : StoneCech X → Y := stoneCechExtend ht
hh : Continuous h
⊢ (g ∘ h) ∘ stoneCechUnit = f ∘ stoneCechUnit
[PROOFSTEP]
rw [comp.assoc, stoneCechExtend_extends ht, ← comp.assoc, hs, comp.left_id]
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
⊢ ExtremallyDisconnected X
[PROOFSTEP]
refine' { open_closure := fun U hU => _ }
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
⊢ IsOpen (closure U)
[PROOFSTEP]
let Z₁ : Set (X × Bool) := Uᶜ ×ˢ { true }
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
⊢ IsOpen (closure U)
[PROOFSTEP]
let Z₂ : Set (X × Bool) := closure U ×ˢ { false }
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
⊢ IsOpen (closure U)
[PROOFSTEP]
let Z : Set (X × Bool) := Z₁ ∪ Z₂
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
⊢ IsOpen (closure U)
[PROOFSTEP]
have hZ₁₂ : Disjoint Z₁ Z₂ := disjoint_left.2 fun x hx₁ hx₂ => by cases hx₁.2.symm.trans hx₂.2
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
x : X × Bool
hx₁ : x ∈ Z₁
hx₂ : x ∈ Z₂
⊢ False
[PROOFSTEP]
cases hx₁.2.symm.trans hx₂.2
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
⊢ IsOpen (closure U)
[PROOFSTEP]
have hZ₁ : IsClosed Z₁ := hU.isClosed_compl.prod (T1Space.t1 _)
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
⊢ IsOpen (closure U)
[PROOFSTEP]
have hZ₂ : IsClosed Z₂ := isClosed_closure.prod (T1Space.t1 false)
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
⊢ IsOpen (closure U)
[PROOFSTEP]
have hZ : IsClosed Z := hZ₁.union hZ₂
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
⊢ IsOpen (closure U)
[PROOFSTEP]
let f : Z → X := Prod.fst ∘ Subtype.val
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
⊢ IsOpen (closure U)
[PROOFSTEP]
have f_cont : Continuous f := continuous_fst.comp continuous_subtype_val
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
⊢ IsOpen (closure U)
[PROOFSTEP]
have f_sur : Surjective f := by
intro x
by_cases hx : x ∈ U
· exact ⟨⟨(x, false), Or.inr ⟨subset_closure hx, mem_singleton _⟩⟩, rfl⟩
· exact ⟨⟨(x, true), Or.inl ⟨hx, mem_singleton _⟩⟩, rfl⟩
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
⊢ Surjective f
[PROOFSTEP]
intro x
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
x : X
⊢ ∃ a, f a = x
[PROOFSTEP]
by_cases hx : x ∈ U
[GOAL]
case pos
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
x : X
hx : x ∈ U
⊢ ∃ a, f a = x
[PROOFSTEP]
exact ⟨⟨(x, false), Or.inr ⟨subset_closure hx, mem_singleton _⟩⟩, rfl⟩
[GOAL]
case neg
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
x : X
hx : ¬x ∈ U
⊢ ∃ a, f a = x
[PROOFSTEP]
exact ⟨⟨(x, true), Or.inl ⟨hx, mem_singleton _⟩⟩, rfl⟩
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
⊢ IsOpen (closure U)
[PROOFSTEP]
haveI : CompactSpace Z := isCompact_iff_compactSpace.mp hZ.isCompact
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
⊢ IsOpen (closure U)
[PROOFSTEP]
obtain ⟨g, hg, g_sec⟩ := h continuous_id f_cont f_sur
[GOAL]
case intro.intro
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
⊢ IsOpen (closure U)
[PROOFSTEP]
let φ := Subtype.val ∘ g
[GOAL]
case intro.intro
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
⊢ IsOpen (closure U)
[PROOFSTEP]
have hφ : Continuous φ := continuous_subtype_val.comp hg
[GOAL]
case intro.intro
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
⊢ IsOpen (closure U)
[PROOFSTEP]
have hφ₁ : ∀ x, (φ x).1 = x := congr_fun g_sec
[GOAL]
case intro.intro
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
⊢ IsOpen (closure U)
[PROOFSTEP]
suffices closure U = φ ⁻¹' Z₂
by
rw [this, preimage_comp, ← isClosed_compl_iff, ← preimage_compl, ← preimage_subtype_coe_eq_compl Subset.rfl]
· exact hZ₁.preimage hφ
· rw [hZ₁₂.inter_eq, inter_empty]
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this✝ : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
this : closure U = φ ⁻¹' Z₂
⊢ IsOpen (closure U)
[PROOFSTEP]
rw [this, preimage_comp, ← isClosed_compl_iff, ← preimage_compl, ← preimage_subtype_coe_eq_compl Subset.rfl]
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this✝ : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
this : closure U = φ ⁻¹' Z₂
⊢ IsClosed (g ⁻¹' (Subtype.val ⁻¹' Z₁))
[PROOFSTEP]
exact hZ₁.preimage hφ
[GOAL]
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this✝ : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
this : closure U = φ ⁻¹' Z₂
⊢ (Z₁ ∪ Z₂) ∩ (Z₁ ∩ Z₂) = ∅
[PROOFSTEP]
rw [hZ₁₂.inter_eq, inter_empty]
[GOAL]
case intro.intro
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
⊢ closure U = φ ⁻¹' Z₂
[PROOFSTEP]
refine' (closure_minimal _ <| hZ₂.preimage hφ).antisymm fun x hx => _
[GOAL]
case intro.intro.refine'_1
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
⊢ U ⊆ φ ⁻¹' Z₂
[PROOFSTEP]
intro x hx
[GOAL]
case intro.intro.refine'_1
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
x : X
hx : x ∈ U
⊢ x ∈ φ ⁻¹' Z₂
[PROOFSTEP]
have : φ x ∈ Z₁ ∪ Z₂ :=
(g x).2
-- Porting note: Originally `simpa [hx, hφ₁] using this`
[GOAL]
case intro.intro.refine'_1
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this✝ : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
x : X
hx : x ∈ U
this : φ x ∈ Z₁ ∪ Z₂
⊢ x ∈ φ ⁻¹' Z₂
[PROOFSTEP]
cases' this with hφ hφ
[GOAL]
case intro.intro.refine'_1.inl
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ✝ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
x : X
hx : x ∈ U
hφ : φ x ∈ Z₁
⊢ x ∈ φ ⁻¹' Z₂
[PROOFSTEP]
exact ((hφ₁ x ▸ hφ.1) hx).elim
[GOAL]
case intro.intro.refine'_1.inr
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ✝ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
x : X
hx : x ∈ U
hφ : φ x ∈ Z₂
⊢ x ∈ φ ⁻¹' Z₂
[PROOFSTEP]
exact hφ
[GOAL]
case intro.intro.refine'_2
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
x : X
hx : x ∈ φ ⁻¹' Z₂
⊢ x ∈ closure U
[PROOFSTEP]
rw [← hφ₁ x]
[GOAL]
case intro.intro.refine'_2
X : Type u
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
inst✝ : T2Space X
h : Projective X
U : Set X
hU : IsOpen U
Z₁ : Set (X × Bool) := Uᶜ ×ˢ {true}
Z₂ : Set (X × Bool) := closure U ×ˢ {false}
Z : Set (X × Bool) := Z₁ ∪ Z₂
hZ₁₂ : Disjoint Z₁ Z₂
hZ₁ : IsClosed Z₁
hZ₂ : IsClosed Z₂
hZ : IsClosed Z
f : ↑Z → X := Prod.fst ∘ Subtype.val
f_cont : Continuous f
f_sur : Surjective f
this : CompactSpace ↑Z
g : X → ↑Z
hg : Continuous g
g_sec : f ∘ g = id
φ : X → X × Bool := Subtype.val ∘ g
hφ : Continuous φ
hφ₁ : ∀ (x : X), (φ x).fst = x
x : X
hx : x ∈ φ ⁻¹' Z₂
⊢ (φ x).fst ∈ closure U
[PROOFSTEP]
exact hx.1
[GOAL]
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
⊢ ∃ E, CompactSpace ↑E ∧ π '' E = univ ∧ ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π '' E₀ ≠ univ
[PROOFSTEP]
let S : Set <| Set D := {E : Set D | IsClosed E ∧ π '' E = univ}
[GOAL]
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
⊢ ∃ E, CompactSpace ↑E ∧ π '' E = univ ∧ ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π '' E₀ ≠ univ
[PROOFSTEP]
suffices ∀ (C : Set <| Set D) (_ : C ⊆ S) (_ : IsChain (· ⊆ ·) C), ∃ s ∈ S, ∀ c ∈ C, s ⊆ c
by
rcases zorn_superset S this with ⟨E, ⟨E_closed, E_surj⟩, E_min⟩
refine ⟨E, isCompact_iff_compactSpace.mp E_closed.isCompact, E_surj, ?_⟩
intro E₀ E₀_min E₀_closed
contrapose! E₀_min
exact eq_univ_of_coe_eq <| E_min E₀ ⟨E₀_closed.trans E_closed, image_coe_eq_restrict_image ▸ E₀_min⟩ coe_subset
[GOAL]
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
this : ∀ (C : Set (Set D)), C ⊆ S → IsChain (fun x x_1 => x ⊆ x_1) C → ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
⊢ ∃ E, CompactSpace ↑E ∧ π '' E = univ ∧ ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π '' E₀ ≠ univ
[PROOFSTEP]
rcases zorn_superset S this with ⟨E, ⟨E_closed, E_surj⟩, E_min⟩
[GOAL]
case intro.intro.intro
X : Type u
inst✝⁵ : TopologicalSpace X
A D E✝ : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E✝
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
this : ∀ (C : Set (Set D)), C ⊆ S → IsChain (fun x x_1 => x ⊆ x_1) C → ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
E : Set D
E_min : ∀ (a : Set D), a ∈ S → a ⊆ E → a = E
E_closed : IsClosed E
E_surj : π '' E = univ
⊢ ∃ E, CompactSpace ↑E ∧ π '' E = univ ∧ ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π '' E₀ ≠ univ
[PROOFSTEP]
refine ⟨E, isCompact_iff_compactSpace.mp E_closed.isCompact, E_surj, ?_⟩
[GOAL]
case intro.intro.intro
X : Type u
inst✝⁵ : TopologicalSpace X
A D E✝ : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E✝
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
this : ∀ (C : Set (Set D)), C ⊆ S → IsChain (fun x x_1 => x ⊆ x_1) C → ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
E : Set D
E_min : ∀ (a : Set D), a ∈ S → a ⊆ E → a = E
E_closed : IsClosed E
E_surj : π '' E = univ
⊢ ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π '' E₀ ≠ univ
[PROOFSTEP]
intro E₀ E₀_min E₀_closed
[GOAL]
case intro.intro.intro
X : Type u
inst✝⁵ : TopologicalSpace X
A D E✝ : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E✝
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
this : ∀ (C : Set (Set D)), C ⊆ S → IsChain (fun x x_1 => x ⊆ x_1) C → ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
E : Set D
E_min : ∀ (a : Set D), a ∈ S → a ⊆ E → a = E
E_closed : IsClosed E
E_surj : π '' E = univ
E₀ : Set ↑E
E₀_min : E₀ ≠ univ
E₀_closed : IsClosed E₀
⊢ restrict E π '' E₀ ≠ univ
[PROOFSTEP]
contrapose! E₀_min
[GOAL]
case intro.intro.intro
X : Type u
inst✝⁵ : TopologicalSpace X
A D E✝ : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E✝
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
this : ∀ (C : Set (Set D)), C ⊆ S → IsChain (fun x x_1 => x ⊆ x_1) C → ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
E : Set D
E_min : ∀ (a : Set D), a ∈ S → a ⊆ E → a = E
E_closed : IsClosed E
E_surj : π '' E = univ
E₀ : Set ↑E
E₀_closed : IsClosed E₀
E₀_min : restrict E π '' E₀ = univ
⊢ E₀ = univ
[PROOFSTEP]
exact eq_univ_of_coe_eq <| E_min E₀ ⟨E₀_closed.trans E_closed, image_coe_eq_restrict_image ▸ E₀_min⟩ coe_subset
[GOAL]
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
⊢ ∀ (C : Set (Set D)), C ⊆ S → IsChain (fun x x_1 => x ⊆ x_1) C → ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
[PROOFSTEP]
intro C C_sub C_chain
[GOAL]
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
⊢ ∃ s, s ∈ S ∧ ∀ (c : Set D), c ∈ C → s ⊆ c
[PROOFSTEP]
refine
⟨iInter (fun c : C => c), ⟨isClosed_iInter fun ⟨_, h⟩ => (C_sub h).left, ?_⟩, fun c hc _ h => mem_iInter.mp h ⟨c, hc⟩⟩
-- prove intersection of chain is mapped onto $A$
[GOAL]
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
⊢ π '' ⋂ (c : ↑C), ↑c = univ
[PROOFSTEP]
by_cases hC : Nonempty C
[GOAL]
case pos
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
⊢ π '' ⋂ (c : ↑C), ↑c = univ
[PROOFSTEP]
refine
eq_univ_of_forall fun a =>
inter_nonempty_iff_exists_left.mp
?_
-- apply Cantor's intersection theorem
[GOAL]
case pos
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
⊢ Set.Nonempty ((⋂ (c : ↑C), ↑c) ∩ fun a_1 => π a_1 = a)
[PROOFSTEP]
refine
iInter_inter (ι := C) (π ⁻¹' { a }) _ ▸
IsCompact.nonempty_iInter_of_directed_nonempty_compact_closed _ ?_ (fun c => ?_) (fun c => IsClosed.isCompact ?_)
(fun c => ?_)
[GOAL]
case pos.refine_1
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
⊢ Directed (fun x x_1 => x ⊇ x_1) fun i => ↑i ∩ π ⁻¹' {a}
[PROOFSTEP]
replace C_chain : IsChain (· ⊇ ·) C := C_chain.symm
[GOAL]
case pos.refine_1
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
hC : Nonempty ↑C
a : A
C_chain : IsChain (fun x x_1 => x ⊇ x_1) C
⊢ Directed (fun x x_1 => x ⊇ x_1) fun i => ↑i ∩ π ⁻¹' {a}
[PROOFSTEP]
have : ∀ s t : Set D, s ⊇ t → _ ⊇ _ := fun _ _ => inter_subset_inter_left <| π ⁻¹' { a }
[GOAL]
case pos.refine_1
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
hC : Nonempty ↑C
a : A
C_chain : IsChain (fun x x_1 => x ⊇ x_1) C
this : ∀ (s t : Set D), s ⊇ t → s ∩ π ⁻¹' {a} ⊇ t ∩ π ⁻¹' {a}
⊢ Directed (fun x x_1 => x ⊇ x_1) fun i => ↑i ∩ π ⁻¹' {a}
[PROOFSTEP]
exact (directedOn_iff_directed.mp C_chain.directedOn).mono_comp (· ⊇ ·) this
[GOAL]
case pos.refine_2
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
c : ↑C
⊢ Set.Nonempty (↑c ∩ π ⁻¹' {a})
[PROOFSTEP]
rw [← image_inter_nonempty_iff, (C_sub c.mem).right, univ_inter]
[GOAL]
case pos.refine_2
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
c : ↑C
⊢ Set.Nonempty {a}
[PROOFSTEP]
exact singleton_nonempty a
[GOAL]
case pos.refine_3
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
c : ↑C
⊢ IsClosed (↑c ∩ π ⁻¹' {a})
case pos.refine_4
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
c : ↑C
⊢ IsClosed (↑c ∩ π ⁻¹' {a})
[PROOFSTEP]
all_goals exact (C_sub c.mem).left.inter <| (T1Space.t1 a).preimage π_cont
[GOAL]
case pos.refine_3
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
c : ↑C
⊢ IsClosed (↑c ∩ π ⁻¹' {a})
[PROOFSTEP]
exact (C_sub c.mem).left.inter <| (T1Space.t1 a).preimage π_cont
[GOAL]
case pos.refine_4
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : Nonempty ↑C
a : A
c : ↑C
⊢ IsClosed (↑c ∩ π ⁻¹' {a})
[PROOFSTEP]
exact (C_sub c.mem).left.inter <| (T1Space.t1 a).preimage π_cont
[GOAL]
case neg
X : Type u
inst✝⁵ : TopologicalSpace X
A D E : Type u
inst✝⁴ : TopologicalSpace A
inst✝³ : TopologicalSpace D
inst✝² : TopologicalSpace E
inst✝¹ : T1Space A
inst✝ : CompactSpace D
π : D → A
π_cont : Continuous π
π_surj : Surjective π
S : Set (Set D) := {E | IsClosed E ∧ π '' E = univ}
C : Set (Set D)
C_sub : C ⊆ S
C_chain : IsChain (fun x x_1 => x ⊆ x_1) C
hC : ¬Nonempty ↑C
⊢ π '' ⋂ (c : ↑C), ↑c = univ
[PROOFSTEP]
rw [@iInter_of_empty _ _ <| not_nonempty_iff.mp hC, image_univ_of_surjective π_surj]
[GOAL]
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
⊢ ρ '' G ⊆ closure (ρ '' Gᶜ)ᶜ
[PROOFSTEP]
by_cases G_empty : G = ∅
[GOAL]
case pos
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : G = ∅
⊢ ρ '' G ⊆ closure (ρ '' Gᶜ)ᶜ
[PROOFSTEP]
simpa only [G_empty, image_empty] using empty_subset _
[GOAL]
case neg
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
⊢ ρ '' G ⊆ closure (ρ '' Gᶜ)ᶜ
[PROOFSTEP]
intro a ha
[GOAL]
case neg
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
a : A
ha : a ∈ ρ '' G
⊢ a ∈ closure (ρ '' Gᶜ)ᶜ
[PROOFSTEP]
rw [mem_closure_iff]
-- let $N$ be a neighbourhood of $a$
[GOAL]
case neg
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
a : A
ha : a ∈ ρ '' G
⊢ ∀ (o : Set A), IsOpen o → a ∈ o → Set.Nonempty (o ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
intro N N_open hN
[GOAL]
case neg
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
a : A
ha : a ∈ ρ '' G
N : Set A
N_open : IsOpen N
hN : a ∈ N
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
rcases(G.mem_image ρ a).mp ha with ⟨e, he, rfl⟩
[GOAL]
case neg.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
have nonempty : (G ∩ ρ ⁻¹' N).Nonempty := ⟨e, mem_inter he <| mem_preimage.mpr hN⟩
[GOAL]
case neg.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
have is_open : IsOpen <| G ∩ ρ ⁻¹' N := hG.inter <| N_open.preimage ρ_cont
[GOAL]
case neg.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
have ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ := zorn_subset _ (compl_ne_univ.mpr nonempty) is_open.isClosed_compl
[GOAL]
case neg.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
rcases nonempty_compl.mpr ne_univ with
⟨x, hx⟩
-- prove $x \in N \cap (A \setminus \rho(E \setminus G))$
[GOAL]
case neg.intro.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
x : A
hx : x ∈ (ρ '' (G ∩ ρ ⁻¹' N)ᶜ)ᶜ
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
have hx' : x ∈ (ρ '' Gᶜ)ᶜ := fun h => hx <| image_subset ρ (by simp) h
[GOAL]
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
x : A
hx : x ∈ (ρ '' (G ∩ ρ ⁻¹' N)ᶜ)ᶜ
h : x ∈ ρ '' Gᶜ
⊢ Gᶜ ⊆ (G ∩ ρ ⁻¹' N)ᶜ
[PROOFSTEP]
simp
[GOAL]
case neg.intro.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
x : A
hx : x ∈ (ρ '' (G ∩ ρ ⁻¹' N)ᶜ)ᶜ
hx' : x ∈ (ρ '' Gᶜ)ᶜ
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
rcases ρ_surj x with ⟨y, rfl⟩
[GOAL]
case neg.intro.intro.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
y : E
hx : ρ y ∈ (ρ '' (G ∩ ρ ⁻¹' N)ᶜ)ᶜ
hx' : ρ y ∈ (ρ '' Gᶜ)ᶜ
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
have hy : y ∈ G ∩ ρ ⁻¹' N := by simpa using mt (mem_image_of_mem ρ) <| mem_compl hx
[GOAL]
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
y : E
hx : ρ y ∈ (ρ '' (G ∩ ρ ⁻¹' N)ᶜ)ᶜ
hx' : ρ y ∈ (ρ '' Gᶜ)ᶜ
⊢ y ∈ G ∩ ρ ⁻¹' N
[PROOFSTEP]
simpa using mt (mem_image_of_mem ρ) <| mem_compl hx
[GOAL]
case neg.intro.intro.intro.intro
X : Type u
inst✝³ : TopologicalSpace X
A D E : Type u
inst✝² : TopologicalSpace A
inst✝¹ : TopologicalSpace D
inst✝ : TopologicalSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
G : Set E
hG : IsOpen G
G_empty : ¬G = ∅
N : Set A
N_open : IsOpen N
e : E
he : e ∈ G
ha : ρ e ∈ ρ '' G
hN : ρ e ∈ N
nonempty : Set.Nonempty (G ∩ ρ ⁻¹' N)
is_open : IsOpen (G ∩ ρ ⁻¹' N)
ne_univ : ρ '' (G ∩ ρ ⁻¹' N)ᶜ ≠ univ
y : E
hx : ρ y ∈ (ρ '' (G ∩ ρ ⁻¹' N)ᶜ)ᶜ
hx' : ρ y ∈ (ρ '' Gᶜ)ᶜ
hy : y ∈ G ∩ ρ ⁻¹' N
⊢ Set.Nonempty (N ∩ (ρ '' Gᶜ)ᶜ)
[PROOFSTEP]
exact ⟨ρ y, mem_inter (mem_preimage.mp <| mem_of_mem_inter_right hy) hx'⟩
[GOAL]
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
⊢ Injective ρ
[PROOFSTEP]
intro x₁ x₂ hρx
[GOAL]
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
⊢ x₁ = x₂
[PROOFSTEP]
by_contra hx
[GOAL]
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
⊢ False
[PROOFSTEP]
rcases t2_separation hx with
⟨G₁, G₂, G₁_open, G₂_open, hx₁, hx₂, disj⟩
-- prove $A \setminus \rho(E - G_1)$ and $A \setminus \rho(E - G_2)$ are disjoint
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
⊢ False
[PROOFSTEP]
have G₁_comp : IsCompact G₁ᶜ := IsClosed.isCompact G₁_open.isClosed_compl
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
⊢ False
[PROOFSTEP]
have G₂_comp : IsCompact G₂ᶜ := IsClosed.isCompact G₂_open.isClosed_compl
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
⊢ False
[PROOFSTEP]
have G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ := (G₁_comp.image ρ_cont).isClosed.isOpen_compl
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
⊢ False
[PROOFSTEP]
have G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ := (G₂_comp.image ρ_cont).isClosed.isOpen_compl
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ
⊢ False
[PROOFSTEP]
have disj' : Disjoint (ρ '' G₁ᶜ)ᶜ (ρ '' G₂ᶜ)ᶜ := by
rw [disjoint_iff_inter_eq_empty, ← compl_union, ← image_union, ← compl_inter, disjoint_iff_inter_eq_empty.mp disj,
compl_empty, compl_empty_iff, image_univ_of_surjective ρ_surj]
-- apply Lemma 2.2 to prove their closures are disjoint
[GOAL]
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ
⊢ Disjoint (ρ '' G₁ᶜ)ᶜ (ρ '' G₂ᶜ)ᶜ
[PROOFSTEP]
rw [disjoint_iff_inter_eq_empty, ← compl_union, ← image_union, ← compl_inter, disjoint_iff_inter_eq_empty.mp disj,
compl_empty, compl_empty_iff, image_univ_of_surjective ρ_surj]
-- apply Lemma 2.2 to prove their closures are disjoint
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ
disj' : Disjoint (ρ '' G₁ᶜ)ᶜ (ρ '' G₂ᶜ)ᶜ
⊢ False
[PROOFSTEP]
have disj'' : Disjoint (closure (ρ '' G₁ᶜ)ᶜ) (closure (ρ '' G₂ᶜ)ᶜ) :=
disjoint_closure_of_disjoint_IsOpen disj' G₁_open' G₂_open'
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ
disj' : Disjoint (ρ '' G₁ᶜ)ᶜ (ρ '' G₂ᶜ)ᶜ
disj'' : Disjoint (closure (ρ '' G₁ᶜ)ᶜ) (closure (ρ '' G₂ᶜ)ᶜ)
⊢ False
[PROOFSTEP]
have hx₁' :=
image_subset_closure_compl_image_compl_of_isOpen ρ_cont ρ_surj zorn_subset G₁_open <| mem_image_of_mem ρ hx₁
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ
disj' : Disjoint (ρ '' G₁ᶜ)ᶜ (ρ '' G₂ᶜ)ᶜ
disj'' : Disjoint (closure (ρ '' G₁ᶜ)ᶜ) (closure (ρ '' G₂ᶜ)ᶜ)
hx₁' : ρ x₁ ∈ closure (ρ '' G₁ᶜ)ᶜ
⊢ False
[PROOFSTEP]
have hx₂' :=
image_subset_closure_compl_image_compl_of_isOpen ρ_cont ρ_surj zorn_subset G₂_open <| mem_image_of_mem ρ hx₂
[GOAL]
case intro.intro.intro.intro.intro.intro
X : Type u
inst✝⁷ : TopologicalSpace X
A D E : Type u
inst✝⁶ : TopologicalSpace A
inst✝⁵ : TopologicalSpace D
inst✝⁴ : TopologicalSpace E
inst✝³ : ExtremallyDisconnected A
inst✝² : T2Space A
inst✝¹ : T2Space E
inst✝ : CompactSpace E
ρ : E → A
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
zorn_subset : ∀ (E₀ : Set E), E₀ ≠ univ → IsClosed E₀ → ρ '' E₀ ≠ univ
x₁ x₂ : E
hρx : ρ x₁ = ρ x₂
hx : ¬x₁ = x₂
G₁ G₂ : Set E
G₁_open : IsOpen G₁
G₂_open : IsOpen G₂
hx₁ : x₁ ∈ G₁
hx₂ : x₂ ∈ G₂
disj : Disjoint G₁ G₂
G₁_comp : IsCompact G₁ᶜ
G₂_comp : IsCompact G₂ᶜ
G₁_open' : IsOpen (ρ '' G₁ᶜ)ᶜ
G₂_open' : IsOpen (ρ '' G₂ᶜ)ᶜ
disj' : Disjoint (ρ '' G₁ᶜ)ᶜ (ρ '' G₂ᶜ)ᶜ
disj'' : Disjoint (closure (ρ '' G₁ᶜ)ᶜ) (closure (ρ '' G₂ᶜ)ᶜ)
hx₁' : ρ x₁ ∈ closure (ρ '' G₁ᶜ)ᶜ
hx₂' : ρ x₂ ∈ closure (ρ '' G₂ᶜ)ᶜ
⊢ False
[PROOFSTEP]
exact disj''.ne_of_mem hx₁' hx₂' hρx
[GOAL]
X : Type u
inst✝⁶ : TopologicalSpace X
A D E : Type u
inst✝⁵ : TopologicalSpace A
inst✝⁴ : TopologicalSpace D
inst✝³ : TopologicalSpace E
inst✝² : ExtremallyDisconnected A
inst✝¹ : CompactSpace A
inst✝ : T2Space A
⊢ Projective A
[PROOFSTEP]
intro B C _ _ _ _ _ _ φ f φ_cont f_cont f_surj
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D E : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D
inst✝⁹ : TopologicalSpace E
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
let D : Set <| A × B := {x | φ x.fst = f x.snd}
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
have D_comp : CompactSpace D :=
isCompact_iff_compactSpace.mp (isClosed_eq (φ_cont.comp continuous_fst) (f_cont.comp continuous_snd)).isCompact
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
let π₁ : D → A := Prod.fst ∘ Subtype.val
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
have π₁_cont : Continuous π₁ := continuous_fst.comp continuous_subtype_val
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
have π₁_surj : π₁.Surjective := fun a => ⟨⟨⟨a, _⟩, (f_surj <| φ a).choose_spec.symm⟩, rfl⟩
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
rcases exists_compact_surjective_zorn_subset π₁_cont π₁_surj with
⟨E, _, E_onto, E_min⟩
-- apply Lemma 2.3 to get homeomorphism $\pi_1|_E : E \to A$
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
let ρ : E → A := E.restrict π₁
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
have ρ_cont : Continuous ρ := π₁_cont.continuousOn.restrict
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
have ρ_surj : ρ.Surjective := fun a => by rcases(E_onto ▸ mem_univ a : a ∈ π₁ '' E) with ⟨d, ⟨hd, rfl⟩⟩;
exact ⟨⟨d, hd⟩, rfl⟩
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
a : A
⊢ ∃ a_1, ρ a_1 = a
[PROOFSTEP]
rcases(E_onto ▸ mem_univ a : a ∈ π₁ '' E) with ⟨d, ⟨hd, rfl⟩⟩
[GOAL]
case intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
d : ↑D
hd : d ∈ E
⊢ ∃ a, ρ a = π₁ d
[PROOFSTEP]
exact ⟨⟨d, hd⟩, rfl⟩
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
let ρ' := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
let π₂ : D → B := Prod.snd ∘ Subtype.val
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
π₂ : ↑D → B := Prod.snd ∘ Subtype.val
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
have π₂_cont : Continuous π₂ := continuous_snd.comp continuous_subtype_val
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
π₂ : ↑D → B := Prod.snd ∘ Subtype.val
π₂_cont : Continuous π₂
⊢ ∃ h, Continuous h ∧ f ∘ h = φ
[PROOFSTEP]
refine ⟨E.restrict π₂ ∘ ρ'.symm, ⟨π₂_cont.continuousOn.restrict.comp ρ'.symm.continuous, ?_⟩⟩
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
π₂ : ↑D → B := Prod.snd ∘ Subtype.val
π₂_cont : Continuous π₂
⊢ f ∘ restrict E π₂ ∘ ↑(Homeomorph.symm ρ') = φ
[PROOFSTEP]
suffices f ∘ E.restrict π₂ = φ ∘ ρ' by rw [← comp.assoc, this, comp.assoc, Homeomorph.self_comp_symm, comp.right_id]
[GOAL]
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
π₂ : ↑D → B := Prod.snd ∘ Subtype.val
π₂_cont : Continuous π₂
this : f ∘ restrict E π₂ = φ ∘ ↑ρ'
⊢ f ∘ restrict E π₂ ∘ ↑(Homeomorph.symm ρ') = φ
[PROOFSTEP]
rw [← comp.assoc, this, comp.assoc, Homeomorph.self_comp_symm, comp.right_id]
[GOAL]
case intro.intro.intro
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
π₂ : ↑D → B := Prod.snd ∘ Subtype.val
π₂_cont : Continuous π₂
⊢ f ∘ restrict E π₂ = φ ∘ ↑ρ'
[PROOFSTEP]
ext x
[GOAL]
case intro.intro.intro.h
X : Type u
inst✝¹² : TopologicalSpace X
A D✝ E✝ : Type u
inst✝¹¹ : TopologicalSpace A
inst✝¹⁰ : TopologicalSpace D✝
inst✝⁹ : TopologicalSpace E✝
inst✝⁸ : ExtremallyDisconnected A
inst✝⁷ : CompactSpace A
inst✝⁶ : T2Space A
B C : Type u
inst✝⁵ : TopologicalSpace B
inst✝⁴ : TopologicalSpace C
inst✝³ : CompactSpace B
inst✝² : T2Space B
inst✝¹ : CompactSpace C
inst✝ : T2Space C
φ : A → C
f : B → C
φ_cont : Continuous φ
f_cont : Continuous f
f_surj : Surjective f
D : Set (A × B) := {x | φ x.fst = f x.snd}
D_comp : CompactSpace ↑D
π₁ : ↑D → A := Prod.fst ∘ Subtype.val
π₁_cont : Continuous π₁
π₁_surj : Surjective π₁
E : Set ↑D
left✝ : CompactSpace ↑E
E_onto : π₁ '' E = univ
E_min : ∀ (E₀ : Set ↑E), E₀ ≠ univ → IsClosed E₀ → restrict E π₁ '' E₀ ≠ univ
ρ : ↑E → A := restrict E π₁
ρ_cont : Continuous ρ
ρ_surj : Surjective ρ
ρ' : ↑E ≃ₜ A := ExtremallyDisconnected.homeoCompactToT2 ρ_cont ρ_surj E_min
π₂ : ↑D → B := Prod.snd ∘ Subtype.val
π₂_cont : Continuous π₂
x : ↑E
⊢ (f ∘ restrict E π₂) x = (φ ∘ ↑ρ') x
[PROOFSTEP]
exact x.val.mem.symm
[GOAL]
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀ : ∀ (i : ι), ExtremallyDisconnected (π i)
⊢ ExtremallyDisconnected ((i : ι) × π i)
[PROOFSTEP]
constructor
[GOAL]
case open_closure
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀ : ∀ (i : ι), ExtremallyDisconnected (π i)
⊢ ∀ (U : Set ((i : ι) × π i)), IsOpen U → IsOpen (closure U)
[PROOFSTEP]
intro s hs
[GOAL]
case open_closure
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : IsOpen s
⊢ IsOpen (closure s)
[PROOFSTEP]
rw [isOpen_sigma_iff] at hs ⊢
[GOAL]
case open_closure
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
⊢ ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' closure s)
[PROOFSTEP]
intro i
[GOAL]
case open_closure
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
⊢ IsOpen (Sigma.mk i ⁻¹' closure s)
[PROOFSTEP]
rcases h₀ i with ⟨h₀⟩
[GOAL]
case open_closure.mk
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
⊢ IsOpen (Sigma.mk i ⁻¹' closure s)
[PROOFSTEP]
have h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
[GOAL]
case h₁
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
⊢ IsOpen (closure (Sigma.mk i ⁻¹' s))
[PROOFSTEP]
apply h₀
[GOAL]
case h₁.a
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
⊢ IsOpen (Sigma.mk i ⁻¹' s)
[PROOFSTEP]
exact hs i
[GOAL]
case open_closure.mk
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
⊢ IsOpen (Sigma.mk i ⁻¹' closure s)
[PROOFSTEP]
suffices h₂ : Sigma.mk i ⁻¹' closure s = closure (Sigma.mk i ⁻¹' s)
[GOAL]
case open_closure.mk
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
h₂ : Sigma.mk i ⁻¹' closure s = closure (Sigma.mk i ⁻¹' s)
⊢ IsOpen (Sigma.mk i ⁻¹' closure s)
[PROOFSTEP]
rwa [h₂]
[GOAL]
case h₂
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
⊢ Sigma.mk i ⁻¹' closure s = closure (Sigma.mk i ⁻¹' s)
[PROOFSTEP]
apply IsOpenMap.preimage_closure_eq_closure_preimage
[GOAL]
case h₂.hf
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
⊢ IsOpenMap (Sigma.mk i)
case h₂.hfc
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
⊢ Continuous (Sigma.mk i)
[PROOFSTEP]
intro U _
[GOAL]
case h₂.hf
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
⊢ IsOpen (Sigma.mk i '' U)
[PROOFSTEP]
rw [isOpen_sigma_iff]
[GOAL]
case h₂.hf
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
⊢ ∀ (i_1 : ι), IsOpen (Sigma.mk i_1 ⁻¹' (Sigma.mk i '' U))
[PROOFSTEP]
intro j
[GOAL]
case h₂.hf
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
j : ι
⊢ IsOpen (Sigma.mk j ⁻¹' (Sigma.mk i '' U))
[PROOFSTEP]
by_cases ij : i = j
[GOAL]
case pos
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
j : ι
ij : i = j
⊢ IsOpen (Sigma.mk j ⁻¹' (Sigma.mk i '' U))
[PROOFSTEP]
rw [← ij]
[GOAL]
case pos
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
j : ι
ij : i = j
⊢ IsOpen (Sigma.mk i ⁻¹' (Sigma.mk i '' U))
[PROOFSTEP]
rw [sigma_mk_preimage_image_eq_self]
[GOAL]
case pos
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
j : ι
ij : i = j
⊢ IsOpen U
[PROOFSTEP]
assumption
[GOAL]
case neg
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
j : ι
ij : ¬i = j
⊢ IsOpen (Sigma.mk j ⁻¹' (Sigma.mk i '' U))
[PROOFSTEP]
rw [sigma_mk_preimage_image' ij]
[GOAL]
case neg
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
U : Set (π i)
a✝ : IsOpen U
j : ι
ij : ¬i = j
⊢ IsOpen ∅
[PROOFSTEP]
apply isOpen_empty
[GOAL]
case h₂.hfc
X : Type u
inst✝¹ : TopologicalSpace X
ι : Type ?u.17123
π : ι → Type u_1
inst✝ : (i : ι) → TopologicalSpace (π i)
h₀✝ : ∀ (i : ι), ExtremallyDisconnected (π i)
s : Set ((i : ι) × π i)
hs : ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
i : ι
h₀ : ∀ (U : Set (π i)), IsOpen U → IsOpen (closure U)
h₁ : IsOpen (closure (Sigma.mk i ⁻¹' s))
⊢ Continuous (Sigma.mk i)
[PROOFSTEP]
continuity
| {"mathlib_filename": "Mathlib.Topology.ExtremallyDisconnected", "llama_tokens": 41674} |
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
⊢ 𝓝 as = traverse 𝓝 as
[PROOFSTEP]
refine' nhds_mkOfNhds _ _ _ _
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
⊢ pure ≤ traverse 𝓝
[PROOFSTEP]
intro l
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as l : List α
⊢ pure l ≤ traverse 𝓝 l
[PROOFSTEP]
induction l
[GOAL]
case refine'_1.nil
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
⊢ pure [] ≤ traverse 𝓝 []
case refine'_1.cons
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
head✝ : α
tail✝ : List α
tail_ih✝ : pure tail✝ ≤ traverse 𝓝 tail✝
⊢ pure (head✝ :: tail✝) ≤ traverse 𝓝 (head✝ :: tail✝)
[PROOFSTEP]
case nil => exact le_rfl
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
⊢ pure [] ≤ traverse 𝓝 []
[PROOFSTEP]
case nil => exact le_rfl
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
⊢ pure [] ≤ traverse 𝓝 []
[PROOFSTEP]
exact le_rfl
[GOAL]
case refine'_1.cons
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
head✝ : α
tail✝ : List α
tail_ih✝ : pure tail✝ ≤ traverse 𝓝 tail✝
⊢ pure (head✝ :: tail✝) ≤ traverse 𝓝 (head✝ :: tail✝)
[PROOFSTEP]
case cons a l
ih =>
suffices List.cons <$> pure a <*> pure l ≤ List.cons <$> 𝓝 a <*> traverse 𝓝 l by simpa only [functor_norm] using this
exact Filter.seq_mono (Filter.map_mono <| pure_le_nhds a) ih
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
a : α
l : List α
ih : pure l ≤ traverse 𝓝 l
⊢ pure (a :: l) ≤ traverse 𝓝 (a :: l)
[PROOFSTEP]
case cons a l
ih =>
suffices List.cons <$> pure a <*> pure l ≤ List.cons <$> 𝓝 a <*> traverse 𝓝 l by simpa only [functor_norm] using this
exact Filter.seq_mono (Filter.map_mono <| pure_le_nhds a) ih
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
a : α
l : List α
ih : pure l ≤ traverse 𝓝 l
⊢ pure (a :: l) ≤ traverse 𝓝 (a :: l)
[PROOFSTEP]
suffices List.cons <$> pure a <*> pure l ≤ List.cons <$> 𝓝 a <*> traverse 𝓝 l by simpa only [functor_norm] using this
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
a : α
l : List α
ih : pure l ≤ traverse 𝓝 l
this : (Seq.seq (List.cons <$> pure a) fun x => pure l) ≤ Seq.seq (List.cons <$> 𝓝 a) fun x => traverse 𝓝 l
⊢ pure (a :: l) ≤ traverse 𝓝 (a :: l)
[PROOFSTEP]
simpa only [functor_norm] using this
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
a : α
l : List α
ih : pure l ≤ traverse 𝓝 l
⊢ (Seq.seq (List.cons <$> pure a) fun x => pure l) ≤ Seq.seq (List.cons <$> 𝓝 a) fun x => traverse 𝓝 l
[PROOFSTEP]
exact Filter.seq_mono (Filter.map_mono <| pure_le_nhds a) ih
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as : List α
⊢ ∀ (a : List α) (s : Set (List α)),
s ∈ traverse 𝓝 a → ∃ t, t ∈ traverse 𝓝 a ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
intro l s hs
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as l : List α
s : Set (List α)
hs : s ∈ traverse 𝓝 l
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
rcases(mem_traverse_iff _ _).1 hs with ⟨u, hu, hus⟩
[GOAL]
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
as l : List α
s : Set (List α)
hs : s ∈ traverse 𝓝 l
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
clear as hs
[GOAL]
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
have : ∃ v : List (Set α), l.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) v ∧ sequence v ⊆ s
[GOAL]
case this
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
⊢ ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v ∧ sequence v ⊆ s
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
this : ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v ∧ sequence v ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
induction hu generalizing s
[GOAL]
case this.nil
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
u : List (Set α)
s : Set (List α)
hus : sequence [] ⊆ s
⊢ ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) [] v ∧ sequence v ⊆ s
case this.cons
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
u : List (Set α)
a✝² : α
b✝ : Set α
l₁✝ : List α
l₂✝ : List (Set α)
a✝¹ : b✝ ∈ 𝓝 a✝²
a✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l₁✝ l₂✝
a_ih✝ : ∀ (s : Set (List α)), sequence l₂✝ ⊆ s → ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l₁✝ v ∧ sequence v ⊆ s
s : Set (List α)
hus : sequence (b✝ :: l₂✝) ⊆ s
⊢ ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) (a✝² :: l₁✝) v ∧ sequence v ⊆ s
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
this : ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v ∧ sequence v ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
case nil _hs =>
exists []
simp only [List.forall₂_nil_left_iff, exists_eq_left]
exact
⟨trivial, hus⟩
-- porting note -- renamed reordered variables based on previous types
[GOAL]
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
_hs : TopologicalSpace β
l : List α
u : List (Set α)
s : Set (List α)
hus : sequence [] ⊆ s
⊢ ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) [] v ∧ sequence v ⊆ s
[PROOFSTEP]
case nil _hs =>
exists []
simp only [List.forall₂_nil_left_iff, exists_eq_left]
exact
⟨trivial, hus⟩
-- porting note -- renamed reordered variables based on previous types
[GOAL]
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
_hs : TopologicalSpace β
l : List α
u : List (Set α)
s : Set (List α)
hus : sequence [] ⊆ s
⊢ ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) [] v ∧ sequence v ⊆ s
[PROOFSTEP]
exists []
[GOAL]
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
_hs : TopologicalSpace β
l : List α
u : List (Set α)
s : Set (List α)
hus : sequence [] ⊆ s
⊢ List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) [] [] ∧ sequence [] ⊆ s
[PROOFSTEP]
simp only [List.forall₂_nil_left_iff, exists_eq_left]
[GOAL]
α : Type u_1
β : Type u_2
inst✝ : TopologicalSpace α
_hs : TopologicalSpace β
l : List α
u : List (Set α)
s : Set (List α)
hus : sequence [] ⊆ s
⊢ True ∧ sequence [] ⊆ s
[PROOFSTEP]
exact
⟨trivial, hus⟩
-- porting note -- renamed reordered variables based on previous types
[GOAL]
case this.cons
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
u : List (Set α)
a✝² : α
b✝ : Set α
l₁✝ : List α
l₂✝ : List (Set α)
a✝¹ : b✝ ∈ 𝓝 a✝²
a✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l₁✝ l₂✝
a_ih✝ : ∀ (s : Set (List α)), sequence l₂✝ ⊆ s → ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l₁✝ v ∧ sequence v ⊆ s
s : Set (List α)
hus : sequence (b✝ :: l₂✝) ⊆ s
⊢ ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) (a✝² :: l₁✝) v ∧ sequence v ⊆ s
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
this : ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v ∧ sequence v ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
case cons a s as ss hts h ht _ ih =>
rcases mem_nhds_iff.1 ht with ⟨u, hut, hu⟩
rcases ih _ Subset.rfl with ⟨v, hv, hvss⟩
exact ⟨u :: v, List.Forall₂.cons hu hv, Subset.trans (Set.seq_mono (Set.image_subset _ hut) hvss) hus⟩
[GOAL]
α : Type u_1
β : Type u_2
a : TopologicalSpace α
s✝ : TopologicalSpace β
l : List α
u : List (Set α)
as : α
ss : Set α
hts : List α
h : List (Set α)
ht : ss ∈ 𝓝 as
a✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) hts h
ih : ∀ (s : Set (List α)), sequence h ⊆ s → ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) hts v ∧ sequence v ⊆ s
s : Set (List α)
hus : sequence (ss :: h) ⊆ s
⊢ ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) (as :: hts) v ∧ sequence v ⊆ s
[PROOFSTEP]
case cons a s as ss hts h ht _ ih =>
rcases mem_nhds_iff.1 ht with ⟨u, hut, hu⟩
rcases ih _ Subset.rfl with ⟨v, hv, hvss⟩
exact ⟨u :: v, List.Forall₂.cons hu hv, Subset.trans (Set.seq_mono (Set.image_subset _ hut) hvss) hus⟩
[GOAL]
α : Type u_1
β : Type u_2
a : TopologicalSpace α
s✝ : TopologicalSpace β
l : List α
u : List (Set α)
as : α
ss : Set α
hts : List α
h : List (Set α)
ht : ss ∈ 𝓝 as
a✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) hts h
ih : ∀ (s : Set (List α)), sequence h ⊆ s → ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) hts v ∧ sequence v ⊆ s
s : Set (List α)
hus : sequence (ss :: h) ⊆ s
⊢ ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) (as :: hts) v ∧ sequence v ⊆ s
[PROOFSTEP]
rcases mem_nhds_iff.1 ht with ⟨u, hut, hu⟩
[GOAL]
case intro.intro
α : Type u_1
β : Type u_2
a : TopologicalSpace α
s✝ : TopologicalSpace β
l : List α
u✝ : List (Set α)
as : α
ss : Set α
hts : List α
h : List (Set α)
ht : ss ∈ 𝓝 as
a✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) hts h
ih : ∀ (s : Set (List α)), sequence h ⊆ s → ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) hts v ∧ sequence v ⊆ s
s : Set (List α)
hus : sequence (ss :: h) ⊆ s
u : Set α
hut : u ⊆ ss
hu : IsOpen u ∧ as ∈ u
⊢ ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) (as :: hts) v ∧ sequence v ⊆ s
[PROOFSTEP]
rcases ih _ Subset.rfl with ⟨v, hv, hvss⟩
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
a : TopologicalSpace α
s✝ : TopologicalSpace β
l : List α
u✝ : List (Set α)
as : α
ss : Set α
hts : List α
h : List (Set α)
ht : ss ∈ 𝓝 as
a✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) hts h
ih : ∀ (s : Set (List α)), sequence h ⊆ s → ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) hts v ∧ sequence v ⊆ s
s : Set (List α)
hus : sequence (ss :: h) ⊆ s
u : Set α
hut : u ⊆ ss
hu : IsOpen u ∧ as ∈ u
v : List (Set α)
hv : List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) hts v
hvss : sequence v ⊆ sequence h
⊢ ∃ v, List.Forall₂ (fun a_1 s => IsOpen s ∧ a_1 ∈ s) (as :: hts) v ∧ sequence v ⊆ s
[PROOFSTEP]
exact ⟨u :: v, List.Forall₂.cons hu hv, Subset.trans (Set.seq_mono (Set.image_subset _ hut) hvss) hus⟩
[GOAL]
case refine'_2.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
this : ∃ v, List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v ∧ sequence v ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
rcases this with ⟨v, hv, hvs⟩
[GOAL]
case refine'_2.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
⊢ ∃ t, t ∈ traverse 𝓝 l ∧ t ⊆ s ∧ ∀ (a' : List α), a' ∈ t → s ∈ traverse 𝓝 a'
[PROOFSTEP]
refine' ⟨sequence v, mem_traverse _ _ _, hvs, _⟩
[GOAL]
case refine'_2.intro.intro.intro.intro.refine'_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
⊢ List.Forall₂ (fun b c => id c ∈ 𝓝 b) l v
[PROOFSTEP]
exact hv.imp fun a s ⟨hs, ha⟩ => IsOpen.mem_nhds hs ha
[GOAL]
case refine'_2.intro.intro.intro.intro.refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u : List (Set α)
hu : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u
hus : sequence u ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
⊢ ∀ (a' : List α), a' ∈ sequence v → s ∈ traverse 𝓝 a'
[PROOFSTEP]
intro u hu
[GOAL]
case refine'_2.intro.intro.intro.intro.refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
u : List α
hu : u ∈ sequence v
⊢ s ∈ traverse 𝓝 u
[PROOFSTEP]
have hu := (List.mem_traverse _ _).1 hu
[GOAL]
case refine'_2.intro.intro.intro.intro.refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
⊢ s ∈ traverse 𝓝 u
[PROOFSTEP]
have : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) u v :=
by
refine' List.Forall₂.flip _
replace hv := hv.flip
simp only [List.forall₂_and_left, flip] at hv ⊢
exact ⟨hv.1, hu.flip⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
⊢ List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) u v
[PROOFSTEP]
refine' List.Forall₂.flip _
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
⊢ List.Forall₂ (flip fun a s => IsOpen s ∧ a ∈ s) v u
[PROOFSTEP]
replace hv := hv.flip
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
hv : List.Forall₂ (fun s a => IsOpen s ∧ a ∈ s) v l
⊢ List.Forall₂ (flip fun a s => IsOpen s ∧ a ∈ s) v u
[PROOFSTEP]
simp only [List.forall₂_and_left, flip] at hv ⊢
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
hv : (∀ (a : Set α), a ∈ v → IsOpen a) ∧ List.Forall₂ (fun a b => b ∈ a) v l
⊢ (∀ (a : Set α), a ∈ v → IsOpen a) ∧ List.Forall₂ (fun a b => b ∈ a) v u
[PROOFSTEP]
exact ⟨hv.1, hu.flip⟩
[GOAL]
case refine'_2.intro.intro.intro.intro.refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
this : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) u v
⊢ s ∈ traverse 𝓝 u
[PROOFSTEP]
refine' mem_of_superset _ hvs
[GOAL]
case refine'_2.intro.intro.intro.intro.refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
s : Set (List α)
u✝ : List (Set α)
hu✝¹ : List.Forall₂ (fun b s => s ∈ 𝓝 b) l u✝
hus : sequence u✝ ⊆ s
v : List (Set α)
hv : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) l v
hvs : sequence v ⊆ s
u : List α
hu✝ : u ∈ sequence v
hu : List.Forall₂ (fun b a => b ∈ id a) u v
this : List.Forall₂ (fun a s => IsOpen s ∧ a ∈ s) u v
⊢ sequence v ∈ traverse 𝓝 u
[PROOFSTEP]
exact mem_traverse _ _ (this.imp fun a s ⟨hs, ha⟩ => IsOpen.mem_nhds hs ha)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ 𝓝 [] = pure []
[PROOFSTEP]
rw [nhds_list, List.traverse_nil _]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
l : List α
⊢ 𝓝 (a :: l) = Seq.seq (List.cons <$> 𝓝 a) fun x => 𝓝 l
[PROOFSTEP]
rw [nhds_list, List.traverse_cons _, ← nhds_list]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
l : List α
⊢ Tendsto (fun p => p.fst :: p.snd) (𝓝 a ×ˢ 𝓝 l) (𝓝 (a :: l))
[PROOFSTEP]
rw [nhds_cons, Tendsto, Filter.map_prod]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
l : List α
⊢ Filter.seq (Filter.map (fun a b => (a, b).fst :: (a, b).snd) (𝓝 a)) (𝓝 l) ≤ Seq.seq (cons <$> 𝓝 a) fun x => 𝓝 l
[PROOFSTEP]
exact le_rfl
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
b : Filter β
a : α
l : List α
⊢ Tendsto f (𝓝 (a :: l)) b ↔ Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) b
[PROOFSTEP]
have : 𝓝 (a :: l) = (𝓝 a ×ˢ 𝓝 l).map fun p : α × List α => p.1 :: p.2 :=
by
simp only [nhds_cons, Filter.prod_eq, (Filter.map_def _ _).symm, (Filter.seq_eq_filter_seq _ _).symm]
simp [-Filter.map_def, (· ∘ ·), functor_norm]
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
b : Filter β
a : α
l : List α
⊢ 𝓝 (a :: l) = Filter.map (fun p => p.fst :: p.snd) (𝓝 a ×ˢ 𝓝 l)
[PROOFSTEP]
simp only [nhds_cons, Filter.prod_eq, (Filter.map_def _ _).symm, (Filter.seq_eq_filter_seq _ _).symm]
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
b : Filter β
a : α
l : List α
⊢ (Seq.seq (cons <$> 𝓝 a) fun x => 𝓝 l) = (fun p => p.fst :: p.snd) <$> Seq.seq (Prod.mk <$> 𝓝 a) fun x => 𝓝 l
[PROOFSTEP]
simp [-Filter.map_def, (· ∘ ·), functor_norm]
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
b : Filter β
a : α
l : List α
this : 𝓝 (a :: l) = Filter.map (fun p => p.fst :: p.snd) (𝓝 a ×ˢ 𝓝 l)
⊢ Tendsto f (𝓝 (a :: l)) b ↔ Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) b
[PROOFSTEP]
rw [this, Filter.tendsto_map'_iff]
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
b : Filter β
a : α
l : List α
this : 𝓝 (a :: l) = Filter.map (fun p => p.fst :: p.snd) (𝓝 a ×ˢ 𝓝 l)
⊢ Tendsto (f ∘ fun p => p.fst :: p.snd) (𝓝 a ×ˢ 𝓝 l) b ↔ Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) b
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
r : List α → Filter β
h_nil : Tendsto f (pure []) (r [])
h_cons : ∀ (l : List α) (a : α), Tendsto f (𝓝 l) (r l) → Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) (r (a :: l))
⊢ Tendsto f (𝓝 []) (r [])
[PROOFSTEP]
rwa [nhds_nil]
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
r : List α → Filter β
h_nil : Tendsto f (pure []) (r [])
h_cons : ∀ (l : List α) (a : α), Tendsto f (𝓝 l) (r l) → Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) (r (a :: l))
a : α
l : List α
⊢ Tendsto f (𝓝 (a :: l)) (r (a :: l))
[PROOFSTEP]
rw [tendsto_cons_iff]
[GOAL]
α : Type u_1
β✝ : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
β : Type u_3
f : List α → β
r : List α → Filter β
h_nil : Tendsto f (pure []) (r [])
h_cons : ∀ (l : List α) (a : α), Tendsto f (𝓝 l) (r l) → Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) (r (a :: l))
a : α
l : List α
⊢ Tendsto (fun p => f (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) (r (a :: l))
[PROOFSTEP]
exact h_cons l a (@tendsto_nhds _ _ _ h_nil h_cons l)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ ∀ (l : List α), ContinuousAt length l
[PROOFSTEP]
simp only [ContinuousAt, nhds_discrete]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ ∀ (l : List α), Tendsto length (𝓝 l) (pure (length l))
[PROOFSTEP]
refine' tendsto_nhds _ _
[GOAL]
case refine'_1
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ Tendsto length (pure []) (pure (length []))
[PROOFSTEP]
exact tendsto_pure_pure _ _
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ ∀ (l : List α) (a : α),
Tendsto length (𝓝 l) (pure (length l)) →
Tendsto (fun p => length (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) (pure (length (a :: l)))
[PROOFSTEP]
intro l a ih
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
a : α
ih : Tendsto length (𝓝 l) (pure (length l))
⊢ Tendsto (fun p => length (p.fst :: p.snd)) (𝓝 a ×ˢ 𝓝 l) (pure (length (a :: l)))
[PROOFSTEP]
dsimp only [List.length]
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
a : α
ih : Tendsto length (𝓝 l) (pure (length l))
⊢ Tendsto (fun p => length p.snd + 1) (𝓝 a ×ˢ 𝓝 l) (pure (length l + 1))
[PROOFSTEP]
refine' Tendsto.comp (tendsto_pure_pure (fun x => x + 1) _) _
[GOAL]
case refine'_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
l : List α
a : α
ih : Tendsto length (𝓝 l) (pure (length l))
⊢ Tendsto (fun p => Nat.add (length p.snd) 0) (𝓝 a ×ˢ 𝓝 l) (pure (length l))
[PROOFSTEP]
refine' Tendsto.comp ih tendsto_snd
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
n : ℕ
⊢ Tendsto (fun p => insertNth (n + 1) p.fst p.snd) (𝓝 a ×ˢ 𝓝 []) (𝓝 (insertNth (n + 1) a []))
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
n : ℕ
a' : α
l : List α
⊢ Tendsto (fun p => insertNth (n + 1) p.fst p.snd) (𝓝 a ×ˢ 𝓝 (a' :: l)) (𝓝 (insertNth (n + 1) a (a' :: l)))
[PROOFSTEP]
have : 𝓝 a ×ˢ 𝓝 (a' :: l) = (𝓝 a ×ˢ (𝓝 a' ×ˢ 𝓝 l)).map fun p : α × α × List α => (p.1, p.2.1 :: p.2.2) :=
by
simp only [nhds_cons, Filter.prod_eq, ← Filter.map_def, ← Filter.seq_eq_filter_seq]
simp [-Filter.map_def, (· ∘ ·), functor_norm]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
n : ℕ
a' : α
l : List α
⊢ 𝓝 a ×ˢ 𝓝 (a' :: l) = Filter.map (fun p => (p.fst, p.snd.fst :: p.snd.snd)) (𝓝 a ×ˢ 𝓝 a' ×ˢ 𝓝 l)
[PROOFSTEP]
simp only [nhds_cons, Filter.prod_eq, ← Filter.map_def, ← Filter.seq_eq_filter_seq]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
n : ℕ
a' : α
l : List α
⊢ (Seq.seq (Prod.mk <$> 𝓝 a) fun x => Seq.seq (cons <$> 𝓝 a') fun x => 𝓝 l) =
(fun p => (p.fst, p.snd.fst :: p.snd.snd)) <$>
Seq.seq (Prod.mk <$> 𝓝 a) fun x => Seq.seq (Prod.mk <$> 𝓝 a') fun x => 𝓝 l
[PROOFSTEP]
simp [-Filter.map_def, (· ∘ ·), functor_norm]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
n : ℕ
a' : α
l : List α
this : 𝓝 a ×ˢ 𝓝 (a' :: l) = Filter.map (fun p => (p.fst, p.snd.fst :: p.snd.snd)) (𝓝 a ×ˢ 𝓝 a' ×ˢ 𝓝 l)
⊢ Tendsto (fun p => insertNth (n + 1) p.fst p.snd) (𝓝 a ×ˢ 𝓝 (a' :: l)) (𝓝 (insertNth (n + 1) a (a' :: l)))
[PROOFSTEP]
rw [this, tendsto_map'_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
n : ℕ
a' : α
l : List α
this : 𝓝 a ×ˢ 𝓝 (a' :: l) = Filter.map (fun p => (p.fst, p.snd.fst :: p.snd.snd)) (𝓝 a ×ˢ 𝓝 a' ×ˢ 𝓝 l)
⊢ Tendsto ((fun p => insertNth (n + 1) p.fst p.snd) ∘ fun p => (p.fst, p.snd.fst :: p.snd.snd)) (𝓝 a ×ˢ 𝓝 a' ×ˢ 𝓝 l)
(𝓝 (insertNth (n + 1) a (a' :: l)))
[PROOFSTEP]
exact
(tendsto_fst.comp tendsto_snd).cons
((@tendsto_insertNth' _ n l).comp <| tendsto_fst.prod_mk <| tendsto_snd.comp tendsto_snd)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
x✝ : α × List α
a : α
l : List α
⊢ ContinuousAt (fun p => insertNth n p.fst p.snd) (a, l)
[PROOFSTEP]
rw [ContinuousAt, nhds_prod_eq]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
x✝ : α × List α
a : α
l : List α
⊢ Tendsto (fun p => insertNth n p.fst p.snd) (𝓝 a ×ˢ 𝓝 l) (𝓝 (insertNth n (a, l).fst (a, l).snd))
[PROOFSTEP]
exact tendsto_insertNth'
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x✝ : ℕ
⊢ Tendsto (fun l => removeNth l x✝) (𝓝 []) (𝓝 (removeNth [] x✝))
[PROOFSTEP]
rw [nhds_nil]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
x✝ : ℕ
⊢ Tendsto (fun l => removeNth l x✝) (pure []) (𝓝 (removeNth [] x✝))
[PROOFSTEP]
exact tendsto_pure_nhds _ _
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
l : List α
⊢ Tendsto (fun l => removeNth l 0) (𝓝 (a :: l)) (𝓝 (removeNth (a :: l) 0))
[PROOFSTEP]
rw [tendsto_cons_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
a : α
l : List α
⊢ Tendsto (fun p => removeNth (p.fst :: p.snd) 0) (𝓝 a ×ˢ 𝓝 l) (𝓝 (removeNth (a :: l) 0))
[PROOFSTEP]
exact tendsto_snd
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
a : α
l : List α
⊢ Tendsto (fun l => removeNth l (n + 1)) (𝓝 (a :: l)) (𝓝 (removeNth (a :: l) (n + 1)))
[PROOFSTEP]
rw [tendsto_cons_iff]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
a : α
l : List α
⊢ Tendsto (fun p => removeNth (p.fst :: p.snd) (n + 1)) (𝓝 a ×ˢ 𝓝 l) (𝓝 (removeNth (a :: l) (n + 1)))
[PROOFSTEP]
dsimp [removeNth]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
a : α
l : List α
⊢ Tendsto (fun p => p.fst :: removeNth p.snd n) (𝓝 a ×ˢ 𝓝 l) (𝓝 (a :: removeNth l n))
[PROOFSTEP]
exact tendsto_fst.cons ((@tendsto_removeNth n l).comp tendsto_snd)
[GOAL]
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : Monoid α
inst✝ : ContinuousMul α
l : List α
⊢ Tendsto prod (𝓝 l) (𝓝 (prod l))
[PROOFSTEP]
induction' l with x l ih
[GOAL]
case nil
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : Monoid α
inst✝ : ContinuousMul α
⊢ Tendsto prod (𝓝 []) (𝓝 (prod []))
[PROOFSTEP]
simp (config := { contextual := true }) [nhds_nil, mem_of_mem_nhds, tendsto_pure_left]
[GOAL]
case cons
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : Monoid α
inst✝ : ContinuousMul α
x : α
l : List α
ih : Tendsto prod (𝓝 l) (𝓝 (prod l))
⊢ Tendsto prod (𝓝 (x :: l)) (𝓝 (prod (x :: l)))
[PROOFSTEP]
simp_rw [tendsto_cons_iff, prod_cons]
[GOAL]
case cons
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : Monoid α
inst✝ : ContinuousMul α
x : α
l : List α
ih : Tendsto prod (𝓝 l) (𝓝 (prod l))
⊢ Tendsto (fun p => p.fst * prod p.snd) (𝓝 x ×ˢ 𝓝 l) (𝓝 (x * prod l))
[PROOFSTEP]
have := continuous_iff_continuousAt.mp continuous_mul (x, l.prod)
[GOAL]
case cons
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : Monoid α
inst✝ : ContinuousMul α
x : α
l : List α
ih : Tendsto prod (𝓝 l) (𝓝 (prod l))
this : ContinuousAt (fun p => p.fst * p.snd) (x, prod l)
⊢ Tendsto (fun p => p.fst * prod p.snd) (𝓝 x ×ˢ 𝓝 l) (𝓝 (x * prod l))
[PROOFSTEP]
rw [ContinuousAt, nhds_prod_eq] at this
[GOAL]
case cons
α : Type u_1
β : Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : Monoid α
inst✝ : ContinuousMul α
x : α
l : List α
ih : Tendsto prod (𝓝 l) (𝓝 (prod l))
this : Tendsto (fun p => p.fst * p.snd) (𝓝 x ×ˢ 𝓝 (prod l)) (𝓝 ((x, prod l).fst * (x, prod l).snd))
⊢ Tendsto (fun p => p.fst * prod p.snd) (𝓝 x ×ˢ 𝓝 l) (𝓝 (x * prod l))
[PROOFSTEP]
exact this.comp (tendsto_id.prod_map ih)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
⊢ TopologicalSpace (Vector α n)
[PROOFSTEP]
unfold Vector
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
⊢ TopologicalSpace { l // List.length l = n }
[PROOFSTEP]
infer_instance
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
a : α
l : Vector α n
⊢ Tendsto (fun p => p.fst ::ᵥ p.snd) (𝓝 a ×ˢ 𝓝 l) (𝓝 (a ::ᵥ l))
[PROOFSTEP]
rw [tendsto_subtype_rng, cons_val]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
a : α
l : Vector α n
⊢ Tendsto (fun x => ↑(x.fst ::ᵥ x.snd)) (𝓝 a ×ˢ 𝓝 l) (𝓝 (a :: ↑l))
[PROOFSTEP]
exact tendsto_fst.cons (Tendsto.comp continuousAt_subtype_val tendsto_snd)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
a : α
l : List α
hl : List.length l = n
⊢ Tendsto (fun p => insertNth p.fst i p.snd) (𝓝 a ×ˢ 𝓝 { val := l, property := hl })
(𝓝 (insertNth a i { val := l, property := hl }))
[PROOFSTEP]
rw [insertNth, tendsto_subtype_rng]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
a : α
l : List α
hl : List.length l = n
⊢ Tendsto (fun x => ↑(insertNth x.fst i x.snd)) (𝓝 a ×ˢ 𝓝 { val := l, property := hl })
(𝓝
↑{ val := List.insertNth (↑i) a ↑{ val := l, property := hl },
property := (_ : List.length (List.insertNth (↑i) a ↑{ val := l, property := hl }) = n + 1) })
[PROOFSTEP]
simp [insertNth_val]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
a : α
l : List α
hl : List.length l = n
⊢ Tendsto (fun x => List.insertNth (↑i) x.fst ↑x.snd) (𝓝 a ×ˢ 𝓝 { val := l, property := hl })
(𝓝 (List.insertNth (↑i) a l))
[PROOFSTEP]
exact List.tendsto_insertNth tendsto_fst (Tendsto.comp continuousAt_subtype_val tendsto_snd : _)
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
x✝ : α × Vector α n
a : α
l : Vector α n
⊢ ContinuousAt (fun p => insertNth p.fst i p.snd) (a, l)
[PROOFSTEP]
rw [ContinuousAt, nhds_prod_eq]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
x✝ : α × Vector α n
a : α
l : Vector α n
⊢ Tendsto (fun p => insertNth p.fst i p.snd) (𝓝 a ×ˢ 𝓝 l) (𝓝 (insertNth (a, l).fst i (a, l).snd))
[PROOFSTEP]
exact tendsto_insertNth
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
l : List α
hl : List.length l = n + 1
⊢ ContinuousAt (removeNth i) { val := l, property := hl }
[PROOFSTEP]
rw [ContinuousAt, removeNth, tendsto_subtype_rng]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
l : List α
hl : List.length l = n + 1
⊢ Tendsto (fun x => ↑(removeNth i x)) (𝓝 { val := l, property := hl })
(𝓝
↑(match { val := l, property := hl } with
| { val := l, property := p } =>
{ val := List.removeNth l ↑i, property := (_ : List.length (List.removeNth l ↑i) = n + 1 - 1) }))
[PROOFSTEP]
simp only [Vector.removeNth_val]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
n : ℕ
i : Fin (n + 1)
l : List α
hl : List.length l = n + 1
⊢ Tendsto (fun x => List.removeNth ↑x ↑i) (𝓝 { val := l, property := hl }) (𝓝 (List.removeNth l ↑i))
[PROOFSTEP]
exact Tendsto.comp List.tendsto_removeNth continuousAt_subtype_val
| {"mathlib_filename": "Mathlib.Topology.List", "llama_tokens": 15851} |
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
⊢ IsPreconnected s
[PROOFSTEP]
rintro u v hu hv hs ⟨z, zs, zu⟩ ⟨y, ys, yv⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have xs : x ∈ s := by
rcases H y ys with ⟨t, ts, xt, -, -⟩
exact ts xt
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
⊢ x ∈ s
[PROOFSTEP]
rcases H y ys with ⟨t, ts, xt, -, -⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
t : Set α
ts : t ⊆ s
xt : x ∈ t
⊢ x ∈ s
[PROOFSTEP]
exact ts xt
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
cases hs xs
[GOAL]
case intro.intro.intro.intro.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
h✝ : x ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
case intro.intro.intro.intro.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
h✝ : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
case inl xu =>
rcases H y ys with ⟨t, ts, xt, yt, ht⟩
have := ht u v hu hv (ts.trans hs) ⟨x, xt, xu⟩ ⟨y, yt, yv⟩
exact this.imp fun z hz => ⟨ts hz.1, hz.2⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xu : x ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
case inl xu =>
rcases H y ys with ⟨t, ts, xt, yt, ht⟩
have := ht u v hu hv (ts.trans hs) ⟨x, xt, xu⟩ ⟨y, yt, yv⟩
exact this.imp fun z hz => ⟨ts hz.1, hz.2⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xu : x ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases H y ys with ⟨t, ts, xt, yt, ht⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xu : x ∈ u
t : Set α
ts : t ⊆ s
xt : x ∈ t
yt : y ∈ t
ht : IsPreconnected t
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have := ht u v hu hv (ts.trans hs) ⟨x, xt, xu⟩ ⟨y, yt, yv⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xu : x ∈ u
t : Set α
ts : t ⊆ s
xt : x ∈ t
yt : y ∈ t
ht : IsPreconnected t
this : Set.Nonempty (t ∩ (u ∩ v))
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact this.imp fun z hz => ⟨ts hz.1, hz.2⟩
[GOAL]
case intro.intro.intro.intro.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
h✝ : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
case inr xv =>
rcases H z zs with ⟨t, ts, xt, zt, ht⟩
have := ht v u hv hu (ts.trans <| by rwa [union_comm]) ⟨x, xt, xv⟩ ⟨z, zt, zu⟩
exact this.imp fun _ h => ⟨ts h.1, h.2.2, h.2.1⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xv : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
case inr xv =>
rcases H z zs with ⟨t, ts, xt, zt, ht⟩
have := ht v u hv hu (ts.trans <| by rwa [union_comm]) ⟨x, xt, xv⟩ ⟨z, zt, zu⟩
exact this.imp fun _ h => ⟨ts h.1, h.2.2, h.2.1⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xv : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases H z zs with ⟨t, ts, xt, zt, ht⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xv : x ∈ v
t : Set α
ts : t ⊆ s
xt : x ∈ t
zt : z ∈ t
ht : IsPreconnected t
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have := ht v u hv hu (ts.trans <| by rwa [union_comm]) ⟨x, xt, xv⟩ ⟨z, zt, zu⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xv : x ∈ v
t : Set α
ts : t ⊆ s
xt : x ∈ t
zt : z ∈ t
ht : IsPreconnected t
⊢ s ⊆ v ∪ u
[PROOFSTEP]
rwa [union_comm]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
x : α
H : ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
z : α
zs : z ∈ s
zu : z ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
xs : x ∈ s
xv : x ∈ v
t : Set α
ts : t ⊆ s
xt : x ∈ t
zt : z ∈ t
ht : IsPreconnected t
this : Set.Nonempty (t ∩ (v ∩ u))
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact this.imp fun _ h => ⟨ts h.1, h.2.2, h.2.1⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
H : ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
⊢ IsPreconnected s
[PROOFSTEP]
rcases eq_empty_or_nonempty s with (rfl | ⟨x, hx⟩)
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
H : ∀ (x : α), x ∈ ∅ → ∀ (y : α), y ∈ ∅ → ∃ t, t ⊆ ∅ ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
⊢ IsPreconnected ∅
case inr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
H : ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → ∃ t, t ⊆ s ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
x : α
hx : x ∈ s
⊢ IsPreconnected s
[PROOFSTEP]
exacts [isPreconnected_empty, isPreconnected_of_forall x fun y => H x hx y]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
c : Set (Set α)
H1 : ∀ (s : Set α), s ∈ c → x ∈ s
H2 : ∀ (s : Set α), s ∈ c → IsPreconnected s
⊢ IsPreconnected (⋃₀ c)
[PROOFSTEP]
apply isPreconnected_of_forall x
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
c : Set (Set α)
H1 : ∀ (s : Set α), s ∈ c → x ∈ s
H2 : ∀ (s : Set α), s ∈ c → IsPreconnected s
⊢ ∀ (y : α), y ∈ ⋃₀ c → ∃ t, t ⊆ ⋃₀ c ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
[PROOFSTEP]
rintro y ⟨s, sc, ys⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v : Set α
x : α
c : Set (Set α)
H1 : ∀ (s : Set α), s ∈ c → x ∈ s
H2 : ∀ (s : Set α), s ∈ c → IsPreconnected s
y : α
s : Set α
sc : s ∈ c
ys : y ∈ s
⊢ ∃ t, t ⊆ ⋃₀ c ∧ x ∈ t ∧ y ∈ t ∧ IsPreconnected t
[PROOFSTEP]
exact ⟨s, subset_sUnion_of_mem sc, H1 s sc, ys, H2 s sc⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
x : α
s t : Set α
H1 : x ∈ s
H2 : x ∈ t
H3 : IsPreconnected s
H4 : IsPreconnected t
⊢ ∀ (s_1 : Set α), s_1 ∈ {s, t} → x ∈ s_1
[PROOFSTEP]
rintro r (rfl | rfl | h)
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t✝ u v : Set α
x : α
t : Set α
H2 : x ∈ t
H4 : IsPreconnected t
r : Set α
H1 : x ∈ r
H3 : IsPreconnected r
⊢ x ∈ r
[PROOFSTEP]
assumption
[GOAL]
case inr.refl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
x : α
s t : Set α
H1 : x ∈ s
H2 : x ∈ t
H3 : IsPreconnected s
H4 : IsPreconnected t
⊢ x ∈ t
[PROOFSTEP]
assumption
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
x : α
s t : Set α
H1 : x ∈ s
H2 : x ∈ t
H3 : IsPreconnected s
H4 : IsPreconnected t
⊢ ∀ (s_1 : Set α), s_1 ∈ {s, t} → IsPreconnected s_1
[PROOFSTEP]
rintro r (rfl | rfl | h)
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t✝ u v : Set α
x : α
t : Set α
H2 : x ∈ t
H4 : IsPreconnected t
r : Set α
H1 : x ∈ r
H3 : IsPreconnected r
⊢ IsPreconnected r
[PROOFSTEP]
assumption
[GOAL]
case inr.refl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
x : α
s t : Set α
H1 : x ∈ s
H2 : x ∈ t
H3 : IsPreconnected s
H4 : IsPreconnected t
⊢ IsPreconnected t
[PROOFSTEP]
assumption
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s t : Set α
H : Set.Nonempty (s ∩ t)
hs : IsPreconnected s
ht : IsPreconnected t
⊢ IsPreconnected (s ∪ t)
[PROOFSTEP]
rcases H with ⟨x, hxs, hxt⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s t : Set α
hs : IsPreconnected s
ht : IsPreconnected t
x : α
hxs : x ∈ s
hxt : x ∈ t
⊢ IsPreconnected (s ∪ t)
[PROOFSTEP]
exact hs.union x hxs hxt ht
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s t : Set α
H : Set.Nonempty (s ∩ t)
Hs : IsConnected s
Ht : IsConnected t
⊢ IsConnected (s ∪ t)
[PROOFSTEP]
rcases H with ⟨x, hx⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s t : Set α
Hs : IsConnected s
Ht : IsConnected t
x : α
hx : x ∈ s ∩ t
⊢ IsConnected (s ∪ t)
[PROOFSTEP]
refine' ⟨⟨x, mem_union_left t (mem_of_mem_inter_left hx)⟩, _⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s t : Set α
Hs : IsConnected s
Ht : IsConnected t
x : α
hx : x ∈ s ∩ t
⊢ IsPreconnected (s ∪ t)
[PROOFSTEP]
exact Hs.isPreconnected.union x (mem_of_mem_inter_left hx) (mem_of_mem_inter_right hx) Ht.isPreconnected
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
S : Set (Set α)
K : DirectedOn (fun x x_1 => x ⊆ x_1) S
H : ∀ (s : Set α), s ∈ S → IsPreconnected s
⊢ IsPreconnected (⋃₀ S)
[PROOFSTEP]
rintro u v hu hv Huv ⟨a, ⟨s, hsS, has⟩, hau⟩ ⟨b, ⟨t, htS, hbt⟩, hbv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ : Set α
S : Set (Set α)
K : DirectedOn (fun x x_1 => x ⊆ x_1) S
H : ∀ (s : Set α), s ∈ S → IsPreconnected s
u v : Set α
hu : IsOpen u
hv : IsOpen v
Huv : ⋃₀ S ⊆ u ∪ v
a : α
hau : a ∈ u
s : Set α
hsS : s ∈ S
has : a ∈ s
b : α
hbv : b ∈ v
t : Set α
htS : t ∈ S
hbt : b ∈ t
⊢ Set.Nonempty (⋃₀ S ∩ (u ∩ v))
[PROOFSTEP]
obtain ⟨r, hrS, hsr, htr⟩ : ∃ r ∈ S, s ⊆ r ∧ t ⊆ r := K s hsS t htS
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ : Set α
S : Set (Set α)
K : DirectedOn (fun x x_1 => x ⊆ x_1) S
H : ∀ (s : Set α), s ∈ S → IsPreconnected s
u v : Set α
hu : IsOpen u
hv : IsOpen v
Huv : ⋃₀ S ⊆ u ∪ v
a : α
hau : a ∈ u
s : Set α
hsS : s ∈ S
has : a ∈ s
b : α
hbv : b ∈ v
t : Set α
htS : t ∈ S
hbt : b ∈ t
r : Set α
hrS : r ∈ S
hsr : s ⊆ r
htr : t ⊆ r
⊢ Set.Nonempty (⋃₀ S ∩ (u ∩ v))
[PROOFSTEP]
have Hnuv : (r ∩ (u ∩ v)).Nonempty :=
H _ hrS u v hu hv ((subset_sUnion_of_mem hrS).trans Huv) ⟨a, hsr has, hau⟩ ⟨b, htr hbt, hbv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ : Set α
S : Set (Set α)
K : DirectedOn (fun x x_1 => x ⊆ x_1) S
H : ∀ (s : Set α), s ∈ S → IsPreconnected s
u v : Set α
hu : IsOpen u
hv : IsOpen v
Huv : ⋃₀ S ⊆ u ∪ v
a : α
hau : a ∈ u
s : Set α
hsS : s ∈ S
has : a ∈ s
b : α
hbv : b ∈ v
t : Set α
htS : t ∈ S
hbt : b ∈ t
r : Set α
hrS : r ∈ S
hsr : s ⊆ r
htr : t ⊆ r
Hnuv : Set.Nonempty (r ∩ (u ∩ v))
⊢ Set.Nonempty (⋃₀ S ∩ (u ∩ v))
[PROOFSTEP]
have Kruv : r ∩ (u ∩ v) ⊆ ⋃₀ S ∩ (u ∩ v) := inter_subset_inter_left _ (subset_sUnion_of_mem hrS)
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ : Set α
S : Set (Set α)
K : DirectedOn (fun x x_1 => x ⊆ x_1) S
H : ∀ (s : Set α), s ∈ S → IsPreconnected s
u v : Set α
hu : IsOpen u
hv : IsOpen v
Huv : ⋃₀ S ⊆ u ∪ v
a : α
hau : a ∈ u
s : Set α
hsS : s ∈ S
has : a ∈ s
b : α
hbv : b ∈ v
t : Set α
htS : t ∈ S
hbt : b ∈ t
r : Set α
hrS : r ∈ S
hsr : s ⊆ r
htr : t ⊆ r
Hnuv : Set.Nonempty (r ∩ (u ∩ v))
Kruv : r ∩ (u ∩ v) ⊆ ⋃₀ S ∩ (u ∩ v)
⊢ Set.Nonempty (⋃₀ S ∩ (u ∩ v))
[PROOFSTEP]
exact Hnuv.mono Kruv
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
⊢ IsPreconnected (⋃ (n : ι) (_ : n ∈ t), s n)
[PROOFSTEP]
let R := fun i j : ι => (s i ∩ s j).Nonempty ∧ i ∈ t
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
⊢ IsPreconnected (⋃ (n : ι) (_ : n ∈ t), s n)
[PROOFSTEP]
have P : ∀ i, i ∈ t → ∀ j, j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ j ∈ p, s j) :=
fun i hi j hj h => by
induction h
case refl =>
refine ⟨{ i }, singleton_subset_iff.mpr hi, mem_singleton i, mem_singleton i, ?_⟩
rw [biUnion_singleton]
exact H i hi
case tail j k _ hjk ih =>
obtain ⟨p, hpt, hip, hjp, hp⟩ := ih hjk.2
refine ⟨insert k p, insert_subset_iff.mpr ⟨hj, hpt⟩, mem_insert_of_mem k hip, mem_insert k p, ?_⟩
rw [biUnion_insert]
refine (H k hj).union' (hjk.1.mono ?_) hp
rw [inter_comm]
exact inter_subset_inter_right _ (subset_biUnion_of_mem hjp)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j : ι
hj : j ∈ t
h : ReflTransGen R i j
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
induction h
[GOAL]
case refl
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j : ι
hj : i ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ i ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
case tail
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j b✝ c✝ : ι
a✝¹ : ReflTransGen R i b✝
a✝ : R b✝ c✝
a_ih✝ : b✝ ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ b✝ ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : c✝ ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ c✝ ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
case refl =>
refine ⟨{ i }, singleton_subset_iff.mpr hi, mem_singleton i, mem_singleton i, ?_⟩
rw [biUnion_singleton]
exact H i hi
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j : ι
hj : i ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ i ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
case refl =>
refine ⟨{ i }, singleton_subset_iff.mpr hi, mem_singleton i, mem_singleton i, ?_⟩
rw [biUnion_singleton]
exact H i hi
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j : ι
hj : i ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ i ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
refine ⟨{ i }, singleton_subset_iff.mpr hi, mem_singleton i, mem_singleton i, ?_⟩
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j : ι
hj : i ∈ t
⊢ IsPreconnected (⋃ (j : ι) (_ : j ∈ {i}), s j)
[PROOFSTEP]
rw [biUnion_singleton]
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j : ι
hj : i ∈ t
⊢ IsPreconnected (s i)
[PROOFSTEP]
exact H i hi
[GOAL]
case tail
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j b✝ c✝ : ι
a✝¹ : ReflTransGen R i b✝
a✝ : R b✝ c✝
a_ih✝ : b✝ ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ b✝ ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : c✝ ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ c✝ ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
case tail j k _ hjk ih =>
obtain ⟨p, hpt, hip, hjp, hp⟩ := ih hjk.2
refine ⟨insert k p, insert_subset_iff.mpr ⟨hj, hpt⟩, mem_insert_of_mem k hip, mem_insert k p, ?_⟩
rw [biUnion_insert]
refine (H k hj).union' (hjk.1.mono ?_) hp
rw [inter_comm]
exact inter_subset_inter_right _ (subset_biUnion_of_mem hjp)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ k ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
case tail j k _ hjk ih =>
obtain ⟨p, hpt, hip, hjp, hp⟩ := ih hjk.2
refine ⟨insert k p, insert_subset_iff.mpr ⟨hj, hpt⟩, mem_insert_of_mem k hip, mem_insert k p, ?_⟩
rw [biUnion_insert]
refine (H k hj).union' (hjk.1.mono ?_) hp
rw [inter_comm]
exact inter_subset_inter_right _ (subset_biUnion_of_mem hjp)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ k ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
obtain ⟨p, hpt, hip, hjp, hp⟩ := ih hjk.2
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
p : Set ι
hpt : p ⊆ t
hip : i ∈ p
hjp : j ∈ p
hp : IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ ∃ p, p ⊆ t ∧ i ∈ p ∧ k ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
[PROOFSTEP]
refine ⟨insert k p, insert_subset_iff.mpr ⟨hj, hpt⟩, mem_insert_of_mem k hip, mem_insert k p, ?_⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
p : Set ι
hpt : p ⊆ t
hip : i ∈ p
hjp : j ∈ p
hp : IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ IsPreconnected (⋃ (j : ι) (_ : j ∈ insert k p), s j)
[PROOFSTEP]
rw [biUnion_insert]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
p : Set ι
hpt : p ⊆ t
hip : i ∈ p
hjp : j ∈ p
hp : IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ IsPreconnected (s k ∪ ⋃ (x : ι) (_ : x ∈ p), s x)
[PROOFSTEP]
refine (H k hj).union' (hjk.1.mono ?_) hp
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
p : Set ι
hpt : p ⊆ t
hip : i ∈ p
hjp : j ∈ p
hp : IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ s j ∩ s k ⊆ s k ∩ ⋃ (x : ι) (_ : x ∈ p), s x
[PROOFSTEP]
rw [inter_comm]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
i : ι
hi : i ∈ t
j✝ j k : ι
a✝ : ReflTransGen R i j
hjk : R j k
ih : j ∈ t → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
hj : k ∈ t
p : Set ι
hpt : p ⊆ t
hip : i ∈ p
hjp : j ∈ p
hp : IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ s k ∩ s j ⊆ s k ∩ ⋃ (x : ι) (_ : x ∈ p), s x
[PROOFSTEP]
exact inter_subset_inter_right _ (subset_biUnion_of_mem hjp)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
P :
∀ (i : ι),
i ∈ t →
∀ (j : ι), j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ IsPreconnected (⋃ (n : ι) (_ : n ∈ t), s n)
[PROOFSTEP]
refine' isPreconnected_of_forall_pair _
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
P :
∀ (i : ι),
i ∈ t →
∀ (j : ι), j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ ∀ (x : α),
x ∈ ⋃ (n : ι) (_ : n ∈ t), s n →
∀ (y : α),
y ∈ ⋃ (n : ι) (_ : n ∈ t), s n →
∃ t_1, t_1 ⊆ ⋃ (n : ι) (_ : n ∈ t), s n ∧ x ∈ t_1 ∧ y ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
intro x hx y hy
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
P :
∀ (i : ι),
i ∈ t →
∀ (j : ι), j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
x : α
hx : x ∈ ⋃ (n : ι) (_ : n ∈ t), s n
y : α
hy : y ∈ ⋃ (n : ι) (_ : n ∈ t), s n
⊢ ∃ t_1, t_1 ⊆ ⋃ (n : ι) (_ : n ∈ t), s n ∧ x ∈ t_1 ∧ y ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
obtain ⟨i : ι, hi : i ∈ t, hxi : x ∈ s i⟩ := mem_iUnion₂.1 hx
[GOAL]
case intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
P :
∀ (i : ι),
i ∈ t →
∀ (j : ι), j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
x : α
hx : x ∈ ⋃ (n : ι) (_ : n ∈ t), s n
y : α
hy : y ∈ ⋃ (n : ι) (_ : n ∈ t), s n
i : ι
hi : i ∈ t
hxi : x ∈ s i
⊢ ∃ t_1, t_1 ⊆ ⋃ (n : ι) (_ : n ∈ t), s n ∧ x ∈ t_1 ∧ y ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
obtain ⟨j : ι, hj : j ∈ t, hyj : y ∈ s j⟩ := mem_iUnion₂.1 hy
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
P :
∀ (i : ι),
i ∈ t →
∀ (j : ι), j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
x : α
hx : x ∈ ⋃ (n : ι) (_ : n ∈ t), s n
y : α
hy : y ∈ ⋃ (n : ι) (_ : n ∈ t), s n
i : ι
hi : i ∈ t
hxi : x ∈ s i
j : ι
hj : j ∈ t
hyj : y ∈ s j
⊢ ∃ t_1, t_1 ⊆ ⋃ (n : ι) (_ : n ∈ t), s n ∧ x ∈ t_1 ∧ y ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
obtain ⟨p, hpt, hip, hjp, hp⟩ := P i hi j hj (K i hi j hj)
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v : Set α
ι : Type u_3
t : Set ι
s : ι → Set α
H : ∀ (i : ι), i ∈ t → IsPreconnected (s i)
K : ∀ (i : ι), i ∈ t → ∀ (j : ι), j ∈ t → ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
R : ι → ι → Prop := fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t
P :
∀ (i : ι),
i ∈ t →
∀ (j : ι), j ∈ t → ReflTransGen R i j → ∃ p, p ⊆ t ∧ i ∈ p ∧ j ∈ p ∧ IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
x : α
hx : x ∈ ⋃ (n : ι) (_ : n ∈ t), s n
y : α
hy : y ∈ ⋃ (n : ι) (_ : n ∈ t), s n
i : ι
hi : i ∈ t
hxi : x ∈ s i
j : ι
hj : j ∈ t
hyj : y ∈ s j
p : Set ι
hpt : p ⊆ t
hip : i ∈ p
hjp : j ∈ p
hp : IsPreconnected (⋃ (j : ι) (_ : j ∈ p), s j)
⊢ ∃ t_1, t_1 ⊆ ⋃ (n : ι) (_ : n ∈ t), s n ∧ x ∈ t_1 ∧ y ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
exact ⟨⋃ j ∈ p, s j, biUnion_subset_biUnion_left hpt, mem_biUnion hip hxi, mem_biUnion hjp hyj, hp⟩
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v : Set α
ι : Type u_3
s : ι → Set α
H : ∀ (i : ι), IsPreconnected (s i)
K : ∀ (i j : ι), ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j)) i j
⊢ IsPreconnected (⋃ (n : ι), s n)
[PROOFSTEP]
rw [← biUnion_univ]
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v : Set α
ι : Type u_3
s : ι → Set α
H : ∀ (i : ι), IsPreconnected (s i)
K : ∀ (i j : ι), ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j)) i j
⊢ IsPreconnected (⋃ (x : ι) (_ : x ∈ univ), s x)
[PROOFSTEP]
exact IsPreconnected.biUnion_of_reflTransGen (fun i _ => H i) fun i _ j _ => by simpa [mem_univ] using K i j
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v : Set α
ι : Type u_3
s : ι → Set α
H : ∀ (i : ι), IsPreconnected (s i)
K : ∀ (i j : ι), ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j)) i j
i : ι
x✝¹ : i ∈ univ
j : ι
x✝ : j ∈ univ
⊢ ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ univ) i j
[PROOFSTEP]
simpa [mem_univ] using K i j
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
H : ∀ (n : β), IsPreconnected (s n)
K : ∀ (n : β), Set.Nonempty (s n ∩ s (succ n))
i✝ j i : β
x✝ : i ∈ Ico j i✝
⊢ Set.Nonempty (s (succ i) ∩ s i)
[PROOFSTEP]
rw [inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
H : ∀ (n : β), IsPreconnected (s n)
K : ∀ (n : β), Set.Nonempty (s n ∩ s (succ n))
i✝ j i : β
x✝ : i ∈ Ico j i✝
⊢ Set.Nonempty (s i ∩ s (succ i))
[PROOFSTEP]
exact K i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
s✝ t u v : Set α
inst✝³ : LinearOrder β
inst✝² : SuccOrder β
inst✝¹ : IsSuccArchimedean β
inst✝ : Nonempty β
s : β → Set α
H : ∀ (n : β), IsConnected (s n)
K : ∀ (n : β), Set.Nonempty (s n ∩ s (succ n))
i✝ j i : β
x✝ : i ∈ Ico j i✝
⊢ Set.Nonempty (s (succ i) ∩ s i)
[PROOFSTEP]
rw [inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
s✝ t u v : Set α
inst✝³ : LinearOrder β
inst✝² : SuccOrder β
inst✝¹ : IsSuccArchimedean β
inst✝ : Nonempty β
s : β → Set α
H : ∀ (n : β), IsConnected (s n)
K : ∀ (n : β), Set.Nonempty (s n ∩ s (succ n))
i✝ j i : β
x✝ : i ∈ Ico j i✝
⊢ Set.Nonempty (s i ∩ s (succ i))
[PROOFSTEP]
exact K i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
⊢ IsPreconnected (⋃ (n : β) (_ : n ∈ t), s n)
[PROOFSTEP]
have h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t := fun hi hj hk => ht.out hi hj (Ico_subset_Icc_self hk)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t
⊢ IsPreconnected (⋃ (n : β) (_ : n ∈ t), s n)
[PROOFSTEP]
have h2 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → succ k ∈ t := fun hi hj hk =>
ht.out hi hj ⟨hk.1.trans <| le_succ _, succ_le_of_lt hk.2⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t
h2 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → succ k ∈ t
⊢ IsPreconnected (⋃ (n : β) (_ : n ∈ t), s n)
[PROOFSTEP]
have h3 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → (s k ∩ s (succ k)).Nonempty := fun hi hj hk =>
K _ (h1 hi hj hk) (h2 hi hj hk)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t
h2 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → succ k ∈ t
h3 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → Set.Nonempty (s k ∩ s (succ k))
⊢ IsPreconnected (⋃ (n : β) (_ : n ∈ t), s n)
[PROOFSTEP]
refine' IsPreconnected.biUnion_of_reflTransGen H fun i hi j hj => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t
h2 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → succ k ∈ t
h3 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → Set.Nonempty (s k ∩ s (succ k))
i : β
hi : i ∈ t
j : β
hj : j ∈ t
⊢ ReflTransGen (fun i j => Set.Nonempty (s i ∩ s j) ∧ i ∈ t) i j
[PROOFSTEP]
exact
reflTransGen_of_succ _ (fun k hk => ⟨h3 hi hj hk, h1 hi hj hk⟩) fun k hk =>
⟨by rw [inter_comm]; exact h3 hj hi hk, h2 hj hi hk⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t
h2 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → succ k ∈ t
h3 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → Set.Nonempty (s k ∩ s (succ k))
i : β
hi : i ∈ t
j : β
hj : j ∈ t
k : β
hk : k ∈ Ico j i
⊢ Set.Nonempty (s (succ k) ∩ s k)
[PROOFSTEP]
rw [inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝² : LinearOrder β
inst✝¹ : SuccOrder β
inst✝ : IsSuccArchimedean β
s : β → Set α
t : Set β
ht : OrdConnected t
H : ∀ (n : β), n ∈ t → IsPreconnected (s n)
K : ∀ (n : β), n ∈ t → succ n ∈ t → Set.Nonempty (s n ∩ s (succ n))
h1 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → k ∈ t
h2 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → succ k ∈ t
h3 : ∀ {i j k : β}, i ∈ t → j ∈ t → k ∈ Ico i j → Set.Nonempty (s k ∩ s (succ k))
i : β
hi : i ∈ t
j : β
hj : j ∈ t
k : β
hk : k ∈ Ico j i
⊢ Set.Nonempty (s k ∩ s (succ k))
[PROOFSTEP]
exact h3 hj hi hk
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
⊢ IsPreconnected (f '' s)
[PROOFSTEP]
rintro u v hu hv huv ⟨_, ⟨x, xs, rfl⟩, xu⟩ ⟨_, ⟨y, ys, rfl⟩, yv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
huv : f '' s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rcases continuousOn_iff'.1 hf u hu with ⟨u', hu', u'_eq⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
huv : f '' s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rcases continuousOn_iff'.1 hf v hv with
⟨v', hv', v'_eq⟩
-- Reformulate `huv : f '' s ⊆ u ∪ v` in terms of `u'` and `v'`
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
huv : f '' s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
replace huv : s ⊆ u' ∪ v'
[GOAL]
case huv
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
huv : f '' s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
⊢ s ⊆ u' ∪ v'
[PROOFSTEP]
rw [image_subset_iff, preimage_union] at huv
[GOAL]
case huv
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ f ⁻¹' u ∪ f ⁻¹' v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
⊢ s ⊆ u' ∪ v'
[PROOFSTEP]
replace huv := subset_inter huv Subset.rfl
[GOAL]
case huv
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ (f ⁻¹' u ∪ f ⁻¹' v) ∩ s
⊢ s ⊆ u' ∪ v'
[PROOFSTEP]
rw [inter_distrib_right, u'_eq, v'_eq, ← inter_distrib_right] at huv
[GOAL]
case huv
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ (u' ∪ v') ∩ s
⊢ s ⊆ u' ∪ v'
[PROOFSTEP]
exact
(subset_inter_iff.1 huv).1
-- Now `s ⊆ u' ∪ v'`, so we can apply `‹IsPreconnected s›`
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
obtain ⟨z, hz⟩ : (s ∩ (u' ∩ v')).Nonempty :=
by
refine H u' v' hu' hv' huv ⟨x, ?_⟩ ⟨y, ?_⟩ <;> rw [inter_comm]
exacts [u'_eq ▸ ⟨xu, xs⟩, v'_eq ▸ ⟨yv, ys⟩]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
⊢ Set.Nonempty (s ∩ (u' ∩ v'))
[PROOFSTEP]
refine H u' v' hu' hv' huv ⟨x, ?_⟩ ⟨y, ?_⟩
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
⊢ x ∈ s ∩ u'
[PROOFSTEP]
rw [inter_comm]
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
⊢ y ∈ s ∩ v'
[PROOFSTEP]
rw [inter_comm]
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
⊢ x ∈ u' ∩ s
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
⊢ y ∈ v' ∩ s
[PROOFSTEP]
exacts [u'_eq ▸ ⟨xu, xs⟩, v'_eq ▸ ⟨yv, ys⟩]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
z : α
hz : z ∈ s ∩ (u' ∩ v')
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rw [← inter_self s, inter_assoc, inter_left_comm s u', ← inter_assoc, inter_comm s, inter_comm s, ← u'_eq, ← v'_eq] at
hz
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
H : IsPreconnected s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
xs : x ∈ s
xu : f x ∈ u
y : α
ys : y ∈ s
yv : f y ∈ v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
huv : s ⊆ u' ∪ v'
z : α
hz : z ∈ f ⁻¹' u ∩ s ∩ (f ⁻¹' v ∩ s)
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨f z, ⟨z, hz.1.2, rfl⟩, hz.1.1, hz.2.1⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ IsPreconnected s →
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
[PROOFSTEP]
rintro h t t' ht ht' htt' ⟨x, xs, xt⟩ ⟨y, ys, yt'⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
⊢ Set.Nonempty (s ∩ (t ∩ t'))
[PROOFSTEP]
rw [← not_disjoint_iff_nonempty_inter, ← subset_compl_iff_disjoint_right, compl_inter]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
⊢ ¬s ⊆ tᶜ ∪ t'ᶜ
[PROOFSTEP]
intro h'
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
h' : s ⊆ tᶜ ∪ t'ᶜ
⊢ False
[PROOFSTEP]
have xt' : x ∉ t' := (h' xs).resolve_left (absurd xt)
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
h' : s ⊆ tᶜ ∪ t'ᶜ
xt' : ¬x ∈ t'
⊢ False
[PROOFSTEP]
have yt : y ∉ t := (h' ys).resolve_right (absurd yt')
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
h' : s ⊆ tᶜ ∪ t'ᶜ
xt' : ¬x ∈ t'
yt : ¬y ∈ t
⊢ False
[PROOFSTEP]
have := h _ _ ht.isOpen_compl ht'.isOpen_compl h' ⟨y, ys, yt⟩ ⟨x, xs, xt'⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
h' : s ⊆ tᶜ ∪ t'ᶜ
xt' : ¬x ∈ t'
yt : ¬y ∈ t
this : Set.Nonempty (s ∩ (tᶜ ∩ t'ᶜ))
⊢ False
[PROOFSTEP]
rw [← compl_union] at this
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
h : IsPreconnected s
t t' : Set α
ht : IsClosed t
ht' : IsClosed t'
htt' : s ⊆ t ∪ t'
x : α
xs : x ∈ s
xt : x ∈ t
y : α
ys : y ∈ s
yt' : y ∈ t'
h' : s ⊆ tᶜ ∪ t'ᶜ
xt' : ¬x ∈ t'
yt : ¬y ∈ t
this : Set.Nonempty (s ∩ (t ∪ t')ᶜ)
⊢ False
[PROOFSTEP]
exact this.ne_empty htt'.disjoint_compl_right.inter_eq
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ (∀ (t t' : Set α),
IsClosed t →
IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))) →
IsPreconnected s
[PROOFSTEP]
rintro h u v hu hv huv ⟨x, xs, xu⟩ ⟨y, ys, yv⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rw [← not_disjoint_iff_nonempty_inter, ← subset_compl_iff_disjoint_right, compl_inter]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
⊢ ¬s ⊆ uᶜ ∪ vᶜ
[PROOFSTEP]
intro h'
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
h' : s ⊆ uᶜ ∪ vᶜ
⊢ False
[PROOFSTEP]
have xv : x ∉ v := (h' xs).elim (absurd xu) id
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
h' : s ⊆ uᶜ ∪ vᶜ
xv : ¬x ∈ v
⊢ False
[PROOFSTEP]
have yu : y ∉ u := (h' ys).elim id (absurd yv)
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
h' : s ⊆ uᶜ ∪ vᶜ
xv : ¬x ∈ v
yu : ¬y ∈ u
⊢ False
[PROOFSTEP]
have := h _ _ hu.isClosed_compl hv.isClosed_compl h' ⟨y, ys, yu⟩ ⟨x, xs, xv⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
h' : s ⊆ uᶜ ∪ vᶜ
xv : ¬x ∈ v
yu : ¬y ∈ u
this : Set.Nonempty (s ∩ (uᶜ ∩ vᶜ))
⊢ False
[PROOFSTEP]
rw [← compl_union] at this
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : s ⊆ u ∪ v
x : α
xs : x ∈ s
xu : x ∈ u
y : α
ys : y ∈ s
yv : y ∈ v
h' : s ⊆ uᶜ ∪ vᶜ
xv : ¬x ∈ v
yu : ¬y ∈ u
this : Set.Nonempty (s ∩ (u ∪ v)ᶜ)
⊢ False
[PROOFSTEP]
exact this.ne_empty huv.disjoint_compl_right.inter_eq
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
⊢ IsPreconnected (f '' s) ↔ IsPreconnected s
[PROOFSTEP]
refine' ⟨fun h => _, fun h => h.image _ hf.continuous.continuousOn⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
⊢ IsPreconnected s
[PROOFSTEP]
rintro u v hu' hv' huv ⟨x, hxs, hxu⟩ ⟨y, hys, hyv⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
u v : Set α
hu' : IsOpen u
hv' : IsOpen v
huv : s ⊆ u ∪ v
x : α
hxs : x ∈ s
hxu : x ∈ u
y : α
hys : y ∈ s
hyv : y ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases hf.isOpen_iff.1 hu' with ⟨u, hu, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
v : Set α
hv' : IsOpen v
x : α
hxs : x ∈ s
y : α
hys : y ∈ s
hyv : y ∈ v
u : Set β
hu : IsOpen u
hu' : IsOpen (f ⁻¹' u)
huv : s ⊆ f ⁻¹' u ∪ v
hxu : x ∈ f ⁻¹' u
⊢ Set.Nonempty (s ∩ (f ⁻¹' u ∩ v))
[PROOFSTEP]
rcases hf.isOpen_iff.1 hv' with ⟨v, hv, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
x : α
hxs : x ∈ s
y : α
hys : y ∈ s
u : Set β
hu : IsOpen u
hu' : IsOpen (f ⁻¹' u)
hxu : x ∈ f ⁻¹' u
v : Set β
hv : IsOpen v
hv' : IsOpen (f ⁻¹' v)
hyv : y ∈ f ⁻¹' v
huv : s ⊆ f ⁻¹' u ∪ f ⁻¹' v
⊢ Set.Nonempty (s ∩ (f ⁻¹' u ∩ f ⁻¹' v))
[PROOFSTEP]
replace huv : f '' s ⊆ u ∪ v
[GOAL]
case huv
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
x : α
hxs : x ∈ s
y : α
hys : y ∈ s
u : Set β
hu : IsOpen u
hu' : IsOpen (f ⁻¹' u)
hxu : x ∈ f ⁻¹' u
v : Set β
hv : IsOpen v
hv' : IsOpen (f ⁻¹' v)
hyv : y ∈ f ⁻¹' v
huv : s ⊆ f ⁻¹' u ∪ f ⁻¹' v
⊢ f '' s ⊆ u ∪ v
[PROOFSTEP]
rwa [image_subset_iff]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
x : α
hxs : x ∈ s
y : α
hys : y ∈ s
u : Set β
hu : IsOpen u
hu' : IsOpen (f ⁻¹' u)
hxu : x ∈ f ⁻¹' u
v : Set β
hv : IsOpen v
hv' : IsOpen (f ⁻¹' v)
hyv : y ∈ f ⁻¹' v
huv : f '' s ⊆ u ∪ v
⊢ Set.Nonempty (s ∩ (f ⁻¹' u ∩ f ⁻¹' v))
[PROOFSTEP]
rcases h u v hu hv huv ⟨f x, mem_image_of_mem _ hxs, hxu⟩ ⟨f y, mem_image_of_mem _ hys, hyv⟩ with
⟨_, ⟨z, hzs, rfl⟩, hzuv⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Inducing f
h : IsPreconnected (f '' s)
x : α
hxs : x ∈ s
y : α
hys : y ∈ s
u : Set β
hu : IsOpen u
hu' : IsOpen (f ⁻¹' u)
hxu : x ∈ f ⁻¹' u
v : Set β
hv : IsOpen v
hv' : IsOpen (f ⁻¹' v)
hyv : y ∈ f ⁻¹' v
huv : f '' s ⊆ u ∪ v
z : α
hzs : z ∈ s
hzuv : f z ∈ u ∩ v
⊢ Set.Nonempty (s ∩ (f ⁻¹' u ∩ f ⁻¹' v))
[PROOFSTEP]
exact ⟨z, hzs, hzuv⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
hsf : s ⊆ range f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
⊢ Set.Nonempty (f ⁻¹' s ∩ (u ∩ v))
[PROOFSTEP]
replace hsf : f '' (f ⁻¹' s) = s := image_preimage_eq_of_subset hsf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (f ⁻¹' s ∩ (u ∩ v))
[PROOFSTEP]
obtain ⟨_, has, ⟨a, hau, rfl⟩, hav⟩ : (s ∩ (f '' u ∩ f '' v)).Nonempty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (s ∩ (f '' u ∩ f '' v))
[PROOFSTEP]
refine hs (f '' u) (f '' v) (hf u hu) (hf v hv) ?_ ?_ ?_
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ s ⊆ f '' u ∪ f '' v
[PROOFSTEP]
simpa only [hsf, image_union] using image_subset f hsuv
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (s ∩ f '' u)
[PROOFSTEP]
simpa only [image_preimage_inter] using hsu.image f
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (s ∩ f '' v)
[PROOFSTEP]
simpa only [image_preimage_inter] using hsv.image f
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsOpenMap f
u v : Set α
hu : IsOpen u
hv : IsOpen v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
a : α
hau : a ∈ u
has : f a ∈ s
hav : f a ∈ f '' v
⊢ Set.Nonempty (f ⁻¹' s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨a, has, hau, hinj.mem_set_image.1 hav⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
hsf : s ⊆ range f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
⊢ Set.Nonempty (f ⁻¹' s ∩ (u ∩ v))
[PROOFSTEP]
replace hsf : f '' (f ⁻¹' s) = s := image_preimage_eq_of_subset hsf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (f ⁻¹' s ∩ (u ∩ v))
[PROOFSTEP]
obtain ⟨_, has, ⟨a, hau, rfl⟩, hav⟩ : (s ∩ (f '' u ∩ f '' v)).Nonempty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (s ∩ (f '' u ∩ f '' v))
[PROOFSTEP]
refine isPreconnected_closed_iff.1 hs (f '' u) (f '' v) (hf u hu) (hf v hv) ?_ ?_ ?_
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ s ⊆ f '' u ∪ f '' v
[PROOFSTEP]
simpa only [hsf, image_union] using image_subset f hsuv
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (s ∩ f '' u)
[PROOFSTEP]
simpa only [image_preimage_inter] using hsu.image f
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
⊢ Set.Nonempty (s ∩ f '' v)
[PROOFSTEP]
simpa only [image_preimage_inter] using hsv.image f
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : TopologicalSpace β
s : Set β
hs : IsPreconnected s
f : α → β
hinj : Injective f
hf : IsClosedMap f
u v : Set α
hu : IsClosed u
hv : IsClosed v
hsuv : f ⁻¹' s ⊆ u ∪ v
hsu : Set.Nonempty (f ⁻¹' s ∩ u)
hsv : Set.Nonempty (f ⁻¹' s ∩ v)
hsf : f '' (f ⁻¹' s) = s
a : α
hau : a ∈ u
has : f a ∈ s
hav : f a ∈ f '' v
⊢ Set.Nonempty (f ⁻¹' s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨a, has, hau, hinj.mem_set_image.1 hav⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hs : IsPreconnected s
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
specialize hs u v hu hv hsuv
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hs : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
obtain hsu | hsu := (s ∩ u).eq_empty_or_nonempty
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hs : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
hsu : s ∩ u = ∅
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
exact Or.inr ((Set.disjoint_iff_inter_eq_empty.2 hsu).subset_right_of_subset_union hsuv)
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hs : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
hsu : Set.Nonempty (s ∩ u)
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
replace hs := mt (hs hsu)
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hs : ¬Set.Nonempty (s ∩ (u ∩ v)) → ¬Set.Nonempty (s ∩ v)
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
simp_rw [Set.not_nonempty_iff_eq_empty, ← Set.disjoint_iff_inter_eq_empty, disjoint_iff_inter_eq_empty.1 huv] at hs
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hs : Disjoint s ∅ → Disjoint s v
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
exact Or.inl ((hs s.disjoint_empty).subset_left_of_subset_union hsuv)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hs : IsPreconnected s
⊢ Disjoint s v
[PROOFSTEP]
by_contra hsv
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hs : IsPreconnected s
hsv : ¬Disjoint s v
⊢ False
[PROOFSTEP]
rw [not_disjoint_iff_nonempty_inter] at hsv
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hs : IsPreconnected s
hsv : Set.Nonempty (s ∩ v)
⊢ False
[PROOFSTEP]
obtain ⟨x, _, hx⟩ := hs u v hu hv hsuv hsu hsv
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hu : IsOpen u
hv : IsOpen v
huv : Disjoint u v
hsuv : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hs : IsPreconnected s
hsv : Set.Nonempty (s ∩ v)
x : α
left✝ : x ∈ s
hx : x ∈ u ∩ v
⊢ False
[PROOFSTEP]
exact Set.disjoint_iff.1 huv hx
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s t : Set α
hs : IsPreconnected s
ht : IsClopen t
hne : Set.Nonempty (s ∩ t)
⊢ s ⊆ t ∪ tᶜ
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
⊢ s ⊆ u
[PROOFSTEP]
have A : s ⊆ u ∪ (closure u)ᶜ := by
intro x hx
by_cases xu : x ∈ u
· exact Or.inl xu
· right
intro h'x
exact xu (h (mem_inter h'x hx))
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
⊢ s ⊆ u ∪ (closure u)ᶜ
[PROOFSTEP]
intro x hx
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
x : α
hx : x ∈ s
⊢ x ∈ u ∪ (closure u)ᶜ
[PROOFSTEP]
by_cases xu : x ∈ u
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
x : α
hx : x ∈ s
xu : x ∈ u
⊢ x ∈ u ∪ (closure u)ᶜ
[PROOFSTEP]
exact Or.inl xu
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
x : α
hx : x ∈ s
xu : ¬x ∈ u
⊢ x ∈ u ∪ (closure u)ᶜ
[PROOFSTEP]
right
[GOAL]
case neg.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
x : α
hx : x ∈ s
xu : ¬x ∈ u
⊢ x ∈ (closure u)ᶜ
[PROOFSTEP]
intro h'x
[GOAL]
case neg.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
x : α
hx : x ∈ s
xu : ¬x ∈ u
h'x : x ∈ closure u
⊢ False
[PROOFSTEP]
exact xu (h (mem_inter h'x hx))
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
A : s ⊆ u ∪ (closure u)ᶜ
⊢ s ⊆ u
[PROOFSTEP]
apply hs.subset_left_of_subset_union hu isClosed_closure.isOpen_compl _ A h'u
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
hs : IsPreconnected s
hu : IsOpen u
h'u : Set.Nonempty (s ∩ u)
h : closure u ∩ s ⊆ u
A : s ⊆ u ∪ (closure u)ᶜ
⊢ Disjoint u (closure u)ᶜ
[PROOFSTEP]
exact disjoint_compl_right.mono_right (compl_subset_compl.2 subset_closure)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
⊢ IsPreconnected (s ×ˢ t)
[PROOFSTEP]
apply isPreconnected_of_forall_pair
[GOAL]
case H
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
⊢ ∀ (x : α × β), x ∈ s ×ˢ t → ∀ (y : α × β), y ∈ s ×ˢ t → ∃ t_1, t_1 ⊆ s ×ˢ t ∧ x ∈ t_1 ∧ y ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
rintro ⟨a₁, b₁⟩ ⟨ha₁, hb₁⟩ ⟨a₂, b₂⟩ ⟨ha₂, hb₂⟩
[GOAL]
case H.mk.intro.mk.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
a₁ : α
b₁ : β
ha₁ : (a₁, b₁).fst ∈ s
hb₁ : (a₁, b₁).snd ∈ t
a₂ : α
b₂ : β
ha₂ : (a₂, b₂).fst ∈ s
hb₂ : (a₂, b₂).snd ∈ t
⊢ ∃ t_1, t_1 ⊆ s ×ˢ t ∧ (a₁, b₁) ∈ t_1 ∧ (a₂, b₂) ∈ t_1 ∧ IsPreconnected t_1
[PROOFSTEP]
refine' ⟨Prod.mk a₁ '' t ∪ flip Prod.mk b₂ '' s, _, .inl ⟨b₁, hb₁, rfl⟩, .inr ⟨a₂, ha₂, rfl⟩, _⟩
[GOAL]
case H.mk.intro.mk.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
a₁ : α
b₁ : β
ha₁ : (a₁, b₁).fst ∈ s
hb₁ : (a₁, b₁).snd ∈ t
a₂ : α
b₂ : β
ha₂ : (a₂, b₂).fst ∈ s
hb₂ : (a₂, b₂).snd ∈ t
⊢ Prod.mk a₁ '' t ∪ flip Prod.mk b₂ '' s ⊆ s ×ˢ t
[PROOFSTEP]
rintro _ (⟨y, hy, rfl⟩ | ⟨x, hx, rfl⟩)
[GOAL]
case H.mk.intro.mk.intro.refine'_1.inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
a₁ : α
b₁ : β
ha₁ : (a₁, b₁).fst ∈ s
hb₁ : (a₁, b₁).snd ∈ t
a₂ : α
b₂ : β
ha₂ : (a₂, b₂).fst ∈ s
hb₂ : (a₂, b₂).snd ∈ t
y : β
hy : y ∈ t
⊢ (a₁, y) ∈ s ×ˢ t
case H.mk.intro.mk.intro.refine'_1.inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
a₁ : α
b₁ : β
ha₁ : (a₁, b₁).fst ∈ s
hb₁ : (a₁, b₁).snd ∈ t
a₂ : α
b₂ : β
ha₂ : (a₂, b₂).fst ∈ s
hb₂ : (a₂, b₂).snd ∈ t
x : α
hx : x ∈ s
⊢ flip Prod.mk b₂ x ∈ s ×ˢ t
[PROOFSTEP]
exacts [⟨ha₁, hy⟩, ⟨hx, hb₂⟩]
[GOAL]
case H.mk.intro.mk.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : TopologicalSpace β
s : Set α
t : Set β
hs : IsPreconnected s
ht : IsPreconnected t
a₁ : α
b₁ : β
ha₁ : (a₁, b₁).fst ∈ s
hb₁ : (a₁, b₁).snd ∈ t
a₂ : α
b₂ : β
ha₂ : (a₂, b₂).fst ∈ s
hb₂ : (a₂, b₂).snd ∈ t
⊢ IsPreconnected (Prod.mk a₁ '' t ∪ flip Prod.mk b₂ '' s)
[PROOFSTEP]
exact
(ht.image _ (Continuous.Prod.mk _).continuousOn).union (a₁, b₂) ⟨b₂, hb₂, rfl⟩ ⟨a₁, ha₁, rfl⟩
(hs.image _ (continuous_id.prod_mk continuous_const).continuousOn)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
⊢ IsPreconnected (pi univ s)
[PROOFSTEP]
rintro u v uo vo hsuv ⟨f, hfs, hfu⟩ ⟨g, hgs, hgv⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
rcases exists_finset_piecewise_mem_of_mem_nhds (uo.mem_nhds hfu) g with ⟨I, hI⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I : Finset ι
hI : Finset.piecewise I f g ∈ u
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
induction' I using Finset.induction_on with i I _ ihI
[GOAL]
case intro.intro.intro.intro.intro.empty
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I : Finset ι
hI✝ : Finset.piecewise I f g ∈ u
hI : Finset.piecewise ∅ f g ∈ u
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
refine' ⟨g, hgs, ⟨_, hgv⟩⟩
[GOAL]
case intro.intro.intro.intro.intro.empty
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I : Finset ι
hI✝ : Finset.piecewise I f g ∈ u
hI : Finset.piecewise ∅ f g ∈ u
⊢ g ∈ u
[PROOFSTEP]
simpa using hI
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : Finset.piecewise (insert i I) f g ∈ u
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
rw [Finset.piecewise_insert] at hI
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
have := I.piecewise_mem_set_pi hfs hgs
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
refine' (hsuv this).elim ihI fun h => _
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
set S := update (I.piecewise f g) i '' s i
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
have hsub : S ⊆ pi univ s := by
refine' image_subset_iff.2 fun z hz => _
rwa [update_preimage_univ_pi]
exact fun j _ => this j trivial
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
⊢ S ⊆ pi univ s
[PROOFSTEP]
refine' image_subset_iff.2 fun z hz => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
z : π i
hz : z ∈ s i
⊢ z ∈ update (Finset.piecewise I f g) i ⁻¹' pi univ s
[PROOFSTEP]
rwa [update_preimage_univ_pi]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
z : π i
hz : z ∈ s i
⊢ ∀ (j : ι), j ≠ i → Finset.piecewise I f g j ∈ s j
[PROOFSTEP]
exact fun j _ => this j trivial
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
hsub : S ⊆ pi univ s
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
have hconn : IsPreconnected S := (hs i).image _ (continuous_const.update i continuous_id).continuousOn
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
hsub : S ⊆ pi univ s
hconn : IsPreconnected S
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
have hSu : (S ∩ u).Nonempty := ⟨_, mem_image_of_mem _ (hfs _ trivial), hI⟩
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
hsub : S ⊆ pi univ s
hconn : IsPreconnected S
hSu : Set.Nonempty (S ∩ u)
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
have hSv : (S ∩ v).Nonempty := ⟨_, ⟨_, this _ trivial, update_eq_self _ _⟩, h⟩
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
hsub : S ⊆ pi univ s
hconn : IsPreconnected S
hSu : Set.Nonempty (S ∩ u)
hSv : Set.Nonempty (S ∩ v)
⊢ Set.Nonempty (pi univ s ∩ (u ∩ v))
[PROOFSTEP]
refine' (hconn u v uo vo (hsub.trans hsuv) hSu hSv).mono _
[GOAL]
case intro.intro.intro.intro.intro.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u✝ v✝ : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hs : ∀ (i : ι), IsPreconnected (s i)
u v : Set ((i : ι) → π i)
uo : IsOpen u
vo : IsOpen v
hsuv : pi univ s ⊆ u ∪ v
f : (i : ι) → π i
hfs : f ∈ pi univ s
hfu : f ∈ u
g : (i : ι) → π i
hgs : g ∈ pi univ s
hgv : g ∈ v
I✝ : Finset ι
hI✝ : Finset.piecewise I✝ f g ∈ u
i : ι
I : Finset ι
a✝ : ¬i ∈ I
ihI : Finset.piecewise I f g ∈ u → Set.Nonempty (pi univ s ∩ (u ∩ v))
hI : update (Finset.piecewise I f g) i (f i) ∈ u
this : Finset.piecewise I f g ∈ pi univ s
h : Finset.piecewise I f g ∈ v
S : Set ((a : ι) → π a) := update (Finset.piecewise I f g) i '' s i
hsub : S ⊆ pi univ s
hconn : IsPreconnected S
hSu : Set.Nonempty (S ∩ u)
hSv : Set.Nonempty (S ∩ v)
⊢ S ∩ (u ∩ v) ⊆ pi univ s ∩ (u ∩ v)
[PROOFSTEP]
exact inter_subset_inter_left _ hsub
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
⊢ IsConnected (pi univ s) ↔ ∀ (i : ι), IsConnected (s i)
[PROOFSTEP]
simp only [IsConnected, ← univ_pi_nonempty_iff, forall_and, and_congr_right_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
⊢ Set.Nonempty (pi univ s) → (IsPreconnected (pi univ s) ↔ ∀ (x : ι), IsPreconnected (s x))
[PROOFSTEP]
refine' fun hne => ⟨fun hc i => _, isPreconnected_univ_pi⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hne : Set.Nonempty (pi univ s)
hc : IsPreconnected (pi univ s)
i : ι
⊢ IsPreconnected (s i)
[PROOFSTEP]
rw [← eval_image_univ_pi hne]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
hne : Set.Nonempty (pi univ s)
hc : IsPreconnected (pi univ s)
i : ι
⊢ IsPreconnected ((fun f => f i) '' pi univ s)
[PROOFSTEP]
exact hc.image _ (continuous_apply _).continuousOn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
⊢ IsConnected s ↔ ∃ i t, IsConnected t ∧ s = mk i '' t
[PROOFSTEP]
refine' ⟨fun hs => _, _⟩
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
hs : IsConnected s
⊢ ∃ i t, IsConnected t ∧ s = mk i '' t
[PROOFSTEP]
obtain ⟨⟨i, x⟩, hx⟩ := hs.nonempty
[GOAL]
case refine'_1.intro.mk
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
hs : IsConnected s
i : ι
x : π i
hx : { fst := i, snd := x } ∈ s
⊢ ∃ i t, IsConnected t ∧ s = mk i '' t
[PROOFSTEP]
have : s ⊆ range (Sigma.mk i) := hs.isPreconnected.subset_clopen isClopen_range_sigmaMk ⟨⟨i, x⟩, hx, x, rfl⟩
[GOAL]
case refine'_1.intro.mk
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
hs : IsConnected s
i : ι
x : π i
hx : { fst := i, snd := x } ∈ s
this : s ⊆ range (mk i)
⊢ ∃ i t, IsConnected t ∧ s = mk i '' t
[PROOFSTEP]
exact
⟨i, Sigma.mk i ⁻¹' s, hs.preimage_of_openMap sigma_mk_injective isOpenMap_sigmaMk this,
(Set.image_preimage_eq_of_subset this).symm⟩
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
⊢ (∃ i t, IsConnected t ∧ s = mk i '' t) → IsConnected s
[PROOFSTEP]
rintro ⟨i, t, ht, rfl⟩
[GOAL]
case refine'_2.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
i : ι
t : Set (π i)
ht : IsConnected t
⊢ IsConnected (mk i '' t)
[PROOFSTEP]
exact ht.image _ continuous_sigmaMk.continuousOn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
⊢ IsPreconnected s ↔ ∃ i t, IsPreconnected t ∧ s = mk i '' t
[PROOFSTEP]
refine' ⟨fun hs => _, _⟩
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
hs : IsPreconnected s
⊢ ∃ i t, IsPreconnected t ∧ s = mk i '' t
[PROOFSTEP]
obtain rfl | h := s.eq_empty_or_nonempty
[GOAL]
case refine'_1.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
hs : IsPreconnected ∅
⊢ ∃ i t, IsPreconnected t ∧ ∅ = mk i '' t
[PROOFSTEP]
exact ⟨Classical.choice hι, ∅, isPreconnected_empty, (Set.image_empty _).symm⟩
[GOAL]
case refine'_1.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
hs : IsPreconnected s
h : Set.Nonempty s
⊢ ∃ i t, IsPreconnected t ∧ s = mk i '' t
[PROOFSTEP]
obtain ⟨a, t, ht, rfl⟩ := Sigma.isConnected_iff.1 ⟨h, hs⟩
[GOAL]
case refine'_1.inr.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
a : ι
t : Set (π a)
ht : IsConnected t
hs : IsPreconnected (mk a '' t)
h : Set.Nonempty (mk a '' t)
⊢ ∃ i t_1, IsPreconnected t_1 ∧ mk a '' t = mk i '' t_1
[PROOFSTEP]
refine' ⟨a, t, ht.isPreconnected, rfl⟩
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
s : Set ((i : ι) × π i)
⊢ (∃ i t, IsPreconnected t ∧ s = mk i '' t) → IsPreconnected s
[PROOFSTEP]
rintro ⟨a, t, ht, rfl⟩
[GOAL]
case refine'_2.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
hι : Nonempty ι
inst✝ : (i : ι) → TopologicalSpace (π i)
a : ι
t : Set (π a)
ht : IsPreconnected t
⊢ IsPreconnected (mk a '' t)
[PROOFSTEP]
exact ht.image _ continuous_sigmaMk.continuousOn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
⊢ IsConnected s ↔ (∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t
[PROOFSTEP]
refine' ⟨fun hs => _, _⟩
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
⊢ (∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t
[PROOFSTEP]
obtain ⟨x | x, hx⟩ := hs.nonempty
[GOAL]
case refine'_1.intro.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : α
hx : inl x ∈ s
⊢ (∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t
[PROOFSTEP]
have h : s ⊆ range Sum.inl := hs.isPreconnected.subset_clopen isClopen_range_inl ⟨.inl x, hx, x, rfl⟩
[GOAL]
case refine'_1.intro.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : α
hx : inl x ∈ s
h : s ⊆ range inl
⊢ (∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t
[PROOFSTEP]
refine' Or.inl ⟨Sum.inl ⁻¹' s, _, _⟩
[GOAL]
case refine'_1.intro.inl.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : α
hx : inl x ∈ s
h : s ⊆ range inl
⊢ IsConnected (inl ⁻¹' s)
[PROOFSTEP]
exact hs.preimage_of_openMap Sum.inl_injective isOpenMap_inl h
[GOAL]
case refine'_1.intro.inl.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : α
hx : inl x ∈ s
h : s ⊆ range inl
⊢ s = inl '' (inl ⁻¹' s)
[PROOFSTEP]
exact (image_preimage_eq_of_subset h).symm
[GOAL]
case refine'_1.intro.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : β
hx : inr x ∈ s
⊢ (∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t
[PROOFSTEP]
have h : s ⊆ range Sum.inr := hs.isPreconnected.subset_clopen isClopen_range_inr ⟨.inr x, hx, x, rfl⟩
[GOAL]
case refine'_1.intro.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : β
hx : inr x ∈ s
h : s ⊆ range inr
⊢ (∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t
[PROOFSTEP]
refine' Or.inr ⟨Sum.inr ⁻¹' s, _, _⟩
[GOAL]
case refine'_1.intro.inr.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : β
hx : inr x ∈ s
h : s ⊆ range inr
⊢ IsConnected (inr ⁻¹' s)
[PROOFSTEP]
exact hs.preimage_of_openMap Sum.inr_injective isOpenMap_inr h
[GOAL]
case refine'_1.intro.inr.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsConnected s
x : β
hx : inr x ∈ s
h : s ⊆ range inr
⊢ s = inr '' (inr ⁻¹' s)
[PROOFSTEP]
exact (image_preimage_eq_of_subset h).symm
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
⊢ ((∃ t, IsConnected t ∧ s = inl '' t) ∨ ∃ t, IsConnected t ∧ s = inr '' t) → IsConnected s
[PROOFSTEP]
rintro (⟨t, ht, rfl⟩ | ⟨t, ht, rfl⟩)
[GOAL]
case refine'_2.inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
t : Set α
ht : IsConnected t
⊢ IsConnected (inl '' t)
[PROOFSTEP]
exact ht.image _ continuous_inl.continuousOn
[GOAL]
case refine'_2.inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
t : Set β
ht : IsConnected t
⊢ IsConnected (inr '' t)
[PROOFSTEP]
exact ht.image _ continuous_inr.continuousOn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
⊢ IsPreconnected s ↔ (∃ t, IsPreconnected t ∧ s = inl '' t) ∨ ∃ t, IsPreconnected t ∧ s = inr '' t
[PROOFSTEP]
refine' ⟨fun hs => _, _⟩
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsPreconnected s
⊢ (∃ t, IsPreconnected t ∧ s = inl '' t) ∨ ∃ t, IsPreconnected t ∧ s = inr '' t
[PROOFSTEP]
obtain rfl | h := s.eq_empty_or_nonempty
[GOAL]
case refine'_1.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : TopologicalSpace β
hs : IsPreconnected ∅
⊢ (∃ t, IsPreconnected t ∧ ∅ = inl '' t) ∨ ∃ t, IsPreconnected t ∧ ∅ = inr '' t
[PROOFSTEP]
exact Or.inl ⟨∅, isPreconnected_empty, (Set.image_empty _).symm⟩
[GOAL]
case refine'_1.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
hs : IsPreconnected s
h : Set.Nonempty s
⊢ (∃ t, IsPreconnected t ∧ s = inl '' t) ∨ ∃ t, IsPreconnected t ∧ s = inr '' t
[PROOFSTEP]
obtain ⟨t, ht, rfl⟩ | ⟨t, ht, rfl⟩ := Sum.isConnected_iff.1 ⟨h, hs⟩
[GOAL]
case refine'_1.inr.inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
t : Set α
ht : IsConnected t
hs : IsPreconnected (inl '' t)
h : Set.Nonempty (inl '' t)
⊢ (∃ t_1, IsPreconnected t_1 ∧ inl '' t = inl '' t_1) ∨ ∃ t_1, IsPreconnected t_1 ∧ inl '' t = inr '' t_1
[PROOFSTEP]
exact Or.inl ⟨t, ht.isPreconnected, rfl⟩
[GOAL]
case refine'_1.inr.inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
t : Set β
ht : IsConnected t
hs : IsPreconnected (inr '' t)
h : Set.Nonempty (inr '' t)
⊢ (∃ t_1, IsPreconnected t_1 ∧ inr '' t = inl '' t_1) ∨ ∃ t_1, IsPreconnected t_1 ∧ inr '' t = inr '' t_1
[PROOFSTEP]
exact Or.inr ⟨t, ht.isPreconnected, rfl⟩
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : TopologicalSpace β
s : Set (α ⊕ β)
⊢ ((∃ t, IsPreconnected t ∧ s = inl '' t) ∨ ∃ t, IsPreconnected t ∧ s = inr '' t) → IsPreconnected s
[PROOFSTEP]
rintro (⟨t, ht, rfl⟩ | ⟨t, ht, rfl⟩)
[GOAL]
case refine'_2.inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
t : Set α
ht : IsPreconnected t
⊢ IsPreconnected (inl '' t)
[PROOFSTEP]
exact ht.image _ continuous_inl.continuousOn
[GOAL]
case refine'_2.inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
t : Set β
ht : IsPreconnected t
⊢ IsPreconnected (inr '' t)
[PROOFSTEP]
exact ht.image _ continuous_inr.continuousOn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hx : x ∈ F
⊢ x ∈ connectedComponentIn F x
[PROOFSTEP]
simp [connectedComponentIn_eq_image hx, mem_connectedComponent, hx]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
⊢ Set.Nonempty (connectedComponentIn F x) ↔ x ∈ F
[PROOFSTEP]
rw [connectedComponentIn]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
⊢ Set.Nonempty (if h : x ∈ F then Subtype.val '' connectedComponent { val := x, property := h } else ∅) ↔ x ∈ F
[PROOFSTEP]
split_ifs
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
h✝ : x ∈ F
⊢ Set.Nonempty (Subtype.val '' connectedComponent { val := x, property := h✝ }) ↔ x ∈ F
[PROOFSTEP]
simp [connectedComponent_nonempty, *]
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
h✝ : ¬x ∈ F
⊢ Set.Nonempty ∅ ↔ x ∈ F
[PROOFSTEP]
simp [connectedComponent_nonempty, *]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v F : Set α
x : α
⊢ connectedComponentIn F x ⊆ F
[PROOFSTEP]
rw [connectedComponentIn]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v F : Set α
x : α
⊢ (if h : x ∈ F then Subtype.val '' connectedComponent { val := x, property := h } else ∅) ⊆ F
[PROOFSTEP]
split_ifs
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v F : Set α
x : α
h✝ : x ∈ F
⊢ Subtype.val '' connectedComponent { val := x, property := h✝ } ⊆ F
[PROOFSTEP]
simp
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v F : Set α
x : α
h✝ : ¬x ∈ F
⊢ ∅ ⊆ F
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
⊢ IsPreconnected (connectedComponentIn F x)
[PROOFSTEP]
rw [connectedComponentIn]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
⊢ IsPreconnected (if h : x ∈ F then Subtype.val '' connectedComponent { val := x, property := h } else ∅)
[PROOFSTEP]
split_ifs
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
h✝ : x ∈ F
⊢ IsPreconnected (Subtype.val '' connectedComponent { val := x, property := h✝ })
[PROOFSTEP]
exact inducing_subtype_val.isPreconnected_image.mpr isPreconnected_connectedComponent
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
h✝ : ¬x ∈ F
⊢ IsPreconnected ∅
[PROOFSTEP]
exact isPreconnected_empty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
⊢ IsConnected (connectedComponentIn F x) ↔ x ∈ F
[PROOFSTEP]
simp_rw [← connectedComponentIn_nonempty_iff, IsConnected, isPreconnected_connectedComponentIn, and_true_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
⊢ s ⊆ connectedComponentIn F x
[PROOFSTEP]
have : IsPreconnected (((↑) : F → α) ⁻¹' s) :=
by
refine' inducing_subtype_val.isPreconnected_image.mp _
rwa [Subtype.image_preimage_coe, inter_eq_left_iff_subset.mpr hsF]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
⊢ IsPreconnected (Subtype.val ⁻¹' s)
[PROOFSTEP]
refine' inducing_subtype_val.isPreconnected_image.mp _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
⊢ IsPreconnected (Subtype.val '' (Subtype.val ⁻¹' s))
[PROOFSTEP]
rwa [Subtype.image_preimage_coe, inter_eq_left_iff_subset.mpr hsF]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this : IsPreconnected (Subtype.val ⁻¹' s)
⊢ s ⊆ connectedComponentIn F x
[PROOFSTEP]
have h2xs : (⟨x, hsF hxs⟩ : F) ∈ (↑) ⁻¹' s := by
rw [mem_preimage]
exact hxs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this : IsPreconnected (Subtype.val ⁻¹' s)
⊢ { val := x, property := (_ : x ∈ F) } ∈ Subtype.val ⁻¹' s
[PROOFSTEP]
rw [mem_preimage]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this : IsPreconnected (Subtype.val ⁻¹' s)
⊢ ↑{ val := x, property := (_ : x ∈ F) } ∈ s
[PROOFSTEP]
exact hxs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this : IsPreconnected (Subtype.val ⁻¹' s)
h2xs : { val := x, property := (_ : x ∈ F) } ∈ Subtype.val ⁻¹' s
⊢ s ⊆ connectedComponentIn F x
[PROOFSTEP]
have := this.subset_connectedComponent h2xs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this✝ : IsPreconnected (Subtype.val ⁻¹' s)
h2xs : { val := x, property := (_ : x ∈ F) } ∈ Subtype.val ⁻¹' s
this : Subtype.val ⁻¹' s ⊆ connectedComponent { val := x, property := (_ : x ∈ F) }
⊢ s ⊆ connectedComponentIn F x
[PROOFSTEP]
rw [connectedComponentIn_eq_image (hsF hxs)]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this✝ : IsPreconnected (Subtype.val ⁻¹' s)
h2xs : { val := x, property := (_ : x ∈ F) } ∈ Subtype.val ⁻¹' s
this : Subtype.val ⁻¹' s ⊆ connectedComponent { val := x, property := (_ : x ∈ F) }
⊢ s ⊆ Subtype.val '' connectedComponent { val := x, property := (_ : x ∈ F) }
[PROOFSTEP]
refine' Subset.trans _ (image_subset _ this)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hs : IsPreconnected s
hxs : x ∈ s
hsF : s ⊆ F
this✝ : IsPreconnected (Subtype.val ⁻¹' s)
h2xs : { val := x, property := (_ : x ∈ F) } ∈ Subtype.val ⁻¹' s
this : Subtype.val ⁻¹' s ⊆ connectedComponent { val := x, property := (_ : x ∈ F) }
⊢ s ⊆ Subtype.val '' (Subtype.val ⁻¹' s)
[PROOFSTEP]
rw [Subtype.image_preimage_coe, inter_eq_left_iff_subset.mpr hsF]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x y : α
F : Set α
h : y ∈ connectedComponentIn F x
⊢ connectedComponentIn F x = connectedComponentIn F y
[PROOFSTEP]
have hx : x ∈ F := connectedComponentIn_nonempty_iff.mp ⟨y, h⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x y : α
F : Set α
h : y ∈ connectedComponentIn F x
hx : x ∈ F
⊢ connectedComponentIn F x = connectedComponentIn F y
[PROOFSTEP]
simp_rw [connectedComponentIn_eq_image hx] at h ⊢
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x y : α
F : Set α
hx : x ∈ F
h : y ∈ Subtype.val '' connectedComponent { val := x, property := hx }
⊢ Subtype.val '' connectedComponent { val := x, property := hx } = connectedComponentIn F y
[PROOFSTEP]
obtain ⟨⟨y, hy⟩, h2y, rfl⟩ := h
[GOAL]
case intro.mk.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F : Set α
hx : x ∈ F
y : α
hy : y ∈ F
h2y : { val := y, property := hy } ∈ connectedComponent { val := x, property := hx }
⊢ Subtype.val '' connectedComponent { val := x, property := hx } = connectedComponentIn F ↑{ val := y, property := hy }
[PROOFSTEP]
simp_rw [connectedComponentIn_eq_image hy, connectedComponent_eq h2y]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F G : Set α
h : F ⊆ G
⊢ connectedComponentIn F x ⊆ connectedComponentIn G x
[PROOFSTEP]
by_cases hx : x ∈ F
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F G : Set α
h : F ⊆ G
hx : x ∈ F
⊢ connectedComponentIn F x ⊆ connectedComponentIn G x
[PROOFSTEP]
rw [connectedComponentIn_eq_image hx, connectedComponentIn_eq_image (h hx), ←
show ((↑) : G → α) ∘ inclusion h = (↑) from rfl, image_comp]
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F G : Set α
h : F ⊆ G
hx : x ∈ F
⊢ Subtype.val '' (inclusion h '' connectedComponent { val := x, property := hx }) ⊆
Subtype.val '' connectedComponent { val := x, property := (_ : x ∈ G) }
[PROOFSTEP]
exact image_subset _ ((continuous_inclusion h).image_connectedComponent_subset ⟨x, hx⟩)
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F G : Set α
h : F ⊆ G
hx : ¬x ∈ F
⊢ connectedComponentIn F x ⊆ connectedComponentIn G x
[PROOFSTEP]
rw [connectedComponentIn_eq_empty hx]
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
F G : Set α
h : F ⊆ G
hx : ¬x ∈ F
⊢ ∅ ⊆ connectedComponentIn G x
[PROOFSTEP]
exact Set.empty_subset _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : TopologicalSpace β
f : α → β
hf : Surjective f
hf' : Continuous f
⊢ ConnectedSpace β
[PROOFSTEP]
rw [connectedSpace_iff_univ, ← hf.range_eq]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : TopologicalSpace β
f : α → β
hf : Surjective f
hf' : Continuous f
⊢ IsConnected (range f)
[PROOFSTEP]
exact isConnected_range hf'
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ ConnectedSpace α ↔ ∃ x, connectedComponent x = univ
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ ConnectedSpace α → ∃ x, connectedComponent x = univ
[PROOFSTEP]
rintro ⟨⟨x⟩⟩
[GOAL]
case mp.mk.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
toPreconnectedSpace✝ : PreconnectedSpace α
x : α
⊢ ∃ x, connectedComponent x = univ
[PROOFSTEP]
exact ⟨x, eq_univ_of_univ_subset <| isPreconnected_univ.subset_connectedComponent (mem_univ x)⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∃ x, connectedComponent x = univ) → ConnectedSpace α
[PROOFSTEP]
rintro ⟨x, h⟩
[GOAL]
case mpr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
h : connectedComponent x = univ
⊢ ConnectedSpace α
[PROOFSTEP]
haveI : PreconnectedSpace α := ⟨by rw [← h]; exact isPreconnected_connectedComponent⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
h : connectedComponent x = univ
⊢ IsPreconnected univ
[PROOFSTEP]
rw [← h]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
h : connectedComponent x = univ
⊢ IsPreconnected (connectedComponent x)
[PROOFSTEP]
exact isPreconnected_connectedComponent
[GOAL]
case mpr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
h : connectedComponent x = univ
this : PreconnectedSpace α
⊢ ConnectedSpace α
[PROOFSTEP]
exact ⟨⟨x⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ PreconnectedSpace α ↔ ∀ (x : α), connectedComponent x = univ
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ PreconnectedSpace α → ∀ (x : α), connectedComponent x = univ
[PROOFSTEP]
intro h x
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : PreconnectedSpace α
x : α
⊢ connectedComponent x = univ
[PROOFSTEP]
exact eq_univ_of_univ_subset <| isPreconnected_univ.subset_connectedComponent (mem_univ x)
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α), connectedComponent x = univ) → PreconnectedSpace α
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
⊢ PreconnectedSpace α
[PROOFSTEP]
cases' isEmpty_or_nonempty α with hα hα
[GOAL]
case mpr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
hα : IsEmpty α
⊢ PreconnectedSpace α
[PROOFSTEP]
exact ⟨by rw [univ_eq_empty_iff.mpr hα]; exact isPreconnected_empty⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
hα : IsEmpty α
⊢ IsPreconnected univ
[PROOFSTEP]
rw [univ_eq_empty_iff.mpr hα]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
hα : IsEmpty α
⊢ IsPreconnected ∅
[PROOFSTEP]
exact isPreconnected_empty
[GOAL]
case mpr.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
hα : Nonempty α
⊢ PreconnectedSpace α
[PROOFSTEP]
exact ⟨by rw [← h (Classical.choice hα)]; exact isPreconnected_connectedComponent⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
hα : Nonempty α
⊢ IsPreconnected univ
[PROOFSTEP]
rw [← h (Classical.choice hα)]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), connectedComponent x = univ
hα : Nonempty α
⊢ IsPreconnected (connectedComponent (Classical.choice hα))
[PROOFSTEP]
exact isPreconnected_connectedComponent
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s t u v : Set α
inst✝² : TopologicalSpace β
inst✝¹ : PreconnectedSpace α
inst✝ : PreconnectedSpace β
⊢ IsPreconnected univ
[PROOFSTEP]
rw [← univ_prod_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s t u v : Set α
inst✝² : TopologicalSpace β
inst✝¹ : PreconnectedSpace α
inst✝ : PreconnectedSpace β
⊢ IsPreconnected (univ ×ˢ univ)
[PROOFSTEP]
exact isPreconnected_univ.prod isPreconnected_univ
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), PreconnectedSpace (π i)
⊢ IsPreconnected univ
[PROOFSTEP]
rw [← pi_univ univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), PreconnectedSpace (π i)
⊢ IsPreconnected (pi univ fun i => univ)
[PROOFSTEP]
exact isPreconnected_univ_pi fun i => isPreconnected_univ
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) × π i
hf : Continuous f
⊢ ∃ i g, Continuous g ∧ f = Sigma.mk i ∘ g
[PROOFSTEP]
obtain ⟨i, hi⟩ : ∃ i, range f ⊆ range (.mk i)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) × π i
hf : Continuous f
⊢ ∃ i, range f ⊆ range (Sigma.mk i)
[PROOFSTEP]
rcases Sigma.isConnected_iff.1 (isConnected_range hf) with ⟨i, s, -, hs⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) × π i
hf : Continuous f
i : ι
s : Set (π i)
hs : range f = Sigma.mk i '' s
⊢ ∃ i, range f ⊆ range (Sigma.mk i)
[PROOFSTEP]
exact ⟨i, hs.trans_subset (image_subset_range _ _)⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) × π i
hf : Continuous f
i : ι
hi : range f ⊆ range (Sigma.mk i)
⊢ ∃ i g, Continuous g ∧ f = Sigma.mk i ∘ g
[PROOFSTEP]
rcases range_subset_range_iff_exists_comp.1 hi with ⟨g, rfl⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
i : ι
g : α → π i
hf : Continuous (Sigma.mk i ∘ g)
hi : range (Sigma.mk i ∘ g) ⊆ range (Sigma.mk i)
⊢ ∃ i_1 g_1, Continuous g_1 ∧ Sigma.mk i ∘ g = Sigma.mk i_1 ∘ g_1
[PROOFSTEP]
refine ⟨i, g, ?_, rfl⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : ConnectedSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
i : ι
g : α → π i
hf : Continuous (Sigma.mk i ∘ g)
hi : range (Sigma.mk i ∘ g) ⊆ range (Sigma.mk i)
⊢ Continuous g
[PROOFSTEP]
rwa [← embedding_sigmaMk.continuous_iff] at hf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t✝ u v : Set α
inst✝ : PreconnectedSpace α
s t : Set α
⊢ IsOpen s → IsOpen t → s ∪ t = univ → Set.Nonempty s → Set.Nonempty t → Set.Nonempty (s ∩ t)
[PROOFSTEP]
simpa only [univ_inter, univ_subset_iff] using @PreconnectedSpace.isPreconnected_univ α _ _ s t
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : Set α
hs : IsClopen s
h : ¬(s = ∅ ∨ s = univ)
h2 : sᶜ = ∅
⊢ s = univ
[PROOFSTEP]
rw [← compl_compl s, h2, compl_empty]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : Set α
⊢ s = ∅ ∨ s = univ → IsClopen s
[PROOFSTEP]
rintro (rfl | rfl) <;> [exact isClopen_empty; exact isClopen_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : Set α
⊢ s = ∅ ∨ s = univ → IsClopen s
[PROOFSTEP]
rintro (rfl | rfl)
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : PreconnectedSpace α
⊢ IsClopen ∅
[PROOFSTEP]
exact isClopen_empty
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : PreconnectedSpace α
⊢ IsClopen univ
[PROOFSTEP]
exact isClopen_univ
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
⊢ Subsingleton ι
[PROOFSTEP]
replace h_nonempty : ∀ i, s i ≠ ∅ := by intro i; rw [← nonempty_iff_ne_empty]; exact h_nonempty i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
⊢ ∀ (i : ι), s i ≠ ∅
[PROOFSTEP]
intro i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
i : ι
⊢ s i ≠ ∅
[PROOFSTEP]
rw [← nonempty_iff_ne_empty]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
i : ι
⊢ Set.Nonempty (s i)
[PROOFSTEP]
exact h_nonempty i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
⊢ Subsingleton ι
[PROOFSTEP]
rw [← not_nontrivial_iff_subsingleton]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
⊢ ¬Nontrivial ι
[PROOFSTEP]
by_contra contra
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
contra : Nontrivial ι
⊢ False
[PROOFSTEP]
obtain ⟨i, j, h_ne⟩ := contra
[GOAL]
case mk.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
i j : ι
h_ne : i ≠ j
⊢ False
[PROOFSTEP]
replace h_ne : s i ∩ s j = ∅ := by
simpa only [← bot_eq_empty, eq_bot_iff, ← inf_eq_inter, ← disjoint_iff_inf_le] using h_disj h_ne
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
i j : ι
h_ne : i ≠ j
⊢ s i ∩ s j = ∅
[PROOFSTEP]
simpa only [← bot_eq_empty, eq_bot_iff, ← inf_eq_inter, ← disjoint_iff_inf_le] using h_disj h_ne
[GOAL]
case mk.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
i j : ι
h_ne : s i ∩ s j = ∅
⊢ False
[PROOFSTEP]
cases' isClopen_iff.mp (h_clopen i) with hi hi
[GOAL]
case mk.intro.intro.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
i j : ι
h_ne : s i ∩ s j = ∅
hi : s i = ∅
⊢ False
[PROOFSTEP]
exact h_nonempty i hi
[GOAL]
case mk.intro.intro.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
i j : ι
h_ne : s i ∩ s j = ∅
hi : s i = univ
⊢ False
[PROOFSTEP]
rw [hi, univ_inter] at h_ne
[GOAL]
case mk.intro.intro.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_disj : Pairwise (Disjoint on s)
h_clopen : ∀ (i : ι), IsClopen (s i)
h_nonempty : ∀ (i : ι), s i ≠ ∅
i j : ι
h_ne : s j = ∅
hi : s i = univ
⊢ False
[PROOFSTEP]
exact h_nonempty j h_ne
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_open : ∀ (i : ι), IsOpen (s i)
h_Union : ⋃ (i : ι), s i = univ
⊢ Subsingleton ι
[PROOFSTEP]
refine' subsingleton_of_disjoint_isClopen h_nonempty h_disj (fun i ↦ ⟨h_open i, _⟩)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_open : ∀ (i : ι), IsOpen (s i)
h_Union : ⋃ (i : ι), s i = univ
i : ι
⊢ IsClosed (s i)
[PROOFSTEP]
rw [← isOpen_compl_iff, compl_eq_univ_diff, ← h_Union, iUnion_diff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_open : ∀ (i : ι), IsOpen (s i)
h_Union : ⋃ (i : ι), s i = univ
i : ι
⊢ IsOpen (⋃ (i_1 : ι), s i_1 \ s i)
[PROOFSTEP]
refine' isOpen_iUnion (fun j ↦ _)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_open : ∀ (i : ι), IsOpen (s i)
h_Union : ⋃ (i : ι), s i = univ
i j : ι
⊢ IsOpen (s j \ s i)
[PROOFSTEP]
rcases eq_or_ne i j with rfl | h_ne
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_open : ∀ (i : ι), IsOpen (s i)
h_Union : ⋃ (i : ι), s i = univ
i : ι
⊢ IsOpen (s i \ s i)
[PROOFSTEP]
simp
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
h_open : ∀ (i : ι), IsOpen (s i)
h_Union : ⋃ (i : ι), s i = univ
i j : ι
h_ne : i ≠ j
⊢ IsOpen (s j \ s i)
[PROOFSTEP]
simpa only [(h_disj h_ne.symm).sdiff_eq_left] using h_open j
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
inst✝ : Finite ι
h_closed : ∀ (i : ι), IsClosed (s i)
h_Union : ⋃ (i : ι), s i = univ
⊢ Subsingleton ι
[PROOFSTEP]
refine' subsingleton_of_disjoint_isClopen h_nonempty h_disj (fun i ↦ ⟨_, h_closed i⟩)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
inst✝ : Finite ι
h_closed : ∀ (i : ι), IsClosed (s i)
h_Union : ⋃ (i : ι), s i = univ
i : ι
⊢ IsOpen (s i)
[PROOFSTEP]
rw [← isClosed_compl_iff, compl_eq_univ_diff, ← h_Union, iUnion_diff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
inst✝ : Finite ι
h_closed : ∀ (i : ι), IsClosed (s i)
h_Union : ⋃ (i : ι), s i = univ
i : ι
⊢ IsClosed (⋃ (i_1 : ι), s i_1 \ s i)
[PROOFSTEP]
refine' isClosed_iUnion (fun j ↦ _)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
inst✝ : Finite ι
h_closed : ∀ (i : ι), IsClosed (s i)
h_Union : ⋃ (i : ι), s i = univ
i j : ι
⊢ IsClosed (s j \ s i)
[PROOFSTEP]
rcases eq_or_ne i j with rfl | h_ne
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
inst✝ : Finite ι
h_closed : ∀ (i : ι), IsClosed (s i)
h_Union : ⋃ (i : ι), s i = univ
i : ι
⊢ IsClosed (s i \ s i)
[PROOFSTEP]
simp
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : PreconnectedSpace α
s : ι → Set α
h_nonempty : ∀ (i : ι), Set.Nonempty (s i)
h_disj : Pairwise (Disjoint on s)
inst✝ : Finite ι
h_closed : ∀ (i : ι), IsClosed (s i)
h_Union : ⋃ (i : ι), s i = univ
i j : ι
h_ne : i ≠ j
⊢ IsClosed (s j \ s i)
[PROOFSTEP]
simpa only [(h_disj h_ne.symm).sdiff_eq_left] using h_closed j
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : PreconnectedSpace α
s : Set α
⊢ Set.Nonempty (frontier s) ↔ Set.Nonempty s ∧ s ≠ univ
[PROOFSTEP]
simp only [nonempty_iff_ne_empty, Ne.def, frontier_eq_empty_iff, not_or]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
h : IsPreconnected s
⊢ IsPreconnected univ
[PROOFSTEP]
rwa [← inducing_subtype_val.isPreconnected_image, image_univ, Subtype.range_val]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
h : PreconnectedSpace ↑s
⊢ IsPreconnected s
[PROOFSTEP]
simpa using isPreconnected_univ.image ((↑) : s → α) continuous_subtype_val.continuousOn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
⊢ P x y
[PROOFSTEP]
let u := {z | P x z}
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
⊢ P x y
[PROOFSTEP]
have A : IsOpen u := by
apply isOpen_iff_mem_nhds.2 (fun z hz ↦ ?_)
filter_upwards [h z] with t ht
exact h' hz ht.1
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
⊢ IsOpen u
[PROOFSTEP]
apply isOpen_iff_mem_nhds.2 (fun z hz ↦ ?_)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
z : α
hz : z ∈ u
⊢ u ∈ 𝓝 z
[PROOFSTEP]
filter_upwards [h z] with t ht
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
z : α
hz : z ∈ u
t : α
ht : P z t ∧ P t z
⊢ P x t
[PROOFSTEP]
exact h' hz ht.1
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
⊢ P x y
[PROOFSTEP]
have B : IsClosed u := by
apply isClosed_iff_nhds.2 (fun z hz ↦ ?_)
rcases hz _ (h z) with ⟨t, ht, h't⟩
exact h' h't ht.2
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
⊢ IsClosed u
[PROOFSTEP]
apply isClosed_iff_nhds.2 (fun z hz ↦ ?_)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
z : α
hz : ∀ (U : Set α), U ∈ 𝓝 z → Set.Nonempty (U ∩ u)
⊢ z ∈ u
[PROOFSTEP]
rcases hz _ (h z) with ⟨t, ht, h't⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
z : α
hz : ∀ (U : Set α), U ∈ 𝓝 z → Set.Nonempty (U ∩ u)
t : α
ht : t ∈ {x | (fun y => P z y ∧ P y z) x}
h't : t ∈ u
⊢ z ∈ u
[PROOFSTEP]
exact h' h't ht.2
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
B : IsClosed u
⊢ P x y
[PROOFSTEP]
have C : u.Nonempty := ⟨x, (mem_of_mem_nhds (h x)).1⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
B : IsClosed u
C : Set.Nonempty u
⊢ P x y
[PROOFSTEP]
have D : u = Set.univ := IsClopen.eq_univ ⟨A, B⟩ C
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
B : IsClosed u
C : Set.Nonempty u
D : u = univ
⊢ P x y
[PROOFSTEP]
show y ∈ u
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u✝ v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y ∧ P y x
h' : Transitive P
x y : α
u : Set α := {z | P x z}
A : IsOpen u
B : IsClosed u
C : Set.Nonempty u
D : u = univ
⊢ y ∈ u
[PROOFSTEP]
simp [D]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y
h' : Transitive P
h'' : Symmetric P
x y : α
⊢ P x y
[PROOFSTEP]
refine PreconnectedSpace.induction₂' P (fun z ↦ ?_) h' x y
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y
h' : Transitive P
h'' : Symmetric P
x y z : α
⊢ ∀ᶠ (y : α) in 𝓝 z, P z y ∧ P y z
[PROOFSTEP]
filter_upwards [h z] with a ha
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : PreconnectedSpace α
P : α → α → Prop
h : ∀ (x : α), ∀ᶠ (y : α) in 𝓝 x, P x y
h' : Transitive P
h'' : Symmetric P
x y z a : α
ha : P z a
⊢ P z a ∧ P a z
[PROOFSTEP]
refine ⟨ha, h'' ha⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
⊢ P x y
[PROOFSTEP]
let Q : s → s → Prop := fun a b ↦ P a b
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
⊢ P x y
[PROOFSTEP]
show Q ⟨x, hx⟩ ⟨y, hy⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
⊢ Q { val := x, property := hx } { val := y, property := hy }
[PROOFSTEP]
have : PreconnectedSpace s := Subtype.preconnectedSpace hs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
this : PreconnectedSpace ↑s
⊢ Q { val := x, property := hx } { val := y, property := hy }
[PROOFSTEP]
apply PreconnectedSpace.induction₂'
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
this : PreconnectedSpace ↑s
⊢ ∀ (x : { x // x ∈ s }), ∀ᶠ (y : { x // x ∈ s }) in 𝓝 x, Q x y ∧ Q y x
[PROOFSTEP]
rintro ⟨x, hx⟩
[GOAL]
case h.mk
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x✝ y : α
hx✝ : x✝ ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
this : PreconnectedSpace ↑s
x : α
hx : x ∈ s
⊢ ∀ᶠ (y : { x // x ∈ s }) in 𝓝 { val := x, property := hx },
Q { val := x, property := hx } y ∧ Q y { val := x, property := hx }
[PROOFSTEP]
have Z := h x hx
[GOAL]
case h.mk
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x✝ y : α
hx✝ : x✝ ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
this : PreconnectedSpace ↑s
x : α
hx : x ∈ s
Z : ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
⊢ ∀ᶠ (y : { x // x ∈ s }) in 𝓝 { val := x, property := hx },
Q { val := x, property := hx } y ∧ Q y { val := x, property := hx }
[PROOFSTEP]
rwa [nhdsWithin_eq_map_subtype_coe] at Z
[GOAL]
case h'
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
this : PreconnectedSpace ↑s
⊢ Transitive Q
[PROOFSTEP]
rintro ⟨a, ha⟩ ⟨b, hb⟩ ⟨c, hc⟩ hab hbc
[GOAL]
case h'.mk.mk.mk
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y ∧ P y x
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
x y : α
hx : x ∈ s
hy : y ∈ s
Q : ↑s → ↑s → Prop := fun a b => P ↑a ↑b
this : PreconnectedSpace ↑s
a : α
ha : a ∈ s
b : α
hb : b ∈ s
c : α
hc : c ∈ s
hab : Q { val := a, property := ha } { val := b, property := hb }
hbc : Q { val := b, property := hb } { val := c, property := hc }
⊢ Q { val := a, property := ha } { val := c, property := hc }
[PROOFSTEP]
exact h' a b c ha hb hc hab hbc
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
h'' : ∀ (x y : α), x ∈ s → y ∈ s → P x y → P y x
x y : α
hx : x ∈ s
hy : y ∈ s
⊢ P x y
[PROOFSTEP]
apply hs.induction₂' P (fun z hz ↦ ?_) h' hx hy
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
h'' : ∀ (x y : α), x ∈ s → y ∈ s → P x y → P y x
x y : α
hx : x ∈ s
hy : y ∈ s
z : α
hz : z ∈ s
⊢ ∀ᶠ (y : α) in 𝓝[s] z, P z y ∧ P y z
[PROOFSTEP]
filter_upwards [h z hz, self_mem_nhdsWithin] with a ha h'a
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsPreconnected s
P : α → α → Prop
h : ∀ (x : α), x ∈ s → ∀ᶠ (y : α) in 𝓝[s] x, P x y
h' : ∀ (x y z : α), x ∈ s → y ∈ s → z ∈ s → P x y → P y z → P x z
h'' : ∀ (x y : α), x ∈ s → y ∈ s → P x y → P y x
x y : α
hx : x ∈ s
hy : y ∈ s
z : α
hz : z ∈ s
a : α
ha : P z a
h'a : a ∈ s
⊢ P z a ∧ P a z
[PROOFSTEP]
exact ⟨ha, h'' z a hz h'a ha⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ IsPreconnected s ↔ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ IsPreconnected s → ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ (∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v) → IsPreconnected s
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
h : IsPreconnected s
⊢ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
intro u v hu hv hs huv
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h : IsPreconnected s
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
specialize h u v hu hv hs
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
contrapose! huv
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
huv : ¬s ⊆ u ∧ ¬s ⊆ v
⊢ s ∩ (u ∩ v) ≠ ∅
[PROOFSTEP]
rw [← nonempty_iff_ne_empty]
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
huv : ¬s ⊆ u ∧ ¬s ⊆ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
simp [not_subset] at huv
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
huv : (∃ a, a ∈ s ∧ ¬a ∈ u) ∧ ∃ a, a ∈ s ∧ ¬a ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases huv with ⟨⟨x, hxs, hxu⟩, ⟨y, hys, hyv⟩⟩
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
x : α
hxs : x ∈ s
hxu : ¬x ∈ u
y : α
hys : y ∈ s
hyv : ¬y ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have hxv : x ∈ v := or_iff_not_imp_left.mp (hs hxs) hxu
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
x : α
hxs : x ∈ s
hxu : ¬x ∈ u
y : α
hys : y ∈ s
hyv : ¬y ∈ v
hxv : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have hyu : y ∈ u := or_iff_not_imp_right.mp (hs hys) hyv
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
x : α
hxs : x ∈ s
hxu : ¬x ∈ u
y : α
hys : y ∈ s
hyv : ¬y ∈ v
hxv : x ∈ v
hyu : y ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact h ⟨y, hys, hyu⟩ ⟨x, hxs, hxv⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
⊢ IsPreconnected s
[PROOFSTEP]
intro u v hu hv hs hsu hsv
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rw [nonempty_iff_ne_empty]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
⊢ s ∩ (u ∩ v) ≠ ∅
[PROOFSTEP]
intro H
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : s ∩ (u ∩ v) = ∅
⊢ False
[PROOFSTEP]
specialize h u v hu hv hs H
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : s ∩ (u ∩ v) = ∅
h : s ⊆ u ∨ s ⊆ v
⊢ False
[PROOFSTEP]
contrapose H
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
h : s ⊆ u ∨ s ⊆ v
H : ¬False
⊢ ¬s ∩ (u ∩ v) = ∅
[PROOFSTEP]
apply Nonempty.ne_empty
[GOAL]
case mpr.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
h : s ⊆ u ∨ s ⊆ v
H : ¬False
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
cases' h with h h
[GOAL]
case mpr.a.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : ¬False
h : s ⊆ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases hsv with ⟨x, hxs, hxv⟩
[GOAL]
case mpr.a.inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
H : ¬False
h : s ⊆ u
x : α
hxs : x ∈ s
hxv : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨x, hxs, ⟨h hxs, hxv⟩⟩
[GOAL]
case mpr.a.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : ¬False
h : s ⊆ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases hsu with ⟨x, hxs, hxu⟩
[GOAL]
case mpr.a.inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsv : Set.Nonempty (s ∩ v)
H : ¬False
h : s ⊆ v
x : α
hxs : x ∈ s
hxu : x ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨x, hxs, ⟨hxu, h hxs⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ IsConnected s ↔
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
[PROOFSTEP]
rw [IsConnected, isPreconnected_iff_subset_of_disjoint]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
⊢ (Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v) ↔
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
[PROOFSTEP]
refine ⟨fun ⟨hne, h⟩ U hU hUo hsU => ?_, fun h => ⟨?_, fun u v hu hv hs hsuv => ?_⟩⟩
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
U : Finset (Set α)
hU : ∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ U → IsOpen u
hsU : s ⊆ ⋃₀ ↑U
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
⊢ ∃ u, u ∈ U ∧ s ⊆ u
[PROOFSTEP]
induction U using Finset.induction_on
[GOAL]
case refine_1.empty
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hU : ∀ (u v : Set α), u ∈ ∅ → v ∈ ∅ → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hsU : s ⊆ ⋃₀ ↑∅
⊢ ∃ u, u ∈ ∅ ∧ s ⊆ u
case refine_1.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝¹ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
a✝² : Set α
s✝ : Finset (Set α)
a✝¹ : ¬a✝² ∈ s✝
a✝ :
(∀ (u v : Set α), u ∈ s✝ → v ∈ s✝ → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ s✝ → IsOpen u) → s ⊆ ⋃₀ ↑s✝ → ∃ u, u ∈ s✝ ∧ s ⊆ u
hU : ∀ (u v : Set α), u ∈ insert a✝² s✝ → v ∈ insert a✝² s✝ → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ insert a✝² s✝ → IsOpen u
hsU : s ⊆ ⋃₀ ↑(insert a✝² s✝)
⊢ ∃ u, u ∈ insert a✝² s✝ ∧ s ⊆ u
[PROOFSTEP]
case empty => exact absurd (by simpa using hsU) hne.not_subset_empty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hU : ∀ (u v : Set α), u ∈ ∅ → v ∈ ∅ → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hsU : s ⊆ ⋃₀ ↑∅
⊢ ∃ u, u ∈ ∅ ∧ s ⊆ u
[PROOFSTEP]
case empty => exact absurd (by simpa using hsU) hne.not_subset_empty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hU : ∀ (u v : Set α), u ∈ ∅ → v ∈ ∅ → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hsU : s ⊆ ⋃₀ ↑∅
⊢ ∃ u, u ∈ ∅ ∧ s ⊆ u
[PROOFSTEP]
exact absurd (by simpa using hsU) hne.not_subset_empty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hU : ∀ (u v : Set α), u ∈ ∅ → v ∈ ∅ → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hsU : s ⊆ ⋃₀ ↑∅
⊢ s ⊆ ∅
[PROOFSTEP]
simpa using hsU
[GOAL]
case refine_1.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝¹ t u v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
a✝² : Set α
s✝ : Finset (Set α)
a✝¹ : ¬a✝² ∈ s✝
a✝ :
(∀ (u v : Set α), u ∈ s✝ → v ∈ s✝ → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ s✝ → IsOpen u) → s ⊆ ⋃₀ ↑s✝ → ∃ u, u ∈ s✝ ∧ s ⊆ u
hU : ∀ (u v : Set α), u ∈ insert a✝² s✝ → v ∈ insert a✝² s✝ → Set.Nonempty (s ∩ (u ∩ v)) → u = v
hUo : ∀ (u : Set α), u ∈ insert a✝² s✝ → IsOpen u
hsU : s ⊆ ⋃₀ ↑(insert a✝² s✝)
⊢ ∃ u, u ∈ insert a✝² s✝ ∧ s ⊆ u
[PROOFSTEP]
case insert u U uU
IH =>
simp only [← ball_cond_comm, Finset.forall_mem_insert, Finset.exists_mem_insert, Finset.coe_insert, sUnion_insert,
implies_true, true_and] at *
refine (h _ hUo.1 (⋃₀ ↑U) (isOpen_sUnion hUo.2) hsU ?_).imp_right ?_
· refine subset_empty_iff.1 fun x ⟨hxs, hxu, v, hvU, hxv⟩ => ?_
exact ne_of_mem_of_not_mem hvU uU (hU.1 v hvU ⟨x, hxs, hxu, hxv⟩).symm
· exact IH (fun u hu => (hU.2 u hu).2) hUo.2
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u : Set α
U : Finset (Set α)
uU : ¬u ∈ U
IH :
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
hU : ∀ (u_1 v : Set α), u_1 ∈ insert u U → v ∈ insert u U → Set.Nonempty (s ∩ (u_1 ∩ v)) → u_1 = v
hUo : ∀ (u_1 : Set α), u_1 ∈ insert u U → IsOpen u_1
hsU : s ⊆ ⋃₀ ↑(insert u U)
⊢ ∃ u_1, u_1 ∈ insert u U ∧ s ⊆ u_1
[PROOFSTEP]
case insert u U uU
IH =>
simp only [← ball_cond_comm, Finset.forall_mem_insert, Finset.exists_mem_insert, Finset.coe_insert, sUnion_insert,
implies_true, true_and] at *
refine (h _ hUo.1 (⋃₀ ↑U) (isOpen_sUnion hUo.2) hsU ?_).imp_right ?_
· refine subset_empty_iff.1 fun x ⟨hxs, hxu, v, hvU, hxv⟩ => ?_
exact ne_of_mem_of_not_mem hvU uU (hU.1 v hvU ⟨x, hxs, hxu, hxv⟩).symm
· exact IH (fun u hu => (hU.2 u hu).2) hUo.2
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v s : Set α
x✝ : Set.Nonempty s ∧ ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
hne : Set.Nonempty s
h : ∀ (u v : Set α), IsOpen u → IsOpen v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u : Set α
U : Finset (Set α)
uU : ¬u ∈ U
IH :
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
hU : ∀ (u_1 v : Set α), u_1 ∈ insert u U → v ∈ insert u U → Set.Nonempty (s ∩ (u_1 ∩ v)) → u_1 = v
hUo : ∀ (u_1 : Set α), u_1 ∈ insert u U → IsOpen u_1
hsU : s ⊆ ⋃₀ ↑(insert u U)
⊢ ∃ u_1, u_1 ∈ insert u U ∧ s ⊆ u_1
[PROOFSTEP]
simp only [← ball_cond_comm, Finset.forall_mem_insert, Finset.exists_mem_insert, Finset.coe_insert, sUnion_insert,
implies_true, true_and] at *
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v s : Set α
hne : Set.Nonempty s
u : Set α
U : Finset (Set α)
uU : ¬u ∈ U
x✝ : Set.Nonempty s ∧ ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
h : ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
IH :
(∀ (a : Set α), a ∈ U → ∀ (b : Set α), b ∈ U → Set.Nonempty (s ∩ (a ∩ b)) → a = b) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
hU :
(∀ (x : Set α), x ∈ U → Set.Nonempty (s ∩ (u ∩ x)) → u = x) ∧
∀ (x : Set α),
x ∈ U → (Set.Nonempty (s ∩ (x ∩ u)) → x = u) ∧ ∀ (x_1 : Set α), x_1 ∈ U → Set.Nonempty (s ∩ (x ∩ x_1)) → x = x_1
hUo : IsOpen u ∧ ∀ (x : Set α), x ∈ U → IsOpen x
hsU : s ⊆ u ∪ ⋃₀ ↑U
⊢ s ⊆ u ∨ ∃ x, x ∈ U ∧ s ⊆ x
[PROOFSTEP]
refine (h _ hUo.1 (⋃₀ ↑U) (isOpen_sUnion hUo.2) hsU ?_).imp_right ?_
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v s : Set α
hne : Set.Nonempty s
u : Set α
U : Finset (Set α)
uU : ¬u ∈ U
x✝ : Set.Nonempty s ∧ ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
h : ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
IH :
(∀ (a : Set α), a ∈ U → ∀ (b : Set α), b ∈ U → Set.Nonempty (s ∩ (a ∩ b)) → a = b) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
hU :
(∀ (x : Set α), x ∈ U → Set.Nonempty (s ∩ (u ∩ x)) → u = x) ∧
∀ (x : Set α),
x ∈ U → (Set.Nonempty (s ∩ (x ∩ u)) → x = u) ∧ ∀ (x_1 : Set α), x_1 ∈ U → Set.Nonempty (s ∩ (x ∩ x_1)) → x = x_1
hUo : IsOpen u ∧ ∀ (x : Set α), x ∈ U → IsOpen x
hsU : s ⊆ u ∪ ⋃₀ ↑U
⊢ s ∩ (u ∩ ⋃₀ ↑U) = ∅
[PROOFSTEP]
refine subset_empty_iff.1 fun x ⟨hxs, hxu, v, hvU, hxv⟩ => ?_
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hne : Set.Nonempty s
u : Set α
U : Finset (Set α)
uU : ¬u ∈ U
x✝¹ : Set.Nonempty s ∧ ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
h : ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
IH :
(∀ (a : Set α), a ∈ U → ∀ (b : Set α), b ∈ U → Set.Nonempty (s ∩ (a ∩ b)) → a = b) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
hU :
(∀ (x : Set α), x ∈ U → Set.Nonempty (s ∩ (u ∩ x)) → u = x) ∧
∀ (x : Set α),
x ∈ U → (Set.Nonempty (s ∩ (x ∩ u)) → x = u) ∧ ∀ (x_1 : Set α), x_1 ∈ U → Set.Nonempty (s ∩ (x ∩ x_1)) → x = x_1
hUo : IsOpen u ∧ ∀ (x : Set α), x ∈ U → IsOpen x
hsU : s ⊆ u ∪ ⋃₀ ↑U
x : α
x✝ : x ∈ s ∩ (u ∩ ⋃₀ ↑U)
hxs : x ∈ s
hxu : x ∈ u
v : Set α
hvU : v ∈ ↑U
hxv : x ∈ v
⊢ x ∈ ∅
[PROOFSTEP]
exact ne_of_mem_of_not_mem hvU uU (hU.1 v hvU ⟨x, hxs, hxu, hxv⟩).symm
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v s : Set α
hne : Set.Nonempty s
u : Set α
U : Finset (Set α)
uU : ¬u ∈ U
x✝ : Set.Nonempty s ∧ ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
h : ∀ (a : Set α), IsOpen a → ∀ (b : Set α), IsOpen b → s ⊆ a ∪ b → s ∩ (a ∩ b) = ∅ → s ⊆ a ∨ s ⊆ b
IH :
(∀ (a : Set α), a ∈ U → ∀ (b : Set α), b ∈ U → Set.Nonempty (s ∩ (a ∩ b)) → a = b) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
hU :
(∀ (x : Set α), x ∈ U → Set.Nonempty (s ∩ (u ∩ x)) → u = x) ∧
∀ (x : Set α),
x ∈ U → (Set.Nonempty (s ∩ (x ∩ u)) → x = u) ∧ ∀ (x_1 : Set α), x_1 ∈ U → Set.Nonempty (s ∩ (x ∩ x_1)) → x = x_1
hUo : IsOpen u ∧ ∀ (x : Set α), x ∈ U → IsOpen x
hsU : s ⊆ u ∪ ⋃₀ ↑U
⊢ s ⊆ ⋃₀ ↑U → ∃ x, x ∈ U ∧ s ⊆ x
[PROOFSTEP]
exact IH (fun u hu => (hU.2 u hu).2) hUo.2
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
⊢ Set.Nonempty s
[PROOFSTEP]
simpa [subset_empty_iff, nonempty_iff_ne_empty] using h ∅
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsuv : s ∩ (u ∩ v) = ∅
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
rw [← not_nonempty_iff_eq_empty] at hsuv
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsuv : ¬Set.Nonempty (s ∩ (u ∩ v))
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
have := hsuv
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsuv this : ¬Set.Nonempty (s ∩ (u ∩ v))
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
rw [inter_comm u] at this
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u v : Set α), u ∈ U → v ∈ U → Set.Nonempty (s ∩ (u ∩ v)) → u = v) →
(∀ (u : Set α), u ∈ U → IsOpen u) → s ⊆ ⋃₀ ↑U → ∃ u, u ∈ U ∧ s ⊆ u
u v : Set α
hu : IsOpen u
hv : IsOpen v
hs : s ⊆ u ∪ v
hsuv : ¬Set.Nonempty (s ∩ (u ∩ v))
this : ¬Set.Nonempty (s ∩ (v ∩ u))
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
simpa [*, or_imp, forall_and] using h { u, v }
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ IsPreconnected s ↔ ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ IsPreconnected s → ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v) → IsPreconnected s
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : IsPreconnected s
⊢ ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
intro u v hu hv hs huv
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ : Set α
h : IsPreconnected s
u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
rw [isPreconnected_closed_iff] at h
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ : Set α
h :
∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
specialize h u v hu hv hs
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
contrapose! huv
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
huv : ¬s ⊆ u ∧ ¬s ⊆ v
⊢ s ∩ (u ∩ v) ≠ ∅
[PROOFSTEP]
rw [← nonempty_iff_ne_empty]
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
huv : ¬s ⊆ u ∧ ¬s ⊆ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
simp [not_subset] at huv
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
huv : (∃ a, a ∈ s ∧ ¬a ∈ u) ∧ ∃ a, a ∈ s ∧ ¬a ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases huv with ⟨⟨x, hxs, hxu⟩, ⟨y, hys, hyv⟩⟩
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
x : α
hxs : x ∈ s
hxu : ¬x ∈ u
y : α
hys : y ∈ s
hyv : ¬y ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have hxv : x ∈ v := or_iff_not_imp_left.mp (hs hxs) hxu
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
x : α
hxs : x ∈ s
hxu : ¬x ∈ u
y : α
hys : y ∈ s
hyv : ¬y ∈ v
hxv : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
have hyu : y ∈ u := or_iff_not_imp_right.mp (hs hys) hyv
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
h : Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
x : α
hxs : x ∈ s
hxu : ¬x ∈ u
y : α
hys : y ∈ s
hyv : ¬y ∈ v
hxv : x ∈ v
hyu : y ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact h ⟨y, hys, hyu⟩ ⟨x, hxs, hxv⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
⊢ IsPreconnected s
[PROOFSTEP]
rw [isPreconnected_closed_iff]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
⊢ ∀ (t t' : Set α),
IsClosed t → IsClosed t' → s ⊆ t ∪ t' → Set.Nonempty (s ∩ t) → Set.Nonempty (s ∩ t') → Set.Nonempty (s ∩ (t ∩ t'))
[PROOFSTEP]
intro u v hu hv hs hsu hsv
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ : Set α
h : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rw [nonempty_iff_ne_empty]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ : Set α
h : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
⊢ s ∩ (u ∩ v) ≠ ∅
[PROOFSTEP]
intro H
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ : Set α
h : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : s ∩ (u ∩ v) = ∅
⊢ False
[PROOFSTEP]
specialize h u v hu hv hs H
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : s ∩ (u ∩ v) = ∅
h : s ⊆ u ∨ s ⊆ v
⊢ False
[PROOFSTEP]
contrapose H
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
h : s ⊆ u ∨ s ⊆ v
H : ¬False
⊢ ¬s ∩ (u ∩ v) = ∅
[PROOFSTEP]
apply Nonempty.ne_empty
[GOAL]
case mpr.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
h : s ⊆ u ∨ s ⊆ v
H : ¬False
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
cases' h with h h
[GOAL]
case mpr.a.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : ¬False
h : s ⊆ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases hsv with ⟨x, hxs, hxv⟩
[GOAL]
case mpr.a.inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
H : ¬False
h : s ⊆ u
x : α
hxs : x ∈ s
hxv : x ∈ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨x, hxs, ⟨h hxs, hxv⟩⟩
[GOAL]
case mpr.a.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsu : Set.Nonempty (s ∩ u)
hsv : Set.Nonempty (s ∩ v)
H : ¬False
h : s ⊆ v
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rcases hsu with ⟨x, hxs, hxu⟩
[GOAL]
case mpr.a.inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u✝ v✝ u v : Set α
hu : IsClosed u
hv : IsClosed v
hs : s ⊆ u ∪ v
hsv : Set.Nonempty (s ∩ v)
H : ¬False
h : s ⊆ v
x : α
hxs : x ∈ s
hxu : x ∈ u
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨x, hxs, ⟨hxu, h hxs⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsClosed s
⊢ IsPreconnected s ↔ ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
refine isPreconnected_iff_subset_of_disjoint_closed.trans ⟨?_, ?_⟩
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsClosed s
⊢ (∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v) →
∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
intro H u v hu hv hss huv
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : IsClosed s
⊢ (∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v) →
∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
intro H u v hu hv hss huv
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : Disjoint u v
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
apply H u v hu hv hss
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → s ∩ (u ∩ v) = ∅ → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : Disjoint u v
⊢ s ∩ (u ∩ v) = ∅
[PROOFSTEP]
rw [huv.inter_eq, inter_empty]
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
have H1 := H (u ∩ s) (v ∩ s)
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
H1 : IsClosed (u ∩ s) → IsClosed (v ∩ s) → s ⊆ u ∩ s ∪ v ∩ s → Disjoint (u ∩ s) (v ∩ s) → s ⊆ u ∩ s ∨ s ⊆ v ∩ s
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
rw [subset_inter_iff, subset_inter_iff] at H1
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
H1 : IsClosed (u ∩ s) → IsClosed (v ∩ s) → s ⊆ u ∩ s ∪ v ∩ s → Disjoint (u ∩ s) (v ∩ s) → s ⊆ u ∧ s ⊆ s ∨ s ⊆ v ∧ s ⊆ s
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
simp only [Subset.refl, and_true] at H1
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
H1 : IsClosed (u ∩ s) → IsClosed (v ∩ s) → s ⊆ u ∩ s ∪ v ∩ s → Disjoint (u ∩ s) (v ∩ s) → s ⊆ u ∨ s ⊆ v
⊢ s ⊆ u ∨ s ⊆ v
[PROOFSTEP]
apply H1 (hu.inter hs) (hv.inter hs)
[GOAL]
case refine_2.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
H1 : IsClosed (u ∩ s) → IsClosed (v ∩ s) → s ⊆ u ∩ s ∪ v ∩ s → Disjoint (u ∩ s) (v ∩ s) → s ⊆ u ∨ s ⊆ v
⊢ s ⊆ u ∩ s ∪ v ∩ s
[PROOFSTEP]
rw [← inter_distrib_right]
[GOAL]
case refine_2.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
H1 : IsClosed (u ∩ s) → IsClosed (v ∩ s) → s ⊆ u ∩ s ∪ v ∩ s → Disjoint (u ∩ s) (v ∩ s) → s ⊆ u ∨ s ⊆ v
⊢ s ⊆ (u ∪ v) ∩ s
[PROOFSTEP]
exact subset_inter hss Subset.rfl
[GOAL]
case refine_2.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : IsClosed s
H : ∀ (u v : Set α), IsClosed u → IsClosed v → s ⊆ u ∪ v → Disjoint u v → s ⊆ u ∨ s ⊆ v
u v : Set α
hu : IsClosed u
hv : IsClosed v
hss : s ⊆ u ∪ v
huv : s ∩ (u ∩ v) = ∅
H1 : IsClosed (u ∩ s) → IsClosed (v ∩ s) → s ⊆ u ∩ s ∪ v ∩ s → Disjoint (u ∩ s) (v ∩ s) → s ⊆ u ∨ s ⊆ v
⊢ Disjoint (u ∩ s) (v ∩ s)
[PROOFSTEP]
rwa [disjoint_iff_inter_eq_empty, ← inter_inter_distrib_right, inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
⊢ IsConnected (f ⁻¹' connectedComponent t)
[PROOFSTEP]
have hf : Surjective f := Surjective.of_comp fun t : β => (connected_fibers t).1
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
⊢ IsConnected (f ⁻¹' connectedComponent t)
[PROOFSTEP]
refine ⟨Nonempty.preimage connectedComponent_nonempty hf, ?_⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
⊢ IsPreconnected (f ⁻¹' connectedComponent t)
[PROOFSTEP]
have hT : IsClosed (f ⁻¹' connectedComponent t) := (hcl (connectedComponent t)).1 isClosed_connectedComponent
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
⊢ IsPreconnected (f ⁻¹' connectedComponent t)
[PROOFSTEP]
rw [isPreconnected_iff_subset_of_fully_disjoint_closed hT]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u v : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
⊢ ∀ (u v : Set α),
IsClosed u →
IsClosed v →
f ⁻¹' connectedComponent t ⊆ u ∪ v →
Disjoint u v → f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
intro u v hu hv huv uv_disj
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
let T₁ := {t' ∈ connectedComponent t | f ⁻¹' { t' } ⊆ u}
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
let T₂ := {t' ∈ connectedComponent t | f ⁻¹' { t' } ⊆ v}
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have fiber_decomp : ∀ t' ∈ connectedComponent t, f ⁻¹' { t' } ⊆ u ∨ f ⁻¹' { t' } ⊆ v :=
by
intro t' ht'
apply isPreconnected_iff_subset_of_disjoint_closed.1 (connected_fibers t').2 u v hu hv
· exact Subset.trans (preimage_mono (singleton_subset_iff.2 ht')) huv
rw [uv_disj.inter_eq, inter_empty]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
⊢ ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
[PROOFSTEP]
intro t' ht'
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
t' : β
ht' : t' ∈ connectedComponent t
⊢ f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
[PROOFSTEP]
apply isPreconnected_iff_subset_of_disjoint_closed.1 (connected_fibers t').2 u v hu hv
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
t' : β
ht' : t' ∈ connectedComponent t
⊢ f ⁻¹' {t'} ⊆ u ∪ v
[PROOFSTEP]
exact Subset.trans (preimage_mono (singleton_subset_iff.2 ht')) huv
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
t' : β
ht' : t' ∈ connectedComponent t
⊢ f ⁻¹' {t'} ∩ (u ∩ v) = ∅
[PROOFSTEP]
rw [uv_disj.inter_eq, inter_empty]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u :=
by
apply eq_of_subset_of_subset
· rw [← biUnion_preimage_singleton]
refine' iUnion₂_subset fun t' ht' => subset_inter _ ht'.2
rw [hf.preimage_subset_preimage_iff, singleton_subset_iff]
exact ht'.1
rintro a ⟨hat, hau⟩
constructor
· exact mem_preimage.1 hat
refine (fiber_decomp (f a) (mem_preimage.1 hat)).resolve_right fun h => ?_
exact
uv_disj.subset_compl_right hau
(h rfl)
-- This proof is exactly the same as the above (modulo some symmetry)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
⊢ f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
[PROOFSTEP]
apply eq_of_subset_of_subset
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
⊢ f ⁻¹' T₁ ⊆ f ⁻¹' connectedComponent t ∩ u
[PROOFSTEP]
rw [← biUnion_preimage_singleton]
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
⊢ ⋃ (y : β) (_ : y ∈ T₁), f ⁻¹' {y} ⊆ f ⁻¹' connectedComponent t ∩ u
[PROOFSTEP]
refine' iUnion₂_subset fun t' ht' => subset_inter _ ht'.2
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
t' : β
ht' : t' ∈ T₁
⊢ f ⁻¹' {t'} ⊆ f ⁻¹' connectedComponent t
[PROOFSTEP]
rw [hf.preimage_subset_preimage_iff, singleton_subset_iff]
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
t' : β
ht' : t' ∈ T₁
⊢ t' ∈ connectedComponent t
[PROOFSTEP]
exact ht'.1
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
⊢ f ⁻¹' connectedComponent t ∩ u ⊆ f ⁻¹' T₁
[PROOFSTEP]
rintro a ⟨hat, hau⟩
[GOAL]
case a.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hau : a ∈ u
⊢ a ∈ f ⁻¹' T₁
[PROOFSTEP]
constructor
[GOAL]
case a.intro.left
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hau : a ∈ u
⊢ f a ∈ connectedComponent t
[PROOFSTEP]
exact mem_preimage.1 hat
[GOAL]
case a.intro.right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hau : a ∈ u
⊢ f ⁻¹' {f a} ⊆ u
[PROOFSTEP]
refine (fiber_decomp (f a) (mem_preimage.1 hat)).resolve_right fun h => ?_
[GOAL]
case a.intro.right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hau : a ∈ u
h : f ⁻¹' {f a} ⊆ v
⊢ False
[PROOFSTEP]
exact
uv_disj.subset_compl_right hau
(h rfl)
-- This proof is exactly the same as the above (modulo some symmetry)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v :=
by
apply eq_of_subset_of_subset
· rw [← biUnion_preimage_singleton]
refine' iUnion₂_subset fun t' ht' => subset_inter _ ht'.2
rw [hf.preimage_subset_preimage_iff, singleton_subset_iff]
exact ht'.1
rintro a ⟨hat, hav⟩
constructor
· exact mem_preimage.1 hat
· refine (fiber_decomp (f a) (mem_preimage.1 hat)).resolve_left fun h => ?_
exact
uv_disj.subset_compl_left hav
(h rfl)
-- Now we show T₁, T₂ are closed, cover connectedComponent t and are disjoint.
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
⊢ f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
[PROOFSTEP]
apply eq_of_subset_of_subset
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
⊢ f ⁻¹' T₂ ⊆ f ⁻¹' connectedComponent t ∩ v
[PROOFSTEP]
rw [← biUnion_preimage_singleton]
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
⊢ ⋃ (y : β) (_ : y ∈ T₂), f ⁻¹' {y} ⊆ f ⁻¹' connectedComponent t ∩ v
[PROOFSTEP]
refine' iUnion₂_subset fun t' ht' => subset_inter _ ht'.2
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
t' : β
ht' : t' ∈ T₂
⊢ f ⁻¹' {t'} ⊆ f ⁻¹' connectedComponent t
[PROOFSTEP]
rw [hf.preimage_subset_preimage_iff, singleton_subset_iff]
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
t' : β
ht' : t' ∈ T₂
⊢ t' ∈ connectedComponent t
[PROOFSTEP]
exact ht'.1
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
⊢ f ⁻¹' connectedComponent t ∩ v ⊆ f ⁻¹' T₂
[PROOFSTEP]
rintro a ⟨hat, hav⟩
[GOAL]
case a.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hav : a ∈ v
⊢ a ∈ f ⁻¹' T₂
[PROOFSTEP]
constructor
[GOAL]
case a.intro.left
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hav : a ∈ v
⊢ f a ∈ connectedComponent t
[PROOFSTEP]
exact mem_preimage.1 hat
[GOAL]
case a.intro.right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hav : a ∈ v
⊢ f ⁻¹' {f a} ⊆ v
[PROOFSTEP]
refine (fiber_decomp (f a) (mem_preimage.1 hat)).resolve_left fun h => ?_
[GOAL]
case a.intro.right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
a : α
hat : a ∈ f ⁻¹' connectedComponent t
hav : a ∈ v
h : f ⁻¹' {f a} ⊆ u
⊢ False
[PROOFSTEP]
exact
uv_disj.subset_compl_left hav
(h rfl)
-- Now we show T₁, T₂ are closed, cover connectedComponent t and are disjoint.
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have hT₁ : IsClosed T₁ := (hcl T₁).2 (T₁_u.symm ▸ IsClosed.inter hT hu)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have hT₂ : IsClosed T₂ := (hcl T₂).2 (T₂_v.symm ▸ IsClosed.inter hT hv)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have T_decomp : connectedComponent t ⊆ T₁ ∪ T₂ := fun t' ht' =>
by
rw [mem_union t' T₁ T₂]
cases' fiber_decomp t' ht' with htu htv
· left
exact ⟨ht', htu⟩
right
exact ⟨ht', htv⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
t' : β
ht' : t' ∈ connectedComponent t
⊢ t' ∈ T₁ ∪ T₂
[PROOFSTEP]
rw [mem_union t' T₁ T₂]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
t' : β
ht' : t' ∈ connectedComponent t
⊢ t' ∈ T₁ ∨ t' ∈ T₂
[PROOFSTEP]
cases' fiber_decomp t' ht' with htu htv
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
t' : β
ht' : t' ∈ connectedComponent t
htu : f ⁻¹' {t'} ⊆ u
⊢ t' ∈ T₁ ∨ t' ∈ T₂
[PROOFSTEP]
left
[GOAL]
case inl.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
t' : β
ht' : t' ∈ connectedComponent t
htu : f ⁻¹' {t'} ⊆ u
⊢ t' ∈ T₁
[PROOFSTEP]
exact ⟨ht', htu⟩
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
t' : β
ht' : t' ∈ connectedComponent t
htv : f ⁻¹' {t'} ⊆ v
⊢ t' ∈ T₁ ∨ t' ∈ T₂
[PROOFSTEP]
right
[GOAL]
case inr.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
t' : β
ht' : t' ∈ connectedComponent t
htv : f ⁻¹' {t'} ⊆ v
⊢ t' ∈ T₂
[PROOFSTEP]
exact ⟨ht', htv⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
have T_disjoint : Disjoint T₁ T₂ := by
refine' Disjoint.of_preimage hf _
rw [T₁_u, T₂_v, disjoint_iff_inter_eq_empty, ← inter_inter_distrib_left, uv_disj.inter_eq, inter_empty]
-- Now we do cases on whether (connectedComponent t) is a subset of T₁ or T₂ to show
-- that the preimage is a subset of u or v.
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
⊢ Disjoint T₁ T₂
[PROOFSTEP]
refine' Disjoint.of_preimage hf _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
⊢ Disjoint (f ⁻¹' T₁) (f ⁻¹' T₂)
[PROOFSTEP]
rw [T₁_u, T₂_v, disjoint_iff_inter_eq_empty, ← inter_inter_distrib_left, uv_disj.inter_eq, inter_empty]
-- Now we do cases on whether (connectedComponent t) is a subset of T₁ or T₂ to show
-- that the preimage is a subset of u or v.
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
cases'
(isPreconnected_iff_subset_of_fully_disjoint_closed isClosed_connectedComponent).1 isPreconnected_connectedComponent
T₁ T₂ hT₁ hT₂ T_decomp T_disjoint with
h h
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₁
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
left
[GOAL]
case inl.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₁
⊢ f ⁻¹' connectedComponent t ⊆ u
[PROOFSTEP]
rw [Subset.antisymm_iff] at T₁_u
[GOAL]
case inl.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ ⊆ f ⁻¹' connectedComponent t ∩ u ∧ f ⁻¹' connectedComponent t ∩ u ⊆ f ⁻¹' T₁
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₁
⊢ f ⁻¹' connectedComponent t ⊆ u
[PROOFSTEP]
suffices f ⁻¹' connectedComponent t ⊆ f ⁻¹' T₁ from (this.trans T₁_u.1).trans (inter_subset_right _ _)
[GOAL]
case inl.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ ⊆ f ⁻¹' connectedComponent t ∩ u ∧ f ⁻¹' connectedComponent t ∩ u ⊆ f ⁻¹' T₁
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₁
⊢ f ⁻¹' connectedComponent t ⊆ f ⁻¹' T₁
[PROOFSTEP]
exact preimage_mono h
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₂
⊢ f ⁻¹' connectedComponent t ⊆ u ∨ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
right
[GOAL]
case inr.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ = f ⁻¹' connectedComponent t ∩ v
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₂
⊢ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
rw [Subset.antisymm_iff] at T₂_v
[GOAL]
case inr.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ ⊆ f ⁻¹' connectedComponent t ∩ v ∧ f ⁻¹' connectedComponent t ∩ v ⊆ f ⁻¹' T₂
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₂
⊢ f ⁻¹' connectedComponent t ⊆ v
[PROOFSTEP]
suffices f ⁻¹' connectedComponent t ⊆ f ⁻¹' T₂ from (this.trans T₂_v.1).trans (inter_subset_right _ _)
[GOAL]
case inr.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t✝ u✝ v✝ : Set α
inst✝ : TopologicalSpace β
f : α → β
connected_fibers : ∀ (t : β), IsConnected (f ⁻¹' {t})
hcl : ∀ (T : Set β), IsClosed T ↔ IsClosed (f ⁻¹' T)
t : β
hf : Surjective f
hT : IsClosed (f ⁻¹' connectedComponent t)
u v : Set α
hu : IsClosed u
hv : IsClosed v
huv : f ⁻¹' connectedComponent t ⊆ u ∪ v
uv_disj : Disjoint u v
T₁ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ u}
T₂ : Set β := {t' | t' ∈ connectedComponent t ∧ f ⁻¹' {t'} ⊆ v}
fiber_decomp : ∀ (t' : β), t' ∈ connectedComponent t → f ⁻¹' {t'} ⊆ u ∨ f ⁻¹' {t'} ⊆ v
T₁_u : f ⁻¹' T₁ = f ⁻¹' connectedComponent t ∩ u
T₂_v : f ⁻¹' T₂ ⊆ f ⁻¹' connectedComponent t ∩ v ∧ f ⁻¹' connectedComponent t ∩ v ⊆ f ⁻¹' T₂
hT₁ : IsClosed T₁
hT₂ : IsClosed T₂
T_decomp : connectedComponent t ⊆ T₁ ∪ T₂
T_disjoint : Disjoint T₁ T₂
h : connectedComponent t ⊆ T₂
⊢ f ⁻¹' connectedComponent t ⊆ f ⁻¹' T₂
[PROOFSTEP]
exact preimage_mono h
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : TopologicalSpace β
f : α → β
hf : QuotientMap f
h_fibers : ∀ (y : β), IsConnected (f ⁻¹' {y})
a : α
⊢ f '' connectedComponent a = connectedComponent (f a)
[PROOFSTEP]
rw [← hf.preimage_connectedComponent h_fibers, image_preimage_eq _ hf.surjective]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ LocallyConnectedSpace α ↔ ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ⊆ U ∧ IsOpen V ∧ x ∈ V ∧ IsConnected V
[PROOFSTEP]
simp_rw [locallyConnectedSpace_iff_open_connected_basis]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α), Filter.HasBasis (𝓝 x) (fun s => IsOpen s ∧ x ∈ s ∧ IsConnected s) id) ↔
∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ⊆ U ∧ IsOpen V ∧ x ∈ V ∧ IsConnected V
[PROOFSTEP]
refine forall_congr' fun _ => ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x✝ : α
⊢ Filter.HasBasis (𝓝 x✝) (fun s => IsOpen s ∧ x✝ ∈ s ∧ IsConnected s) id ↔
∀ (U : Set α), U ∈ 𝓝 x✝ → ∃ V, V ⊆ U ∧ IsOpen V ∧ x✝ ∈ V ∧ IsConnected V
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x✝ : α
⊢ Filter.HasBasis (𝓝 x✝) (fun s => IsOpen s ∧ x✝ ∈ s ∧ IsConnected s) id →
∀ (U : Set α), U ∈ 𝓝 x✝ → ∃ V, V ⊆ U ∧ IsOpen V ∧ x✝ ∈ V ∧ IsConnected V
[PROOFSTEP]
intro h U hU
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x✝ : α
h : Filter.HasBasis (𝓝 x✝) (fun s => IsOpen s ∧ x✝ ∈ s ∧ IsConnected s) id
U : Set α
hU : U ∈ 𝓝 x✝
⊢ ∃ V, V ⊆ U ∧ IsOpen V ∧ x✝ ∈ V ∧ IsConnected V
[PROOFSTEP]
rcases h.mem_iff.mp hU with ⟨V, hV, hVU⟩
[GOAL]
case mp.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x✝ : α
h : Filter.HasBasis (𝓝 x✝) (fun s => IsOpen s ∧ x✝ ∈ s ∧ IsConnected s) id
U : Set α
hU : U ∈ 𝓝 x✝
V : Set α
hV : IsOpen V ∧ x✝ ∈ V ∧ IsConnected V
hVU : id V ⊆ U
⊢ ∃ V, V ⊆ U ∧ IsOpen V ∧ x✝ ∈ V ∧ IsConnected V
[PROOFSTEP]
exact ⟨V, hVU, hV⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x✝ : α
⊢ (∀ (U : Set α), U ∈ 𝓝 x✝ → ∃ V, V ⊆ U ∧ IsOpen V ∧ x✝ ∈ V ∧ IsConnected V) →
Filter.HasBasis (𝓝 x✝) (fun s => IsOpen s ∧ x✝ ∈ s ∧ IsConnected s) id
[PROOFSTEP]
exact fun h =>
⟨fun U =>
⟨fun hU =>
let ⟨V, hVU, hV⟩ := h U hU
⟨V, hV, hVU⟩,
fun ⟨V, ⟨hV, hxV, _⟩, hVU⟩ => mem_nhds_iff.mpr ⟨V, hVU, hV, hxV⟩⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
h : F ∈ 𝓝 x
⊢ connectedComponentIn F x ∈ 𝓝 x
[PROOFSTEP]
rw [(LocallyConnectedSpace.open_connected_basis x).mem_iff] at h
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
h : ∃ i, (IsOpen i ∧ x ∈ i ∧ IsConnected i) ∧ id i ⊆ F
⊢ connectedComponentIn F x ∈ 𝓝 x
[PROOFSTEP]
rcases h with ⟨s, ⟨h1s, hxs, h2s⟩, hsF⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s✝ t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
s : Set α
hsF : id s ⊆ F
h1s : IsOpen s
hxs : x ∈ s
h2s : IsConnected s
⊢ connectedComponentIn F x ∈ 𝓝 x
[PROOFSTEP]
exact mem_nhds_iff.mpr ⟨s, h2s.isPreconnected.subset_connectedComponentIn hxs hsF, h1s, hxs⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
hF : IsOpen F
⊢ IsOpen (connectedComponentIn F x)
[PROOFSTEP]
rw [isOpen_iff_mem_nhds]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
hF : IsOpen F
⊢ ∀ (a : α), a ∈ connectedComponentIn F x → connectedComponentIn F x ∈ 𝓝 a
[PROOFSTEP]
intro y hy
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
hF : IsOpen F
y : α
hy : y ∈ connectedComponentIn F x
⊢ connectedComponentIn F x ∈ 𝓝 y
[PROOFSTEP]
rw [connectedComponentIn_eq hy]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
F : Set α
x : α
hF : IsOpen F
y : α
hy : y ∈ connectedComponentIn F x
⊢ connectedComponentIn F y ∈ 𝓝 y
[PROOFSTEP]
exact connectedComponentIn_mem_nhds (hF.mem_nhds <| connectedComponentIn_subset F x hy)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
x : α
⊢ IsOpen (connectedComponent x)
[PROOFSTEP]
rw [← connectedComponentIn_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
inst✝ : LocallyConnectedSpace α
x : α
⊢ IsOpen (connectedComponentIn univ x)
[PROOFSTEP]
exact isOpen_univ.connectedComponentIn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ LocallyConnectedSpace α ↔ ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ LocallyConnectedSpace α → ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : LocallyConnectedSpace α
⊢ ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
[PROOFSTEP]
exact fun F hF x _ => hF.connectedComponentIn
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)) → LocallyConnectedSpace α
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
⊢ LocallyConnectedSpace α
[PROOFSTEP]
rw [locallyConnectedSpace_iff_open_connected_subsets]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
⊢ ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ⊆ U ∧ IsOpen V ∧ x ∈ V ∧ IsConnected V
[PROOFSTEP]
refine' fun x U hU =>
⟨connectedComponentIn (interior U) x, (connectedComponentIn_subset _ _).trans interior_subset,
h _ isOpen_interior x _, mem_connectedComponentIn _, isConnected_connectedComponentIn_iff.mpr _⟩
[GOAL]
case mpr.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
x : α
U : Set α
hU : U ∈ 𝓝 x
⊢ x ∈ interior U
[PROOFSTEP]
exact mem_interior_iff_mem_nhds.mpr hU
[GOAL]
case mpr.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
x : α
U : Set α
hU : U ∈ 𝓝 x
⊢ x ∈ interior U
[PROOFSTEP]
exact mem_interior_iff_mem_nhds.mpr hU
[GOAL]
case mpr.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
x : α
U : Set α
hU : U ∈ 𝓝 x
⊢ x ∈ interior U
[PROOFSTEP]
exact mem_interior_iff_mem_nhds.mpr hU
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ LocallyConnectedSpace α ↔ ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ LocallyConnectedSpace α → ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
[PROOFSTEP]
rw [locallyConnectedSpace_iff_open_connected_subsets]
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ⊆ U ∧ IsOpen V ∧ x ∈ V ∧ IsConnected V) →
∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
[PROOFSTEP]
intro h x U hxU
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ⊆ U ∧ IsOpen V ∧ x ∈ V ∧ IsConnected V
x : α
U : Set α
hxU : U ∈ 𝓝 x
⊢ ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
[PROOFSTEP]
rcases h x U hxU with ⟨V, hVU, hV₁, hxV, hV₂⟩
[GOAL]
case mp.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ⊆ U ∧ IsOpen V ∧ x ∈ V ∧ IsConnected V
x : α
U : Set α
hxU : U ∈ 𝓝 x
V : Set α
hVU : V ⊆ U
hV₁ : IsOpen V
hxV : x ∈ V
hV₂ : IsConnected V
⊢ ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
[PROOFSTEP]
exact ⟨V, hV₁.mem_nhds hxV, hV₂.isPreconnected, hVU⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U) → LocallyConnectedSpace α
[PROOFSTEP]
rw [locallyConnectedSpace_iff_connectedComponentIn_open]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U) →
∀ (F : Set α), IsOpen F → ∀ (x : α), x ∈ F → IsOpen (connectedComponentIn F x)
[PROOFSTEP]
refine' fun h U hU x _ => isOpen_iff_mem_nhds.mpr fun y hy => _
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
U : Set α
hU : IsOpen U
x : α
x✝ : x ∈ U
y : α
hy : y ∈ connectedComponentIn U x
⊢ connectedComponentIn U x ∈ 𝓝 y
[PROOFSTEP]
rw [connectedComponentIn_eq hy]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
U : Set α
hU : IsOpen U
x : α
x✝ : x ∈ U
y : α
hy : y ∈ connectedComponentIn U x
⊢ connectedComponentIn U y ∈ 𝓝 y
[PROOFSTEP]
rcases h y U (hU.mem_nhds <| (connectedComponentIn_subset _ _) hy) with ⟨V, hVy, hV, hVU⟩
[GOAL]
case mpr.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U
U : Set α
hU : IsOpen U
x : α
x✝ : x ∈ U
y : α
hy : y ∈ connectedComponentIn U x
V : Set α
hVy : V ∈ 𝓝 y
hV : IsPreconnected V
hVU : V ⊆ U
⊢ connectedComponentIn U y ∈ 𝓝 y
[PROOFSTEP]
exact Filter.mem_of_superset hVy (hV.subset_connectedComponentIn (mem_of_mem_nhds hVy) hVU)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ LocallyConnectedSpace α ↔ ∀ (x : α), Filter.HasBasis (𝓝 x) (fun s => s ∈ 𝓝 x ∧ IsPreconnected s) id
[PROOFSTEP]
rw [locallyConnectedSpace_iff_connected_subsets]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α) (U : Set α), U ∈ 𝓝 x → ∃ V, V ∈ 𝓝 x ∧ IsPreconnected V ∧ V ⊆ U) ↔
∀ (x : α), Filter.HasBasis (𝓝 x) (fun s => s ∈ 𝓝 x ∧ IsPreconnected s) id
[PROOFSTEP]
exact forall_congr' <| fun x => Filter.hasBasis_self.symm
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
ι : Type u_3
b : α → ι → Set α
p : α → ι → Prop
hbasis : ∀ (x : α), Filter.HasBasis (𝓝 x) (p x) (b x)
hconnected : ∀ (x : α) (i : ι), p x i → IsPreconnected (b x i)
⊢ LocallyConnectedSpace α
[PROOFSTEP]
rw [locallyConnectedSpace_iff_connected_basis]
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
ι : Type u_3
b : α → ι → Set α
p : α → ι → Prop
hbasis : ∀ (x : α), Filter.HasBasis (𝓝 x) (p x) (b x)
hconnected : ∀ (x : α) (i : ι), p x i → IsPreconnected (b x i)
⊢ ∀ (x : α), Filter.HasBasis (𝓝 x) (fun s => s ∈ 𝓝 x ∧ IsPreconnected s) id
[PROOFSTEP]
exact fun x =>
(hbasis x).to_hasBasis (fun i hi => ⟨b x i, ⟨(hbasis x).mem_of_mem hi, hconnected x i hi⟩, subset_rfl⟩) fun s hs =>
⟨(hbasis x).index s hs.1, ⟨(hbasis x).property_index hs.1, (hbasis x).set_index_subset hs.1⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s t u v : Set α
inst✝² : TopologicalSpace β
inst✝¹ : TotallyDisconnectedSpace α
inst✝ : TotallyDisconnectedSpace β
⊢ TotallyDisconnectedSpace (α ⊕ β)
[PROOFSTEP]
refine' ⟨fun s _ hs => _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s✝ t u v : Set α
inst✝² : TopologicalSpace β
inst✝¹ : TotallyDisconnectedSpace α
inst✝ : TotallyDisconnectedSpace β
s : Set (α ⊕ β)
x✝ : s ⊆ univ
hs : IsPreconnected s
⊢ Set.Subsingleton s
[PROOFSTEP]
obtain ⟨t, ht, rfl⟩ | ⟨t, ht, rfl⟩ := Sum.isPreconnected_iff.1 hs
[GOAL]
case inl.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s t✝ u v : Set α
inst✝² : TopologicalSpace β
inst✝¹ : TotallyDisconnectedSpace α
inst✝ : TotallyDisconnectedSpace β
t : Set α
ht : IsPreconnected t
x✝ : Sum.inl '' t ⊆ univ
hs : IsPreconnected (Sum.inl '' t)
⊢ Set.Subsingleton (Sum.inl '' t)
[PROOFSTEP]
exact ht.subsingleton.image _
[GOAL]
case inr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
s t✝ u v : Set α
inst✝² : TopologicalSpace β
inst✝¹ : TotallyDisconnectedSpace α
inst✝ : TotallyDisconnectedSpace β
t : Set β
ht : IsPreconnected t
x✝ : Sum.inr '' t ⊆ univ
hs : IsPreconnected (Sum.inr '' t)
⊢ Set.Subsingleton (Sum.inr '' t)
[PROOFSTEP]
exact ht.subsingleton.image _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), TotallyDisconnectedSpace (π i)
⊢ TotallyDisconnectedSpace ((i : ι) × π i)
[PROOFSTEP]
refine' ⟨fun s _ hs => _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), TotallyDisconnectedSpace (π i)
s : Set ((i : ι) × π i)
x✝ : s ⊆ univ
hs : IsPreconnected s
⊢ Set.Subsingleton s
[PROOFSTEP]
obtain rfl | h := s.eq_empty_or_nonempty
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), TotallyDisconnectedSpace (π i)
x✝ : ∅ ⊆ univ
hs : IsPreconnected ∅
⊢ Set.Subsingleton ∅
[PROOFSTEP]
exact subsingleton_empty
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s✝ t u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), TotallyDisconnectedSpace (π i)
s : Set ((i : ι) × π i)
x✝ : s ⊆ univ
hs : IsPreconnected s
h : Set.Nonempty s
⊢ Set.Subsingleton s
[PROOFSTEP]
obtain ⟨a, t, ht, rfl⟩ := Sigma.isConnected_iff.1 ⟨h, hs⟩
[GOAL]
case inr.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t✝ u v : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), TotallyDisconnectedSpace (π i)
a : ι
t : Set (π a)
ht : IsConnected t
x✝ : Sigma.mk a '' t ⊆ univ
hs : IsPreconnected (Sigma.mk a '' t)
h : Set.Nonempty (Sigma.mk a '' t)
⊢ Set.Subsingleton (Sigma.mk a '' t)
[PROOFSTEP]
exact
ht.isPreconnected.subsingleton.image
_
-- porting note: reformulated using `Pairwise`
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
⊢ IsTotallyDisconnected univ
[PROOFSTEP]
rintro S - hS
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
hS : IsPreconnected S
⊢ Set.Subsingleton S
[PROOFSTEP]
unfold Set.Subsingleton
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
hS : IsPreconnected S
⊢ ∀ ⦃x : X⦄, x ∈ S → ∀ ⦃y : X⦄, y ∈ S → x = y
[PROOFSTEP]
by_contra' h_contra
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
hS : IsPreconnected S
h_contra : Exists fun ⦃x⦄ => x ∈ S ∧ Exists fun ⦃y⦄ => y ∈ S ∧ x ≠ y
⊢ False
[PROOFSTEP]
rcases h_contra with ⟨x, hx, y, hy, hxy⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
hS : IsPreconnected S
x : X
hx : x ∈ S
y : X
hy : y ∈ S
hxy : x ≠ y
⊢ False
[PROOFSTEP]
obtain ⟨U, h_clopen, hxU, hyU⟩ := hX hxy
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
hS : IsPreconnected S
x : X
hx : x ∈ S
y : X
hy : y ∈ S
hxy : x ≠ y
U : Set X
h_clopen : IsClopen U
hxU : x ∈ U
hyU : ¬y ∈ U
⊢ False
[PROOFSTEP]
specialize hS U Uᶜ h_clopen.1 h_clopen.compl.1 (fun a _ => em (a ∈ U)) ⟨x, hx, hxU⟩ ⟨y, hy, hyU⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
x : X
hx : x ∈ S
y : X
hy : y ∈ S
hxy : x ≠ y
U : Set X
h_clopen : IsClopen U
hxU : x ∈ U
hyU : ¬y ∈ U
hS : Set.Nonempty (S ∩ (U ∩ Uᶜ))
⊢ False
[PROOFSTEP]
rw [inter_compl_self, Set.inter_empty] at hS
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
s t u v : Set α
X : Type u_3
inst✝ : TopologicalSpace X
hX : Pairwise fun x y => ∃ U, IsClopen U ∧ x ∈ U ∧ ¬y ∈ U
S : Set X
x : X
hx : x ∈ S
y : X
hy : y ∈ S
hxy : x ≠ y
U : Set X
h_clopen : IsClopen U
hxU : x ∈ U
hyU : ¬y ∈ U
hS : Set.Nonempty ∅
⊢ False
[PROOFSTEP]
exact Set.not_nonempty_empty hS
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ TotallyDisconnectedSpace α ↔ ∀ (x : α), Set.Subsingleton (connectedComponent x)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ TotallyDisconnectedSpace α → ∀ (x : α), Set.Subsingleton (connectedComponent x)
[PROOFSTEP]
intro h x
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : TotallyDisconnectedSpace α
x : α
⊢ Set.Subsingleton (connectedComponent x)
[PROOFSTEP]
apply h.1
[GOAL]
case mp.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : TotallyDisconnectedSpace α
x : α
⊢ connectedComponent x ⊆ univ
[PROOFSTEP]
exact subset_univ _
[GOAL]
case mp.a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : TotallyDisconnectedSpace α
x : α
⊢ IsPreconnected (connectedComponent x)
[PROOFSTEP]
exact isPreconnected_connectedComponent
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α), Set.Subsingleton (connectedComponent x)) → TotallyDisconnectedSpace α
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), Set.Subsingleton (connectedComponent x)
⊢ TotallyDisconnectedSpace α
[PROOFSTEP]
constructor
[GOAL]
case mpr.isTotallyDisconnected_univ
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), Set.Subsingleton (connectedComponent x)
⊢ IsTotallyDisconnected univ
[PROOFSTEP]
intro s s_sub hs
[GOAL]
case mpr.isTotallyDisconnected_univ
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v : Set α
h : ∀ (x : α), Set.Subsingleton (connectedComponent x)
s : Set α
s_sub : s ⊆ univ
hs : IsPreconnected s
⊢ Set.Subsingleton s
[PROOFSTEP]
rcases eq_empty_or_nonempty s with (rfl | ⟨x, x_in⟩)
[GOAL]
case mpr.isTotallyDisconnected_univ.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
h : ∀ (x : α), Set.Subsingleton (connectedComponent x)
s_sub : ∅ ⊆ univ
hs : IsPreconnected ∅
⊢ Set.Subsingleton ∅
[PROOFSTEP]
exact subsingleton_empty
[GOAL]
case mpr.isTotallyDisconnected_univ.inr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v : Set α
h : ∀ (x : α), Set.Subsingleton (connectedComponent x)
s : Set α
s_sub : s ⊆ univ
hs : IsPreconnected s
x : α
x_in : x ∈ s
⊢ Set.Subsingleton s
[PROOFSTEP]
exact (h x).anti (hs.subset_connectedComponent x_in)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ TotallyDisconnectedSpace α ↔ ∀ (x : α), connectedComponent x = {x}
[PROOFSTEP]
rw [totallyDisconnectedSpace_iff_connectedComponent_subsingleton]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
⊢ (∀ (x : α), Set.Subsingleton (connectedComponent x)) ↔ ∀ (x : α), connectedComponent x = {x}
[PROOFSTEP]
refine forall_congr' fun x => ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
⊢ Set.Subsingleton (connectedComponent x) ↔ connectedComponent x = {x}
[PROOFSTEP]
rw [subsingleton_iff_singleton]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s t u v : Set α
x : α
⊢ x ∈ connectedComponent x
[PROOFSTEP]
exact mem_connectedComponent
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
H : IsTotallySeparated s
⊢ IsTotallyDisconnected s
[PROOFSTEP]
intro t hts ht x x_in y y_in
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
H : IsTotallySeparated s
t : Set α
hts : t ⊆ s
ht : IsPreconnected t
x : α
x_in : x ∈ t
y : α
y_in : y ∈ t
⊢ x = y
[PROOFSTEP]
by_contra h
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u v s : Set α
H : IsTotallySeparated s
t : Set α
hts : t ⊆ s
ht : IsPreconnected t
x : α
x_in : x ∈ t
y : α
y_in : y ∈ t
h : ¬x = y
⊢ False
[PROOFSTEP]
obtain ⟨u : Set α, v : Set α, hu : IsOpen u, hv : IsOpen v, hxu : x ∈ u, hyv : y ∈ v, hs : s ⊆ u ∪ v, huv⟩ :=
H x (hts x_in) y (hts y_in) h
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
H : IsTotallySeparated s
t : Set α
hts : t ⊆ s
ht : IsPreconnected t
x : α
x_in : x ∈ t
y : α
y_in : y ∈ t
h : ¬x = y
u v : Set α
hu : IsOpen u
hv : IsOpen v
hxu : x ∈ u
hyv : y ∈ v
hs : s ⊆ u ∪ v
huv : Disjoint u v
⊢ False
[PROOFSTEP]
refine' (ht _ _ hu hv (hts.trans hs) ⟨x, x_in, hxu⟩ ⟨y, y_in, hyv⟩).ne_empty _
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t✝ u✝ v✝ s : Set α
H : IsTotallySeparated s
t : Set α
hts : t ⊆ s
ht : IsPreconnected t
x : α
x_in : x ∈ t
y : α
y_in : y ∈ t
h : ¬x = y
u v : Set α
hu : IsOpen u
hv : IsOpen v
hxu : x ∈ u
hyv : y ∈ v
hs : s ⊆ u ∪ v
huv : Disjoint u v
⊢ t ∩ (u ∩ v) = ∅
[PROOFSTEP]
rw [huv.inter_eq, inter_empty]
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
s t u v : Set α✝
α : Type u_3
inst✝¹ : TopologicalSpace α
inst✝ : TotallySeparatedSpace α
x y : α
hxy : x ≠ y
⊢ ∃ U, IsClopen U ∧ x ∈ U ∧ y ∈ Uᶜ
[PROOFSTEP]
obtain ⟨U, V, hU, hV, Ux, Vy, f, disj⟩ :=
TotallySeparatedSpace.isTotallySeparated_univ x (Set.mem_univ x) y (Set.mem_univ y) hxy
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
s t u v : Set α✝
α : Type u_3
inst✝¹ : TopologicalSpace α
inst✝ : TotallySeparatedSpace α
x y : α
hxy : x ≠ y
U V : Set α
hU : IsOpen U
hV : IsOpen V
Ux : x ∈ U
Vy : y ∈ V
f : univ ⊆ U ∪ V
disj : Disjoint U V
⊢ ∃ U, IsClopen U ∧ x ∈ U ∧ y ∈ Uᶜ
[PROOFSTEP]
have clopen_U := isClopen_inter_of_disjoint_cover_clopen isClopen_univ f hU hV disj
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
s t u v : Set α✝
α : Type u_3
inst✝¹ : TopologicalSpace α
inst✝ : TotallySeparatedSpace α
x y : α
hxy : x ≠ y
U V : Set α
hU : IsOpen U
hV : IsOpen V
Ux : x ∈ U
Vy : y ∈ V
f : univ ⊆ U ∪ V
disj : Disjoint U V
clopen_U : IsClopen (univ ∩ U)
⊢ ∃ U, IsClopen U ∧ x ∈ U ∧ y ∈ Uᶜ
[PROOFSTEP]
rw [univ_inter _] at clopen_U
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
s t u v : Set α✝
α : Type u_3
inst✝¹ : TopologicalSpace α
inst✝ : TotallySeparatedSpace α
x y : α
hxy : x ≠ y
U V : Set α
hU : IsOpen U
hV : IsOpen V
Ux : x ∈ U
Vy : y ∈ V
f : univ ⊆ U ∪ V
disj : Disjoint U V
clopen_U : IsClopen U
⊢ ∃ U, IsClopen U ∧ x ∈ U ∧ y ∈ Uᶜ
[PROOFSTEP]
rw [← Set.subset_compl_iff_disjoint_right, subset_compl_comm] at disj
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
s t u v : Set α✝
α : Type u_3
inst✝¹ : TopologicalSpace α
inst✝ : TotallySeparatedSpace α
x y : α
hxy : x ≠ y
U V : Set α
hU : IsOpen U
hV : IsOpen V
Ux : x ∈ U
Vy : y ∈ V
f : univ ⊆ U ∪ V
disj : V ⊆ Uᶜ
clopen_U : IsClopen U
⊢ ∃ U, IsClopen U ∧ x ∈ U ∧ y ∈ Uᶜ
[PROOFSTEP]
exact ⟨U, clopen_U, Ux, disj Vy⟩
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α✝
s t u v : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
x : α
⊢ connectedComponent x = connectedComponent x
[PROOFSTEP]
trivial
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
h : Continuous f
⊢ ∀ (a b : α), Setoid.r a b → f a = f b
[PROOFSTEP]
convert h.image_eq_of_connectedComponent_eq
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
x : α
⊢ ConnectedComponents.mk ⁻¹' {ConnectedComponents.mk x} = connectedComponent x
[PROOFSTEP]
ext y
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
x y : α
⊢ y ∈ ConnectedComponents.mk ⁻¹' {ConnectedComponents.mk x} ↔ y ∈ connectedComponent x
[PROOFSTEP]
rw [mem_preimage, mem_singleton_iff, ConnectedComponents.coe_eq_coe']
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
U : Set α
⊢ ConnectedComponents.mk ⁻¹' (ConnectedComponents.mk '' U) = ⋃ (x : α) (_ : x ∈ U), connectedComponent x
[PROOFSTEP]
simp only [connectedComponents_preimage_singleton, preimage_iUnion₂, image_eq_iUnion]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
⊢ TotallyDisconnectedSpace (ConnectedComponents α)
[PROOFSTEP]
rw [totallyDisconnectedSpace_iff_connectedComponent_singleton]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
⊢ ∀ (x : ConnectedComponents α), connectedComponent x = {x}
[PROOFSTEP]
refine' ConnectedComponents.surjective_coe.forall.2 fun x => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
x : α
⊢ connectedComponent (mk x) = {mk x}
[PROOFSTEP]
rw [← ConnectedComponents.quotientMap_coe.image_connectedComponent, ← connectedComponents_preimage_singleton,
image_preimage_eq _ ConnectedComponents.surjective_coe]
[GOAL]
case h_fibers
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
x : α
⊢ ∀ (y : ConnectedComponents α), IsConnected (mk ⁻¹' {y})
[PROOFSTEP]
refine' ConnectedComponents.surjective_coe.forall.2 fun y => _
[GOAL]
case h_fibers
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
x y : α
⊢ IsConnected (mk ⁻¹' {mk y})
[PROOFSTEP]
rw [connectedComponents_preimage_singleton]
[GOAL]
case h_fibers
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
inst✝ : TotallyDisconnectedSpace β
f : α → β
x y : α
⊢ IsConnected (connectedComponent y)
[PROOFSTEP]
exact isConnected_connectedComponent
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
⊢ IsPreconnected s
[PROOFSTEP]
unfold IsPreconnected
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
⊢ ∀ (u v : Set α),
IsOpen u → IsOpen v → s ⊆ u ∪ v → Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
by_contra'
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u v s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
this :
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∪ v ∧ Set.Nonempty (s ∩ u) ∧ Set.Nonempty (s ∩ v) ∧ ¬Set.Nonempty (s ∩ (u ∩ v))
⊢ False
[PROOFSTEP]
rcases this with ⟨u, v, u_op, v_op, hsuv, ⟨x, x_in_s, x_in_u⟩, ⟨y, y_in_s, y_in_v⟩, H⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : ¬Set.Nonempty (s ∩ (u ∩ v))
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
⊢ False
[PROOFSTEP]
rw [not_nonempty_iff_eq_empty] at H
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
⊢ False
[PROOFSTEP]
have hy : y ∉ u := fun y_in_u => eq_empty_iff_forall_not_mem.mp H y ⟨y_in_s, ⟨y_in_u, y_in_v⟩⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
hy : ¬y ∈ u
⊢ False
[PROOFSTEP]
have : ContinuousOn u.boolIndicator s :=
by
apply (continuousOn_boolIndicator_iff_clopen _ _).mpr ⟨_, _⟩
· exact u_op.preimage continuous_subtype_val
· rw [preimage_subtype_coe_eq_compl hsuv H]
exact (v_op.preimage continuous_subtype_val).isClosed_compl
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
hy : ¬y ∈ u
⊢ ContinuousOn (boolIndicator u) s
[PROOFSTEP]
apply (continuousOn_boolIndicator_iff_clopen _ _).mpr ⟨_, _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
hy : ¬y ∈ u
⊢ IsOpen (Subtype.val ⁻¹' u)
[PROOFSTEP]
exact u_op.preimage continuous_subtype_val
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
hy : ¬y ∈ u
⊢ IsClosed (Subtype.val ⁻¹' u)
[PROOFSTEP]
rw [preimage_subtype_coe_eq_compl hsuv H]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
hy : ¬y ∈ u
⊢ IsClosed (Subtype.val ⁻¹' v)ᶜ
[PROOFSTEP]
exact (v_op.preimage continuous_subtype_val).isClosed_compl
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝ : TopologicalSpace α
s✝ t u✝ v✝ s : Set α
hs : ∀ (f : α → Bool), ContinuousOn f s → ∀ (x : α), x ∈ s → ∀ (y : α), y ∈ s → f x = f y
u v : Set α
u_op : IsOpen u
v_op : IsOpen v
hsuv : s ⊆ u ∪ v
x : α
x_in_s : x ∈ s
x_in_u : x ∈ u
H : s ∩ (u ∩ v) = ∅
y : α
y_in_s : y ∈ s
y_in_v : y ∈ v
hy : ¬y ∈ u
this : ContinuousOn (boolIndicator u) s
⊢ False
[PROOFSTEP]
simpa [(u.mem_iff_boolIndicator _).mp x_in_u, (u.not_mem_iff_boolIndicator _).mp hy] using hs _ this x x_in_s y y_in_s
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
S : Set α
hS : IsPreconnected S
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hc : ContinuousOn f S
hTm : MapsTo f S T
x y : α
hx : x ∈ S
hy : y ∈ S
⊢ f x = f y
[PROOFSTEP]
let F : S → T := hTm.restrict f S T
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
S : Set α
hS : IsPreconnected S
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hc : ContinuousOn f S
hTm : MapsTo f S T
x y : α
hx : x ∈ S
hy : y ∈ S
F : ↑S → ↑T := MapsTo.restrict f S T hTm
⊢ f x = f y
[PROOFSTEP]
suffices F ⟨x, hx⟩ = F ⟨y, hy⟩ by rwa [← Subtype.coe_inj] at this
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
S : Set α
hS : IsPreconnected S
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hc : ContinuousOn f S
hTm : MapsTo f S T
x y : α
hx : x ∈ S
hy : y ∈ S
F : ↑S → ↑T := MapsTo.restrict f S T hTm
this : F { val := x, property := hx } = F { val := y, property := hy }
⊢ f x = f y
[PROOFSTEP]
rwa [← Subtype.coe_inj] at this
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
S : Set α
hS : IsPreconnected S
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hc : ContinuousOn f S
hTm : MapsTo f S T
x y : α
hx : x ∈ S
hy : y ∈ S
F : ↑S → ↑T := MapsTo.restrict f S T hTm
⊢ F { val := x, property := hx } = F { val := y, property := hy }
[PROOFSTEP]
exact (isPreconnected_iff_preconnectedSpace.mp hS).constant (hc.restrict_mapsTo _)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
S : Set α
hS : IsPreconnected S
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hc : ContinuousOn f S
hTm : MapsTo f S T
hne : Set.Nonempty T
⊢ ∃ y, y ∈ T ∧ EqOn f (const α y) S
[PROOFSTEP]
rcases S.eq_empty_or_nonempty with (rfl | ⟨x, hx⟩)
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hne : Set.Nonempty T
hS : IsPreconnected ∅
hc : ContinuousOn f ∅
hTm : MapsTo f ∅ T
⊢ ∃ y, y ∈ T ∧ EqOn f (const α y) ∅
[PROOFSTEP]
exact hne.imp fun _ hy => ⟨hy, eqOn_empty _ _⟩
[GOAL]
case inr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
s t u v : Set α
inst✝¹ : TopologicalSpace β
S : Set α
hS : IsPreconnected S
T : Set β
inst✝ : DiscreteTopology ↑T
f : α → β
hc : ContinuousOn f S
hTm : MapsTo f S T
hne : Set.Nonempty T
x : α
hx : x ∈ S
⊢ ∃ y, y ∈ T ∧ EqOn f (const α y) S
[PROOFSTEP]
exact ⟨f x, hTm hx, fun x' hx' => hS.constant_of_mapsTo hc hTm hx' hx⟩
| {"mathlib_filename": "Mathlib.Topology.Connected", "llama_tokens": 134115} |
[GOAL]
α : Type u
T : Set (Set α)
empty_mem : ∅ ∈ T
sInter_mem : ∀ (A : Set (Set α)), A ⊆ T → ⋂₀ A ∈ T
union_mem : ∀ (A : Set α), A ∈ T → ∀ (B : Set α), B ∈ T → A ∪ B ∈ T
⊢ (fun X => Xᶜ ∈ T) univ
[PROOFSTEP]
simp [empty_mem]
[GOAL]
α : Type u
T : Set (Set α)
empty_mem : ∅ ∈ T
sInter_mem : ∀ (A : Set (Set α)), A ⊆ T → ⋂₀ A ∈ T
union_mem : ∀ (A : Set α), A ∈ T → ∀ (B : Set α), B ∈ T → A ∪ B ∈ T
s t : Set α
hs : (fun X => Xᶜ ∈ T) s
ht : (fun X => Xᶜ ∈ T) t
⊢ (fun X => Xᶜ ∈ T) (s ∩ t)
[PROOFSTEP]
simpa only [compl_inter] using union_mem sᶜ hs tᶜ ht
[GOAL]
α : Type u
T : Set (Set α)
empty_mem : ∅ ∈ T
sInter_mem : ∀ (A : Set (Set α)), A ⊆ T → ⋂₀ A ∈ T
union_mem : ∀ (A : Set α), A ∈ T → ∀ (B : Set α), B ∈ T → A ∪ B ∈ T
s : Set (Set α)
hs : ∀ (t : Set α), t ∈ s → (fun X => Xᶜ ∈ T) t
⊢ (fun X => Xᶜ ∈ T) (⋃₀ s)
[PROOFSTEP]
simp only [Set.compl_sUnion]
[GOAL]
α : Type u
T : Set (Set α)
empty_mem : ∅ ∈ T
sInter_mem : ∀ (A : Set (Set α)), A ⊆ T → ⋂₀ A ∈ T
union_mem : ∀ (A : Set α), A ∈ T → ∀ (B : Set α), B ∈ T → A ∪ B ∈ T
s : Set (Set α)
hs : ∀ (t : Set α), t ∈ s → (fun X => Xᶜ ∈ T) t
⊢ ⋂₀ (compl '' s) ∈ T
[PROOFSTEP]
exact sInter_mem (compl '' s) fun z ⟨y, hy, hz⟩ => hz ▸ hs y hy
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
t t' : TopologicalSpace α
h : ∀ (s : Set α), IsOpen s ↔ IsOpen s
⊢ t = t'
[PROOFSTEP]
ext
[GOAL]
case a.h.a
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
t t' : TopologicalSpace α
h : ∀ (s : Set α), IsOpen s ↔ IsOpen s
x✝ : Set α
⊢ IsOpen x✝ ↔ IsOpen x✝
[PROOFSTEP]
exact h _
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
h₁ : IsOpen s₁
h₂ : IsOpen s₂
⊢ IsOpen (s₁ ∪ s₂)
[PROOFSTEP]
rw [union_eq_iUnion]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
h₁ : IsOpen s₁
h₂ : IsOpen s₂
⊢ IsOpen (⋃ (b : Bool), bif b then s₁ else s₂)
[PROOFSTEP]
exact isOpen_iUnion (Bool.forall_bool.2 ⟨h₂, h₁⟩)
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ IsOpen ∅
[PROOFSTEP]
rw [← sUnion_empty]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ IsOpen (⋃₀ ∅)
[PROOFSTEP]
exact isOpen_sUnion fun a => False.elim
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set (Set α)
hs : Set.Finite s
x✝ : ∀ (t : Set α), t ∈ ∅ → IsOpen t
⊢ IsOpen (⋂₀ ∅)
[PROOFSTEP]
rw [sInter_empty]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set (Set α)
hs : Set.Finite s
x✝ : ∀ (t : Set α), t ∈ ∅ → IsOpen t
⊢ IsOpen univ
[PROOFSTEP]
exact isOpen_univ
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝¹ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set (Set α)
hs : Set.Finite s
a✝ : Set α
s✝ : Set (Set α)
x✝¹ : ¬a✝ ∈ s✝
x✝ : Set.Finite s✝
ih : (∀ (t : Set α), t ∈ s✝ → IsOpen t) → IsOpen (⋂₀ s✝)
h : ∀ (t : Set α), t ∈ insert a✝ s✝ → IsOpen t
⊢ IsOpen (⋂₀ insert a✝ s✝)
[PROOFSTEP]
simp only [sInter_insert, ball_insert_iff] at h ⊢
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝¹ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set (Set α)
hs : Set.Finite s
a✝ : Set α
s✝ : Set (Set α)
x✝¹ : ¬a✝ ∈ s✝
x✝ : Set.Finite s✝
ih : (∀ (t : Set α), t ∈ s✝ → IsOpen t) → IsOpen (⋂₀ s✝)
h : IsOpen a✝ ∧ ∀ (x : Set α), x ∈ s✝ → IsOpen x
⊢ IsOpen (a✝ ∩ ⋂₀ s✝)
[PROOFSTEP]
exact h.1.inter (ih h.2)
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : Prop
⊢ IsOpen {_a | p}
[PROOFSTEP]
by_cases p
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : Prop
⊢ IsOpen {_a | p}
[PROOFSTEP]
by_cases p
[GOAL]
case pos
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : Prop
h : p
⊢ IsOpen {_a | p}
[PROOFSTEP]
simp [*]
[GOAL]
case neg
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : Prop
h : ¬p
⊢ IsOpen {_a | p}
[PROOFSTEP]
simp [*]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ IsClosed s₁ → IsClosed s₂ → IsClosed (s₁ ∪ s₂)
[PROOFSTEP]
simpa only [← isOpen_compl_iff, compl_union] using IsOpen.inter
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set (Set α)
⊢ (∀ (t : Set α), t ∈ s → IsClosed t) → IsClosed (⋂₀ s)
[PROOFSTEP]
simpa only [← isOpen_compl_iff, compl_sInter, sUnion_image] using isOpen_biUnion
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ IsClosed sᶜ ↔ IsOpen s
[PROOFSTEP]
rw [← isOpen_compl_iff, compl_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
h₁ : IsClosed s₁
h₂ : IsClosed s₂
⊢ IsClosed (s₁ ∩ s₂)
[PROOFSTEP]
rw [← isOpen_compl_iff] at *
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
h₁ : IsOpen s₁ᶜ
h₂ : IsOpen s₂ᶜ
⊢ IsOpen (s₁ ∩ s₂)ᶜ
[PROOFSTEP]
rw [compl_inter]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
h₁ : IsOpen s₁ᶜ
h₂ : IsOpen s₂ᶜ
⊢ IsOpen (s₁ᶜ ∪ s₂ᶜ)
[PROOFSTEP]
exact IsOpen.union h₁ h₂
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set β
f : β → Set α
hs : Set.Finite s
h : ∀ (i : β), i ∈ s → IsClosed (f i)
⊢ IsClosed (⋃ (i : β) (_ : i ∈ s), f i)
[PROOFSTEP]
simp only [← isOpen_compl_iff, compl_iUnion] at *
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set β
f : β → Set α
hs : Set.Finite s
h : ∀ (i : β), i ∈ s → IsOpen (f i)ᶜ
⊢ IsOpen (⋂ (i : β) (_ : i ∈ s), (f i)ᶜ)
[PROOFSTEP]
exact isOpen_biInter hs h
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
inst✝ : Finite ι
s : ι → Set α
h : ∀ (i : ι), IsClosed (s i)
⊢ IsClosed (⋃ (i : ι), s i)
[PROOFSTEP]
simp only [← isOpen_compl_iff, compl_iUnion] at *
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
inst✝ : Finite ι
s : ι → Set α
h : ∀ (i : ι), IsOpen (s i)ᶜ
⊢ IsOpen (⋂ (i : ι), (s i)ᶜ)
[PROOFSTEP]
exact isOpen_iInter h
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p q : α → Prop
hp : IsOpen {x | p x}
hq : IsClosed {x | q x}
⊢ IsClosed {x | p x → q x}
[PROOFSTEP]
simpa only [imp_iff_not_or] using hp.isClosed_compl.union hq
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
x : α
⊢ x ∈ interior s ↔ ∃ t, t ⊆ s ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
simp only [interior, mem_sUnion, mem_setOf_eq, and_assoc, and_left_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ s ⊆ interior s ↔ IsOpen s
[PROOFSTEP]
simp only [interior_eq_iff_isOpen.symm, Subset.antisymm_iff, interior_subset, true_and]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ interior (⋂ (i : ι) (_ : i ∈ s), f i) = ⋂ (i : ι) (_ : i ∈ s), interior (f i)
[PROOFSTEP]
classical
refine' s.induction_on (by simp) _
intro i s _ h₂
simp [h₂]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ interior (⋂ (i : ι) (_ : i ∈ s), f i) = ⋂ (i : ι) (_ : i ∈ s), interior (f i)
[PROOFSTEP]
refine' s.induction_on (by simp) _
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ interior (⋂ (i : ι) (_ : i ∈ ∅), f i) = ⋂ (i : ι) (_ : i ∈ ∅), interior (f i)
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ ∀ ⦃a : ι⦄ {s : Finset ι},
¬a ∈ s →
interior (⋂ (i : ι) (_ : i ∈ s), f i) = ⋂ (i : ι) (_ : i ∈ s), interior (f i) →
interior (⋂ (i : ι) (_ : i ∈ insert a s), f i) = ⋂ (i : ι) (_ : i ∈ insert a s), interior (f i)
[PROOFSTEP]
intro i s _ h₂
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝¹ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s✝ : Finset ι
f : ι → Set α
i : ι
s : Finset ι
a✝ : ¬i ∈ s
h₂ : interior (⋂ (i : ι) (_ : i ∈ s), f i) = ⋂ (i : ι) (_ : i ∈ s), interior (f i)
⊢ interior (⋂ (i_1 : ι) (_ : i_1 ∈ insert i s), f i_1) = ⋂ (i_1 : ι) (_ : i_1 ∈ insert i s), interior (f i_1)
[PROOFSTEP]
simp [h₂]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
⊢ interior (⋂ (i : ι), f i) = ⋂ (i : ι), interior (f i)
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
val✝ : Fintype ι
⊢ interior (⋂ (i : ι), f i) = ⋂ (i : ι), interior (f i)
[PROOFSTEP]
convert Finset.univ.interior_iInter f
[GOAL]
case h.e'_2.h.e'_3.h.e'_3.h
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
val✝ : Fintype ι
x✝ : ι
⊢ f x✝ = ⋂ (_ : x✝ ∈ Finset.univ), f x✝
[PROOFSTEP]
simp
[GOAL]
case h.e'_3.h.e'_3.h
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
val✝ : Fintype ι
x✝ : ι
⊢ interior (f x✝) = ⋂ (_ : x✝ ∈ Finset.univ), interior (f x✝)
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
h₁ : IsClosed s
h₂ : interior t = ∅
x : α
x✝ : x ∈ interior (s ∪ t)
u : Set α
hu₁ : IsOpen u
hu₂ : u ⊆ s ∪ t
hx₁ : x ∈ u
hx₂ : ¬x ∈ s
this : u \ s ⊆ t
⊢ u \ s ⊆ interior t
[PROOFSTEP]
rwa [(IsOpen.sdiff hu₁ h₁).subset_interior_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
h₁ : IsClosed s
h₂ : interior t = ∅
x : α
x✝ : x ∈ interior (s ∪ t)
u : Set α
hu₁ : IsOpen u
hu₂ : u ⊆ s ∪ t
hx₁ : x ∈ u
hx₂ : ¬x ∈ s
this✝ : u \ s ⊆ t
this : u \ s ⊆ interior t
⊢ u \ s ⊆ ∅
[PROOFSTEP]
rwa [h₂] at this
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ IsOpen s ↔ ∀ (x : α), x ∈ s → ∃ t, t ⊆ s ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
rw [← subset_interior_iff_isOpen]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ s ⊆ interior s ↔ ∀ (x : α), x ∈ s → ∃ t, t ⊆ s ∧ IsOpen t ∧ x ∈ t
[PROOFSTEP]
simp only [subset_def, mem_interior]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
S : Set (Set α)
⊢ interior (⋂₀ S) = interior (⋂ (s : Set α) (_ : s ∈ S), s)
[PROOFSTEP]
rw [sInter_eq_biInter]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ s \ t ⊆ closure t ↔ s ⊆ closure t
[PROOFSTEP]
rw [diff_subset_iff, union_eq_self_of_subset_left subset_closure]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : closure s ⊆ s
⊢ IsClosed s
[PROOFSTEP]
rw [subset_closure.antisymm h]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : closure s ⊆ s
⊢ IsClosed (closure s)
[PROOFSTEP]
exact isClosed_closure
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ Set.Nonempty (closure s) ↔ Set.Nonempty s
[PROOFSTEP]
simp only [nonempty_iff_ne_empty, Ne.def, closure_empty_iff]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ closure (⋃ (i : ι) (_ : i ∈ s), f i) = ⋃ (i : ι) (_ : i ∈ s), closure (f i)
[PROOFSTEP]
classical
refine' s.induction_on (by simp) _
intro i s _ h₂
simp [h₂]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ closure (⋃ (i : ι) (_ : i ∈ s), f i) = ⋃ (i : ι) (_ : i ∈ s), closure (f i)
[PROOFSTEP]
refine' s.induction_on (by simp) _
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ closure (⋃ (i : ι) (_ : i ∈ ∅), f i) = ⋃ (i : ι) (_ : i ∈ ∅), closure (f i)
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s : Finset ι
f : ι → Set α
⊢ ∀ ⦃a : ι⦄ {s : Finset ι},
¬a ∈ s →
closure (⋃ (i : ι) (_ : i ∈ s), f i) = ⋃ (i : ι) (_ : i ∈ s), closure (f i) →
closure (⋃ (i : ι) (_ : i ∈ insert a s), f i) = ⋃ (i : ι) (_ : i ∈ insert a s), closure (f i)
[PROOFSTEP]
intro i s _ h₂
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s✝¹ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
s✝ : Finset ι
f : ι → Set α
i : ι
s : Finset ι
a✝ : ¬i ∈ s
h₂ : closure (⋃ (i : ι) (_ : i ∈ s), f i) = ⋃ (i : ι) (_ : i ∈ s), closure (f i)
⊢ closure (⋃ (i_1 : ι) (_ : i_1 ∈ insert i s), f i_1) = ⋃ (i_1 : ι) (_ : i_1 ∈ insert i s), closure (f i_1)
[PROOFSTEP]
simp [h₂]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
⊢ closure (⋃ (i : ι), f i) = ⋃ (i : ι), closure (f i)
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
val✝ : Fintype ι
⊢ closure (⋃ (i : ι), f i) = ⋃ (i : ι), closure (f i)
[PROOFSTEP]
convert Finset.univ.closure_biUnion f
[GOAL]
case h.e'_2.h.e'_3.h.e'_3.h
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
val✝ : Fintype ι
x✝ : ι
⊢ f x✝ = ⋃ (_ : x✝ ∈ Finset.univ), f x✝
[PROOFSTEP]
simp
[GOAL]
case h.e'_3.h.e'_3.h
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
inst✝ : Finite ι
f : ι → Set α
val✝ : Fintype ι
x✝ : ι
⊢ closure (f x✝) = ⋃ (_ : x✝ ∈ Finset.univ), closure (f x✝)
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ closure s = (interior sᶜ)ᶜ
[PROOFSTEP]
rw [interior, closure, compl_sUnion, compl_image_set_of]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ ⋂₀ {t | IsClosed t ∧ s ⊆ t} = ⋂₀ {s_1 | IsOpen s_1ᶜ ∧ s_1ᶜ ⊆ sᶜ}
[PROOFSTEP]
simp only [compl_subset_compl, isOpen_compl_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ interior sᶜ = (closure s)ᶜ
[PROOFSTEP]
simp [closure_eq_compl_interior_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ closure sᶜ = (interior s)ᶜ
[PROOFSTEP]
simp [closure_eq_compl_interior_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
l : Filter α
h : l = ⊥
⊢ Filter.lift' ⊥ closure = ⊥
[PROOFSTEP]
rw [lift'_bot (monotone_closure _), closure_empty, principal_empty]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ interior s = ∅ ↔ Dense sᶜ
[PROOFSTEP]
rw [dense_iff_closure_eq, closure_compl, compl_univ_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : Dense s
⊢ Dense sᶜᶜ
[PROOFSTEP]
rwa [compl_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ Dense (closure s) ↔ Dense s
[PROOFSTEP]
rw [Dense, Dense, closure_closure]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ Dense s ↔ ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ Dense s → ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ (∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)) → Dense s
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : Dense s
⊢ ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
[PROOFSTEP]
rintro U U_op ⟨x, x_in⟩
[GOAL]
case mp.intro
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : Dense s
U : Set α
U_op : IsOpen U
x : α
x_in : x ∈ U
⊢ Set.Nonempty (U ∩ s)
[PROOFSTEP]
exact mem_closure_iff.1 (h _) U U_op x_in
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
⊢ Dense s
[PROOFSTEP]
intro x
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
x : α
⊢ x ∈ closure s
[PROOFSTEP]
rw [mem_closure_iff]
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
x : α
⊢ ∀ (o : Set α), IsOpen o → x ∈ o → Set.Nonempty (o ∩ s)
[PROOFSTEP]
intro U U_op x_in
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : ∀ (U : Set α), IsOpen U → Set.Nonempty U → Set.Nonempty (U ∩ s)
x : α
U : Set α
U_op : IsOpen U
x_in : x ∈ U
⊢ Set.Nonempty (U ∩ s)
[PROOFSTEP]
exact h U U_op ⟨_, x_in⟩
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
⊢ Dense {x}ᶜ ↔ ¬IsOpen {x}
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
⊢ Dense {x}ᶜ → ¬IsOpen {x}
[PROOFSTEP]
intro hd ho
[GOAL]
case mp
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
hd : Dense {x}ᶜ
ho : IsOpen {x}
⊢ False
[PROOFSTEP]
exact (hd.inter_open_nonempty _ ho (singleton_nonempty _)).ne_empty (inter_compl_self _)
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
⊢ ¬IsOpen {x} → Dense {x}ᶜ
[PROOFSTEP]
refine' fun ho => dense_iff_inter_open.2 fun U hU hne => inter_compl_nonempty_iff.2 fun hUx => _
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
ho : ¬IsOpen {x}
U : Set α
hU : IsOpen U
hne : Set.Nonempty U
hUx : U ⊆ {x}
⊢ False
[PROOFSTEP]
obtain rfl : U = { x }
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
ho : ¬IsOpen {x}
U : Set α
hU : IsOpen U
hne : Set.Nonempty U
hUx : U ⊆ {x}
⊢ U = {x}
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
ho : ¬IsOpen {x}
hU : IsOpen {x}
hne : Set.Nonempty {x}
hUx : {x} ⊆ {x}
⊢ False
[PROOFSTEP]
exact eq_singleton_iff_nonempty_unique_mem.2 ⟨hne, hUx⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
ho : ¬IsOpen {x}
hU : IsOpen {x}
hne : Set.Nonempty {x}
hUx : {x} ⊆ {x}
⊢ False
[PROOFSTEP]
exact ho hU
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ closure s \ frontier s = interior s
[PROOFSTEP]
rw [frontier, diff_diff_right_self, inter_eq_self_of_subset_right interior_subset_closure]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ s \ frontier s = interior s
[PROOFSTEP]
rw [frontier, diff_diff_right, diff_eq_empty.2 subset_closure, inter_eq_self_of_subset_right interior_subset,
empty_union]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ frontier s = closure s ∩ closure sᶜ
[PROOFSTEP]
rw [closure_compl, frontier, diff_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ frontier sᶜ = frontier s
[PROOFSTEP]
simp only [frontier_eq_closure_inter_closure, compl_compl, inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ frontier univ = ∅
[PROOFSTEP]
simp [frontier]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
⊢ frontier ∅ = ∅
[PROOFSTEP]
simp [frontier]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ frontier (s ∩ t) ⊆ frontier s ∩ closure t ∪ closure s ∩ frontier t
[PROOFSTEP]
simp only [frontier_eq_closure_inter_closure, compl_inter, closure_union]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ closure (s ∩ t) ∩ (closure sᶜ ∪ closure tᶜ) ⊆
closure s ∩ closure sᶜ ∩ closure t ∪ closure s ∩ (closure t ∩ closure tᶜ)
[PROOFSTEP]
refine' (inter_subset_inter_left _ (closure_inter_subset_inter_closure s t)).trans_eq _
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ closure s ∩ closure t ∩ (closure sᶜ ∪ closure tᶜ) =
closure s ∩ closure sᶜ ∩ closure t ∪ closure s ∩ (closure t ∩ closure tᶜ)
[PROOFSTEP]
simp only [inter_distrib_left, inter_distrib_right, inter_assoc, inter_comm (closure t)]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ frontier (s ∪ t) ⊆ frontier s ∩ closure tᶜ ∪ closure sᶜ ∩ frontier t
[PROOFSTEP]
simpa only [frontier_compl, ← compl_union] using frontier_inter_subset sᶜ tᶜ
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
hs : IsClosed s
⊢ frontier s = s \ interior s
[PROOFSTEP]
rw [frontier, hs.closure_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
hs : IsOpen s
⊢ frontier s = closure s \ s
[PROOFSTEP]
rw [frontier, hs.interior_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
hs : IsOpen s
⊢ s ∩ frontier s = ∅
[PROOFSTEP]
rw [hs.frontier_eq, inter_diff_self]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ IsClosed (frontier s)
[PROOFSTEP]
rw [frontier_eq_closure_inter_closure]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ IsClosed (closure s ∩ closure sᶜ)
[PROOFSTEP]
exact IsClosed.inter isClosed_closure isClosed_closure
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
⊢ interior (frontier s) = ∅
[PROOFSTEP]
have A : frontier s = s \ interior s := h.frontier_eq
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
⊢ interior (frontier s) = ∅
[PROOFSTEP]
have B : interior (frontier s) ⊆ interior s := by rw [A]; exact interior_mono (diff_subset _ _)
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
⊢ interior (frontier s) ⊆ interior s
[PROOFSTEP]
rw [A]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
⊢ interior (s \ interior s) ⊆ interior s
[PROOFSTEP]
exact interior_mono (diff_subset _ _)
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
B : interior (frontier s) ⊆ interior s
⊢ interior (frontier s) = ∅
[PROOFSTEP]
have C : interior (frontier s) ⊆ frontier s := interior_subset
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
B : interior (frontier s) ⊆ interior s
C : interior (frontier s) ⊆ frontier s
⊢ interior (frontier s) = ∅
[PROOFSTEP]
have : interior (frontier s) ⊆ interior s ∩ (s \ interior s) := subset_inter B (by simpa [A] using C)
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
B : interior (frontier s) ⊆ interior s
C : interior (frontier s) ⊆ frontier s
⊢ interior (frontier s) ⊆ s \ interior s
[PROOFSTEP]
simpa [A] using C
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
h : IsClosed s
A : frontier s = s \ interior s
B : interior (frontier s) ⊆ interior s
C : interior (frontier s) ⊆ frontier s
this : interior (frontier s) ⊆ interior s ∩ (s \ interior s)
⊢ interior (frontier s) = ∅
[PROOFSTEP]
rwa [inter_diff_self, subset_empty_iff] at this
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ frontier s = (interior s)ᶜ ∩ (interior sᶜ)ᶜ
[PROOFSTEP]
rw [← frontier_compl, ← closure_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ frontier sᶜ = closure sᶜ ∩ (interior sᶜ)ᶜ
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ (frontier s)ᶜ = interior s ∪ interior sᶜ
[PROOFSTEP]
rw [frontier_eq_inter_compl_interior]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ ((interior s)ᶜ ∩ (interior sᶜ)ᶜ)ᶜ = interior s ∪ interior sᶜ
[PROOFSTEP]
simp only [compl_inter, compl_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ 𝓝 a = ⨅ (s : Set α) (_ : IsOpen s) (_ : a ∈ s), 𝓟 s
[PROOFSTEP]
simp only [nhds_def, mem_setOf_eq, @and_comm (a ∈ _), iInf_and]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ HasBasis (𝓝 a) (fun s => a ∈ s ∧ IsOpen s) fun s => s
[PROOFSTEP]
rw [nhds_def]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ HasBasis (⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ IsOpen s}), 𝓟 s) (fun s => a ∈ s ∧ IsOpen s) fun s => s
[PROOFSTEP]
exact
hasBasis_biInf_principal
(fun s ⟨has, hs⟩ t ⟨hat, ht⟩ =>
⟨s ∩ t, ⟨⟨has, hat⟩, IsOpen.inter hs ht⟩, ⟨inter_subset_left _ _, inter_subset_right _ _⟩⟩)
⟨univ, ⟨mem_univ a, isOpen_univ⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
t : Set α
⊢ (∃ x, (a ∈ xᶜ ∧ IsOpen xᶜ) ∧ xᶜ ⊆ t) ↔ ∃ i, (¬a ∈ i ∧ IsClosed i) ∧ iᶜ ⊆ t
[PROOFSTEP]
simp only [isOpen_compl_iff, mem_compl_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
a : α
⊢ f ≤ 𝓝 a ↔ ∀ (s : Set α), a ∈ s → IsOpen s → s ∈ f
[PROOFSTEP]
simp [nhds_def]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
a : α
s : Set α
h : a ∈ s
o : IsOpen s
sf : 𝓟 s ≤ f
⊢ 𝓝 a ≤ f
[PROOFSTEP]
rw [nhds_def]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
a : α
s : Set α
h : a ∈ s
o : IsOpen s
sf : 𝓟 s ≤ f
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ IsOpen s}), 𝓟 s ≤ f
[PROOFSTEP]
exact iInf₂_le_of_le s ⟨h, o⟩ sf
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
p : α → Prop
⊢ (∃ t, t ⊆ {x | (fun x => p x) x} ∧ IsOpen t ∧ a ∈ t) ↔ ∃ t, (∀ (x : α), x ∈ t → p x) ∧ IsOpen t ∧ a ∈ t
[PROOFSTEP]
simp only [subset_def, exists_prop, mem_setOf_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ HasBasis (𝓝 a) (fun s => s ∈ 𝓝 a ∧ IsOpen s) fun x => x
[PROOFSTEP]
convert nhds_basis_opens a using 2
[GOAL]
case h.e'_4.h.a
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
x✝ : Set α
⊢ x✝ ∈ 𝓝 a ∧ IsOpen x✝ ↔ a ∈ x✝ ∧ IsOpen x✝
[PROOFSTEP]
exact and_congr_left_iff.2 IsOpen.mem_nhds_iff
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s U : Set α
h : U ∈ ⨆ (x : α) (_ : x ∈ s), 𝓝 x
⊢ ∀ (x : α), x ∈ s → U ∈ 𝓝 x
[PROOFSTEP]
simpa using h
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : α → Prop
a : α
⊢ (∃ᶠ (y : α) in 𝓝 a, ∃ᶠ (x : α) in 𝓝 y, p x) ↔ ∃ᶠ (x : α) in 𝓝 a, p x
[PROOFSTEP]
rw [← not_iff_not]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : α → Prop
a : α
⊢ (¬∃ᶠ (y : α) in 𝓝 a, ∃ᶠ (x : α) in 𝓝 y, p x) ↔ ¬∃ᶠ (x : α) in 𝓝 a, p x
[PROOFSTEP]
simp only [not_frequently, eventually_eventually_nhds]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
P : Set α → Prop
hP : ∀ (s t : Set α), s ⊆ t → P s → P t
⊢ (∀ (i : Set α), x ∈ i ∧ IsOpen i → P i) ↔ ∀ (s : Set α), IsOpen s → x ∈ s → P s
[PROOFSTEP]
simp only [@and_comm (x ∈ _), and_imp]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝² : TopologicalSpace α
inst✝¹ : Nonempty β
inst✝ : SemilatticeSup β
f : β → α
a : α
⊢ (∀ (ib : Set α), a ∈ ib ∧ IsOpen ib → ∃ ia, True ∧ ∀ (x : β), x ∈ Ici ia → f x ∈ ib) ↔
∀ (U : Set α), a ∈ U → IsOpen U → ∃ N, ∀ (n : β), N ≤ n → f n ∈ U
[PROOFSTEP]
simp only [and_imp, exists_prop, true_and_iff, mem_Ici, ge_iff_le]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
F : Filter α
⊢ ClusterPt x F ↔ ¬Disjoint (𝓝 x) F
[PROOFSTEP]
rw [disjoint_iff, ClusterPt, neBot_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
s : Set α
⊢ ClusterPt x (𝓟 s) ↔ ∃ᶠ (y : α) in 𝓝 x, y ∈ s
[PROOFSTEP]
simp only [clusterPt_principal_iff, frequently_iff, Set.Nonempty, exists_prop, mem_inter_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
x : α
f : Filter α
H : f ≤ 𝓝 x
inst✝ : NeBot f
⊢ ClusterPt x f
[PROOFSTEP]
rwa [ClusterPt, inf_eq_right.mpr H]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
f : Filter α
H : 𝓝 x ≤ f
⊢ ClusterPt x f
[PROOFSTEP]
simp only [ClusterPt, inf_eq_left.mpr H, nhds_neBot]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
x : α
F : Filter ι
u : ι → α
⊢ MapClusterPt x F u ↔ ∀ (s : Set α), s ∈ 𝓝 x → ∃ᶠ (a : ι) in F, u a ∈ s
[PROOFSTEP]
simp_rw [MapClusterPt, ClusterPt, inf_neBot_iff_frequently_left, frequently_map]
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
ι : Type u_1
x : α
F : Filter ι
u : ι → α
⊢ (∀ {p : α → Prop}, (∀ᶠ (x : α) in 𝓝 x, p x) → ∃ᶠ (a : ι) in F, p (u a)) ↔
∀ (s : Set α), s ∈ 𝓝 x → ∃ᶠ (a : ι) in F, u a ∈ s
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
δ : Type u_2
F : Filter ι
φ : δ → ι
p : Filter δ
x : α
u : ι → α
inst✝ : NeBot p
h : Tendsto φ p F
H : Tendsto (u ∘ φ) p (𝓝 x)
⊢ MapClusterPt x F u
[PROOFSTEP]
have :=
calc
map (u ∘ φ) p = map u (map φ p) := map_map
_ ≤ map u F := map_mono h
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
δ : Type u_2
F : Filter ι
φ : δ → ι
p : Filter δ
x : α
u : ι → α
inst✝ : NeBot p
h : Tendsto φ p F
H : Tendsto (u ∘ φ) p (𝓝 x)
this : map (u ∘ φ) p ≤ map u F
⊢ MapClusterPt x F u
[PROOFSTEP]
have : map (u ∘ φ) p ≤ 𝓝 x ⊓ map u F := le_inf H this
[GOAL]
α : Type u
β : Type v
ι✝ : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
ι : Type u_1
δ : Type u_2
F : Filter ι
φ : δ → ι
p : Filter δ
x : α
u : ι → α
inst✝ : NeBot p
h : Tendsto φ p F
H : Tendsto (u ∘ φ) p (𝓝 x)
this✝ : map (u ∘ φ) p ≤ map u F
this : map (u ∘ φ) p ≤ 𝓝 x ⊓ map u F
⊢ MapClusterPt x F u
[PROOFSTEP]
exact neBot_of_le this
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
F : Filter α
⊢ AccPt x F ↔ ClusterPt x (𝓟 {x}ᶜ ⊓ F)
[PROOFSTEP]
rw [AccPt, nhdsWithin, ClusterPt, inf_assoc]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
C : Set α
⊢ AccPt x (𝓟 C) ↔ ClusterPt x (𝓟 (C \ {x}))
[PROOFSTEP]
rw [acc_iff_cluster, inf_principal, inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
C : Set α
⊢ ClusterPt x (𝓟 (C ∩ {x}ᶜ)) ↔ ClusterPt x (𝓟 (C \ {x}))
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
C : Set α
⊢ AccPt x (𝓟 C) ↔ ∀ (U : Set α), U ∈ 𝓝 x → ∃ y, y ∈ U ∩ C ∧ y ≠ x
[PROOFSTEP]
simp [acc_principal_iff_cluster, clusterPt_principal_iff, Set.Nonempty, exists_prop, and_assoc, @and_comm (¬_ = x)]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
x : α
C : Set α
⊢ AccPt x (𝓟 C) ↔ ∃ᶠ (y : α) in 𝓝 x, y ≠ x ∧ y ∈ C
[PROOFSTEP]
simp [acc_principal_iff_cluster, clusterPt_principal_iff_frequently, and_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
x : α
⊢ x ∈ interior s ↔ x ∈ {a | s ∈ 𝓝 a}
[PROOFSTEP]
simp only [mem_interior, mem_nhds_iff, mem_setOf_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ {a | s ∈ 𝓝 a} = {a | 𝓝 a ≤ 𝓟 s}
[PROOFSTEP]
simp only [le_principal_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
p : α → Prop
⊢ IsOpen {x | ∀ᶠ (y : α) in 𝓝 x, p y}
[PROOFSTEP]
simp only [← interior_setOf_eq, isOpen_interior]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s V : Set α
⊢ s ⊆ interior V ↔ ∀ (x : α), x ∈ s → V ∈ 𝓝 x
[PROOFSTEP]
simp_rw [subset_def, mem_interior_iff_mem_nhds]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ s ⊆ interior s ↔ ∀ (a : α), a ∈ s → 𝓝 a ≤ 𝓟 s
[PROOFSTEP]
rw [interior_eq_nhds]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ s ⊆ {a | 𝓝 a ≤ 𝓟 s} ↔ ∀ (a : α), a ∈ s → 𝓝 a ≤ 𝓟 s
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ IsOpen s ↔ ∀ (x : α), x ∈ s → ∀ (l : Ultrafilter α), ↑l ≤ 𝓝 x → s ∈ l
[PROOFSTEP]
simp_rw [isOpen_iff_mem_nhds, ← mem_iff_ultrafilter]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ IsOpen {a} ↔ 𝓝 a = pure a
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ IsOpen {a} → 𝓝 a = pure a
[PROOFSTEP]
intro h
[GOAL]
case mp
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
h : IsOpen {a}
⊢ 𝓝 a = pure a
[PROOFSTEP]
apply le_antisymm _ (pure_le_nhds a)
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
h : IsOpen {a}
⊢ 𝓝 a ≤ pure a
[PROOFSTEP]
rw [le_pure_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
h : IsOpen {a}
⊢ {a} ∈ 𝓝 a
[PROOFSTEP]
exact h.mem_nhds (mem_singleton a)
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
⊢ 𝓝 a = pure a → IsOpen {a}
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
h : 𝓝 a = pure a
⊢ IsOpen {a}
[PROOFSTEP]
simp [isOpen_iff_nhds, h]
[GOAL]
α✝ : Type u
β : Type v
ι : Sort w
a✝ : α✝
s s₁ s₂ t : Set α✝
p p₁ p₂ : α✝ → Prop
inst✝¹ : TopologicalSpace α✝
α : Type u_1
inst✝ : TopologicalSpace α
a : α
⊢ IsOpen {a} ↔ 𝓝[{a}ᶜ] a = ⊥
[PROOFSTEP]
rw [isOpen_singleton_iff_nhds_eq_pure, nhdsWithin, ← mem_iff_inf_principal_compl, ← le_pure_iff, nhds_neBot.le_pure_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
a : α
⊢ a ∈ closure s ↔ ∃ᶠ (x : α) in 𝓝 a, x ∈ s
[PROOFSTEP]
rw [Filter.Frequently, Filter.Eventually, ← mem_interior_iff_mem_nhds, closure_eq_compl_interior_compl]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
a : α
⊢ a ∈ (interior sᶜ)ᶜ ↔ ¬a ∈ interior {x | ¬x ∈ s}
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ IsClosed s ↔ ∀ (x : α), (∃ᶠ (y : α) in 𝓝 x, y ∈ s) → x ∈ s
[PROOFSTEP]
rw [← closure_subset_iff_isClosed]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ closure s ⊆ s ↔ ∀ (x : α), (∃ᶠ (y : α) in 𝓝 x, y ∈ s) → x ∈ s
[PROOFSTEP]
refine' forall_congr' fun x => _
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
x : α
⊢ x ∈ closure s → x ∈ s ↔ (∃ᶠ (y : α) in 𝓝 x, y ∈ s) → x ∈ s
[PROOFSTEP]
rw [mem_closure_iff_frequently]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
⊢ IsClosed {x | ClusterPt x f}
[PROOFSTEP]
simp only [ClusterPt, inf_neBot_iff_frequently_left, setOf_forall, imp_iff_not_or]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
⊢ IsClosed (⋂ (i : α → Prop), {x | (¬∀ᶠ (x : α) in 𝓝 x, i x) ∨ ∃ᶠ (x : α) in f, i x})
[PROOFSTEP]
refine' isClosed_iInter fun p => IsClosed.union _ _
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
p : α → Prop
⊢ IsClosed fun x => (∀ᶠ (x : α) in 𝓝 x, p x) → False
[PROOFSTEP]
apply isClosed_compl_iff.2
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
p : α → Prop
⊢ IsClosed fun x => (∀ᶠ (x : α) in f, ¬(fun x => p x) x) → False
[PROOFSTEP]
apply isClosed_compl_iff.2
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
p : α → Prop
⊢ IsOpen fun x => sets (𝓝 x) {x | (fun x => p x) x}
case refine'_2
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : Filter α
p : α → Prop
⊢ IsOpen fun x => sets f {x | (fun x => ¬(fun x => p x) x) x}
[PROOFSTEP]
exacts [isOpen_setOf_eventually_nhds, isOpen_const]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
x : α
inst✝ : NeBot (𝓝[{x}ᶜ] x)
⊢ Dense {x}ᶜ
[PROOFSTEP]
intro y
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
x : α
inst✝ : NeBot (𝓝[{x}ᶜ] x)
y : α
⊢ y ∈ closure {x}ᶜ
[PROOFSTEP]
rcases eq_or_ne y x with (rfl | hne)
[GOAL]
case inl
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
y : α
inst✝ : NeBot (𝓝[{y}ᶜ] y)
⊢ y ∈ closure {y}ᶜ
[PROOFSTEP]
rwa [mem_closure_iff_nhdsWithin_neBot]
[GOAL]
case inr
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝¹ : TopologicalSpace α
x : α
inst✝ : NeBot (𝓝[{x}ᶜ] x)
y : α
hne : y ≠ x
⊢ y ∈ closure {x}ᶜ
[PROOFSTEP]
exact subset_closure hne
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
a : α
⊢ a ∈ closure s ↔ ∀ (t : Set α), t ∈ 𝓝 a → ∃ y, ↑y ∈ t
[PROOFSTEP]
simp only [mem_closure_iff_nhds, Set.inter_nonempty_iff_exists_right, SetCoe.exists, exists_prop]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
A : Set α
x : α
⊢ x ∈ closure A ↔ NeBot (comap Subtype.val (𝓝 x))
[PROOFSTEP]
simp_rw [mem_closure_iff_nhds, comap_neBot_iff, Set.inter_nonempty_iff_exists_right, SetCoe.exists, exists_prop]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t✝ : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
p : ι → Prop
s : ι → Set α
h : HasBasis (𝓝 a) p s
t : Set α
⊢ (∀ ⦃i : ι⦄, p i → ∀ ⦃j : Unit⦄, True → Set.Nonempty (s i ∩ t)) ↔ ∀ (i : ι), p i → Set.Nonempty (s i ∩ t)
[PROOFSTEP]
simp only [exists_prop, forall_const]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t✝ : Set α
p✝ p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
a : α
p : ι → Prop
s : ι → Set α
h : HasBasis (𝓝 a) p s
t : Set α
⊢ (∀ (i : ι), p i → Set.Nonempty (s i ∩ t)) ↔ ∀ (i : ι), p i → ∃ y, y ∈ t ∧ y ∈ s i
[PROOFSTEP]
simp only [Set.Nonempty, mem_inter_iff, exists_prop, and_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
F : Filter α
a : α
⊢ ClusterPt a F ↔ ∀ (s : Set α), s ∈ F → a ∈ closure s
[PROOFSTEP]
simp_rw [ClusterPt, inf_neBot_iff, mem_closure_iff_nhds]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
F : Filter α
a : α
⊢ (∀ ⦃s : Set α⦄, s ∈ 𝓝 a → ∀ ⦃s' : Set α⦄, s' ∈ F → Set.Nonempty (s ∩ s')) ↔
∀ (s : Set α), s ∈ F → ∀ (t : Set α), t ∈ 𝓝 a → Set.Nonempty (t ∩ s)
[PROOFSTEP]
rw [forall₂_swap]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
F : Filter α
a : α
⊢ ClusterPt a F ↔ pure a ≤ Filter.lift' F closure
[PROOFSTEP]
simp_rw [clusterPt_iff_forall_mem_closure, (hasBasis_pure _).le_basis_iff F.basis_sets.lift'_closure, id,
singleton_subset_iff, true_and, exists_const]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
F : Filter α
a : α
⊢ ClusterPt a F ↔ NeBot (Filter.lift' F closure ⊓ pure a)
[PROOFSTEP]
rw [clusterPt_iff_lift'_closure, ← Ultrafilter.coe_pure, inf_comm, Ultrafilter.inf_neBot_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
F : Filter α
a : α
⊢ ClusterPt a (Filter.lift' F closure) ↔ ClusterPt a F
[PROOFSTEP]
simp [clusterPt_iff_lift'_closure, lift'_lift'_assoc (monotone_closure α) (monotone_closure α)]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
x : α
⊢ x ∈ closure s ↔ ∃ u, s ∈ u ∧ ↑u ≤ 𝓝 x
[PROOFSTEP]
simp [closure_eq_cluster_pts, ClusterPt, ← exists_ultrafilter_iff, and_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ closure s ⊆ s ↔ ∀ (a : α), ClusterPt a (𝓟 s) → a ∈ s
[PROOFSTEP]
simp only [subset_def, mem_closure_iff_clusterPt]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s : Set α
⊢ IsClosed s ↔ ∀ (x : α), (∀ (U : Set α), U ∈ 𝓝 x → Set.Nonempty (U ∩ s)) → x ∈ s
[PROOFSTEP]
simp_rw [isClosed_iff_clusterPt, ClusterPt, inf_principal_neBot_iff]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
h : IsClosed t
⊢ interior (s ∪ t) ⊆ interior s ∪ t
[PROOFSTEP]
simpa only [union_comm _ t] using h.interior_union_left
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
h : IsOpen s
⊢ (closure (s ∩ t))ᶜ ⊆ (s ∩ closure t)ᶜ
[PROOFSTEP]
simpa only [← interior_compl, compl_inter] using IsClosed.interior_union_left h.isClosed_compl
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
h : IsOpen t
⊢ closure s ∩ t ⊆ closure (s ∩ t)
[PROOFSTEP]
simpa only [inter_comm t] using h.inter_closure
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
hs : Dense s
ht : IsOpen t
⊢ t = t ∩ closure s
[PROOFSTEP]
rw [hs.closure_eq, inter_univ]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁✝ s₂✝ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s₁ s₂ : Set α
x : α
h : x ∈ closure (s₁ ∪ s₂)
h₁ : s₁ᶜ ∈ 𝓝 x
⊢ x ∈ closure s₂
[PROOFSTEP]
rw [mem_closure_iff_nhds_neBot] at *
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁✝ s₂✝ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s₁ s₂ : Set α
x : α
h : 𝓝 x ⊓ 𝓟 (s₁ ∪ s₂) ≠ ⊥
h₁ : s₁ᶜ ∈ 𝓝 x
⊢ 𝓝 x ⊓ 𝓟 s₂ ≠ ⊥
[PROOFSTEP]
rwa [←
calc
𝓝 x ⊓ principal (s₁ ∪ s₂) = 𝓝 x ⊓ (principal s₁ ⊔ principal s₂) := by rw [sup_principal]
_ = 𝓝 x ⊓ principal s₁ ⊔ 𝓝 x ⊓ principal s₂ := inf_sup_left
_ = ⊥ ⊔ 𝓝 x ⊓ principal s₂ := by rw [inf_principal_eq_bot.mpr h₁]
_ = 𝓝 x ⊓ principal s₂ := bot_sup_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁✝ s₂✝ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s₁ s₂ : Set α
x : α
h : 𝓝 x ⊓ 𝓟 (s₁ ∪ s₂) ≠ ⊥
h₁ : s₁ᶜ ∈ 𝓝 x
⊢ 𝓝 x ⊓ 𝓟 (s₁ ∪ s₂) = 𝓝 x ⊓ (𝓟 s₁ ⊔ 𝓟 s₂)
[PROOFSTEP]
rw [sup_principal]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s s₁✝ s₂✝ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s₁ s₂ : Set α
x : α
h : 𝓝 x ⊓ 𝓟 (s₁ ∪ s₂) ≠ ⊥
h₁ : s₁ᶜ ∈ 𝓝 x
⊢ 𝓝 x ⊓ 𝓟 s₁ ⊔ 𝓝 x ⊓ 𝓟 s₂ = ⊥ ⊔ 𝓝 x ⊓ 𝓟 s₂
[PROOFSTEP]
rw [inf_principal_eq_bot.mpr h₁]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
hs : Dense s
ht : Dense t
hso : IsOpen s
x : α
⊢ x ∈ closure (s ∩ closure t)
[PROOFSTEP]
simp [hs.closure_eq, ht.closure_eq]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ closure s \ closure t = (closure t)ᶜ ∩ closure s
[PROOFSTEP]
simp only [diff_eq, inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
s t : Set α
⊢ closure ((closure t)ᶜ ∩ s) = closure (s \ closure t)
[PROOFSTEP]
simp only [diff_eq, inter_comm]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : ∀ (x : β), ¬x ∈ s → f x = a
⊢ Tendsto f (l ⊓ 𝓟 s) (𝓝 a) ↔ Tendsto f l (𝓝 a)
[PROOFSTEP]
rw [tendsto_iff_comap, tendsto_iff_comap]
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : ∀ (x : β), ¬x ∈ s → f x = a
⊢ l ⊓ 𝓟 s ≤ comap f (𝓝 a) ↔ l ≤ comap f (𝓝 a)
[PROOFSTEP]
replace h : 𝓟 sᶜ ≤ comap f (𝓝 a)
[GOAL]
case h
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : ∀ (x : β), ¬x ∈ s → f x = a
⊢ 𝓟 sᶜ ≤ comap f (𝓝 a)
[PROOFSTEP]
rintro U ⟨t, ht, htU⟩ x hx
[GOAL]
case h.intro.intro
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : ∀ (x : β), ¬x ∈ s → f x = a
U : Set β
t : Set α
ht : t ∈ 𝓝 a
htU : f ⁻¹' t ⊆ U
x : β
hx : x ∈ sᶜ
⊢ x ∈ U
[PROOFSTEP]
have : f x ∈ t := (h x hx).symm ▸ mem_of_mem_nhds ht
[GOAL]
case h.intro.intro
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t✝ : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : ∀ (x : β), ¬x ∈ s → f x = a
U : Set β
t : Set α
ht : t ∈ 𝓝 a
htU : f ⁻¹' t ⊆ U
x : β
hx : x ∈ sᶜ
this : f x ∈ t
⊢ x ∈ U
[PROOFSTEP]
exact htU this
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : 𝓟 sᶜ ≤ comap f (𝓝 a)
⊢ l ⊓ 𝓟 s ≤ comap f (𝓝 a) ↔ l ≤ comap f (𝓝 a)
[PROOFSTEP]
refine' ⟨fun h' => _, le_trans inf_le_left⟩
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : 𝓟 sᶜ ≤ comap f (𝓝 a)
h' : l ⊓ 𝓟 s ≤ comap f (𝓝 a)
⊢ l ≤ comap f (𝓝 a)
[PROOFSTEP]
have := sup_le h' h
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : 𝓟 sᶜ ≤ comap f (𝓝 a)
h' : l ⊓ 𝓟 s ≤ comap f (𝓝 a)
this : l ⊓ 𝓟 s ⊔ 𝓟 sᶜ ≤ comap f (𝓝 a)
⊢ l ≤ comap f (𝓝 a)
[PROOFSTEP]
rw [sup_inf_right, sup_principal, union_compl_self, principal_univ, inf_top_eq, sup_le_iff] at this
[GOAL]
α : Type u
β : Type v
ι : Sort w
a✝ : α
s✝ s₁ s₂ t : Set α
p p₁ p₂ : α → Prop
inst✝ : TopologicalSpace α
f : β → α
l : Filter β
s : Set β
a : α
h : 𝓟 sᶜ ≤ comap f (𝓝 a)
h' : l ⊓ 𝓟 s ≤ comap f (𝓝 a)
this : l ≤ comap f (𝓝 a) ∧ 𝓟 sᶜ ≤ comap f (𝓝 a)
⊢ l ≤ comap f (𝓝 a)
[PROOFSTEP]
exact this.1
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f g : α → β
h : Continuous f
h' : ∀ (x : α), f x = g x
⊢ Continuous g
[PROOFSTEP]
convert h
[GOAL]
case h.e'_5
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f g : α → β
h : Continuous f
h' : ∀ (x : α), f x = g x
⊢ g = f
[PROOFSTEP]
ext
[GOAL]
case h.e'_5.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f g : α → β
h : Continuous f
h' : ∀ (x : α), f x = g x
x✝ : α
⊢ g x✝ = f x✝
[PROOFSTEP]
rw [h']
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f g : α → β
x : α
h : f =ᶠ[𝓝 x] g
⊢ ContinuousAt f x ↔ ContinuousAt g x
[PROOFSTEP]
simp only [ContinuousAt, tendsto_congr' h, h.eq_of_nhds]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
M₀ : Type u_5
inst✝ : Zero M₀
a : α
f : α → M₀
⊢ f =ᶠ[𝓝 a] 0 ↔ ¬a ∈ closure (Function.support f)
[PROOFSTEP]
rw [← mem_compl_iff, ← interior_compl, mem_interior_iff_mem_nhds, Function.compl_support]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
M₀ : Type u_5
inst✝ : Zero M₀
a : α
f : α → M₀
⊢ f =ᶠ[𝓝 a] 0 ↔ {x | f x = 0} ∈ 𝓝 a
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : β → γ
f : α → β
x : α
y : β
hg : ContinuousAt g y
hf : ContinuousAt f x
hy : f x = y
⊢ ContinuousAt (g ∘ f) x
[PROOFSTEP]
subst hy
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
g : β → γ
f : α → β
x : α
hf : ContinuousAt f x
hg : ContinuousAt g (f x)
⊢ ContinuousAt (g ∘ f) x
[PROOFSTEP]
exact hg.comp hf
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
⊢ (∀ (x : Set β), IsOpen xᶜ → IsOpen (f ⁻¹' xᶜ)) ↔ ∀ (s : Set β), IsClosed s → IsClosed (f ⁻¹' s)
[PROOFSTEP]
simp only [isOpen_compl_iff, preimage_compl]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
⊢ Continuous f ↔ ∀ (x : α) (g : Ultrafilter α), ↑g ≤ 𝓝 x → Tendsto f (↑g) (𝓝 (f x))
[PROOFSTEP]
simp only [continuous_iff_continuousAt, continuousAt_iff_ultrafilter]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : Continuous f
t : Set β
⊢ closure (f ⁻¹' t) ⊆ f ⁻¹' closure t
[PROOFSTEP]
rw [← (isClosed_closure.preimage hf).closure_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
hf : Continuous f
t : Set β
⊢ closure (f ⁻¹' t) ⊆ closure (f ⁻¹' closure t)
[PROOFSTEP]
exact closure_mono (preimage_mono subset_closure)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
t : Set β
f : α → β
h : MapsTo f s t
hc : Continuous f
⊢ MapsTo f (closure s) (closure t)
[PROOFSTEP]
simp only [MapsTo, mem_closure_iff_clusterPt]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
s : Set α
t : Set β
f : α → β
h : MapsTo f s t
hc : Continuous f
⊢ ∀ ⦃x : α⦄, ClusterPt x (𝓟 s) → ClusterPt (f x) (𝓟 t)
[PROOFSTEP]
exact fun x hx => hx.map hc.continuousAt (tendsto_principal_principal.2 h)
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
s : Set α
h : Continuous f
⊢ closure s ⊆ f ⁻¹' closure (f '' s)
[PROOFSTEP]
rw [← Set.image_subset_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
f : α → β
s : Set α
h : Continuous f
⊢ f '' closure s ⊆ closure (f '' s)
[PROOFSTEP]
exact image_closure_subset_closure_image h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f : κ → β
g : β → γ
hf : Surjective f
x : β
⊢ x ∈ closure (range f)
[PROOFSTEP]
simp [hf.range_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f : κ → β
g : β → γ
s : Set α
h : Dense s
⊢ DenseRange Subtype.val
[PROOFSTEP]
simpa only [DenseRange, Subtype.range_coe_subtype]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f✝ : κ → β
g : β → γ
f : α → β
hf : Continuous f
s : Set α
hs : Dense s
⊢ range f ⊆ closure (f '' s)
[PROOFSTEP]
rw [← image_univ, ← hs.closure_eq]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f✝ : κ → β
g : β → γ
f : α → β
hf : Continuous f
s : Set α
hs : Dense s
⊢ f '' closure s ⊆ closure (f '' s)
[PROOFSTEP]
exact image_closure_subset_closure_image hf
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f : κ → β
g : β → γ
hf : DenseRange f
s : Set β
hs : IsOpen s
⊢ s ⊆ closure (f '' (f ⁻¹' s))
[PROOFSTEP]
rw [image_preimage_eq_inter_range]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f : κ → β
g : β → γ
hf : DenseRange f
s : Set β
hs : IsOpen s
⊢ s ⊆ closure (s ∩ range f)
[PROOFSTEP]
exact hf.open_subset_closure_inter hs
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f✝ : κ → β
g✝ g : β → γ
f : κ → β
hg : DenseRange g
hf : DenseRange f
cg : Continuous g
⊢ DenseRange (g ∘ f)
[PROOFSTEP]
rw [DenseRange, range_comp]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
κ : Type u_5
ι : Type u_6
f✝ : κ → β
g✝ g : β → γ
f : κ → β
hg : DenseRange g
hf : DenseRange f
cg : Continuous g
⊢ Dense (g '' range f)
[PROOFSTEP]
exact hg.dense_image cg hf
| {"mathlib_filename": "Mathlib.Topology.Basic", "llama_tokens": 30525} |
[GOAL]
α : Type u
⊢ ∀ (t₁ : Set (Ultrafilter α)),
t₁ ∈ ultrafilterBasis α →
∀ (t₂ : Set (Ultrafilter α)),
t₂ ∈ ultrafilterBasis α →
∀ (x : Ultrafilter α), x ∈ t₁ ∩ t₂ → ∃ t₃, t₃ ∈ ultrafilterBasis α ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
rintro _ ⟨a, rfl⟩ _ ⟨b, rfl⟩ u ⟨ua, ub⟩
[GOAL]
case intro.intro.intro
α : Type u
a b : Set α
u : Ultrafilter α
ua : u ∈ (fun s => {u | s ∈ u}) a
ub : u ∈ (fun s => {u | s ∈ u}) b
⊢ ∃ t₃, t₃ ∈ ultrafilterBasis α ∧ u ∈ t₃ ∧ t₃ ⊆ (fun s => {u | s ∈ u}) a ∩ (fun s => {u | s ∈ u}) b
[PROOFSTEP]
refine' ⟨_, ⟨a ∩ b, rfl⟩, inter_mem ua ub, fun v hv => ⟨_, _⟩⟩
[GOAL]
case intro.intro.intro.refine'_1
α : Type u
a b : Set α
u : Ultrafilter α
ua : u ∈ (fun s => {u | s ∈ u}) a
ub : u ∈ (fun s => {u | s ∈ u}) b
v : Ultrafilter α
hv : v ∈ (fun s => {u | s ∈ u}) (a ∩ b)
⊢ v ∈ (fun s => {u | s ∈ u}) a
[PROOFSTEP]
apply mem_of_superset hv
[GOAL]
case intro.intro.intro.refine'_2
α : Type u
a b : Set α
u : Ultrafilter α
ua : u ∈ (fun s => {u | s ∈ u}) a
ub : u ∈ (fun s => {u | s ∈ u}) b
v : Ultrafilter α
hv : v ∈ (fun s => {u | s ∈ u}) (a ∩ b)
⊢ v ∈ (fun s => {u | s ∈ u}) b
[PROOFSTEP]
apply mem_of_superset hv
[GOAL]
case intro.intro.intro.refine'_1
α : Type u
a b : Set α
u : Ultrafilter α
ua : u ∈ (fun s => {u | s ∈ u}) a
ub : u ∈ (fun s => {u | s ∈ u}) b
v : Ultrafilter α
hv : v ∈ (fun s => {u | s ∈ u}) (a ∩ b)
⊢ a ∩ b ⊆ a
[PROOFSTEP]
simp [inter_subset_right a b]
[GOAL]
case intro.intro.intro.refine'_2
α : Type u
a b : Set α
u : Ultrafilter α
ua : u ∈ (fun s => {u | s ∈ u}) a
ub : u ∈ (fun s => {u | s ∈ u}) b
v : Ultrafilter α
hv : v ∈ (fun s => {u | s ∈ u}) (a ∩ b)
⊢ a ∩ b ⊆ b
[PROOFSTEP]
simp [inter_subset_right a b]
[GOAL]
α : Type u
s : Set α
⊢ IsClosed {u | s ∈ u}
[PROOFSTEP]
rw [← isOpen_compl_iff]
[GOAL]
α : Type u
s : Set α
⊢ IsOpen {u | s ∈ u}ᶜ
[PROOFSTEP]
convert ultrafilter_isOpen_basic sᶜ using 1
[GOAL]
case h.e'_3
α : Type u
s : Set α
⊢ {u | s ∈ u}ᶜ = {u | sᶜ ∈ u}
[PROOFSTEP]
ext u
[GOAL]
case h.e'_3.h
α : Type u
s : Set α
u : Ultrafilter α
⊢ u ∈ {u | s ∈ u}ᶜ ↔ u ∈ {u | sᶜ ∈ u}
[PROOFSTEP]
exact Ultrafilter.compl_mem_iff_not_mem.symm
[GOAL]
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
⊢ ↑u ≤ 𝓝 x ↔ x = joinM u
[PROOFSTEP]
rw [eq_comm, ← Ultrafilter.coe_le_coe]
[GOAL]
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
⊢ ↑u ≤ 𝓝 x ↔ ↑(joinM u) ≤ ↑x
[PROOFSTEP]
change ↑u ≤ 𝓝 x ↔ ∀ s ∈ x, {v : Ultrafilter α | s ∈ v} ∈ u
[GOAL]
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
⊢ ↑u ≤ 𝓝 x ↔ ∀ (s : Set α), s ∈ x → {v | s ∈ v} ∈ u
[PROOFSTEP]
simp only [TopologicalSpace.nhds_generateFrom, le_iInf_iff, ultrafilterBasis, le_principal_iff, mem_setOf_eq]
[GOAL]
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
⊢ (∀ (i : Set (Ultrafilter α)), (x ∈ i ∧ i ∈ range fun s => {u | s ∈ u}) → i ∈ ↑u) ↔
∀ (s : Set α), s ∈ x → {v | s ∈ v} ∈ u
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
⊢ (∀ (i : Set (Ultrafilter α)), (x ∈ i ∧ i ∈ range fun s => {u | s ∈ u}) → i ∈ ↑u) →
∀ (s : Set α), s ∈ x → {v | s ∈ v} ∈ u
[PROOFSTEP]
intro h a ha
[GOAL]
case mp
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
h : ∀ (i : Set (Ultrafilter α)), (x ∈ i ∧ i ∈ range fun s => {u | s ∈ u}) → i ∈ ↑u
a : Set α
ha : a ∈ x
⊢ {v | a ∈ v} ∈ u
[PROOFSTEP]
exact h _ ⟨ha, a, rfl⟩
[GOAL]
case mpr
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
⊢ (∀ (s : Set α), s ∈ x → {v | s ∈ v} ∈ u) →
∀ (i : Set (Ultrafilter α)), (x ∈ i ∧ i ∈ range fun s => {u | s ∈ u}) → i ∈ ↑u
[PROOFSTEP]
rintro h a ⟨xi, a, rfl⟩
[GOAL]
case mpr.intro.intro
α : Type u
u : Ultrafilter (Ultrafilter α)
x : Ultrafilter α
h : ∀ (s : Set α), s ∈ x → {v | s ∈ v} ∈ u
a : Set α
xi : x ∈ (fun s => {u | s ∈ u}) a
⊢ (fun s => {u | s ∈ u}) a ∈ ↑u
[PROOFSTEP]
exact h _ xi
[GOAL]
α : Type u
⊢ TotallyDisconnectedSpace (Ultrafilter α)
[PROOFSTEP]
rw [totallyDisconnectedSpace_iff_connectedComponent_singleton]
[GOAL]
α : Type u
⊢ ∀ (x : Ultrafilter α), connectedComponent x = {x}
[PROOFSTEP]
intro A
[GOAL]
α : Type u
A : Ultrafilter α
⊢ connectedComponent A = {A}
[PROOFSTEP]
simp only [Set.eq_singleton_iff_unique_mem, mem_connectedComponent, true_and_iff]
[GOAL]
α : Type u
A : Ultrafilter α
⊢ ∀ (x : Ultrafilter α), x ∈ connectedComponent A → x = A
[PROOFSTEP]
intro B hB
[GOAL]
α : Type u
A B : Ultrafilter α
hB : B ∈ connectedComponent A
⊢ B = A
[PROOFSTEP]
rw [← Ultrafilter.coe_le_coe]
[GOAL]
α : Type u
A B : Ultrafilter α
hB : B ∈ connectedComponent A
⊢ ↑B ≤ ↑A
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u
A B : Ultrafilter α
hB : B ∈ connectedComponent A
s : Set α
hs : s ∈ ↑A
⊢ s ∈ ↑B
[PROOFSTEP]
rw [connectedComponent_eq_iInter_clopen, Set.mem_iInter] at hB
[GOAL]
α : Type u
A B : Ultrafilter α
hB : ∀ (i : { Z // IsClopen Z ∧ A ∈ Z }), B ∈ ↑i
s : Set α
hs : s ∈ ↑A
⊢ s ∈ ↑B
[PROOFSTEP]
let Z := {F : Ultrafilter α | s ∈ F}
[GOAL]
α : Type u
A B : Ultrafilter α
hB : ∀ (i : { Z // IsClopen Z ∧ A ∈ Z }), B ∈ ↑i
s : Set α
hs : s ∈ ↑A
Z : Set (Ultrafilter α) := {F | s ∈ F}
⊢ s ∈ ↑B
[PROOFSTEP]
have hZ : IsClopen Z := ⟨ultrafilter_isOpen_basic s, ultrafilter_isClosed_basic s⟩
[GOAL]
α : Type u
A B : Ultrafilter α
hB : ∀ (i : { Z // IsClopen Z ∧ A ∈ Z }), B ∈ ↑i
s : Set α
hs : s ∈ ↑A
Z : Set (Ultrafilter α) := {F | s ∈ F}
hZ : IsClopen Z
⊢ s ∈ ↑B
[PROOFSTEP]
exact hB ⟨Z, hZ, hs⟩
[GOAL]
α : Type u
b : Ultrafilter α
⊢ Tendsto pure (↑b) (𝓝 b)
[PROOFSTEP]
rw [Tendsto, ← coe_map, ultrafilter_converges_iff]
[GOAL]
α : Type u
b : Ultrafilter α
⊢ b = joinM (map pure b)
[PROOFSTEP]
ext s
[GOAL]
case h
α : Type u
b : Ultrafilter α
s : Set α
⊢ s ∈ b ↔ s ∈ joinM (map pure b)
[PROOFSTEP]
change s ∈ b ↔ {t | s ∈ t} ∈ map pure b
[GOAL]
case h
α : Type u
b : Ultrafilter α
s : Set α
⊢ s ∈ b ↔ {t | s ∈ t} ∈ map pure b
[PROOFSTEP]
simp_rw [mem_map, preimage_setOf_eq, mem_pure, setOf_mem_eq]
[GOAL]
α : Type u
b : Ultrafilter α
⊢ comap pure (𝓝 b) ≤ ↑b
[PROOFSTEP]
rw [TopologicalSpace.nhds_generateFrom]
[GOAL]
α : Type u
b : Ultrafilter α
⊢ comap pure (⨅ (s : Set (Ultrafilter α)) (_ : s ∈ {s | b ∈ s ∧ s ∈ ultrafilterBasis α}), 𝓟 s) ≤ ↑b
[PROOFSTEP]
simp only [comap_iInf, comap_principal]
[GOAL]
α : Type u
b : Ultrafilter α
⊢ ⨅ (i : Set (Ultrafilter α)) (_ : i ∈ {s | b ∈ s ∧ s ∈ ultrafilterBasis α}), 𝓟 (pure ⁻¹' i) ≤ ↑b
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u
b : Ultrafilter α
s : Set α
hs : s ∈ ↑b
⊢ s ∈ ⨅ (i : Set (Ultrafilter α)) (_ : i ∈ {s | b ∈ s ∧ s ∈ ultrafilterBasis α}), 𝓟 (pure ⁻¹' i)
[PROOFSTEP]
rw [← le_principal_iff]
[GOAL]
α : Type u
b : Ultrafilter α
s : Set α
hs : s ∈ ↑b
⊢ ⨅ (i : Set (Ultrafilter α)) (_ : i ∈ {s | b ∈ s ∧ s ∈ ultrafilterBasis α}), 𝓟 (pure ⁻¹' i) ≤ 𝓟 s
[PROOFSTEP]
refine' iInf_le_of_le {u | s ∈ u} _
[GOAL]
α : Type u
b : Ultrafilter α
s : Set α
hs : s ∈ ↑b
⊢ ⨅ (_ : {u | s ∈ u} ∈ {s | b ∈ s ∧ s ∈ ultrafilterBasis α}), 𝓟 (pure ⁻¹' {u | s ∈ u}) ≤ 𝓟 s
[PROOFSTEP]
refine' iInf_le_of_le ⟨hs, ⟨s, rfl⟩⟩ _
[GOAL]
α : Type u
b : Ultrafilter α
s : Set α
hs : s ∈ ↑b
⊢ 𝓟 (pure ⁻¹' {u | s ∈ u}) ≤ 𝓟 s
[PROOFSTEP]
exact principal_mono.2 fun a => id
[GOAL]
α : Type u
⊢ Function.Injective pure
[PROOFSTEP]
intro x y h
[GOAL]
α : Type u
x y : α
h : pure x = pure y
⊢ x = y
[PROOFSTEP]
have : { x } ∈ (pure x : Ultrafilter α) := singleton_mem_pure
[GOAL]
α : Type u
x y : α
h : pure x = pure y
this : {x} ∈ pure x
⊢ x = y
[PROOFSTEP]
rw [h] at this
[GOAL]
α : Type u
x y : α
h : pure x = pure y
this : {x} ∈ pure y
⊢ x = y
[PROOFSTEP]
exact (mem_singleton_iff.mp (mem_pure.mp this)).symm
[GOAL]
α : Type u
⊢ induced pure Ultrafilter.topologicalSpace = ⊥
[PROOFSTEP]
apply eq_bot_of_singletons_open
[GOAL]
case h
α : Type u
⊢ ∀ (x : α), IsOpen {x}
[PROOFSTEP]
intro x
[GOAL]
case h
α : Type u
x : α
⊢ IsOpen {x}
[PROOFSTEP]
use{u : Ultrafilter α | { x } ∈ u}, ultrafilter_isOpen_basic _
[GOAL]
case right
α : Type u
x : α
⊢ pure ⁻¹' {u | {x} ∈ u} = {x}
[PROOFSTEP]
simp
[GOAL]
α : Type u
γ : Type u_1
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
f : α → γ
⊢ Ultrafilter.extend f ∘ pure = f
[PROOFSTEP]
letI : TopologicalSpace α := ⊥
[GOAL]
α : Type u
γ : Type u_1
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
f : α → γ
this : TopologicalSpace α := ⊥
⊢ Ultrafilter.extend f ∘ pure = f
[PROOFSTEP]
haveI : DiscreteTopology α := ⟨rfl⟩
[GOAL]
α : Type u
γ : Type u_1
inst✝¹ : TopologicalSpace γ
inst✝ : T2Space γ
f : α → γ
this✝ : TopologicalSpace α := ⊥
this : DiscreteTopology α
⊢ Ultrafilter.extend f ∘ pure = f
[PROOFSTEP]
exact funext (denseInducing_pure.extend_eq continuous_of_discreteTopology)
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
⊢ Continuous (Ultrafilter.extend f)
[PROOFSTEP]
have h : ∀ b : Ultrafilter α, ∃ c, Tendsto f (comap pure (𝓝 b)) (𝓝 c) :=
fun b =>
-- b.map f is an ultrafilter on γ, which is compact, so it converges to some c in γ.
let ⟨c, _, h'⟩ := isCompact_univ.ultrafilter_le_nhds (b.map f) (by rw [le_principal_iff]; exact univ_mem)
⟨c, le_trans (map_mono (ultrafilter_comap_pure_nhds _)) h'⟩
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
⊢ ↑(Ultrafilter.map f b) ≤ 𝓟 univ
[PROOFSTEP]
rw [le_principal_iff]
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
⊢ univ ∈ ↑(Ultrafilter.map f b)
[PROOFSTEP]
exact univ_mem
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
h : ∀ (b : Ultrafilter α), ∃ c, Tendsto f (comap pure (𝓝 b)) (𝓝 c)
⊢ Continuous (Ultrafilter.extend f)
[PROOFSTEP]
letI : TopologicalSpace α := ⊥
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
h : ∀ (b : Ultrafilter α), ∃ c, Tendsto f (comap pure (𝓝 b)) (𝓝 c)
this : TopologicalSpace α := ⊥
⊢ Continuous (Ultrafilter.extend f)
[PROOFSTEP]
haveI : NormalSpace γ := normalOfCompactT2
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
h : ∀ (b : Ultrafilter α), ∃ c, Tendsto f (comap pure (𝓝 b)) (𝓝 c)
this✝ : TopologicalSpace α := ⊥
this : NormalSpace γ
⊢ Continuous (Ultrafilter.extend f)
[PROOFSTEP]
exact denseInducing_pure.continuous_extend h
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
⊢ ↑(Ultrafilter.map f b) ≤ 𝓝 c
[PROOFSTEP]
let b' : Ultrafilter (Ultrafilter α) := b.map pure
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
⊢ ↑(Ultrafilter.map f b) ≤ 𝓝 c
[PROOFSTEP]
have t : ↑b' ≤ 𝓝 b := ultrafilter_converges_iff.mpr (bind_pure _).symm
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
t : ↑b' ≤ 𝓝 b
⊢ ↑(Ultrafilter.map f b) ≤ 𝓝 c
[PROOFSTEP]
rw [← h]
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
t : ↑b' ≤ 𝓝 b
⊢ ↑(Ultrafilter.map f b) ≤ 𝓝 (Ultrafilter.extend f b)
[PROOFSTEP]
have := (continuous_ultrafilter_extend f).tendsto b
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
t : ↑b' ≤ 𝓝 b
this : Tendsto (Ultrafilter.extend f) (𝓝 b) (𝓝 (Ultrafilter.extend f b))
⊢ ↑(Ultrafilter.map f b) ≤ 𝓝 (Ultrafilter.extend f b)
[PROOFSTEP]
refine' le_trans _ (le_trans (map_mono t) this)
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
t : ↑b' ≤ 𝓝 b
this : Tendsto (Ultrafilter.extend f) (𝓝 b) (𝓝 (Ultrafilter.extend f b))
⊢ ↑(Ultrafilter.map f b) ≤ map (Ultrafilter.extend f) ↑b'
[PROOFSTEP]
change _ ≤ map (Ultrafilter.extend f ∘ pure) ↑b
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
t : ↑b' ≤ 𝓝 b
this : Tendsto (Ultrafilter.extend f) (𝓝 b) (𝓝 (Ultrafilter.extend f b))
⊢ ↑(Ultrafilter.map f b) ≤ map (Ultrafilter.extend f ∘ pure) ↑b
[PROOFSTEP]
rw [ultrafilter_extend_extends]
[GOAL]
α : Type u
γ : Type u_1
inst✝² : TopologicalSpace γ
inst✝¹ : T2Space γ
inst✝ : CompactSpace γ
f : α → γ
b : Ultrafilter α
c : γ
h : Ultrafilter.extend f b = c
b' : Ultrafilter (Ultrafilter α) := Ultrafilter.map pure b
t : ↑b' ≤ 𝓝 b
this : Tendsto (Ultrafilter.extend f) (𝓝 b) (𝓝 (Ultrafilter.extend f b))
⊢ ↑(Ultrafilter.map f b) ≤ map f ↑b
[PROOFSTEP]
exact le_rfl
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
⊢ TopologicalSpace (StoneCech α)
[PROOFSTEP]
unfold StoneCech
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
⊢ TopologicalSpace (Quotient (stoneCechSetoid α))
[PROOFSTEP]
infer_instance
[GOAL]
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : Inhabited α
⊢ Inhabited (StoneCech α)
[PROOFSTEP]
unfold StoneCech
[GOAL]
α : Type u
inst✝¹ : TopologicalSpace α
inst✝ : Inhabited α
⊢ Inhabited (Quotient (stoneCechSetoid α))
[PROOFSTEP]
infer_instance
[GOAL]
α : Type u
inst✝⁵ : TopologicalSpace α
γ : Type u
inst✝⁴ : TopologicalSpace γ
inst✝³ : T2Space γ
inst✝² : CompactSpace γ
γ' : Type u
inst✝¹ : TopologicalSpace γ'
inst✝ : T2Space γ'
f : α → γ
hf : Continuous f
g₁ g₂ : StoneCech α → γ'
h₁ : Continuous g₁
h₂ : Continuous g₂
h : g₁ ∘ stoneCechUnit = g₂ ∘ stoneCechUnit
⊢ g₁ = g₂
[PROOFSTEP]
apply Continuous.ext_on denseRange_stoneCechUnit h₁ h₂
[GOAL]
α : Type u
inst✝⁵ : TopologicalSpace α
γ : Type u
inst✝⁴ : TopologicalSpace γ
inst✝³ : T2Space γ
inst✝² : CompactSpace γ
γ' : Type u
inst✝¹ : TopologicalSpace γ'
inst✝ : T2Space γ'
f : α → γ
hf : Continuous f
g₁ g₂ : StoneCech α → γ'
h₁ : Continuous g₁
h₂ : Continuous g₂
h : g₁ ∘ stoneCechUnit = g₂ ∘ stoneCechUnit
⊢ EqOn g₁ g₂ (range stoneCechUnit)
[PROOFSTEP]
rintro x ⟨x, rfl⟩
[GOAL]
case intro
α : Type u
inst✝⁵ : TopologicalSpace α
γ : Type u
inst✝⁴ : TopologicalSpace γ
inst✝³ : T2Space γ
inst✝² : CompactSpace γ
γ' : Type u
inst✝¹ : TopologicalSpace γ'
inst✝ : T2Space γ'
f : α → γ
hf : Continuous f
g₁ g₂ : StoneCech α → γ'
h₁ : Continuous g₁
h₂ : Continuous g₂
h : g₁ ∘ stoneCechUnit = g₂ ∘ stoneCechUnit
x : α
⊢ g₁ (stoneCechUnit x) = g₂ (stoneCechUnit x)
[PROOFSTEP]
apply congr_fun h x
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f u = Ultrafilter.extend f (pure x)
[PROOFSTEP]
skip
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f u = Ultrafilter.extend f (pure x)
[PROOFSTEP]
trans f x
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f u = f x
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ f x = Ultrafilter.extend f (pure x)
[PROOFSTEP]
swap
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ f x = Ultrafilter.extend f (pure x)
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f u = f x
[PROOFSTEP]
symm
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f (pure x) = f x
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f u = f x
[PROOFSTEP]
all_goals refine' ultrafilter_extend_eq_iff.mpr (le_trans (map_mono _) (hf.tendsto _))
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f (pure x) = f x
[PROOFSTEP]
refine' ultrafilter_extend_eq_iff.mpr (le_trans (map_mono _) (hf.tendsto _))
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f u = f x
[PROOFSTEP]
refine' ultrafilter_extend_eq_iff.mpr (le_trans (map_mono _) (hf.tendsto _))
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ ↑(pure x) ≤ 𝓝 x
[PROOFSTEP]
apply pure_le_nhds
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
u : Ultrafilter α
x : α
ux : ↑u ≤ 𝓝 x
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ ↑u ≤ 𝓝 x
[PROOFSTEP]
exact ux
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
x : α
g : Ultrafilter α
gx : ↑g ≤ 𝓝 x
⊢ Tendsto stoneCechUnit (↑g) (𝓝 (stoneCechUnit x))
[PROOFSTEP]
have : (g.map pure).toFilter ≤ 𝓝 g := by
rw [ultrafilter_converges_iff]
exact (bind_pure _).symm
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
x : α
g : Ultrafilter α
gx : ↑g ≤ 𝓝 x
⊢ ↑(Ultrafilter.map pure g) ≤ 𝓝 g
[PROOFSTEP]
rw [ultrafilter_converges_iff]
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
x : α
g : Ultrafilter α
gx : ↑g ≤ 𝓝 x
⊢ g = joinM (Ultrafilter.map pure g)
[PROOFSTEP]
exact (bind_pure _).symm
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
x : α
g : Ultrafilter α
gx : ↑g ≤ 𝓝 x
this : ↑(Ultrafilter.map pure g) ≤ 𝓝 g
⊢ Tendsto stoneCechUnit (↑g) (𝓝 (stoneCechUnit x))
[PROOFSTEP]
have : (g.map stoneCechUnit : Filter (StoneCech α)) ≤ 𝓝 ⟦g⟧ :=
continuousAt_iff_ultrafilter.mp (continuous_quotient_mk'.tendsto g) _ this
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
x : α
g : Ultrafilter α
gx : ↑g ≤ 𝓝 x
this✝ : ↑(Ultrafilter.map pure g) ≤ 𝓝 g
this : ↑(Ultrafilter.map stoneCechUnit g) ≤ 𝓝 (Quotient.mk (stoneCechSetoid α) g)
⊢ Tendsto stoneCechUnit (↑g) (𝓝 (stoneCechUnit x))
[PROOFSTEP]
rwa [show ⟦g⟧ = ⟦pure x⟧ from Quotient.sound <| convergent_eqv_pure gx] at this
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
⊢ T2Space (StoneCech α)
[PROOFSTEP]
rw [t2_iff_ultrafilter]
[GOAL]
α : Type u
inst✝ : TopologicalSpace α
⊢ ∀ {x y : StoneCech α} (f : Ultrafilter (StoneCech α)), ↑f ≤ 𝓝 x → ↑f ≤ 𝓝 y → x = y
[PROOFSTEP]
rintro ⟨x⟩ ⟨y⟩ g gx gy
[GOAL]
case mk.mk
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
⊢ Quot.mk Setoid.r x = Quot.mk Setoid.r y
[PROOFSTEP]
apply Quotient.sound
[GOAL]
case mk.mk.a
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
⊢ x ≈ y
[PROOFSTEP]
intro γ tγ h₁ h₂ f hf
[GOAL]
case mk.mk.a
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f x = Ultrafilter.extend f y
[PROOFSTEP]
skip
[GOAL]
case mk.mk.a
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
⊢ Ultrafilter.extend f x = Ultrafilter.extend f y
[PROOFSTEP]
let ff := stoneCechExtend hf
[GOAL]
case mk.mk.a
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
ff : StoneCech α → γ := stoneCechExtend hf
⊢ Ultrafilter.extend f x = Ultrafilter.extend f y
[PROOFSTEP]
change ff ⟦x⟧ = ff ⟦y⟧
[GOAL]
case mk.mk.a
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
ff : StoneCech α → γ := stoneCechExtend hf
⊢ ff (Quotient.mk (stoneCechSetoid α) x) = ff (Quotient.mk (stoneCechSetoid α) y)
[PROOFSTEP]
have lim := fun (z : Ultrafilter α) (gz : (g : Filter (StoneCech α)) ≤ 𝓝 ⟦z⟧) =>
((continuous_stoneCechExtend hf).tendsto _).mono_left gz
[GOAL]
case mk.mk.a
α : Type u
inst✝ : TopologicalSpace α
x✝ : StoneCech α
x : Ultrafilter α
y✝ : StoneCech α
y : Ultrafilter α
g : Ultrafilter (StoneCech α)
gx : ↑g ≤ 𝓝 (Quot.mk Setoid.r x)
gy : ↑g ≤ 𝓝 (Quot.mk Setoid.r y)
γ : Type u
tγ : TopologicalSpace γ
h₁ : T2Space γ
h₂ : CompactSpace γ
f : α → γ
hf : Continuous f
ff : StoneCech α → γ := stoneCechExtend hf
lim :
∀ (z : Ultrafilter α),
↑g ≤ 𝓝 (Quotient.mk (stoneCechSetoid α) z) →
Tendsto (stoneCechExtend hf) (↑g) (𝓝 (stoneCechExtend hf (Quotient.mk (stoneCechSetoid α) z)))
⊢ ff (Quotient.mk (stoneCechSetoid α) x) = ff (Quotient.mk (stoneCechSetoid α) y)
[PROOFSTEP]
exact tendsto_nhds_unique (lim x gx) (lim y gy)
| {"mathlib_filename": "Mathlib.Topology.StoneCech", "llama_tokens": 11109} |
{"mathlib_filename": "Mathlib.Topology.Tactic", "llama_tokens": 0} |
|
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
hα : DiscreteTopology α
hβ : DiscreteTopology β
⊢ coinduced inl inst✝¹ = ⊥ ∧ coinduced inr inst✝ = ⊥
[PROOFSTEP]
simp [hα.eq_bot, hβ.eq_bot]
[GOAL]
α : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
β : α → Type v
inst✝ : (a : α) → TopologicalSpace (β a)
h : ∀ (a : α), DiscreteTopology (β a)
x✝ : α
⊢ coinduced (mk x✝) ((fun a => inst✝ a) x✝) = ⊥
[PROOFSTEP]
simp only [(h _).eq_bot, coinduced_bot]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
s t : Set α
x : ↑s
⊢ 𝓝[Subtype.val ⁻¹' t] x = ⊥ ↔ 𝓝[t] ↑x ⊓ 𝓟 s = ⊥
[PROOFSTEP]
rw [inf_principal_eq_bot_iff_comap, nhdsWithin, nhdsWithin, comap_inf, comap_principal, nhds_induced]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
S : Set α
x : ↑S
⊢ 𝓝[{x}ᶜ] x = ⊥ ↔ 𝓝[{↑x}ᶜ] ↑x ⊓ 𝓟 S = ⊥
[PROOFSTEP]
rw [← nhdsWithin_subtype_eq_bot_iff, preimage_compl, ← image_singleton, Subtype.coe_injective.preimage_image]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
S : Set α
x : ↑S
⊢ NeBot (𝓝[{x}ᶜ] x) ↔ NeBot (𝓝[{↑x}ᶜ] ↑x ⊓ 𝓟 S)
[PROOFSTEP]
rw [neBot_iff, neBot_iff, not_iff_not, nhds_ne_subtype_eq_bot_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
S : Set α
⊢ DiscreteTopology ↑S ↔ ∀ (x : α), x ∈ S → 𝓝[{x}ᶜ] x ⊓ 𝓟 S = ⊥
[PROOFSTEP]
simp_rw [discreteTopology_iff_nhds_ne, SetCoe.forall', nhds_ne_subtype_eq_bot_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
⊢ (fun s => Set.Nonempty s → Set.Finite sᶜ) univ
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s t : Set (CofiniteTopology α)
⊢ (fun s => Set.Nonempty s → Set.Finite sᶜ) s →
(fun s => Set.Nonempty s → Set.Finite sᶜ) t → (fun s => Set.Nonempty s → Set.Finite sᶜ) (s ∩ t)
[PROOFSTEP]
rintro hs ht ⟨x, hxs, hxt⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s t : Set (CofiniteTopology α)
hs : Set.Nonempty s → Set.Finite sᶜ
ht : Set.Nonempty t → Set.Finite tᶜ
x : CofiniteTopology α
hxs : x ∈ s
hxt : x ∈ t
⊢ Set.Finite (s ∩ t)ᶜ
[PROOFSTEP]
rw [compl_inter]
[GOAL]
case intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s t : Set (CofiniteTopology α)
hs : Set.Nonempty s → Set.Finite sᶜ
ht : Set.Nonempty t → Set.Finite tᶜ
x : CofiniteTopology α
hxs : x ∈ s
hxt : x ∈ t
⊢ Set.Finite (sᶜ ∪ tᶜ)
[PROOFSTEP]
exact (hs ⟨x, hxs⟩).union (ht ⟨x, hxt⟩)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
⊢ ∀ (s : Set (Set (CofiniteTopology α))),
(∀ (t : Set (CofiniteTopology α)), t ∈ s → (fun s => Set.Nonempty s → Set.Finite sᶜ) t) →
(fun s => Set.Nonempty s → Set.Finite sᶜ) (⋃₀ s)
[PROOFSTEP]
rintro s h ⟨x, t, hts, hzt⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s : Set (Set (CofiniteTopology α))
h : ∀ (t : Set (CofiniteTopology α)), t ∈ s → (fun s => Set.Nonempty s → Set.Finite sᶜ) t
x : CofiniteTopology α
t : Set (CofiniteTopology α)
hts : t ∈ s
hzt : x ∈ t
⊢ Set.Finite (⋃₀ s)ᶜ
[PROOFSTEP]
rw [Set.compl_sUnion]
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s : Set (Set (CofiniteTopology α))
h : ∀ (t : Set (CofiniteTopology α)), t ∈ s → (fun s => Set.Nonempty s → Set.Finite sᶜ) t
x : CofiniteTopology α
t : Set (CofiniteTopology α)
hts : t ∈ s
hzt : x ∈ t
⊢ Set.Finite (⋂₀ (compl '' s))
[PROOFSTEP]
exact Set.Finite.sInter (mem_image_of_mem _ hts) (h t hts ⟨x, hzt⟩)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s : Set (CofiniteTopology α)
⊢ IsOpen s ↔ s = ∅ ∨ Set.Finite sᶜ
[PROOFSTEP]
simp only [isOpen_iff, nonempty_iff_ne_empty, or_iff_not_imp_left]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
s : Set (CofiniteTopology α)
⊢ IsClosed s ↔ s = univ ∨ Set.Finite s
[PROOFSTEP]
simp only [← isOpen_compl_iff, isOpen_iff', compl_compl, compl_empty_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
⊢ 𝓝 a = pure a ⊔ cofinite
[PROOFSTEP]
ext U
[GOAL]
case a
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
U : Set (CofiniteTopology α)
⊢ U ∈ 𝓝 a ↔ U ∈ pure a ⊔ cofinite
[PROOFSTEP]
rw [mem_nhds_iff]
[GOAL]
case a
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
U : Set (CofiniteTopology α)
⊢ (∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t) ↔ U ∈ pure a ⊔ cofinite
[PROOFSTEP]
constructor
[GOAL]
case a.mp
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
U : Set (CofiniteTopology α)
⊢ (∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t) → U ∈ pure a ⊔ cofinite
[PROOFSTEP]
rintro ⟨V, hVU, V_op, haV⟩
[GOAL]
case a.mp.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
U V : Set (CofiniteTopology α)
hVU : V ⊆ U
V_op : IsOpen V
haV : a ∈ V
⊢ U ∈ pure a ⊔ cofinite
[PROOFSTEP]
exact mem_sup.mpr ⟨hVU haV, mem_of_superset (V_op ⟨_, haV⟩) hVU⟩
[GOAL]
case a.mpr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
U : Set (CofiniteTopology α)
⊢ U ∈ pure a ⊔ cofinite → ∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t
[PROOFSTEP]
rintro ⟨hU : a ∈ U, hU' : Uᶜ.Finite⟩
[GOAL]
case a.mpr.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
U : Set (CofiniteTopology α)
hU : a ∈ U
hU' : Set.Finite Uᶜ
⊢ ∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t
[PROOFSTEP]
exact ⟨U, Subset.rfl, fun _ => hU', hU⟩
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
a : CofiniteTopology α
s : Set (CofiniteTopology α)
⊢ s ∈ 𝓝 a ↔ a ∈ s ∧ Set.Finite sᶜ
[PROOFSTEP]
simp [nhds_eq]
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.27593
β : Type ?u.27599
γ : Type ?u.27605
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
⊢ Sort ?u.27607
[PROOFSTEP]
haveI := ta1
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.27593
β : Type ?u.27599
γ : Type ?u.27605
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
this : TopologicalSpace α
⊢ Sort ?u.27607
[PROOFSTEP]
haveI := tb1
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.27593
β : Type ?u.27599
γ : Type ?u.27605
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
this✝ : TopologicalSpace α
this : TopologicalSpace β
⊢ Sort ?u.27607
[PROOFSTEP]
exact Continuous fun p : α × β => f p.1 p.2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.27593
β : Type ?u.27599
γ : Type ?u.27605
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
⊢ Sort ?u.27610
[PROOFSTEP]
haveI := ta1 ⊓ ta2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.27593
β : Type ?u.27599
γ : Type ?u.27605
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
this : TopologicalSpace α
⊢ Sort ?u.27610
[PROOFSTEP]
haveI := tb1 ⊓ tb2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.27593
β : Type ?u.27599
γ : Type ?u.27605
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
this✝ : TopologicalSpace α
this : TopologicalSpace β
⊢ Sort ?u.27610
[PROOFSTEP]
exact Continuous fun p : α × β => f p.1 p.2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have ha := @continuous_inf_dom_left _ _ id ta1 ta2 ta1 (@continuous_id _ (id _))
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
ha : Continuous id
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have hb := @continuous_inf_dom_left _ _ id tb1 tb2 tb1 (@continuous_id _ (id _))
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
ha : Continuous id
hb : Continuous id
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have h_continuous_id := @Continuous.prod_map _ _ _ _ ta1 tb1 (ta1 ⊓ ta2) (tb1 ⊓ tb2) _ _ ha hb
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
ha : Continuous id
hb : Continuous id
h_continuous_id : Continuous fun x => (id x.fst, id x.snd)
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
exact @Continuous.comp _ _ _ (id _) (id _) _ _ _ h h_continuous_id
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28286
β : Type ?u.28292
γ : Type ?u.28298
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
⊢ Sort ?u.28300
[PROOFSTEP]
haveI := ta2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28286
β : Type ?u.28292
γ : Type ?u.28298
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
this : TopologicalSpace α
⊢ Sort ?u.28300
[PROOFSTEP]
haveI := tb2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28286
β : Type ?u.28292
γ : Type ?u.28298
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
this✝ : TopologicalSpace α
this : TopologicalSpace β
⊢ Sort ?u.28300
[PROOFSTEP]
exact Continuous fun p : α × β => f p.1 p.2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28286
β : Type ?u.28292
γ : Type ?u.28298
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
⊢ Sort ?u.28303
[PROOFSTEP]
haveI := ta1 ⊓ ta2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28286
β : Type ?u.28292
γ : Type ?u.28298
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
this : TopologicalSpace α
⊢ Sort ?u.28303
[PROOFSTEP]
haveI := tb1 ⊓ tb2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28286
β : Type ?u.28292
γ : Type ?u.28298
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
this✝ : TopologicalSpace α
this : TopologicalSpace β
⊢ Sort ?u.28303
[PROOFSTEP]
exact Continuous fun p : α × β => f p.1 p.2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have ha := @continuous_inf_dom_right _ _ id ta1 ta2 ta2 (@continuous_id _ (id _))
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
ha : Continuous id
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have hb := @continuous_inf_dom_right _ _ id tb1 tb2 tb2 (@continuous_id _ (id _))
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
ha : Continuous id
hb : Continuous id
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have h_continuous_id := @Continuous.prod_map _ _ _ _ ta2 tb2 (ta1 ⊓ ta2) (tb1 ⊓ tb2) _ _ ha hb
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
ta1 ta2 : TopologicalSpace α
tb1 tb2 : TopologicalSpace β
tc1 : TopologicalSpace γ
h : Continuous fun p => f p.fst p.snd
ha : Continuous id
hb : Continuous id
h_continuous_id : Continuous fun x => (id x.fst, id x.snd)
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
exact @Continuous.comp _ _ _ (id _) (id _) _ _ _ h h_continuous_id
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28980
β : Type ?u.28984
γ : Type ?u.28993
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha : ta ∈ tas
hb : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
⊢ Sort ?u.29158
[PROOFSTEP]
haveI := sInf tas
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28980
β : Type ?u.28984
γ : Type ?u.28993
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha : ta ∈ tas
hb : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
this : TopologicalSpace α
⊢ Sort ?u.29158
[PROOFSTEP]
haveI := sInf tbs
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type ?u.28980
β : Type ?u.28984
γ : Type ?u.28993
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha : ta ∈ tas
hb : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
this✝ : TopologicalSpace α
this : TopologicalSpace β
⊢ Sort ?u.29158
[PROOFSTEP]
exact @Continuous _ _ _ tc fun p : α × β => f p.1 p.2
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha : ta ∈ tas
hb : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have ha := continuous_sInf_dom ha continuous_id
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha✝ : ta ∈ tas
hb : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
ha : Continuous id
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have hb := continuous_sInf_dom hb continuous_id
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha✝ : ta ∈ tas
hb✝ : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
ha : Continuous id
hb : Continuous id
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
have h_continuous_id := @Continuous.prod_map _ _ _ _ ta tb (sInf tas) (sInf tbs) _ _ ha hb
[GOAL]
α✝ : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
γ : Type u_7
f : α → β → γ
tas : Set (TopologicalSpace α)
tbs : Set (TopologicalSpace β)
ta : TopologicalSpace α
tb : TopologicalSpace β
tc : TopologicalSpace γ
ha✝ : ta ∈ tas
hb✝ : tb ∈ tbs
hf : Continuous fun p => f p.fst p.snd
ha : Continuous id
hb : Continuous id
h_continuous_id : Continuous fun x => (id x.fst, id x.snd)
⊢ Continuous fun p => f p.fst p.snd
[PROOFSTEP]
exact @Continuous.comp _ _ _ (id _) (id _) _ _ _ hf h_continuous_id
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
⊢ 𝓝 (a, b) = 𝓝 a ×ˢ 𝓝 b
[PROOFSTEP]
dsimp only [SProd.sprod]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
⊢ 𝓝 (a, b) = Filter.prod (𝓝 a) (𝓝 b)
[PROOFSTEP]
rw [Filter.prod, instTopologicalSpaceProd,
nhds_inf (t₁ := TopologicalSpace.induced Prod.fst _) (t₂ := TopologicalSpace.induced Prod.snd _), nhds_induced,
nhds_induced]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
s : Set α
t : Set β
⊢ 𝓝[s ×ˢ t] (a, b) = 𝓝[s] a ×ˢ 𝓝[t] b
[PROOFSTEP]
simp only [nhdsWithin, nhds_prod_eq, ← prod_inf_prod, prod_principal_principal]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
inst✝² : TopologicalSpace ε
inst✝¹ : TopologicalSpace ζ
inst✝ : DiscreteTopology α
f : α → β → γ
hf : ∀ (a : α), Continuous (f a)
⊢ Continuous (uncurry f)
[PROOFSTEP]
apply continuous_iff_continuousAt.2
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
inst✝² : TopologicalSpace ε
inst✝¹ : TopologicalSpace ζ
inst✝ : DiscreteTopology α
f : α → β → γ
hf : ∀ (a : α), Continuous (f a)
⊢ ∀ (x : α × β), ContinuousAt (uncurry f) x
[PROOFSTEP]
rintro ⟨a, x⟩
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
inst✝² : TopologicalSpace ε
inst✝¹ : TopologicalSpace ζ
inst✝ : DiscreteTopology α
f : α → β → γ
hf : ∀ (a : α), Continuous (f a)
a : α
x : β
⊢ ContinuousAt (uncurry f) (a, x)
[PROOFSTEP]
change map _ _ ≤ _
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
inst✝² : TopologicalSpace ε
inst✝¹ : TopologicalSpace ζ
inst✝ : DiscreteTopology α
f : α → β → γ
hf : ∀ (a : α), Continuous (f a)
a : α
x : β
⊢ map (uncurry f) (𝓝 (a, x)) ≤ 𝓝 (uncurry f (a, x))
[PROOFSTEP]
rw [nhds_prod_eq, nhds_discrete, Filter.map_pure_prod]
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
inst✝² : TopologicalSpace ε
inst✝¹ : TopologicalSpace ζ
inst✝ : DiscreteTopology α
f : α → β → γ
hf : ∀ (a : α), Continuous (f a)
a : α
x : β
⊢ map (f a) (𝓝 x) ≤ 𝓝 (uncurry f (a, x))
[PROOFSTEP]
exact (hf a).continuousAt
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
s : Set (α × β)
⊢ s ∈ 𝓝 (a, b) ↔ ∃ u, u ∈ 𝓝 a ∧ ∃ v, v ∈ 𝓝 b ∧ u ×ˢ v ⊆ s
[PROOFSTEP]
rw [nhds_prod_eq, mem_prod_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
ιa : Type u_5
ιb : Type u_6
pa : ιa → Prop
pb : ιb → Prop
sa : ιa → Set α
sb : ιb → Set β
a : α
b : β
ha : HasBasis (𝓝 a) pa sa
hb : HasBasis (𝓝 b) pb sb
⊢ HasBasis (𝓝 (a, b)) (fun i => pa i.fst ∧ pb i.snd) fun i => sa i.fst ×ˢ sb i.snd
[PROOFSTEP]
rw [nhds_prod_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
ιa : Type u_5
ιb : Type u_6
pa : ιa → Prop
pb : ιb → Prop
sa : ιa → Set α
sb : ιb → Set β
a : α
b : β
ha : HasBasis (𝓝 a) pa sa
hb : HasBasis (𝓝 b) pb sb
⊢ HasBasis (𝓝 a ×ˢ 𝓝 b) (fun i => pa i.fst ∧ pb i.snd) fun i => sa i.fst ×ˢ sb i.snd
[PROOFSTEP]
exact ha.prod hb
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
s : Set (α × β)
⊢ (∃ i, ((a ∈ i.fst ∧ IsOpen i.fst) ∧ b ∈ i.snd ∧ IsOpen i.snd) ∧ i.fst ×ˢ i.snd ⊆ s) ↔
∃ u v, IsOpen u ∧ a ∈ u ∧ IsOpen v ∧ b ∈ v ∧ u ×ˢ v ⊆ s
[PROOFSTEP]
simp only [Prod.exists, and_comm, and_assoc, and_left_comm]
[GOAL]
α✝ : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
seq : α → β × γ
f : Filter α
x : β × γ
⊢ Tendsto seq f (𝓝 x) ↔ Tendsto (fun n => (seq n).fst) f (𝓝 x.fst) ∧ Tendsto (fun n => (seq n).snd) f (𝓝 x.snd)
[PROOFSTEP]
rw [nhds_prod_eq, Filter.tendsto_prod_iff']
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁷ : TopologicalSpace α
inst✝⁶ : TopologicalSpace β
inst✝⁵ : TopologicalSpace γ
inst✝⁴ : TopologicalSpace δ
inst✝³ : TopologicalSpace ε
inst✝² : TopologicalSpace ζ
inst✝¹ : DiscreteTopology α
inst✝ : DiscreteTopology β
x✝ : α × β
a : α
b : β
⊢ 𝓝 (a, b) = pure (a, b)
[PROOFSTEP]
rw [nhds_prod_eq, nhds_discrete α, nhds_discrete β, prod_pure_pure]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
a : α
b : β
⊢ s ×ˢ t ∈ 𝓝 (a, b) ↔ s ∈ 𝓝 a ∧ t ∈ 𝓝 b
[PROOFSTEP]
rw [nhds_prod_eq, prod_mem_prod_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
⊢ 𝓝 (a, b) = map Prod.swap (𝓝 (b, a))
[PROOFSTEP]
rw [nhds_prod_eq, Filter.prod_comm, nhds_prod_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
b : β
⊢ map (fun p => (p.snd, p.fst)) (𝓝 b ×ˢ 𝓝 a) = map Prod.swap (𝓝 b ×ˢ 𝓝 a)
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
γ : Type u_5
a : α
b : β
f : Filter γ
ma : γ → α
mb : γ → β
ha : Tendsto ma f (𝓝 a)
hb : Tendsto mb f (𝓝 b)
⊢ Tendsto (fun c => (ma c, mb c)) f (𝓝 (a, b))
[PROOFSTEP]
rw [nhds_prod_eq]
[GOAL]
α : Type u
β : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ✝
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
γ : Type u_5
a : α
b : β
f : Filter γ
ma : γ → α
mb : γ → β
ha : Tendsto ma f (𝓝 a)
hb : Tendsto mb f (𝓝 b)
⊢ Tendsto (fun c => (ma c, mb c)) f (𝓝 a ×ˢ 𝓝 b)
[PROOFSTEP]
exact Filter.Tendsto.prod_mk ha hb
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
p : α × β → Prop
x : α
y : β
h : ∀ᶠ (x : α × β) in 𝓝 (x, y), p x
⊢ ∀ᶠ (x' : α) in 𝓝 x, ∀ᶠ (y' : β) in 𝓝 y, p (x', y')
[PROOFSTEP]
rw [nhds_prod_eq] at h
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
p : α × β → Prop
x : α
y : β
h : ∀ᶠ (x : α × β) in 𝓝 x ×ˢ 𝓝 y, p x
⊢ ∀ᶠ (x' : α) in 𝓝 x, ∀ᶠ (y' : β) in 𝓝 y, p (x', y')
[PROOFSTEP]
exact h.curry
[GOAL]
α✝ : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
s : Set (Set α)
t : Set (Set β)
hs : ⋃₀ s = univ
ht : ⋃₀ t = univ
G : TopologicalSpace (α × β) := generateFrom {g | ∃ u, u ∈ s ∧ ∃ v, v ∈ t ∧ g = u ×ˢ v}
u : Set α
hu : u ∈ s
⊢ ⋃ (v : Set β) (_ : v ∈ t), u ×ˢ v = Prod.fst ⁻¹' u
[PROOFSTEP]
simp_rw [← prod_iUnion, ← sUnion_eq_biUnion, ht, prod_univ]
[GOAL]
α✝ : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
s : Set (Set α)
t : Set (Set β)
hs : ⋃₀ s = univ
ht : ⋃₀ t = univ
G : TopologicalSpace (α × β) := generateFrom {g | ∃ u, u ∈ s ∧ ∃ v, v ∈ t ∧ g = u ×ˢ v}
u : Set α
hu : u ∈ s
this : ⋃ (v : Set β) (_ : v ∈ t), u ×ˢ v = Prod.fst ⁻¹' u
⊢ TopologicalSpace.IsOpen (Prod.fst ⁻¹' u)
[PROOFSTEP]
rw [← this]
[GOAL]
α✝ : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
s : Set (Set α)
t : Set (Set β)
hs : ⋃₀ s = univ
ht : ⋃₀ t = univ
G : TopologicalSpace (α × β) := generateFrom {g | ∃ u, u ∈ s ∧ ∃ v, v ∈ t ∧ g = u ×ˢ v}
u : Set α
hu : u ∈ s
this : ⋃ (v : Set β) (_ : v ∈ t), u ×ˢ v = Prod.fst ⁻¹' u
⊢ TopologicalSpace.IsOpen (⋃ (v : Set β) (_ : v ∈ t), u ×ˢ v)
[PROOFSTEP]
exact isOpen_iUnion fun v => isOpen_iUnion fun hv => GenerateOpen.basic _ ⟨_, hu, _, hv, rfl⟩
[GOAL]
α✝ : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
s : Set (Set α)
t : Set (Set β)
hs : ⋃₀ s = univ
ht : ⋃₀ t = univ
G : TopologicalSpace (α × β) := generateFrom {g | ∃ u, u ∈ s ∧ ∃ v, v ∈ t ∧ g = u ×ˢ v}
v : Set β
hv : v ∈ t
⊢ ⋃ (u : Set α) (_ : u ∈ s), u ×ˢ v = Prod.snd ⁻¹' v
[PROOFSTEP]
simp_rw [← iUnion_prod_const, ← sUnion_eq_biUnion, hs, univ_prod]
[GOAL]
α✝ : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
s : Set (Set α)
t : Set (Set β)
hs : ⋃₀ s = univ
ht : ⋃₀ t = univ
G : TopologicalSpace (α × β) := generateFrom {g | ∃ u, u ∈ s ∧ ∃ v, v ∈ t ∧ g = u ×ˢ v}
v : Set β
hv : v ∈ t
this : ⋃ (u : Set α) (_ : u ∈ s), u ×ˢ v = Prod.snd ⁻¹' v
⊢ TopologicalSpace.IsOpen (Prod.snd ⁻¹' v)
[PROOFSTEP]
rw [← this]
[GOAL]
α✝ : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α✝
inst✝⁴ : TopologicalSpace β✝
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
α : Type u_5
β : Type u_6
s : Set (Set α)
t : Set (Set β)
hs : ⋃₀ s = univ
ht : ⋃₀ t = univ
G : TopologicalSpace (α × β) := generateFrom {g | ∃ u, u ∈ s ∧ ∃ v, v ∈ t ∧ g = u ×ˢ v}
v : Set β
hv : v ∈ t
this : ⋃ (u : Set α) (_ : u ∈ s), u ×ˢ v = Prod.snd ⁻¹' v
⊢ TopologicalSpace.IsOpen (⋃ (u : Set α) (_ : u ∈ s), u ×ˢ v)
[PROOFSTEP]
exact isOpen_iUnion fun u => isOpen_iUnion fun hu => GenerateOpen.basic _ ⟨_, hu, _, hv, rfl⟩
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
t : Set α
ht : t ∈ fun s' => inst✝⁵.1 s'
⊢ IsOpen t ∧ IsOpen univ ∧ Prod.fst ⁻¹' t = t ×ˢ univ
[PROOFSTEP]
simpa [Set.prod_eq] using ht
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
t : Set β
ht : t ∈ fun s' => inst✝⁴.1 s'
⊢ IsOpen univ ∧ IsOpen t ∧ Prod.snd ⁻¹' t = univ ×ˢ t
[PROOFSTEP]
simpa [Set.prod_eq] using ht
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set (α × β)
⊢ (∀ (a : α × β), a ∈ s → s ∈ 𝓝 a) ↔
∀ (a : α) (b : β), (a, b) ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ a ∈ u ∧ b ∈ v ∧ u ×ˢ v ⊆ s
[PROOFSTEP]
simp_rw [Prod.forall, mem_nhds_prod_iff', and_left_comm]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
⊢ instTopologicalSpaceProd = induced (fun p => (f p.fst, g p.snd)) instTopologicalSpaceProd
[PROOFSTEP]
delta instTopologicalSpaceProd
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
⊢ induced Prod.fst (induced f inst✝⁴) ⊓ induced Prod.snd (induced g inst✝²) =
induced (fun p => (f p.fst, g p.snd)) (induced Prod.fst inst✝⁴ ⊓ induced Prod.snd inst✝²)
[PROOFSTEP]
simp_rw [induced_inf, induced_compose]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
⊢ induced (f ∘ Prod.fst) inst✝⁴ ⊓ induced (g ∘ Prod.snd) inst✝² =
induced (Prod.fst ∘ fun p => (f p.fst, g p.snd)) inst✝⁴ ⊓ induced (Prod.snd ∘ fun p => (f p.fst, g p.snd)) inst✝²
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁶ : TopologicalSpace α
inst✝⁵ : TopologicalSpace β
inst✝⁴ : TopologicalSpace γ
inst✝³ : TopologicalSpace δ
inst✝² : TopologicalSpace ε
inst✝¹ : TopologicalSpace ζ
inst✝ : DiscreteTopology α
f : α → β → γ
h : ∀ (a : α), Continuous (f a)
x✝ : α × β
a : α
b : β
⊢ ContinuousAt (uncurry f) (a, b)
[PROOFSTEP]
simp only [ContinuousAt, nhds_prod_eq, nhds_discrete α, pure_prod, tendsto_map'_iff, (· ∘ ·), uncurry, (h a).tendsto]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set (α × α)
x : α
hx : s ∈ 𝓝 (x, x)
⊢ ∃ U, IsOpen U ∧ x ∈ U ∧ U ×ˢ U ⊆ s
[PROOFSTEP]
simpa [nhds_prod_eq, (nhds_basis_opens x).prod_self.mem_iff, and_assoc, and_left_comm] using hx
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
x : α × β
⊢ map Prod.fst (𝓝[Prod.snd ⁻¹' {x.snd}] x) = 𝓝 x.fst
[PROOFSTEP]
refine' le_antisymm (continuousAt_fst.mono_left inf_le_left) fun s hs => _
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
x : α × β
s : Set α
hs : s ∈ map Prod.fst (𝓝[Prod.snd ⁻¹' {x.snd}] x)
⊢ s ∈ 𝓝 x.fst
[PROOFSTEP]
rcases x with ⟨x, y⟩
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
x : α
y : β
hs : s ∈ map Prod.fst (𝓝[Prod.snd ⁻¹' {(x, y).snd}] (x, y))
⊢ s ∈ 𝓝 (x, y).fst
[PROOFSTEP]
rw [mem_map, nhdsWithin, mem_inf_principal, mem_nhds_prod_iff] at hs
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
x : α
y : β
hs : ∃ u, u ∈ 𝓝 x ∧ ∃ v, v ∈ 𝓝 y ∧ u ×ˢ v ⊆ {x_1 | x_1 ∈ Prod.snd ⁻¹' {(x, y).snd} → x_1 ∈ Prod.fst ⁻¹' s}
⊢ s ∈ 𝓝 (x, y).fst
[PROOFSTEP]
rcases hs with ⟨u, hu, v, hv, H⟩
[GOAL]
case mk.intro.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
x : α
y : β
u : Set α
hu : u ∈ 𝓝 x
v : Set β
hv : v ∈ 𝓝 y
H : u ×ˢ v ⊆ {x_1 | x_1 ∈ Prod.snd ⁻¹' {(x, y).snd} → x_1 ∈ Prod.fst ⁻¹' s}
⊢ s ∈ 𝓝 (x, y).fst
[PROOFSTEP]
simp only [prod_subset_iff, mem_singleton_iff, mem_setOf_eq, mem_preimage] at H
[GOAL]
case mk.intro.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
x : α
y : β
u : Set α
hu : u ∈ 𝓝 x
v : Set β
hv : v ∈ 𝓝 y
H : ∀ (x : α), x ∈ u → ∀ (y_1 : β), y_1 ∈ v → y_1 = y → x ∈ s
⊢ s ∈ 𝓝 (x, y).fst
[PROOFSTEP]
exact mem_of_superset hu fun z hz => H _ hz _ (mem_of_mem_nhds hv) rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
x : α × β
⊢ map Prod.snd (𝓝[Prod.fst ⁻¹' {x.fst}] x) = 𝓝 x.snd
[PROOFSTEP]
refine' le_antisymm (continuousAt_snd.mono_left inf_le_left) fun s hs => _
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
x : α × β
s : Set β
hs : s ∈ map Prod.snd (𝓝[Prod.fst ⁻¹' {x.fst}] x)
⊢ s ∈ 𝓝 x.snd
[PROOFSTEP]
rcases x with ⟨x, y⟩
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set β
x : α
y : β
hs : s ∈ map Prod.snd (𝓝[Prod.fst ⁻¹' {(x, y).fst}] (x, y))
⊢ s ∈ 𝓝 (x, y).snd
[PROOFSTEP]
rw [mem_map, nhdsWithin, mem_inf_principal, mem_nhds_prod_iff] at hs
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set β
x : α
y : β
hs : ∃ u, u ∈ 𝓝 x ∧ ∃ v, v ∈ 𝓝 y ∧ u ×ˢ v ⊆ {x_1 | x_1 ∈ Prod.fst ⁻¹' {(x, y).fst} → x_1 ∈ Prod.snd ⁻¹' s}
⊢ s ∈ 𝓝 (x, y).snd
[PROOFSTEP]
rcases hs with ⟨u, hu, v, hv, H⟩
[GOAL]
case mk.intro.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set β
x : α
y : β
u : Set α
hu : u ∈ 𝓝 x
v : Set β
hv : v ∈ 𝓝 y
H : u ×ˢ v ⊆ {x_1 | x_1 ∈ Prod.fst ⁻¹' {(x, y).fst} → x_1 ∈ Prod.snd ⁻¹' s}
⊢ s ∈ 𝓝 (x, y).snd
[PROOFSTEP]
simp only [prod_subset_iff, mem_singleton_iff, mem_setOf_eq, mem_preimage] at H
[GOAL]
case mk.intro.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set β
x : α
y : β
u : Set α
hu : u ∈ 𝓝 x
v : Set β
hv : v ∈ 𝓝 y
H : ∀ (x_1 : α), x_1 ∈ u → ∀ (y : β), y ∈ v → x_1 = x → y ∈ s
⊢ s ∈ 𝓝 (x, y).snd
[PROOFSTEP]
exact mem_of_superset hv fun z hz => H _ (mem_of_mem_nhds hu) _ hz rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
⊢ IsOpen (s ×ˢ t) ↔ IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
[PROOFSTEP]
cases' (s ×ˢ t).eq_empty_or_nonempty with h h
[GOAL]
case inl
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : s ×ˢ t = ∅
⊢ IsOpen (s ×ˢ t) ↔ IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
[PROOFSTEP]
simp [h, prod_eq_empty_iff.1 h]
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
⊢ IsOpen (s ×ˢ t) ↔ IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
[PROOFSTEP]
have st : s.Nonempty ∧ t.Nonempty := prod_nonempty_iff.1 h
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
⊢ IsOpen (s ×ˢ t) ↔ IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
[PROOFSTEP]
constructor
[GOAL]
case inr.mp
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
⊢ IsOpen (s ×ˢ t) → IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
[PROOFSTEP]
intro (H : IsOpen (s ×ˢ t))
[GOAL]
case inr.mp
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
[PROOFSTEP]
refine' Or.inl ⟨_, _⟩
[GOAL]
case inr.mp.refine'_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen s
case inr.mp.refine'_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen t
[PROOFSTEP]
show IsOpen s
[GOAL]
case inr.mp.refine'_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen s
[PROOFSTEP]
rw [← fst_image_prod s st.2]
[GOAL]
case inr.mp.refine'_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen (Prod.fst '' s ×ˢ t)
[PROOFSTEP]
exact isOpenMap_fst _ H
[GOAL]
case inr.mp.refine'_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen t
[PROOFSTEP]
show IsOpen t
[GOAL]
case inr.mp.refine'_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen t
[PROOFSTEP]
rw [← snd_image_prod st.1 t]
[GOAL]
case inr.mp.refine'_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen (s ×ˢ t)
⊢ IsOpen (Prod.snd '' s ×ˢ t)
[PROOFSTEP]
exact isOpenMap_snd _ H
[GOAL]
case inr.mpr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
⊢ IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅ → IsOpen (s ×ˢ t)
[PROOFSTEP]
intro H
[GOAL]
case inr.mpr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen s ∧ IsOpen t ∨ s = ∅ ∨ t = ∅
⊢ IsOpen (s ×ˢ t)
[PROOFSTEP]
simp only [st.1.ne_empty, st.2.ne_empty, not_false_iff, or_false_iff] at H
[GOAL]
case inr.mpr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
h : Set.Nonempty (s ×ˢ t)
st : Set.Nonempty s ∧ Set.Nonempty t
H : IsOpen s ∧ IsOpen t
⊢ IsOpen (s ×ˢ t)
[PROOFSTEP]
exact H.1.prod H.2
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
x✝ : α × β
a : α
b : β
⊢ (a, b) ∈ closure (s ×ˢ t) ↔ (a, b) ∈ closure s ×ˢ closure t
[PROOFSTEP]
simp_rw [mem_prod, mem_closure_iff_nhdsWithin_neBot, nhdsWithin_prod_eq, prod_neBot]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
x✝ : α × β
a : α
b : β
⊢ (a, b) ∈ interior (s ×ˢ t) ↔ (a, b) ∈ interior s ×ˢ interior t
[PROOFSTEP]
simp only [mem_interior_iff_mem_nhds, mem_prod, prod_mem_nhds_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
⊢ frontier (s ×ˢ t) = closure s ×ˢ frontier t ∪ frontier s ×ˢ closure t
[PROOFSTEP]
simp only [frontier, closure_prod_eq, interior_prod_eq, prod_diff_prod]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
⊢ frontier (s ×ˢ univ) = frontier s ×ˢ univ
[PROOFSTEP]
simp [frontier_prod_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set β
⊢ frontier (univ ×ˢ s) = univ ×ˢ frontier s
[PROOFSTEP]
simp [frontier_prod_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β → γ
a : α
b : β
s : Set α
t : Set β
u : Set γ
hf : Continuous (uncurry f)
ha : a ∈ closure s
hb : b ∈ closure t
h : ∀ (a : α), a ∈ s → ∀ (b : β), b ∈ t → f a b ∈ u
⊢ (a, b) ∈ closure (s ×ˢ t)
[PROOFSTEP]
simpa only [closure_prod_eq] using mk_mem_prod ha hb
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s₁ : Set α
s₂ : Set β
h₁ : IsClosed s₁
h₂ : IsClosed s₂
⊢ closure (s₁ ×ˢ s₂) = s₁ ×ˢ s₂
[PROOFSTEP]
simp only [h₁.closure_eq, h₂.closure_eq, closure_prod_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
hs : Dense s
ht : Dense t
x : α × β
⊢ x ∈ closure (s ×ˢ t)
[PROOFSTEP]
rw [closure_prod_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
s : Set α
t : Set β
hs : Dense s
ht : Dense t
x : α × β
⊢ x ∈ closure s ×ˢ closure t
[PROOFSTEP]
exact ⟨hs x.1, ht x.2⟩
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
ι : Type u_5
κ : Type u_6
f : ι → β
g : κ → γ
hf : DenseRange f
hg : DenseRange g
⊢ DenseRange (Prod.map f g)
[PROOFSTEP]
simpa only [DenseRange, prod_range_range_eq] using hf.prod hg
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
hf : Inducing f
hg : Inducing g
x✝ : α × γ
a : α
b : γ
⊢ 𝓝 (a, b) = comap (Prod.map f g) (𝓝 (Prod.map f g (a, b)))
[PROOFSTEP]
simp_rw [Prod.map, nhds_prod_eq, hf.nhds_eq_comap, hg.nhds_eq_comap, prod_comap_comap_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
a : α
f : β → γ
⊢ (Inducing fun x => (a, f x)) ↔ Inducing f
[PROOFSTEP]
simp_rw [inducing_iff, instTopologicalSpaceProd, induced_inf, induced_compose, Function.comp, induced_const, top_inf_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
b : β
f : α → γ
⊢ (Inducing fun x => (f x, b)) ↔ Inducing f
[PROOFSTEP]
simp_rw [inducing_iff, instTopologicalSpaceProd, induced_inf, induced_compose, Function.comp, induced_const, inf_top_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
hf : _root_.Embedding f
hg : _root_.Embedding g
src✝ : Inducing (Prod.map f g) := Inducing.prod_map hf.toInducing hg.toInducing
x✝¹ x✝ : α × γ
x₁ : α
x₂ : γ
y₁ : α
y₂ : γ
⊢ Prod.map f g (x₁, x₂) = Prod.map f g (y₁, y₂) → (x₁, x₂) = (y₁, y₂)
[PROOFSTEP]
simp [hf.inj.eq_iff, hg.inj.eq_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
hf : IsOpenMap f
hg : IsOpenMap g
⊢ IsOpenMap fun p => (f p.fst, g p.snd)
[PROOFSTEP]
rw [isOpenMap_iff_nhds_le]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
hf : IsOpenMap f
hg : IsOpenMap g
⊢ ∀ (a : α × γ), 𝓝 (f a.fst, g a.snd) ≤ map (fun p => (f p.fst, g p.snd)) (𝓝 a)
[PROOFSTEP]
rintro ⟨a, b⟩
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
hf : IsOpenMap f
hg : IsOpenMap g
a : α
b : γ
⊢ 𝓝 (f (a, b).fst, g (a, b).snd) ≤ map (fun p => (f p.fst, g p.snd)) (𝓝 (a, b))
[PROOFSTEP]
rw [nhds_prod_eq, nhds_prod_eq, ← Filter.prod_map_map_eq]
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
inst✝³ : TopologicalSpace γ
inst✝² : TopologicalSpace δ
inst✝¹ : TopologicalSpace ε
inst✝ : TopologicalSpace ζ
f : α → β
g : γ → δ
hf : IsOpenMap f
hg : IsOpenMap g
a : α
b : γ
⊢ 𝓝 (f (a, b).fst) ×ˢ 𝓝 (g (a, b).snd) ≤ map f (𝓝 a) ×ˢ map g (𝓝 b)
[PROOFSTEP]
exact Filter.prod_mono (hf.nhds_le a) (hg.nhds_le b)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
s : Set (α ⊕ β)
⊢ IsClosed s ↔ IsClosed (inl ⁻¹' s) ∧ IsClosed (inr ⁻¹' s)
[PROOFSTEP]
simp only [← isOpen_compl_iff, isOpen_sum_iff, preimage_compl]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
u : Set α
hu : IsOpen u
⊢ IsOpen (inl '' u)
[PROOFSTEP]
simpa [isOpen_sum_iff, preimage_image_eq u Sum.inl_injective]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
u : Set β
hu : IsOpen u
⊢ IsOpen (inr '' u)
[PROOFSTEP]
simpa [isOpen_sum_iff, preimage_image_eq u Sum.inr_injective]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
⊢ IsClosed (range inl)
[PROOFSTEP]
rw [← isOpen_compl_iff, compl_range_inl]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
⊢ IsOpen (range inr)
[PROOFSTEP]
exact isOpen_range_inr
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
⊢ IsClosed (range inr)
[PROOFSTEP]
rw [← isOpen_compl_iff, compl_range_inr]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
⊢ IsOpen (range inl)
[PROOFSTEP]
exact isOpen_range_inl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α ⊕ β → γ
⊢ IsOpenMap f ↔ (IsOpenMap fun a => f (inl a)) ∧ IsOpenMap fun b => f (inr b)
[PROOFSTEP]
simp only [isOpenMap_iff_nhds_le, Sum.forall, nhds_inl, nhds_inr, Filter.map_map, comp]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : TopologicalSpace γ
inst✝ : TopologicalSpace δ
f : α → γ
g : β → γ
⊢ IsOpenMap (Sum.elim f g) ↔ IsOpenMap f ∧ IsOpenMap g
[PROOFSTEP]
simp only [isOpenMap_sum, elim_inl, elim_inr]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
h : IsClosed {a | p a}
⊢ IsClosed (range Subtype.val)
[PROOFSTEP]
rwa [Subtype.range_coe_subtype]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : IsClosedMap f
T : Set β
⊢ IsClosedMap (Set.restrictPreimage T f)
[PROOFSTEP]
rw [isClosedMap_iff_clusterPt] at hcl ⊢
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
T : Set β
⊢ ∀ (s : Set ↑(f ⁻¹' T)) (y : ↑T),
MapClusterPt y (𝓟 s) (Set.restrictPreimage T f) → ∃ x, Set.restrictPreimage T f x = y ∧ ClusterPt x (𝓟 s)
[PROOFSTEP]
intro A ⟨y, hyT⟩ hy
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
T : Set β
A : Set ↑(f ⁻¹' T)
y : β
hyT : y ∈ T
hy : MapClusterPt { val := y, property := hyT } (𝓟 A) (Set.restrictPreimage T f)
⊢ ∃ x, Set.restrictPreimage T f x = { val := y, property := hyT } ∧ ClusterPt x (𝓟 A)
[PROOFSTEP]
rw [restrictPreimage, MapClusterPt, ← inducing_subtype_val.mapClusterPt_iff, MapClusterPt, map_map,
MapsTo.restrict_commutes, ← map_map, ← MapClusterPt, map_principal] at hy
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
T : Set β
A : Set ↑(f ⁻¹' T)
y : β
hyT : y ∈ T
hy : MapClusterPt (↑{ val := y, property := hyT }) (𝓟 (Subtype.val '' A)) f
⊢ ∃ x, Set.restrictPreimage T f x = { val := y, property := hyT } ∧ ClusterPt x (𝓟 A)
[PROOFSTEP]
rcases hcl _ y hy with ⟨x, hxy, hx⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
T : Set β
A : Set ↑(f ⁻¹' T)
y : β
hyT : y ∈ T
hy : MapClusterPt (↑{ val := y, property := hyT }) (𝓟 (Subtype.val '' A)) f
x : α
hxy : f x = y
hx : ClusterPt x (𝓟 (Subtype.val '' A))
⊢ ∃ x, Set.restrictPreimage T f x = { val := y, property := hyT } ∧ ClusterPt x (𝓟 A)
[PROOFSTEP]
have hxT : f x ∈ T := hxy ▸ hyT
[GOAL]
case intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
T : Set β
A : Set ↑(f ⁻¹' T)
y : β
hyT : y ∈ T
hy : MapClusterPt (↑{ val := y, property := hyT }) (𝓟 (Subtype.val '' A)) f
x : α
hxy : f x = y
hx : ClusterPt x (𝓟 (Subtype.val '' A))
hxT : f x ∈ T
⊢ ∃ x, Set.restrictPreimage T f x = { val := y, property := hyT } ∧ ClusterPt x (𝓟 A)
[PROOFSTEP]
refine ⟨⟨x, hxT⟩, Subtype.ext hxy, ?_⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
f : α → β
hcl : ∀ (s : Set α) (y : β), MapClusterPt y (𝓟 s) f → ∃ x, f x = y ∧ ClusterPt x (𝓟 s)
T : Set β
A : Set ↑(f ⁻¹' T)
y : β
hyT : y ∈ T
hy : MapClusterPt (↑{ val := y, property := hyT }) (𝓟 (Subtype.val '' A)) f
x : α
hxy : f x = y
hx : ClusterPt x (𝓟 (Subtype.val '' A))
hxT : f x ∈ T
⊢ ClusterPt { val := x, property := hxT } (𝓟 A)
[PROOFSTEP]
rwa [← inducing_subtype_val.mapClusterPt_iff, MapClusterPt, map_principal]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
s : Set α
t : Set ↑s
⊢ Dense t ↔ s ⊆ closure (val '' t)
[PROOFSTEP]
rw [inducing_subtype_val.dense_iff, SetCoe.forall]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
s : Set α
t : Set ↑s
⊢ (∀ (x : α) (h : x ∈ s), ↑{ val := x, property := h } ∈ closure (val '' t)) ↔ s ⊆ closure (val '' t)
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
s : Set α
a : ↑s
⊢ map Subtype.val (𝓝 a) = 𝓝[s] ↑a
[PROOFSTEP]
rw [inducing_subtype_val.map_nhds_eq, Subtype.range_val]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
a : α
ha : p a
h : ∀ᶠ (x : α) in 𝓝 a, p x
⊢ range Subtype.val ∈ 𝓝 ↑{ val := a, property := ha }
[PROOFSTEP]
rw [Subtype.range_val]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : TopologicalSpace γ
p : α → Prop
a : α
ha : p a
h : ∀ᶠ (x : α) in 𝓝 a, p x
⊢ (fun x => p x) ∈ 𝓝 ↑{ val := a, property := ha }
[PROOFSTEP]
exact h
[GOAL]
α : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β✝
inst✝ : TopologicalSpace γ
p✝ : α → Prop
β : Type u_5
p : α → Prop
b : Filter β
f : β → Subtype p
a : α
ha : p a
⊢ Tendsto f b (𝓝 { val := a, property := ha }) ↔ Tendsto (fun x => ↑(f x)) b (𝓝 ↑{ val := a, property := ha })
[PROOFSTEP]
rw [nhds_subtype_eq_comap, tendsto_comap_iff]
[GOAL]
α : Type u
β✝ : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β✝
inst✝ : TopologicalSpace γ
p✝ : α → Prop
β : Type u_5
p : α → Prop
b : Filter β
f : β → Subtype p
a : α
ha : p a
⊢ Tendsto (Subtype.val ∘ f) b (𝓝 a) ↔ Tendsto (fun x => ↑(f x)) b (𝓝 ↑{ val := a, property := ha })
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
⊢ Continuous f ↔ ∀ (i : ι), Continuous fun a => f a i
[PROOFSTEP]
simp only [continuous_iInf_rng, continuous_induced_rng, comp]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
a : (i : ι) → π i
⊢ 𝓝 a = Filter.pi fun i => 𝓝 (a i)
[PROOFSTEP]
simp only [nhds_iInf, nhds_induced, Filter.pi]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
f : β → (i : ι) → π i
g : (i : ι) → π i
u : Filter β
⊢ Tendsto f u (𝓝 g) ↔ ∀ (x : ι), Tendsto (fun i => f i x) u (𝓝 (g x))
[PROOFSTEP]
rw [nhds_pi, Filter.tendsto_pi]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
inst✝ : DecidableEq ι
l : Filter β
f : β → (i : ι) → π i
x : (i : ι) → π i
hf : Tendsto f l (𝓝 x)
i : ι
g : β → π i
xi : π i
hg : Tendsto g l (𝓝 xi)
j : ι
⊢ Tendsto (fun i_1 => Function.update (f i_1) i (g i_1) j) l (𝓝 (Function.update x i xi j))
[PROOFSTEP]
rcases eq_or_ne j i with (rfl | hj)
[GOAL]
case inl
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
inst✝ : DecidableEq ι
l : Filter β
f : β → (i : ι) → π i
x : (i : ι) → π i
hf : Tendsto f l (𝓝 x)
j : ι
g : β → π j
xi : π j
hg : Tendsto g l (𝓝 xi)
⊢ Tendsto (fun i => Function.update (f i) j (g i) j) l (𝓝 (Function.update x j xi j))
[PROOFSTEP]
simp [*, hf.apply]
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
inst✝ : DecidableEq ι
l : Filter β
f : β → (i : ι) → π i
x : (i : ι) → π i
hf : Tendsto f l (𝓝 x)
i : ι
g : β → π i
xi : π i
hg : Tendsto g l (𝓝 xi)
j : ι
hj : j ≠ i
⊢ Tendsto (fun i_1 => Function.update (f i_1) i (g i_1) j) l (𝓝 (Function.update x i xi j))
[PROOFSTEP]
simp [*, hf.apply]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
n : ℕ
π : Fin (n + 1) → Type u_8
inst✝ : (i : Fin (n + 1)) → TopologicalSpace (π i)
i : Fin (n + 1)
f : β → π i
l : Filter β
x : π i
hf : Tendsto f l (𝓝 x)
g : β → (j : Fin n) → π (Fin.succAbove i j)
y : (j : Fin n) → π (Fin.succAbove i j)
hg : Tendsto g l (𝓝 y)
j : Fin (n + 1)
⊢ Tendsto (fun i_1 => Fin.insertNth i (f i_1) (g i_1) i) l (𝓝 (Fin.insertNth i x y i))
[PROOFSTEP]
simpa
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
n : ℕ
π : Fin (n + 1) → Type u_8
inst✝ : (i : Fin (n + 1)) → TopologicalSpace (π i)
i : Fin (n + 1)
f : β → π i
l : Filter β
x : π i
hf : Tendsto f l (𝓝 x)
g : β → (j : Fin n) → π (Fin.succAbove i j)
y : (j : Fin n) → π (Fin.succAbove i j)
hg : Tendsto g l (𝓝 y)
j : Fin (n + 1)
⊢ ∀ (j : Fin n),
Tendsto (fun i_1 => Fin.insertNth i (f i_1) (g i_1) (Fin.succAbove i j)) l
(𝓝 (Fin.insertNth i x y (Fin.succAbove i j)))
[PROOFSTEP]
simpa using tendsto_pi_nhds.1 hg
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
i : Set ι
s : (a : ι) → Set (π a)
hi : Set.Finite i
hs : ∀ (a : ι), a ∈ i → IsOpen (s a)
⊢ IsOpen (Set.pi i s)
[PROOFSTEP]
rw [pi_def]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
i : Set ι
s : (a : ι) → Set (π a)
hi : Set.Finite i
hs : ∀ (a : ι), a ∈ i → IsOpen (s a)
⊢ IsOpen (⋂ (a : ι) (_ : a ∈ i), eval a ⁻¹' s a)
[PROOFSTEP]
exact isOpen_biInter hi fun a ha => (hs _ ha).preimage (continuous_apply _)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
⊢ IsOpen s ↔ ∀ (f : (a : ι) → π a), f ∈ s → ∃ I u, (∀ (a : ι), a ∈ I → IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi (↑I) u ⊆ s
[PROOFSTEP]
rw [isOpen_iff_nhds]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
⊢ (∀ (a : (a : ι) → π a), a ∈ s → 𝓝 a ≤ 𝓟 s) ↔
∀ (f : (a : ι) → π a), f ∈ s → ∃ I u, (∀ (a : ι), a ∈ I → IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi (↑I) u ⊆ s
[PROOFSTEP]
simp_rw [le_principal_iff, nhds_pi, Filter.mem_pi', mem_nhds_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
⊢ (∀ (a : (a : ι) → π a), a ∈ s → ∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s) ↔
∀ (f : (a : ι) → π a), f ∈ s → ∃ I u, (∀ (a : ι), a ∈ I → IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi (↑I) u ⊆ s
[PROOFSTEP]
refine ball_congr fun a _ => ⟨?_, ?_⟩
[GOAL]
case refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
⊢ (∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s) →
∃ I u, (∀ (a_2 : ι), a_2 ∈ I → IsOpen (u a_2) ∧ a a_2 ∈ u a_2) ∧ Set.pi (↑I) u ⊆ s
[PROOFSTEP]
rintro ⟨I, t, ⟨h1, h2⟩⟩
[GOAL]
case refine_1.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
⊢ ∃ I u, (∀ (a_1 : ι), a_1 ∈ I → IsOpen (u a_1) ∧ a a_1 ∈ u a_1) ∧ Set.pi (↑I) u ⊆ s
[PROOFSTEP]
refine ⟨I, fun a => eval a '' (I : Set ι).pi fun a => (h1 a).choose, fun i hi => ?_, ?_⟩
[GOAL]
case refine_1.intro.intro.intro.refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : i ∈ I
⊢ IsOpen
((fun a_1 => eval a_1 '' Set.pi ↑I fun a_2 => Exists.choose (_ : ∃ t_1, t_1 ⊆ t a_2 ∧ IsOpen t_1 ∧ a a_2 ∈ t_1))
i) ∧
a i ∈
(fun a_1 => eval a_1 '' Set.pi ↑I fun a_2 => Exists.choose (_ : ∃ t_1, t_1 ⊆ t a_2 ∧ IsOpen t_1 ∧ a a_2 ∈ t_1)) i
[PROOFSTEP]
simp_rw [Set.eval_image_pi (Finset.mem_coe.mpr hi) (pi_nonempty_iff.mpr fun i => ⟨_, fun _ => (h1 i).choose_spec.2.2⟩)]
[GOAL]
case refine_1.intro.intro.intro.refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : i ∈ I
⊢ IsOpen (Exists.choose (_ : ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1)) ∧
a i ∈ Exists.choose (_ : ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1)
[PROOFSTEP]
exact (h1 i).choose_spec.2
[GOAL]
case refine_1.intro.intro.intro.refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
⊢ (Set.pi ↑I fun a_1 =>
eval a_1 '' Set.pi ↑I fun a_2 => Exists.choose (_ : ∃ t_1, t_1 ⊆ t a_2 ∧ IsOpen t_1 ∧ a a_2 ∈ t_1)) ⊆
s
[PROOFSTEP]
exact Subset.trans (Set.pi_mono fun i hi => (Set.eval_image_pi_subset hi).trans (h1 i).choose_spec.1) h2
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
⊢ (∃ I u, (∀ (a_1 : ι), a_1 ∈ I → IsOpen (u a_1) ∧ a a_1 ∈ u a_1) ∧ Set.pi (↑I) u ⊆ s) →
∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s
[PROOFSTEP]
rintro ⟨I, t, ⟨h1, h2⟩⟩
[GOAL]
case refine_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
⊢ ∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s
[PROOFSTEP]
refine ⟨I, fun a => ite (a ∈ I) (t a) Set.univ, fun i => ?_, ?_⟩
[GOAL]
case refine_2.intro.intro.intro.refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
⊢ ∃ t_1, t_1 ⊆ (fun a => if a ∈ I then t a else univ) i ∧ IsOpen t_1 ∧ a i ∈ t_1
[PROOFSTEP]
by_cases hi : i ∈ I
[GOAL]
case pos
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : i ∈ I
⊢ ∃ t_1, t_1 ⊆ (fun a => if a ∈ I then t a else univ) i ∧ IsOpen t_1 ∧ a i ∈ t_1
[PROOFSTEP]
use t i
[GOAL]
case h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : i ∈ I
⊢ t i ⊆ (fun a => if a ∈ I then t a else univ) i ∧ IsOpen (t i) ∧ a i ∈ t i
[PROOFSTEP]
simp_rw [if_pos hi]
[GOAL]
case h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : i ∈ I
⊢ t i ⊆ t i ∧ IsOpen (t i) ∧ a i ∈ t i
[PROOFSTEP]
exact ⟨Subset.rfl, (h1 i) hi⟩
[GOAL]
case neg
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : ¬i ∈ I
⊢ ∃ t_1, t_1 ⊆ (fun a => if a ∈ I then t a else univ) i ∧ IsOpen t_1 ∧ a i ∈ t_1
[PROOFSTEP]
use Set.univ
[GOAL]
case h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : ¬i ∈ I
⊢ univ ⊆ (fun a => if a ∈ I then t a else univ) i ∧ IsOpen univ ∧ a i ∈ univ
[PROOFSTEP]
simp_rw [if_neg hi]
[GOAL]
case h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
i : ι
hi : ¬i ∈ I
⊢ univ ⊆ univ ∧ IsOpen univ ∧ a i ∈ univ
[PROOFSTEP]
exact ⟨Subset.rfl, isOpen_univ, mem_univ _⟩
[GOAL]
case refine_2.intro.intro.intro.refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
⊢ (Set.pi ↑I fun a => if a ∈ I then t a else univ) ⊆ s
[PROOFSTEP]
rw [← Set.univ_pi_ite]
[GOAL]
case refine_2.intro.intro.intro.refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
s : Set ((a : ι) → π a)
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), a_1 ∈ I → IsOpen (t a_1) ∧ a a_1 ∈ t a_1
h2 : Set.pi (↑I) t ⊆ s
⊢ (Set.pi univ fun i => if i ∈ ↑I then if i ∈ I then t i else univ else univ) ⊆ s
[PROOFSTEP]
simp only [← ite_and, ← Finset.mem_coe, and_self_iff, Set.univ_pi_ite, h2]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
⊢ IsOpen s ↔ ∀ (f : (a : ι) → π a), f ∈ s → ∃ u, (∀ (a : ι), IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi univ u ⊆ s
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
⊢ IsOpen s ↔ ∀ (f : (a : ι) → π a), f ∈ s → ∃ u, (∀ (a : ι), IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi univ u ⊆ s
[PROOFSTEP]
rw [isOpen_iff_nhds]
[GOAL]
case intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
⊢ (∀ (a : (a : ι) → π a), a ∈ s → 𝓝 a ≤ 𝓟 s) ↔
∀ (f : (a : ι) → π a), f ∈ s → ∃ u, (∀ (a : ι), IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi univ u ⊆ s
[PROOFSTEP]
simp_rw [le_principal_iff, nhds_pi, Filter.mem_pi', mem_nhds_iff]
[GOAL]
case intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
⊢ (∀ (a : (a : ι) → π a), a ∈ s → ∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s) ↔
∀ (f : (a : ι) → π a), f ∈ s → ∃ u, (∀ (a : ι), IsOpen (u a) ∧ f a ∈ u a) ∧ Set.pi univ u ⊆ s
[PROOFSTEP]
refine ball_congr fun a _ => ⟨?_, ?_⟩
[GOAL]
case intro.refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
a : (a : ι) → π a
x✝ : a ∈ s
⊢ (∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s) →
∃ u, (∀ (a_2 : ι), IsOpen (u a_2) ∧ a a_2 ∈ u a_2) ∧ Set.pi univ u ⊆ s
[PROOFSTEP]
rintro ⟨I, t, ⟨h1, h2⟩⟩
[GOAL]
case intro.refine_1.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
⊢ ∃ u, (∀ (a_1 : ι), IsOpen (u a_1) ∧ a a_1 ∈ u a_1) ∧ Set.pi univ u ⊆ s
[PROOFSTEP]
refine
⟨fun i => (h1 i).choose,
⟨fun i => (h1 i).choose_spec.2, (Set.pi_mono fun i _ => (h1 i).choose_spec.1).trans (Subset.trans ?_ h2)⟩⟩
[GOAL]
case intro.refine_1.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
⊢ (Set.pi univ fun i => t i) ⊆ Set.pi (↑I) t
[PROOFSTEP]
rw [← Set.pi_inter_compl (I : Set ι)]
[GOAL]
case intro.refine_1.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
a : (a : ι) → π a
x✝ : a ∈ s
I : Finset ι
t : (i : ι) → Set (π i)
h1 : ∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1
h2 : Set.pi (↑I) t ⊆ s
⊢ ((Set.pi ↑I fun i => t i) ∩ Set.pi (↑I)ᶜ fun i => t i) ⊆ Set.pi (↑I) t
[PROOFSTEP]
exact inter_subset_left _ _
[GOAL]
case intro.refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
a : (a : ι) → π a
x✝ : a ∈ s
⊢ (∃ u, (∀ (a_1 : ι), IsOpen (u a_1) ∧ a a_1 ∈ u a_1) ∧ Set.pi univ u ⊆ s) →
∃ I t, (∀ (i : ι), ∃ t_1, t_1 ⊆ t i ∧ IsOpen t_1 ∧ a i ∈ t_1) ∧ Set.pi (↑I) t ⊆ s
[PROOFSTEP]
exact fun ⟨u, ⟨h1, _⟩⟩ => ⟨Finset.univ, u, ⟨fun i => ⟨u i, ⟨rfl.subset, h1 i⟩⟩, by rwa [Finset.coe_univ]⟩⟩
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : Finite ι
s : Set ((a : ι) → π a)
val✝ : Fintype ι
a : (a : ι) → π a
x✝¹ : a ∈ s
x✝ : ∃ u, (∀ (a_1 : ι), IsOpen (u a_1) ∧ a a_1 ∈ u a_1) ∧ Set.pi univ u ⊆ s
u : (a : ι) → Set (π a)
h1 : ∀ (a_1 : ι), IsOpen (u a_1) ∧ a a_1 ∈ u a_1
right✝ : Set.pi univ u ⊆ s
⊢ Set.pi (↑Finset.univ) u ⊆ s
[PROOFSTEP]
rwa [Finset.coe_univ]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
i : Set ι
s : (a : ι) → Set (π a)
hs : ∀ (a : ι), a ∈ i → IsClosed (s a)
⊢ IsClosed (Set.pi i s)
[PROOFSTEP]
rw [pi_def]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
i : Set ι
s : (a : ι) → Set (π a)
hs : ∀ (a : ι), a ∈ i → IsClosed (s a)
⊢ IsClosed (⋂ (a : ι) (_ : a ∈ i), eval a ⁻¹' s a)
[PROOFSTEP]
exact isClosed_biInter fun a ha => (hs _ ha).preimage (continuous_apply _)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
I : Set ι
s : (i : ι) → Set (π i)
a : (i : ι) → π i
hs : Set.pi I s ∈ 𝓝 a
i : ι
hi : i ∈ I
⊢ s i ∈ 𝓝 (a i)
[PROOFSTEP]
rw [nhds_pi] at hs
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
I : Set ι
s : (i : ι) → Set (π i)
a : (i : ι) → π i
hs : Set.pi I s ∈ Filter.pi fun i => 𝓝 (a i)
i : ι
hi : i ∈ I
⊢ s i ∈ 𝓝 (a i)
[PROOFSTEP]
exact mem_of_pi_mem_pi hs hi
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
i : Set ι
s : (a : ι) → Set (π a)
x : (a : ι) → π a
hi : Set.Finite i
hs : ∀ (a : ι), a ∈ i → s a ∈ 𝓝 (x a)
⊢ Set.pi i s ∈ 𝓝 x
[PROOFSTEP]
rw [pi_def, biInter_mem hi]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
i : Set ι
s : (a : ι) → Set (π a)
x : (a : ι) → π a
hi : Set.Finite i
hs : ∀ (a : ι), a ∈ i → s a ∈ 𝓝 (x a)
⊢ ∀ (i_1 : ι), i_1 ∈ i → eval i_1 ⁻¹' s i_1 ∈ 𝓝 x
[PROOFSTEP]
exact fun a ha => (continuous_apply a).continuousAt (hs a ha)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (π i)
a : (i : ι) → π i
⊢ Set.pi I s ∈ 𝓝 a ↔ ∀ (i : ι), i ∈ I → s i ∈ 𝓝 (a i)
[PROOFSTEP]
rw [nhds_pi, pi_mem_pi_iff hI]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (π i)
⊢ interior (Set.pi I s) = Set.pi I fun i => interior (s i)
[PROOFSTEP]
ext a
[GOAL]
case h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
I : Set ι
hI : Set.Finite I
s : (i : ι) → Set (π i)
a : (i : ι) → π i
⊢ a ∈ interior (Set.pi I s) ↔ a ∈ Set.pi I fun i => interior (s i)
[PROOFSTEP]
simp only [Set.mem_pi, mem_interior_iff_mem_nhds, set_pi_mem_nhds_iff hI]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : DecidableEq ι
s : Set ((a : ι) → π a)
x : (a : ι) → π a
hs : s ∈ 𝓝 x
y : (a : ι) → π a
⊢ ∃ I, Finset.piecewise I x y ∈ s
[PROOFSTEP]
simp only [nhds_pi, Filter.mem_pi'] at hs
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : DecidableEq ι
s : Set ((a : ι) → π a)
x y : (a : ι) → π a
hs : ∃ I t, (∀ (i : ι), t i ∈ 𝓝 (x i)) ∧ Set.pi (↑I) t ⊆ s
⊢ ∃ I, Finset.piecewise I x y ∈ s
[PROOFSTEP]
rcases hs with ⟨I, t, htx, hts⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : DecidableEq ι
s : Set ((a : ι) → π a)
x y : (a : ι) → π a
I : Finset ι
t : (i : ι) → Set (π i)
htx : ∀ (i : ι), t i ∈ 𝓝 (x i)
hts : Set.pi (↑I) t ⊆ s
⊢ ∃ I, Finset.piecewise I x y ∈ s
[PROOFSTEP]
refine' ⟨I, hts fun i hi => _⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝ : DecidableEq ι
s : Set ((a : ι) → π a)
x y : (a : ι) → π a
I : Finset ι
t : (i : ι) → Set (π i)
htx : ∀ (i : ι), t i ∈ 𝓝 (x i)
hts : Set.pi (↑I) t ⊆ s
i : ι
hi : i ∈ ↑I
⊢ Finset.piecewise I x y i ∈ t i
[PROOFSTEP]
simpa [Finset.mem_coe.1 hi] using mem_of_mem_nhds (htx i)
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
⊢ Pi.topologicalSpace = generateFrom {t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s}
[PROOFSTEP]
refine le_antisymm ?_ ?_
[GOAL]
case refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
⊢ Pi.topologicalSpace ≤ generateFrom {t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s}
[PROOFSTEP]
apply le_generateFrom
[GOAL]
case refine_1.h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
⊢ ∀ (s : Set ((a : ι) → π a)), s ∈ {t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s} → IsOpen s
[PROOFSTEP]
rintro _ ⟨s, i, hi, rfl⟩
[GOAL]
case refine_1.h.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
s : (a : ι) → Set (π a)
i : Finset ι
hi : ∀ (a : ι), a ∈ i → s a ∈ g a
⊢ IsOpen (Set.pi (↑i) s)
[PROOFSTEP]
letI := fun a => generateFrom (g a)
[GOAL]
case refine_1.h.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
s : (a : ι) → Set (π a)
i : Finset ι
hi : ∀ (a : ι), a ∈ i → s a ∈ g a
this : (a : ι) → TopologicalSpace (π a) := fun a => generateFrom (g a)
⊢ IsOpen (Set.pi (↑i) s)
[PROOFSTEP]
exact isOpen_set_pi i.finite_toSet (fun a ha => GenerateOpen.basic _ (hi a ha))
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
⊢ generateFrom {t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s} ≤ Pi.topologicalSpace
[PROOFSTEP]
refine le_iInf fun a => coinduced_le_iff_le_induced.1 <| le_generateFrom fun s hs => ?_
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
a : ι
s : Set (π a)
hs : s ∈ g a
⊢ IsOpen s
[PROOFSTEP]
refine GenerateOpen.basic _ ⟨update (fun a => univ) a s, { a }, ?_⟩
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
a : ι
s : Set (π a)
hs : s ∈ g a
⊢ (∀ (a_1 : ι), a_1 ∈ {a} → update (fun a => univ) a s a_1 ∈ g a_1) ∧
(fun f => f a) ⁻¹' s = Set.pi (↑{a}) (update (fun a => univ) a s)
[PROOFSTEP]
simp [hs]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
⊢ Pi.topologicalSpace = Pi.topologicalSpace
[PROOFSTEP]
simp only [generateFrom_setOf_isOpen]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
⊢ Pi.topologicalSpace = generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
[PROOFSTEP]
cases nonempty_fintype ι
[GOAL]
case intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
⊢ Pi.topologicalSpace = generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
[PROOFSTEP]
rw [pi_generateFrom_eq]
[GOAL]
case intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
⊢ generateFrom {t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s} =
generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
[PROOFSTEP]
refine' le_antisymm (generateFrom_anti _) (le_generateFrom _)
[GOAL]
case intro.refine'_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
⊢ {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s} ⊆
{t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s}
[PROOFSTEP]
exact fun s ⟨t, ht, Eq⟩ => ⟨t, Finset.univ, by simp [ht, Eq]⟩
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
s : Set ((i : ι) → π i)
x✝ : s ∈ {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
t : (a : ι) → Set (π a)
ht : ∀ (a : ι), t a ∈ g a
Eq : s = Set.pi univ t
⊢ (∀ (a : ι), a ∈ Finset.univ → t a ∈ g a) ∧ s = Set.pi (↑Finset.univ) t
[PROOFSTEP]
simp [ht, Eq]
[GOAL]
case intro.refine'_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
⊢ ∀ (s : Set ((i : ι) → π i)), s ∈ {t | ∃ s i, (∀ (a : ι), a ∈ i → s a ∈ g a) ∧ t = Set.pi (↑i) s} → IsOpen s
[PROOFSTEP]
rintro s ⟨t, i, ht, rfl⟩
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
⊢ IsOpen (Set.pi (↑i) t)
[PROOFSTEP]
letI := generateFrom {t | ∃ s : ∀ a, Set (π a), (∀ a, s a ∈ g a) ∧ t = pi univ s}
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
⊢ IsOpen (Set.pi (↑i) t)
[PROOFSTEP]
refine isOpen_iff_forall_mem_open.2 fun f hf => ?_
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
⊢ ∃ t_1, t_1 ⊆ Set.pi (↑i) t ∧ IsOpen t_1 ∧ f ∈ t_1
[PROOFSTEP]
choose c hcg hfc using fun a => sUnion_eq_univ_iff.1 (hg a) (f a)
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
⊢ ∃ t_1, t_1 ⊆ Set.pi (↑i) t ∧ IsOpen t_1 ∧ f ∈ t_1
[PROOFSTEP]
refine ⟨pi i t ∩ pi ((↑i)ᶜ : Set ι) c, inter_subset_left _ _, ?_, ⟨hf, fun a _ => hfc a⟩⟩
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
⊢ IsOpen (Set.pi (↑i) t ∩ Set.pi (↑i)ᶜ c)
[PROOFSTEP]
rw [← univ_pi_piecewise]
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
⊢ IsOpen (Set.pi univ (piecewise (↑i) t c))
[PROOFSTEP]
refine GenerateOpen.basic _ ⟨_, fun a => ?_, rfl⟩
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
a : ι
⊢ piecewise (↑i) t c a ∈ g a
[PROOFSTEP]
by_cases a ∈ i
[GOAL]
case intro.refine'_2.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
a : ι
⊢ piecewise (↑i) t c a ∈ g a
[PROOFSTEP]
by_cases a ∈ i
[GOAL]
case pos
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
a : ι
h : a ∈ i
⊢ piecewise (↑i) t c a ∈ g a
[PROOFSTEP]
simp [*]
[GOAL]
case neg
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π✝ : ι → Type u_6
κ : Type u_7
inst✝² : TopologicalSpace α
inst✝¹ : (i : ι) → TopologicalSpace (π✝ i)
f✝ : α → (i : ι) → π✝ i
π : ι → Type u_8
g : (a : ι) → Set (Set (π a))
inst✝ : Finite ι
hg : ∀ (a : ι), ⋃₀ g a = univ
val✝ : Fintype ι
t : (a : ι) → Set (π a)
i : Finset ι
ht : ∀ (a : ι), a ∈ i → t a ∈ g a
this : TopologicalSpace ((i : ι) → π i) := generateFrom {t | ∃ s, (∀ (a : ι), s a ∈ g a) ∧ t = Set.pi univ s}
f : (i : ι) → π i
hf : f ∈ Set.pi (↑i) t
c : (a : ι) → Set (π a)
hcg : ∀ (a : ι), c a ∈ g a
hfc : ∀ (a : ι), f a ∈ c a
a : ι
h : ¬a ∈ i
⊢ piecewise (↑i) t c a ∈ g a
[PROOFSTEP]
simp [*]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
X : Type u_8
f : X → (i : ι) → π i
⊢ induced f Pi.topologicalSpace = ⨅ (i : ι), induced (fun x => f x i) inferInstance
[PROOFSTEP]
erw [induced_iInf]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
X : Type u_8
f : X → (i : ι) → π i
⊢ ⨅ (i : ι), induced f (induced (fun f => f i) ((fun a => inst✝ a) i)) =
⨅ (i : ι), induced (fun x => f x i) inferInstance
[PROOFSTEP]
simp only [induced_compose]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝¹ : TopologicalSpace α
inst✝ : (i : ι) → TopologicalSpace (π i)
f✝ : α → (i : ι) → π i
X : Type u_8
f : X → (i : ι) → π i
⊢ ⨅ (i : ι), induced ((fun f => f i) ∘ f) (inst✝ i) = ⨅ (i : ι), induced (fun x => f x i) inferInstance
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝³ : TopologicalSpace α
inst✝² : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝¹ : Finite ι
inst✝ : ∀ (i : ι), DiscreteTopology (π i)
x : (i : ι) → π i
⊢ IsOpen {x}
[PROOFSTEP]
rw [← univ_pi_singleton]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
π : ι → Type u_6
κ : Type u_7
inst✝³ : TopologicalSpace α
inst✝² : (i : ι) → TopologicalSpace (π i)
f : α → (i : ι) → π i
inst✝¹ : Finite ι
inst✝ : ∀ (i : ι), DiscreteTopology (π i)
x : (i : ι) → π i
⊢ IsOpen (Set.pi univ fun i => {x i})
[PROOFSTEP]
exact isOpen_set_pi finite_univ fun i _ => (isOpen_discrete {x i})
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set (Sigma σ)
⊢ IsOpen s ↔ ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
[PROOFSTEP]
delta instTopologicalSpaceSigma
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set (Sigma σ)
⊢ IsOpen s ↔ ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
[PROOFSTEP]
rw [isOpen_iSup_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set (Sigma σ)
⊢ (∀ (i : ι), IsOpen s) ↔ ∀ (i : ι), IsOpen (Sigma.mk i ⁻¹' s)
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set (Sigma σ)
⊢ IsClosed s ↔ ∀ (i : ι), IsClosed (Sigma.mk i ⁻¹' s)
[PROOFSTEP]
simp only [← isOpen_compl_iff, isOpen_sigma_iff, preimage_compl]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
⊢ IsOpenMap (Sigma.mk i)
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsOpen s
⊢ IsOpen (Sigma.mk i '' s)
[PROOFSTEP]
rw [isOpen_sigma_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsOpen s
⊢ ∀ (i_1 : ι), IsOpen (Sigma.mk i_1 ⁻¹' (Sigma.mk i '' s))
[PROOFSTEP]
intro j
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsOpen s
j : ι
⊢ IsOpen (Sigma.mk j ⁻¹' (Sigma.mk i '' s))
[PROOFSTEP]
rcases eq_or_ne j i with (rfl | hne)
[GOAL]
case inl
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
j : ι
s : Set (σ j)
hs : IsOpen s
⊢ IsOpen (Sigma.mk j ⁻¹' (Sigma.mk j '' s))
[PROOFSTEP]
rwa [Set.preimage_image_eq _ sigma_mk_injective]
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsOpen s
j : ι
hne : j ≠ i
⊢ IsOpen (Sigma.mk j ⁻¹' (Sigma.mk i '' s))
[PROOFSTEP]
rw [preimage_image_sigmaMk_of_ne hne]
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsOpen s
j : ι
hne : j ≠ i
⊢ IsOpen ∅
[PROOFSTEP]
exact isOpen_empty
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
⊢ IsClosedMap (Sigma.mk i)
[PROOFSTEP]
intro s hs
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsClosed s
⊢ IsClosed (Sigma.mk i '' s)
[PROOFSTEP]
rw [isClosed_sigma_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsClosed s
⊢ ∀ (i_1 : ι), IsClosed (Sigma.mk i_1 ⁻¹' (Sigma.mk i '' s))
[PROOFSTEP]
intro j
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsClosed s
j : ι
⊢ IsClosed (Sigma.mk j ⁻¹' (Sigma.mk i '' s))
[PROOFSTEP]
rcases eq_or_ne j i with (rfl | hne)
[GOAL]
case inl
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
j : ι
s : Set (σ j)
hs : IsClosed s
⊢ IsClosed (Sigma.mk j ⁻¹' (Sigma.mk j '' s))
[PROOFSTEP]
rwa [Set.preimage_image_eq _ sigma_mk_injective]
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsClosed s
j : ι
hne : j ≠ i
⊢ IsClosed (Sigma.mk j ⁻¹' (Sigma.mk i '' s))
[PROOFSTEP]
rw [preimage_image_sigmaMk_of_ne hne]
[GOAL]
case inr
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
i : ι
s : Set (σ i)
hs : IsClosed s
j : ι
hne : j ≠ i
⊢ IsClosed ∅
[PROOFSTEP]
exact isClosed_empty
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
x : Sigma σ
⊢ 𝓝 x = Filter.map (mk x.fst) (𝓝 x.snd)
[PROOFSTEP]
cases x
[GOAL]
case mk
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
fst✝ : ι
snd✝ : σ fst✝
⊢ 𝓝 { fst := fst✝, snd := snd✝ } = Filter.map (mk { fst := fst✝, snd := snd✝ }.fst) (𝓝 { fst := fst✝, snd := snd✝ }.snd)
[PROOFSTEP]
apply Sigma.nhds_mk
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set ι
⊢ IsOpen (Sigma.fst ⁻¹' s)
[PROOFSTEP]
rw [← biUnion_of_singleton s, preimage_iUnion₂]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set ι
⊢ IsOpen (⋃ (i : ι) (_ : i ∈ s), Sigma.fst ⁻¹' {i})
[PROOFSTEP]
simp only [← range_sigmaMk]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
s : Set ι
⊢ IsOpen (⋃ (i : ι) (_ : i ∈ s), range (Sigma.mk i))
[PROOFSTEP]
exact isOpen_biUnion fun _ _ => isOpen_range_sigmaMk
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
⊢ Continuous f ↔ ∀ (i : ι), Continuous fun a => f { fst := i, snd := a }
[PROOFSTEP]
delta instTopologicalSpaceSigma
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
⊢ Continuous f ↔ ∀ (i : ι), Continuous fun a => f { fst := i, snd := a }
[PROOFSTEP]
rw [continuous_iSup_dom]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
⊢ (∀ (i : ι), Continuous f) ↔ ∀ (i : ι), Continuous fun a => f { fst := i, snd := a }
[PROOFSTEP]
exact forall_congr' fun _ => continuous_coinduced_dom
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
⊢ Inducing f ↔ (∀ (i : ι), Inducing (f ∘ Sigma.mk i)) ∧ ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
[PROOFSTEP]
refine ⟨fun h ↦ ⟨fun i ↦ h.comp embedding_sigmaMk.1, fun i ↦ ?_⟩, ?_⟩
[GOAL]
case refine_1
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
h : Inducing f
i : ι
⊢ ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
[PROOFSTEP]
rcases h.isOpen_iff.1 (isOpen_range_sigmaMk (i := i)) with ⟨U, hUo, hU⟩
[GOAL]
case refine_1.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
h : Inducing f
i : ι
U : Set α
hUo : IsOpen U
hU : f ⁻¹' U = range (Sigma.mk i)
⊢ ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
[PROOFSTEP]
refine ⟨U, hUo, ?_⟩
[GOAL]
case refine_1.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
h : Inducing f
i : ι
U : Set α
hUo : IsOpen U
hU : f ⁻¹' U = range (Sigma.mk i)
⊢ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
[PROOFSTEP]
simpa [Set.ext_iff] using hU
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
⊢ ((∀ (i : ι), Inducing (f ∘ Sigma.mk i)) ∧ ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i) →
Inducing f
[PROOFSTEP]
refine fun ⟨h₁, h₂⟩ ↦ inducing_iff_nhds.2 fun ⟨i, x⟩ ↦ ?_
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
x✝¹ : (∀ (i : ι), Inducing (f ∘ Sigma.mk i)) ∧ ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
h₁ : ∀ (i : ι), Inducing (f ∘ Sigma.mk i)
h₂ : ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
x✝ : Sigma σ
i : ι
x : σ i
⊢ 𝓝 { fst := i, snd := x } = comap f (𝓝 (f { fst := i, snd := x }))
[PROOFSTEP]
rw [Sigma.nhds_mk, (h₁ i).nhds_eq_comap, comp_apply, ← comap_comap, map_comap_of_mem]
[GOAL]
case refine_2
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
x✝¹ : (∀ (i : ι), Inducing (f ∘ Sigma.mk i)) ∧ ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
h₁ : ∀ (i : ι), Inducing (f ∘ Sigma.mk i)
h₂ : ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
x✝ : Sigma σ
i : ι
x : σ i
⊢ range (Sigma.mk i) ∈ comap f (𝓝 (f { fst := i, snd := x }))
[PROOFSTEP]
rcases h₂ i with ⟨U, hUo, hU⟩
[GOAL]
case refine_2.intro.intro
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
x✝¹ : (∀ (i : ι), Inducing (f ∘ Sigma.mk i)) ∧ ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
h₁ : ∀ (i : ι), Inducing (f ∘ Sigma.mk i)
h₂ : ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
x✝ : Sigma σ
i : ι
x : σ i
U : Set α
hUo : IsOpen U
hU : ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
⊢ range (Sigma.mk i) ∈ comap f (𝓝 (f { fst := i, snd := x }))
[PROOFSTEP]
filter_upwards [preimage_mem_comap <| hUo.mem_nhds <| (hU _).2 rfl] with y hy
[GOAL]
case h
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
x✝¹ : (∀ (i : ι), Inducing (f ∘ Sigma.mk i)) ∧ ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
h₁ : ∀ (i : ι), Inducing (f ∘ Sigma.mk i)
h₂ : ∀ (i : ι), ∃ U, IsOpen U ∧ ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
x✝ : Sigma σ
i : ι
x : σ i
U : Set α
hUo : IsOpen U
hU : ∀ (x : Sigma σ), f x ∈ U ↔ x.fst = i
y : Sigma σ
hy : y ∈ f ⁻¹' U
⊢ y ∈ range (Sigma.mk i)
[PROOFSTEP]
simpa [hU] using hy
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f₁ : ι → κ
f₂ : (i : ι) → σ i → τ (f₁ i)
⊢ (∀ (i : ι), Continuous fun a => Sigma.map f₁ f₂ { fst := i, snd := a }) ↔ ∀ (i : ι), Continuous (f₂ i)
[PROOFSTEP]
simp only [Sigma.map, embedding_sigmaMk.continuous_iff, comp]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f : Sigma σ → α
⊢ IsOpenMap f ↔ ∀ (i : ι), IsOpenMap fun a => f { fst := i, snd := a }
[PROOFSTEP]
simp only [isOpenMap_iff_nhds_le, Sigma.forall, Sigma.nhds_eq, map_map, comp]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f₁ : ι → κ
f₂ : (i : ι) → σ i → τ (f₁ i)
h₁ : Injective f₁
⊢ Inducing (Sigma.map f₁ f₂) ↔ ∀ (i : ι), Inducing (f₂ i)
[PROOFSTEP]
simp only [inducing_iff_nhds, Sigma.forall, Sigma.nhds_mk, Sigma.map_mk, ← map_sigma_mk_comap h₁,
map_inj sigma_mk_injective]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f₁ : ι → κ
f₂ : (i : ι) → σ i → τ (f₁ i)
h : Injective f₁
⊢ _root_.Embedding (Sigma.map f₁ f₂) ↔ ∀ (i : ι), _root_.Embedding (f₂ i)
[PROOFSTEP]
simp only [embedding_iff, Injective.sigma_map, inducing_sigma_map h, forall_and, h.sigma_map_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
ι : Type u_5
κ : Type u_6
σ : ι → Type u_7
τ : κ → Type u_8
inst✝² : (i : ι) → TopologicalSpace (σ i)
inst✝¹ : (k : κ) → TopologicalSpace (τ k)
inst✝ : TopologicalSpace α
f₁ : ι → κ
f₂ : (i : ι) → σ i → τ (f₁ i)
h : Injective f₁
⊢ OpenEmbedding (Sigma.map f₁ f₂) ↔ ∀ (i : ι), OpenEmbedding (f₂ i)
[PROOFSTEP]
simp only [openEmbedding_iff_embedding_open, isOpenMap_sigma_map, embedding_sigma_map h, forall_and]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
⊢ IsClosed (range down)
[PROOFSTEP]
simp only [ULift.down_surjective.range_eq, isClosed_univ]
[GOAL]
α : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
γ : Set ↑β
hγ : IsOpen γ
hβ : IsOpen β
⊢ IsOpen (Lean.Internal.coeM γ)
[PROOFSTEP]
rcases isOpen_induced_iff.mp hγ with ⟨δ, hδ, rfl⟩
[GOAL]
case intro.intro
α : Type u
β✝ : Type v
γ : Type u_1
δ✝ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
hβ : IsOpen β
δ : Set α
hδ : IsOpen δ
hγ : IsOpen (Subtype.val ⁻¹' δ)
⊢ IsOpen (Lean.Internal.coeM (Subtype.val ⁻¹' δ))
[PROOFSTEP]
convert IsOpen.inter hβ hδ
[GOAL]
case h.e'_3
α : Type u
β✝ : Type v
γ : Type u_1
δ✝ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
hβ : IsOpen β
δ : Set α
hδ : IsOpen δ
hγ : IsOpen (Subtype.val ⁻¹' δ)
⊢ Lean.Internal.coeM (Subtype.val ⁻¹' δ) = β ∩ δ
[PROOFSTEP]
ext
[GOAL]
case h.e'_3.h
α : Type u
β✝ : Type v
γ : Type u_1
δ✝ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
hβ : IsOpen β
δ : Set α
hδ : IsOpen δ
hγ : IsOpen (Subtype.val ⁻¹' δ)
x✝ : α
⊢ x✝ ∈ Lean.Internal.coeM (Subtype.val ⁻¹' δ) ↔ x✝ ∈ β ∩ δ
[PROOFSTEP]
exact ⟨fun h => ⟨coe_subset h, mem_of_mem_coe h⟩, fun ⟨hβ, hδ⟩ => mem_coe_of_mem hβ hδ⟩
[GOAL]
α : Type u
β✝ : Type v
γ✝ : Type u_1
δ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
γ : Set ↑β
hγ : IsClosed γ
hβ : IsClosed β
⊢ IsClosed (Lean.Internal.coeM γ)
[PROOFSTEP]
rcases isClosed_induced_iff.mp hγ with ⟨δ, hδ, rfl⟩
[GOAL]
case intro.intro
α : Type u
β✝ : Type v
γ : Type u_1
δ✝ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
hβ : IsClosed β
δ : Set α
hδ : IsClosed δ
hγ : IsClosed (Subtype.val ⁻¹' δ)
⊢ IsClosed (Lean.Internal.coeM (Subtype.val ⁻¹' δ))
[PROOFSTEP]
convert IsClosed.inter hβ hδ
[GOAL]
case h.e'_3
α : Type u
β✝ : Type v
γ : Type u_1
δ✝ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
hβ : IsClosed β
δ : Set α
hδ : IsClosed δ
hγ : IsClosed (Subtype.val ⁻¹' δ)
⊢ Lean.Internal.coeM (Subtype.val ⁻¹' δ) = β ∩ δ
[PROOFSTEP]
ext
[GOAL]
case h.e'_3.h
α : Type u
β✝ : Type v
γ : Type u_1
δ✝ : Type u_2
ε : Type u_3
ζ : Type u_4
inst✝ : TopologicalSpace α
β : Set α
hβ : IsClosed β
δ : Set α
hδ : IsClosed δ
hγ : IsClosed (Subtype.val ⁻¹' δ)
x✝ : α
⊢ x✝ ∈ Lean.Internal.coeM (Subtype.val ⁻¹' δ) ↔ x✝ ∈ β ∩ δ
[PROOFSTEP]
exact ⟨fun h => ⟨coe_subset h, mem_of_mem_coe h⟩, fun ⟨hβ, hδ⟩ => mem_coe_of_mem hβ hδ⟩
| {"mathlib_filename": "Mathlib.Topology.Constructions", "llama_tokens": 67119} |
[GOAL]
α : Type u
g : Set (Set α)
a : α
⊢ 𝓝 a = ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s
[PROOFSTEP]
letI := generateFrom g
[GOAL]
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
⊢ 𝓝 a = ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s
[PROOFSTEP]
rw [nhds_def]
[GOAL]
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ IsOpen s}), 𝓟 s = ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s
[PROOFSTEP]
refine le_antisymm (biInf_mono fun s ⟨as, sg⟩ => ⟨as, .basic _ sg⟩) ?_
[GOAL]
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ IsOpen s}), 𝓟 s
[PROOFSTEP]
refine le_iInf₂ fun s ⟨ha, hs⟩ => ?_
[GOAL]
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
x✝ : s ∈ {s | a ∈ s ∧ IsOpen s}
ha : a ∈ s
hs : IsOpen s
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s
[PROOFSTEP]
clear ‹s ∈ {s | a ∈ s ∧ IsOpen s}›
[GOAL]
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
ha : a ∈ s
hs : IsOpen s
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s
[PROOFSTEP]
induction hs with
| basic _ hs => exact iInf₂_le _ ⟨ha, hs⟩
| univ => exact le_top.trans_eq principal_univ.symm
| inter _ _ _ _ hs ht => exact (le_inf (hs ha.1) (ht ha.2)).trans_eq inf_principal
| sUnion _ _ hS =>
let ⟨t, htS, hat⟩ := ha
exact (hS t htS hat).trans (principal_mono.2 <| subset_sUnion_of_mem htS)
[GOAL]
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
ha : a ∈ s
hs : IsOpen s
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s
[PROOFSTEP]
induction hs with
| basic _ hs => exact iInf₂_le _ ⟨ha, hs⟩
| univ => exact le_top.trans_eq principal_univ.symm
| inter _ _ _ _ hs ht => exact (le_inf (hs ha.1) (ht ha.2)).trans_eq inf_principal
| sUnion _ _ hS =>
let ⟨t, htS, hat⟩ := ha
exact (hS t htS hat).trans (principal_mono.2 <| subset_sUnion_of_mem htS)
[GOAL]
case basic
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s s✝ : Set α
hs : s✝ ∈ g
ha : a ∈ s✝
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s✝
[PROOFSTEP]
| basic _ hs => exact iInf₂_le _ ⟨ha, hs⟩
[GOAL]
case basic
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s s✝ : Set α
hs : s✝ ∈ g
ha : a ∈ s✝
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s✝
[PROOFSTEP]
exact iInf₂_le _ ⟨ha, hs⟩
[GOAL]
case univ
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
ha : a ∈ univ
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 univ
[PROOFSTEP]
| univ => exact le_top.trans_eq principal_univ.symm
[GOAL]
case univ
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
ha : a ∈ univ
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 univ
[PROOFSTEP]
exact le_top.trans_eq principal_univ.symm
[GOAL]
case inter
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s s✝ t✝ : Set α
a✝¹ : GenerateOpen g s✝
a✝ : GenerateOpen g t✝
hs : a ∈ s✝ → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s✝
ht : a ∈ t✝ → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 t✝
ha : a ∈ s✝ ∩ t✝
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 (s✝ ∩ t✝)
[PROOFSTEP]
| inter _ _ _ _ hs ht => exact (le_inf (hs ha.1) (ht ha.2)).trans_eq inf_principal
[GOAL]
case inter
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s s✝ t✝ : Set α
a✝¹ : GenerateOpen g s✝
a✝ : GenerateOpen g t✝
hs : a ∈ s✝ → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s✝
ht : a ∈ t✝ → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 t✝
ha : a ∈ s✝ ∩ t✝
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 (s✝ ∩ t✝)
[PROOFSTEP]
exact (le_inf (hs ha.1) (ht ha.2)).trans_eq inf_principal
[GOAL]
case sUnion
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
S✝ : Set (Set α)
a✝ : ∀ (s : Set α), s ∈ S✝ → GenerateOpen g s
hS : ∀ (s : Set α), s ∈ S✝ → a ∈ s → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s
ha : a ∈ ⋃₀ S✝
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 (⋃₀ S✝)
[PROOFSTEP]
| sUnion _ _ hS =>
let ⟨t, htS, hat⟩ := ha
exact (hS t htS hat).trans (principal_mono.2 <| subset_sUnion_of_mem htS)
[GOAL]
case sUnion
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
S✝ : Set (Set α)
a✝ : ∀ (s : Set α), s ∈ S✝ → GenerateOpen g s
hS : ∀ (s : Set α), s ∈ S✝ → a ∈ s → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s
ha : a ∈ ⋃₀ S✝
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 (⋃₀ S✝)
[PROOFSTEP]
let ⟨t, htS, hat⟩ := ha
[GOAL]
case sUnion
α : Type u
g : Set (Set α)
a : α
this : TopologicalSpace α := generateFrom g
s : Set α
S✝ : Set (Set α)
a✝ : ∀ (s : Set α), s ∈ S✝ → GenerateOpen g s
hS : ∀ (s : Set α), s ∈ S✝ → a ∈ s → ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 s
ha : a ∈ ⋃₀ S✝
t : Set α
htS : t ∈ S✝
hat : a ∈ t
⊢ ⨅ (s : Set α) (_ : s ∈ {s | a ∈ s ∧ s ∈ g}), 𝓟 s ≤ 𝓟 (⋃₀ S✝)
[PROOFSTEP]
exact (hS t htS hat).trans (principal_mono.2 <| subset_sUnion_of_mem htS)
[GOAL]
α : Type u
β : Type u_1
m : α → β
f : Filter α
g : Set (Set β)
b : β
h : ∀ (s : Set β), s ∈ g → b ∈ s → m ⁻¹' s ∈ f
⊢ Tendsto m f (𝓝 b)
[PROOFSTEP]
rw [nhds_generateFrom]
[GOAL]
α : Type u
β : Type u_1
m : α → β
f : Filter α
g : Set (Set β)
b : β
h : ∀ (s : Set β), s ∈ g → b ∈ s → m ⁻¹' s ∈ f
⊢ Tendsto m f (⨅ (s : Set β) (_ : s ∈ {s | b ∈ s ∧ s ∈ g}), 𝓟 s)
[PROOFSTEP]
exact tendsto_iInf.2 fun s => tendsto_iInf.2 fun ⟨hbs, hsg⟩ => tendsto_principal.2 <| h s hsg hbs
[GOAL]
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
⊢ 𝓝 a = n a
[PROOFSTEP]
letI := TopologicalSpace.mkOfNhds n
[GOAL]
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
⊢ 𝓝 a = n a
[PROOFSTEP]
apply le_antisymm
[GOAL]
case a
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
⊢ 𝓝 a ≤ n a
[PROOFSTEP]
intros s hs
[GOAL]
case a
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
⊢ n a ≤ 𝓝 a
[PROOFSTEP]
intros s hs
[GOAL]
case a
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ n a
⊢ s ∈ 𝓝 a
[PROOFSTEP]
have h₀ : {b | s ∈ n b} ⊆ s := fun b hb => mem_pure.1 <| h₀ b hb
[GOAL]
case a
α : Type u
n : α → Filter α
a : α
h₀✝ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ n a
h₀ : {b | s ∈ n b} ⊆ s
⊢ s ∈ 𝓝 a
[PROOFSTEP]
have h₁ : {b | s ∈ n b} ∈ 𝓝 a :=
by
refine' IsOpen.mem_nhds (fun b (hb : s ∈ n b) => _) hs
rcases h₁ _ _ hb with ⟨t, ht, -, h⟩
exact mem_of_superset ht h
[GOAL]
α : Type u
n : α → Filter α
a : α
h₀✝ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ n a
h₀ : {b | s ∈ n b} ⊆ s
⊢ {b | s ∈ n b} ∈ 𝓝 a
[PROOFSTEP]
refine' IsOpen.mem_nhds (fun b (hb : s ∈ n b) => _) hs
[GOAL]
α : Type u
n : α → Filter α
a : α
h₀✝ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ n a
h₀ : {b | s ∈ n b} ⊆ s
b : α
hb : s ∈ n b
⊢ {b | s ∈ n b} ∈ n b
[PROOFSTEP]
rcases h₁ _ _ hb with ⟨t, ht, -, h⟩
[GOAL]
case intro.intro.intro
α : Type u
n : α → Filter α
a : α
h₀✝ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ n a
h₀ : {b | s ∈ n b} ⊆ s
b : α
hb : s ∈ n b
t : Set α
ht : t ∈ n b
h : ∀ (a' : α), a' ∈ t → s ∈ n a'
⊢ {b | s ∈ n b} ∈ n b
[PROOFSTEP]
exact mem_of_superset ht h
[GOAL]
case a
α : Type u
n : α → Filter α
a : α
h₀✝ : pure ≤ n
h₁✝ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ n a
h₀ : {b | s ∈ n b} ⊆ s
h₁ : {b | s ∈ n b} ∈ 𝓝 a
⊢ s ∈ 𝓝 a
[PROOFSTEP]
exact mem_of_superset h₁ h₀
[GOAL]
case a
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ 𝓝 a
⊢ s ∈ n a
[PROOFSTEP]
rcases mem_nhds_iff.1 hs with ⟨t, hts, ht, hat⟩
[GOAL]
case a.intro.intro.intro
α : Type u
n : α → Filter α
a : α
h₀ : pure ≤ n
h₁ : ∀ (a : α) (s : Set α), s ∈ n a → ∃ t, t ∈ n a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ n a'
this : TopologicalSpace α := TopologicalSpace.mkOfNhds n
s : Set α
hs : s ∈ 𝓝 a
t : Set α
hts : t ⊆ s
ht : IsOpen t
hat : a ∈ t
⊢ s ∈ n a
[PROOFSTEP]
exact (n a).sets_of_superset (ht _ hat) hts
[GOAL]
α : Type u
inst✝ : DecidableEq α
a₀ : α
l : Filter α
h : pure a₀ ≤ l
b : α
⊢ 𝓝 b = update pure a₀ l b
[PROOFSTEP]
refine' nhds_mkOfNhds _ _ (le_update_iff.mpr ⟨h, fun _ _ => le_rfl⟩) fun a s hs => _
[GOAL]
α : Type u
inst✝ : DecidableEq α
a₀ : α
l : Filter α
h : pure a₀ ≤ l
b a : α
s : Set α
hs : s ∈ update pure a₀ l a
⊢ ∃ t, t ∈ update pure a₀ l a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ update pure a₀ l a'
[PROOFSTEP]
rcases eq_or_ne a a₀ with (rfl | ha)
[GOAL]
case inl
α : Type u
inst✝ : DecidableEq α
l : Filter α
b a : α
s : Set α
h : pure a ≤ l
hs : s ∈ update pure a l a
⊢ ∃ t, t ∈ update pure a l a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ update pure a l a'
[PROOFSTEP]
refine' ⟨s, hs, Subset.rfl, fun b hb => _⟩
[GOAL]
case inl
α : Type u
inst✝ : DecidableEq α
l : Filter α
b✝ a : α
s : Set α
h : pure a ≤ l
hs : s ∈ update pure a l a
b : α
hb : b ∈ s
⊢ s ∈ update pure a l b
[PROOFSTEP]
rcases eq_or_ne b a with (rfl | hb)
[GOAL]
case inl.inl
α : Type u
inst✝ : DecidableEq α
l : Filter α
b✝ : α
s : Set α
b : α
hb : b ∈ s
h : pure b ≤ l
hs : s ∈ update pure b l b
⊢ s ∈ update pure b l b
[PROOFSTEP]
exact hs
[GOAL]
case inl.inr
α : Type u
inst✝ : DecidableEq α
l : Filter α
b✝ a : α
s : Set α
h : pure a ≤ l
hs : s ∈ update pure a l a
b : α
hb✝ : b ∈ s
hb : b ≠ a
⊢ s ∈ update pure a l b
[PROOFSTEP]
rwa [update_noteq hb]
[GOAL]
case inr
α : Type u
inst✝ : DecidableEq α
a₀ : α
l : Filter α
h : pure a₀ ≤ l
b a : α
s : Set α
hs : s ∈ update pure a₀ l a
ha : a ≠ a₀
⊢ ∃ t, t ∈ update pure a₀ l a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ update pure a₀ l a'
[PROOFSTEP]
have hs' := hs
[GOAL]
case inr
α : Type u
inst✝ : DecidableEq α
a₀ : α
l : Filter α
h : pure a₀ ≤ l
b a : α
s : Set α
hs : s ∈ update pure a₀ l a
ha : a ≠ a₀
hs' : s ∈ update pure a₀ l a
⊢ ∃ t, t ∈ update pure a₀ l a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ update pure a₀ l a'
[PROOFSTEP]
rw [update_noteq ha] at hs ⊢
[GOAL]
case inr
α : Type u
inst✝ : DecidableEq α
a₀ : α
l : Filter α
h : pure a₀ ≤ l
b a : α
s : Set α
hs : s ∈ pure a
ha : a ≠ a₀
hs' : s ∈ update pure a₀ l a
⊢ ∃ t, t ∈ pure a ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ update pure a₀ l a'
[PROOFSTEP]
exact ⟨{ a }, rfl, singleton_subset_iff.mpr hs, forall_eq.2 hs'⟩
[GOAL]
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
⊢ 𝓝 a = FilterBasis.filter (B a)
[PROOFSTEP]
rw [TopologicalSpace.nhds_mkOfNhds]
[GOAL]
case h₀
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
⊢ pure ≤ fun x => FilterBasis.filter (B x)
[PROOFSTEP]
intro x n hn
[GOAL]
case h₁
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
⊢ ∀ (a : α) (s : Set α),
s ∈ FilterBasis.filter (B a) →
∃ t, t ∈ FilterBasis.filter (B a) ∧ t ⊆ s ∧ ∀ (a' : α), a' ∈ t → s ∈ FilterBasis.filter (B a')
[PROOFSTEP]
intro x n hn
[GOAL]
case h₀
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ (fun x => FilterBasis.filter (B x)) x
⊢ n ∈ pure x
[PROOFSTEP]
obtain ⟨m, hm₁, hm₂⟩ := (B x).mem_filter_iff.mp hn
[GOAL]
case h₁
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ FilterBasis.filter (B x)
⊢ ∃ t, t ∈ FilterBasis.filter (B x) ∧ t ⊆ n ∧ ∀ (a' : α), a' ∈ t → n ∈ FilterBasis.filter (B a')
[PROOFSTEP]
obtain ⟨m, hm₁, hm₂⟩ := (B x).mem_filter_iff.mp hn
[GOAL]
case h₀.intro.intro
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ (fun x => FilterBasis.filter (B x)) x
m : Set α
hm₁ : m ∈ B x
hm₂ : m ⊆ n
⊢ n ∈ pure x
[PROOFSTEP]
exact hm₂ (h₀ _ _ hm₁)
[GOAL]
case h₁.intro.intro
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ FilterBasis.filter (B x)
m : Set α
hm₁ : m ∈ B x
hm₂ : m ⊆ n
⊢ ∃ t, t ∈ FilterBasis.filter (B x) ∧ t ⊆ n ∧ ∀ (a' : α), a' ∈ t → n ∈ FilterBasis.filter (B a')
[PROOFSTEP]
obtain ⟨n₁, hn₁, hn₂, hn₃⟩ := h₁ x m hm₁
[GOAL]
case h₁.intro.intro.intro.intro.intro
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ FilterBasis.filter (B x)
m : Set α
hm₁ : m ∈ B x
hm₂ : m ⊆ n
n₁ : Set α
hn₁ : n₁ ∈ B x
hn₂ : n₁ ⊆ m
hn₃ : ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ m
⊢ ∃ t, t ∈ FilterBasis.filter (B x) ∧ t ⊆ n ∧ ∀ (a' : α), a' ∈ t → n ∈ FilterBasis.filter (B a')
[PROOFSTEP]
refine' ⟨n₁, (B x).mem_filter_of_mem hn₁, hn₂.trans hm₂, fun x' hx' => (B x').mem_filter_iff.mp _⟩
[GOAL]
case h₁.intro.intro.intro.intro.intro
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ FilterBasis.filter (B x)
m : Set α
hm₁ : m ∈ B x
hm₂ : m ⊆ n
n₁ : Set α
hn₁ : n₁ ∈ B x
hn₂ : n₁ ⊆ m
hn₃ : ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ m
x' : α
hx' : x' ∈ n₁
⊢ n ∈ FilterBasis.filter (B x')
[PROOFSTEP]
obtain ⟨n₂, hn₄, hn₅⟩ := hn₃ x' hx'
[GOAL]
case h₁.intro.intro.intro.intro.intro.intro.intro
α : Type u
B : α → FilterBasis α
a : α
h₀ : ∀ (x : α) (n : Set α), n ∈ B x → x ∈ n
h₁ : ∀ (x : α) (n : Set α), n ∈ B x → ∃ n₁, n₁ ∈ B x ∧ n₁ ⊆ n ∧ ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ n
x : α
n : Set α
hn : n ∈ FilterBasis.filter (B x)
m : Set α
hm₁ : m ∈ B x
hm₂ : m ⊆ n
n₁ : Set α
hn₁ : n₁ ∈ B x
hn₂ : n₁ ⊆ m
hn₃ : ∀ (x' : α), x' ∈ n₁ → ∃ n₂, n₂ ∈ B x' ∧ n₂ ⊆ m
x' : α
hx' : x' ∈ n₁
n₂ : Set α
hn₄ : n₂ ∈ B x'
hn₅ : n₂ ⊆ m
⊢ n ∈ FilterBasis.filter (B x')
[PROOFSTEP]
exact ⟨n₂, hn₄, hn₅.trans hm₂⟩
[GOAL]
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
h : IsOpen U
⊢ U = ∅ ∨ U = univ
[PROOFSTEP]
induction h with
| basic _ h => exact False.elim h
| univ => exact .inr rfl
| inter _ _ _ _ h₁ h₂ => rcases h₁ with (rfl | rfl) <;> rcases h₂ with (rfl | rfl) <;> simp
| sUnion _ _ ih => exact sUnion_mem_empty_univ ih
[GOAL]
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
h : IsOpen U
⊢ U = ∅ ∨ U = univ
[PROOFSTEP]
induction h with
| basic _ h => exact False.elim h
| univ => exact .inr rfl
| inter _ _ _ _ h₁ h₂ => rcases h₁ with (rfl | rfl) <;> rcases h₂ with (rfl | rfl) <;> simp
| sUnion _ _ ih => exact sUnion_mem_empty_univ ih
[GOAL]
case basic
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U s✝ : Set α
h : s✝ ∈ ↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)
⊢ s✝ = ∅ ∨ s✝ = univ
[PROOFSTEP]
| basic _ h => exact False.elim h
[GOAL]
case basic
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U s✝ : Set α
h : s✝ ∈ ↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)
⊢ s✝ = ∅ ∨ s✝ = univ
[PROOFSTEP]
exact False.elim h
[GOAL]
case univ
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
⊢ univ = ∅ ∨ univ = univ
[PROOFSTEP]
| univ => exact .inr rfl
[GOAL]
case univ
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
⊢ univ = ∅ ∨ univ = univ
[PROOFSTEP]
exact .inr rfl
[GOAL]
case inter
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U s✝ t✝ : Set α
a✝¹ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) s✝
a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) t✝
h₁ : s✝ = ∅ ∨ s✝ = univ
h₂ : t✝ = ∅ ∨ t✝ = univ
⊢ s✝ ∩ t✝ = ∅ ∨ s✝ ∩ t✝ = univ
[PROOFSTEP]
| inter _ _ _ _ h₁ h₂ => rcases h₁ with (rfl | rfl) <;> rcases h₂ with (rfl | rfl) <;> simp
[GOAL]
case inter
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U s✝ t✝ : Set α
a✝¹ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) s✝
a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) t✝
h₁ : s✝ = ∅ ∨ s✝ = univ
h₂ : t✝ = ∅ ∨ t✝ = univ
⊢ s✝ ∩ t✝ = ∅ ∨ s✝ ∩ t✝ = univ
[PROOFSTEP]
rcases h₁ with (rfl | rfl)
[GOAL]
case inter.inl
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U t✝ : Set α
a✝¹ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) t✝
h₂ : t✝ = ∅ ∨ t✝ = univ
a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) ∅
⊢ ∅ ∩ t✝ = ∅ ∨ ∅ ∩ t✝ = univ
[PROOFSTEP]
rcases h₂ with (rfl | rfl)
[GOAL]
case inter.inr
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U t✝ : Set α
a✝¹ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) t✝
h₂ : t✝ = ∅ ∨ t✝ = univ
a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) univ
⊢ univ ∩ t✝ = ∅ ∨ univ ∩ t✝ = univ
[PROOFSTEP]
rcases h₂ with (rfl | rfl)
[GOAL]
case inter.inl.inl
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
a✝¹ a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) ∅
⊢ ∅ ∩ ∅ = ∅ ∨ ∅ ∩ ∅ = univ
[PROOFSTEP]
simp
[GOAL]
case inter.inl.inr
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
a✝¹ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) ∅
a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) univ
⊢ ∅ ∩ univ = ∅ ∨ ∅ ∩ univ = univ
[PROOFSTEP]
simp
[GOAL]
case inter.inr.inl
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
a✝¹ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) univ
a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) ∅
⊢ univ ∩ ∅ = ∅ ∨ univ ∩ ∅ = univ
[PROOFSTEP]
simp
[GOAL]
case inter.inr.inr
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
a✝¹ a✝ : GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) univ
⊢ univ ∩ univ = ∅ ∨ univ ∩ univ = univ
[PROOFSTEP]
simp
[GOAL]
case sUnion
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
S✝ : Set (Set α)
a✝ : ∀ (s : Set α), s ∈ S✝ → GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) s
ih : ∀ (s : Set α), s ∈ S✝ → s = ∅ ∨ s = univ
⊢ ⋃₀ S✝ = ∅ ∨ ⋃₀ S✝ = univ
[PROOFSTEP]
| sUnion _ _ ih => exact sUnion_mem_empty_univ ih
[GOAL]
case sUnion
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
S✝ : Set (Set α)
a✝ : ∀ (s : Set α), s ∈ S✝ → GenerateOpen (↑OrderDual.ofDual (↑OrderDual.ofDual ⊥)) s
ih : ∀ (s : Set α), s ∈ S✝ → s = ∅ ∨ s = univ
⊢ ⋃₀ S✝ = ∅ ∨ ⋃₀ S✝ = univ
[PROOFSTEP]
exact sUnion_mem_empty_univ ih
[GOAL]
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
U : Set α
⊢ U = ∅ ∨ U = univ → IsOpen U
[PROOFSTEP]
rintro (rfl | rfl)
[GOAL]
case inl
α✝ : Type ?u.10996
t t₁ t₂ : TopologicalSpace α✝
s : Set α✝
α : Type u_1
⊢ IsOpen ∅
case inr α✝ : Type ?u.10996 t t₁ t₂ : TopologicalSpace α✝ s : Set α✝ α : Type u_1 ⊢ IsOpen univ
[PROOFSTEP]
exacts [@isOpen_empty _ ⊤, @isOpen_univ _ ⊤]
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s✝ : Set α
inst✝¹ : TopologicalSpace α
inst✝ : DiscreteTopology α
s : Set α
⊢ Dense s ↔ s = univ
[PROOFSTEP]
simp [dense_iff_closure_eq]
[GOAL]
α : Type u_2
t t₁ t₂ : TopologicalSpace α
s : Set α
inst✝¹ : TopologicalSpace α
inst✝ : DiscreteTopology α
ι : Type u_1
f : ι → α
⊢ DenseRange f ↔ Surjective f
[PROOFSTEP]
rw [DenseRange, dense_discrete, range_iff_surjective]
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s✝ : Set α
inst✝¹ : TopologicalSpace α
inst✝ : DiscreteTopology α
x : α
s : Set α
⊢ s ∈ 𝓝 x ↔ x ∈ s
[PROOFSTEP]
rw [nhds_discrete, mem_pure]
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s✝ : Set α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
s : Set α
⊢ IsOpen s → IsOpen s
[PROOFSTEP]
rw [@isOpen_iff_mem_nhds _ t₁, @isOpen_iff_mem_nhds α t₂]
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s✝ : Set α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
s : Set α
⊢ (∀ (a : α), a ∈ s → s ∈ 𝓝 a) → ∀ (a : α), a ∈ s → s ∈ 𝓝 a
[PROOFSTEP]
exact fun hs a ha => h _ (hs _ ha)
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s : Set α
inst✝ : TopologicalSpace α
⊢ DiscreteTopology α ↔ ∀ (x : α), {x} ∈ 𝓝 x
[PROOFSTEP]
simp only [← singletons_open_iff_discrete, isOpen_iff_mem_nhds, mem_singleton_iff, forall_eq]
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s : Set α
inst✝ : TopologicalSpace α
⊢ DiscreteTopology α ↔ ∀ (x : α), 𝓝 x = pure x
[PROOFSTEP]
simp only [discreteTopology_iff_singleton_mem_nhds, ← nhds_neBot.le_pure_iff, le_pure_iff]
[GOAL]
α : Type u_1
t t₁ t₂ : TopologicalSpace α
s : Set α
inst✝ : TopologicalSpace α
⊢ DiscreteTopology α ↔ ∀ (x : α), 𝓝[{x}ᶜ] x = ⊥
[PROOFSTEP]
simp only [discreteTopology_iff_singleton_mem_nhds, nhdsWithin, inf_principal_eq_bot, compl_compl]
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace β
⊢ ∀ (s t_1 : Set α),
(fun s => ∃ s', IsOpen s' ∧ f ⁻¹' s' = s) s →
(fun s => ∃ s', IsOpen s' ∧ f ⁻¹' s' = s) t_1 → (fun s => ∃ s', IsOpen s' ∧ f ⁻¹' s' = s) (s ∩ t_1)
[PROOFSTEP]
rintro s₁ s₂ ⟨s'₁, hs₁, rfl⟩ ⟨s'₂, hs₂, rfl⟩
[GOAL]
case intro.intro.intro.intro
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace β
s'₁ : Set β
hs₁ : IsOpen s'₁
s'₂ : Set β
hs₂ : IsOpen s'₂
⊢ ∃ s', IsOpen s' ∧ f ⁻¹' s' = f ⁻¹' s'₁ ∩ f ⁻¹' s'₂
[PROOFSTEP]
exact ⟨s'₁ ∩ s'₂, hs₁.inter hs₂, preimage_inter⟩
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace β
S : Set (Set α)
h : ∀ (t_1 : Set α), t_1 ∈ S → (fun s => ∃ s', IsOpen s' ∧ f ⁻¹' s' = s) t_1
⊢ (fun s => ∃ s', IsOpen s' ∧ f ⁻¹' s' = s) (⋃₀ S)
[PROOFSTEP]
choose! g hgo hfg using h
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace β
S : Set (Set α)
g : Set α → Set β
hgo : ∀ (t_1 : Set α), t_1 ∈ S → IsOpen (g t_1)
hfg : ∀ (t : Set α), t ∈ S → f ⁻¹' g t = t
⊢ ∃ s', IsOpen s' ∧ f ⁻¹' s' = ⋃₀ S
[PROOFSTEP]
refine ⟨⋃ s ∈ S, g s, isOpen_biUnion fun s hs => hgo s hs, ?_⟩
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace β
S : Set (Set α)
g : Set α → Set β
hgo : ∀ (t_1 : Set α), t_1 ∈ S → IsOpen (g t_1)
hfg : ∀ (t : Set α), t ∈ S → f ⁻¹' g t = t
⊢ f ⁻¹' ⋃ (s : Set α) (_ : s ∈ S), g s = ⋃₀ S
[PROOFSTEP]
rw [preimage_iUnion₂, sUnion_eq_biUnion]
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace β
S : Set (Set α)
g : Set α → Set β
hgo : ∀ (t_1 : Set α), t_1 ∈ S → IsOpen (g t_1)
hfg : ∀ (t : Set α), t ∈ S → f ⁻¹' g t = t
⊢ ⋃ (i : Set α) (_ : i ∈ S), f ⁻¹' g i = ⋃ (i : Set α) (_ : i ∈ S), i
[PROOFSTEP]
exact iUnion₂_congr hfg
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
t : TopologicalSpace β
s : Set α
f : α → β
⊢ IsClosed s ↔ ∃ t_1, IsClosed t_1 ∧ f ⁻¹' t_1 = s
[PROOFSTEP]
letI := t.induced f
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
t : TopologicalSpace β
s : Set α
f : α → β
this : TopologicalSpace α := TopologicalSpace.induced f t
⊢ IsClosed s ↔ ∃ t_1, IsClosed t_1 ∧ f ⁻¹' t_1 = s
[PROOFSTEP]
simp only [← isOpen_compl_iff, isOpen_induced_iff]
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
t : TopologicalSpace β
s : Set α
f : α → β
this : TopologicalSpace α := TopologicalSpace.induced f t
⊢ (∃ t_1, IsOpen t_1 ∧ f ⁻¹' t_1 = sᶜ) ↔ ∃ t_1, IsOpen t_1ᶜ ∧ f ⁻¹' t_1 = s
[PROOFSTEP]
exact compl_surjective.exists.trans (by simp only [preimage_compl, compl_inj_iff])
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
t : TopologicalSpace β
s : Set α
f : α → β
this : TopologicalSpace α := TopologicalSpace.induced f t
⊢ (∃ x, IsOpen xᶜ ∧ f ⁻¹' xᶜ = sᶜ) ↔ ∃ t_1, IsOpen t_1ᶜ ∧ f ⁻¹' t_1 = s
[PROOFSTEP]
simp only [preimage_compl, compl_inj_iff]
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
α : Type u
β : Type v
f : α → β
t : TopologicalSpace α
s : Set (Set β)
h : ∀ (t_1 : Set β), t_1 ∈ s → (fun s => IsOpen (f ⁻¹' s)) t_1
⊢ (fun s => IsOpen (f ⁻¹' s)) (⋃₀ s)
[PROOFSTEP]
simpa only [preimage_sUnion] using isOpen_biUnion h
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝ : TopologicalSpace α
π : α → β
s : Set β
a : α
hs : s ∈ 𝓝 (π a)
⊢ π ⁻¹' s ∈ 𝓝 a
[PROOFSTEP]
letI := TopologicalSpace.coinduced π ‹_›
[GOAL]
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝ : TopologicalSpace α
π : α → β
s : Set β
a : α
hs : s ∈ 𝓝 (π a)
this : TopologicalSpace β := TopologicalSpace.coinduced π inst✝
⊢ π ⁻¹' s ∈ 𝓝 a
[PROOFSTEP]
rcases mem_nhds_iff.mp hs with ⟨V, hVs, V_op, mem_V⟩
[GOAL]
case intro.intro.intro
α : Type u_1
β : Type u_2
γ : Type u_3
inst✝ : TopologicalSpace α
π : α → β
s : Set β
a : α
hs : s ∈ 𝓝 (π a)
this : TopologicalSpace β := TopologicalSpace.coinduced π inst✝
V : Set β
hVs : V ⊆ s
V_op : IsOpen V
mem_V : π a ∈ V
⊢ π ⁻¹' s ∈ 𝓝 a
[PROOFSTEP]
exact mem_nhds_iff.mpr ⟨π ⁻¹' V, Set.preimage_mono hVs, V_op, mem_V⟩
[GOAL]
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
t t₁ t₂ : TopologicalSpace α✝
t' : TopologicalSpace β✝
f : α✝ → β✝
g : β✝ → α✝
α : Type u_4
β : Type u_5
e : α ≃ β
⊢ TopologicalSpace.induced ↑e.symm = TopologicalSpace.coinduced ↑e
[PROOFSTEP]
ext t U
[GOAL]
case h.a.h.a
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
t✝ t₁ t₂ : TopologicalSpace α✝
t' : TopologicalSpace β✝
f : α✝ → β✝
g : β✝ → α✝
α : Type u_4
β : Type u_5
e : α ≃ β
t : TopologicalSpace α
U : Set β
⊢ IsOpen U ↔ IsOpen U
[PROOFSTEP]
rw [isOpen_induced_iff, isOpen_coinduced]
[GOAL]
case h.a.h.a
α✝ : Type u_1
β✝ : Type u_2
γ : Type u_3
t✝ t₁ t₂ : TopologicalSpace α✝
t' : TopologicalSpace β✝
f : α✝ → β✝
g : β✝ → α✝
α : Type u_4
β : Type u_5
e : α ≃ β
t : TopologicalSpace α
U : Set β
⊢ (∃ t_1, IsOpen t_1 ∧ ↑e.symm ⁻¹' t_1 = U) ↔ IsOpen (↑e ⁻¹' U)
[PROOFSTEP]
simp only [e.symm.preimage_eq_iff_eq_image, exists_eq_right, ← preimage_equiv_eq_image_symm]
[GOAL]
α✝ : Type u
β✝ : Type v
α : Type u_1
β : Type u_2
t : TopologicalSpace α
b : Set (Set β)
f : α → β
h : ∀ (a : Set β), a ∈ b → IsOpen (f ⁻¹' a)
⊢ t ≤ induced f (generateFrom b)
[PROOFSTEP]
rw [induced_generateFrom_eq]
[GOAL]
α✝ : Type u
β✝ : Type v
α : Type u_1
β : Type u_2
t : TopologicalSpace α
b : Set (Set β)
f : α → β
h : ∀ (a : Set β), a ∈ b → IsOpen (f ⁻¹' a)
⊢ t ≤ generateFrom (preimage f '' b)
[PROOFSTEP]
apply le_generateFrom
[GOAL]
case h
α✝ : Type u
β✝ : Type v
α : Type u_1
β : Type u_2
t : TopologicalSpace α
b : Set (Set β)
f : α → β
h : ∀ (a : Set β), a ∈ b → IsOpen (f ⁻¹' a)
⊢ ∀ (s : Set α), s ∈ preimage f '' b → IsOpen s
[PROOFSTEP]
simp only [mem_image, and_imp, forall_apply_eq_imp_iff₂, exists_imp]
[GOAL]
case h
α✝ : Type u
β✝ : Type v
α : Type u_1
β : Type u_2
t : TopologicalSpace α
b : Set (Set β)
f : α → β
h : ∀ (a : Set β), a ∈ b → IsOpen (f ⁻¹' a)
⊢ ∀ (a : Set β), a ∈ b → IsOpen (f ⁻¹' a)
[PROOFSTEP]
exact h
[GOAL]
α : Type u
β : Type v
a : α
f : Filter α
t : TopologicalSpace α
⊢ nhdsAdjoint a f ≤ t ↔ f ≤ (fun t => 𝓝 a) t
[PROOFSTEP]
rw [le_nhds_iff]
[GOAL]
α : Type u
β : Type v
a : α
f : Filter α
t : TopologicalSpace α
⊢ nhdsAdjoint a f ≤ t ↔ ∀ (s : Set α), a ∈ s → IsOpen s → s ∈ f
[PROOFSTEP]
exact ⟨fun H s hs has => H _ has hs, fun H s has hs => H _ hs has⟩
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
⊢ 𝓝 a = pure a ⊔ f
[PROOFSTEP]
letI := nhdsAdjoint a f
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
⊢ 𝓝 a = pure a ⊔ f
[PROOFSTEP]
ext U
[GOAL]
case a
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
⊢ U ∈ 𝓝 a ↔ U ∈ pure a ⊔ f
[PROOFSTEP]
rw [mem_nhds_iff]
[GOAL]
case a
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
⊢ (∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t) ↔ U ∈ pure a ⊔ f
[PROOFSTEP]
constructor
[GOAL]
case a.mp
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
⊢ (∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t) → U ∈ pure a ⊔ f
[PROOFSTEP]
rintro ⟨t, htU, ht, hat⟩
[GOAL]
case a.mp.intro.intro.intro
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
U t : Set α
htU : t ⊆ U
ht : IsOpen t
hat : a ∈ t
⊢ U ∈ pure a ⊔ f
[PROOFSTEP]
exact ⟨htU hat, mem_of_superset (ht hat) htU⟩
[GOAL]
case a.mpr
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
⊢ U ∈ pure a ⊔ f → ∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t
[PROOFSTEP]
rintro ⟨haU, hU⟩
[GOAL]
case a.mpr.intro
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
haU : U ∈ (pure a).sets
hU : U ∈ f.sets
⊢ ∃ t, t ⊆ U ∧ IsOpen t ∧ a ∈ t
[PROOFSTEP]
exact ⟨U, Subset.rfl, fun _ => hU, haU⟩
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
⊢ 𝓝 b = pure b
[PROOFSTEP]
letI := nhdsAdjoint a f
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
⊢ 𝓝 b = pure b
[PROOFSTEP]
apply le_antisymm
[GOAL]
case a
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
⊢ 𝓝 b ≤ pure b
[PROOFSTEP]
intro U hU
[GOAL]
case a
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
hU : U ∈ pure b
⊢ U ∈ 𝓝 b
[PROOFSTEP]
rw [mem_nhds_iff]
[GOAL]
case a
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
hU : U ∈ pure b
⊢ ∃ t, t ⊆ U ∧ IsOpen t ∧ b ∈ t
[PROOFSTEP]
use{ b }
[GOAL]
case h
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
hU : U ∈ pure b
⊢ {b} ⊆ U ∧ IsOpen {b} ∧ b ∈ {b}
[PROOFSTEP]
simp only [and_true_iff, singleton_subset_iff, mem_singleton]
[GOAL]
case h
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
U : Set α
hU : U ∈ pure b
⊢ b ∈ U ∧ IsOpen {b}
[PROOFSTEP]
refine' ⟨hU, fun ha => (h.symm ha).elim⟩
[GOAL]
case a
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
b : α
h : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
⊢ pure b ≤ 𝓝 b
[PROOFSTEP]
exact @pure_le_nhds α (nhdsAdjoint a f) b
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a b : α
f : Filter α
hb : b ≠ a
⊢ IsOpen {b}
[PROOFSTEP]
letI := nhdsAdjoint a f
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a b : α
f : Filter α
hb : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
⊢ IsOpen {b}
[PROOFSTEP]
rw [isOpen_singleton_iff_nhds_eq_pure]
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a b : α
f : Filter α
hb : b ≠ a
this : TopologicalSpace α := nhdsAdjoint a f
⊢ 𝓝 b = pure b
[PROOFSTEP]
exact nhdsAdjoint_nhds_of_ne a f hb
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ t ≤ nhdsAdjoint a f ↔ 𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → 𝓝 b = pure b
[PROOFSTEP]
rw [le_iff_nhds]
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ (∀ (x : α), 𝓝 x ≤ 𝓝 x) ↔ 𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → 𝓝 b = pure b
[PROOFSTEP]
constructor
[GOAL]
case mp
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ (∀ (x : α), 𝓝 x ≤ 𝓝 x) → 𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → 𝓝 b = pure b
[PROOFSTEP]
intro h
[GOAL]
case mp
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
⊢ 𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → 𝓝 b = pure b
[PROOFSTEP]
constructor
[GOAL]
case mp.left
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
⊢ 𝓝 a ≤ pure a ⊔ f
[PROOFSTEP]
specialize h a
[GOAL]
case mp.left
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : 𝓝 a ≤ 𝓝 a
⊢ 𝓝 a ≤ pure a ⊔ f
[PROOFSTEP]
rwa [nhdsAdjoint_nhds] at h
[GOAL]
case mp.right
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
⊢ ∀ (b : α), b ≠ a → 𝓝 b = pure b
[PROOFSTEP]
intro b hb
[GOAL]
case mp.right
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
b : α
hb : b ≠ a
⊢ 𝓝 b = pure b
[PROOFSTEP]
apply le_antisymm _ (pure_le_nhds b)
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : ∀ (x : α), 𝓝 x ≤ 𝓝 x
b : α
hb : b ≠ a
⊢ 𝓝 b ≤ pure b
[PROOFSTEP]
specialize h b
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
b : α
hb : b ≠ a
h : 𝓝 b ≤ 𝓝 b
⊢ 𝓝 b ≤ pure b
[PROOFSTEP]
rwa [nhdsAdjoint_nhds_of_ne a f hb] at h
[GOAL]
case mpr
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ (𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → 𝓝 b = pure b) → ∀ (x : α), 𝓝 x ≤ 𝓝 x
[PROOFSTEP]
rintro ⟨h, h'⟩ b
[GOAL]
case mpr.intro
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : 𝓝 a ≤ pure a ⊔ f
h' : ∀ (b : α), b ≠ a → 𝓝 b = pure b
b : α
⊢ 𝓝 b ≤ 𝓝 b
[PROOFSTEP]
by_cases hb : b = a
[GOAL]
case pos
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : 𝓝 a ≤ pure a ⊔ f
h' : ∀ (b : α), b ≠ a → 𝓝 b = pure b
b : α
hb : b = a
⊢ 𝓝 b ≤ 𝓝 b
[PROOFSTEP]
rwa [hb, nhdsAdjoint_nhds]
[GOAL]
case neg
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
h : 𝓝 a ≤ pure a ⊔ f
h' : ∀ (b : α), b ≠ a → 𝓝 b = pure b
b : α
hb : ¬b = a
⊢ 𝓝 b ≤ 𝓝 b
[PROOFSTEP]
simp [nhdsAdjoint_nhds_of_ne a f hb, h' b hb]
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ t ≤ nhdsAdjoint a f ↔ 𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → IsOpen {b}
[PROOFSTEP]
change _ ↔ _ ∧ ∀ b : α, b ≠ a → IsOpen { b }
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ t ≤ nhdsAdjoint a f ↔ 𝓝 a ≤ pure a ⊔ f ∧ ∀ (b : α), b ≠ a → IsOpen {b}
[PROOFSTEP]
rw [le_nhdsAdjoint_iff', and_congr_right_iff]
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
⊢ 𝓝 a ≤ pure a ⊔ f → ((∀ (b : α), b ≠ a → 𝓝 b = pure b) ↔ ∀ (b : α), b ≠ a → IsOpen {b})
[PROOFSTEP]
refine fun _ => forall_congr' fun b => ?_
[GOAL]
α✝ : Type u
β : Type v
α : Type u_1
a : α
f : Filter α
t : TopologicalSpace α
x✝ : 𝓝 a ≤ pure a ⊔ f
b : α
⊢ b ≠ a → 𝓝 b = pure b ↔ b ≠ a → IsOpen {b}
[PROOFSTEP]
rw [@isOpen_singleton_iff_nhds_eq_pure α t b]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
g : γ → α
t₂ : TopologicalSpace β
t₁ : TopologicalSpace γ
⊢ Continuous g ↔ Continuous (f ∘ g)
[PROOFSTEP]
simp only [continuous_iff_le_induced, induced_compose]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
g : β → γ
t₁ : TopologicalSpace α
t₂ : TopologicalSpace γ
⊢ Continuous g ↔ Continuous (g ∘ f)
[PROOFSTEP]
simp only [continuous_iff_coinduced_le, coinduced_compose]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ t₂ : TopologicalSpace α
t₃ : TopologicalSpace β
h₁ : t₂ ≤ t₁
h₂ : Continuous f
⊢ Continuous f
[PROOFSTEP]
rw [continuous_iff_le_induced] at h₂ ⊢
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ t₂ : TopologicalSpace α
t₃ : TopologicalSpace β
h₁ : t₂ ≤ t₁
h₂ : t₁ ≤ induced f t₃
⊢ t₂ ≤ induced f t₃
[PROOFSTEP]
exact le_trans h₁ h₂
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ : TopologicalSpace α
t₂ t₃ : TopologicalSpace β
h₁ : t₂ ≤ t₃
h₂ : Continuous f
⊢ Continuous f
[PROOFSTEP]
rw [continuous_iff_coinduced_le] at h₂ ⊢
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ : TopologicalSpace α
t₂ t₃ : TopologicalSpace β
h₁ : t₂ ≤ t₃
h₂ : coinduced f t₁ ≤ t₂
⊢ coinduced f t₁ ≤ t₃
[PROOFSTEP]
exact le_trans h₂ h₁
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ t₂ : TopologicalSpace α
t₃ : TopologicalSpace β
⊢ Continuous f ↔ Continuous f ∧ Continuous f
[PROOFSTEP]
simp only [continuous_iff_le_induced, sup_le_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
T : Set (TopologicalSpace α)
t₂ : TopologicalSpace β
⊢ Continuous f ↔ ∀ (t : TopologicalSpace α), t ∈ T → Continuous f
[PROOFSTEP]
simp only [continuous_iff_le_induced, sSup_le_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ : ι → TopologicalSpace α
t₂ : TopologicalSpace β
⊢ Continuous f ↔ ∀ (i : ι), Continuous f
[PROOFSTEP]
simp only [continuous_iff_le_induced, iSup_le_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ : TopologicalSpace α
t₂ t₃ : TopologicalSpace β
⊢ Continuous f ↔ Continuous f ∧ Continuous f
[PROOFSTEP]
simp only [continuous_iff_coinduced_le, le_inf_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ : TopologicalSpace α
T : Set (TopologicalSpace β)
⊢ Continuous f ↔ ∀ (t : TopologicalSpace β), t ∈ T → Continuous f
[PROOFSTEP]
simp only [continuous_iff_coinduced_le, le_sInf_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f : α → β
ι : Sort u_2
t₁ : TopologicalSpace α
t₂ : ι → TopologicalSpace β
⊢ Continuous f ↔ ∀ (i : ι), Continuous f
[PROOFSTEP]
simp only [continuous_iff_coinduced_le, le_iInf_iff]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
⊢ s ∈ 𝓝 a ↔ ∃ u, u ∈ 𝓝 (f a) ∧ f ⁻¹' u ⊆ s
[PROOFSTEP]
letI := T.induced f
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
this : TopologicalSpace β := induced f T
⊢ s ∈ 𝓝 a ↔ ∃ u, u ∈ 𝓝 (f a) ∧ f ⁻¹' u ⊆ s
[PROOFSTEP]
simp only [mem_nhds_iff, isOpen_induced_iff, exists_prop, Set.mem_setOf_eq]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
this : TopologicalSpace β := induced f T
⊢ (∃ t, t ⊆ s ∧ (∃ t_1, IsOpen t_1 ∧ f ⁻¹' t_1 = t) ∧ a ∈ t) ↔ ∃ u, (∃ t, t ⊆ u ∧ IsOpen t ∧ f a ∈ t) ∧ f ⁻¹' u ⊆ s
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
this : TopologicalSpace β := induced f T
⊢ (∃ t, t ⊆ s ∧ (∃ t_1, IsOpen t_1 ∧ f ⁻¹' t_1 = t) ∧ a ∈ t) → ∃ u, (∃ t, t ⊆ u ∧ IsOpen t ∧ f a ∈ t) ∧ f ⁻¹' u ⊆ s
[PROOFSTEP]
rintro ⟨u, usub, ⟨v, openv, rfl⟩, au⟩
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
this : TopologicalSpace β := induced f T
v : Set α
openv : IsOpen v
usub : f ⁻¹' v ⊆ s
au : a ∈ f ⁻¹' v
⊢ ∃ u, (∃ t, t ⊆ u ∧ IsOpen t ∧ f a ∈ t) ∧ f ⁻¹' u ⊆ s
[PROOFSTEP]
exact ⟨v, ⟨v, Subset.rfl, openv, au⟩, usub⟩
[GOAL]
case mpr
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
this : TopologicalSpace β := induced f T
⊢ (∃ u, (∃ t, t ⊆ u ∧ IsOpen t ∧ f a ∈ t) ∧ f ⁻¹' u ⊆ s) → ∃ t, t ⊆ s ∧ (∃ t_1, IsOpen t_1 ∧ f ⁻¹' t_1 = t) ∧ a ∈ t
[PROOFSTEP]
rintro ⟨u, ⟨v, vsubu, openv, amem⟩, finvsub⟩
[GOAL]
case mpr.intro.intro.intro.intro.intro
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
this : TopologicalSpace β := induced f T
u : Set α
finvsub : f ⁻¹' u ⊆ s
v : Set α
vsubu : v ⊆ u
openv : IsOpen v
amem : f a ∈ v
⊢ ∃ t, t ⊆ s ∧ (∃ t_1, IsOpen t_1 ∧ f ⁻¹' t_1 = t) ∧ a ∈ t
[PROOFSTEP]
exact ⟨f ⁻¹' v, (Set.preimage_mono vsubu).trans finvsub, ⟨⟨v, openv, rfl⟩, amem⟩⟩
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
⊢ 𝓝 a = comap f (𝓝 (f a))
[PROOFSTEP]
ext s
[GOAL]
case a
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
a : β
s : Set β
⊢ s ∈ 𝓝 a ↔ s ∈ comap f (𝓝 (f a))
[PROOFSTEP]
rw [mem_nhds_induced, mem_comap]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
tα : TopologicalSpace α
tβ : TopologicalSpace β
f : β → α
h : ∀ (b : β), 𝓝 b = comap f (𝓝 (f b))
x : β
⊢ 𝓝 x = 𝓝 x
[PROOFSTEP]
rw [h, nhds_induced]
[GOAL]
α : Type u
β : Type v
γ : Type u_1
f✝ : α → β
ι : Sort u_2
T : TopologicalSpace α
f : β → α
hf : Surjective f
a : β
⊢ map f (𝓝 a) = 𝓝 (f a)
[PROOFSTEP]
rw [nhds_induced, map_comap_of_surjective hf]
[GOAL]
α : Type u_1
β : Type u_2
t : TopologicalSpace β
f : α → β
a : α
⊢ map f (𝓝 a) = 𝓝[range f] f a
[PROOFSTEP]
rw [nhds_induced, Filter.map_comap, nhdsWithin]
[GOAL]
α : Type u_1
β : Type u_2
t : TopologicalSpace β
f : α → β
a : α
h : range f ∈ 𝓝 (f a)
⊢ map f (𝓝 a) = 𝓝 (f a)
[PROOFSTEP]
rw [nhds_induced, Filter.map_comap_of_mem h]
[GOAL]
α : Type u_1
β : Type u_2
t✝ : TopologicalSpace β
f✝ : α → β
t : TopologicalSpace β
f : α → β
a : α
s : Set α
⊢ a ∈ closure s ↔ f a ∈ closure (f '' s)
[PROOFSTEP]
letI := t.induced f
[GOAL]
α : Type u_1
β : Type u_2
t✝ : TopologicalSpace β
f✝ : α → β
t : TopologicalSpace β
f : α → β
a : α
s : Set α
this : TopologicalSpace α := induced f t
⊢ a ∈ closure s ↔ f a ∈ closure (f '' s)
[PROOFSTEP]
simp only [mem_closure_iff_frequently, nhds_induced, frequently_comap, mem_image, and_comm]
[GOAL]
α : Type u_1
β : Type u_2
t✝ : TopologicalSpace β
f✝ : α → β
t : TopologicalSpace β
f : α → β
s : Set α
⊢ IsClosed s ↔ ∀ (a : α), f a ∈ closure (f '' s) → a ∈ s
[PROOFSTEP]
letI := t.induced f
[GOAL]
α : Type u_1
β : Type u_2
t✝ : TopologicalSpace β
f✝ : α → β
t : TopologicalSpace β
f : α → β
s : Set α
this : TopologicalSpace α := induced f t
⊢ IsClosed s ↔ ∀ (a : α), f a ∈ closure (f '' s) → a ∈ s
[PROOFSTEP]
simp only [← closure_subset_iff_isClosed, subset_def, closure_induced]
[GOAL]
α : Type u_1
inst✝ : TopologicalSpace α
⊢ ⨅ (s : Set Prop) (_ : s ∈ {s | False ∈ s ∧ s ∈ {{True}}}), 𝓟 s = ⊤
[PROOFSTEP]
simp [@and_comm (_ ∈ _)]
[GOAL]
α : Type u_1
inst✝ : TopologicalSpace α
l : Filter α
p : α → Prop
⊢ Tendsto p l (𝓝 True) ↔ ∀ᶠ (x : α) in l, p x
[PROOFSTEP]
simp
[GOAL]
α : Type u_1
inst✝ : TopologicalSpace α
l : Filter α
p : α → Prop
q : Prop
⊢ Tendsto p l (𝓝 q) ↔ q → ∀ᶠ (x : α) in l, p x
[PROOFSTEP]
by_cases q
[GOAL]
α : Type u_1
inst✝ : TopologicalSpace α
l : Filter α
p : α → Prop
q : Prop
⊢ Tendsto p l (𝓝 q) ↔ q → ∀ᶠ (x : α) in l, p x
[PROOFSTEP]
by_cases q
[GOAL]
case pos
α : Type u_1
inst✝ : TopologicalSpace α
l : Filter α
p : α → Prop
q : Prop
h : q
⊢ Tendsto p l (𝓝 q) ↔ q → ∀ᶠ (x : α) in l, p x
[PROOFSTEP]
simp [*]
[GOAL]
case neg
α : Type u_1
inst✝ : TopologicalSpace α
l : Filter α
p : α → Prop
q : Prop
h : ¬q
⊢ Tendsto p l (𝓝 q) ↔ q → ∀ᶠ (x : α) in l, p x
[PROOFSTEP]
simp [*]
[GOAL]
α : Type u_1
inst✝ : TopologicalSpace α
p : α → Prop
⊢ Continuous p ↔ IsOpen {x | p x}
[PROOFSTEP]
simp only [continuous_iff_continuousAt, ContinuousAt, tendsto_nhds_Prop, isOpen_iff_mem_nhds]
[GOAL]
α : Type u_1
inst✝ : TopologicalSpace α
p : α → Prop
⊢ (∀ (x : α), p x → ∀ᶠ (x : α) in 𝓝 x, p x) ↔ ∀ (a : α), a ∈ {x | p x} → {x | p x} ∈ 𝓝 a
[PROOFSTEP]
rfl
[GOAL]
α : Type u
ι : Sort v
t : ι → TopologicalSpace α
s : Set α
⊢ s ∈ {s | IsOpen s} ↔ s ∈ {x | ∀ (i : ι), IsOpen x}
[PROOFSTEP]
simp [setOf_isOpen_iSup]
[GOAL]
α : Type u
ι : Sort v
t : ι → TopologicalSpace α
s : Set α
⊢ IsClosed s ↔ ∀ (i : ι), IsClosed s
[PROOFSTEP]
simp [← @isOpen_compl_iff _ (⨆ i, t i), ← @isOpen_compl_iff _ (t _), isOpen_iSup_iff]
| {"mathlib_filename": "Mathlib.Topology.Order", "llama_tokens": 24403} |
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
⊢ ∃ v, (∀ (a : ι), IsOpen (v a)) ∧ ⋃ (i : ι), v i = univ ∧ LocallyFinite v ∧ ∀ (a : ι), v a ⊆ u a
[PROOFSTEP]
have :=
ParacompactSpace.locallyFinite_refinement (range u) (fun r ↦ (r : Set X)) (SetCoe.forall.2 <| forall_range_iff.2 uo)
(by rwa [← sUnion_range, Subtype.range_coe])
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
⊢ ⋃ (a : ↑(range u)), (fun r => ↑r) a = univ
[PROOFSTEP]
rwa [← sUnion_range, Subtype.range_coe]
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
this : ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ (fun r => ↑r) a
⊢ ∃ v, (∀ (a : ι), IsOpen (v a)) ∧ ⋃ (i : ι), v i = univ ∧ LocallyFinite v ∧ ∀ (a : ι), v a ⊆ u a
[PROOFSTEP]
simp only [SetCoe.exists, exists_range_iff', iUnion_eq_univ_iff, exists_prop] at this
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
this : ∃ β t, (∀ (b : β), IsOpen (t b)) ∧ (∀ (x : X), ∃ i, x ∈ t i) ∧ LocallyFinite t ∧ ∀ (b : β), ∃ i, t b ⊆ u i
⊢ ∃ v, (∀ (a : ι), IsOpen (v a)) ∧ ⋃ (i : ι), v i = univ ∧ LocallyFinite v ∧ ∀ (a : ι), v a ⊆ u a
[PROOFSTEP]
choose α t hto hXt htf ind hind using this
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
hXt : ∀ (x : X), ∃ i, x ∈ t i
htf : LocallyFinite t
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
⊢ ∃ v, (∀ (a : ι), IsOpen (v a)) ∧ ⋃ (i : ι), v i = univ ∧ LocallyFinite v ∧ ∀ (a : ι), v a ⊆ u a
[PROOFSTEP]
choose t_inv ht_inv using hXt
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
htf : LocallyFinite t
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
⊢ ∃ v, (∀ (a : ι), IsOpen (v a)) ∧ ⋃ (i : ι), v i = univ ∧ LocallyFinite v ∧ ∀ (a : ι), v a ⊆ u a
[PROOFSTEP]
choose U hxU hU using htf
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ ∃ v, (∀ (a : ι), IsOpen (v a)) ∧ ⋃ (i : ι), v i = univ ∧ LocallyFinite v ∧ ∀ (a : ι), v a ⊆ u a
[PROOFSTEP]
refine' ⟨fun i ↦ ⋃ (a : α) (_ : ind a = i), t a, _, _, _, _⟩
[GOAL]
case refine'_1
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ ∀ (a : ι), IsOpen ((fun i => ⋃ (a : α) (_ : ind a = i), t a) a)
[PROOFSTEP]
exact fun a ↦ isOpen_iUnion fun a ↦ isOpen_iUnion fun _ ↦ hto a
[GOAL]
case refine'_2
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ ⋃ (i : ι), (fun i => ⋃ (a : α) (_ : ind a = i), t a) i = univ
[PROOFSTEP]
simp only [eq_univ_iff_forall, mem_iUnion]
[GOAL]
case refine'_2
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ ∀ (x : X), ∃ i i_1 i, x ∈ t i_1
[PROOFSTEP]
exact fun x ↦ ⟨ind (t_inv x), _, rfl, ht_inv _⟩
[GOAL]
case refine'_3
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ LocallyFinite fun i => ⋃ (a : α) (_ : ind a = i), t a
[PROOFSTEP]
refine' fun x ↦ ⟨U x, hxU x, ((hU x).image ind).subset _⟩
[GOAL]
case refine'_3
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
x : X
⊢ {i | Set.Nonempty ((fun i => ⋃ (a : α) (_ : ind a = i), t a) i ∩ U x)} ⊆ ind '' {i | Set.Nonempty (t i ∩ U x)}
[PROOFSTEP]
simp only [subset_def, mem_iUnion, mem_setOf_eq, Set.Nonempty, mem_inter_iff]
[GOAL]
case refine'_3
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
x : X
⊢ ∀ (x_1 : ι), (∃ x_2, (∃ i i_1, x_2 ∈ t i) ∧ x_2 ∈ U x) → x_1 ∈ ind '' {i | ∃ x_2, x_2 ∈ t i ∧ x_2 ∈ U x}
[PROOFSTEP]
rintro i ⟨y, ⟨a, rfl, hya⟩, hyU⟩
[GOAL]
case refine'_3.intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
x y : X
hyU : y ∈ U x
a : α
hya : y ∈ t a
⊢ ind a ∈ ind '' {i | ∃ x_1, x_1 ∈ t i ∧ x_1 ∈ U x}
[PROOFSTEP]
exact mem_image_of_mem _ ⟨y, hya, hyU⟩
[GOAL]
case refine'_4
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ ∀ (a : ι), (fun i => ⋃ (a : α) (_ : ind a = i), t a) a ⊆ u a
[PROOFSTEP]
simp only [subset_def, mem_iUnion]
[GOAL]
case refine'_4
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
⊢ ∀ (a : ι) (x : X), (∃ i i_1, x ∈ t i) → x ∈ u a
[PROOFSTEP]
rintro i x ⟨a, rfl, hxa⟩
[GOAL]
case refine'_4.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
u : ι → Set X
uo : ∀ (a : ι), IsOpen (u a)
uc : ⋃ (i : ι), u i = univ
α : Type v
t : α → Set X
hto : ∀ (b : α), IsOpen (t b)
ind : α → ι
hind : ∀ (b : α), t b ⊆ u (ind b)
t_inv : X → α
ht_inv : ∀ (x : X), x ∈ t (t_inv x)
U : X → Set X
hxU : ∀ (x : X), U x ∈ 𝓝 x
hU : ∀ (x : X), Set.Finite {i | Set.Nonempty (t i ∩ U x)}
x : X
a : α
hxa : x ∈ t a
⊢ x ∈ u (ind a)
[PROOFSTEP]
exact hind _ hxa
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
⊢ ∃ v, (∀ (i : ι), IsOpen (v i)) ∧ s ⊆ ⋃ (i : ι), v i ∧ LocallyFinite v ∧ ∀ (i : ι), v i ⊆ u i
[PROOFSTEP]
have uc : (iUnion fun i => Option.elim' sᶜ u i) = univ :=
by
apply Subset.antisymm (subset_univ _)
· simp_rw [← compl_union_self s, Option.elim', iUnion_option]
apply union_subset_union_right sᶜ us
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
⊢ ⋃ (i : Option ι), Option.elim' sᶜ u i = univ
[PROOFSTEP]
apply Subset.antisymm (subset_univ _)
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
⊢ univ ⊆ ⋃ (i : Option ι), Option.elim' sᶜ u i
[PROOFSTEP]
simp_rw [← compl_union_self s, Option.elim', iUnion_option]
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
⊢ sᶜ ∪ s ⊆ sᶜ ∪ ⋃ (a : ι), u a
[PROOFSTEP]
apply union_subset_union_right sᶜ us
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
uc : ⋃ (i : Option ι), Option.elim' sᶜ u i = univ
⊢ ∃ v, (∀ (i : ι), IsOpen (v i)) ∧ s ⊆ ⋃ (i : ι), v i ∧ LocallyFinite v ∧ ∀ (i : ι), v i ⊆ u i
[PROOFSTEP]
rcases precise_refinement (Option.elim' sᶜ u) (Option.forall.2 ⟨isOpen_compl_iff.2 hs, uo⟩) uc with ⟨v, vo, vc, vf, vu⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
uc : ⋃ (i : Option ι), Option.elim' sᶜ u i = univ
v : Option ι → Set X
vo : ∀ (a : Option ι), IsOpen (v a)
vc : ⋃ (i : Option ι), v i = univ
vf : LocallyFinite v
vu : ∀ (a : Option ι), v a ⊆ Option.elim' sᶜ u a
⊢ ∃ v, (∀ (i : ι), IsOpen (v i)) ∧ s ⊆ ⋃ (i : ι), v i ∧ LocallyFinite v ∧ ∀ (i : ι), v i ⊆ u i
[PROOFSTEP]
refine' ⟨v ∘ some, fun i ↦ vo _, _, vf.comp_injective (Option.some_injective _), fun i ↦ vu _⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
uc : ⋃ (i : Option ι), Option.elim' sᶜ u i = univ
v : Option ι → Set X
vo : ∀ (a : Option ι), IsOpen (v a)
vc : ⋃ (i : Option ι), v i = univ
vf : LocallyFinite v
vu : ∀ (a : Option ι), v a ⊆ Option.elim' sᶜ u a
⊢ s ⊆ ⋃ (i : ι), (v ∘ some) i
[PROOFSTEP]
simp only [iUnion_option, ← compl_subset_iff_union] at vc
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace X
s : Set X
hs : IsClosed s
u : ι → Set X
uo : ∀ (i : ι), IsOpen (u i)
us : s ⊆ ⋃ (i : ι), u i
uc : ⋃ (i : Option ι), Option.elim' sᶜ u i = univ
v : Option ι → Set X
vo : ∀ (a : Option ι), IsOpen (v a)
vf : LocallyFinite v
vu : ∀ (a : Option ι), v a ⊆ Option.elim' sᶜ u a
vc : (v none)ᶜ ⊆ ⋃ (i : ι), v (some i)
⊢ s ⊆ ⋃ (i : ι), (v ∘ some) i
[PROOFSTEP]
exact Subset.trans (subset_compl_comm.1 <| vu Option.none) vc
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
choose U hUo hU using fun a ↦ he.isOpen_iff.1 (ho a)
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
U : α → Set Y
hUo : ∀ (a : α), IsOpen (U a)
hU : ∀ (a : α), e ⁻¹' U a = s a
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
simp only [← hU] at hu ⊢
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
U : α → Set Y
hUo : ∀ (a : α), IsOpen (U a)
hU : ∀ (a : α), e ⁻¹' U a = s a
hu : ⋃ (a : α), e ⁻¹' U a = univ
⊢ ∃ β t h h, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ e ⁻¹' U a
[PROOFSTEP]
have heU : range e ⊆ ⋃ i, U i := by simpa only [range_subset_iff, mem_iUnion, iUnion_eq_univ_iff] using hu
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
U : α → Set Y
hUo : ∀ (a : α), IsOpen (U a)
hU : ∀ (a : α), e ⁻¹' U a = s a
hu : ⋃ (a : α), e ⁻¹' U a = univ
⊢ range e ⊆ ⋃ (i : α), U i
[PROOFSTEP]
simpa only [range_subset_iff, mem_iUnion, iUnion_eq_univ_iff] using hu
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
U : α → Set Y
hUo : ∀ (a : α), IsOpen (U a)
hU : ∀ (a : α), e ⁻¹' U a = s a
hu : ⋃ (a : α), e ⁻¹' U a = univ
heU : range e ⊆ ⋃ (i : α), U i
⊢ ∃ β t h h, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ e ⁻¹' U a
[PROOFSTEP]
rcases precise_refinement_set he.closed_range U hUo heU with ⟨V, hVo, heV, hVf, hVU⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
U : α → Set Y
hUo : ∀ (a : α), IsOpen (U a)
hU : ∀ (a : α), e ⁻¹' U a = s a
hu : ⋃ (a : α), e ⁻¹' U a = univ
heU : range e ⊆ ⋃ (i : α), U i
V : α → Set Y
hVo : ∀ (i : α), IsOpen (V i)
heV : range e ⊆ ⋃ (i : α), V i
hVf : LocallyFinite V
hVU : ∀ (i : α), V i ⊆ U i
⊢ ∃ β t h h, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ e ⁻¹' U a
[PROOFSTEP]
refine
⟨α, fun a ↦ e ⁻¹' (V a), fun a ↦ (hVo a).preimage he.continuous, ?_, hVf.preimage_continuous he.continuous, fun a ↦
⟨a, preimage_mono (hVU a)⟩⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : ParacompactSpace Y
e : X → Y
he : ClosedEmbedding e
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
U : α → Set Y
hUo : ∀ (a : α), IsOpen (U a)
hU : ∀ (a : α), e ⁻¹' U a = s a
hu : ⋃ (a : α), e ⁻¹' U a = univ
heU : range e ⊆ ⋃ (i : α), U i
V : α → Set Y
hVo : ∀ (i : α), IsOpen (V i)
heV : range e ⊆ ⋃ (i : α), V i
hVf : LocallyFinite V
hVU : ∀ (i : α), V i ⊆ U i
⊢ ⋃ (b : α), (fun a => e ⁻¹' V a) b = univ
[PROOFSTEP]
simpa only [range_subset_iff, mem_iUnion, iUnion_eq_univ_iff] using heV
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
have : ∀ (x : X) (y : Y), ∃ (a : α) (U : Set X) (V : Set Y), IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ U ×ˢ V ⊆ s a :=
fun x y ↦ (iUnion_eq_univ_iff.1 hu (x, y)).imp fun a ha ↦ isOpen_prod_iff.1 (ho a) x y ha
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
this : ∀ (x : X) (y : Y), ∃ a U V, IsOpen U ∧ IsOpen V ∧ x ∈ U ∧ y ∈ V ∧ U ×ˢ V ⊆ s a
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
choose a U V hUo hVo hxU hyV hUV using this
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
choose T hT using fun y ↦ CompactSpace.elim_nhds_subcover (U · y) fun x ↦ (hUo x y).mem_nhds (hxU x y)
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
set W : Y → Set Y := fun y ↦ ⋂ x ∈ T y, V x y
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
have hWo : ∀ y, IsOpen (W y) := fun y ↦ isOpen_biInter_finset fun _ _ ↦ hVo _ _
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
have hW : ∀ y, y ∈ W y := fun _ ↦ mem_iInter₂.2 fun _ _ ↦ hyV _ _
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
rcases precise_refinement W hWo (iUnion_eq_univ_iff.2 fun y ↦ ⟨y, hW y⟩) with ⟨E, hEo, hE, hEf, hEA⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
refine
⟨Σ y, T y, fun z ↦ U z.2.1 z.1 ×ˢ E z.1, fun _ ↦ (hUo _ _).prod (hEo _), iUnion_eq_univ_iff.2 fun (x, y) ↦ ?_,
fun (x, y) ↦ ?_, fun ⟨y, x, hx⟩ ↦ ?_⟩
[GOAL]
case intro.intro.intro.intro.refine_1
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y : Y
⊢ ∃ i, (x, y) ∈ (fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i
[PROOFSTEP]
rcases iUnion_eq_univ_iff.1 hE y with ⟨b, hb⟩
[GOAL]
case intro.intro.intro.intro.refine_1.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y b : Y
hb : y ∈ E b
⊢ ∃ i, (x, y) ∈ (fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i
[PROOFSTEP]
rcases iUnion₂_eq_univ_iff.1 (hT b) x with ⟨a, ha, hx⟩
[GOAL]
case intro.intro.intro.intro.refine_1.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a✝ : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a✝ x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y b : Y
hb : y ∈ E b
a : X
ha : a ∈ T b
hx : x ∈ U a b
⊢ ∃ i, (x, y) ∈ (fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i
[PROOFSTEP]
exact ⟨⟨b, a, ha⟩, hx, hb⟩
[GOAL]
case intro.intro.intro.intro.refine_2
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y : Y
⊢ ∃ t, t ∈ 𝓝 (x, y) ∧ Set.Finite {i | Set.Nonempty ((fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i ∩ t)}
[PROOFSTEP]
rcases hEf y with ⟨t, ht, htf⟩
[GOAL]
case intro.intro.intro.intro.refine_2.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y : Y
t : Set Y
ht : t ∈ 𝓝 y
htf : Set.Finite {i | Set.Nonempty (E i ∩ t)}
⊢ ∃ t, t ∈ 𝓝 (x, y) ∧ Set.Finite {i | Set.Nonempty ((fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i ∩ t)}
[PROOFSTEP]
refine ⟨univ ×ˢ t, prod_mem_nhds univ_mem ht, ?_⟩
[GOAL]
case intro.intro.intro.intro.refine_2.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y : Y
t : Set Y
ht : t ∈ 𝓝 y
htf : Set.Finite {i | Set.Nonempty (E i ∩ t)}
⊢ Set.Finite {i | Set.Nonempty ((fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i ∩ univ ×ˢ t)}
[PROOFSTEP]
refine (htf.biUnion fun y _ ↦ finite_range (Sigma.mk y)).subset ?_
[GOAL]
case intro.intro.intro.intro.refine_2.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y : Y
t : Set Y
ht : t ∈ 𝓝 y
htf : Set.Finite {i | Set.Nonempty (E i ∩ t)}
⊢ {i | Set.Nonempty ((fun z => U (↑z.snd) z.fst ×ˢ E z.fst) i ∩ univ ×ˢ t)} ⊆
⋃ (i : Y) (_ : i ∈ {i | Set.Nonempty (E i ∩ t)}), range (Sigma.mk i)
[PROOFSTEP]
rintro ⟨b, a, ha⟩ ⟨⟨c, d⟩, ⟨-, hd : d ∈ E b⟩, -, hdt : d ∈ t⟩
[GOAL]
case intro.intro.intro.intro.refine_2.intro.intro.mk.mk.intro.mk.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a✝ : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a✝ x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : X × Y
x : X
y : Y
t : Set Y
ht : t ∈ 𝓝 y
htf : Set.Finite {i | Set.Nonempty (E i ∩ t)}
b : Y
a : X
ha : a ∈ T b
c : X
d : Y
hd : d ∈ E b
hdt : d ∈ t
⊢ { fst := b, snd := { val := a, property := ha } } ∈
⋃ (i : Y) (_ : i ∈ {i | Set.Nonempty (E i ∩ t)}), range (Sigma.mk i)
[PROOFSTEP]
exact mem_iUnion₂.2 ⟨b, ⟨d, hd, hdt⟩, mem_range_self _⟩
[GOAL]
case intro.intro.intro.intro.refine_3
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : (y : Y) × { x // x ∈ T y }
y : Y
x : X
hx : x ∈ T y
⊢ ∃ a, (fun z => U (↑z.snd) z.fst ×ˢ E z.fst) { fst := y, snd := { val := x, property := hx } } ⊆ s a
[PROOFSTEP]
refine ⟨a x y, (Set.prod_mono Subset.rfl ?_).trans (hUV x y)⟩
[GOAL]
case intro.intro.intro.intro.refine_3
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : CompactSpace X
inst✝ : ParacompactSpace Y
α : Type (max v w)
s : α → Set (X × Y)
ho : ∀ (a : α), IsOpen (s a)
hu : ⋃ (a : α), s a = univ
a : X → Y → α
U : X → Y → Set X
V : X → Y → Set Y
hUo : ∀ (x : X) (y : Y), IsOpen (U x y)
hVo : ∀ (x : X) (y : Y), IsOpen (V x y)
hxU : ∀ (x : X) (y : Y), x ∈ U x y
hyV : ∀ (x : X) (y : Y), y ∈ V x y
hUV : ∀ (x : X) (y : Y), U x y ×ˢ V x y ⊆ s (a x y)
T : Y → Finset X
hT : ∀ (y : Y), ⋃ (x : X) (_ : x ∈ T y), U x y = ⊤
W : Y → Set Y := fun y => ⋂ (x : X) (_ : x ∈ T y), V x y
hWo : ∀ (y : Y), IsOpen (W y)
hW : ∀ (y : Y), y ∈ W y
E : Y → Set Y
hEo : ∀ (a : Y), IsOpen (E a)
hE : ⋃ (i : Y), E i = univ
hEf : LocallyFinite E
hEA : ∀ (a : Y), E a ⊆ W a
x✝ : (y : Y) × { x // x ∈ T y }
y : Y
x : X
hx : x ∈ T y
⊢ E { fst := y, snd := { val := x, property := hx } }.fst ⊆ V x y
[PROOFSTEP]
exact (hEA _).trans (iInter₂_subset x hx)
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : CompactSpace X
⊢ ParacompactSpace X
[PROOFSTEP]
refine' ⟨fun ι s ho hu ↦ _⟩
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : CompactSpace X
ι : Type v
s : ι → Set X
ho : ∀ (a : ι), IsOpen (s a)
hu : ⋃ (a : ι), s a = univ
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
rcases isCompact_univ.elim_finite_subcover _ ho hu.ge with ⟨T, hT⟩
[GOAL]
case intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : CompactSpace X
ι : Type v
s : ι → Set X
ho : ∀ (a : ι), IsOpen (s a)
hu : ⋃ (a : ι), s a = univ
T : Finset ι
hT : univ ⊆ ⋃ (i : ι) (_ : i ∈ T), s i
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
refine' ⟨(T : Set ι), fun t ↦ s t, fun t ↦ ho _, _, locallyFinite_of_finite _, fun t ↦ ⟨t, Subset.rfl⟩⟩
[GOAL]
case intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝² : TopologicalSpace X
inst✝¹ : TopologicalSpace Y
inst✝ : CompactSpace X
ι : Type v
s : ι → Set X
ho : ∀ (a : ι), IsOpen (s a)
hu : ⋃ (a : ι), s a = univ
T : Finset ι
hT : univ ⊆ ⋃ (i : ι) (_ : i ∈ T), s i
⊢ ⋃ (b : ↑↑T), (fun t => s ↑t) b = univ
[PROOFSTEP]
simpa only [iUnion_coe_set, ← univ_subset_iff]
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
classical
-- For technical reasons we prepend two empty sets to the sequence `CompactExhaustion.choice X`
set K' : CompactExhaustion X := CompactExhaustion.choice X
set K : CompactExhaustion X := K'.shiftr.shiftr
set Kdiff := fun n ↦
K (n + 1) \
interior
(K n)
-- Now we restate some properties of `CompactExhaustion` for `K`/`Kdiff`
have hKcov : ∀ x, x ∈ Kdiff (K'.find x + 1) := by
intro x
simpa only [K'.find_shiftr] using diff_subset_diff_right interior_subset (K'.shiftr.mem_diff_shiftr_find x)
have Kdiffc : ∀ n, IsCompact (Kdiff n ∩ s) := fun n ↦ ((K.isCompact _).diff isOpen_interior).inter_right hs
have : ∀ (n) (x : ↑(Kdiff (n + 1) ∩ s)), (K n)ᶜ ∈ 𝓝 (x : X) := fun n x ↦
IsOpen.mem_nhds (K.isClosed n).isOpen_compl fun hx' ↦ x.2.1.2 <| K.subset_interior_succ _ hx'
choose! r hrp hr using fun n (x : ↑(Kdiff (n + 1) ∩ s)) ↦ (hB x x.2.2).mem_iff.1 (this n x)
have hxr : ∀ (n x) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n ⟨x, hx⟩) ∈ 𝓝 x := fun n x hx ↦
(hB x hx.2).mem_of_mem (hrp _ ⟨x, hx⟩)
choose T hT using fun n ↦ (Kdiffc (n + 1)).elim_nhds_subcover' _ (hxr n)
set T' : ∀ n, Set ↑(Kdiff (n + 1) ∩ s) := fun n ↦ T n
refine' ⟨Σ n, T' n, fun a ↦ a.2, fun a ↦ r a.1 a.2, _, _, _⟩
· rintro ⟨n, x, hx⟩
exact ⟨x.2.2, hrp _ _⟩
· refine' fun x hx ↦ mem_iUnion.2 _
rcases mem_iUnion₂.1 (hT _ ⟨hKcov x, hx⟩) with ⟨⟨c, hc⟩, hcT, hcx⟩
exact ⟨⟨_, ⟨c, hc⟩, hcT⟩, hcx⟩
· intro x
refine' ⟨interior (K (K'.find x + 3)), IsOpen.mem_nhds isOpen_interior (K.subset_interior_succ _ (hKcov x).1), _⟩
have : (⋃ k ≤ K'.find x + 2, range (Sigma.mk k) : Set (Σ n, T' n)).Finite :=
(finite_le_nat _).biUnion fun k _ ↦ finite_range _
apply this.subset
rintro ⟨k, c, hc⟩
simp only [mem_iUnion, mem_setOf_eq, mem_image, Subtype.coe_mk]
rintro ⟨x, hxB : x ∈ B c (r k c), hxK⟩
refine' ⟨k, _, ⟨c, hc⟩, rfl⟩
have := (mem_compl_iff _ _).1 (hr k c hxB)
contrapose! this with hnk
exact K.subset hnk (interior_subset hxK)
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
set K' : CompactExhaustion X := CompactExhaustion.choice X
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
set K : CompactExhaustion X := K'.shiftr.shiftr
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
set Kdiff := fun n ↦
K (n + 1) \
interior
(K n)
-- Now we restate some properties of `CompactExhaustion` for `K`/`Kdiff`
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
have hKcov : ∀ x, x ∈ Kdiff (K'.find x + 1) := by
intro x
simpa only [K'.find_shiftr] using diff_subset_diff_right interior_subset (K'.shiftr.mem_diff_shiftr_find x)
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
⊢ ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
[PROOFSTEP]
intro x
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
x : X
⊢ x ∈ Kdiff (CompactExhaustion.find K' x + 1)
[PROOFSTEP]
simpa only [K'.find_shiftr] using diff_subset_diff_right interior_subset (K'.shiftr.mem_diff_shiftr_find x)
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
have Kdiffc : ∀ n, IsCompact (Kdiff n ∩ s) := fun n ↦ ((K.isCompact _).diff isOpen_interior).inter_right hs
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
have : ∀ (n) (x : ↑(Kdiff (n + 1) ∩ s)), (K n)ᶜ ∈ 𝓝 (x : X) := fun n x ↦
IsOpen.mem_nhds (K.isClosed n).isOpen_compl fun hx' ↦ x.2.1.2 <| K.subset_interior_succ _ hx'
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
choose! r hrp hr using fun n (x : ↑(Kdiff (n + 1) ∩ s)) ↦ (hB x x.2.2).mem_iff.1 (this n x)
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
have hxr : ∀ (n x) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n ⟨x, hx⟩) ∈ 𝓝 x := fun n x hx ↦
(hB x hx.2).mem_of_mem (hrp _ ⟨x, hx⟩)
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
choose T hT using fun n ↦ (Kdiffc (n + 1)).elim_nhds_subcover' _ (hxr n)
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
set T' : ∀ n, Set ↑(Kdiff (n + 1) ∩ s) := fun n ↦ T n
[GOAL]
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
⊢ ∃ α c r, (∀ (a : α), c a ∈ s ∧ p (c a) (r a)) ∧ s ⊆ ⋃ (a : α), B (c a) (r a) ∧ LocallyFinite fun a => B (c a) (r a)
[PROOFSTEP]
refine' ⟨Σ n, T' n, fun a ↦ a.2, fun a ↦ r a.1 a.2, _, _, _⟩
[GOAL]
case refine'_1
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
⊢ ∀ (a : (n : ℕ) × ↑(T' n)), (fun a => ↑↑a.snd) a ∈ s ∧ p ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)
[PROOFSTEP]
rintro ⟨n, x, hx⟩
[GOAL]
case refine'_1.mk.mk
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
n : ℕ
x : ↑(Kdiff (n + 1) ∩ s)
hx : x ∈ T' n
⊢ (fun a => ↑↑a.snd) { fst := n, snd := { val := x, property := hx } } ∈ s ∧
p ((fun a => ↑↑a.snd) { fst := n, snd := { val := x, property := hx } })
((fun a => r a.fst ↑a.snd) { fst := n, snd := { val := x, property := hx } })
[PROOFSTEP]
exact ⟨x.2.2, hrp _ _⟩
[GOAL]
case refine'_2
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
⊢ s ⊆ ⋃ (a : (n : ℕ) × ↑(T' n)), B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)
[PROOFSTEP]
refine' fun x hx ↦ mem_iUnion.2 _
[GOAL]
case refine'_2
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
hx : x ∈ s
⊢ ∃ i, x ∈ B ((fun a => ↑↑a.snd) i) ((fun a => r a.fst ↑a.snd) i)
[PROOFSTEP]
rcases mem_iUnion₂.1 (hT _ ⟨hKcov x, hx⟩) with ⟨⟨c, hc⟩, hcT, hcx⟩
[GOAL]
case refine'_2.intro.mk.intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
hx : x ∈ s
c : X
hc : c ∈ Kdiff (CompactExhaustion.find K' x + 1) ∩ s
hcT : { val := c, property := hc } ∈ T (CompactExhaustion.find K' x)
hcx :
x ∈
B (↑{ val := c, property := hc })
(r (CompactExhaustion.find K' x)
{ val := ↑{ val := c, property := hc },
property := (_ : ↑{ val := c, property := hc } ∈ Kdiff (CompactExhaustion.find K' x + 1) ∩ s) })
⊢ ∃ i, x ∈ B ((fun a => ↑↑a.snd) i) ((fun a => r a.fst ↑a.snd) i)
[PROOFSTEP]
exact ⟨⟨_, ⟨c, hc⟩, hcT⟩, hcx⟩
[GOAL]
case refine'_3
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
⊢ LocallyFinite fun a => B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)
[PROOFSTEP]
intro x
[GOAL]
case refine'_3
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
⊢ ∃ t, t ∈ 𝓝 x ∧ Set.Finite {i | Set.Nonempty ((fun a => B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)) i ∩ t)}
[PROOFSTEP]
refine' ⟨interior (K (K'.find x + 3)), IsOpen.mem_nhds isOpen_interior (K.subset_interior_succ _ (hKcov x).1), _⟩
[GOAL]
case refine'_3
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
⊢ Set.Finite
{i |
Set.Nonempty
((fun a => B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)) i ∩
interior (↑K (CompactExhaustion.find K' x + 3)))}
[PROOFSTEP]
have : (⋃ k ≤ K'.find x + 2, range (Sigma.mk k) : Set (Σ n, T' n)).Finite :=
(finite_le_nat _).biUnion fun k _ ↦ finite_range _
[GOAL]
case refine'_3
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x + 2), range (Sigma.mk k))
⊢ Set.Finite
{i |
Set.Nonempty
((fun a => B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)) i ∩
interior (↑K (CompactExhaustion.find K' x + 3)))}
[PROOFSTEP]
apply this.subset
[GOAL]
case refine'_3
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x + 2), range (Sigma.mk k))
⊢ {i |
Set.Nonempty
((fun a => B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)) i ∩
interior (↑K (CompactExhaustion.find K' x + 3)))} ⊆
⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x + 2), range (Sigma.mk k)
[PROOFSTEP]
rintro ⟨k, c, hc⟩
[GOAL]
case refine'_3.mk.mk
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x + 2), range (Sigma.mk k))
k : ℕ
c : ↑(Kdiff (k + 1) ∩ s)
hc : c ∈ T' k
⊢ { fst := k, snd := { val := c, property := hc } } ∈
{i |
Set.Nonempty
((fun a => B ((fun a => ↑↑a.snd) a) ((fun a => r a.fst ↑a.snd) a)) i ∩
interior (↑K (CompactExhaustion.find K' x + 3)))} →
{ fst := k, snd := { val := c, property := hc } } ∈
⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x + 2), range (Sigma.mk k)
[PROOFSTEP]
simp only [mem_iUnion, mem_setOf_eq, mem_image, Subtype.coe_mk]
[GOAL]
case refine'_3.mk.mk
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x + 2), range (Sigma.mk k))
k : ℕ
c : ↑(Kdiff (k + 1) ∩ s)
hc : c ∈ T' k
⊢ Set.Nonempty
(B (↑c) (r k c) ∩
interior
(↑(CompactExhaustion.shiftr (CompactExhaustion.shiftr (CompactExhaustion.choice X)))
(CompactExhaustion.find (CompactExhaustion.choice X) x + 3))) →
∃ i i_1, { fst := k, snd := { val := c, property := hc } } ∈ range (Sigma.mk i)
[PROOFSTEP]
rintro ⟨x, hxB : x ∈ B c (r k c), hxK⟩
[GOAL]
case refine'_3.mk.mk.intro.intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x✝ : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x✝ + 2), range (Sigma.mk k))
k : ℕ
c : ↑(Kdiff (k + 1) ∩ s)
hc : c ∈ T' k
x : X
hxB : x ∈ B (↑c) (r k c)
hxK :
x ∈
interior
(↑(CompactExhaustion.shiftr (CompactExhaustion.shiftr (CompactExhaustion.choice X)))
(CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 3))
⊢ ∃ i i_1, { fst := k, snd := { val := c, property := hc } } ∈ range (Sigma.mk i)
[PROOFSTEP]
refine' ⟨k, _, ⟨c, hc⟩, rfl⟩
[GOAL]
case refine'_3.mk.mk.intro.intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x✝ : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x✝ + 2), range (Sigma.mk k))
k : ℕ
c : ↑(Kdiff (k + 1) ∩ s)
hc : c ∈ T' k
x : X
hxB : x ∈ B (↑c) (r k c)
hxK :
x ∈
interior
(↑(CompactExhaustion.shiftr (CompactExhaustion.shiftr (CompactExhaustion.choice X)))
(CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 3))
⊢ k ≤ CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 2
[PROOFSTEP]
have := (mem_compl_iff _ _).1 (hr k c hxB)
[GOAL]
case refine'_3.mk.mk.intro.intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝¹ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x✝ : X
this✝ : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x✝ + 2), range (Sigma.mk k))
k : ℕ
c : ↑(Kdiff (k + 1) ∩ s)
hc : c ∈ T' k
x : X
hxB : x ∈ B (↑c) (r k c)
hxK :
x ∈
interior
(↑(CompactExhaustion.shiftr (CompactExhaustion.shiftr (CompactExhaustion.choice X)))
(CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 3))
this : ¬x ∈ ↑K k
⊢ k ≤ CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 2
[PROOFSTEP]
contrapose! this with hnk
[GOAL]
case refine'_3.mk.mk.intro.intro
ι✝ : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
ι : X → Type u
p : (x : X) → ι x → Prop
B : (x : X) → ι x → Set X
s : Set X
hs : IsClosed s
hB : ∀ (x : X), x ∈ s → HasBasis (𝓝 x) (p x) (B x)
K' : CompactExhaustion X := CompactExhaustion.choice X
K : CompactExhaustion X := CompactExhaustion.shiftr (CompactExhaustion.shiftr K')
Kdiff : (n : ℕ) → (fun x => Set X) (n + 1) := fun n => ↑K (n + 1) \ interior (↑K n)
hKcov : ∀ (x : X), x ∈ Kdiff (CompactExhaustion.find K' x + 1)
Kdiffc : ∀ (n : ℕ), IsCompact (Kdiff n ∩ s)
this✝ : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), (↑K n)ᶜ ∈ 𝓝 ↑x
r : (n : ℕ) → (x : ↑(Kdiff (n + 1) ∩ s)) → ι ↑x
hrp : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), p (↑x) (r n x)
hr : ∀ (n : ℕ) (x : ↑(Kdiff (n + 1) ∩ s)), B (↑x) (r n x) ⊆ (↑K n)ᶜ
hxr : ∀ (n : ℕ) (x : X) (hx : x ∈ Kdiff (n + 1) ∩ s), B x (r n { val := x, property := hx }) ∈ 𝓝 x
T : (n : ℕ) → Finset ↑(Kdiff (n + 1) ∩ s)
hT :
∀ (n : ℕ),
Kdiff (n + 1) ∩ s ⊆
⋃ (x : ↑(Kdiff (n + 1) ∩ s)) (_ : x ∈ T n), B (↑x) (r n { val := ↑x, property := (_ : ↑x ∈ Kdiff (n + 1) ∩ s) })
T' : (n : ℕ) → Set ↑(Kdiff (n + 1) ∩ s) := fun n => ↑(T n)
x✝ : X
this : Set.Finite (⋃ (k : ℕ) (_ : k ≤ CompactExhaustion.find K' x✝ + 2), range (Sigma.mk k))
k : ℕ
c : ↑(Kdiff (k + 1) ∩ s)
hc : c ∈ T' k
x : X
hxB : x ∈ B (↑c) (r k c)
hxK :
x ∈
interior
(↑(CompactExhaustion.shiftr (CompactExhaustion.shiftr (CompactExhaustion.choice X)))
(CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 3))
hnk : CompactExhaustion.find (CompactExhaustion.choice X) x✝ + 2 < k
⊢ x ∈ ↑(CompactExhaustion.shiftr (CompactExhaustion.shiftr K')) k
[PROOFSTEP]
exact K.subset hnk (interior_subset hxK)
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
⊢ ParacompactSpace X
[PROOFSTEP]
refine' ⟨fun α s ho hc ↦ _⟩
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
hc : ⋃ (a : α), s a = univ
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
choose i hi using iUnion_eq_univ_iff.1 hc
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
hc : ⋃ (a : α), s a = univ
i : X → α
hi : ∀ (x : X), x ∈ s (i x)
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
have : ∀ x : X, (𝓝 x).HasBasis (fun t : Set X ↦ (x ∈ t ∧ IsOpen t) ∧ t ⊆ s (i x)) id := fun x : X ↦
(nhds_basis_opens x).restrict_subset (IsOpen.mem_nhds (ho (i x)) (hi x))
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
hc : ⋃ (a : α), s a = univ
i : X → α
hi : ∀ (x : X), x ∈ s (i x)
this : ∀ (x : X), HasBasis (𝓝 x) (fun t => (x ∈ t ∧ IsOpen t) ∧ t ⊆ s (i x)) id
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
rcases refinement_of_locallyCompact_sigmaCompact_of_nhds_basis this with ⟨β, c, t, hto, htc, htf⟩
[GOAL]
case intro.intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝⁴ : TopologicalSpace X
inst✝³ : TopologicalSpace Y
inst✝² : LocallyCompactSpace X
inst✝¹ : SigmaCompactSpace X
inst✝ : T2Space X
α : Type v
s : α → Set X
ho : ∀ (a : α), IsOpen (s a)
hc : ⋃ (a : α), s a = univ
i : X → α
hi : ∀ (x : X), x ∈ s (i x)
this : ∀ (x : X), HasBasis (𝓝 x) (fun t => (x ∈ t ∧ IsOpen t) ∧ t ⊆ s (i x)) id
β : Type v
c : β → X
t : β → Set X
hto : ∀ (a : β), (c a ∈ t a ∧ IsOpen (t a)) ∧ t a ⊆ s (i (c a))
htc : ⋃ (a : β), id (t a) = univ
htf : LocallyFinite fun a => id (t a)
⊢ ∃ β t x x, LocallyFinite t ∧ ∀ (b : β), ∃ a, t b ⊆ s a
[PROOFSTEP]
exact ⟨β, t, fun x ↦ (hto x).1.2, htc, htf, fun b ↦ ⟨i <| c b, (hto b).2⟩⟩
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
⊢ NormalSpace X
[PROOFSTEP]
have :
∀ s t : Set X,
IsClosed s →
IsClosed t →
(∀ x ∈ s, ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v :=
by
/- For each `x ∈ s` we choose open disjoint `u x ∋ x` and `v x ⊇ t`. The sets `u x` form an
open covering of `s`. We choose a locally finite refinement `u' : s → Set X`, then
`⋃ i, u' i` and `(closure (⋃ i, u' i))ᶜ` are disjoint open neighborhoods of `s` and `t`. -/
intro s t hs _ H
choose u v hu hv hxu htv huv using SetCoe.forall'.1 H
rcases precise_refinement_set hs u hu fun x hx ↦ mem_iUnion.2 ⟨⟨x, hx⟩, hxu _⟩ with ⟨u', hu'o, hcov', hu'fin, hsub⟩
refine'
⟨⋃ i, u' i, (closure (⋃ i, u' i))ᶜ, isOpen_iUnion hu'o, isClosed_closure.isOpen_compl, hcov', _,
disjoint_compl_right.mono le_rfl (compl_le_compl subset_closure)⟩
rw [hu'fin.closure_iUnion, compl_iUnion, subset_iInter_iff]
refine' fun i x hxt hxu ↦ absurd (htv i hxt) (closure_minimal _ (isClosed_compl_iff.2 <| hv _) hxu)
exact fun y hyu hyv ↦
(huv i).le_bot
⟨hsub _ hyu, hyv⟩
-- Now we apply the lemma twice: first to `s` and `t`, then to `t` and each point of `s`.
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
⊢ ∀ (s t : Set X),
IsClosed s →
IsClosed t →
(∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
[PROOFSTEP]
intro s t hs _ H
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
s t : Set X
hs : IsClosed s
a✝ : IsClosed t
H : ∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
[PROOFSTEP]
choose u v hu hv hxu htv huv using SetCoe.forall'.1 H
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
s t : Set X
hs : IsClosed s
a✝ : IsClosed t
H : ∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
u v : ↑s → Set X
hu : ∀ (x : ↑s), IsOpen (u x)
hv : ∀ (x : ↑s), IsOpen (v x)
hxu : ∀ (x : ↑s), ↑x ∈ u x
htv : ∀ (x : ↑s), t ⊆ v x
huv : ∀ (x : ↑s), Disjoint (u x) (v x)
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
[PROOFSTEP]
rcases precise_refinement_set hs u hu fun x hx ↦ mem_iUnion.2 ⟨⟨x, hx⟩, hxu _⟩ with ⟨u', hu'o, hcov', hu'fin, hsub⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
s t : Set X
hs : IsClosed s
a✝ : IsClosed t
H : ∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
u v : ↑s → Set X
hu : ∀ (x : ↑s), IsOpen (u x)
hv : ∀ (x : ↑s), IsOpen (v x)
hxu : ∀ (x : ↑s), ↑x ∈ u x
htv : ∀ (x : ↑s), t ⊆ v x
huv : ∀ (x : ↑s), Disjoint (u x) (v x)
u' : ↑s → Set X
hu'o : ∀ (i : ↑s), IsOpen (u' i)
hcov' : s ⊆ ⋃ (i : ↑s), u' i
hu'fin : LocallyFinite u'
hsub : ∀ (i : ↑s), u' i ⊆ u i
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
[PROOFSTEP]
refine'
⟨⋃ i, u' i, (closure (⋃ i, u' i))ᶜ, isOpen_iUnion hu'o, isClosed_closure.isOpen_compl, hcov', _,
disjoint_compl_right.mono le_rfl (compl_le_compl subset_closure)⟩
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
s t : Set X
hs : IsClosed s
a✝ : IsClosed t
H : ∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
u v : ↑s → Set X
hu : ∀ (x : ↑s), IsOpen (u x)
hv : ∀ (x : ↑s), IsOpen (v x)
hxu : ∀ (x : ↑s), ↑x ∈ u x
htv : ∀ (x : ↑s), t ⊆ v x
huv : ∀ (x : ↑s), Disjoint (u x) (v x)
u' : ↑s → Set X
hu'o : ∀ (i : ↑s), IsOpen (u' i)
hcov' : s ⊆ ⋃ (i : ↑s), u' i
hu'fin : LocallyFinite u'
hsub : ∀ (i : ↑s), u' i ⊆ u i
⊢ t ⊆ (closure (⋃ (i : ↑s), u' i))ᶜ
[PROOFSTEP]
rw [hu'fin.closure_iUnion, compl_iUnion, subset_iInter_iff]
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
s t : Set X
hs : IsClosed s
a✝ : IsClosed t
H : ∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
u v : ↑s → Set X
hu : ∀ (x : ↑s), IsOpen (u x)
hv : ∀ (x : ↑s), IsOpen (v x)
hxu : ∀ (x : ↑s), ↑x ∈ u x
htv : ∀ (x : ↑s), t ⊆ v x
huv : ∀ (x : ↑s), Disjoint (u x) (v x)
u' : ↑s → Set X
hu'o : ∀ (i : ↑s), IsOpen (u' i)
hcov' : s ⊆ ⋃ (i : ↑s), u' i
hu'fin : LocallyFinite u'
hsub : ∀ (i : ↑s), u' i ⊆ u i
⊢ ∀ (i : ↑s), t ⊆ (closure (u' i))ᶜ
[PROOFSTEP]
refine' fun i x hxt hxu ↦ absurd (htv i hxt) (closure_minimal _ (isClosed_compl_iff.2 <| hv _) hxu)
[GOAL]
case intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
s t : Set X
hs : IsClosed s
a✝ : IsClosed t
H : ∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
u v : ↑s → Set X
hu : ∀ (x : ↑s), IsOpen (u x)
hv : ∀ (x : ↑s), IsOpen (v x)
hxu✝ : ∀ (x : ↑s), ↑x ∈ u x
htv : ∀ (x : ↑s), t ⊆ v x
huv : ∀ (x : ↑s), Disjoint (u x) (v x)
u' : ↑s → Set X
hu'o : ∀ (i : ↑s), IsOpen (u' i)
hcov' : s ⊆ ⋃ (i : ↑s), u' i
hu'fin : LocallyFinite u'
hsub : ∀ (i : ↑s), u' i ⊆ u i
i : ↑s
x : X
hxt : x ∈ t
hxu : x ∈ closure (u' i)
⊢ u' i ⊆ (v i)ᶜ
[PROOFSTEP]
exact fun y hyu hyv ↦
(huv i).le_bot
⟨hsub _ hyu, hyv⟩
-- Now we apply the lemma twice: first to `s` and `t`, then to `t` and each point of `s`.
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
this :
∀ (s t : Set X),
IsClosed s →
IsClosed t →
(∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
⊢ NormalSpace X
[PROOFSTEP]
refine' ⟨fun s t hs ht hst ↦ this s t hs ht fun x hx ↦ _⟩
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
this :
∀ (s t : Set X),
IsClosed s →
IsClosed t →
(∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
s t : Set X
hs : IsClosed s
ht : IsClosed t
hst : Disjoint s t
x : X
hx : x ∈ s
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
[PROOFSTEP]
rcases this t { x } ht isClosed_singleton fun y hy ↦
(by
simp_rw [singleton_subset_iff]
exact t2_separation (hst.symm.ne_of_mem hy hx)) with
⟨v, u, hv, hu, htv, hxu, huv⟩
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
this :
∀ (s t : Set X),
IsClosed s →
IsClosed t →
(∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
s t : Set X
hs : IsClosed s
ht : IsClosed t
hst : Disjoint s t
x : X
hx : x ∈ s
y : X
hy : y ∈ t
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ y ∈ u ∧ {x} ⊆ v ∧ Disjoint u v
[PROOFSTEP]
simp_rw [singleton_subset_iff]
[GOAL]
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
this :
∀ (s t : Set X),
IsClosed s →
IsClosed t →
(∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
s t : Set X
hs : IsClosed s
ht : IsClosed t
hst : Disjoint s t
x : X
hx : x ∈ s
y : X
hy : y ∈ t
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ y ∈ u ∧ x ∈ v ∧ Disjoint u v
[PROOFSTEP]
exact t2_separation (hst.symm.ne_of_mem hy hx)
[GOAL]
case intro.intro.intro.intro.intro.intro
ι : Type u
X : Type v
Y : Type w
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : T2Space X
inst✝ : ParacompactSpace X
this :
∀ (s t : Set X),
IsClosed s →
IsClosed t →
(∀ (x : X), x ∈ s → ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v) →
∃ u v, IsOpen u ∧ IsOpen v ∧ s ⊆ u ∧ t ⊆ v ∧ Disjoint u v
s t : Set X
hs : IsClosed s
ht : IsClosed t
hst : Disjoint s t
x : X
hx : x ∈ s
v u : Set X
hv : IsOpen v
hu : IsOpen u
htv : t ⊆ v
hxu : {x} ⊆ u
huv : Disjoint v u
⊢ ∃ u v, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ t ⊆ v ∧ Disjoint u v
[PROOFSTEP]
exact ⟨u, v, hu, hv, singleton_subset_iff.1 hxu, htv, huv.symm⟩
| {"mathlib_filename": "Mathlib.Topology.Paracompact", "llama_tokens": 46078} |
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
[PROOFSTEP]
rw [noetherianSpace_iff, CompleteLattice.wellFounded_iff_isSupFiniteCompact,
CompleteLattice.isSupFiniteCompact_iff_all_elements_compact]
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ (∀ (k : Opens α), CompleteLattice.IsCompactElement k) ↔ ∀ (s : Opens α), IsCompact ↑s
[PROOFSTEP]
exact forall_congr' Opens.isCompactElement_iff
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Set α
⊢ IsCompact s
[PROOFSTEP]
refine isCompact_iff_finite_subcover.2 fun U hUo hs => ?_
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Set α
ι✝ : Type u_1
U : ι✝ → Set α
hUo : ∀ (i : ι✝), IsOpen (U i)
hs : s ⊆ ⋃ (i : ι✝), U i
⊢ ∃ t, s ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
[PROOFSTEP]
rcases((noetherianSpace_iff_opens α).mp ‹_› ⟨⋃ i, U i, isOpen_iUnion hUo⟩).elim_finite_subcover U hUo
Set.Subset.rfl with
⟨t, ht⟩
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Set α
ι✝ : Type u_1
U : ι✝ → Set α
hUo : ∀ (i : ι✝), IsOpen (U i)
hs : s ⊆ ⋃ (i : ι✝), U i
t : Finset ι✝
ht : ↑{ carrier := ⋃ (i : ι✝), U i, is_open' := (_ : IsOpen (⋃ (i : ι✝), U i)) } ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
⊢ ∃ t, s ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
[PROOFSTEP]
exact ⟨t, hs.trans ht⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ TFAE [NoetherianSpace α, WellFounded fun s t => s < t, ∀ (s : Set α), IsCompact s, ∀ (s : Opens α), IsCompact ↑s]
[PROOFSTEP]
tfae_have 1 ↔ 2
[GOAL]
case tfae_1_iff_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ NoetherianSpace α ↔ WellFounded fun s t => s < t
[PROOFSTEP]
refine' (noetherianSpace_iff α).trans (Surjective.wellFounded_iff Opens.compl_bijective.2 _)
[GOAL]
case tfae_1_iff_2
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
⊢ ∀ {a b : Opens α}, a > b ↔ Opens.compl a < Opens.compl b
[PROOFSTEP]
exact (@OrderIso.compl (Set α)).lt_iff_lt.symm
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
⊢ TFAE [NoetherianSpace α, WellFounded fun s t => s < t, ∀ (s : Set α), IsCompact s, ∀ (s : Opens α), IsCompact ↑s]
[PROOFSTEP]
tfae_have 1 ↔ 4
[GOAL]
case tfae_1_iff_4
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
⊢ NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
[PROOFSTEP]
exact noetherianSpace_iff_opens α
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
tfae_1_iff_4 : NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
⊢ TFAE [NoetherianSpace α, WellFounded fun s t => s < t, ∀ (s : Set α), IsCompact s, ∀ (s : Opens α), IsCompact ↑s]
[PROOFSTEP]
tfae_have 1 → 3
[GOAL]
case tfae_1_to_3
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
tfae_1_iff_4 : NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
⊢ NoetherianSpace α → ∀ (s : Set α), IsCompact s
[PROOFSTEP]
exact @NoetherianSpace.isCompact α _
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
tfae_1_iff_4 : NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
tfae_1_to_3 : NoetherianSpace α → ∀ (s : Set α), IsCompact s
⊢ TFAE [NoetherianSpace α, WellFounded fun s t => s < t, ∀ (s : Set α), IsCompact s, ∀ (s : Opens α), IsCompact ↑s]
[PROOFSTEP]
tfae_have 3 → 4
[GOAL]
case tfae_3_to_4
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
tfae_1_iff_4 : NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
tfae_1_to_3 : NoetherianSpace α → ∀ (s : Set α), IsCompact s
⊢ (∀ (s : Set α), IsCompact s) → ∀ (s : Opens α), IsCompact ↑s
[PROOFSTEP]
exact fun h s => h s
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
tfae_1_iff_2 : NoetherianSpace α ↔ WellFounded fun s t => s < t
tfae_1_iff_4 : NoetherianSpace α ↔ ∀ (s : Opens α), IsCompact ↑s
tfae_1_to_3 : NoetherianSpace α → ∀ (s : Set α), IsCompact s
tfae_3_to_4 : (∀ (s : Set α), IsCompact s) → ∀ (s : Opens α), IsCompact ↑s
⊢ TFAE [NoetherianSpace α, WellFounded fun s t => s < t, ∀ (s : Set α), IsCompact s, ∀ (s : Opens α), IsCompact ↑s]
[PROOFSTEP]
tfae_finish
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α✝
inst✝ : TopologicalSpace β
α : Type ?u.3614
⊢ NoetherianSpace (CofiniteTopology α)
[PROOFSTEP]
simp only [noetherianSpace_iff_isCompact, isCompact_iff_ultrafilter_le_nhds, CofiniteTopology.nhds_eq,
Ultrafilter.le_sup_iff, Filter.le_principal_iff]
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α✝
inst✝ : TopologicalSpace β
α : Type ?u.3614
⊢ ∀ (s : Set (CofiniteTopology α)) (f : Ultrafilter (CofiniteTopology α)),
s ∈ ↑f → ∃ a, a ∈ s ∧ (↑f ≤ pure a ∨ ↑f ≤ Filter.cofinite)
[PROOFSTEP]
intro s f hs
[GOAL]
α✝ : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α✝
inst✝ : TopologicalSpace β
α : Type ?u.3614
s : Set (CofiniteTopology α)
f : Ultrafilter (CofiniteTopology α)
hs : s ∈ ↑f
⊢ ∃ a, a ∈ s ∧ (↑f ≤ pure a ∨ ↑f ≤ Filter.cofinite)
[PROOFSTEP]
rcases f.le_cofinite_or_eq_pure with (hf | ⟨a, rfl⟩)
[GOAL]
case inl
α✝ : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α✝
inst✝ : TopologicalSpace β
α : Type ?u.3614
s : Set (CofiniteTopology α)
f : Ultrafilter (CofiniteTopology α)
hs : s ∈ ↑f
hf : ↑f ≤ Filter.cofinite
⊢ ∃ a, a ∈ s ∧ (↑f ≤ pure a ∨ ↑f ≤ Filter.cofinite)
[PROOFSTEP]
rcases Filter.nonempty_of_mem hs with ⟨a, ha⟩
[GOAL]
case inl.intro
α✝ : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α✝
inst✝ : TopologicalSpace β
α : Type ?u.3614
s : Set (CofiniteTopology α)
f : Ultrafilter (CofiniteTopology α)
hs : s ∈ ↑f
hf : ↑f ≤ Filter.cofinite
a : CofiniteTopology α
ha : a ∈ s
⊢ ∃ a, a ∈ s ∧ (↑f ≤ pure a ∨ ↑f ≤ Filter.cofinite)
[PROOFSTEP]
exact ⟨a, ha, Or.inr hf⟩
[GOAL]
case inr.intro
α✝ : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α✝
inst✝ : TopologicalSpace β
α : Type ?u.3614
s : Set (CofiniteTopology α)
a : CofiniteTopology α
hs : s ∈ ↑(pure a)
⊢ ∃ a_1, a_1 ∈ s ∧ (↑(pure a) ≤ pure a_1 ∨ ↑(pure a) ≤ Filter.cofinite)
[PROOFSTEP]
exact ⟨a, hs, Or.inl le_rfl⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set α
⊢ NoetherianSpace ↑s ↔ ∀ (t : Set α), t ⊆ s → IsCompact t
[PROOFSTEP]
simp only [noetherianSpace_iff_isCompact, embedding_subtype_val.isCompact_iff_isCompact_image,
Subtype.forall_set_subtype]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
ι : Type u_3
f : ι → Set α
inst✝ : Finite ι
hf : ∀ (i : ι), NoetherianSpace ↑(f i)
⊢ NoetherianSpace ↑(⋃ (i : ι), f i)
[PROOFSTEP]
simp_rw [noetherianSpace_set_iff] at hf ⊢
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
ι : Type u_3
f : ι → Set α
inst✝ : Finite ι
hf : ∀ (i : ι) (t : Set α), t ⊆ f i → IsCompact t
⊢ ∀ (t : Set α), t ⊆ ⋃ (i : ι), f i → IsCompact t
[PROOFSTEP]
intro t ht
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
ι : Type u_3
f : ι → Set α
inst✝ : Finite ι
hf : ∀ (i : ι) (t : Set α), t ⊆ f i → IsCompact t
t : Set α
ht : t ⊆ ⋃ (i : ι), f i
⊢ IsCompact t
[PROOFSTEP]
rw [← Set.inter_eq_left_iff_subset.mpr ht, Set.inter_iUnion]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
ι : Type u_3
f : ι → Set α
inst✝ : Finite ι
hf : ∀ (i : ι) (t : Set α), t ⊆ f i → IsCompact t
t : Set α
ht : t ⊆ ⋃ (i : ι), f i
⊢ IsCompact (⋃ (i : ι), t ∩ f i)
[PROOFSTEP]
exact isCompact_iUnion fun i => hf i _ (Set.inter_subset_right _ _)
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
apply wellFounded_closeds.induction s
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
⊢ ∀ (x : Closeds α),
(∀ (y : Closeds α), y < x → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S) →
∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ x = sSup S
[PROOFSTEP]
clear s
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
⊢ ∀ (x : Closeds α),
(∀ (y : Closeds α), y < x → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S) →
∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ x = sSup S
[PROOFSTEP]
intro s H
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
rcases eq_or_ne s ⊥ with rfl | h₀
[GOAL]
case inl
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
H : ∀ (y : Closeds α), y < ⊥ → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ ⊥ = sSup S
[PROOFSTEP]
use∅
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
H : ∀ (y : Closeds α), y < ⊥ → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
⊢ Set.Finite ∅ ∧ (∀ (t : Closeds α), t ∈ ∅ → IsIrreducible ↑t) ∧ ⊥ = sSup ∅
[PROOFSTEP]
simp
[GOAL]
case inr
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
by_cases h₁ : IsPreirreducible (s : Set α)
[GOAL]
case pos
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
h₁ : IsPreirreducible ↑s
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
replace h₁ : IsIrreducible (s : Set α) := ⟨Closeds.coe_nonempty.2 h₀, h₁⟩
[GOAL]
case pos
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
h₁ : IsIrreducible ↑s
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
use{ s }
[GOAL]
case h
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
h₁ : IsIrreducible ↑s
⊢ Set.Finite {s} ∧ (∀ (t : Closeds α), t ∈ {s} → IsIrreducible ↑t) ∧ s = sSup {s}
[PROOFSTEP]
simp [h₁]
[GOAL]
case neg
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
h₁ : ¬IsPreirreducible ↑s
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
simp only [isPreirreducible_iff_closed_union_closed, not_forall, not_or] at h₁
[GOAL]
case neg
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
h₁ : ∃ x x_1 h h h, ¬↑s ⊆ x ∧ ¬↑s ⊆ x_1
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
obtain ⟨z₁, z₂, hz₁, hz₂, h, hz₁', hz₂'⟩ := h₁
[GOAL]
case neg.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
z₁ z₂ : Set α
hz₁ : IsClosed z₁
hz₂ : IsClosed z₂
h : ↑s ⊆ z₁ ∪ z₂
hz₁' : ¬↑s ⊆ z₁
hz₂' : ¬↑s ⊆ z₂
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
lift z₁ to Closeds α using hz₁
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
z₂ : Set α
hz₂ : IsClosed z₂
hz₂' : ¬↑s ⊆ z₂
z₁ : Closeds α
h : ↑s ⊆ ↑z₁ ∪ z₂
hz₁' : ¬↑s ⊆ ↑z₁
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
lift z₂ to Closeds α using hz₂
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
z₁ : Closeds α
hz₁' : ¬↑s ⊆ ↑z₁
z₂ : Closeds α
hz₂' : ¬↑s ⊆ ↑z₂
h : ↑s ⊆ ↑z₁ ∪ ↑z₂
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
rcases H (s ⊓ z₁) (inf_lt_left.2 hz₁') with ⟨S₁, hSf₁, hS₁, h₁⟩
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
z₁ : Closeds α
hz₁' : ¬↑s ⊆ ↑z₁
z₂ : Closeds α
hz₂' : ¬↑s ⊆ ↑z₂
h : ↑s ⊆ ↑z₁ ∪ ↑z₂
S₁ : Set (Closeds α)
hSf₁ : Set.Finite S₁
hS₁ : ∀ (t : Closeds α), t ∈ S₁ → IsIrreducible ↑t
h₁ : s ⊓ z₁ = sSup S₁
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
rcases H (s ⊓ z₂) (inf_lt_left.2 hz₂') with ⟨S₂, hSf₂, hS₂, h₂⟩
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
z₁ : Closeds α
hz₁' : ¬↑s ⊆ ↑z₁
z₂ : Closeds α
hz₂' : ¬↑s ⊆ ↑z₂
h : ↑s ⊆ ↑z₁ ∪ ↑z₂
S₁ : Set (Closeds α)
hSf₁ : Set.Finite S₁
hS₁ : ∀ (t : Closeds α), t ∈ S₁ → IsIrreducible ↑t
h₁ : s ⊓ z₁ = sSup S₁
S₂ : Set (Closeds α)
hSf₂ : Set.Finite S₂
hS₂ : ∀ (t : Closeds α), t ∈ S₂ → IsIrreducible ↑t
h₂ : s ⊓ z₂ = sSup S₂
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ s = sSup S
[PROOFSTEP]
refine ⟨S₁ ∪ S₂, hSf₁.union hSf₂, Set.union_subset_iff.2 ⟨hS₁, hS₂⟩, ?_⟩
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
H : ∀ (y : Closeds α), y < s → ∃ S, Set.Finite S ∧ (∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t) ∧ y = sSup S
h₀ : s ≠ ⊥
z₁ : Closeds α
hz₁' : ¬↑s ⊆ ↑z₁
z₂ : Closeds α
hz₂' : ¬↑s ⊆ ↑z₂
h : ↑s ⊆ ↑z₁ ∪ ↑z₂
S₁ : Set (Closeds α)
hSf₁ : Set.Finite S₁
hS₁ : ∀ (t : Closeds α), t ∈ S₁ → IsIrreducible ↑t
h₁ : s ⊓ z₁ = sSup S₁
S₂ : Set (Closeds α)
hSf₂ : Set.Finite S₂
hS₂ : ∀ (t : Closeds α), t ∈ S₂ → IsIrreducible ↑t
h₂ : s ⊓ z₂ = sSup S₂
⊢ s = sSup (S₁ ∪ S₂)
[PROOFSTEP]
rwa [sSup_union, ← h₁, ← h₂, ← inf_sup_left, left_eq_inf]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Set α
hs : IsClosed s
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Set α), t ∈ S → IsClosed t) ∧ (∀ (t : Set α), t ∈ S → IsIrreducible t) ∧ s = ⋃₀ S
[PROOFSTEP]
lift s to Closeds α using hs
[GOAL]
case intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
⊢ ∃ S, Set.Finite S ∧ (∀ (t : Set α), t ∈ S → IsClosed t) ∧ (∀ (t : Set α), t ∈ S → IsIrreducible t) ∧ ↑s = ⋃₀ S
[PROOFSTEP]
rcases NoetherianSpace.exists_finite_set_closeds_irreducible s with ⟨S, hSf, hS, rfl⟩
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
S : Set (Closeds α)
hSf : Set.Finite S
hS : ∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t
⊢ ∃ S_1,
Set.Finite S_1 ∧
(∀ (t : Set α), t ∈ S_1 → IsClosed t) ∧ (∀ (t : Set α), t ∈ S_1 → IsIrreducible t) ∧ ↑(sSup S) = ⋃₀ S_1
[PROOFSTEP]
refine ⟨(↑) '' S, hSf.image _, Set.ball_image_iff.2 fun S _ => S.2, Set.ball_image_iff.2 hS, ?_⟩
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
S : Set (Closeds α)
hSf : Set.Finite S
hS : ∀ (t : Closeds α), t ∈ S → IsIrreducible ↑t
⊢ ↑(sSup S) = ⋃₀ (SetLike.coe '' S)
[PROOFSTEP]
lift S to Finset (Closeds α) using hSf
[GOAL]
case intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
S : Finset (Closeds α)
hS : ∀ (t : Closeds α), t ∈ ↑S → IsIrreducible ↑t
⊢ ↑(sSup ↑S) = ⋃₀ (SetLike.coe '' ↑S)
[PROOFSTEP]
simp [← Finset.sup_id_eq_sSup, Closeds.coe_finset_sup]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Closeds α
⊢ ∃ S, (∀ (k : { x // x ∈ S }), IsIrreducible ↑↑k) ∧ s = Finset.sup S id
[PROOFSTEP]
simpa [Set.exists_finite_iff_finset, Finset.sup_id_eq_sSup] using
NoetherianSpace.exists_finite_set_closeds_irreducible s
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
⊢ Set.Finite (irreducibleComponents α)
[PROOFSTEP]
obtain ⟨S : Set (Set α), hSf, hSc, hSi, hSU⟩ :=
NoetherianSpace.exists_finite_set_isClosed_irreducible isClosed_univ (α := α)
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
S : Set (Set α)
hSf : Set.Finite S
hSc : ∀ (t : Set α), t ∈ S → IsClosed t
hSi : ∀ (t : Set α), t ∈ S → IsIrreducible t
hSU : Set.univ = ⋃₀ S
⊢ Set.Finite (irreducibleComponents α)
[PROOFSTEP]
refine hSf.subset fun s hs => ?_
[GOAL]
case intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
S : Set (Set α)
hSf : Set.Finite S
hSc : ∀ (t : Set α), t ∈ S → IsClosed t
hSi : ∀ (t : Set α), t ∈ S → IsIrreducible t
hSU : Set.univ = ⋃₀ S
s : Set α
hs : s ∈ irreducibleComponents α
⊢ s ∈ S
[PROOFSTEP]
lift S to Finset (Set α) using hSf
[GOAL]
case intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Set α
hs : s ∈ irreducibleComponents α
S : Finset (Set α)
hSc : ∀ (t : Set α), t ∈ ↑S → IsClosed t
hSi : ∀ (t : Set α), t ∈ ↑S → IsIrreducible t
hSU : Set.univ = ⋃₀ ↑S
⊢ s ∈ ↑S
[PROOFSTEP]
rcases isIrreducible_iff_sUnion_closed.1 hs.1 S hSc (hSU ▸ Set.subset_univ _) with ⟨t, htS, ht⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
inst✝ : NoetherianSpace α
s : Set α
hs : s ∈ irreducibleComponents α
S : Finset (Set α)
hSc : ∀ (t : Set α), t ∈ ↑S → IsClosed t
hSi : ∀ (t : Set α), t ∈ ↑S → IsIrreducible t
hSU : Set.univ = ⋃₀ ↑S
t : Set α
htS : t ∈ S
ht : s ⊆ t
⊢ s ∈ ↑S
[PROOFSTEP]
rwa [ht.antisymm (hs.2 (hSi _ htS) ht)]
| {"mathlib_filename": "Mathlib.Topology.NoetherianSpace", "llama_tokens": 10444} |
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → sᶜ ∈ 𝓝 a ⊓ f
⊢ sᶜ ∈ f
[PROOFSTEP]
contrapose! hf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
f : Filter α
hf : ¬sᶜ ∈ f
⊢ ∃ a, a ∈ s ∧ ¬sᶜ ∈ 𝓝 a ⊓ f
[PROOFSTEP]
simp only [not_mem_iff_inf_principal_compl, compl_compl, inf_assoc] at hf ⊢
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
f : Filter α
hf : NeBot (f ⊓ 𝓟 s)
⊢ ∃ a, a ∈ s ∧ NeBot (𝓝 a ⊓ (f ⊓ 𝓟 s))
[PROOFSTEP]
exact @hs _ hf inf_le_right
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
⊢ sᶜ ∈ f
[PROOFSTEP]
refine' hs.compl_mem_sets fun a ha => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
a : α
ha : a ∈ s
⊢ sᶜ ∈ 𝓝 a ⊓ f
[PROOFSTEP]
rcases hf a ha with ⟨t, ht, hst⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hs : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
a : α
ha : a ∈ s
t : Set α
ht : t ∈ 𝓝[s] a
hst : tᶜ ∈ f
⊢ sᶜ ∈ 𝓝 a ⊓ f
[PROOFSTEP]
replace ht := mem_inf_principal.1 ht
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hs : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
a : α
ha : a ∈ s
t : Set α
hst : tᶜ ∈ f
ht : {x | x ∈ s → x ∈ t} ∈ 𝓝 a
⊢ sᶜ ∈ 𝓝 a ⊓ f
[PROOFSTEP]
apply mem_inf_of_inter ht hst
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hs : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
a : α
ha : a ∈ s
t : Set α
hst : tᶜ ∈ f
ht : {x | x ∈ s → x ∈ t} ∈ 𝓝 a
⊢ {x | x ∈ s → x ∈ t} ∩ tᶜ ⊆ sᶜ
[PROOFSTEP]
rintro x ⟨h₁, h₂⟩ hs
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hs✝ : IsCompact s
f : Filter α
hf : ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
a : α
ha : a ∈ s
t : Set α
hst : tᶜ ∈ f
ht : {x | x ∈ s → x ∈ t} ∈ 𝓝 a
x : α
h₁ : x ∈ {x | x ∈ s → x ∈ t}
h₂ : x ∈ tᶜ
hs : x ∈ s
⊢ False
[PROOFSTEP]
exact h₂ (h₁ hs)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
p : Set α → Prop
he : p ∅
hmono : ∀ ⦃s t : Set α⦄, s ⊆ t → p t → p s
hunion : ∀ ⦃s t : Set α⦄, p s → p t → p (s ∪ t)
hnhds : ∀ (x : α), x ∈ s → ∃ t, t ∈ 𝓝[s] x ∧ p t
⊢ p s
[PROOFSTEP]
let f : Filter α :=
{ sets := {t | p tᶜ}
univ_sets := by simpa
sets_of_superset := fun ht₁ ht => hmono (compl_subset_compl.2 ht) ht₁
inter_sets := fun ht₁ ht₂ => by simp [compl_inter, hunion ht₁ ht₂] }
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
p : Set α → Prop
he : p ∅
hmono : ∀ ⦃s t : Set α⦄, s ⊆ t → p t → p s
hunion : ∀ ⦃s t : Set α⦄, p s → p t → p (s ∪ t)
hnhds : ∀ (x : α), x ∈ s → ∃ t, t ∈ 𝓝[s] x ∧ p t
⊢ univ ∈ {t | p tᶜ}
[PROOFSTEP]
simpa
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
p : Set α → Prop
he : p ∅
hmono : ∀ ⦃s t : Set α⦄, s ⊆ t → p t → p s
hunion : ∀ ⦃s t : Set α⦄, p s → p t → p (s ∪ t)
hnhds : ∀ (x : α), x ∈ s → ∃ t, t ∈ 𝓝[s] x ∧ p t
x✝ y✝ : Set α
ht₁ : x✝ ∈ {t | p tᶜ}
ht₂ : y✝ ∈ {t | p tᶜ}
⊢ x✝ ∩ y✝ ∈ {t | p tᶜ}
[PROOFSTEP]
simp [compl_inter, hunion ht₁ ht₂]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
p : Set α → Prop
he : p ∅
hmono : ∀ ⦃s t : Set α⦄, s ⊆ t → p t → p s
hunion : ∀ ⦃s t : Set α⦄, p s → p t → p (s ∪ t)
hnhds : ∀ (x : α), x ∈ s → ∃ t, t ∈ 𝓝[s] x ∧ p t
f : Filter α :=
{ sets := {t | p tᶜ}, univ_sets := (_ : univ ∈ {t | p tᶜ}),
sets_of_superset := (_ : ∀ {x y : Set α}, x ∈ {t | p tᶜ} → x ⊆ y → p yᶜ),
inter_sets := (_ : ∀ {x y : Set α}, x ∈ {t | p tᶜ} → y ∈ {t | p tᶜ} → p (x ∩ y)ᶜ) }
⊢ p s
[PROOFSTEP]
have : sᶜ ∈ f := hs.compl_mem_sets_of_nhdsWithin (by simpa using hnhds)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
p : Set α → Prop
he : p ∅
hmono : ∀ ⦃s t : Set α⦄, s ⊆ t → p t → p s
hunion : ∀ ⦃s t : Set α⦄, p s → p t → p (s ∪ t)
hnhds : ∀ (x : α), x ∈ s → ∃ t, t ∈ 𝓝[s] x ∧ p t
f : Filter α :=
{ sets := {t | p tᶜ}, univ_sets := (_ : univ ∈ {t | p tᶜ}),
sets_of_superset := (_ : ∀ {x y : Set α}, x ∈ {t | p tᶜ} → x ⊆ y → p yᶜ),
inter_sets := (_ : ∀ {x y : Set α}, x ∈ {t | p tᶜ} → y ∈ {t | p tᶜ} → p (x ∩ y)ᶜ) }
⊢ ∀ (a : α), a ∈ s → ∃ t, t ∈ 𝓝[s] a ∧ tᶜ ∈ f
[PROOFSTEP]
simpa using hnhds
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
p : Set α → Prop
he : p ∅
hmono : ∀ ⦃s t : Set α⦄, s ⊆ t → p t → p s
hunion : ∀ ⦃s t : Set α⦄, p s → p t → p (s ∪ t)
hnhds : ∀ (x : α), x ∈ s → ∃ t, t ∈ 𝓝[s] x ∧ p t
f : Filter α :=
{ sets := {t | p tᶜ}, univ_sets := (_ : univ ∈ {t | p tᶜ}),
sets_of_superset := (_ : ∀ {x y : Set α}, x ∈ {t | p tᶜ} → x ⊆ y → p yᶜ),
inter_sets := (_ : ∀ {x y : Set α}, x ∈ {t | p tᶜ} → y ∈ {t | p tᶜ} → p (x ∩ y)ᶜ) }
this : sᶜ ∈ f
⊢ p s
[PROOFSTEP]
rwa [← compl_compl s]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsClosed t
⊢ IsCompact (s ∩ t)
[PROOFSTEP]
intro f hnf hstf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsClosed t
f : Filter α
hnf : NeBot f
hstf : f ≤ 𝓟 (s ∩ t)
⊢ ∃ a, a ∈ s ∩ t ∧ ClusterPt a f
[PROOFSTEP]
obtain ⟨a, hsa, ha⟩ : ∃ a ∈ s, ClusterPt a f := hs (le_trans hstf (le_principal_iff.2 (inter_subset_left _ _)))
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsClosed t
f : Filter α
hnf : NeBot f
hstf : f ≤ 𝓟 (s ∩ t)
a : α
hsa : a ∈ s
ha : ClusterPt a f
⊢ ∃ a, a ∈ s ∩ t ∧ ClusterPt a f
[PROOFSTEP]
have : a ∈ t := ht.mem_of_nhdsWithin_neBot <| ha.mono <| le_trans hstf (le_principal_iff.2 (inter_subset_right _ _))
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsClosed t
f : Filter α
hnf : NeBot f
hstf : f ≤ 𝓟 (s ∩ t)
a : α
hsa : a ∈ s
ha : ClusterPt a f
this : a ∈ t
⊢ ∃ a, a ∈ s ∩ t ∧ ClusterPt a f
[PROOFSTEP]
exact ⟨a, ⟨hsa, this⟩, ha⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
⊢ IsCompact (f '' s)
[PROOFSTEP]
intro l lne ls
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
⊢ ∃ a, a ∈ f '' s ∧ ClusterPt a l
[PROOFSTEP]
have : NeBot (l.comap f ⊓ 𝓟 s) := comap_inf_principal_neBot_of_image_mem lne (le_principal_iff.1 ls)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this : NeBot (comap f l ⊓ 𝓟 s)
⊢ ∃ a, a ∈ f '' s ∧ ClusterPt a l
[PROOFSTEP]
obtain ⟨a, has, ha⟩ : ∃ a ∈ s, ClusterPt a (l.comap f ⊓ 𝓟 s) := @hs _ this inf_le_right
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
⊢ ∃ a, a ∈ f '' s ∧ ClusterPt a l
[PROOFSTEP]
haveI := ha.neBot
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this✝ : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
this : NeBot (𝓝 a ⊓ (comap f l ⊓ 𝓟 s))
⊢ ∃ a, a ∈ f '' s ∧ ClusterPt a l
[PROOFSTEP]
use f a, mem_image_of_mem f has
[GOAL]
case right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this✝ : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
this : NeBot (𝓝 a ⊓ (comap f l ⊓ 𝓟 s))
⊢ ClusterPt (f a) l
[PROOFSTEP]
have : Tendsto f (𝓝 a ⊓ (comap f l ⊓ 𝓟 s)) (𝓝 (f a) ⊓ l) :=
by
convert (hf a has).inf (@tendsto_comap _ _ f l) using 1
rw [nhdsWithin]
ac_rfl
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this✝ : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
this : NeBot (𝓝 a ⊓ (comap f l ⊓ 𝓟 s))
⊢ Tendsto f (𝓝 a ⊓ (comap f l ⊓ 𝓟 s)) (𝓝 (f a) ⊓ l)
[PROOFSTEP]
convert (hf a has).inf (@tendsto_comap _ _ f l) using 1
[GOAL]
case h.e'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this✝ : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
this : NeBot (𝓝 a ⊓ (comap f l ⊓ 𝓟 s))
⊢ 𝓝 a ⊓ (comap f l ⊓ 𝓟 s) = 𝓝[s] a ⊓ comap f l
[PROOFSTEP]
rw [nhdsWithin]
[GOAL]
case h.e'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this✝ : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
this : NeBot (𝓝 a ⊓ (comap f l ⊓ 𝓟 s))
⊢ 𝓝 a ⊓ (comap f l ⊓ 𝓟 s) = 𝓝 a ⊓ 𝓟 s ⊓ comap f l
[PROOFSTEP]
ac_rfl
[GOAL]
case right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hs : IsCompact s
hf : ContinuousOn f s
l : Filter β
lne : NeBot l
ls : l ≤ 𝓟 (f '' s)
this✝¹ : NeBot (comap f l ⊓ 𝓟 s)
a : α
has : a ∈ s
ha : ClusterPt a (comap f l ⊓ 𝓟 s)
this✝ : NeBot (𝓝 a ⊓ (comap f l ⊓ 𝓟 s))
this : Tendsto f (𝓝 a ⊓ (comap f l ⊓ 𝓟 s)) (𝓝 (f a) ⊓ l)
⊢ ClusterPt (f a) l
[PROOFSTEP]
exact this.neBot
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ IsCompact s ↔ ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
refine' (forall_neBot_le_iff _).trans _
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ Monotone fun f => ∃ a, a ∈ s ∧ ClusterPt a f
[PROOFSTEP]
rintro f g hle ⟨a, has, haf⟩
[GOAL]
case refine'_1.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f g : Filter α
hle : f ≤ g
a : α
has : a ∈ s
haf : ClusterPt a f
⊢ ∃ a, a ∈ s ∧ ClusterPt a g
[PROOFSTEP]
exact ⟨a, has, haf.mono hle⟩
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ (∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ClusterPt a ↑f) ↔
∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
simp only [Ultrafilter.clusterPt_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hs : IsCompact s
U : α → Set α
hU : ∀ (x : α), x ∈ s → U x ∈ 𝓝 x
t : Finset ↑s
ht : s ⊆ ⋃ (x : ↑s) (_ : x ∈ t), U ↑x
⊢ s ⊆ ⋃ (x : α) (_ : x ∈ Finset.image Subtype.val t), U x
[PROOFSTEP]
rwa [Finset.set_biUnion_finset_image]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
l : Filter α
hs : IsCompact s
⊢ Disjoint (𝓝ˢ s) l ↔ ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
[PROOFSTEP]
refine' ⟨fun h x hx => h.mono_left <| nhds_le_nhdsSet hx, fun H => _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
l : Filter α
hs : IsCompact s
H : ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
⊢ Disjoint (𝓝ˢ s) l
[PROOFSTEP]
choose! U hxU hUl using fun x hx => (nhds_basis_opens x).disjoint_iff_left.1 (H x hx)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
l : Filter α
hs : IsCompact s
H : ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
U : α → Set α
hxU : ∀ (x : α), x ∈ s → x ∈ U x ∧ IsOpen (U x)
hUl : ∀ (x : α), x ∈ s → (U x)ᶜ ∈ l
⊢ Disjoint (𝓝ˢ s) l
[PROOFSTEP]
choose hxU hUo using hxU
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
l : Filter α
hs : IsCompact s
H : ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
U : α → Set α
hUl : ∀ (x : α), x ∈ s → (U x)ᶜ ∈ l
hxU : ∀ (x : α), x ∈ s → x ∈ U x
hUo : ∀ (x : α), x ∈ s → IsOpen (U x)
⊢ Disjoint (𝓝ˢ s) l
[PROOFSTEP]
rcases hs.elim_nhds_subcover U fun x hx => (hUo x hx).mem_nhds (hxU x hx) with ⟨t, hts, hst⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
l : Filter α
hs : IsCompact s
H : ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
U : α → Set α
hUl : ∀ (x : α), x ∈ s → (U x)ᶜ ∈ l
hxU : ∀ (x : α), x ∈ s → x ∈ U x
hUo : ∀ (x : α), x ∈ s → IsOpen (U x)
t : Finset α
hts : ∀ (x : α), x ∈ t → x ∈ s
hst : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
⊢ Disjoint (𝓝ˢ s) l
[PROOFSTEP]
refine' (hasBasis_nhdsSet _).disjoint_iff_left.2 ⟨⋃ x ∈ t, U x, ⟨isOpen_biUnion fun x hx => hUo x (hts x hx), hst⟩, _⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
l : Filter α
hs : IsCompact s
H : ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
U : α → Set α
hUl : ∀ (x : α), x ∈ s → (U x)ᶜ ∈ l
hxU : ∀ (x : α), x ∈ s → x ∈ U x
hUo : ∀ (x : α), x ∈ s → IsOpen (U x)
t : Finset α
hts : ∀ (x : α), x ∈ t → x ∈ s
hst : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
⊢ (⋃ (x : α) (_ : x ∈ t), U x)ᶜ ∈ l
[PROOFSTEP]
rw [compl_iUnion₂, biInter_finset_mem]
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
l : Filter α
hs : IsCompact s
H : ∀ (x : α), x ∈ s → Disjoint (𝓝 x) l
U : α → Set α
hUl : ∀ (x : α), x ∈ s → (U x)ᶜ ∈ l
hxU : ∀ (x : α), x ∈ s → x ∈ U x
hUo : ∀ (x : α), x ∈ s → IsOpen (U x)
t : Finset α
hts : ∀ (x : α), x ∈ t → x ∈ s
hst : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
⊢ ∀ (i : α), i ∈ t → (U i)ᶜ ∈ l
[PROOFSTEP]
exact fun x hx => hUl x (hts x hx)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
l : Filter α
hs : IsCompact s
⊢ Disjoint l (𝓝ˢ s) ↔ ∀ (x : α), x ∈ s → Disjoint l (𝓝 x)
[PROOFSTEP]
simpa only [disjoint_comm] using hs.disjoint_nhdsSet_left
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : s ∩ ⋂ (i : ι), Z i = ∅
hdZ : Directed (fun x x_1 => x ⊇ x_1) Z
⊢ s ⊆ ⋃ (i : ι), (compl ∘ Z) i
[PROOFSTEP]
simpa only [subset_def, not_forall, eq_empty_iff_forall_not_mem, mem_iUnion, exists_prop, mem_inter_iff, not_and,
iff_self_iff, mem_iInter, mem_compl_iff] using hsZ
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
ι : Type v
hι : Nonempty ι
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : s ∩ ⋂ (i : ι), Z i = ∅
hdZ : Directed (fun x x_1 => x ⊇ x_1) Z
t : ι
ht : s ⊆ (compl ∘ Z) t
⊢ s ∩ Z t = ∅
[PROOFSTEP]
simpa only [subset_def, not_forall, eq_empty_iff_forall_not_mem, mem_iUnion, exists_prop, mem_inter_iff, not_and,
iff_self_iff, mem_iInter, mem_compl_iff] using ht
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
ι : Type v
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : s ∩ ⋂ (i : ι), Z i = ∅
⊢ s ∩ ⋂ (i : Finset ι) (i_1 : ι) (_ : i_1 ∈ i), Z i_1 = ∅
[PROOFSTEP]
rwa [← iInter_eq_iInter_finset]
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
ι : Type u_3
f : ι → Set α
hf : LocallyFinite f
s : Set α
hs : IsCompact s
⊢ Set.Finite {i | Set.Nonempty (f i ∩ s)}
[PROOFSTEP]
choose U hxU hUf using hf
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
ι : Type u_3
f : ι → Set α
s : Set α
hs : IsCompact s
U : α → Set α
hxU : ∀ (x : α), U x ∈ 𝓝 x
hUf : ∀ (x : α), Set.Finite {i | Set.Nonempty (f i ∩ U x)}
⊢ Set.Finite {i | Set.Nonempty (f i ∩ s)}
[PROOFSTEP]
rcases hs.elim_nhds_subcover U fun x _ => hxU x with ⟨t, -, hsU⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
ι : Type u_3
f : ι → Set α
s : Set α
hs : IsCompact s
U : α → Set α
hxU : ∀ (x : α), U x ∈ 𝓝 x
hUf : ∀ (x : α), Set.Finite {i | Set.Nonempty (f i ∩ U x)}
t : Finset α
hsU : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
⊢ Set.Finite {i | Set.Nonempty (f i ∩ s)}
[PROOFSTEP]
refine' (t.finite_toSet.biUnion fun x _ => hUf x).subset _
[GOAL]
case intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
ι : Type u_3
f : ι → Set α
s : Set α
hs : IsCompact s
U : α → Set α
hxU : ∀ (x : α), U x ∈ 𝓝 x
hUf : ∀ (x : α), Set.Finite {i | Set.Nonempty (f i ∩ U x)}
t : Finset α
hsU : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
⊢ {i | Set.Nonempty (f i ∩ s)} ⊆ ⋃ (i : α) (_ : i ∈ ↑t), {i_1 | Set.Nonempty (f i_1 ∩ U i)}
[PROOFSTEP]
rintro i ⟨x, hx⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
ι : Type u_3
f : ι → Set α
s : Set α
hs : IsCompact s
U : α → Set α
hxU : ∀ (x : α), U x ∈ 𝓝 x
hUf : ∀ (x : α), Set.Finite {i | Set.Nonempty (f i ∩ U x)}
t : Finset α
hsU : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
i : ι
x : α
hx : x ∈ f i ∩ s
⊢ i ∈ ⋃ (i : α) (_ : i ∈ ↑t), {i_1 | Set.Nonempty (f i_1 ∩ U i)}
[PROOFSTEP]
rcases mem_iUnion₂.1 (hsU hx.2) with ⟨c, hct, hcx⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
ι : Type u_3
f : ι → Set α
s : Set α
hs : IsCompact s
U : α → Set α
hxU : ∀ (x : α), U x ∈ 𝓝 x
hUf : ∀ (x : α), Set.Finite {i | Set.Nonempty (f i ∩ U x)}
t : Finset α
hsU : s ⊆ ⋃ (x : α) (_ : x ∈ t), U x
i : ι
x : α
hx : x ∈ f i ∩ s
c : α
hct : c ∈ t
hcx : x ∈ U c
⊢ i ∈ ⋃ (i : α) (_ : i ∈ ↑t), {i_1 | Set.Nonempty (f i_1 ∩ U i)}
[PROOFSTEP]
exact mem_biUnion hct ⟨x, hx.1, hcx⟩
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
ι : Type v
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : ∀ (t : Finset ι), Set.Nonempty (s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i)
⊢ Set.Nonempty (s ∩ ⋂ (i : ι), Z i)
[PROOFSTEP]
simp only [nonempty_iff_ne_empty] at hsZ ⊢
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
ι : Type v
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : ∀ (t : Finset ι), s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i ≠ ∅
⊢ s ∩ ⋂ (i : ι), Z i ≠ ∅
[PROOFSTEP]
apply mt (hs.elim_finite_subfamily_closed Z hZc)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
ι : Type v
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : ∀ (t : Finset ι), s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i ≠ ∅
⊢ ¬∃ t, s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i = ∅
[PROOFSTEP]
push_neg
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
ι : Type v
hs : IsCompact s
Z : ι → Set α
hZc : ∀ (i : ι), IsClosed (Z i)
hsZ : ∀ (t : Finset ι), s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i ≠ ∅
⊢ ∀ (t : Finset ι), s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i ≠ ∅
[PROOFSTEP]
exact hsZ
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZn : ∀ (i : ι), Set.Nonempty (Z i)
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
⊢ Set.Nonempty (⋂ (i : ι), Z i)
[PROOFSTEP]
let i₀ := hι.some
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZn : ∀ (i : ι), Set.Nonempty (Z i)
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
⊢ Set.Nonempty (⋂ (i : ι), Z i)
[PROOFSTEP]
suffices (Z i₀ ∩ ⋂ i, Z i).Nonempty by rwa [inter_eq_right_iff_subset.mpr (iInter_subset _ i₀)] at this
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZn : ∀ (i : ι), Set.Nonempty (Z i)
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
this : Set.Nonempty (Z i₀ ∩ ⋂ (i : ι), Z i)
⊢ Set.Nonempty (⋂ (i : ι), Z i)
[PROOFSTEP]
rwa [inter_eq_right_iff_subset.mpr (iInter_subset _ i₀)] at this
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZn : ∀ (i : ι), Set.Nonempty (Z i)
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
⊢ Set.Nonempty (Z i₀ ∩ ⋂ (i : ι), Z i)
[PROOFSTEP]
simp only [nonempty_iff_ne_empty] at hZn ⊢
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
hZn : ∀ (i : ι), Z i ≠ ∅
⊢ Z (Nonempty.some hι) ∩ ⋂ (i : ι), Z i ≠ ∅
[PROOFSTEP]
apply mt ((hZc i₀).elim_directed_family_closed Z hZcl)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
hZn : ∀ (i : ι), Z i ≠ ∅
⊢ ¬(Directed (fun x x_1 => x ⊇ x_1) Z → ∃ i, Z i₀ ∩ Z i = ∅)
[PROOFSTEP]
push_neg
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
hZn : ∀ (i : ι), Z i ≠ ∅
⊢ Directed (fun x x_1 => x ⊇ x_1) Z ∧ ∀ (i : ι), Z (Nonempty.some hι) ∩ Z i ≠ ∅
[PROOFSTEP]
simp only [← nonempty_iff_ne_empty] at hZn ⊢
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
hZn : ∀ (i : ι), Set.Nonempty (Z i)
⊢ Directed (fun x x_1 => x ⊇ x_1) Z ∧ ∀ (i : ι), Set.Nonempty (Z (Nonempty.some hι) ∩ Z i)
[PROOFSTEP]
refine' ⟨hZd, fun i => _⟩
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
hZn : ∀ (i : ι), Set.Nonempty (Z i)
i : ι
⊢ Set.Nonempty (Z (Nonempty.some hι) ∩ Z i)
[PROOFSTEP]
rcases hZd i₀ i with ⟨j, hji₀, hji⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
ι : Type v
hι : Nonempty ι
Z : ι → Set α
hZd : Directed (fun x x_1 => x ⊇ x_1) Z
hZc : ∀ (i : ι), IsCompact (Z i)
hZcl : ∀ (i : ι), IsClosed (Z i)
i₀ : ι := Nonempty.some hι
hZn : ∀ (i : ι), Set.Nonempty (Z i)
i j : ι
hji₀ : Z i₀ ⊇ Z j
hji : Z i ⊇ Z j
⊢ Set.Nonempty (Z (Nonempty.some hι) ∩ Z i)
[PROOFSTEP]
exact (hZn j).mono (subset_inter hji₀ hji)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : Set ι
c : ι → Set α
hs : IsCompact s
hc₁ : ∀ (i : ι), i ∈ b → IsOpen (c i)
hc₂ : s ⊆ ⋃ (i : ι) (_ : i ∈ b), c i
⊢ ∃ b', b' ⊆ b ∧ Set.Finite b' ∧ s ⊆ ⋃ (i : ι) (_ : i ∈ b'), c i
[PROOFSTEP]
simp only [Subtype.forall', biUnion_eq_iUnion] at hc₁ hc₂
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : Set ι
c : ι → Set α
hs : IsCompact s
hc₁ : ∀ (x : { a // a ∈ b }), IsOpen (c ↑x)
hc₂ : s ⊆ ⋃ (x : ↑b), c ↑x
⊢ ∃ b', b' ⊆ b ∧ Set.Finite b' ∧ s ⊆ ⋃ (i : ι) (_ : i ∈ b'), c i
[PROOFSTEP]
rcases hs.elim_finite_subcover (fun i => c i : b → Set α) hc₁ hc₂ with ⟨d, hd⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : Set ι
c : ι → Set α
hs : IsCompact s
hc₁ : ∀ (x : { a // a ∈ b }), IsOpen (c ↑x)
hc₂ : s ⊆ ⋃ (x : ↑b), c ↑x
d : Finset ↑b
hd : s ⊆ ⋃ (i : ↑b) (_ : i ∈ d), c ↑i
⊢ ∃ b', b' ⊆ b ∧ Set.Finite b' ∧ s ⊆ ⋃ (i : ι) (_ : i ∈ b'), c i
[PROOFSTEP]
refine' ⟨Subtype.val '' d.toSet, _, d.finite_toSet.image _, _⟩
[GOAL]
case intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : Set ι
c : ι → Set α
hs : IsCompact s
hc₁ : ∀ (x : { a // a ∈ b }), IsOpen (c ↑x)
hc₂ : s ⊆ ⋃ (x : ↑b), c ↑x
d : Finset ↑b
hd : s ⊆ ⋃ (i : ↑b) (_ : i ∈ d), c ↑i
⊢ Subtype.val '' ↑d ⊆ b
[PROOFSTEP]
simp
[GOAL]
case intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : Set ι
c : ι → Set α
hs : IsCompact s
hc₁ : ∀ (x : { a // a ∈ b }), IsOpen (c ↑x)
hc₂ : s ⊆ ⋃ (x : ↑b), c ↑x
d : Finset ↑b
hd : s ⊆ ⋃ (i : ↑b) (_ : i ∈ d), c ↑i
⊢ s ⊆ ⋃ (i : ι) (_ : i ∈ Subtype.val '' ↑d), c i
[PROOFSTEP]
rwa [biUnion_image]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
h : ∀ {ι : Type u} (U : ι → Set α), (∀ (i : ι), IsOpen (U i)) → s ⊆ ⋃ (i : ι), U i → ∃ t, s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
⊢ ∃ a, a ∈ s ∧ ClusterPt a f
[PROOFSTEP]
contrapose! h
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
h : ∀ (a : α), a ∈ s → ¬ClusterPt a f
⊢ Exists fun {ι} =>
∃ U, (∀ (i : ι), IsOpen (U i)) ∧ s ⊆ ⋃ (i : ι), U i ∧ ∀ (t : Finset ι), ¬s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i
[PROOFSTEP]
simp only [ClusterPt, not_neBot, ← disjoint_iff, SetCoe.forall', (nhds_basis_opens _).disjoint_iff_left] at h
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
h : ∀ (x : ↑s), ∃ i, (↑x ∈ i ∧ IsOpen i) ∧ iᶜ ∈ f
⊢ Exists fun {ι} =>
∃ U, (∀ (i : ι), IsOpen (U i)) ∧ s ⊆ ⋃ (i : ι), U i ∧ ∀ (t : Finset ι), ¬s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i
[PROOFSTEP]
choose U hU hUf using h
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
U : ↑s → Set α
hU : ∀ (x : ↑s), ↑x ∈ U x ∧ IsOpen (U x)
hUf : ∀ (x : ↑s), (U x)ᶜ ∈ f
⊢ Exists fun {ι} =>
∃ U, (∀ (i : ι), IsOpen (U i)) ∧ s ⊆ ⋃ (i : ι), U i ∧ ∀ (t : Finset ι), ¬s ⊆ ⋃ (i : ι) (_ : i ∈ t), U i
[PROOFSTEP]
refine ⟨s, U, fun x => (hU x).2, fun x hx => mem_iUnion.2 ⟨⟨x, hx⟩, (hU _).1⟩, fun t ht => ?_⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
U : ↑s → Set α
hU : ∀ (x : ↑s), ↑x ∈ U x ∧ IsOpen (U x)
hUf : ∀ (x : ↑s), (U x)ᶜ ∈ f
t : Finset ↑s
ht : s ⊆ ⋃ (i : ↑s) (_ : i ∈ t), U i
⊢ False
[PROOFSTEP]
refine compl_not_mem (le_principal_iff.1 hfs) ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
U : ↑s → Set α
hU : ∀ (x : ↑s), ↑x ∈ U x ∧ IsOpen (U x)
hUf : ∀ (x : ↑s), (U x)ᶜ ∈ f
t : Finset ↑s
ht : s ⊆ ⋃ (i : ↑s) (_ : i ∈ t), U i
⊢ sᶜ ∈ f
[PROOFSTEP]
refine mem_of_superset ((biInter_finset_mem t).2 fun x _ => hUf x) ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
U : ↑s → Set α
hU : ∀ (x : ↑s), ↑x ∈ U x ∧ IsOpen (U x)
hUf : ∀ (x : ↑s), (U x)ᶜ ∈ f
t : Finset ↑s
ht : s ⊆ ⋃ (i : ↑s) (_ : i ∈ t), U i
⊢ ⋂ (i : ↑s) (_ : i ∈ t), (U i)ᶜ ⊆ sᶜ
[PROOFSTEP]
rw [subset_compl_comm, compl_iInter₂]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
f : Filter α
hf : NeBot f
hfs : f ≤ 𝓟 s
U : ↑s → Set α
hU : ∀ (x : ↑s), ↑x ∈ U x ∧ IsOpen (U x)
hUf : ∀ (x : ↑s), (U x)ᶜ ∈ f
t : Finset ↑s
ht : s ⊆ ⋃ (i : ↑s) (_ : i ∈ t), U i
⊢ s ⊆ ⋃ (i : ↑s) (_ : i ∈ t), (U i)ᶜᶜ
[PROOFSTEP]
simpa only [compl_compl]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
h :
∀ {ι : Type u} (Z : ι → Set α),
(∀ (i : ι), IsClosed (Z i)) → s ∩ ⋂ (i : ι), Z i = ∅ → ∃ t, s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i = ∅
ι✝ : Type u
U : ι✝ → Set α
hUo : ∀ (i : ι✝), IsOpen (U i)
hsU : s ⊆ ⋃ (i : ι✝), U i
⊢ ∃ t, s ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
[PROOFSTEP]
rw [← disjoint_compl_right_iff_subset, compl_iUnion, disjoint_iff] at hsU
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
h :
∀ {ι : Type u} (Z : ι → Set α),
(∀ (i : ι), IsClosed (Z i)) → s ∩ ⋂ (i : ι), Z i = ∅ → ∃ t, s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i = ∅
ι✝ : Type u
U : ι✝ → Set α
hUo : ∀ (i : ι✝), IsOpen (U i)
hsU : s ⊓ ⋂ (i : ι✝), (U i)ᶜ = ⊥
⊢ ∃ t, s ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
[PROOFSTEP]
rcases h (fun i => (U i)ᶜ) (fun i => (hUo _).isClosed_compl) hsU with ⟨t, ht⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
h :
∀ {ι : Type u} (Z : ι → Set α),
(∀ (i : ι), IsClosed (Z i)) → s ∩ ⋂ (i : ι), Z i = ∅ → ∃ t, s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i = ∅
ι✝ : Type u
U : ι✝ → Set α
hUo : ∀ (i : ι✝), IsOpen (U i)
hsU : s ⊓ ⋂ (i : ι✝), (U i)ᶜ = ⊥
t : Finset ι✝
ht : s ∩ ⋂ (i : ι✝) (_ : i ∈ t), (U i)ᶜ = ∅
⊢ ∃ t, s ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
[PROOFSTEP]
refine ⟨t, ?_⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
h :
∀ {ι : Type u} (Z : ι → Set α),
(∀ (i : ι), IsClosed (Z i)) → s ∩ ⋂ (i : ι), Z i = ∅ → ∃ t, s ∩ ⋂ (i : ι) (_ : i ∈ t), Z i = ∅
ι✝ : Type u
U : ι✝ → Set α
hUo : ∀ (i : ι✝), IsOpen (U i)
hsU : s ⊓ ⋂ (i : ι✝), (U i)ᶜ = ⊥
t : Finset ι✝
ht : s ∩ ⋂ (i : ι✝) (_ : i ∈ t), (U i)ᶜ = ∅
⊢ s ⊆ ⋃ (i : ι✝) (_ : i ∈ t), U i
[PROOFSTEP]
rwa [← disjoint_compl_right_iff_subset, compl_iUnion₂, disjoint_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
⊢ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ K → P x y
[PROOFSTEP]
refine' hK.induction_on _ _ _ _
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
⊢ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ ∅ → P x y
[PROOFSTEP]
exact eventually_of_forall fun x y => False.elim
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
⊢ ∀ ⦃s t : Set β⦄, s ⊆ t → (∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y) → ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y
[PROOFSTEP]
intro s t hst ht
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
s t : Set β
hst : s ⊆ t
ht : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
⊢ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y
[PROOFSTEP]
refine' ht.mono fun x h y hys => h y <| hst hys
[GOAL]
case refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
⊢ ∀ ⦃s t : Set β⦄,
(∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y) →
(∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y) → ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s ∪ t → P x y
[PROOFSTEP]
intro s t hs ht
[GOAL]
case refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
s t : Set β
hs : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y
ht : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
⊢ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s ∪ t → P x y
[PROOFSTEP]
filter_upwards [hs, ht]
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
s t : Set β
hs : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y
ht : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
⊢ ∀ (a : α), (∀ (y : β), y ∈ s → P a y) → (∀ (y : β), y ∈ t → P a y) → ∀ (y : β), y ∈ s ∪ t → P a y
[PROOFSTEP]
rintro x h1 h2 y (hys | hyt)
[GOAL]
case h.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
s t : Set β
hs : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y
ht : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
x : α
h1 : ∀ (y : β), y ∈ s → P x y
h2 : ∀ (y : β), y ∈ t → P x y
y : β
hys : y ∈ s
⊢ P x y
case h.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
s t : Set β
hs : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ s → P x y
ht : ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
x : α
h1 : ∀ (y : β), y ∈ s → P x y
h2 : ∀ (y : β), y ∈ t → P x y
y : β
hyt : y ∈ t
⊢ P x y
[PROOFSTEP]
exacts [h1 y hys, h2 y hyt]
[GOAL]
case refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
⊢ ∀ (x : β), x ∈ K → ∃ t, t ∈ 𝓝[K] x ∧ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
[PROOFSTEP]
intro y hyK
[GOAL]
case refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
hP : ∀ (y : β), y ∈ K → ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
y : β
hyK : y ∈ K
⊢ ∃ t, t ∈ 𝓝[K] y ∧ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
[PROOFSTEP]
specialize hP y hyK
[GOAL]
case refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
y : β
hyK : y ∈ K
hP : ∀ᶠ (z : α × β) in 𝓝 (x₀, y), P z.fst z.snd
⊢ ∃ t, t ∈ 𝓝[K] y ∧ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
[PROOFSTEP]
rw [nhds_prod_eq, eventually_prod_iff] at hP
[GOAL]
case refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
y : β
hyK : y ∈ K
hP :
∃ pa,
(∀ᶠ (x : α) in 𝓝 x₀, pa x) ∧
∃ pb, (∀ᶠ (y : β) in 𝓝 y, pb y) ∧ ∀ {x : α}, pa x → ∀ {y : β}, pb y → P (x, y).fst (x, y).snd
⊢ ∃ t, t ∈ 𝓝[K] y ∧ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
[PROOFSTEP]
rcases hP with ⟨p, hp, q, hq, hpq⟩
[GOAL]
case refine'_4.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x₀ : α
K : Set β
hK : IsCompact K
P : α → β → Prop
y : β
hyK : y ∈ K
p : α → Prop
hp : ∀ᶠ (x : α) in 𝓝 x₀, p x
q : β → Prop
hq : ∀ᶠ (y : β) in 𝓝 y, q y
hpq : ∀ {x : α}, p x → ∀ {y : β}, q y → P (x, y).fst (x, y).snd
⊢ ∃ t, t ∈ 𝓝[K] y ∧ ∀ᶠ (x : α) in 𝓝 x₀, ∀ (y : β), y ∈ t → P x y
[PROOFSTEP]
exact ⟨{y | q y}, mem_nhdsWithin_of_mem_nhds hq, eventually_of_mem hp @hpq⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
a : α
f : Filter α
hf : NeBot f
hfa : f ≤ 𝓟 {a}
⊢ 𝓟 {a} ≤ 𝓝 a
[PROOFSTEP]
simpa only [principal_singleton] using pure_le_nhds a
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
s : Set ι
f : ι → Set α
hs : Set.Finite s
hf : ∀ (i : ι), i ∈ s → IsCompact (f i)
l : Ultrafilter α
hl : ↑l ≤ 𝓟 (⋃ (i : ι) (_ : i ∈ s), f i)
⊢ ∃ a, a ∈ ⋃ (i : ι) (_ : i ∈ s), f i ∧ ↑l ≤ 𝓝 a
[PROOFSTEP]
rw [le_principal_iff, Ultrafilter.mem_coe, Ultrafilter.finite_biUnion_mem_iff hs] at hl
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
s : Set ι
f : ι → Set α
hs : Set.Finite s
hf : ∀ (i : ι), i ∈ s → IsCompact (f i)
l : Ultrafilter α
hl : ∃ i, i ∈ s ∧ f i ∈ l
⊢ ∃ a, a ∈ ⋃ (i : ι) (_ : i ∈ s), f i ∧ ↑l ≤ 𝓝 a
[PROOFSTEP]
rcases hl with ⟨i, his, hi⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
s : Set ι
f : ι → Set α
hs : Set.Finite s
hf : ∀ (i : ι), i ∈ s → IsCompact (f i)
l : Ultrafilter α
i : ι
his : i ∈ s
hi : f i ∈ l
⊢ ∃ a, a ∈ ⋃ (i : ι) (_ : i ∈ s), f i ∧ ↑l ≤ 𝓝 a
[PROOFSTEP]
rcases(hf i his).ultrafilter_le_nhds _ (le_principal_iff.2 hi) with ⟨x, hxi, hlx⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
s : Set ι
f : ι → Set α
hs : Set.Finite s
hf : ∀ (i : ι), i ∈ s → IsCompact (f i)
l : Ultrafilter α
i : ι
his : i ∈ s
hi : f i ∈ l
x : α
hxi : x ∈ f i
hlx : ↑l ≤ 𝓝 x
⊢ ∃ a, a ∈ ⋃ (i : ι) (_ : i ∈ s), f i ∧ ↑l ≤ 𝓝 a
[PROOFSTEP]
exact ⟨x, mem_iUnion₂.2 ⟨i, his, hxi⟩, hlx⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
S : Set (Set α)
hf : Set.Finite S
hc : ∀ (s : Set α), s ∈ S → IsCompact s
⊢ IsCompact (⋃₀ S)
[PROOFSTEP]
rw [sUnion_eq_biUnion]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
S : Set (Set α)
hf : Set.Finite S
hc : ∀ (s : Set α), s ∈ S → IsCompact s
⊢ IsCompact (⋃ (i : Set α) (_ : i ∈ S), i)
[PROOFSTEP]
exact hf.isCompact_biUnion hc
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : DiscreteTopology α
s : Set α
hs : IsCompact s
⊢ Set.Finite s
[PROOFSTEP]
have : ∀ x : α, ({ x } : Set α) ∈ 𝓝 x := by simp [nhds_discrete]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : DiscreteTopology α
s : Set α
hs : IsCompact s
⊢ ∀ (x : α), {x} ∈ 𝓝 x
[PROOFSTEP]
simp [nhds_discrete]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : DiscreteTopology α
s : Set α
hs : IsCompact s
this : ∀ (x : α), {x} ∈ 𝓝 x
⊢ Set.Finite s
[PROOFSTEP]
rcases hs.elim_nhds_subcover (fun x => { x }) fun x _ => this x with ⟨t, _, hst⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : DiscreteTopology α
s : Set α
hs : IsCompact s
this : ∀ (x : α), {x} ∈ 𝓝 x
t : Finset α
left✝ : ∀ (x : α), x ∈ t → x ∈ s
hst : s ⊆ ⋃ (x : α) (_ : x ∈ t), {x}
⊢ Set.Finite s
[PROOFSTEP]
simp only [← t.set_biUnion_coe, biUnion_of_singleton] at hst
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : DiscreteTopology α
s : Set α
hs : IsCompact s
this : ∀ (x : α), {x} ∈ 𝓝 x
t : Finset α
left✝ : ∀ (x : α), x ∈ t → x ∈ s
hst : s ⊆ ↑t
⊢ Set.Finite s
[PROOFSTEP]
exact t.finite_toSet.subset hst
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsCompact t
⊢ IsCompact (s ∪ t)
[PROOFSTEP]
rw [union_eq_iUnion]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsCompact t
⊢ IsCompact (⋃ (b : Bool), bif b then s else t)
[PROOFSTEP]
exact isCompact_iUnion fun b => by cases b <;> assumption
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsCompact t
b : Bool
⊢ IsCompact (bif b then s else t)
[PROOFSTEP]
cases b
[GOAL]
case false
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsCompact t
⊢ IsCompact (bif false then s else t)
[PROOFSTEP]
assumption
[GOAL]
case true
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hs : IsCompact s
ht : IsCompact t
⊢ IsCompact (bif true then s else t)
[PROOFSTEP]
assumption
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
⊢ ∃ i, V i ⊆ U
[PROOFSTEP]
obtain ⟨W, hsubW, W_op, hWU⟩ := exists_open_set_nhds hU
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
⊢ ∃ i, V i ⊆ U
[PROOFSTEP]
suffices : ∃ i, V i ⊆ W
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
this : ∃ i, V i ⊆ W
⊢ ∃ i, V i ⊆ U
[PROOFSTEP]
exact this.imp fun i hi => hi.trans hWU
[GOAL]
case this
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
⊢ ∃ i, V i ⊆ W
[PROOFSTEP]
by_contra' H
[GOAL]
case this
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), ¬V i ⊆ W
⊢ False
[PROOFSTEP]
replace H : ∀ i, (V i ∩ Wᶜ).Nonempty := fun i => Set.inter_compl_nonempty_iff.mpr (H i)
[GOAL]
case this
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
⊢ False
[PROOFSTEP]
have : (⋂ i, V i ∩ Wᶜ).Nonempty :=
by
refine'
IsCompact.nonempty_iInter_of_directed_nonempty_compact_closed _ (fun i j => _) H
(fun i => (hV_cpct i).inter_right W_op.isClosed_compl) fun i => (hV_closed i).inter W_op.isClosed_compl
rcases hV i j with ⟨k, hki, hkj⟩
refine' ⟨k, ⟨fun x => _, fun x => _⟩⟩ <;> simp only [and_imp, mem_inter_iff, mem_compl_iff] <;> tauto
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
⊢ Set.Nonempty (⋂ (i : ι), V i ∩ Wᶜ)
[PROOFSTEP]
refine'
IsCompact.nonempty_iInter_of_directed_nonempty_compact_closed _ (fun i j => _) H
(fun i => (hV_cpct i).inter_right W_op.isClosed_compl) fun i => (hV_closed i).inter W_op.isClosed_compl
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
i j : ι
⊢ ∃ z, (fun x x_1 => x ⊇ x_1) (V i ∩ Wᶜ) (V z ∩ Wᶜ) ∧ (fun x x_1 => x ⊇ x_1) (V j ∩ Wᶜ) (V z ∩ Wᶜ)
[PROOFSTEP]
rcases hV i j with ⟨k, hki, hkj⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
i j k : ι
hki : V i ⊇ V k
hkj : V j ⊇ V k
⊢ ∃ z, (fun x x_1 => x ⊇ x_1) (V i ∩ Wᶜ) (V z ∩ Wᶜ) ∧ (fun x x_1 => x ⊇ x_1) (V j ∩ Wᶜ) (V z ∩ Wᶜ)
[PROOFSTEP]
refine' ⟨k, ⟨fun x => _, fun x => _⟩⟩
[GOAL]
case intro.intro.refine'_1
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
i j k : ι
hki : V i ⊇ V k
hkj : V j ⊇ V k
x : α
⊢ x ∈ V k ∩ Wᶜ → x ∈ V i ∩ Wᶜ
[PROOFSTEP]
simp only [and_imp, mem_inter_iff, mem_compl_iff]
[GOAL]
case intro.intro.refine'_2
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
i j k : ι
hki : V i ⊇ V k
hkj : V j ⊇ V k
x : α
⊢ x ∈ V k ∩ Wᶜ → x ∈ V j ∩ Wᶜ
[PROOFSTEP]
simp only [and_imp, mem_inter_iff, mem_compl_iff]
[GOAL]
case intro.intro.refine'_1
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
i j k : ι
hki : V i ⊇ V k
hkj : V j ⊇ V k
x : α
⊢ x ∈ V k → ¬x ∈ W → x ∈ V i ∧ ¬x ∈ W
[PROOFSTEP]
tauto
[GOAL]
case intro.intro.refine'_2
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
i j k : ι
hki : V i ⊇ V k
hkj : V j ⊇ V k
x : α
⊢ x ∈ V k → ¬x ∈ W → x ∈ V j ∧ ¬x ∈ W
[PROOFSTEP]
tauto
[GOAL]
case this
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
this : Set.Nonempty (⋂ (i : ι), V i ∩ Wᶜ)
⊢ False
[PROOFSTEP]
have : ¬⋂ i : ι, V i ⊆ W := by simpa [← iInter_inter, inter_compl_nonempty_iff]
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
this : Set.Nonempty (⋂ (i : ι), V i ∩ Wᶜ)
⊢ ¬⋂ (i : ι), V i ⊆ W
[PROOFSTEP]
simpa [← iInter_inter, inter_compl_nonempty_iff]
[GOAL]
case this
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : Nonempty ι
V : ι → Set α
hV : Directed (fun x x_1 => x ⊇ x_1) V
hV_cpct : ∀ (i : ι), IsCompact (V i)
hV_closed : ∀ (i : ι), IsClosed (V i)
U : Set α
hU : ∀ (x : α), x ∈ ⋂ (i : ι), V i → U ∈ 𝓝 x
W : Set α
hsubW : ⋂ (i : ι), V i ⊆ W
W_op : IsOpen W
hWU : W ⊆ U
H : ∀ (i : ι), Set.Nonempty (V i ∩ Wᶜ)
this✝ : Set.Nonempty (⋂ (i : ι), V i ∩ Wᶜ)
this : ¬⋂ (i : ι), V i ⊆ W
⊢ False
[PROOFSTEP]
contradiction
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
⊢ IsCompact U ∧ IsOpen U ↔ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
⊢ IsCompact U ∧ IsOpen U → ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
rintro ⟨h₁, h₂⟩
[GOAL]
case mp.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
⊢ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
obtain ⟨β, f, e, hf⟩ := hb.open_eq_iUnion h₂
[GOAL]
case mp.intro.intro.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f : β → Set α
e : U = ⋃ (i : β), f i
hf : ∀ (i : β), f i ∈ range b
⊢ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
choose f' hf' using hf
[GOAL]
case mp.intro.intro.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f : β → Set α
e : U = ⋃ (i : β), f i
f' : β → ι
hf' : ∀ (i : β), b (f' i) = f i
⊢ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
have : b ∘ f' = f := funext hf'
[GOAL]
case mp.intro.intro.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f : β → Set α
e : U = ⋃ (i : β), f i
f' : β → ι
hf' : ∀ (i : β), b (f' i) = f i
this : b ∘ f' = f
⊢ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
subst this
[GOAL]
case mp.intro.intro.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
⊢ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
obtain ⟨t, ht⟩ := h₁.elim_finite_subcover (b ∘ f') (fun i => hb.isOpen (Set.mem_range_self _)) (by rw [e])
[GOAL]
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
⊢ U ⊆ ⋃ (i : β), (b ∘ f') i
[PROOFSTEP]
rw [e]
[GOAL]
case mp.intro.intro.intro.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
⊢ ∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i
[PROOFSTEP]
refine' ⟨t.image f', Set.Finite.intro inferInstance, le_antisymm _ _⟩
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_1
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
⊢ U ≤ ⋃ (i : ι) (_ : i ∈ ↑(Finset.image f' t)), b i
[PROOFSTEP]
refine' Set.Subset.trans ht _
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_1
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
⊢ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i ⊆ ⋃ (i : ι) (_ : i ∈ ↑(Finset.image f' t)), b i
[PROOFSTEP]
simp only [Set.iUnion_subset_iff]
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_1
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
⊢ ∀ (i : β), i ∈ t → (b ∘ f') i ⊆ ⋃ (i : ι) (_ : i ∈ ↑(Finset.image f' t)), b i
[PROOFSTEP]
intro i hi
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_1
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
i : β
hi : i ∈ t
⊢ (b ∘ f') i ⊆ ⋃ (i : ι) (_ : i ∈ ↑(Finset.image f' t)), b i
[PROOFSTEP]
erw [← Set.iUnion_subtype (fun x : ι => x ∈ t.image f') fun i => b i.1]
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_1
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
i : β
hi : i ∈ t
⊢ (b ∘ f') i ⊆ ⋃ (x : { x // x ∈ Finset.image f' t }), b ↑x
[PROOFSTEP]
exact Set.subset_iUnion (fun i : t.image f' => b i) ⟨_, Finset.mem_image_of_mem _ hi⟩
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_2
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
⊢ ⋃ (i : ι) (_ : i ∈ ↑(Finset.image f' t)), b i ≤ U
[PROOFSTEP]
apply Set.iUnion₂_subset
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_2.h
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
⊢ ∀ (i : ι), i ∈ ↑(Finset.image f' t) → b i ⊆ U
[PROOFSTEP]
rintro i hi
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_2.h
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
i : ι
hi : i ∈ ↑(Finset.image f' t)
⊢ b i ⊆ U
[PROOFSTEP]
obtain ⟨j, -, rfl⟩ := Finset.mem_image.mp hi
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_2.h.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
j : β
hi : f' j ∈ ↑(Finset.image f' t)
⊢ b (f' j) ⊆ U
[PROOFSTEP]
rw [e]
[GOAL]
case mp.intro.intro.intro.intro.intro.refine'_2.h.intro.intro
α : Type u
β✝ : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β✝
s t✝ : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
h₁ : IsCompact U
h₂ : IsOpen U
β : Type u
f' : β → ι
e : U = ⋃ (i : β), (b ∘ f') i
hf' : ∀ (i : β), b (f' i) = (b ∘ f') i
t : Finset β
ht : U ⊆ ⋃ (i : β) (_ : i ∈ t), (b ∘ f') i
j : β
hi : f' j ∈ ↑(Finset.image f' t)
⊢ b (f' j) ⊆ ⋃ (i : β), (b ∘ f') i
[PROOFSTEP]
exact Set.subset_iUnion (b ∘ f') j
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
U : Set α
⊢ (∃ s, Set.Finite s ∧ U = ⋃ (i : ι) (_ : i ∈ s), b i) → IsCompact U ∧ IsOpen U
[PROOFSTEP]
rintro ⟨s, hs, rfl⟩
[GOAL]
case mpr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
s : Set ι
hs : Set.Finite s
⊢ IsCompact (⋃ (i : ι) (_ : i ∈ s), b i) ∧ IsOpen (⋃ (i : ι) (_ : i ∈ s), b i)
[PROOFSTEP]
constructor
[GOAL]
case mpr.intro.intro.left
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
s : Set ι
hs : Set.Finite s
⊢ IsCompact (⋃ (i : ι) (_ : i ∈ s), b i)
[PROOFSTEP]
exact hs.isCompact_biUnion fun i _ => hb' i
[GOAL]
case mpr.intro.intro.right
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
b : ι → Set α
hb : IsTopologicalBasis (range b)
hb' : ∀ (i : ι), IsCompact (b i)
s : Set ι
hs : Set.Finite s
⊢ IsOpen (⋃ (i : ι) (_ : i ∈ s), b i)
[PROOFSTEP]
exact isOpen_biUnion fun i _ => hb.isOpen (Set.mem_range_self _)
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α✝
inst✝² : TopologicalSpace β
s t : Set α✝
α : Type u_3
inst✝¹ : TopologicalSpace α
inst✝ : DiscreteTopology α
⊢ cocompact α = cofinite
[PROOFSTEP]
simp only [cocompact, hasBasis_cofinite.eq_biInf, isCompact_iff_finite]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
⊢ IsCompact (insert b (range f))
[PROOFSTEP]
intro l hne hle
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
by_cases hb : ClusterPt b l
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
hb : ClusterPt b l
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
exact ⟨b, Or.inl rfl, hb⟩
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
hb : ¬ClusterPt b l
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
simp only [clusterPt_iff, not_forall, ← not_disjoint_iff_nonempty_inter, not_not] at hb
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
hb : ∃ x h x_1 h, Disjoint x x_1
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
rcases hb with ⟨s, hsb, t, htl, hd⟩
[GOAL]
case neg.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
rcases mem_cocompact.1 (hf hsb) with ⟨K, hKc, hKs⟩
[GOAL]
case neg.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
have : f '' K ∈ l := by
filter_upwards [htl, le_principal_iff.1 hle] with y hyt hyf
rcases hyf with (rfl | ⟨x, rfl⟩)
exacts [(hd.le_bot ⟨mem_of_mem_nhds hsb, hyt⟩).elim,
mem_image_of_mem _ (not_not.1 fun hxK => hd.le_bot ⟨hKs hxK, hyt⟩)]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
⊢ f '' K ∈ l
[PROOFSTEP]
filter_upwards [htl, le_principal_iff.1 hle] with y hyt hyf
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
y : β
hyt : y ∈ t
hyf : y ∈ insert b (range f)
⊢ y ∈ f '' K
[PROOFSTEP]
rcases hyf with (rfl | ⟨x, rfl⟩)
[GOAL]
case h.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
hfc : Continuous f
l : Filter β
hne : NeBot l
s t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
y : β
hyt : y ∈ t
hf : Tendsto f (cocompact α) (𝓝 y)
hle : l ≤ 𝓟 (insert y (range f))
hsb : s ∈ 𝓝 y
⊢ y ∈ f '' K
case h.inr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
x : α
hyt : f x ∈ t
⊢ f x ∈ f '' K
[PROOFSTEP]
exacts [(hd.le_bot ⟨mem_of_mem_nhds hsb, hyt⟩).elim, mem_image_of_mem _ (not_not.1 fun hxK => hd.le_bot ⟨hKs hxK, hyt⟩)]
[GOAL]
case neg.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
this : f '' K ∈ l
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
rcases hKc.image hfc (le_principal_iff.2 this) with ⟨y, hy, hyl⟩
[GOAL]
case neg.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ : Set α
f : α → β
b : β
hf : Tendsto f (cocompact α) (𝓝 b)
hfc : Continuous f
l : Filter β
hne : NeBot l
hle : l ≤ 𝓟 (insert b (range f))
s : Set β
hsb : s ∈ 𝓝 b
t : Set β
htl : t ∈ l
hd : Disjoint s t
K : Set α
hKc : IsCompact K
hKs : Kᶜ ⊆ f ⁻¹' s
this : f '' K ∈ l
y : β
hy : y ∈ f '' K
hyl : ClusterPt y l
⊢ ∃ a, a ∈ insert b (range f) ∧ ClusterPt a l
[PROOFSTEP]
exact ⟨y, Or.inr <| image_subset_range _ _ hy, hyl⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : ι → α
a : α
hf : Tendsto f cofinite (𝓝 a)
⊢ IsCompact (insert a (range f))
[PROOFSTEP]
letI : TopologicalSpace ι := ⊥
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : ι → α
a : α
hf : Tendsto f cofinite (𝓝 a)
this : TopologicalSpace ι := ⊥
⊢ IsCompact (insert a (range f))
[PROOFSTEP]
haveI h : DiscreteTopology ι := ⟨rfl⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : ι → α
a : α
hf : Tendsto f cofinite (𝓝 a)
this : TopologicalSpace ι := ⊥
h : DiscreteTopology ι
⊢ IsCompact (insert a (range f))
[PROOFSTEP]
rw [← cocompact_eq_cofinite ι] at hf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : ι → α
a : α
this : TopologicalSpace ι := ⊥
hf : Tendsto f (cocompact ι) (𝓝 a)
h : DiscreteTopology ι
⊢ IsCompact (insert a (range f))
[PROOFSTEP]
exact hf.isCompact_insert_range_of_cocompact continuous_of_discreteTopology
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ HasBasis (coclosedCompact α) (fun s => IsClosed s ∧ IsCompact s) compl
[PROOFSTEP]
simp only [Filter.coclosedCompact, iInf_and']
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ HasBasis (⨅ (s : Set α) (_ : IsClosed s ∧ IsCompact s), 𝓟 sᶜ) (fun s => IsClosed s ∧ IsCompact s) compl
[PROOFSTEP]
refine' hasBasis_biInf_principal' _ ⟨∅, isClosed_empty, isCompact_empty⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ ∀ (i : Set α),
IsClosed i ∧ IsCompact i →
∀ (j : Set α), IsClosed j ∧ IsCompact j → ∃ k, (IsClosed k ∧ IsCompact k) ∧ kᶜ ⊆ iᶜ ∧ kᶜ ⊆ jᶜ
[PROOFSTEP]
rintro s ⟨hs₁, hs₂⟩ t ⟨ht₁, ht₂⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
hs₁ : IsClosed s
hs₂ : IsCompact s
t : Set α
ht₁ : IsClosed t
ht₂ : IsCompact t
⊢ ∃ k, (IsClosed k ∧ IsCompact k) ∧ kᶜ ⊆ sᶜ ∧ kᶜ ⊆ tᶜ
[PROOFSTEP]
exact
⟨s ∪ t,
⟨⟨hs₁.union ht₁, hs₂.union ht₂⟩, compl_subset_compl.2 (subset_union_left _ _),
compl_subset_compl.2 (subset_union_right _ _)⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ s ∈ coclosedCompact α ↔ ∃ t, IsClosed t ∧ IsCompact t ∧ tᶜ ⊆ s
[PROOFSTEP]
simp only [hasBasis_coclosedCompact.mem_iff, and_assoc]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ s ∈ coclosedCompact α ↔ ∃ t, IsClosed t ∧ IsCompact t ∧ sᶜ ⊆ t
[PROOFSTEP]
simp only [mem_coclosedCompact, compl_subset_comm]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ IsBounded s ↔ ∃ t, IsCompact t ∧ s ⊆ t
[PROOFSTEP]
change sᶜ ∈ Filter.cocompact α ↔ _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ sᶜ ∈ cocompact α ↔ ∃ t, IsCompact t ∧ s ⊆ t
[PROOFSTEP]
rw [Filter.mem_cocompact]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ (∃ t, IsCompact t ∧ tᶜ ⊆ sᶜ) ↔ ∃ t, IsCompact t ∧ s ⊆ t
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
H : NhdsContainBoxes s t
n : Set (β × α)
hn : IsOpen n
hp : t ×ˢ s ⊆ n
⊢ s ×ˢ t ⊆ Prod.swap ⁻¹' n
[PROOFSTEP]
rwa [← image_subset_iff, image_swap_prod]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
H : NhdsContainBoxes s t
n : Set (β × α)
hn : IsOpen n
hp : t ×ˢ s ⊆ n
u : Set α
v : Set β
uo : IsOpen u
vo : IsOpen v
su : s ⊆ u
tv : t ⊆ v
p : u ×ˢ v ⊆ Prod.swap ⁻¹' n
⊢ v ×ˢ u ⊆ n
[PROOFSTEP]
rwa [← image_subset_iff, image_swap_prod] at p
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x : α
y : β
n : Set (α × β)
hn : IsOpen n
hp : {x} ×ˢ {y} ⊆ n
⊢ (x, y) ∈ {x} ×ˢ {y}
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x : α
y : β
n : Set (α × β)
hn : IsOpen n
hp : {x} ×ˢ {y} ⊆ n
u : Set α
v : Set β
uo : IsOpen u
vo : IsOpen v
xu : x ∈ u
yv : y ∈ v
hp' : u ×ˢ v ⊆ n
⊢ {x} ⊆ u
[PROOFSTEP]
simpa
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
x : α
y : β
n : Set (α × β)
hn : IsOpen n
hp : {x} ×ˢ {y} ⊆ n
u : Set α
v : Set β
uo : IsOpen u
vo : IsOpen v
xu : x ∈ u
yv : y ∈ v
hp' : u ×ˢ v ⊆ n
⊢ {y} ⊆ v
[PROOFSTEP]
simpa
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
hs : IsCompact s
t : Set β
H : ∀ (x : α), x ∈ s → NhdsContainBoxes {x} t
n : Set (α × β)
hn : IsOpen n
hp : s ×ˢ t ⊆ n
x✝ : ↑s
x : α
hx : x ∈ s
⊢ {x} ⊆ s
[PROOFSTEP]
simpa
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
hs : IsCompact s
t : Set β
H : ∀ (x : α), x ∈ s → NhdsContainBoxes {x} t
n : Set (α × β)
hn : IsOpen n
hp : s ×ˢ t ⊆ n
this : ∀ (x : ↑s), ∃ uv, IsOpen uv.fst ∧ IsOpen uv.snd ∧ {↑x} ⊆ uv.fst ∧ t ⊆ uv.snd ∧ uv.fst ×ˢ uv.snd ⊆ n
uvs : ↑s → Set α × Set β
h :
∀ (x : ↑s),
IsOpen (uvs x).fst ∧ IsOpen (uvs x).snd ∧ {↑x} ⊆ (uvs x).fst ∧ t ⊆ (uvs x).snd ∧ (uvs x).fst ×ˢ (uvs x).snd ⊆ n
x : α
hx : x ∈ s
⊢ x ∈ (uvs { val := x, property := hx }).fst
[PROOFSTEP]
simpa using (h ⟨x, hx⟩).2.2.1
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
hs : IsCompact s
t : Set β
H : ∀ (x : α), x ∈ s → NhdsContainBoxes {x} t
n : Set (α × β)
hn : IsOpen n
hp : s ×ˢ t ⊆ n
this✝² : ∀ (x : ↑s), ∃ uv, IsOpen uv.fst ∧ IsOpen uv.snd ∧ {↑x} ⊆ uv.fst ∧ t ⊆ uv.snd ∧ uv.fst ×ˢ uv.snd ⊆ n
uvs : ↑s → Set α × Set β
h :
∀ (x : ↑s),
IsOpen (uvs x).fst ∧ IsOpen (uvs x).snd ∧ {↑x} ⊆ (uvs x).fst ∧ t ⊆ (uvs x).snd ∧ (uvs x).fst ×ˢ (uvs x).snd ⊆ n
us_cover : s ⊆ ⋃ (i : ↑s), (uvs i).fst
s0 : Finset ↑s
s0_cover : s ⊆ ⋃ (i : ↑s) (_ : i ∈ s0), (uvs i).fst
u : Set α := ⋃ (i : ↑s) (_ : i ∈ s0), (uvs i).fst
v : Set β := ⋂ (i : ↑s) (_ : i ∈ s0), (uvs i).snd
this✝¹ : IsOpen u
this✝ : IsOpen v
this : t ⊆ v
x✝¹ : α × β
x' : α
y' : β
x✝ : (x', y') ∈ u ×ˢ v
hx' : (x', y').fst ∈ u
hy' : (x', y').snd ∈ v
⊢ ∃ i, i ∈ s0 ∧ x' ∈ (uvs i).fst
[PROOFSTEP]
simpa using hx'
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : CompactSpace α
f : Filter α
inst✝ : NeBot f
⊢ ∃ x, ClusterPt x f
[PROOFSTEP]
simpa using isCompact_univ (show f ≤ 𝓟 univ by simp)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : CompactSpace α
f : Filter α
inst✝ : NeBot f
⊢ f ≤ 𝓟 univ
[PROOFSTEP]
simp
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
U : α → Set α
hU : ∀ (x : α), U x ∈ 𝓝 x
⊢ ∃ t, ⋃ (x : α) (_ : x ∈ t), U x = ⊤
[PROOFSTEP]
obtain ⟨t, -, s⟩ := IsCompact.elim_nhds_subcover isCompact_univ U fun x _ => hU x
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : CompactSpace α
U : α → Set α
hU : ∀ (x : α), U x ∈ 𝓝 x
t : Finset α
s : univ ⊆ ⋃ (x : α) (_ : x ∈ t), U x
⊢ ∃ t, ⋃ (x : α) (_ : x ∈ t), U x = ⊤
[PROOFSTEP]
exact ⟨t, top_unique s⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
h :
∀ {ι : Type u} (Z : ι → Set α), (∀ (i : ι), IsClosed (Z i)) → ⋂ (i : ι), Z i = ∅ → ∃ t, ⋂ (i : ι) (_ : i ∈ t), Z i = ∅
ι✝ : Type u
Z : ι✝ → Set α
⊢ (∀ (i : ι✝), IsClosed (Z i)) → univ ∩ ⋂ (i : ι✝), Z i = ∅ → ∃ t, univ ∩ ⋂ (i : ι✝) (_ : i ∈ t), Z i = ∅
[PROOFSTEP]
simpa using h Z
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : NoncompactSpace α
⊢ NeBot (cocompact α)
[PROOFSTEP]
refine' Filter.hasBasis_cocompact.neBot_iff.2 fun hs => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : NoncompactSpace α
i✝ : Set α
hs : IsCompact i✝
⊢ Set.Nonempty i✝ᶜ
[PROOFSTEP]
contrapose hs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : NoncompactSpace α
i✝ : Set α
hs : ¬Set.Nonempty i✝ᶜ
⊢ ¬IsCompact i✝
[PROOFSTEP]
rw [not_nonempty_iff_eq_empty, compl_empty_iff] at hs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : NoncompactSpace α
i✝ : Set α
hs : i✝ = univ
⊢ ¬IsCompact i✝
[PROOFSTEP]
rw [hs]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : NoncompactSpace α
i✝ : Set α
hs : i✝ = univ
⊢ ¬IsCompact univ
[PROOFSTEP]
exact noncompact_univ α
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ NeBot (cocompact ℤ)
[PROOFSTEP]
simp only [Filter.cocompact_eq_cofinite, Filter.cofinite_neBot]
-- Note: We can't make this into an instance because it loops with `Finite.compactSpace`.
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α✝
inst✝³ : TopologicalSpace β
s t : Set α✝
α : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : CompactSpace α
inst✝ : Infinite α
⊢ ∃ z, NeBot (𝓝[{z}ᶜ] z)
[PROOFSTEP]
by_contra' H
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α✝
inst✝³ : TopologicalSpace β
s t : Set α✝
α : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : CompactSpace α
inst✝ : Infinite α
H : ∀ (z : α), ¬NeBot (𝓝[{z}ᶜ] z)
⊢ False
[PROOFSTEP]
simp_rw [not_neBot] at H
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α✝
inst✝³ : TopologicalSpace β
s t : Set α✝
α : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : CompactSpace α
inst✝ : Infinite α
H : ∀ (z : α), 𝓝[{z}ᶜ] z = ⊥
⊢ False
[PROOFSTEP]
haveI := discreteTopology_iff_nhds_ne.2 H
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α✝
inst✝³ : TopologicalSpace β
s t : Set α✝
α : Type u_3
inst✝² : TopologicalSpace α
inst✝¹ : CompactSpace α
inst✝ : Infinite α
H : ∀ (z : α), 𝓝[{z}ᶜ] z = ⊥
this : DiscreteTopology α
⊢ False
[PROOFSTEP]
exact Infinite.not_finite (finite_of_compact_of_discrete : Finite α)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : CompactSpace α
f : ι → Set α
hf : LocallyFinite f
⊢ Set.Finite {i | Set.Nonempty (f i)}
[PROOFSTEP]
simpa only [inter_univ] using hf.finite_nonempty_inter_compact isCompact_univ
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
ι : Type u_3
inst✝ : CompactSpace α
f : ι → Set α
hf : LocallyFinite f
hne : ∀ (i : ι), Set.Nonempty (f i)
⊢ Set.Finite univ
[PROOFSTEP]
simpa only [hne] using hf.finite_nonempty_of_compact
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hf : Continuous f
⊢ comap f (cocompact β) ≤ cocompact α
[PROOFSTEP]
rw [(Filter.hasBasis_cocompact.comap f).le_basis_iff Filter.hasBasis_cocompact]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hf : Continuous f
⊢ ∀ (i' : Set α), IsCompact i' → ∃ i, IsCompact i ∧ f ⁻¹' iᶜ ⊆ i'ᶜ
[PROOFSTEP]
intro t ht
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
f : α → β
hf : Continuous f
t : Set α
ht : IsCompact t
⊢ ∃ i, IsCompact i ∧ f ⁻¹' iᶜ ⊆ tᶜ
[PROOFSTEP]
refine' ⟨f '' t, ht.image hf, _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
f : α → β
hf : Continuous f
t : Set α
ht : IsCompact t
⊢ f ⁻¹' (f '' t)ᶜ ⊆ tᶜ
[PROOFSTEP]
simpa using t.subset_preimage_image f
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
f : α → β
hf : Continuous f
⊢ IsCompact (range f)
[PROOFSTEP]
rw [← image_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
f : α → β
hf : Continuous f
⊢ IsCompact (f '' univ)
[PROOFSTEP]
exact isCompact_univ.image hf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs : IsClosed s
⊢ IsClosed (Prod.snd '' s)
[PROOFSTEP]
rw [← isOpen_compl_iff, isOpen_iff_mem_nhds]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs : IsClosed s
⊢ ∀ (a : Y), a ∈ (Prod.snd '' s)ᶜ → (Prod.snd '' s)ᶜ ∈ 𝓝 a
[PROOFSTEP]
intro y hy
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs : IsClosed s
y : Y
hy : y ∈ (Prod.snd '' s)ᶜ
⊢ (Prod.snd '' s)ᶜ ∈ 𝓝 y
[PROOFSTEP]
have : univ ×ˢ { y } ⊆ sᶜ
[GOAL]
case this
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs : IsClosed s
y : Y
hy : y ∈ (Prod.snd '' s)ᶜ
⊢ univ ×ˢ {y} ⊆ sᶜ
[PROOFSTEP]
exact fun (x, y') ⟨_, rfl⟩ hs => hy ⟨(x, y'), hs, rfl⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs : IsClosed s
y : Y
hy : y ∈ (Prod.snd '' s)ᶜ
this : univ ×ˢ {y} ⊆ sᶜ
⊢ (Prod.snd '' s)ᶜ ∈ 𝓝 y
[PROOFSTEP]
rcases generalized_tube_lemma isCompact_univ isCompact_singleton hs.isOpen_compl this with ⟨U, V, -, hVo, hU, hV, hs⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs✝ : IsClosed s
y : Y
hy : y ∈ (Prod.snd '' s)ᶜ
this : univ ×ˢ {y} ⊆ sᶜ
U : Set X
V : Set Y
hVo : IsOpen V
hU : univ ⊆ U
hV : {y} ⊆ V
hs : U ×ˢ V ⊆ sᶜ
⊢ (Prod.snd '' s)ᶜ ∈ 𝓝 y
[PROOFSTEP]
refine mem_nhds_iff.2 ⟨V, ?_, hVo, hV rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs✝ : IsClosed s
y : Y
hy : y ∈ (Prod.snd '' s)ᶜ
this : univ ×ˢ {y} ⊆ sᶜ
U : Set X
V : Set Y
hVo : IsOpen V
hU : univ ⊆ U
hV : {y} ⊆ V
hs : U ×ˢ V ⊆ sᶜ
⊢ V ⊆ (Prod.snd '' s)ᶜ
[PROOFSTEP]
rintro _ hzV ⟨z, hzs, rfl⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : CompactSpace X
Y : Type u_4
inst✝ : TopologicalSpace Y
s : Set (X × Y)
hs✝ : IsClosed s
y : Y
hy : y ∈ (Prod.snd '' s)ᶜ
this : univ ×ˢ {y} ⊆ sᶜ
U : Set X
V : Set Y
hVo : IsOpen V
hU : univ ⊆ U
hV : {y} ⊆ V
hs : U ×ˢ V ⊆ sᶜ
z : X × Y
hzs : z ∈ s
hzV : z.snd ∈ V
⊢ False
[PROOFSTEP]
exact hs ⟨hU trivial, hzV⟩ hzs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
f : α → β
hf : Inducing f
s : Set α
⊢ IsCompact (f '' s) ↔ IsCompact s
[PROOFSTEP]
refine ⟨fun hs F F_ne_bot F_le => ?_, fun hs => hs.image hf.continuous⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
f : α → β
hf : Inducing f
s : Set α
hs : IsCompact (f '' s)
F : Filter α
F_ne_bot : NeBot F
F_le : F ≤ 𝓟 s
⊢ ∃ a, a ∈ s ∧ ClusterPt a F
[PROOFSTEP]
obtain ⟨_, ⟨x, x_in : x ∈ s, rfl⟩, hx : ClusterPt (f x) (map f F)⟩ := hs ((map_mono F_le).trans_eq map_principal)
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t : Set α
f : α → β
hf : Inducing f
s : Set α
hs : IsCompact (f '' s)
F : Filter α
F_ne_bot : NeBot F
F_le : F ≤ 𝓟 s
x : α
x_in : x ∈ s
hx : ClusterPt (f x) (map f F)
⊢ ∃ a, a ∈ s ∧ ClusterPt a F
[PROOFSTEP]
exact ⟨x, x_in, hf.mapClusterPt_iff.1 hx⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hf : ClosedEmbedding f
K : Set β
hK : IsCompact K
⊢ IsCompact (f ⁻¹' K)
[PROOFSTEP]
replace hK := hK.inter_right hf.closed_range
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
f : α → β
hf : ClosedEmbedding f
K : Set β
hK : IsCompact (K ∩ range f)
⊢ IsCompact (f ⁻¹' K)
[PROOFSTEP]
rwa [← hf.toInducing.isCompact_iff, image_preimage_eq_inter_range]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ IsCompact s ↔ IsCompact univ
[PROOFSTEP]
rw [isCompact_iff_isCompact_in_subtype, image_univ, Subtype.range_coe]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
hs' : Set.Infinite s
⊢ ∃ z, z ∈ s ∧ NeBot (𝓝[{z}ᶜ] z ⊓ 𝓟 s)
[PROOFSTEP]
by_contra' H
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
hs' : Set.Infinite s
H : ∀ (z : α), z ∈ s → ¬NeBot (𝓝[{z}ᶜ] z ⊓ 𝓟 s)
⊢ False
[PROOFSTEP]
simp_rw [not_neBot] at H
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
hs : IsCompact s
hs' : Set.Infinite s
H : ∀ (z : α), z ∈ s → 𝓝[{z}ᶜ] z ⊓ 𝓟 s = ⊥
⊢ False
[PROOFSTEP]
exact hs' (hs.finite <| discreteTopology_subtype_iff.mpr H)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
h : CompactSpace β
f : α → β
hf : ClosedEmbedding f
⊢ IsCompact univ
[PROOFSTEP]
rw [← hf.toInducing.isCompact_iff, image_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
h : CompactSpace β
f : α → β
hf : ClosedEmbedding f
⊢ IsCompact (range f)
[PROOFSTEP]
exact hf.closed_range.isCompact
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : IsCompact s
ht : IsCompact t
⊢ IsCompact (s ×ˢ t)
[PROOFSTEP]
rw [isCompact_iff_ultrafilter_le_nhds] at hs ht ⊢
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
⊢ ∀ (f : Ultrafilter (α × β)), ↑f ≤ 𝓟 (s ×ˢ t) → ∃ a, a ∈ s ×ˢ t ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
intro f hfs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : ↑f ≤ 𝓟 (s ×ˢ t)
⊢ ∃ a, a ∈ s ×ˢ t ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
rw [le_principal_iff] at hfs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : s ×ˢ t ∈ ↑f
⊢ ∃ a, a ∈ s ×ˢ t ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
obtain ⟨a : α, sa : a ∈ s, ha : map Prod.fst f.1 ≤ 𝓝 a⟩ :=
hs (f.map Prod.fst) (le_principal_iff.2 <| mem_map.2 <| mem_of_superset hfs fun x => And.left)
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : s ×ˢ t ∈ ↑f
a : α
sa : a ∈ s
ha : map Prod.fst ↑f ≤ 𝓝 a
⊢ ∃ a, a ∈ s ×ˢ t ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
obtain ⟨b : β, tb : b ∈ t, hb : map Prod.snd f.1 ≤ 𝓝 b⟩ :=
ht (f.map Prod.snd) (le_principal_iff.2 <| mem_map.2 <| mem_of_superset hfs fun x => And.right)
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : s ×ˢ t ∈ ↑f
a : α
sa : a ∈ s
ha : map Prod.fst ↑f ≤ 𝓝 a
b : β
tb : b ∈ t
hb : map Prod.snd ↑f ≤ 𝓝 b
⊢ ∃ a, a ∈ s ×ˢ t ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
rw [map_le_iff_le_comap] at ha hb
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : s ×ˢ t ∈ ↑f
a : α
sa : a ∈ s
ha : ↑f ≤ comap Prod.fst (𝓝 a)
b : β
tb : b ∈ t
hb : ↑f ≤ comap Prod.snd (𝓝 b)
⊢ ∃ a, a ∈ s ×ˢ t ∧ ↑f ≤ 𝓝 a
[PROOFSTEP]
refine' ⟨⟨a, b⟩, ⟨sa, tb⟩, _⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : s ×ˢ t ∈ ↑f
a : α
sa : a ∈ s
ha : ↑f ≤ comap Prod.fst (𝓝 a)
b : β
tb : b ∈ t
hb : ↑f ≤ comap Prod.snd (𝓝 b)
⊢ ↑f ≤ 𝓝 (a, b)
[PROOFSTEP]
rw [nhds_prod_eq]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t✝ s : Set α
t : Set β
hs : ∀ (f : Ultrafilter α), ↑f ≤ 𝓟 s → ∃ a, a ∈ s ∧ ↑f ≤ 𝓝 a
ht : ∀ (f : Ultrafilter β), ↑f ≤ 𝓟 t → ∃ a, a ∈ t ∧ ↑f ≤ 𝓝 a
f : Ultrafilter (α × β)
hfs : s ×ˢ t ∈ ↑f
a : α
sa : a ∈ s
ha : ↑f ≤ comap Prod.fst (𝓝 a)
b : β
tb : b ∈ t
hb : ↑f ≤ comap Prod.snd (𝓝 b)
⊢ ↑f ≤ 𝓝 a ×ˢ 𝓝 b
[PROOFSTEP]
exact le_inf ha hb
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : CompactSpace α
inst✝ : CompactSpace β
⊢ IsCompact univ
[PROOFSTEP]
rw [← univ_prod_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : CompactSpace α
inst✝ : CompactSpace β
⊢ IsCompact (univ ×ˢ univ)
[PROOFSTEP]
exact isCompact_univ.prod isCompact_univ
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : CompactSpace α
inst✝ : CompactSpace β
⊢ IsCompact univ
[PROOFSTEP]
rw [← range_inl_union_range_inr]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : CompactSpace α
inst✝ : CompactSpace β
⊢ IsCompact (range Sum.inl ∪ range Sum.inr)
[PROOFSTEP]
exact (isCompact_range continuous_inl).union (isCompact_range continuous_inr)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
⊢ CompactSpace ((i : ι) × π i)
[PROOFSTEP]
refine' ⟨_⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
⊢ IsCompact univ
[PROOFSTEP]
rw [Sigma.univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
⊢ IsCompact (⋃ (a : ι), range (Sigma.mk a))
[PROOFSTEP]
exact isCompact_iUnion fun i => isCompact_range continuous_sigmaMk
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ Filter.coprod (cocompact α) (cocompact β) = cocompact (α × β)
[PROOFSTEP]
ext S
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
S : Set (α × β)
⊢ S ∈ Filter.coprod (cocompact α) (cocompact β) ↔ S ∈ cocompact (α × β)
[PROOFSTEP]
simp only [mem_coprod_iff, exists_prop, mem_comap, Filter.mem_cocompact]
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
S : Set (α × β)
⊢ ((∃ t₁, (∃ t, IsCompact t ∧ tᶜ ⊆ t₁) ∧ Prod.fst ⁻¹' t₁ ⊆ S) ∧
∃ t₂, (∃ t, IsCompact t ∧ tᶜ ⊆ t₂) ∧ Prod.snd ⁻¹' t₂ ⊆ S) ↔
∃ t, IsCompact t ∧ tᶜ ⊆ S
[PROOFSTEP]
constructor
[GOAL]
case a.mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
S : Set (α × β)
⊢ ((∃ t₁, (∃ t, IsCompact t ∧ tᶜ ⊆ t₁) ∧ Prod.fst ⁻¹' t₁ ⊆ S) ∧
∃ t₂, (∃ t, IsCompact t ∧ tᶜ ⊆ t₂) ∧ Prod.snd ⁻¹' t₂ ⊆ S) →
∃ t, IsCompact t ∧ tᶜ ⊆ S
[PROOFSTEP]
rintro ⟨⟨A, ⟨t, ht, hAt⟩, hAS⟩, B, ⟨t', ht', hBt'⟩, hBS⟩
[GOAL]
case a.mp.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S : Set (α × β)
A : Set α
hAS : Prod.fst ⁻¹' A ⊆ S
t : Set α
ht : IsCompact t
hAt : tᶜ ⊆ A
B : Set β
hBS : Prod.snd ⁻¹' B ⊆ S
t' : Set β
ht' : IsCompact t'
hBt' : t'ᶜ ⊆ B
⊢ ∃ t, IsCompact t ∧ tᶜ ⊆ S
[PROOFSTEP]
refine' ⟨t ×ˢ t', ht.prod ht', _⟩
[GOAL]
case a.mp.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S : Set (α × β)
A : Set α
hAS : Prod.fst ⁻¹' A ⊆ S
t : Set α
ht : IsCompact t
hAt : tᶜ ⊆ A
B : Set β
hBS : Prod.snd ⁻¹' B ⊆ S
t' : Set β
ht' : IsCompact t'
hBt' : t'ᶜ ⊆ B
⊢ (t ×ˢ t')ᶜ ⊆ S
[PROOFSTEP]
refine' Subset.trans _ (union_subset hAS hBS)
[GOAL]
case a.mp.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S : Set (α × β)
A : Set α
hAS : Prod.fst ⁻¹' A ⊆ S
t : Set α
ht : IsCompact t
hAt : tᶜ ⊆ A
B : Set β
hBS : Prod.snd ⁻¹' B ⊆ S
t' : Set β
ht' : IsCompact t'
hBt' : t'ᶜ ⊆ B
⊢ (t ×ˢ t')ᶜ ⊆ Prod.fst ⁻¹' A ∪ Prod.snd ⁻¹' B
[PROOFSTEP]
rw [compl_subset_comm] at hAt hBt' ⊢
[GOAL]
case a.mp.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S : Set (α × β)
A : Set α
hAS : Prod.fst ⁻¹' A ⊆ S
t : Set α
ht : IsCompact t
hAt : Aᶜ ⊆ t
B : Set β
hBS : Prod.snd ⁻¹' B ⊆ S
t' : Set β
ht' : IsCompact t'
hBt' : Bᶜ ⊆ t'
⊢ (Prod.fst ⁻¹' A ∪ Prod.snd ⁻¹' B)ᶜ ⊆ t ×ˢ t'
[PROOFSTEP]
refine' Subset.trans (fun x => _) (Set.prod_mono hAt hBt')
[GOAL]
case a.mp.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S : Set (α × β)
A : Set α
hAS : Prod.fst ⁻¹' A ⊆ S
t : Set α
ht : IsCompact t
hAt : Aᶜ ⊆ t
B : Set β
hBS : Prod.snd ⁻¹' B ⊆ S
t' : Set β
ht' : IsCompact t'
hBt' : Bᶜ ⊆ t'
x : α × β
⊢ x ∈ (Prod.fst ⁻¹' A ∪ Prod.snd ⁻¹' B)ᶜ → x ∈ Aᶜ ×ˢ Bᶜ
[PROOFSTEP]
simp only [compl_union, mem_inter_iff, mem_prod, mem_preimage, mem_compl_iff]
[GOAL]
case a.mp.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S : Set (α × β)
A : Set α
hAS : Prod.fst ⁻¹' A ⊆ S
t : Set α
ht : IsCompact t
hAt : Aᶜ ⊆ t
B : Set β
hBS : Prod.snd ⁻¹' B ⊆ S
t' : Set β
ht' : IsCompact t'
hBt' : Bᶜ ⊆ t'
x : α × β
⊢ ¬x.fst ∈ A ∧ ¬x.snd ∈ B → ¬x.fst ∈ A ∧ ¬x.snd ∈ B
[PROOFSTEP]
tauto
[GOAL]
case a.mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
S : Set (α × β)
⊢ (∃ t, IsCompact t ∧ tᶜ ⊆ S) →
(∃ t₁, (∃ t, IsCompact t ∧ tᶜ ⊆ t₁) ∧ Prod.fst ⁻¹' t₁ ⊆ S) ∧
∃ t₂, (∃ t, IsCompact t ∧ tᶜ ⊆ t₂) ∧ Prod.snd ⁻¹' t₂ ⊆ S
[PROOFSTEP]
rintro ⟨t, ht, htS⟩
[GOAL]
case a.mpr.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ (∃ t₁, (∃ t, IsCompact t ∧ tᶜ ⊆ t₁) ∧ Prod.fst ⁻¹' t₁ ⊆ S) ∧ ∃ t₂, (∃ t, IsCompact t ∧ tᶜ ⊆ t₂) ∧ Prod.snd ⁻¹' t₂ ⊆ S
[PROOFSTEP]
refine' ⟨⟨(Prod.fst '' t)ᶜ, _, _⟩, ⟨(Prod.snd '' t)ᶜ, _, _⟩⟩
[GOAL]
case a.mpr.intro.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ ∃ t_1, IsCompact t_1 ∧ t_1ᶜ ⊆ (Prod.fst '' t)ᶜ
[PROOFSTEP]
exact ⟨Prod.fst '' t, ht.image continuous_fst, Subset.rfl⟩
[GOAL]
case a.mpr.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ Prod.fst ⁻¹' (Prod.fst '' t)ᶜ ⊆ S
[PROOFSTEP]
rw [preimage_compl]
[GOAL]
case a.mpr.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ (Prod.fst ⁻¹' (Prod.fst '' t))ᶜ ⊆ S
[PROOFSTEP]
rw [compl_subset_comm] at htS ⊢
[GOAL]
case a.mpr.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : Sᶜ ⊆ t
⊢ Sᶜ ⊆ Prod.fst ⁻¹' (Prod.fst '' t)
[PROOFSTEP]
exact htS.trans (subset_preimage_image Prod.fst _)
[GOAL]
case a.mpr.intro.intro.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ ∃ t_1, IsCompact t_1 ∧ t_1ᶜ ⊆ (Prod.snd '' t)ᶜ
[PROOFSTEP]
exact ⟨Prod.snd '' t, ht.image continuous_snd, Subset.rfl⟩
[GOAL]
case a.mpr.intro.intro.refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ Prod.snd ⁻¹' (Prod.snd '' t)ᶜ ⊆ S
[PROOFSTEP]
rw [preimage_compl]
[GOAL]
case a.mpr.intro.intro.refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : tᶜ ⊆ S
⊢ (Prod.snd ⁻¹' (Prod.snd '' t))ᶜ ⊆ S
[PROOFSTEP]
rw [compl_subset_comm] at htS ⊢
[GOAL]
case a.mpr.intro.intro.refine'_4
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
S t : Set (α × β)
ht : IsCompact t
htS : Sᶜ ⊆ t
⊢ Sᶜ ⊆ Prod.snd ⁻¹' (Prod.snd '' t)
[PROOFSTEP]
exact htS.trans (subset_preimage_image Prod.snd _)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
⊢ NoncompactSpace (α × β) ↔ NoncompactSpace α ∧ Nonempty β ∨ Nonempty α ∧ NoncompactSpace β
[PROOFSTEP]
simp [← Filter.cocompact_neBot_iff, ← Filter.coprod_cocompact, Filter.coprod_neBot_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
⊢ (∀ (i : ι), IsCompact (s i)) → IsCompact {x | ∀ (i : ι), x i ∈ s i}
[PROOFSTEP]
simp only [isCompact_iff_ultrafilter_le_nhds, nhds_pi, Filter.pi, exists_prop, mem_setOf_eq, le_iInf_iff,
le_principal_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
⊢ (∀ (i : ι) (f : Ultrafilter (π i)), s i ∈ ↑f → ∃ a, a ∈ s i ∧ ↑f ≤ 𝓝 a) →
∀ (f : Ultrafilter ((i : ι) → π i)),
{x | ∀ (i : ι), x i ∈ s i} ∈ ↑f → ∃ a, (∀ (i : ι), a i ∈ s i) ∧ ∀ (i : ι), ↑f ≤ comap (Function.eval i) (𝓝 (a i))
[PROOFSTEP]
intro h f hfs
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι) (f : Ultrafilter (π i)), s i ∈ ↑f → ∃ a, a ∈ s i ∧ ↑f ≤ 𝓝 a
f : Ultrafilter ((i : ι) → π i)
hfs : {x | ∀ (i : ι), x i ∈ s i} ∈ ↑f
⊢ ∃ a, (∀ (i : ι), a i ∈ s i) ∧ ∀ (i : ι), ↑f ≤ comap (Function.eval i) (𝓝 (a i))
[PROOFSTEP]
have : ∀ i : ι, ∃ a, a ∈ s i ∧ Tendsto (Function.eval i) f (𝓝 a) :=
by
refine fun i => h i (f.map _) (mem_map.2 ?_)
exact mem_of_superset hfs fun x hx => hx i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι) (f : Ultrafilter (π i)), s i ∈ ↑f → ∃ a, a ∈ s i ∧ ↑f ≤ 𝓝 a
f : Ultrafilter ((i : ι) → π i)
hfs : {x | ∀ (i : ι), x i ∈ s i} ∈ ↑f
⊢ ∀ (i : ι), ∃ a, a ∈ s i ∧ Tendsto (Function.eval i) (↑f) (𝓝 a)
[PROOFSTEP]
refine fun i => h i (f.map _) (mem_map.2 ?_)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι) (f : Ultrafilter (π i)), s i ∈ ↑f → ∃ a, a ∈ s i ∧ ↑f ≤ 𝓝 a
f : Ultrafilter ((i : ι) → π i)
hfs : {x | ∀ (i : ι), x i ∈ s i} ∈ ↑f
i : ι
⊢ Function.eval i ⁻¹' s i ∈ ↑f
[PROOFSTEP]
exact mem_of_superset hfs fun x hx => hx i
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι) (f : Ultrafilter (π i)), s i ∈ ↑f → ∃ a, a ∈ s i ∧ ↑f ≤ 𝓝 a
f : Ultrafilter ((i : ι) → π i)
hfs : {x | ∀ (i : ι), x i ∈ s i} ∈ ↑f
this : ∀ (i : ι), ∃ a, a ∈ s i ∧ Tendsto (Function.eval i) (↑f) (𝓝 a)
⊢ ∃ a, (∀ (i : ι), a i ∈ s i) ∧ ∀ (i : ι), ↑f ≤ comap (Function.eval i) (𝓝 (a i))
[PROOFSTEP]
choose a ha using this
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι) (f : Ultrafilter (π i)), s i ∈ ↑f → ∃ a, a ∈ s i ∧ ↑f ≤ 𝓝 a
f : Ultrafilter ((i : ι) → π i)
hfs : {x | ∀ (i : ι), x i ∈ s i} ∈ ↑f
a : (i : ι) → π i
ha : ∀ (i : ι), a i ∈ s i ∧ Tendsto (Function.eval i) (↑f) (𝓝 (a i))
⊢ ∃ a, (∀ (i : ι), a i ∈ s i) ∧ ∀ (i : ι), ↑f ≤ comap (Function.eval i) (𝓝 (a i))
[PROOFSTEP]
exact ⟨a, fun i => (ha i).left, fun i => (ha i).right.le_comap⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι), IsCompact (s i)
⊢ IsCompact (Set.pi univ s)
[PROOFSTEP]
convert isCompact_pi_infinite h
[GOAL]
case h.e'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : (i : ι) → TopologicalSpace (π i)
s : (i : ι) → Set (π i)
h : ∀ (i : ι), IsCompact (s i)
⊢ Set.pi univ s = {x | ∀ (i : ι), x i ∈ s i}
[PROOFSTEP]
simp only [← mem_univ_pi, setOf_mem_eq]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
⊢ IsCompact univ
[PROOFSTEP]
rw [← pi_univ univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
⊢ IsCompact (Set.pi univ fun i => univ)
[PROOFSTEP]
exact isCompact_univ_pi fun i => isCompact_univ
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
δ : Type u_3
κ : δ → Type u_4
inst✝ : (d : δ) → TopologicalSpace (κ d)
⊢ (Filter.coprodᵢ fun d => cocompact (κ d)) = cocompact ((d : δ) → κ d)
[PROOFSTEP]
refine' le_antisymm (iSup_le fun i => Filter.comap_cocompact_le (continuous_apply i)) _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
δ : Type u_3
κ : δ → Type u_4
inst✝ : (d : δ) → TopologicalSpace (κ d)
⊢ cocompact ((d : δ) → κ d) ≤ Filter.coprodᵢ fun d => cocompact (κ d)
[PROOFSTEP]
refine' compl_surjective.forall.2 fun s H => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s✝ t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
δ : Type u_3
κ : δ → Type u_4
inst✝ : (d : δ) → TopologicalSpace (κ d)
s : Set ((i : δ) → κ i)
H : sᶜ ∈ Filter.coprodᵢ fun d => cocompact (κ d)
⊢ sᶜ ∈ cocompact ((d : δ) → κ d)
[PROOFSTEP]
simp only [compl_mem_coprodᵢ, Filter.mem_cocompact, compl_subset_compl, image_subset_iff] at H ⊢
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s✝ t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
δ : Type u_3
κ : δ → Type u_4
inst✝ : (d : δ) → TopologicalSpace (κ d)
s : Set ((i : δ) → κ i)
H : ∀ (i : δ), ∃ t, IsCompact t ∧ s ⊆ Function.eval i ⁻¹' t
⊢ ∃ t, IsCompact t ∧ s ⊆ t
[PROOFSTEP]
choose K hKc htK using H
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s✝ t : Set α
inst✝¹ : (i : ι) → TopologicalSpace (π i)
δ : Type u_3
κ : δ → Type u_4
inst✝ : (d : δ) → TopologicalSpace (κ d)
s : Set ((i : δ) → κ i)
K : (i : δ) → Set (κ i)
hKc : ∀ (i : δ), IsCompact (K i)
htK : ∀ (i : δ), s ⊆ Function.eval i ⁻¹' K i
⊢ ∃ t, IsCompact t ∧ s ⊆ t
[PROOFSTEP]
exact ⟨Set.pi univ K, isCompact_univ_pi hKc, fun f hf i _ => htK i hf⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
r : α → α → Prop
inst✝ : CompactSpace α
⊢ IsCompact univ
[PROOFSTEP]
rw [← range_quot_mk]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
r : α → α → Prop
inst✝ : CompactSpace α
⊢ IsCompact (range (mk r))
[PROOFSTEP]
exact isCompact_range continuous_quot_mk
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace α
x : α
⊢ ∀ (t : Set α), t ∈ 𝓝 x → ∃ r, r ∈ 𝓝 x ∧ IsCompact r ∧ r ⊆ t
[PROOFSTEP]
simpa only [and_comm] using LocallyCompactSpace.local_compact_nhds x
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : Finite ι
t : (i : ι) → π i
n : Set ((i : ι) → π i)
hn : n ∈ 𝓝 t
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
rw [nhds_pi, Filter.mem_pi] at hn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : Finite ι
t : (i : ι) → π i
n : Set ((i : ι) → π i)
hn : ∃ I, Set.Finite I ∧ ∃ t_1, (∀ (i : ι), t_1 i ∈ 𝓝 (t i)) ∧ Set.pi I t_1 ⊆ n
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
obtain ⟨s, -, n', hn', hsub⟩ := hn
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : Finite ι
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
choose n'' hn'' hsub' hc using fun i => LocallyCompactSpace.local_compact_nhds (t i) (n' i) (hn' i)
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : Finite ι
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
refine' ⟨(Set.univ : Set ι).pi n'', _, subset_trans (fun _ h => _) hsub, isCompact_univ_pi hc⟩
[GOAL]
case intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : Finite ι
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
⊢ Set.pi univ n'' ∈ 𝓝 t
[PROOFSTEP]
exact (set_pi_mem_nhds_iff (@Set.finite_univ ι _) _).mpr fun i _ => hn'' i
[GOAL]
case intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : Finite ι
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
x✝ : (i : ι) → π i
h : x✝ ∈ Set.pi univ n''
⊢ x✝ ∈ Set.pi s n'
[PROOFSTEP]
exact fun i _ => hsub' i (h i trivial)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
hn : n ∈ 𝓝 t
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
rw [nhds_pi, Filter.mem_pi] at hn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
hn : ∃ I, Set.Finite I ∧ ∃ t_1, (∀ (i : ι), t_1 i ∈ 𝓝 (t i)) ∧ Set.pi I t_1 ⊆ n
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
obtain ⟨s, hs, n', hn', hsub⟩ := hn
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
choose n'' hn'' hsub' hc using fun i => LocallyCompactSpace.local_compact_nhds (t i) (n' i) (hn' i)
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
⊢ ∃ s, s ∈ 𝓝 t ∧ s ⊆ n ∧ IsCompact s
[PROOFSTEP]
refine' ⟨s.pi n'', _, subset_trans (fun _ => _) hsub, _⟩
[GOAL]
case intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
⊢ Set.pi s n'' ∈ 𝓝 t
[PROOFSTEP]
exact (set_pi_mem_nhds_iff hs _).mpr fun i _ => hn'' i
[GOAL]
case intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
x✝ : (i : ι) → π i
⊢ x✝ ∈ Set.pi s n'' → x✝ ∈ Set.pi s n'
[PROOFSTEP]
exact forall₂_imp fun i _ hi' => hsub' i hi'
[GOAL]
case intro.intro.intro.intro.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
⊢ IsCompact (Set.pi s n'')
[PROOFSTEP]
rw [← Set.univ_pi_ite]
[GOAL]
case intro.intro.intro.intro.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
⊢ IsCompact (Set.pi univ fun i => if i ∈ s then n'' i else univ)
[PROOFSTEP]
refine' isCompact_univ_pi fun i => _
[GOAL]
case intro.intro.intro.intro.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
i : ι
⊢ IsCompact (if i ∈ s then n'' i else univ)
[PROOFSTEP]
by_cases h : i ∈ s
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
i : ι
h : i ∈ s
⊢ IsCompact (if i ∈ s then n'' i else univ)
[PROOFSTEP]
rw [if_pos h]
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
i : ι
h : i ∈ s
⊢ IsCompact (n'' i)
[PROOFSTEP]
exact hc i
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
i : ι
h : ¬i ∈ s
⊢ IsCompact (if i ∈ s then n'' i else univ)
[PROOFSTEP]
rw [if_neg h]
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s✝ t✝ : Set α
inst✝² : (i : ι) → TopologicalSpace (π i)
inst✝¹ : ∀ (i : ι), LocallyCompactSpace (π i)
inst✝ : ∀ (i : ι), CompactSpace (π i)
t : (i : ι) → π i
n : Set ((i : ι) → π i)
s : Set ι
hs : Set.Finite s
n' : (i : ι) → Set (π i)
hn' : ∀ (i : ι), n' i ∈ 𝓝 (t i)
hsub : Set.pi s n' ⊆ n
n'' : (i : ι) → Set (π i)
hn'' : ∀ (i : ι), n'' i ∈ 𝓝 (t i)
hsub' : ∀ (i : ι), n'' i ⊆ n' i
hc : ∀ (i : ι), IsCompact (n'' i)
i : ι
h : ¬i ∈ s
⊢ IsCompact univ
[PROOFSTEP]
exact CompactSpace.isCompact_univ
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace α
x : α
U : Set α
hU : IsOpen U
hx : x ∈ U
⊢ ∃ K, IsCompact K ∧ x ∈ interior K ∧ K ⊆ U
[PROOFSTEP]
rcases LocallyCompactSpace.local_compact_nhds x U (hU.mem_nhds hx) with ⟨K, h1K, h2K, h3K⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace α
x : α
U : Set α
hU : IsOpen U
hx : x ∈ U
K : Set α
h1K : K ∈ 𝓝 x
h2K : K ⊆ U
h3K : IsCompact K
⊢ ∃ K, IsCompact K ∧ x ∈ interior K ∧ K ⊆ U
[PROOFSTEP]
exact ⟨K, h3K, mem_interior_iff_mem_nhds.2 h1K, h2K⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hα : LocallyCompactSpace α
K U : Set α
hK : IsCompact K
hU : IsOpen U
h_KU : K ⊆ U
⊢ ∃ L, IsCompact L ∧ K ⊆ interior L ∧ L ⊆ U
[PROOFSTEP]
choose V hVc hxV hKV using fun x : K => exists_compact_subset hU (h_KU x.2)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hα : LocallyCompactSpace α
K U : Set α
hK : IsCompact K
hU : IsOpen U
h_KU : K ⊆ U
V : ↑K → Set α
hVc : ∀ (x : ↑K), IsCompact (V x)
hxV : ∀ (x : ↑K), ↑x ∈ interior (V x)
hKV : ∀ (x : ↑K), V x ⊆ U
⊢ ∃ L, IsCompact L ∧ K ⊆ interior L ∧ L ⊆ U
[PROOFSTEP]
have : K ⊆ ⋃ x, interior (V x) := fun x hx => mem_iUnion.2 ⟨⟨x, hx⟩, hxV _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
hα : LocallyCompactSpace α
K U : Set α
hK : IsCompact K
hU : IsOpen U
h_KU : K ⊆ U
V : ↑K → Set α
hVc : ∀ (x : ↑K), IsCompact (V x)
hxV : ∀ (x : ↑K), ↑x ∈ interior (V x)
hKV : ∀ (x : ↑K), V x ⊆ U
this : K ⊆ ⋃ (x : ↑K), interior (V x)
⊢ ∃ L, IsCompact L ∧ K ⊆ interior L ∧ L ⊆ U
[PROOFSTEP]
rcases hK.elim_finite_subcover _ (fun x => @isOpen_interior α _ (V x)) this with ⟨t, ht⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hα : LocallyCompactSpace α
K U : Set α
hK : IsCompact K
hU : IsOpen U
h_KU : K ⊆ U
V : ↑K → Set α
hVc : ∀ (x : ↑K), IsCompact (V x)
hxV : ∀ (x : ↑K), ↑x ∈ interior (V x)
hKV : ∀ (x : ↑K), V x ⊆ U
this : K ⊆ ⋃ (x : ↑K), interior (V x)
t : Finset ↑K
ht : K ⊆ ⋃ (i : ↑K) (_ : i ∈ t), interior (V i)
⊢ ∃ L, IsCompact L ∧ K ⊆ interior L ∧ L ⊆ U
[PROOFSTEP]
refine' ⟨_, t.isCompact_biUnion fun x _ => hVc x, fun x hx => _, Set.iUnion₂_subset fun i _ => hKV i⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hα : LocallyCompactSpace α
K U : Set α
hK : IsCompact K
hU : IsOpen U
h_KU : K ⊆ U
V : ↑K → Set α
hVc : ∀ (x : ↑K), IsCompact (V x)
hxV : ∀ (x : ↑K), ↑x ∈ interior (V x)
hKV : ∀ (x : ↑K), V x ⊆ U
this : K ⊆ ⋃ (x : ↑K), interior (V x)
t : Finset ↑K
ht : K ⊆ ⋃ (i : ↑K) (_ : i ∈ t), interior (V i)
x : α
hx : x ∈ K
⊢ x ∈ interior (⋃ (i : ↑K) (_ : i ∈ t), V i)
[PROOFSTEP]
rcases mem_iUnion₂.1 (ht hx) with ⟨y, hyt, hy⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t✝ : Set α
hα : LocallyCompactSpace α
K U : Set α
hK : IsCompact K
hU : IsOpen U
h_KU : K ⊆ U
V : ↑K → Set α
hVc : ∀ (x : ↑K), IsCompact (V x)
hxV : ∀ (x : ↑K), ↑x ∈ interior (V x)
hKV : ∀ (x : ↑K), V x ⊆ U
this : K ⊆ ⋃ (x : ↑K), interior (V x)
t : Finset ↑K
ht : K ⊆ ⋃ (i : ↑K) (_ : i ∈ t), interior (V i)
x : α
hx : x ∈ K
y : ↑K
hyt : y ∈ t
hy : x ∈ interior (V y)
⊢ x ∈ interior (⋃ (i : ↑K) (_ : i ∈ t), V i)
[PROOFSTEP]
exact interior_mono (subset_iUnion₂ y hyt) hy
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : ClosedEmbedding f
⊢ ∀ (x : α), HasBasis (𝓝 x) (fun s => s ∈ 𝓝 (f x) ∧ IsCompact s) fun s => f ⁻¹' s
[PROOFSTEP]
intro x
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : ClosedEmbedding f
x : α
⊢ HasBasis (𝓝 x) (fun s => s ∈ 𝓝 (f x) ∧ IsCompact s) fun s => f ⁻¹' s
[PROOFSTEP]
rw [hf.toInducing.nhds_eq_comap]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : ClosedEmbedding f
x : α
⊢ HasBasis (comap f (𝓝 (f x))) (fun s => s ∈ 𝓝 (f x) ∧ IsCompact s) fun s => f ⁻¹' s
[PROOFSTEP]
exact (compact_basis_nhds _).comap _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
⊢ LocallyCompactSpace α
[PROOFSTEP]
have : ∀ x : α, (𝓝 x).HasBasis (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s :=
by
intro x
rw [hf.toInducing.nhds_eq_comap]
exact ((compact_basis_nhds _).restrict_subset <| hf.open_range.mem_nhds <| mem_range_self _).comap _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
⊢ ∀ (x : α), HasBasis (𝓝 x) (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s
[PROOFSTEP]
intro x
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
x : α
⊢ HasBasis (𝓝 x) (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s
[PROOFSTEP]
rw [hf.toInducing.nhds_eq_comap]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
x : α
⊢ HasBasis (comap f (𝓝 (f x))) (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s
[PROOFSTEP]
exact ((compact_basis_nhds _).restrict_subset <| hf.open_range.mem_nhds <| mem_range_self _).comap _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
this : ∀ (x : α), HasBasis (𝓝 x) (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s
⊢ LocallyCompactSpace α
[PROOFSTEP]
refine' locallyCompactSpace_of_hasBasis this fun x s hs => _
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
this : ∀ (x : α), HasBasis (𝓝 x) (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s
x : α
s : Set β
hs : (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f
⊢ IsCompact (f ⁻¹' s)
[PROOFSTEP]
rw [← hf.toInducing.isCompact_iff, image_preimage_eq_of_subset hs.2]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : LocallyCompactSpace β
f : α → β
hf : OpenEmbedding f
this : ∀ (x : α), HasBasis (𝓝 x) (fun s => (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f) fun s => f ⁻¹' s
x : α
s : Set β
hs : (s ∈ 𝓝 (f x) ∧ IsCompact s) ∧ s ⊆ range f
⊢ IsCompact s
[PROOFSTEP]
exact hs.1.2
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
F : Ultrafilter α
⊢ ↑F ≤ 𝓝 (lim F)
[PROOFSTEP]
rcases isCompact_univ.ultrafilter_le_nhds F (by simp) with ⟨x, -, h⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
F : Ultrafilter α
⊢ ↑F ≤ 𝓟 univ
[PROOFSTEP]
simp
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
F : Ultrafilter α
x : α
h : ↑F ≤ 𝓝 x
⊢ ↑F ≤ 𝓝 (lim F)
[PROOFSTEP]
exact le_nhds_lim ⟨x, h⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
⊢ ∃ V, V ⊆ S ∧ Set.Nonempty V ∧ IsClosed V ∧ ∀ (V' : Set α), V' ⊆ V → Set.Nonempty V' → IsClosed V' → V' = V
[PROOFSTEP]
let opens := {U : Set α | Sᶜ ⊆ U ∧ IsOpen U ∧ Uᶜ.Nonempty}
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
⊢ ∃ V, V ⊆ S ∧ Set.Nonempty V ∧ IsClosed V ∧ ∀ (V' : Set α), V' ⊆ V → Set.Nonempty V' → IsClosed V' → V' = V
[PROOFSTEP]
obtain ⟨U, ⟨Uc, Uo, Ucne⟩, h⟩ :=
zorn_subset opens fun c hc hz => by
by_cases hcne : c.Nonempty
· obtain ⟨U₀, hU₀⟩ := hcne
haveI : Nonempty { U // U ∈ c } := ⟨⟨U₀, hU₀⟩⟩
obtain ⟨U₀compl, -, -⟩ := hc hU₀
use⋃₀ c
refine' ⟨⟨_, _, _⟩, fun U hU a ha => ⟨U, hU, ha⟩⟩
· exact fun a ha => ⟨U₀, hU₀, U₀compl ha⟩
· exact isOpen_sUnion fun _ h => (hc h).2.1
· convert_to (⋂ U : { U // U ∈ c }, U.1ᶜ).Nonempty
· ext
simp only [not_exists, exists_prop, not_and, Set.mem_iInter, Subtype.forall, mem_setOf_eq, mem_compl_iff,
mem_sUnion]
apply IsCompact.nonempty_iInter_of_directed_nonempty_compact_closed
· rintro ⟨U, hU⟩ ⟨U', hU'⟩
obtain ⟨V, hVc, hVU, hVU'⟩ := hz.directedOn U hU U' hU'
exact ⟨⟨V, hVc⟩, Set.compl_subset_compl.mpr hVU, Set.compl_subset_compl.mpr hVU'⟩
· exact fun U => (hc U.2).2.2
· exact fun U => (hc U.2).2.1.isClosed_compl.isCompact
· exact fun U => (hc U.2).2.1.isClosed_compl
· use Sᶜ
refine' ⟨⟨Set.Subset.refl _, isOpen_compl_iff.mpr hS, _⟩, fun U Uc => (hcne ⟨U, Uc⟩).elim⟩
rw [compl_compl]
exact hne
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
⊢ ∃ ub, ub ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ub
[PROOFSTEP]
by_cases hcne : c.Nonempty
[GOAL]
case pos
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
hcne : Set.Nonempty c
⊢ ∃ ub, ub ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ub
[PROOFSTEP]
obtain ⟨U₀, hU₀⟩ := hcne
[GOAL]
case pos.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
⊢ ∃ ub, ub ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ub
[PROOFSTEP]
haveI : Nonempty { U // U ∈ c } := ⟨⟨U₀, hU₀⟩⟩
[GOAL]
case pos.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
⊢ ∃ ub, ub ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ub
[PROOFSTEP]
obtain ⟨U₀compl, -, -⟩ := hc hU₀
[GOAL]
case pos.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ ∃ ub, ub ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ub
[PROOFSTEP]
use⋃₀ c
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ ⋃₀ c ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ⋃₀ c
[PROOFSTEP]
refine' ⟨⟨_, _, _⟩, fun U hU a ha => ⟨U, hU, ha⟩⟩
[GOAL]
case h.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ Sᶜ ⊆ ⋃₀ c
[PROOFSTEP]
exact fun a ha => ⟨U₀, hU₀, U₀compl ha⟩
[GOAL]
case h.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ IsOpen (⋃₀ c)
[PROOFSTEP]
exact isOpen_sUnion fun _ h => (hc h).2.1
[GOAL]
case h.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ Set.Nonempty (⋃₀ c)ᶜ
[PROOFSTEP]
convert_to (⋂ U : { U // U ∈ c }, U.1ᶜ).Nonempty
[GOAL]
case h.e'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ (⋃₀ c)ᶜ = ⋂ (U : { U // U ∈ c }), (↑U)ᶜ
[PROOFSTEP]
ext
[GOAL]
case h.e'_2.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
x✝ : α
⊢ x✝ ∈ (⋃₀ c)ᶜ ↔ x✝ ∈ ⋂ (U : { U // U ∈ c }), (↑U)ᶜ
[PROOFSTEP]
simp only [not_exists, exists_prop, not_and, Set.mem_iInter, Subtype.forall, mem_setOf_eq, mem_compl_iff, mem_sUnion]
[GOAL]
case h.refine'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ Set.Nonempty (⋂ (U : { U // U ∈ c }), (↑U)ᶜ)
[PROOFSTEP]
apply IsCompact.nonempty_iInter_of_directed_nonempty_compact_closed
[GOAL]
case h.refine'_3.hZd
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ Directed (fun x x_1 => x ⊇ x_1) fun i => (↑i)ᶜ
[PROOFSTEP]
rintro ⟨U, hU⟩ ⟨U', hU'⟩
[GOAL]
case h.refine'_3.hZd.mk.mk
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
U : Set α
hU : U ∈ c
U' : Set α
hU' : U' ∈ c
⊢ ∃ z,
(fun x x_1 => x ⊇ x_1) ((fun i => (↑i)ᶜ) { val := U, property := hU }) ((fun i => (↑i)ᶜ) z) ∧
(fun x x_1 => x ⊇ x_1) ((fun i => (↑i)ᶜ) { val := U', property := hU' }) ((fun i => (↑i)ᶜ) z)
[PROOFSTEP]
obtain ⟨V, hVc, hVU, hVU'⟩ := hz.directedOn U hU U' hU'
[GOAL]
case h.refine'_3.hZd.mk.mk.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
U : Set α
hU : U ∈ c
U' : Set α
hU' : U' ∈ c
V : Set α
hVc : V ∈ c
hVU : U ⊆ V
hVU' : U' ⊆ V
⊢ ∃ z,
(fun x x_1 => x ⊇ x_1) ((fun i => (↑i)ᶜ) { val := U, property := hU }) ((fun i => (↑i)ᶜ) z) ∧
(fun x x_1 => x ⊇ x_1) ((fun i => (↑i)ᶜ) { val := U', property := hU' }) ((fun i => (↑i)ᶜ) z)
[PROOFSTEP]
exact ⟨⟨V, hVc⟩, Set.compl_subset_compl.mpr hVU, Set.compl_subset_compl.mpr hVU'⟩
[GOAL]
case h.refine'_3.hZn
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ ∀ (i : { U // U ∈ c }), Set.Nonempty (↑i)ᶜ
[PROOFSTEP]
exact fun U => (hc U.2).2.2
[GOAL]
case h.refine'_3.hZc
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ ∀ (i : { U // U ∈ c }), IsCompact (↑i)ᶜ
[PROOFSTEP]
exact fun U => (hc U.2).2.1.isClosed_compl.isCompact
[GOAL]
case h.refine'_3.hZcl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
U₀ : Set α
hU₀ : U₀ ∈ c
this : Nonempty { U // U ∈ c }
U₀compl : Sᶜ ⊆ U₀
⊢ ∀ (i : { U // U ∈ c }), IsClosed (↑i)ᶜ
[PROOFSTEP]
exact fun U => (hc U.2).2.1.isClosed_compl
[GOAL]
case neg
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
hcne : ¬Set.Nonempty c
⊢ ∃ ub, ub ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ ub
[PROOFSTEP]
use Sᶜ
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
hcne : ¬Set.Nonempty c
⊢ Sᶜ ∈ opens ∧ ∀ (s : Set α), s ∈ c → s ⊆ Sᶜ
[PROOFSTEP]
refine' ⟨⟨Set.Subset.refl _, isOpen_compl_iff.mpr hS, _⟩, fun U Uc => (hcne ⟨U, Uc⟩).elim⟩
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
hcne : ¬Set.Nonempty c
⊢ Set.Nonempty Sᶜᶜ
[PROOFSTEP]
rw [compl_compl]
[GOAL]
case h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
c : Set (Set α)
hc : c ⊆ opens
hz : IsChain (fun x x_1 => x ⊆ x_1) c
hcne : ¬Set.Nonempty c
⊢ Set.Nonempty S
[PROOFSTEP]
exact hne
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
⊢ ∃ V, V ⊆ S ∧ Set.Nonempty V ∧ IsClosed V ∧ ∀ (V' : Set α), V' ⊆ V → Set.Nonempty V' → IsClosed V' → V' = V
[PROOFSTEP]
refine' ⟨Uᶜ, Set.compl_subset_comm.mp Uc, Ucne, Uo.isClosed_compl, _⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
⊢ ∀ (V' : Set α), V' ⊆ Uᶜ → Set.Nonempty V' → IsClosed V' → V' = Uᶜ
[PROOFSTEP]
intro V' V'sub V'ne V'cls
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
V' : Set α
V'sub : V' ⊆ Uᶜ
V'ne : Set.Nonempty V'
V'cls : IsClosed V'
⊢ V' = Uᶜ
[PROOFSTEP]
have : V'ᶜ = U := by
refine' h V'ᶜ ⟨_, isOpen_compl_iff.mpr V'cls, _⟩ (Set.subset_compl_comm.mp V'sub)
exact Set.Subset.trans Uc (Set.subset_compl_comm.mp V'sub)
simp only [compl_compl, V'ne]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
V' : Set α
V'sub : V' ⊆ Uᶜ
V'ne : Set.Nonempty V'
V'cls : IsClosed V'
⊢ V'ᶜ = U
[PROOFSTEP]
refine' h V'ᶜ ⟨_, isOpen_compl_iff.mpr V'cls, _⟩ (Set.subset_compl_comm.mp V'sub)
[GOAL]
case refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
V' : Set α
V'sub : V' ⊆ Uᶜ
V'ne : Set.Nonempty V'
V'cls : IsClosed V'
⊢ Sᶜ ⊆ V'ᶜ
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
V' : Set α
V'sub : V' ⊆ Uᶜ
V'ne : Set.Nonempty V'
V'cls : IsClosed V'
⊢ Set.Nonempty V'ᶜᶜ
[PROOFSTEP]
exact Set.Subset.trans Uc (Set.subset_compl_comm.mp V'sub)
[GOAL]
case refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
V' : Set α
V'sub : V' ⊆ Uᶜ
V'ne : Set.Nonempty V'
V'cls : IsClosed V'
⊢ Set.Nonempty V'ᶜᶜ
[PROOFSTEP]
simp only [compl_compl, V'ne]
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : CompactSpace α
S : Set α
hS : IsClosed S
hne : Set.Nonempty S
opens : Set (Set α) := {U | Sᶜ ⊆ U ∧ IsOpen U ∧ Set.Nonempty Uᶜ}
U : Set α
h : ∀ (a : Set α), a ∈ opens → U ⊆ a → a = U
Uc : Sᶜ ⊆ U
Uo : IsOpen U
Ucne : Set.Nonempty Uᶜ
V' : Set α
V'sub : V' ⊆ Uᶜ
V'ne : Set.Nonempty V'
V'cls : IsClosed V'
this : V'ᶜ = U
⊢ V' = Uᶜ
[PROOFSTEP]
rw [← this, compl_compl]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : LocallyCompactSpace α
inst✝ : SecondCountableTopology α
⊢ SigmaCompactSpace α
[PROOFSTEP]
choose K hKc hxK using fun x : α => exists_compact_mem_nhds x
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : LocallyCompactSpace α
inst✝ : SecondCountableTopology α
K : α → Set α
hKc : ∀ (x : α), IsCompact (K x)
hxK : ∀ (x : α), K x ∈ 𝓝 x
⊢ SigmaCompactSpace α
[PROOFSTEP]
rcases countable_cover_nhds hxK with ⟨s, hsc, hsU⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s✝ t : Set α
inst✝¹ : LocallyCompactSpace α
inst✝ : SecondCountableTopology α
K : α → Set α
hKc : ∀ (x : α), IsCompact (K x)
hxK : ∀ (x : α), K x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (x : α) (_ : x ∈ s), K x = univ
⊢ SigmaCompactSpace α
[PROOFSTEP]
refine' SigmaCompactSpace.of_countable _ (hsc.image K) (ball_image_iff.2 fun x _ => hKc x) _
[GOAL]
case intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s✝ t : Set α
inst✝¹ : LocallyCompactSpace α
inst✝ : SecondCountableTopology α
K : α → Set α
hKc : ∀ (x : α), IsCompact (K x)
hxK : ∀ (x : α), K x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (x : α) (_ : x ∈ s), K x = univ
⊢ ⋃₀ (K '' s) = univ
[PROOFSTEP]
rwa [sUnion_image]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
⊢ ⋃ (n : ℕ), compactCovering α n = univ
[PROOFSTEP]
rw [compactCovering, iUnion_accumulate]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
⊢ ⋃ (x : ℕ), Exists.choose (_ : ∃ K, (∀ (n : ℕ), IsCompact (K n)) ∧ ⋃ (n : ℕ), K n = univ) x = univ
[PROOFSTEP]
exact (Classical.choose_spec SigmaCompactSpace.exists_compact_covering).2
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : SigmaCompactSpace α
inst✝ : SigmaCompactSpace β
⊢ ⋃ (n : ℕ), (fun n => compactCovering α n ×ˢ compactCovering β n) n = univ
[PROOFSTEP]
simp only [iUnion_prod_of_monotone (compactCovering_subset α) (compactCovering_subset β), iUnion_compactCovering,
univ_prod_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
⊢ SigmaCompactSpace ((i : ι) → π i)
[PROOFSTEP]
refine'
⟨⟨fun n => Set.pi univ fun i => compactCovering (π i) n, fun n =>
isCompact_univ_pi fun i => isCompact_compactCovering (π i) _, _⟩⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
⊢ ⋃ (n : ℕ), (fun n => Set.pi univ fun i => compactCovering (π i) n) n = univ
[PROOFSTEP]
rw [iUnion_univ_pi_of_monotone]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
⊢ (Set.pi univ fun i => ⋃ (j : ℕ), compactCovering (π i) j) = univ
[PROOFSTEP]
simp only [iUnion_compactCovering, pi_univ]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Finite ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
⊢ ∀ (i : ι), Monotone fun n => compactCovering (π i) n
[PROOFSTEP]
exact fun i => compactCovering_subset (π i)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
s t : Set α
inst✝¹ : SigmaCompactSpace α
inst✝ : SigmaCompactSpace β
⊢ ⋃ (n : ℕ), (fun n => Sum.inl '' compactCovering α n ∪ Sum.inr '' compactCovering β n) n = univ
[PROOFSTEP]
simp only [iUnion_union_distrib, ← image_iUnion, iUnion_compactCovering, image_univ, range_inl_union_range_inr]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
⊢ SigmaCompactSpace ((i : ι) × π i)
[PROOFSTEP]
cases isEmpty_or_nonempty ι
[GOAL]
case inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : IsEmpty ι
⊢ SigmaCompactSpace ((i : ι) × π i)
[PROOFSTEP]
infer_instance
[GOAL]
case inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
⊢ SigmaCompactSpace ((i : ι) × π i)
[PROOFSTEP]
rcases exists_surjective_nat ι with ⟨f, hf⟩
[GOAL]
case inr.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
⊢ SigmaCompactSpace ((i : ι) × π i)
[PROOFSTEP]
refine' ⟨⟨fun n => ⋃ k ≤ n, Sigma.mk (f k) '' compactCovering (π (f k)) n, fun n => _, _⟩⟩
[GOAL]
case inr.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
n : ℕ
⊢ IsCompact ((fun n => ⋃ (k : ℕ) (_ : k ≤ n), Sigma.mk (f k) '' compactCovering (π (f k)) n) n)
[PROOFSTEP]
refine' (finite_le_nat _).isCompact_biUnion fun k _ => _
[GOAL]
case inr.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
n k : ℕ
x✝ : k ∈ {i | i ≤ n}
⊢ IsCompact (Sigma.mk (f k) '' compactCovering (π (f k)) n)
[PROOFSTEP]
exact (isCompact_compactCovering _ _).image continuous_sigmaMk
[GOAL]
case inr.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
⊢ ⋃ (n : ℕ), (fun n => ⋃ (k : ℕ) (_ : k ≤ n), Sigma.mk (f k) '' compactCovering (π (f k)) n) n = univ
[PROOFSTEP]
simp only [iUnion_eq_univ_iff, Sigma.forall, mem_iUnion]
[GOAL]
case inr.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
⊢ ∀ (a : ι) (b : π a), ∃ i i_1 i_2, { fst := a, snd := b } ∈ Sigma.mk (f i_1) '' compactCovering (π (f i_1)) i
[PROOFSTEP]
rw [hf.forall]
-- porting note: `simp only` failed to use `hf.forall`
[GOAL]
case inr.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
⊢ ∀ (x : ℕ) (b : π (f x)), ∃ i i_1 i_2, { fst := f x, snd := b } ∈ Sigma.mk (f i_1) '' compactCovering (π (f i_1)) i
[PROOFSTEP]
intro k y
[GOAL]
case inr.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
k : ℕ
y : π (f k)
⊢ ∃ i i_1 i_2, { fst := f k, snd := y } ∈ Sigma.mk (f i_1) '' compactCovering (π (f i_1)) i
[PROOFSTEP]
rcases exists_mem_compactCovering y with ⟨n, hn⟩
[GOAL]
case inr.intro.refine'_2.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
k : ℕ
y : π (f k)
n : ℕ
hn : y ∈ compactCovering (π (f k)) n
⊢ ∃ i i_1 i_2, { fst := f k, snd := y } ∈ Sigma.mk (f i_1) '' compactCovering (π (f i_1)) i
[PROOFSTEP]
refine' ⟨max k n, k, le_max_left _ _, mem_image_of_mem _ _⟩
[GOAL]
case inr.intro.refine'_2.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁵ : TopologicalSpace α
inst✝⁴ : TopologicalSpace β
s t : Set α
inst✝³ : SigmaCompactSpace α
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), SigmaCompactSpace (π i)
h✝ : Nonempty ι
f : ℕ → ι
hf : Function.Surjective f
k : ℕ
y : π (f k)
n : ℕ
hn : y ∈ compactCovering (π (f k)) n
⊢ y ∈ compactCovering (π (f k)) (max k n)
[PROOFSTEP]
exact compactCovering_subset _ (le_max_right _ _) hn
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
e : β → α
he : ClosedEmbedding e
⊢ ⋃ (n : ℕ), (fun n => e ⁻¹' compactCovering α n) n = univ
[PROOFSTEP]
rw [← preimage_iUnion, iUnion_compactCovering, preimage_univ]
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
ι : Type u_3
f : ι → Set α
hf : LocallyFinite f
hne : ∀ (i : ι), Set.Nonempty (f i)
⊢ Set.Countable univ
[PROOFSTEP]
have := fun n => hf.finite_nonempty_inter_compact (isCompact_compactCovering α n)
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
ι : Type u_3
f : ι → Set α
hf : LocallyFinite f
hne : ∀ (i : ι), Set.Nonempty (f i)
this : ∀ (n : ℕ), Set.Finite {i | Set.Nonempty (f i ∩ compactCovering α n)}
⊢ Set.Countable univ
[PROOFSTEP]
refine (countable_iUnion fun n => (this n).countable).mono fun i _ => ?_
[GOAL]
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
ι : Type u_3
f : ι → Set α
hf : LocallyFinite f
hne : ∀ (i : ι), Set.Nonempty (f i)
this : ∀ (n : ℕ), Set.Finite {i | Set.Nonempty (f i ∩ compactCovering α n)}
i : ι
x✝ : i ∈ univ
⊢ i ∈ ⋃ (i : ℕ), {i_1 | Set.Nonempty (f i_1 ∩ compactCovering α i)}
[PROOFSTEP]
rcases hne i with ⟨x, hx⟩
[GOAL]
case intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
ι : Type u_3
f : ι → Set α
hf : LocallyFinite f
hne : ∀ (i : ι), Set.Nonempty (f i)
this : ∀ (n : ℕ), Set.Finite {i | Set.Nonempty (f i ∩ compactCovering α n)}
i : ι
x✝ : i ∈ univ
x : α
hx : x ∈ f i
⊢ i ∈ ⋃ (i : ℕ), {i_1 | Set.Nonempty (f i_1 ∩ compactCovering α i)}
[PROOFSTEP]
rcases iUnion_eq_univ_iff.1 (iUnion_compactCovering α) x with ⟨n, hn⟩
[GOAL]
case intro.intro
α : Type u
β : Type v
ι✝ : Type u_1
π : ι✝ → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
ι : Type u_3
f : ι → Set α
hf : LocallyFinite f
hne : ∀ (i : ι), Set.Nonempty (f i)
this : ∀ (n : ℕ), Set.Finite {i | Set.Nonempty (f i ∩ compactCovering α n)}
i : ι
x✝ : i ∈ univ
x : α
hx : x ∈ f i
n : ℕ
hn : x ∈ compactCovering α n
⊢ i ∈ ⋃ (i : ℕ), {i_1 | Set.Nonempty (f i_1 ∩ compactCovering α i)}
[PROOFSTEP]
exact mem_iUnion.2 ⟨n, x, hx, hn⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
s : Set α
hs : IsClosed s
hf : ∀ (x : α), x ∈ s → f x ∈ 𝓝[s] x
⊢ ∃ t x, Set.Countable t ∧ s ⊆ ⋃ (x : α) (_ : x ∈ t), f x
[PROOFSTEP]
simp only [nhdsWithin, mem_inf_principal] at hf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
s : Set α
hs : IsClosed s
hf : ∀ (x : α), x ∈ s → {x_1 | x_1 ∈ s → x_1 ∈ f x} ∈ 𝓝 x
⊢ ∃ t x, Set.Countable t ∧ s ⊆ ⋃ (x : α) (_ : x ∈ t), f x
[PROOFSTEP]
choose t ht hsub using fun n =>
((isCompact_compactCovering α n).inter_right hs).elim_nhds_subcover _ fun x hx => hf x hx.right
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
s : Set α
hs : IsClosed s
hf : ∀ (x : α), x ∈ s → {x_1 | x_1 ∈ s → x_1 ∈ f x} ∈ 𝓝 x
t : ℕ → Finset α
ht : ∀ (n : ℕ) (x : α), x ∈ t n → x ∈ compactCovering α n ∩ s
hsub : ∀ (n : ℕ), compactCovering α n ∩ s ⊆ ⋃ (x : α) (_ : x ∈ t n), {x_1 | x_1 ∈ s → x_1 ∈ f x}
⊢ ∃ t x, Set.Countable t ∧ s ⊆ ⋃ (x : α) (_ : x ∈ t), f x
[PROOFSTEP]
refine'
⟨⋃ n, (t n : Set α), iUnion_subset fun n x hx => (ht n x hx).2, countable_iUnion fun n => (t n).countable_toSet,
fun x hx => mem_iUnion₂.2 _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
s : Set α
hs : IsClosed s
hf : ∀ (x : α), x ∈ s → {x_1 | x_1 ∈ s → x_1 ∈ f x} ∈ 𝓝 x
t : ℕ → Finset α
ht : ∀ (n : ℕ) (x : α), x ∈ t n → x ∈ compactCovering α n ∩ s
hsub : ∀ (n : ℕ), compactCovering α n ∩ s ⊆ ⋃ (x : α) (_ : x ∈ t n), {x_1 | x_1 ∈ s → x_1 ∈ f x}
x : α
hx : x ∈ s
⊢ ∃ i j, x ∈ f i
[PROOFSTEP]
rcases exists_mem_compactCovering x with ⟨n, hn⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
s : Set α
hs : IsClosed s
hf : ∀ (x : α), x ∈ s → {x_1 | x_1 ∈ s → x_1 ∈ f x} ∈ 𝓝 x
t : ℕ → Finset α
ht : ∀ (n : ℕ) (x : α), x ∈ t n → x ∈ compactCovering α n ∩ s
hsub : ∀ (n : ℕ), compactCovering α n ∩ s ⊆ ⋃ (x : α) (_ : x ∈ t n), {x_1 | x_1 ∈ s → x_1 ∈ f x}
x : α
hx : x ∈ s
n : ℕ
hn : x ∈ compactCovering α n
⊢ ∃ i j, x ∈ f i
[PROOFSTEP]
rcases mem_iUnion₂.1 (hsub n ⟨hn, hx⟩) with ⟨y, hyt : y ∈ t n, hyf : x ∈ s → x ∈ f y⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
s : Set α
hs : IsClosed s
hf : ∀ (x : α), x ∈ s → {x_1 | x_1 ∈ s → x_1 ∈ f x} ∈ 𝓝 x
t : ℕ → Finset α
ht : ∀ (n : ℕ) (x : α), x ∈ t n → x ∈ compactCovering α n ∩ s
hsub : ∀ (n : ℕ), compactCovering α n ∩ s ⊆ ⋃ (x : α) (_ : x ∈ t n), {x_1 | x_1 ∈ s → x_1 ∈ f x}
x : α
hx : x ∈ s
n : ℕ
hn : x ∈ compactCovering α n
y : α
hyt : y ∈ t n
hyf : x ∈ s → x ∈ f y
⊢ ∃ i j, x ∈ f i
[PROOFSTEP]
exact ⟨y, mem_iUnion.2 ⟨n, hyt⟩, hyf hx⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
⊢ ∃ s, Set.Countable s ∧ ⋃ (x : α) (_ : x ∈ s), f x = univ
[PROOFSTEP]
simp only [← nhdsWithin_univ] at hf
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝[univ] x
⊢ ∃ s, Set.Countable s ∧ ⋃ (x : α) (_ : x ∈ s), f x = univ
[PROOFSTEP]
rcases countable_cover_nhdsWithin_of_sigma_compact isClosed_univ fun x _ => hf x with ⟨s, -, hsc, hsU⟩
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
inst✝ : SigmaCompactSpace α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝[univ] x
s : Set α
hsc : Set.Countable s
hsU : univ ⊆ ⋃ (x : α) (_ : x ∈ s), f x
⊢ ∃ s, Set.Countable s ∧ ⋃ (x : α) (_ : x ∈ s), f x = univ
[PROOFSTEP]
exact ⟨s, hsc, univ_subset_iff.1 hsU⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t : Set α
K : CompactExhaustion α
x : α
⊢ ¬CompactExhaustion.find (shiftr K) x ≤ CompactExhaustion.find K x
[PROOFSTEP]
simp only [find_shiftr, not_le, Nat.lt_succ_self]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
K : CompactExhaustion α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : LocallyCompactSpace X
inst✝ : SigmaCompactSpace X
⊢ CompactExhaustion X
[PROOFSTEP]
apply Classical.choice
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
K : CompactExhaustion α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : LocallyCompactSpace X
inst✝ : SigmaCompactSpace X
⊢ Nonempty (CompactExhaustion X)
[PROOFSTEP]
let K : ℕ → { s : Set X // IsCompact s } := fun n =>
Nat.recOn n ⟨∅, isCompact_empty⟩ fun n s =>
⟨(exists_compact_superset s.2).choose ∪ compactCovering X n,
(exists_compact_superset s.2).choose_spec.1.union (isCompact_compactCovering _ _)⟩
[GOAL]
case a
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
K✝ : CompactExhaustion α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : LocallyCompactSpace X
inst✝ : SigmaCompactSpace X
K : ℕ → { s // IsCompact s } :=
fun n =>
Nat.recOn n { val := ∅, property := (_ : IsCompact ∅) } fun n s =>
{ val := Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n,
property := (_ : IsCompact (Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n)) }
⊢ Nonempty (CompactExhaustion X)
[PROOFSTEP]
refine' ⟨⟨fun n => (K n).1, fun n => (K n).2, fun n => _, _⟩⟩
[GOAL]
case a.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
K✝ : CompactExhaustion α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : LocallyCompactSpace X
inst✝ : SigmaCompactSpace X
K : ℕ → { s // IsCompact s } :=
fun n =>
Nat.recOn n { val := ∅, property := (_ : IsCompact ∅) } fun n s =>
{ val := Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n,
property := (_ : IsCompact (Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n)) }
n : ℕ
⊢ (fun n => ↑(K n)) n ⊆ interior ((fun n => ↑(K n)) (n + 1))
[PROOFSTEP]
exact Subset.trans (exists_compact_superset (K n).2).choose_spec.2 (interior_mono <| subset_union_left _ _)
[GOAL]
case a.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
K✝ : CompactExhaustion α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : LocallyCompactSpace X
inst✝ : SigmaCompactSpace X
K : ℕ → { s // IsCompact s } :=
fun n =>
Nat.recOn n { val := ∅, property := (_ : IsCompact ∅) } fun n s =>
{ val := Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n,
property := (_ : IsCompact (Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n)) }
⊢ ⋃ (n : ℕ), (fun n => ↑(K n)) n = univ
[PROOFSTEP]
refine' univ_subset_iff.1 (iUnion_compactCovering X ▸ _)
[GOAL]
case a.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝⁴ : TopologicalSpace α
inst✝³ : TopologicalSpace β
s t : Set α
K✝ : CompactExhaustion α
X : Type u_3
inst✝² : TopologicalSpace X
inst✝¹ : LocallyCompactSpace X
inst✝ : SigmaCompactSpace X
K : ℕ → { s // IsCompact s } :=
fun n =>
Nat.recOn n { val := ∅, property := (_ : IsCompact ∅) } fun n s =>
{ val := Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n,
property := (_ : IsCompact (Exists.choose (_ : ∃ K', IsCompact K' ∧ ↑s ⊆ interior K') ∪ compactCovering X n)) }
⊢ ⋃ (n : ℕ), compactCovering X n ⊆ ⋃ (n : ℕ), (fun n => ↑(K n)) n
[PROOFSTEP]
exact iUnion_mono' fun n => ⟨n + 1, subset_union_right _ _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ IsClopen s ↔ frontier s = ∅
[PROOFSTEP]
rw [IsClopen, ← closure_eq_iff_isClosed, ← interior_eq_iff_isOpen, frontier, diff_eq_empty]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ interior s = s ∧ closure s = s ↔ closure s ⊆ interior s
[PROOFSTEP]
refine' ⟨fun h => (h.2.trans h.1.symm).subset, fun h => _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : closure s ⊆ interior s
⊢ interior s = s ∧ closure s = s
[PROOFSTEP]
exact ⟨interior_subset.antisymm (subset_closure.trans h), (h.trans interior_subset).antisymm subset_closure⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
⊢ IsClopen (Z ∩ a)
[PROOFSTEP]
refine' ⟨IsOpen.inter h.1 ha, _⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
⊢ IsClosed (Z ∩ a)
[PROOFSTEP]
have : IsClosed (Z ∩ bᶜ) := IsClosed.inter h.2 (isClosed_compl_iff.2 hb)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
this : IsClosed (Z ∩ bᶜ)
⊢ IsClosed (Z ∩ a)
[PROOFSTEP]
convert this using 1
[GOAL]
case h.e'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
this : IsClosed (Z ∩ bᶜ)
⊢ Z ∩ a = Z ∩ bᶜ
[PROOFSTEP]
refine' (inter_subset_inter_right Z hab.subset_compl_right).antisymm _
[GOAL]
case h.e'_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
this : IsClosed (Z ∩ bᶜ)
⊢ Z ∩ bᶜ ⊆ Z ∩ a
[PROOFSTEP]
rintro x ⟨hx₁, hx₂⟩
[GOAL]
case h.e'_3.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
this : IsClosed (Z ∩ bᶜ)
x : α
hx₁ : x ∈ Z
hx₂ : x ∈ bᶜ
⊢ x ∈ Z ∩ a
[PROOFSTEP]
exact ⟨hx₁, by simpa [not_mem_of_mem_compl hx₂] using cover hx₁⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z a b : Set α
h : IsClopen Z
cover : Z ⊆ a ∪ b
ha : IsOpen a
hb : IsOpen b
hab : Disjoint a b
this : IsClosed (Z ∩ bᶜ)
x : α
hx₁ : x ∈ Z
hx₂ : x ∈ bᶜ
⊢ x ∈ a
[PROOFSTEP]
simpa [not_mem_of_mem_compl hx₂] using cover hx₁
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
⊢ Continuous (boolIndicator U) ↔ IsClopen U
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
⊢ Continuous (boolIndicator U) → IsClopen U
[PROOFSTEP]
intro hc
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hc : Continuous (boolIndicator U)
⊢ IsClopen U
[PROOFSTEP]
rw [← U.preimage_boolIndicator_true]
[GOAL]
case mp
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hc : Continuous (boolIndicator U)
⊢ IsClopen (boolIndicator U ⁻¹' {true})
[PROOFSTEP]
exact ⟨(isOpen_discrete _).preimage hc, (isClosed_discrete _).preimage hc⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
⊢ IsClopen U → Continuous (boolIndicator U)
[PROOFSTEP]
refine' fun hU => ⟨fun s _ => _⟩
[GOAL]
case mpr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
⊢ IsOpen (boolIndicator U ⁻¹' s)
[PROOFSTEP]
rcases U.preimage_boolIndicator s with (h | h | h | h)
[GOAL]
case mpr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = univ
⊢ IsOpen (boolIndicator U ⁻¹' s)
[PROOFSTEP]
rw [h]
[GOAL]
case mpr.inr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = U
⊢ IsOpen (boolIndicator U ⁻¹' s)
[PROOFSTEP]
rw [h]
[GOAL]
case mpr.inr.inr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = Uᶜ
⊢ IsOpen (boolIndicator U ⁻¹' s)
[PROOFSTEP]
rw [h]
[GOAL]
case mpr.inr.inr.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = ∅
⊢ IsOpen (boolIndicator U ⁻¹' s)
[PROOFSTEP]
rw [h]
[GOAL]
case mpr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = univ
⊢ IsOpen univ
case mpr.inr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = U
⊢ IsOpen U
case mpr.inr.inr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = Uᶜ
⊢ IsOpen Uᶜ
case mpr.inr.inr.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
U : Set X
hU : IsClopen U
s : Set Bool
x✝ : IsOpen s
h : boolIndicator U ⁻¹' s = ∅
⊢ IsOpen ∅
[PROOFSTEP]
exacts [isOpen_univ, hU.1, hU.2.isOpen_compl, isOpen_empty]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
s U : Set X
⊢ ContinuousOn (boolIndicator U) s ↔ IsClopen (Subtype.val ⁻¹' U)
[PROOFSTEP]
rw [continuousOn_iff_continuous_restrict, ← continuous_boolIndicator_iff_clopen]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t : Set α
X : Type u_3
inst✝ : TopologicalSpace X
s U : Set X
⊢ Continuous (restrict s (boolIndicator U)) ↔ Continuous (boolIndicator (Subtype.val ⁻¹' U))
[PROOFSTEP]
rfl
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ Set.Nonempty (closure s ∩ u) → Set.Nonempty (closure s ∩ v) → Set.Nonempty (closure s ∩ (u ∩ v)) ↔
Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
iterate 3 rw [closure_inter_open_nonempty_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ Set.Nonempty (closure s ∩ u) → Set.Nonempty (closure s ∩ v) → Set.Nonempty (closure s ∩ (u ∩ v)) ↔
Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
rw [closure_inter_open_nonempty_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ Set.Nonempty (s ∩ u) → Set.Nonempty (closure s ∩ v) → Set.Nonempty (closure s ∩ (u ∩ v)) ↔
Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ IsOpen u
[PROOFSTEP]
rw [closure_inter_open_nonempty_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (closure s ∩ (u ∩ v)) ↔
Set.Nonempty (s ∩ u) → Set.Nonempty (s ∩ v) → Set.Nonempty (s ∩ (u ∩ v))
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ IsOpen v
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ IsOpen u
[PROOFSTEP]
rw [closure_inter_open_nonempty_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ IsOpen (u ∩ v)
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ IsOpen v
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s u v : Set α
hu : IsOpen u
hv : IsOpen v
⊢ IsOpen u
[PROOFSTEP]
exacts [hu.inter hv, hv, hu]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : s ∈ irreducibleComponents α
⊢ IsClosed s
[PROOFSTEP]
rw [← closure_eq_iff_isClosed, eq_comm]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : s ∈ irreducibleComponents α
⊢ s = closure s
[PROOFSTEP]
exact subset_closure.antisymm (H.2 H.1.closure subset_closure)
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
⊢ irreducibleComponents α = maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
[PROOFSTEP]
ext s
[GOAL]
case h
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
⊢ s ∈ irreducibleComponents α ↔ s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
[PROOFSTEP]
constructor
[GOAL]
case h.mp
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
⊢ s ∈ irreducibleComponents α → s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
[PROOFSTEP]
intro H
[GOAL]
case h.mp
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
H : s ∈ irreducibleComponents α
⊢ s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
[PROOFSTEP]
exact ⟨⟨isClosed_of_mem_irreducibleComponents _ H, H.1⟩, fun x h e => H.2 h.2 e⟩
[GOAL]
case h.mpr
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
⊢ s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s} → s ∈ irreducibleComponents α
[PROOFSTEP]
intro H
[GOAL]
case h.mpr
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
H : s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
⊢ s ∈ irreducibleComponents α
[PROOFSTEP]
refine' ⟨H.1.2, fun x h e => _⟩
[GOAL]
case h.mpr
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
H : s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
x : Set α
h : x ∈ {s | IsIrreducible s}
e : (fun x x_1 => x ≤ x_1) s x
⊢ (fun x x_1 => x ≤ x_1) x s
[PROOFSTEP]
have : closure x ≤ s := H.2 ⟨isClosed_closure, h.closure⟩ (e.trans subset_closure)
[GOAL]
case h.mpr
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s✝ t : Set α✝
α : Type u_3
inst✝ : TopologicalSpace α
s : Set α
H : s ∈ maximals (fun x x_1 => x ≤ x_1) {s | IsClosed s ∧ IsIrreducible s}
x : Set α
h : x ∈ {s | IsIrreducible s}
e : (fun x x_1 => x ≤ x_1) s x
this : closure x ≤ s
⊢ (fun x x_1 => x ≤ x_1) x s
[PROOFSTEP]
exact le_trans subset_closure this
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
s✝ t✝ : Set α
inst✝ : PreirreducibleSpace α
s t : Set α
⊢ IsOpen s → IsOpen t → Set.Nonempty s → Set.Nonempty t → Set.Nonempty (s ∩ t)
[PROOFSTEP]
simpa only [univ_inter, univ_subset_iff] using @PreirreducibleSpace.isPreirreducible_univ α _ _ s t
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
⊢ IsPreirreducible (f '' s)
[PROOFSTEP]
rintro u v hu hv ⟨_, ⟨⟨x, hx, rfl⟩, hxu⟩⟩ ⟨_, ⟨⟨y, hy, rfl⟩, hyv⟩⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : f x ∈ u
y : α
hy : y ∈ s
hyv : f y ∈ v
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rw [← mem_preimage] at hxu hyv
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rcases continuousOn_iff'.1 hf u hu with ⟨u', hu', u'_eq⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rcases continuousOn_iff'.1 hf v hv with ⟨v', hv', v'_eq⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
have := H u' v' hu' hv'
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (s ∩ u') → Set.Nonempty (s ∩ v') → Set.Nonempty (s ∩ (u' ∩ v'))
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rw [inter_comm s u', ← u'_eq] at this
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (s ∩ v') → Set.Nonempty (s ∩ (u' ∩ v'))
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rw [inter_comm s v', ← v'_eq] at this
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
rcases this ⟨x, hxu, hx⟩ ⟨y, hyv, hy⟩ with ⟨z, hzs, hzu', hzv'⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ Set.Nonempty (f '' s ∩ (u ∩ v))
[PROOFSTEP]
refine' ⟨f z, mem_image_of_mem f hzs, _, _⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ f z ∈ u
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ f z ∈ v
[PROOFSTEP]
all_goals
rw [← mem_preimage]
apply mem_of_mem_inter_left
show z ∈ _ ∩ s
simp [*]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ f z ∈ u
[PROOFSTEP]
rw [← mem_preimage]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ z ∈ f ⁻¹' u
[PROOFSTEP]
apply mem_of_mem_inter_left
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ z ∈ f ⁻¹' u ∩ ?intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1.b
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1.b
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ Set α
[PROOFSTEP]
show z ∈ _ ∩ s
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_1.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ z ∈ f ⁻¹' u ∩ s
[PROOFSTEP]
simp [*]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ f z ∈ v
[PROOFSTEP]
rw [← mem_preimage]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ z ∈ f ⁻¹' v
[PROOFSTEP]
apply mem_of_mem_inter_left
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ z ∈ f ⁻¹' v ∩ ?intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2.b
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2.b
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ Set α
[PROOFSTEP]
show z ∈ _ ∩ s
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refine'_2.h
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
H : IsPreirreducible s
f : α → β
hf : ContinuousOn f s
u v : Set β
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ s
hxu : x ∈ f ⁻¹' u
y : α
hy : y ∈ s
hyv : y ∈ f ⁻¹' v
u' : Set α
hu' : IsOpen u'
u'_eq : f ⁻¹' u ∩ s = u' ∩ s
v' : Set α
hv' : IsOpen v'
v'_eq : f ⁻¹' v ∩ s = v' ∩ s
this : Set.Nonempty (f ⁻¹' u ∩ s) → Set.Nonempty (f ⁻¹' v ∩ s) → Set.Nonempty (s ∩ (u' ∩ v'))
z : α
hzs : z ∈ s
hzu' : z ∈ u'
hzv' : z ∈ v'
⊢ z ∈ f ⁻¹' v ∩ s
[PROOFSTEP]
simp [*]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsPreirreducible s
⊢ IsPreirreducible univ
[PROOFSTEP]
rintro _ _ ⟨u, hu, rfl⟩ ⟨v, hv, rfl⟩ ⟨⟨x, hxs⟩, -, hxu⟩ ⟨⟨y, hys⟩, -, hyv⟩
[GOAL]
case intro.intro.intro.intro.intro.mk.intro.intro.mk.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsPreirreducible s
u : Set α
hu : IsOpen u
v : Set α
hv : IsOpen v
x : α
hxs : x ∈ s
hxu : { val := x, property := hxs } ∈ val ⁻¹' u
y : α
hys : y ∈ s
hyv : { val := y, property := hys } ∈ val ⁻¹' v
⊢ Set.Nonempty (univ ∩ (val ⁻¹' u ∩ val ⁻¹' v))
[PROOFSTEP]
rcases h u v hu hv ⟨x, hxs, hxu⟩ ⟨y, hys, hyv⟩ with ⟨z, hzs, ⟨hzu, hzv⟩⟩
[GOAL]
case intro.intro.intro.intro.intro.mk.intro.intro.mk.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsPreirreducible s
u : Set α
hu : IsOpen u
v : Set α
hv : IsOpen v
x : α
hxs : x ∈ s
hxu : { val := x, property := hxs } ∈ val ⁻¹' u
y : α
hys : y ∈ s
hyv : { val := y, property := hys } ∈ val ⁻¹' v
z : α
hzs : z ∈ s
hzu : z ∈ u
hzv : z ∈ v
⊢ Set.Nonempty (univ ∩ (val ⁻¹' u ∩ val ⁻¹' v))
[PROOFSTEP]
exact ⟨⟨z, hzs⟩, ⟨Set.mem_univ _, ⟨hzu, hzv⟩⟩⟩
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t : Set α✝
α : Type ?u.291097
inst✝ : Infinite α
u v : Set (CofiniteTopology α)
⊢ IsOpen u → IsOpen v → Set.Nonempty (univ ∩ u) → Set.Nonempty (univ ∩ v) → Set.Nonempty (univ ∩ (u ∩ v))
[PROOFSTEP]
haveI : Infinite (CofiniteTopology α) := ‹_›
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t : Set α✝
α : Type ?u.291097
inst✝ : Infinite α
u v : Set (CofiniteTopology α)
this : Infinite (CofiniteTopology α)
⊢ IsOpen u → IsOpen v → Set.Nonempty (univ ∩ u) → Set.Nonempty (univ ∩ v) → Set.Nonempty (univ ∩ (u ∩ v))
[PROOFSTEP]
simp only [CofiniteTopology.isOpen_iff, univ_inter]
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t : Set α✝
α : Type ?u.291097
inst✝ : Infinite α
u v : Set (CofiniteTopology α)
this : Infinite (CofiniteTopology α)
⊢ (Set.Nonempty u → Set.Finite uᶜ) →
(Set.Nonempty v → Set.Finite vᶜ) → Set.Nonempty u → Set.Nonempty v → Set.Nonempty (u ∩ v)
[PROOFSTEP]
intro hu hv hu' hv'
[GOAL]
α✝ : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝² : TopologicalSpace α✝
inst✝¹ : TopologicalSpace β
s t : Set α✝
α : Type ?u.291097
inst✝ : Infinite α
u v : Set (CofiniteTopology α)
this : Infinite (CofiniteTopology α)
hu : Set.Nonempty u → Set.Finite uᶜ
hv : Set.Nonempty v → Set.Finite vᶜ
hu' : Set.Nonempty u
hv' : Set.Nonempty v
⊢ Set.Nonempty (u ∩ v)
[PROOFSTEP]
simpa only [compl_union, compl_compl] using ((hu hu').union (hv hv')).infinite_compl.nonempty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ IsIrreducible s ↔
∀ (U : Finset (Set α)),
(∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
[PROOFSTEP]
refine ⟨fun h U hu hU => ?_, fun h => ⟨?_, ?_⟩⟩
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
U : Finset (Set α)
hu : ∀ (u : Set α), u ∈ U → IsOpen u
hU : ∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑U)
[PROOFSTEP]
induction U using Finset.induction_on
[GOAL]
case refine_1.empty
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
hu : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hU : ∀ (u : Set α), u ∈ ∅ → Set.Nonempty (s ∩ u)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑∅)
case refine_1.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝¹ t s : Set α
h : IsIrreducible s
a✝² : Set α
s✝ : Finset (Set α)
a✝¹ : ¬a✝² ∈ s✝
a✝ : (∀ (u : Set α), u ∈ s✝ → IsOpen u) → (∀ (u : Set α), u ∈ s✝ → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑s✝)
hu : ∀ (u : Set α), u ∈ insert a✝² s✝ → IsOpen u
hU : ∀ (u : Set α), u ∈ insert a✝² s✝ → Set.Nonempty (s ∩ u)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑(insert a✝² s✝))
[PROOFSTEP]
case empty => simpa using h.nonempty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
hu : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hU : ∀ (u : Set α), u ∈ ∅ → Set.Nonempty (s ∩ u)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑∅)
[PROOFSTEP]
case empty => simpa using h.nonempty
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
hu : ∀ (u : Set α), u ∈ ∅ → IsOpen u
hU : ∀ (u : Set α), u ∈ ∅ → Set.Nonempty (s ∩ u)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑∅)
[PROOFSTEP]
simpa using h.nonempty
[GOAL]
case refine_1.insert
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝¹ t s : Set α
h : IsIrreducible s
a✝² : Set α
s✝ : Finset (Set α)
a✝¹ : ¬a✝² ∈ s✝
a✝ : (∀ (u : Set α), u ∈ s✝ → IsOpen u) → (∀ (u : Set α), u ∈ s✝ → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑s✝)
hu : ∀ (u : Set α), u ∈ insert a✝² s✝ → IsOpen u
hU : ∀ (u : Set α), u ∈ insert a✝² s✝ → Set.Nonempty (s ∩ u)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑(insert a✝² s✝))
[PROOFSTEP]
case insert u U _ IH =>
rw [Finset.coe_insert, sInter_insert]
rw [Finset.forall_mem_insert] at hu hU
exact h.2 _ _ hu.1 (isOpen_sInter U.finite_toSet hu.2) hU.1 (IH hu.2 hU.2)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
u : Set α
U : Finset (Set α)
a✝ : ¬u ∈ U
IH : (∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
hu : ∀ (u_1 : Set α), u_1 ∈ insert u U → IsOpen u_1
hU : ∀ (u_1 : Set α), u_1 ∈ insert u U → Set.Nonempty (s ∩ u_1)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑(insert u U))
[PROOFSTEP]
case insert u U _ IH =>
rw [Finset.coe_insert, sInter_insert]
rw [Finset.forall_mem_insert] at hu hU
exact h.2 _ _ hu.1 (isOpen_sInter U.finite_toSet hu.2) hU.1 (IH hu.2 hU.2)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
u : Set α
U : Finset (Set α)
a✝ : ¬u ∈ U
IH : (∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
hu : ∀ (u_1 : Set α), u_1 ∈ insert u U → IsOpen u_1
hU : ∀ (u_1 : Set α), u_1 ∈ insert u U → Set.Nonempty (s ∩ u_1)
⊢ Set.Nonempty (s ∩ ⋂₀ ↑(insert u U))
[PROOFSTEP]
rw [Finset.coe_insert, sInter_insert]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
u : Set α
U : Finset (Set α)
a✝ : ¬u ∈ U
IH : (∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
hu : ∀ (u_1 : Set α), u_1 ∈ insert u U → IsOpen u_1
hU : ∀ (u_1 : Set α), u_1 ∈ insert u U → Set.Nonempty (s ∩ u_1)
⊢ Set.Nonempty (s ∩ (u ∩ ⋂₀ ↑U))
[PROOFSTEP]
rw [Finset.forall_mem_insert] at hu hU
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h : IsIrreducible s
u : Set α
U : Finset (Set α)
a✝ : ¬u ∈ U
IH : (∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
hu : IsOpen u ∧ ∀ (x : Set α), x ∈ U → IsOpen x
hU : Set.Nonempty (s ∩ u) ∧ ∀ (x : Set α), x ∈ U → Set.Nonempty (s ∩ x)
⊢ Set.Nonempty (s ∩ (u ∩ ⋂₀ ↑U))
[PROOFSTEP]
exact h.2 _ _ hu.1 (isOpen_sInter U.finite_toSet hu.2) hU.1 (IH hu.2 hU.2)
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
⊢ Set.Nonempty s
[PROOFSTEP]
simpa using h ∅
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
⊢ IsPreirreducible s
[PROOFSTEP]
intro u v hu hv hu' hv'
[GOAL]
case refine_3
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
h :
∀ (U : Finset (Set α)),
(∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)
u v : Set α
hu : IsOpen u
hv : IsOpen v
hu' : Set.Nonempty (s ∩ u)
hv' : Set.Nonempty (s ∩ v)
⊢ Set.Nonempty (s ∩ (u ∩ v))
[PROOFSTEP]
simpa [*] using h { u, v }
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ IsPreirreducible s ↔ ∀ (z₁ z₂ : Set α), IsClosed z₁ → IsClosed z₂ → s ⊆ z₁ ∪ z₂ → s ⊆ z₁ ∨ s ⊆ z₂
[PROOFSTEP]
refine
compl_surjective.forall.trans <| forall_congr' fun z₁ => compl_surjective.forall.trans <| forall_congr' fun z₂ => ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s z₁ z₂ : Set α
⊢ IsOpen z₁ᶜ → IsOpen z₂ᶜ → Set.Nonempty (s ∩ z₁ᶜ) → Set.Nonempty (s ∩ z₂ᶜ) → Set.Nonempty (s ∩ (z₁ᶜ ∩ z₂ᶜ)) ↔
IsClosed z₁ → IsClosed z₂ → s ⊆ z₁ ∪ z₂ → s ⊆ z₁ ∨ s ⊆ z₂
[PROOFSTEP]
simp only [isOpen_compl_iff, ← compl_union, inter_compl_nonempty_iff]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s z₁ z₂ : Set α
⊢ IsClosed z₁ → IsClosed z₂ → ¬s ⊆ z₁ → ¬s ⊆ z₂ → ¬s ⊆ z₁ ∪ z₂ ↔
IsClosed z₁ → IsClosed z₂ → s ⊆ z₁ ∪ z₂ → s ⊆ z₁ ∨ s ⊆ z₂
[PROOFSTEP]
refine forall₂_congr fun _ _ => ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s z₁ z₂ : Set α
x✝¹ : IsClosed z₁
x✝ : IsClosed z₂
⊢ ¬s ⊆ z₁ → ¬s ⊆ z₂ → ¬s ⊆ z₁ ∪ z₂ ↔ s ⊆ z₁ ∪ z₂ → s ⊆ z₁ ∨ s ⊆ z₂
[PROOFSTEP]
rw [← and_imp, ← not_or, not_imp_not]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ IsIrreducible s ↔ ∀ (Z : Finset (Set α)), (∀ (z : Set α), z ∈ Z → IsClosed z) → s ⊆ ⋃₀ ↑Z → ∃ z, z ∈ Z ∧ s ⊆ z
[PROOFSTEP]
simp only [isIrreducible_iff_sInter]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
⊢ (∀ (U : Finset (Set α)),
(∀ (u : Set α), u ∈ U → IsOpen u) → (∀ (u : Set α), u ∈ U → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑U)) ↔
∀ (Z : Finset (Set α)), (∀ (z : Set α), z ∈ Z → IsClosed z) → s ⊆ ⋃₀ ↑Z → ∃ z, z ∈ Z ∧ s ⊆ z
[PROOFSTEP]
refine ((@compl_involutive (Set α) _).toPerm _).finsetCongr.forall_congr fun {Z} => ?_
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
Z : Finset (Set α)
⊢ (∀ (u : Set α), u ∈ Z → IsOpen u) → (∀ (u : Set α), u ∈ Z → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑Z) ↔
(∀ (z : Set α),
z ∈ ↑(Equiv.finsetCongr (Function.Involutive.toPerm compl (_ : Function.Involutive compl))) Z → IsClosed z) →
s ⊆ ⋃₀ ↑(↑(Equiv.finsetCongr (Function.Involutive.toPerm compl (_ : Function.Involutive compl))) Z) →
∃ z, z ∈ ↑(Equiv.finsetCongr (Function.Involutive.toPerm compl (_ : Function.Involutive compl))) Z ∧ s ⊆ z
[PROOFSTEP]
simp_rw [Equiv.finsetCongr_apply, Finset.forall_mem_map, Finset.mem_map, Finset.coe_map, sUnion_image,
Equiv.coe_toEmbedding, Function.Involutive.coe_toPerm, isClosed_compl_iff, exists_exists_and_eq_and]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
Z : Finset (Set α)
⊢ (∀ (u : Set α), u ∈ Z → IsOpen u) → (∀ (u : Set α), u ∈ Z → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑Z) ↔
(∀ (u : Set α), u ∈ Z → IsOpen u) → s ⊆ ⋃ (x : Set α) (_ : x ∈ ↑Z), xᶜ → ∃ a, a ∈ Z ∧ s ⊆ aᶜ
[PROOFSTEP]
refine forall_congr' fun _ => Iff.trans ?_ not_imp_not
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s✝ t s : Set α
Z : Finset (Set α)
x✝ : ∀ (u : Set α), u ∈ Z → IsOpen u
⊢ (∀ (u : Set α), u ∈ Z → Set.Nonempty (s ∩ u)) → Set.Nonempty (s ∩ ⋂₀ ↑Z) ↔
(¬∃ a, a ∈ Z ∧ s ⊆ aᶜ) → ¬s ⊆ ⋃ (x : Set α) (_ : x ∈ ↑Z), xᶜ
[PROOFSTEP]
simp only [not_exists, not_and, ← compl_iInter₂, ← sInter_eq_biInter, subset_compl_iff_disjoint_right,
not_disjoint_iff_nonempty_inter]
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U : Set α
hS : IsPreirreducible S
hU : IsOpen U
h : Set.Nonempty (S ∩ U)
⊢ S ⊆ closure (S ∩ U)
[PROOFSTEP]
by_contra h'
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U : Set α
hS : IsPreirreducible S
hU : IsOpen U
h : Set.Nonempty (S ∩ U)
h' : ¬S ⊆ closure (S ∩ U)
⊢ False
[PROOFSTEP]
obtain ⟨x, h₁, h₂, h₃⟩ := hS _ (closure (S ∩ U))ᶜ hU isClosed_closure.isOpen_compl h (inter_compl_nonempty_iff.mpr h')
[GOAL]
case intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U : Set α
hS : IsPreirreducible S
hU : IsOpen U
h : Set.Nonempty (S ∩ U)
h' : ¬S ⊆ closure (S ∩ U)
x : α
h₁ : x ∈ S
h₂ : x ∈ U
h₃ : x ∈ (closure (S ∩ U))ᶜ
⊢ False
[PROOFSTEP]
exact h₃ (subset_closure ⟨h₁, h₂⟩)
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hZ : IsPreirreducible Z
hU : Set.Nonempty U
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
⊢ IsIrreducible S
[PROOFSTEP]
obtain ⟨z, hz⟩ := hU
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hZ : IsPreirreducible Z
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
⊢ IsIrreducible S
[PROOFSTEP]
replace hZ : IsIrreducible Z := ⟨⟨z, h₂ (h₁ hz)⟩, hZ⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
⊢ IsIrreducible S
[PROOFSTEP]
refine' ⟨⟨z, h₁ hz⟩, _⟩
[GOAL]
case intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
⊢ IsPreirreducible S
[PROOFSTEP]
rintro u v hu hv ⟨x, hx, hx'⟩ ⟨y, hy, hy'⟩
[GOAL]
case intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
⊢ Set.Nonempty (S ∩ (u ∩ v))
[PROOFSTEP]
obtain ⟨a, -, ha'⟩ : Set.Nonempty (Z ∩ ⋂₀ ↑({ U, u, v } : Finset (Set α)))
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
⊢ Set.Nonempty (Z ∩ ⋂₀ ↑{U, u, v})
[PROOFSTEP]
refine isIrreducible_iff_sInter.mp hZ { U, u, v } ?_ ?_
[GOAL]
case refine_1
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
⊢ ∀ (u_1 : Set α), u_1 ∈ {U, u, v} → IsOpen u_1
[PROOFSTEP]
simp [*]
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
⊢ ∀ (u_1 : Set α), u_1 ∈ {U, u, v} → Set.Nonempty (Z ∩ u_1)
[PROOFSTEP]
intro U H
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U✝ Z : Set α
hU' : IsOpen U✝
h₁ : U✝ ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U✝
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
U : Set α
H : U ∈ {U✝, u, v}
⊢ Set.Nonempty (Z ∩ U)
[PROOFSTEP]
simp only [Finset.mem_insert, Finset.mem_singleton] at H
[GOAL]
case refine_2
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U✝ Z : Set α
hU' : IsOpen U✝
h₁ : U✝ ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U✝
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
U : Set α
H : U = U✝ ∨ U = u ∨ U = v
⊢ Set.Nonempty (Z ∩ U)
[PROOFSTEP]
rcases H with (rfl | rfl | rfl)
[GOAL]
case refine_2.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S Z : Set α
h₂ : S ⊆ Z
z : α
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
U : Set α
hU' : IsOpen U
h₁ : U ⊆ S
hz : z ∈ U
⊢ Set.Nonempty (Z ∩ U)
case refine_2.inr.inl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U✝ Z : Set α
hU' : IsOpen U✝
h₁ : U✝ ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U✝
hZ : IsIrreducible Z
v : Set α
hv : IsOpen v
x : α
hx : x ∈ S
y : α
hy : y ∈ S
hy' : y ∈ v
U : Set α
hu : IsOpen U
hx' : x ∈ U
⊢ Set.Nonempty (Z ∩ U)
case refine_2.inr.inr
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U✝ Z : Set α
hU' : IsOpen U✝
h₁ : U✝ ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U✝
hZ : IsIrreducible Z
u : Set α
hu : IsOpen u
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
U : Set α
hv : IsOpen U
hy' : y ∈ U
⊢ Set.Nonempty (Z ∩ U)
[PROOFSTEP]
exacts [⟨z, h₂ (h₁ hz), hz⟩, ⟨x, h₂ hx, hx'⟩, ⟨y, h₂ hy, hy'⟩]
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
a : α
ha' : a ∈ ⋂₀ ↑{U, u, v}
⊢ Set.Nonempty (S ∩ (u ∩ v))
[PROOFSTEP]
replace ha' : a ∈ U ∧ a ∈ u ∧ a ∈ v := by simpa using ha'
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
a : α
ha' : a ∈ ⋂₀ ↑{U, u, v}
⊢ a ∈ U ∧ a ∈ u ∧ a ∈ v
[PROOFSTEP]
simpa using ha'
[GOAL]
case intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t S U Z : Set α
hU' : IsOpen U
h₁ : U ⊆ S
h₂ : S ⊆ Z
z : α
hz : z ∈ U
hZ : IsIrreducible Z
u v : Set α
hu : IsOpen u
hv : IsOpen v
x : α
hx : x ∈ S
hx' : x ∈ u
y : α
hy : y ∈ S
hy' : y ∈ v
a : α
ha' : a ∈ U ∧ a ∈ u ∧ a ∈ v
⊢ Set.Nonempty (S ∩ (u ∩ v))
[PROOFSTEP]
exact ⟨a, h₁ ha'.1, ha'.2⟩
[GOAL]
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z : Set α
hZ : IsPreirreducible Z
f : β → α
hf : OpenEmbedding f
⊢ IsPreirreducible (f ⁻¹' Z)
[PROOFSTEP]
rintro U V hU hV ⟨x, hx, hx'⟩ ⟨y, hy, hy'⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z : Set α
hZ : IsPreirreducible Z
f : β → α
hf : OpenEmbedding f
U V : Set β
hU : IsOpen U
hV : IsOpen V
x : β
hx : x ∈ f ⁻¹' Z
hx' : x ∈ U
y : β
hy : y ∈ f ⁻¹' Z
hy' : y ∈ V
⊢ Set.Nonempty (f ⁻¹' Z ∩ (U ∩ V))
[PROOFSTEP]
obtain ⟨_, h₁, ⟨z, h₂, rfl⟩, ⟨z', h₃, h₄⟩⟩ :=
hZ _ _ (hf.isOpenMap _ hU) (hf.isOpenMap _ hV) ⟨f x, hx, Set.mem_image_of_mem f hx'⟩
⟨f y, hy, Set.mem_image_of_mem f hy'⟩
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z : Set α
hZ : IsPreirreducible Z
f : β → α
hf : OpenEmbedding f
U V : Set β
hU : IsOpen U
hV : IsOpen V
x : β
hx : x ∈ f ⁻¹' Z
hx' : x ∈ U
y : β
hy : y ∈ f ⁻¹' Z
hy' : y ∈ V
z : β
h₂ : z ∈ U
h₁ : f z ∈ Z
z' : β
h₃ : z' ∈ V
h₄ : f z' = f z
⊢ Set.Nonempty (f ⁻¹' Z ∩ (U ∩ V))
[PROOFSTEP]
cases hf.inj h₄
[GOAL]
case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.intro.refl
α : Type u
β : Type v
ι : Type u_1
π : ι → Type u_2
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s t Z : Set α
hZ : IsPreirreducible Z
f : β → α
hf : OpenEmbedding f
U V : Set β
hU : IsOpen U
hV : IsOpen V
x : β
hx : x ∈ f ⁻¹' Z
hx' : x ∈ U
y : β
hy : y ∈ f ⁻¹' Z
hy' : y ∈ V
z : β
h₂ : z ∈ U
h₁ : f z ∈ Z
h₃ : z ∈ V
h₄ : f z = f z
⊢ Set.Nonempty (f ⁻¹' Z ∩ (U ∩ V))
[PROOFSTEP]
exact ⟨z, h₁, h₂, h₃⟩
| {"mathlib_filename": "Mathlib.Topology.SubsetProperties", "llama_tokens": 116943} |
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ IsTopologicalBasis (insert ∅ s)
[PROOFSTEP]
refine' ⟨_, by rw [sUnion_insert, empty_union, h.sUnion_eq], _⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ ⋃₀ insert ∅ s = univ
[PROOFSTEP]
rw [sUnion_insert, empty_union, h.sUnion_eq]
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ ∀ (t₁ : Set α),
t₁ ∈ insert ∅ s →
∀ (t₂ : Set α), t₂ ∈ insert ∅ s → ∀ (x : α), x ∈ t₁ ∩ t₂ → ∃ t₃, t₃ ∈ insert ∅ s ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
rintro t₁ (rfl | h₁) t₂ (rfl | h₂) x ⟨hx₁, hx₂⟩
[GOAL]
case refine'_1.inl.inl.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
x : α
hx₁ hx₂ : x ∈ ∅
⊢ ∃ t₃, t₃ ∈ insert ∅ s ∧ x ∈ t₃ ∧ t₃ ⊆ ∅ ∩ ∅
[PROOFSTEP]
cases hx₁
[GOAL]
case refine'_1.inl.inr.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t₂ : Set α
h₂ : t₂ ∈ s
x : α
hx₁ : x ∈ ∅
hx₂ : x ∈ t₂
⊢ ∃ t₃, t₃ ∈ insert ∅ s ∧ x ∈ t₃ ∧ t₃ ⊆ ∅ ∩ t₂
[PROOFSTEP]
cases hx₁
[GOAL]
case refine'_1.inr.inl.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t₁ : Set α
h₁ : t₁ ∈ s
x : α
hx₁ : x ∈ t₁
hx₂ : x ∈ ∅
⊢ ∃ t₃, t₃ ∈ insert ∅ s ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ ∅
[PROOFSTEP]
cases hx₂
[GOAL]
case refine'_1.inr.inr.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t₁ : Set α
h₁ : t₁ ∈ s
t₂ : Set α
h₂ : t₂ ∈ s
x : α
hx₁ : x ∈ t₁
hx₂ : x ∈ t₂
⊢ ∃ t₃, t₃ ∈ insert ∅ s ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
obtain ⟨t₃, h₃, hs⟩ := h.exists_subset_inter _ h₁ _ h₂ x ⟨hx₁, hx₂⟩
[GOAL]
case refine'_1.inr.inr.intro.intro.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t₁ : Set α
h₁ : t₁ ∈ s
t₂ : Set α
h₂ : t₂ ∈ s
x : α
hx₁ : x ∈ t₁
hx₂ : x ∈ t₂
t₃ : Set α
h₃ : t₃ ∈ s
hs : x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
⊢ ∃ t₃, t₃ ∈ insert ∅ s ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
exact ⟨t₃, .inr h₃, hs⟩
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ t = generateFrom (insert ∅ s)
[PROOFSTEP]
rw [h.eq_generateFrom]
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ generateFrom s = generateFrom (insert ∅ s)
[PROOFSTEP]
refine' le_antisymm (le_generateFrom fun t => _) (generateFrom_anti <| subset_insert ∅ s)
[GOAL]
case refine'_2
α : Type u
t✝ : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t : Set α
⊢ t ∈ insert ∅ s → IsOpen t
[PROOFSTEP]
rintro (rfl | ht)
[GOAL]
case refine'_2.inl
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ IsOpen ∅
[PROOFSTEP]
exact @isOpen_empty _ (generateFrom s)
[GOAL]
case refine'_2.inr
α : Type u
t✝ : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t : Set α
ht : t ∈ s
⊢ IsOpen t
[PROOFSTEP]
exact .basic t ht
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ IsTopologicalBasis (s \ {∅})
[PROOFSTEP]
refine' ⟨_, by rw [sUnion_diff_singleton_empty, h.sUnion_eq], _⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ ⋃₀ (s \ {∅}) = univ
[PROOFSTEP]
rw [sUnion_diff_singleton_empty, h.sUnion_eq]
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ ∀ (t₁ : Set α),
t₁ ∈ s \ {∅} → ∀ (t₂ : Set α), t₂ ∈ s \ {∅} → ∀ (x : α), x ∈ t₁ ∩ t₂ → ∃ t₃, t₃ ∈ s \ {∅} ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
rintro t₁ ⟨h₁, -⟩ t₂ ⟨h₂, -⟩ x hx
[GOAL]
case refine'_1.intro.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t₁ : Set α
h₁ : t₁ ∈ s
t₂ : Set α
h₂ : t₂ ∈ s
x : α
hx : x ∈ t₁ ∩ t₂
⊢ ∃ t₃, t₃ ∈ s \ {∅} ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
obtain ⟨t₃, h₃, hs⟩ := h.exists_subset_inter _ h₁ _ h₂ x hx
[GOAL]
case refine'_1.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t₁ : Set α
h₁ : t₁ ∈ s
t₂ : Set α
h₂ : t₂ ∈ s
x : α
hx : x ∈ t₁ ∩ t₂
t₃ : Set α
h₃ : t₃ ∈ s
hs : x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
⊢ ∃ t₃, t₃ ∈ s \ {∅} ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
exact ⟨t₃, ⟨h₃, Nonempty.ne_empty ⟨x, hs.1⟩⟩, hs⟩
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ t = generateFrom (s \ {∅})
[PROOFSTEP]
rw [h.eq_generateFrom]
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
⊢ generateFrom s = generateFrom (s \ {∅})
[PROOFSTEP]
refine' le_antisymm (generateFrom_anti <| diff_subset s _) (le_generateFrom fun t ht => _)
[GOAL]
case refine'_2
α : Type u
t✝ : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t : Set α
ht : t ∈ s
⊢ IsOpen t
[PROOFSTEP]
obtain rfl | he := eq_or_ne t ∅
[GOAL]
case refine'_2.inl
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
ht : ∅ ∈ s
⊢ IsOpen ∅
[PROOFSTEP]
exact @isOpen_empty _ (generateFrom _)
[GOAL]
case refine'_2.inr
α : Type u
t✝ : TopologicalSpace α
s : Set (Set α)
h : IsTopologicalBasis s
t : Set α
ht : t ∈ s
he : t ≠ ∅
⊢ IsOpen t
[PROOFSTEP]
exact .basic t ⟨ht, he⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set (Set α)
hs : t = generateFrom s
⊢ IsTopologicalBasis ((fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s})
[PROOFSTEP]
subst t
[GOAL]
α : Type u
s : Set (Set α)
⊢ IsTopologicalBasis ((fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s})
[PROOFSTEP]
letI := generateFrom s
[GOAL]
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
⊢ IsTopologicalBasis ((fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s})
[PROOFSTEP]
refine' ⟨_, _, le_antisymm (le_generateFrom _) <| generateFrom_anti fun t ht => _⟩
[GOAL]
case refine'_1
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
⊢ ∀ (t₁ : Set α),
t₁ ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s} →
∀ (t₂ : Set α),
t₂ ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s} →
∀ (x : α), x ∈ t₁ ∩ t₂ → ∃ t₃, t₃ ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s} ∧ x ∈ t₃ ∧ t₃ ⊆ t₁ ∩ t₂
[PROOFSTEP]
rintro _ ⟨t₁, ⟨hft₁, ht₁b⟩, rfl⟩ _ ⟨t₂, ⟨hft₂, ht₂b⟩, rfl⟩ x h
[GOAL]
case refine'_1.intro.intro.intro.intro.intro.intro
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
t₁ : Set (Set α)
hft₁ : Set.Finite t₁
ht₁b : t₁ ⊆ s
t₂ : Set (Set α)
hft₂ : Set.Finite t₂
ht₂b : t₂ ⊆ s
x : α
h : x ∈ (fun f => ⋂₀ f) t₁ ∩ (fun f => ⋂₀ f) t₂
⊢ ∃ t₃, t₃ ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s} ∧ x ∈ t₃ ∧ t₃ ⊆ (fun f => ⋂₀ f) t₁ ∩ (fun f => ⋂₀ f) t₂
[PROOFSTEP]
exact ⟨_, ⟨_, ⟨hft₁.union hft₂, union_subset ht₁b ht₂b⟩, sInter_union t₁ t₂⟩, h, Subset.rfl⟩
[GOAL]
case refine'_2
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
⊢ ⋃₀ ((fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s}) = univ
[PROOFSTEP]
rw [sUnion_image, iUnion₂_eq_univ_iff]
[GOAL]
case refine'_2
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
⊢ ∀ (a : α), ∃ i j, a ∈ ⋂₀ i
[PROOFSTEP]
exact fun x => ⟨∅, ⟨finite_empty, empty_subset _⟩, sInter_empty.substr <| mem_univ x⟩
[GOAL]
case refine'_3
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
⊢ ∀ (s_1 : Set α), s_1 ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s} → IsOpen s_1
[PROOFSTEP]
rintro _ ⟨t, ⟨hft, htb⟩, rfl⟩
[GOAL]
case refine'_3.intro.intro.intro
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
t : Set (Set α)
hft : Set.Finite t
htb : t ⊆ s
⊢ IsOpen ((fun f => ⋂₀ f) t)
[PROOFSTEP]
apply isOpen_sInter
[GOAL]
case refine'_3.intro.intro.intro.hs
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
t : Set (Set α)
hft : Set.Finite t
htb : t ⊆ s
⊢ Set.Finite t
case refine'_3.intro.intro.intro.a
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
t : Set (Set α)
hft : Set.Finite t
htb : t ⊆ s
⊢ ∀ (t_1 : Set α), t_1 ∈ t → IsOpen t_1
[PROOFSTEP]
exacts [hft, fun s hs => GenerateOpen.basic _ <| htb hs]
[GOAL]
case refine'_4
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
t : Set α
ht : t ∈ s
⊢ t ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s}
[PROOFSTEP]
rw [← sInter_singleton t]
[GOAL]
case refine'_4
α : Type u
s : Set (Set α)
this : TopologicalSpace α := generateFrom s
t : Set α
ht : t ∈ s
⊢ ⋂₀ {t} ∈ (fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ s}
[PROOFSTEP]
exact ⟨{ t }, ⟨finite_singleton t, singleton_subset_iff.2 ht⟩, rfl⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
⊢ IsTopologicalBasis s
[PROOFSTEP]
refine' ⟨fun t₁ ht₁ t₂ ht₂ x hx => h_nhds _ _ hx (IsOpen.inter (h_open _ ht₁) (h_open _ ht₂)), _, _⟩
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
⊢ ⋃₀ s = univ
[PROOFSTEP]
refine' sUnion_eq_univ_iff.2 fun a => _
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
a : α
⊢ ∃ b, b ∈ s ∧ a ∈ b
[PROOFSTEP]
rcases h_nhds a univ trivial isOpen_univ with ⟨u, h₁, h₂, -⟩
[GOAL]
case refine'_1.intro.intro.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
a : α
u : Set α
h₁ : u ∈ s
h₂ : a ∈ u
⊢ ∃ b, b ∈ s ∧ a ∈ b
[PROOFSTEP]
exact ⟨u, h₁, h₂⟩
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
⊢ t = generateFrom s
[PROOFSTEP]
refine' (le_generateFrom h_open).antisymm fun u hu => _
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
u : Set α
hu : IsOpen u
⊢ IsOpen u
[PROOFSTEP]
refine' (@isOpen_iff_nhds α (generateFrom s) u).mpr fun a ha => _
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
u : Set α
hu : IsOpen u
a : α
ha : a ∈ u
⊢ 𝓝 a ≤ 𝓟 u
[PROOFSTEP]
rcases h_nhds a u ha hu with ⟨v, hvs, hav, hvu⟩
[GOAL]
case refine'_2.intro.intro.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
u : Set α
hu : IsOpen u
a : α
ha : a ∈ u
v : Set α
hvs : v ∈ s
hav : a ∈ v
hvu : v ⊆ u
⊢ 𝓝 a ≤ 𝓟 u
[PROOFSTEP]
rw [nhds_generateFrom]
[GOAL]
case refine'_2.intro.intro.intro
α : Type u
t : TopologicalSpace α
s : Set (Set α)
h_open : ∀ (u : Set α), u ∈ s → IsOpen u
h_nhds : ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ s ∧ a ∈ v ∧ v ⊆ u
u : Set α
hu : IsOpen u
a : α
ha : a ∈ u
v : Set α
hvs : v ∈ s
hav : a ∈ v
hvu : v ⊆ u
⊢ ⨅ (s_1 : Set α) (_ : s_1 ∈ {s_2 | a ∈ s_2 ∧ s_2 ∈ s}), 𝓟 s_1 ≤ 𝓟 u
[PROOFSTEP]
exact iInf₂_le_of_le v ⟨hav, hvs⟩ (le_principal_iff.2 hvu)
[GOAL]
α : Type u
t : TopologicalSpace α
a : α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
⊢ s ∈ 𝓝 a ↔ ∃ t, t ∈ b ∧ a ∈ t ∧ t ⊆ s
[PROOFSTEP]
change s ∈ (𝓝 a).sets ↔ ∃ t ∈ b, a ∈ t ∧ t ⊆ s
[GOAL]
α : Type u
t : TopologicalSpace α
a : α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
⊢ s ∈ (𝓝 a).sets ↔ ∃ t, t ∈ b ∧ a ∈ t ∧ t ⊆ s
[PROOFSTEP]
rw [hb.eq_generateFrom, nhds_generateFrom, biInf_sets_eq]
[GOAL]
α : Type u
t : TopologicalSpace α
a : α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
⊢ s ∈ ⋃ (i : Set α) (_ : i ∈ {s | a ∈ s ∧ s ∈ b}), (𝓟 i).sets ↔ ∃ t, t ∈ b ∧ a ∈ t ∧ t ⊆ s
[PROOFSTEP]
simp [and_assoc, and_left_comm]
[GOAL]
case h
α : Type u
t : TopologicalSpace α
a : α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
⊢ DirectedOn ((fun s => 𝓟 s) ⁻¹'o fun x x_1 => x ≥ x_1) {s | a ∈ s ∧ s ∈ b}
[PROOFSTEP]
rintro s ⟨hs₁, hs₂⟩ t ⟨ht₁, ht₂⟩
[GOAL]
case h.intro.intro
α : Type u
t✝ : TopologicalSpace α
a : α
s✝ : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
s : Set α
hs₁ : a ∈ s
hs₂ : s ∈ b
t : Set α
ht₁ : a ∈ t
ht₂ : t ∈ b
⊢ ∃ z,
z ∈ {s | a ∈ s ∧ s ∈ b} ∧
((fun s => 𝓟 s) ⁻¹'o fun x x_1 => x ≥ x_1) s z ∧ ((fun s => 𝓟 s) ⁻¹'o fun x x_1 => x ≥ x_1) t z
[PROOFSTEP]
let ⟨u, hu₁, hu₂, hu₃⟩ := hb.1 _ hs₂ _ ht₂ _ ⟨hs₁, ht₁⟩
[GOAL]
case h.intro.intro
α : Type u
t✝ : TopologicalSpace α
a : α
s✝ : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
s : Set α
hs₁ : a ∈ s
hs₂ : s ∈ b
t : Set α
ht₁ : a ∈ t
ht₂ : t ∈ b
u : Set α
hu₁ : u ∈ b
hu₂ : a ∈ u
hu₃ : u ⊆ s ∩ t
⊢ ∃ z,
z ∈ {s | a ∈ s ∧ s ∈ b} ∧
((fun s => 𝓟 s) ⁻¹'o fun x x_1 => x ≥ x_1) s z ∧ ((fun s => 𝓟 s) ⁻¹'o fun x x_1 => x ≥ x_1) t z
[PROOFSTEP]
exact
⟨u, ⟨hu₂, hu₁⟩, le_principal_iff.2 (hu₃.trans (inter_subset_left _ _)),
le_principal_iff.2 (hu₃.trans (inter_subset_right _ _))⟩
[GOAL]
case ne
α : Type u
t : TopologicalSpace α
a : α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
⊢ Set.Nonempty {s | a ∈ s ∧ s ∈ b}
[PROOFSTEP]
rcases eq_univ_iff_forall.1 hb.sUnion_eq a with ⟨i, h1, h2⟩
[GOAL]
case ne.intro.intro
α : Type u
t : TopologicalSpace α
a : α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
i : Set α
h1 : i ∈ b
h2 : a ∈ i
⊢ Set.Nonempty {s | a ∈ s ∧ s ∈ b}
[PROOFSTEP]
exact ⟨i, h2, h1⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
⊢ IsOpen s ↔ ∀ (a : α), a ∈ s → ∃ t, t ∈ b ∧ a ∈ t ∧ t ⊆ s
[PROOFSTEP]
simp [isOpen_iff_mem_nhds, hb.mem_nhds_iff]
[GOAL]
α : Type u
t : TopologicalSpace α
b : Set (Set α)
hb : IsTopologicalBasis b
a : α
s : Set α
⊢ (∃ t, t ∈ b ∧ a ∈ t ∧ t ⊆ s) ↔ ∃ i, (i ∈ b ∧ a ∈ i) ∧ i ⊆ s
[PROOFSTEP]
simp only [and_assoc]
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
hs : s ∈ b
⊢ IsOpen s
[PROOFSTEP]
rw [hb.eq_generateFrom]
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set α
b : Set (Set α)
hb : IsTopologicalBasis b
hs : s ∈ b
⊢ IsOpen s
[PROOFSTEP]
exact .basic s hs
[GOAL]
α : Type u
t : TopologicalSpace α
B : Set (Set α)
hB : IsTopologicalBasis B
u : Set α
ou : IsOpen u
⊢ u = ⋃ (i : ↑{s | s ∈ B ∧ s ⊆ u}), ↑i
[PROOFSTEP]
rw [← sUnion_eq_iUnion]
[GOAL]
α : Type u
t : TopologicalSpace α
B : Set (Set α)
hB : IsTopologicalBasis B
u : Set α
ou : IsOpen u
⊢ u = ⋃₀ {s | s ∈ B ∧ s ⊆ u}
[PROOFSTEP]
apply hB.open_eq_sUnion' ou
[GOAL]
α : Type u
t : TopologicalSpace α
b : Set (Set α)
hb : IsTopologicalBasis b
s : Set α
a : α
⊢ (∀ (i : Set α), i ∈ b ∧ a ∈ i → Set.Nonempty (i ∩ s)) ↔ ∀ (o : Set α), o ∈ b → a ∈ o → Set.Nonempty (o ∩ s)
[PROOFSTEP]
simp only [and_imp]
[GOAL]
α : Type u
t : TopologicalSpace α
b : Set (Set α)
hb : IsTopologicalBasis b
s : Set α
⊢ Dense s ↔ ∀ (o : Set α), o ∈ b → Set.Nonempty o → Set.Nonempty (o ∩ s)
[PROOFSTEP]
simp only [Dense, hb.mem_closure_iff]
[GOAL]
α : Type u
t : TopologicalSpace α
b : Set (Set α)
hb : IsTopologicalBasis b
s : Set α
⊢ (∀ (x : α) (o : Set α), o ∈ b → x ∈ o → Set.Nonempty (o ∩ s)) ↔
∀ (o : Set α), o ∈ b → Set.Nonempty o → Set.Nonempty (o ∩ s)
[PROOFSTEP]
exact ⟨fun h o hb ⟨a, ha⟩ => h a o hb ha, fun h a o hb ha => h o hb ⟨a, ha⟩⟩
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B : Set (Set α)
hB : IsTopologicalBasis B
f : α → β
⊢ IsOpenMap f ↔ ∀ (s : Set α), s ∈ B → IsOpen (f '' s)
[PROOFSTEP]
refine' ⟨fun H o ho => H _ (hB.isOpen ho), fun hf o ho => _⟩
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B : Set (Set α)
hB : IsTopologicalBasis B
f : α → β
hf : ∀ (s : Set α), s ∈ B → IsOpen (f '' s)
o : Set α
ho : IsOpen o
⊢ IsOpen (f '' o)
[PROOFSTEP]
rw [hB.open_eq_sUnion' ho, sUnion_eq_iUnion, image_iUnion]
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B : Set (Set α)
hB : IsTopologicalBasis B
f : α → β
hf : ∀ (s : Set α), s ∈ B → IsOpen (f '' s)
o : Set α
ho : IsOpen o
⊢ IsOpen (⋃ (i : ↑{s | s ∈ B ∧ s ⊆ o}), f '' ↑i)
[PROOFSTEP]
exact isOpen_iUnion fun s => hf s s.2.1
[GOAL]
α : Type u
t : TopologicalSpace α
⊢ ∀ (u : Set α), u ∈ {U | IsOpen U} → IsOpen u
[PROOFSTEP]
tauto
[GOAL]
α : Type u
t : TopologicalSpace α
⊢ ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ {U | IsOpen U} ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
tauto
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B₁ : Set (Set α)
B₂ : Set (Set β)
h₁ : IsTopologicalBasis B₁
h₂ : IsTopologicalBasis B₂
⊢ IsTopologicalBasis (image2 (fun x x_1 => x ×ˢ x_1) B₁ B₂)
[PROOFSTEP]
refine' isTopologicalBasis_of_open_of_nhds _ _
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B₁ : Set (Set α)
B₂ : Set (Set β)
h₁ : IsTopologicalBasis B₁
h₂ : IsTopologicalBasis B₂
⊢ ∀ (u : Set (α × β)), u ∈ image2 (fun x x_1 => x ×ˢ x_1) B₁ B₂ → IsOpen u
[PROOFSTEP]
rintro _ ⟨u₁, u₂, hu₁, hu₂, rfl⟩
[GOAL]
case refine'_1.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B₁ : Set (Set α)
B₂ : Set (Set β)
h₁ : IsTopologicalBasis B₁
h₂ : IsTopologicalBasis B₂
u₁ : Set α
u₂ : Set β
hu₁ : u₁ ∈ B₁
hu₂ : u₂ ∈ B₂
⊢ IsOpen ((fun x x_1 => x ×ˢ x_1) u₁ u₂)
[PROOFSTEP]
exact (h₁.isOpen hu₁).prod (h₂.isOpen hu₂)
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B₁ : Set (Set α)
B₂ : Set (Set β)
h₁ : IsTopologicalBasis B₁
h₂ : IsTopologicalBasis B₂
⊢ ∀ (a : α × β) (u : Set (α × β)), a ∈ u → IsOpen u → ∃ v, v ∈ image2 (fun x x_1 => x ×ˢ x_1) B₁ B₂ ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
rintro ⟨a, b⟩ u hu uo
[GOAL]
case refine'_2.mk
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B₁ : Set (Set α)
B₂ : Set (Set β)
h₁ : IsTopologicalBasis B₁
h₂ : IsTopologicalBasis B₂
a : α
b : β
u : Set (α × β)
hu : (a, b) ∈ u
uo : IsOpen u
⊢ ∃ v, v ∈ image2 (fun x x_1 => x ×ˢ x_1) B₁ B₂ ∧ (a, b) ∈ v ∧ v ⊆ u
[PROOFSTEP]
rcases(h₁.nhds_hasBasis.prod_nhds h₂.nhds_hasBasis).mem_iff.1 (IsOpen.mem_nhds uo hu) with
⟨⟨s, t⟩, ⟨⟨hs, ha⟩, ht, hb⟩, hu⟩
[GOAL]
case refine'_2.mk.intro.mk.intro.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B₁ : Set (Set α)
B₂ : Set (Set β)
h₁ : IsTopologicalBasis B₁
h₂ : IsTopologicalBasis B₂
a : α
b : β
u : Set (α × β)
hu✝ : (a, b) ∈ u
uo : IsOpen u
s : Set α
t : Set β
hu : (s, t).fst ×ˢ (s, t).snd ⊆ u
hs : (s, t).fst ∈ B₁
ha : a ∈ (s, t).fst
ht : (s, t).snd ∈ B₂
hb : b ∈ (s, t).snd
⊢ ∃ v, v ∈ image2 (fun x x_1 => x ×ˢ x_1) B₁ B₂ ∧ (a, b) ∈ v ∧ v ⊆ u
[PROOFSTEP]
exact ⟨s ×ˢ t, mem_image2_of_mem hs ht, ⟨ha, hb⟩, hu⟩
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
⊢ IsTopologicalBasis (preimage f '' T)
[PROOFSTEP]
refine' isTopologicalBasis_of_open_of_nhds _ _
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
⊢ ∀ (u : Set α), u ∈ preimage f '' T → IsOpen u
[PROOFSTEP]
rintro _ ⟨V, hV, rfl⟩
[GOAL]
case refine'_1.intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
V : Set β
hV : V ∈ T
⊢ IsOpen (f ⁻¹' V)
[PROOFSTEP]
rw [hf.isOpen_iff]
[GOAL]
case refine'_1.intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
V : Set β
hV : V ∈ T
⊢ ∃ t, IsOpen t ∧ f ⁻¹' t = f ⁻¹' V
[PROOFSTEP]
refine' ⟨V, h.isOpen hV, rfl⟩
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
⊢ ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ preimage f '' T ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
intro a U ha hU
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
a : α
U : Set α
ha : a ∈ U
hU : IsOpen U
⊢ ∃ v, v ∈ preimage f '' T ∧ a ∈ v ∧ v ⊆ U
[PROOFSTEP]
rw [hf.isOpen_iff] at hU
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
a : α
U : Set α
ha : a ∈ U
hU : ∃ t, IsOpen t ∧ f ⁻¹' t = U
⊢ ∃ v, v ∈ preimage f '' T ∧ a ∈ v ∧ v ⊆ U
[PROOFSTEP]
obtain ⟨V, hV, rfl⟩ := hU
[GOAL]
case refine'_2.intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
a : α
V : Set β
hV : IsOpen V
ha : a ∈ f ⁻¹' V
⊢ ∃ v, v ∈ preimage f '' T ∧ a ∈ v ∧ v ⊆ f ⁻¹' V
[PROOFSTEP]
obtain ⟨S, hS, rfl⟩ := h.open_eq_sUnion hV
[GOAL]
case refine'_2.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
a : α
S : Set (Set β)
hS : S ⊆ T
hV : IsOpen (⋃₀ S)
ha : a ∈ f ⁻¹' ⋃₀ S
⊢ ∃ v, v ∈ preimage f '' T ∧ a ∈ v ∧ v ⊆ f ⁻¹' ⋃₀ S
[PROOFSTEP]
obtain ⟨W, hW, ha⟩ := ha
[GOAL]
case refine'_2.intro.intro.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
f : α → β
T : Set (Set β)
hf : Inducing f
h : IsTopologicalBasis T
a : α
S : Set (Set β)
hS : S ⊆ T
hV : IsOpen (⋃₀ S)
W : Set β
hW : W ∈ S
ha : f a ∈ W
⊢ ∃ v, v ∈ preimage f '' T ∧ a ∈ v ∧ v ⊆ f ⁻¹' ⋃₀ S
[PROOFSTEP]
refine' ⟨f ⁻¹' W, ⟨_, hS hW, rfl⟩, ha, Set.preimage_mono <| Set.subset_sUnion_of_mem hW⟩
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
⊢ IsTopologicalBasis (⋃ (i : ι), image Subtype.val '' b i)
[PROOFSTEP]
refine' isTopologicalBasis_of_open_of_nhds (fun u hu => _) _
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
u : Set α
hu : u ∈ ⋃ (i : ι), image Subtype.val '' b i
⊢ IsOpen u
[PROOFSTEP]
simp only [mem_iUnion, mem_image] at hu
[GOAL]
case refine'_1
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
u : Set α
hu : ∃ i x, x ∈ b i ∧ Subtype.val '' x = u
⊢ IsOpen u
[PROOFSTEP]
rcases hu with ⟨i, s, sb, rfl⟩
[GOAL]
case refine'_1.intro.intro.intro
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
i : ι
s : Set { x // x ∈ U i }
sb : s ∈ b i
⊢ IsOpen (Subtype.val '' s)
[PROOFSTEP]
exact (Uo i).isOpenMap_subtype_val _ ((hb i).isOpen sb)
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
⊢ ∀ (a : α) (u : Set α), a ∈ u → IsOpen u → ∃ v, v ∈ ⋃ (i : ι), image Subtype.val '' b i ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
intro a u ha uo
[GOAL]
case refine'_2
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
a : α
u : Set α
ha : a ∈ u
uo : IsOpen u
⊢ ∃ v, v ∈ ⋃ (i : ι), image Subtype.val '' b i ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
rcases iUnion_eq_univ_iff.1 Uc a with ⟨i, hi⟩
[GOAL]
case refine'_2.intro
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
a : α
u : Set α
ha : a ∈ u
uo : IsOpen u
i : ι
hi : a ∈ U i
⊢ ∃ v, v ∈ ⋃ (i : ι), image Subtype.val '' b i ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
lift a to ↥(U i) using hi
[GOAL]
case refine'_2.intro.intro
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
u : Set α
uo : IsOpen u
i : ι
a : { x // x ∈ U i }
ha : ↑a ∈ u
⊢ ∃ v, v ∈ ⋃ (i : ι), image Subtype.val '' b i ∧ ↑a ∈ v ∧ v ⊆ u
[PROOFSTEP]
rcases(hb i).exists_subset_of_mem_open ha (uo.preimage continuous_subtype_val) with ⟨v, hvb, hav, hvu⟩
[GOAL]
case refine'_2.intro.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
ι : Sort u_1
U : ι → Set α
Uo : ∀ (i : ι), IsOpen (U i)
Uc : ⋃ (i : ι), U i = univ
b : (i : ι) → Set (Set ↑(U i))
hb : ∀ (i : ι), IsTopologicalBasis (b i)
u : Set α
uo : IsOpen u
i : ι
a : { x // x ∈ U i }
ha : ↑a ∈ u
v : Set ↑(U i)
hvb : v ∈ b i
hav : a ∈ v
hvu : v ⊆ Subtype.val ⁻¹' u
⊢ ∃ v, v ∈ ⋃ (i : ι), image Subtype.val '' b i ∧ ↑a ∈ v ∧ v ⊆ u
[PROOFSTEP]
exact ⟨(↑) '' v, mem_iUnion.2 ⟨i, mem_image_of_mem _ hvb⟩, mem_image_of_mem _ hav, image_subset_iff.2 hvu⟩
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B : Set (Set β)
hB : IsTopologicalBasis B
f : α → β
hf : ∀ (s : Set β), s ∈ B → IsOpen (f ⁻¹' s)
⊢ Continuous f
[PROOFSTEP]
rw [hB.eq_generateFrom]
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
B : Set (Set β)
hB : IsTopologicalBasis B
f : α → β
hf : ∀ (s : Set β), s ∈ B → IsOpen (f ⁻¹' s)
⊢ Continuous f
[PROOFSTEP]
exact continuous_generateFrom hf
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝¹ : SeparableSpace α
inst✝ : Nonempty α
⊢ ∃ u, DenseRange u
[PROOFSTEP]
obtain ⟨s : Set α, hs, s_dense⟩ := exists_countable_dense α
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
inst✝¹ : SeparableSpace α
inst✝ : Nonempty α
s : Set α
hs : Set.Countable s
s_dense : Dense s
⊢ ∃ u, DenseRange u
[PROOFSTEP]
cases' Set.countable_iff_exists_subset_range.mp hs with u hu
[GOAL]
case intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝¹ : SeparableSpace α
inst✝ : Nonempty α
s : Set α
hs : Set.Countable s
s_dense : Dense s
u : ℕ → α
hu : s ⊆ range u
⊢ ∃ u, DenseRange u
[PROOFSTEP]
exact ⟨u, s_dense.mono hu⟩
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type ?u.24188
inst✝² : TopologicalSpace β
inst✝¹ : SeparableSpace α
inst✝ : SeparableSpace β
⊢ SeparableSpace (α × β)
[PROOFSTEP]
rcases exists_countable_dense α with ⟨s, hsc, hsd⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
β : Type ?u.24188
inst✝² : TopologicalSpace β
inst✝¹ : SeparableSpace α
inst✝ : SeparableSpace β
s : Set α
hsc : Set.Countable s
hsd : Dense s
⊢ SeparableSpace (α × β)
[PROOFSTEP]
rcases exists_countable_dense β with ⟨t, htc, htd⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type ?u.24188
inst✝² : TopologicalSpace β
inst✝¹ : SeparableSpace α
inst✝ : SeparableSpace β
s : Set α
hsc : Set.Countable s
hsd : Dense s
t : Set β
htc : Set.Countable t
htd : Dense t
⊢ SeparableSpace (α × β)
[PROOFSTEP]
exact ⟨⟨s ×ˢ t, hsc.prod htc, hsd.prod htd⟩⟩
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
choose t htc htd using (exists_countable_dense <| X ·)
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
haveI := fun i ↦ (htc i).to_subtype
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
nontriviality ∀ i, X i
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
inhabit ∀ i, X i
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
classical
set f : (Σ I : Finset ι, ∀ i : I, t i) → ∀ i, X i := fun ⟨I, g⟩ i ↦
if hi : i ∈ I then g ⟨i, hi⟩ else (default : ∀ i, X i) i
refine ⟨⟨range f, countable_range f, dense_iff_inter_open.2 fun U hU ⟨g, hg⟩ ↦ ?_⟩⟩
rcases isOpen_pi_iff.1 hU g hg with ⟨I, u, huo, huU⟩
have : ∀ i : I, ∃ y ∈ t i, y ∈ u i := fun i ↦ (htd i).exists_mem_open (huo i i.2).1 ⟨_, (huo i i.2).2⟩
choose y hyt hyu using this
lift y to ∀ i : I, t i using hyt
refine ⟨f ⟨I, y⟩, huU fun i (hi : i ∈ I) ↦ ?_, mem_range_self _⟩
simp only [dif_pos hi]
exact hyu _
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
set f : (Σ I : Finset ι, ∀ i : I, t i) → ∀ i, X i := fun ⟨I, g⟩ i ↦
if hi : i ∈ I then g ⟨i, hi⟩ else (default : ∀ i, X i) i
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
⊢ SeparableSpace ((i : ι) → X i)
[PROOFSTEP]
refine ⟨⟨range f, countable_range f, dense_iff_inter_open.2 fun U hU ⟨g, hg⟩ ↦ ?_⟩⟩
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
⊢ Set.Nonempty (U ∩ range f)
[PROOFSTEP]
rcases isOpen_pi_iff.1 hU g hg with ⟨I, u, huo, huU⟩
[GOAL]
case intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
I : Finset ι
u : (a : ι) → Set (X a)
huo : ∀ (a : ι), a ∈ I → IsOpen (u a) ∧ g a ∈ u a
huU : Set.pi (↑I) u ⊆ U
⊢ Set.Nonempty (U ∩ range f)
[PROOFSTEP]
have : ∀ i : I, ∃ y ∈ t i, y ∈ u i := fun i ↦ (htd i).exists_mem_open (huo i i.2).1 ⟨_, (huo i i.2).2⟩
[GOAL]
case intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this✝ : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
I : Finset ι
u : (a : ι) → Set (X a)
huo : ∀ (a : ι), a ∈ I → IsOpen (u a) ∧ g a ∈ u a
huU : Set.pi (↑I) u ⊆ U
this : ∀ (i : { x // x ∈ I }), ∃ y, y ∈ t ↑i ∧ y ∈ u ↑i
⊢ Set.Nonempty (U ∩ range f)
[PROOFSTEP]
choose y hyt hyu using this
[GOAL]
case intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
I : Finset ι
u : (a : ι) → Set (X a)
huo : ∀ (a : ι), a ∈ I → IsOpen (u a) ∧ g a ∈ u a
huU : Set.pi (↑I) u ⊆ U
y : (i : { x // x ∈ I }) → X ↑i
hyt : ∀ (i : { x // x ∈ I }), y i ∈ t ↑i
hyu : ∀ (i : { x // x ∈ I }), y i ∈ u ↑i
⊢ Set.Nonempty (U ∩ range f)
[PROOFSTEP]
lift y to ∀ i : I, t i using hyt
[GOAL]
case intro.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
I : Finset ι
u : (a : ι) → Set (X a)
huo : ∀ (a : ι), a ∈ I → IsOpen (u a) ∧ g a ∈ u a
huU : Set.pi (↑I) u ⊆ U
y : (i : { x // x ∈ I }) → ↑(t ↑i)
hyu : ∀ (i : { x // x ∈ I }), (fun i => ↑(y i)) i ∈ u ↑i
⊢ Set.Nonempty (U ∩ range f)
[PROOFSTEP]
refine ⟨f ⟨I, y⟩, huU fun i (hi : i ∈ I) ↦ ?_, mem_range_self _⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
I : Finset ι
u : (a : ι) → Set (X a)
huo : ∀ (a : ι), a ∈ I → IsOpen (u a) ∧ g a ∈ u a
huU : Set.pi (↑I) u ⊆ U
y : (i : { x // x ∈ I }) → ↑(t ↑i)
hyu : ∀ (i : { x // x ∈ I }), (fun i => ↑(y i)) i ∈ u ↑i
i : ι
hi : i ∈ I
⊢ f { fst := I, snd := y } i ∈ u i
[PROOFSTEP]
simp only [dif_pos hi]
[GOAL]
case intro.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
X : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (X i)
inst✝¹ : ∀ (i : ι), SeparableSpace (X i)
inst✝ : Countable ι
t : (x : ι) → Set (X x)
htc : ∀ (x : ι), Set.Countable (t x)
htd : ∀ (x : ι), Dense (t x)
this : ∀ (i : ι), Countable ↑(t i)
✝ : Nontrivial ((i : ι) → X i)
inhabited_h : Inhabited ((i : ι) → X i)
f : (I : Finset ι) × ((i : { x // x ∈ I }) → ↑(t ↑i)) → (i : ι) → X i :=
fun x i =>
match x with
| { fst := I, snd := g } => if hi : i ∈ I then ↑(g { val := i, property := hi }) else default i
U : Set ((i : ι) → X i)
hU : IsOpen U
x✝ : Set.Nonempty U
g : (i : ι) → X i
hg : g ∈ U
I : Finset ι
u : (a : ι) → Set (X a)
huo : ∀ (a : ι), a ∈ I → IsOpen (u a) ∧ g a ∈ u a
huU : Set.pi (↑I) u ⊆ U
y : (i : { x // x ∈ I }) → ↑(t ↑i)
hyu : ∀ (i : { x // x ∈ I }), (fun i => ↑(y i)) i ∈ u ↑i
i : ι
hi : i ∈ I
⊢ ↑(y { val := i, property := (_ : i ∈ I) }) ∈ u i
[PROOFSTEP]
exact hyu _
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : DiscreteTopology α
⊢ SeparableSpace α ↔ Countable α
[PROOFSTEP]
simp [SeparableSpace_iff, countable_univ_iff]
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
⊢ Set.Countable a
[PROOFSTEP]
rcases exists_countable_dense α with ⟨u, ⟨u_encodable⟩, u_dense⟩
[GOAL]
case intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
⊢ Set.Countable a
[PROOFSTEP]
have : ∀ i : a, ∃ y, y ∈ s i ∩ u := fun i => dense_iff_inter_open.1 u_dense (s i) (ha i i.2) (h'a i i.2)
[GOAL]
case intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
this : ∀ (i : ↑a), ∃ y, y ∈ s ↑i ∩ u
⊢ Set.Countable a
[PROOFSTEP]
choose f hfs hfu using this
[GOAL]
case intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
f : ↑a → α
hfs : ∀ (i : ↑a), f i ∈ s ↑i
hfu : ∀ (i : ↑a), f i ∈ u
⊢ Set.Countable a
[PROOFSTEP]
lift f to a → u using hfu
[GOAL]
case intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
f : ↑a → ↑u
hfs : ∀ (i : ↑a), (fun i => ↑(f i)) i ∈ s ↑i
⊢ Set.Countable a
[PROOFSTEP]
have f_inj : Injective f :=
by
refine' injective_iff_pairwise_ne.mpr ((h.subtype _ _).mono fun i j hij hfij => hij.le_bot ⟨hfs i, _⟩)
simp only [congr_arg Subtype.val hfij, hfs j]
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
f : ↑a → ↑u
hfs : ∀ (i : ↑a), (fun i => ↑(f i)) i ∈ s ↑i
⊢ Injective f
[PROOFSTEP]
refine' injective_iff_pairwise_ne.mpr ((h.subtype _ _).mono fun i j hij hfij => hij.le_bot ⟨hfs i, _⟩)
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
f : ↑a → ↑u
hfs : ∀ (i : ↑a), (fun i => ↑(f i)) i ∈ s ↑i
i j : ↑a
hij : (Disjoint on s) ↑i ↑j
hfij : f i = f j
⊢ (fun i => ↑(f i)) i ∈ s ↑j
[PROOFSTEP]
simp only [congr_arg Subtype.val hfij, hfs j]
[GOAL]
case intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SeparableSpace α
ι : Type u_1
s : ι → Set α
a : Set ι
h : PairwiseDisjoint a s
ha : ∀ (i : ι), i ∈ a → IsOpen (s i)
h'a : ∀ (i : ι), i ∈ a → Set.Nonempty (s i)
u : Set α
u_dense : Dense u
u_encodable : Encodable ↑u
f : ↑a → ↑u
hfs : ∀ (i : ↑a), (fun i => ↑(f i)) i ∈ s ↑i
f_inj : Injective f
⊢ Set.Countable a
[PROOFSTEP]
exact ⟨@Encodable.ofInj _ _ u_encodable f f_inj⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s u : Set α
hs : IsSeparable s
hu : u ⊆ s
⊢ IsSeparable u
[PROOFSTEP]
rcases hs with ⟨c, c_count, hs⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
s u : Set α
hu : u ⊆ s
c : Set α
c_count : Set.Countable c
hs : s ⊆ closure c
⊢ IsSeparable u
[PROOFSTEP]
exact ⟨c, c_count, hu.trans hs⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s u : Set α
hs : IsSeparable s
hu : IsSeparable u
⊢ IsSeparable (s ∪ u)
[PROOFSTEP]
rcases hs with ⟨cs, cs_count, hcs⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
s u : Set α
hu : IsSeparable u
cs : Set α
cs_count : Set.Countable cs
hcs : s ⊆ closure cs
⊢ IsSeparable (s ∪ u)
[PROOFSTEP]
rcases hu with ⟨cu, cu_count, hcu⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
s u cs : Set α
cs_count : Set.Countable cs
hcs : s ⊆ closure cs
cu : Set α
cu_count : Set.Countable cu
hcu : u ⊆ closure cu
⊢ IsSeparable (s ∪ u)
[PROOFSTEP]
refine' ⟨cs ∪ cu, cs_count.union cu_count, _⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
s u cs : Set α
cs_count : Set.Countable cs
hcs : s ⊆ closure cs
cu : Set α
cu_count : Set.Countable cu
hcu : u ⊆ closure cu
⊢ s ∪ u ⊆ closure (cs ∪ cu)
[PROOFSTEP]
exact
union_subset (hcs.trans (closure_mono (subset_union_left _ _))) (hcu.trans (closure_mono (subset_union_right _ _)))
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set α
hs : IsSeparable s
⊢ IsSeparable (_root_.closure s)
[PROOFSTEP]
rcases hs with ⟨c, c_count, hs⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
s c : Set α
c_count : Set.Countable c
hs : s ⊆ _root_.closure c
⊢ IsSeparable (_root_.closure s)
[PROOFSTEP]
exact ⟨c, c_count, by simpa using closure_mono hs⟩
[GOAL]
α : Type u
t : TopologicalSpace α
s c : Set α
c_count : Set.Countable c
hs : s ⊆ _root_.closure c
⊢ _root_.closure s ⊆ _root_.closure c
[PROOFSTEP]
simpa using closure_mono hs
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
inst✝ : Countable ι
s : ι → Set α
hs : ∀ (i : ι), IsSeparable (s i)
⊢ IsSeparable (⋃ (i : ι), s i)
[PROOFSTEP]
choose c hc h'c using hs
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
inst✝ : Countable ι
s c : ι → Set α
hc : ∀ (i : ι), Set.Countable (c i)
h'c : ∀ (i : ι), s i ⊆ closure (c i)
⊢ IsSeparable (⋃ (i : ι), s i)
[PROOFSTEP]
refine' ⟨⋃ i, c i, countable_iUnion hc, iUnion_subset_iff.2 fun i => _⟩
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
inst✝ : Countable ι
s c : ι → Set α
hc : ∀ (i : ι), Set.Countable (c i)
h'c : ∀ (i : ι), s i ⊆ closure (c i)
i : ι
⊢ s i ⊆ closure (⋃ (i : ι), c i)
[PROOFSTEP]
exact (h'c i).trans (closure_mono (subset_iUnion _ i))
[GOAL]
α : Type u
t : TopologicalSpace α
⊢ IsSeparable univ ↔ SeparableSpace α
[PROOFSTEP]
constructor
[GOAL]
case mp
α : Type u
t : TopologicalSpace α
⊢ IsSeparable univ → SeparableSpace α
[PROOFSTEP]
rintro ⟨c, c_count, hc⟩
[GOAL]
case mp.intro.intro
α : Type u
t : TopologicalSpace α
c : Set α
c_count : Set.Countable c
hc : univ ⊆ closure c
⊢ SeparableSpace α
[PROOFSTEP]
refine' ⟨⟨c, c_count, by rwa [dense_iff_closure_eq, ← univ_subset_iff]⟩⟩
[GOAL]
α : Type u
t : TopologicalSpace α
c : Set α
c_count : Set.Countable c
hc : univ ⊆ closure c
⊢ Dense c
[PROOFSTEP]
rwa [dense_iff_closure_eq, ← univ_subset_iff]
[GOAL]
case mpr
α : Type u
t : TopologicalSpace α
⊢ SeparableSpace α → IsSeparable univ
[PROOFSTEP]
intro h
[GOAL]
case mpr
α : Type u
t : TopologicalSpace α
h : SeparableSpace α
⊢ IsSeparable univ
[PROOFSTEP]
rcases exists_countable_dense α with ⟨c, c_count, hc⟩
[GOAL]
case mpr.intro.intro
α : Type u
t : TopologicalSpace α
h : SeparableSpace α
c : Set α
c_count : Set.Countable c
hc : Dense c
⊢ IsSeparable univ
[PROOFSTEP]
exact ⟨c, c_count, by rwa [univ_subset_iff, ← dense_iff_closure_eq]⟩
[GOAL]
α : Type u
t : TopologicalSpace α
h : SeparableSpace α
c : Set α
c_count : Set.Countable c
hc : Dense c
⊢ univ ⊆ closure c
[PROOFSTEP]
rwa [univ_subset_iff, ← dense_iff_closure_eq]
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
s : Set α
hs : IsSeparable s
f : α → β
hf : Continuous f
⊢ IsSeparable (f '' s)
[PROOFSTEP]
rcases hs with ⟨c, c_count, hc⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Continuous f
c : Set α
c_count : Set.Countable c
hc : s ⊆ _root_.closure c
⊢ IsSeparable (f '' s)
[PROOFSTEP]
refine' ⟨f '' c, c_count.image _, _⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Continuous f
c : Set α
c_count : Set.Countable c
hc : s ⊆ _root_.closure c
⊢ f '' s ⊆ _root_.closure (f '' c)
[PROOFSTEP]
rw [image_subset_iff]
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝ : TopologicalSpace β
s : Set α
f : α → β
hf : Continuous f
c : Set α
c_count : Set.Countable c
hc : s ⊆ _root_.closure c
⊢ s ⊆ f ⁻¹' _root_.closure (f '' c)
[PROOFSTEP]
exact hc.trans (closure_subset_preimage_closure_image hf)
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set α
inst✝ : SeparableSpace ↑s
⊢ IsSeparable s
[PROOFSTEP]
have : IsSeparable (((↑) : s → α) '' (univ : Set s)) := (isSeparable_of_separableSpace _).image continuous_subtype_val
[GOAL]
α : Type u
t : TopologicalSpace α
s : Set α
inst✝ : SeparableSpace ↑s
this : IsSeparable (Subtype.val '' univ)
⊢ IsSeparable s
[PROOFSTEP]
simpa only [image_univ, Subtype.range_val_subtype] using this
[GOAL]
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
⊢ IsTopologicalBasis {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U}
[PROOFSTEP]
refine' isTopologicalBasis_of_open_of_nhds _ _
[GOAL]
case refine'_1
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
⊢ ∀ (u : Set ((i : ι) → X i)), u ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} → IsOpen u
[PROOFSTEP]
rintro _ ⟨U, F, h1, rfl⟩
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ IsOpen (Set.pi (↑F) U)
[PROOFSTEP]
apply isOpen_set_pi F.finite_toSet
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ ∀ (a : ι), a ∈ ↑F → IsOpen (U a)
[PROOFSTEP]
intro i hi
[GOAL]
case refine'_1.intro.intro.intro
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
i : ι
hi : i ∈ ↑F
⊢ IsOpen (U i)
[PROOFSTEP]
exact (cond i).isOpen (h1 i hi)
[GOAL]
case refine'_2
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
⊢ ∀ (a : (i : ι) → X i) (u : Set ((i : ι) → X i)),
a ∈ u → IsOpen u → ∃ v, v ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
intro a U ha hU
[GOAL]
case refine'_2
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
a : (i : ι) → X i
U : Set ((i : ι) → X i)
ha : a ∈ U
hU : IsOpen U
⊢ ∃ v, v ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} ∧ a ∈ v ∧ v ⊆ U
[PROOFSTEP]
obtain ⟨I, t, hta, htU⟩ : ∃ (I : Finset ι) (t : ∀ i : ι, Set (X i)), (∀ i, t i ∈ 𝓝 (a i)) ∧ Set.pi (↑I) t ⊆ U :=
by
rw [← Filter.mem_pi', ← nhds_pi]
exact hU.mem_nhds ha
[GOAL]
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
a : (i : ι) → X i
U : Set ((i : ι) → X i)
ha : a ∈ U
hU : IsOpen U
⊢ ∃ I t, (∀ (i : ι), t i ∈ 𝓝 (a i)) ∧ Set.pi (↑I) t ⊆ U
[PROOFSTEP]
rw [← Filter.mem_pi', ← nhds_pi]
[GOAL]
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
a : (i : ι) → X i
U : Set ((i : ι) → X i)
ha : a ∈ U
hU : IsOpen U
⊢ U ∈ 𝓝 fun i => a i
[PROOFSTEP]
exact hU.mem_nhds ha
[GOAL]
case refine'_2.intro.intro.intro
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
a : (i : ι) → X i
U : Set ((i : ι) → X i)
ha : a ∈ U
hU : IsOpen U
I : Finset ι
t : (i : ι) → Set (X i)
hta : ∀ (i : ι), t i ∈ 𝓝 (a i)
htU : Set.pi (↑I) t ⊆ U
⊢ ∃ v, v ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} ∧ a ∈ v ∧ v ⊆ U
[PROOFSTEP]
have : ∀ i, ∃ V ∈ T i, a i ∈ V ∧ V ⊆ t i := fun i => (cond i).mem_nhds_iff.1 (hta i)
[GOAL]
case refine'_2.intro.intro.intro
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
a : (i : ι) → X i
U : Set ((i : ι) → X i)
ha : a ∈ U
hU : IsOpen U
I : Finset ι
t : (i : ι) → Set (X i)
hta : ∀ (i : ι), t i ∈ 𝓝 (a i)
htU : Set.pi (↑I) t ⊆ U
this : ∀ (i : ι), ∃ V, V ∈ T i ∧ a i ∈ V ∧ V ⊆ t i
⊢ ∃ v, v ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} ∧ a ∈ v ∧ v ⊆ U
[PROOFSTEP]
choose V hVT haV hVt using this
[GOAL]
case refine'_2.intro.intro.intro
ι : Type u_1
X : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
a : (i : ι) → X i
U : Set ((i : ι) → X i)
ha : a ∈ U
hU : IsOpen U
I : Finset ι
t : (i : ι) → Set (X i)
hta : ∀ (i : ι), t i ∈ 𝓝 (a i)
htU : Set.pi (↑I) t ⊆ U
V : (i : ι) → Set (X i)
hVT : ∀ (i : ι), V i ∈ T i
haV : ∀ (i : ι), a i ∈ V i
hVt : ∀ (i : ι), V i ⊆ t i
⊢ ∃ v, v ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} ∧ a ∈ v ∧ v ⊆ U
[PROOFSTEP]
exact ⟨_, ⟨V, I, fun i _ => hVT i, rfl⟩, fun i _ => haV i, (pi_mono fun i _ => hVt i).trans htU⟩
[GOAL]
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
⊢ IsTopologicalBasis {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i}
[PROOFSTEP]
letI := ⨅ i, induced (f i) (t i)
[GOAL]
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
⊢ IsTopologicalBasis {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i}
[PROOFSTEP]
convert (isTopologicalBasis_pi cond).inducing (inducing_iInf_to_pi f)
[GOAL]
case h.e'_3
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
⊢ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i} =
(preimage fun x i => f i x) '' {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U}
[PROOFSTEP]
ext V
[GOAL]
case h.e'_3.h
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
V : Set β
⊢ V ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i} ↔
V ∈ (preimage fun x i => f i x) '' {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U}
[PROOFSTEP]
constructor
[GOAL]
case h.e'_3.h.mp
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
V : Set β
⊢ V ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i} →
V ∈ (preimage fun x i => f i x) '' {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U}
[PROOFSTEP]
rintro ⟨U, F, h1, rfl⟩
[GOAL]
case h.e'_3.h.mp.intro.intro.intro
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i ∈
(preimage fun x i => f i x) '' {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U}
[PROOFSTEP]
refine' ⟨(F : Set ι).pi U, ⟨U, F, h1, rfl⟩, _⟩
[GOAL]
case h.e'_3.h.mp.intro.intro.intro
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ (fun x i => f i x) ⁻¹' Set.pi (↑F) U = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i
[PROOFSTEP]
simp_rw [pi_def, Set.preimage_iInter]
[GOAL]
case h.e'_3.h.mp.intro.intro.intro
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ ⋂ (i : ι) (_ : i ∈ ↑F), (fun x i => f i x) ⁻¹' (eval i ⁻¹' U i) = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i
[PROOFSTEP]
rfl
[GOAL]
case h.e'_3.h.mpr
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
V : Set β
⊢ V ∈ (preimage fun x i => f i x) '' {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = Set.pi (↑F) U} →
V ∈ {S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i}
[PROOFSTEP]
rintro ⟨U, ⟨U, F, h1, rfl⟩, rfl⟩
[GOAL]
case h.e'_3.h.mpr.intro.intro.intro.intro.intro
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ (fun x i => f i x) ⁻¹' Set.pi (↑F) U ∈
{S | ∃ U F, (∀ (i : ι), i ∈ F → U i ∈ T i) ∧ S = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i}
[PROOFSTEP]
refine' ⟨U, F, h1, _⟩
[GOAL]
case h.e'_3.h.mpr.intro.intro.intro.intro.intro
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ (fun x i => f i x) ⁻¹' Set.pi (↑F) U = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i
[PROOFSTEP]
simp_rw [pi_def, Set.preimage_iInter]
[GOAL]
case h.e'_3.h.mpr.intro.intro.intro.intro.intro
β : Type u_1
ι : Type u_2
X : ι → Type u_3
t : (i : ι) → TopologicalSpace (X i)
T : (i : ι) → Set (Set (X i))
cond : ∀ (i : ι), IsTopologicalBasis (T i)
f : (i : ι) → β → X i
this : TopologicalSpace β := ⨅ (i : ι), induced (f i) (t i)
U : (i : ι) → Set (X i)
F : Finset ι
h1 : ∀ (i : ι), i ∈ F → U i ∈ T i
⊢ ⋂ (i : ι) (_ : i ∈ ↑F), (fun x i => f i x) ⁻¹' (eval i ⁻¹' U i) = ⋂ (i : ι) (_ : i ∈ F), f i ⁻¹' U i
[PROOFSTEP]
rfl
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
⊢ ∃ t, t ⊆ s ∧ Set.Countable t ∧ Dense t ∧ (∀ (x : α), IsBot x → x ∈ s → x ∈ t) ∧ ∀ (x : α), IsTop x → x ∈ s → x ∈ t
[PROOFSTEP]
rcases hs.exists_countable_dense_subset with ⟨t, hts, htc, htd⟩
[GOAL]
case intro.intro.intro
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
t : Set α
hts : t ⊆ s
htc : Set.Countable t
htd : Dense t
⊢ ∃ t, t ⊆ s ∧ Set.Countable t ∧ Dense t ∧ (∀ (x : α), IsBot x → x ∈ s → x ∈ t) ∧ ∀ (x : α), IsTop x → x ∈ s → x ∈ t
[PROOFSTEP]
refine' ⟨(t ∪ ({x | IsBot x} ∪ {x | IsTop x})) ∩ s, _, _, _, _, _⟩
[GOAL]
case intro.intro.intro.refine'_1
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
t : Set α
hts : t ⊆ s
htc : Set.Countable t
htd : Dense t
⊢ (t ∪ ({x | IsBot x} ∪ {x | IsTop x})) ∩ s ⊆ s
case intro.intro.intro.refine'_2
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
t : Set α
hts : t ⊆ s
htc : Set.Countable t
htd : Dense t
⊢ Set.Countable ((t ∪ ({x | IsBot x} ∪ {x | IsTop x})) ∩ s)
case intro.intro.intro.refine'_3
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
t : Set α
hts : t ⊆ s
htc : Set.Countable t
htd : Dense t
⊢ Dense ((t ∪ ({x | IsBot x} ∪ {x | IsTop x})) ∩ s)
case intro.intro.intro.refine'_4
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
t : Set α
hts : t ⊆ s
htc : Set.Countable t
htd : Dense t
⊢ ∀ (x : α), IsBot x → x ∈ s → x ∈ (t ∪ ({x | IsBot x} ∪ {x | IsTop x})) ∩ s
case intro.intro.intro.refine'_5
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : PartialOrder α
s : Set α
inst✝ : SeparableSpace ↑s
hs : Dense s
t : Set α
hts : t ⊆ s
htc : Set.Countable t
htd : Dense t
⊢ ∀ (x : α), IsTop x → x ∈ s → x ∈ (t ∪ ({x | IsBot x} ∪ {x | IsTop x})) ∩ s
[PROOFSTEP]
exacts [inter_subset_right _ _,
(htc.union ((countable_isBot α).union (countable_isTop α))).mono (inter_subset_left _ _),
htd.mono (subset_inter (subset_union_left _ _) hts), fun x hx hxs => ⟨Or.inr <| Or.inl hx, hxs⟩, fun x hx hxs =>
⟨Or.inr <| Or.inr hx, hxs⟩]
[GOAL]
α : Type u_1
inst✝² : TopologicalSpace α
inst✝¹ : SeparableSpace α
inst✝ : PartialOrder α
⊢ ∃ s, Set.Countable s ∧ Dense s ∧ (∀ (x : α), IsBot x → x ∈ s) ∧ ∀ (x : α), IsTop x → x ∈ s
[PROOFSTEP]
simpa using dense_univ.exists_countable_dense_subset_bot_top
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type ?u.70125
inst✝² : TopologicalSpace β
inst✝¹ : FirstCountableTopology α
inst✝ : FirstCountableTopology β
x✝ : α × β
x : α
y : β
⊢ IsCountablyGenerated (𝓝 (x, y))
[PROOFSTEP]
rw [nhds_prod_eq]
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type ?u.70125
inst✝² : TopologicalSpace β
inst✝¹ : FirstCountableTopology α
inst✝ : FirstCountableTopology β
x✝ : α × β
x : α
y : β
⊢ IsCountablyGenerated (𝓝 x ×ˢ 𝓝 y)
[PROOFSTEP]
infer_instance
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
π : ι → Type u_2
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), FirstCountableTopology (π i)
f : (i : ι) → π i
⊢ IsCountablyGenerated (𝓝 f)
[PROOFSTEP]
rw [nhds_pi]
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
π : ι → Type u_2
inst✝² : Countable ι
inst✝¹ : (i : ι) → TopologicalSpace (π i)
inst✝ : ∀ (i : ι), FirstCountableTopology (π i)
f : (i : ι) → π i
⊢ IsCountablyGenerated (Filter.pi fun i => 𝓝 (f i))
[PROOFSTEP]
infer_instance
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
⊢ ∃ b, Set.Countable b ∧ ¬∅ ∈ b ∧ IsTopologicalBasis b
[PROOFSTEP]
obtain ⟨b, hb₁, hb₂⟩ := @SecondCountableTopology.is_open_generated_countable α _ _
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
b : Set (Set α)
hb₁ : Set.Countable b
hb₂ : t = generateFrom b
⊢ ∃ b, Set.Countable b ∧ ¬∅ ∈ b ∧ IsTopologicalBasis b
[PROOFSTEP]
refine' ⟨_, _, not_mem_diff_of_mem _, (isTopologicalBasis_of_subbasis hb₂).diff_empty⟩
[GOAL]
case intro.intro.refine'_1
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
b : Set (Set α)
hb₁ : Set.Countable b
hb₂ : t = generateFrom b
⊢ Set.Countable ((fun f => ⋂₀ f) '' {f | Set.Finite f ∧ f ⊆ b} \ {∅})
case intro.intro.refine'_2
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
b : Set (Set α)
hb₁ : Set.Countable b
hb₂ : t = generateFrom b
⊢ ∅ ∈ {∅}
[PROOFSTEP]
exacts [((countable_setOf_finite_subset hb₁).image _).mono (diff_subset _ _), rfl]
[GOAL]
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
t : TopologicalSpace β
inst✝ : SecondCountableTopology β
f : α → β
⊢ SecondCountableTopology α
[PROOFSTEP]
rcases@SecondCountableTopology.is_open_generated_countable β _ _ with ⟨b, hb, eq⟩
[GOAL]
case intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
t : TopologicalSpace β
inst✝ : SecondCountableTopology β
f : α → β
b : Set (Set β)
hb : Set.Countable b
eq : t = generateFrom b
⊢ SecondCountableTopology α
[PROOFSTEP]
letI := t.induced f
[GOAL]
case intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
t : TopologicalSpace β
inst✝ : SecondCountableTopology β
f : α → β
b : Set (Set β)
hb : Set.Countable b
eq : t = generateFrom b
this : TopologicalSpace α := induced f t
⊢ SecondCountableTopology α
[PROOFSTEP]
refine' { is_open_generated_countable := ⟨preimage f '' b, hb.image _, _⟩ }
[GOAL]
case intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
t : TopologicalSpace β
inst✝ : SecondCountableTopology β
f : α → β
b : Set (Set β)
hb : Set.Countable b
eq : t = generateFrom b
this : TopologicalSpace α := induced f t
⊢ induced f t = generateFrom (preimage f '' b)
[PROOFSTEP]
rw [eq, induced_generateFrom_eq]
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Sort u_1
inst✝ : Countable ι
t : ι → TopologicalSpace α
ht : ∀ (i : ι), SecondCountableTopology α
⊢ SecondCountableTopology α
[PROOFSTEP]
rw [funext fun i => @eq_generateFrom_countableBasis α (t i) (ht i), ← generateFrom_iUnion]
[GOAL]
α : Type u
t✝ : TopologicalSpace α
ι : Sort u_1
inst✝ : Countable ι
t : ι → TopologicalSpace α
ht : ∀ (i : ι), SecondCountableTopology α
⊢ SecondCountableTopology α
[PROOFSTEP]
exact
SecondCountableTopology.mk' <|
countable_iUnion fun i =>
@countable_countableBasis _ (t i)
(ht i)
-- TODO: more fine grained instances for first_countable_topology, separable_space, t2_space, ...
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
⊢ SeparableSpace α
[PROOFSTEP]
choose p hp using fun s : countableBasis α => nonempty_of_mem_countableBasis s.2
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
p : ↑(countableBasis α) → α
hp : ∀ (s : ↑(countableBasis α)), p s ∈ ↑s
⊢ SeparableSpace α
[PROOFSTEP]
exact
⟨⟨range p, countable_range _,
(isBasis_countableBasis α).dense_iff.2 fun o ho _ => ⟨p ⟨o, ho⟩, hp _, mem_range_self _⟩⟩⟩
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
⊢ ∃ T, Set.Countable T ∧ ⋃ (i : ι) (_ : i ∈ T), s i = ⋃ (i : ι), s i
[PROOFSTEP]
let B := {b ∈ countableBasis α | ∃ i, b ⊆ s i}
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
B : Set (Set α) := {b | b ∈ countableBasis α ∧ ∃ i, b ⊆ s i}
⊢ ∃ T, Set.Countable T ∧ ⋃ (i : ι) (_ : i ∈ T), s i = ⋃ (i : ι), s i
[PROOFSTEP]
choose f hf using fun b : B => b.2.2
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
B : Set (Set α) := {b | b ∈ countableBasis α ∧ ∃ i, b ⊆ s i}
f : ↑B → ι
hf : ∀ (b : ↑B), ↑b ⊆ s (f b)
⊢ ∃ T, Set.Countable T ∧ ⋃ (i : ι) (_ : i ∈ T), s i = ⋃ (i : ι), s i
[PROOFSTEP]
haveI : Encodable B := ((countable_countableBasis α).mono (sep_subset _ _)).toEncodable
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
B : Set (Set α) := {b | b ∈ countableBasis α ∧ ∃ i, b ⊆ s i}
f : ↑B → ι
hf : ∀ (b : ↑B), ↑b ⊆ s (f b)
this : Encodable ↑B
⊢ ∃ T, Set.Countable T ∧ ⋃ (i : ι) (_ : i ∈ T), s i = ⋃ (i : ι), s i
[PROOFSTEP]
refine' ⟨_, countable_range f, (iUnion₂_subset_iUnion _ _).antisymm (sUnion_subset _)⟩
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
B : Set (Set α) := {b | b ∈ countableBasis α ∧ ∃ i, b ⊆ s i}
f : ↑B → ι
hf : ∀ (b : ↑B), ↑b ⊆ s (f b)
this : Encodable ↑B
⊢ ∀ (t' : Set α), (t' ∈ range fun i => s i) → t' ⊆ ⋃ (i : ι) (_ : i ∈ range f), s i
[PROOFSTEP]
rintro _ ⟨i, rfl⟩ x xs
[GOAL]
case intro
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
B : Set (Set α) := {b | b ∈ countableBasis α ∧ ∃ i, b ⊆ s i}
f : ↑B → ι
hf : ∀ (b : ↑B), ↑b ⊆ s (f b)
this : Encodable ↑B
i : ι
x : α
xs : x ∈ (fun i => s i) i
⊢ x ∈ ⋃ (i : ι) (_ : i ∈ range f), s i
[PROOFSTEP]
rcases(isBasis_countableBasis α).exists_subset_of_mem_open xs (H _) with ⟨b, hb, xb, bs⟩
[GOAL]
case intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
ι : Type u_1
s : ι → Set α
H : ∀ (i : ι), IsOpen (s i)
B : Set (Set α) := {b | b ∈ countableBasis α ∧ ∃ i, b ⊆ s i}
f : ↑B → ι
hf : ∀ (b : ↑B), ↑b ⊆ s (f b)
this : Encodable ↑B
i : ι
x : α
xs : x ∈ (fun i => s i) i
b : Set α
hb : b ∈ countableBasis α
xb : x ∈ b
bs : b ⊆ (fun i => s i) i
⊢ x ∈ ⋃ (i : ι) (_ : i ∈ range f), s i
[PROOFSTEP]
exact ⟨_, ⟨_, rfl⟩, _, ⟨⟨⟨_, hb, _, bs⟩, rfl⟩, rfl⟩, hf _ xb⟩
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
S : Set (Set α)
H : ∀ (s : Set α), s ∈ S → IsOpen s
T : Set ↑S
cT : Set.Countable T
hT : ⋃ (i : ↑S) (_ : i ∈ T), ↑i = ⋃ (i : ↑S), ↑i
⊢ ⋃₀ (Subtype.val '' T) = ⋃₀ S
[PROOFSTEP]
rwa [sUnion_image, sUnion_eq_iUnion]
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
⊢ ∃ s, Set.Countable s ∧ ⋃ (x : α) (_ : x ∈ s), f x = univ
[PROOFSTEP]
rcases isOpen_iUnion_countable (fun x => interior (f x)) fun x => isOpen_interior with ⟨s, hsc, hsU⟩
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (i : α) (_ : i ∈ s), interior (f i) = ⋃ (i : α), interior (f i)
⊢ ∃ s, Set.Countable s ∧ ⋃ (x : α) (_ : x ∈ s), f x = univ
[PROOFSTEP]
suffices : ⋃ x ∈ s, interior (f x) = univ
[GOAL]
case intro.intro
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (i : α) (_ : i ∈ s), interior (f i) = ⋃ (i : α), interior (f i)
this : ⋃ (x : α) (_ : x ∈ s), interior (f x) = univ
⊢ ∃ s, Set.Countable s ∧ ⋃ (x : α) (_ : x ∈ s), f x = univ
case this
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (i : α) (_ : i ∈ s), interior (f i) = ⋃ (i : α), interior (f i)
⊢ ⋃ (x : α) (_ : x ∈ s), interior (f x) = univ
[PROOFSTEP]
exact ⟨s, hsc, flip eq_univ_of_subset this <| iUnion₂_mono fun _ _ => interior_subset⟩
[GOAL]
case this
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (i : α) (_ : i ∈ s), interior (f i) = ⋃ (i : α), interior (f i)
⊢ ⋃ (x : α) (_ : x ∈ s), interior (f x) = univ
[PROOFSTEP]
simp only [hsU, eq_univ_iff_forall, mem_iUnion]
[GOAL]
case this
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
hf : ∀ (x : α), f x ∈ 𝓝 x
s : Set α
hsc : Set.Countable s
hsU : ⋃ (i : α) (_ : i ∈ s), interior (f i) = ⋃ (i : α), interior (f i)
⊢ ∀ (x : α), ∃ i, x ∈ interior (f i)
[PROOFSTEP]
exact fun x => ⟨x, mem_interior_iff_mem_nhds.2 (hf x)⟩
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
s : Set α
hf : ∀ (x : α), x ∈ s → f x ∈ 𝓝[s] x
⊢ ∃ t, t ⊆ s ∧ Set.Countable t ∧ s ⊆ ⋃ (x : α) (_ : x ∈ t), f x
[PROOFSTEP]
have : ∀ x : s, (↑) ⁻¹' f x ∈ 𝓝 x := fun x => preimage_coe_mem_nhds_subtype.2 (hf x x.2)
[GOAL]
α : Type u
t : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
s : Set α
hf : ∀ (x : α), x ∈ s → f x ∈ 𝓝[s] x
this : ∀ (x : ↑s), Subtype.val ⁻¹' f ↑x ∈ 𝓝 x
⊢ ∃ t, t ⊆ s ∧ Set.Countable t ∧ s ⊆ ⋃ (x : α) (_ : x ∈ t), f x
[PROOFSTEP]
rcases countable_cover_nhds this with ⟨t, htc, htU⟩
[GOAL]
case intro.intro
α : Type u
t✝ : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
s : Set α
hf : ∀ (x : α), x ∈ s → f x ∈ 𝓝[s] x
this : ∀ (x : ↑s), Subtype.val ⁻¹' f ↑x ∈ 𝓝 x
t : Set ↑s
htc : Set.Countable t
htU : ⋃ (x : ↑s) (_ : x ∈ t), Subtype.val ⁻¹' f ↑x = univ
⊢ ∃ t, t ⊆ s ∧ Set.Countable t ∧ s ⊆ ⋃ (x : α) (_ : x ∈ t), f x
[PROOFSTEP]
refine' ⟨(↑) '' t, Subtype.coe_image_subset _ _, htc.image _, fun x hx => _⟩
[GOAL]
case intro.intro
α : Type u
t✝ : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
s : Set α
hf : ∀ (x : α), x ∈ s → f x ∈ 𝓝[s] x
this : ∀ (x : ↑s), Subtype.val ⁻¹' f ↑x ∈ 𝓝 x
t : Set ↑s
htc : Set.Countable t
htU : ⋃ (x : ↑s) (_ : x ∈ t), Subtype.val ⁻¹' f ↑x = univ
x : α
hx : x ∈ s
⊢ x ∈ ⋃ (x : α) (_ : x ∈ Subtype.val '' t), f x
[PROOFSTEP]
simp only [biUnion_image, eq_univ_iff_forall, ← preimage_iUnion, mem_preimage] at htU ⊢
[GOAL]
case intro.intro
α : Type u
t✝ : TopologicalSpace α
inst✝ : SecondCountableTopology α
f : α → Set α
s : Set α
hf : ∀ (x : α), x ∈ s → f x ∈ 𝓝[s] x
this : ∀ (x : ↑s), Subtype.val ⁻¹' f ↑x ∈ 𝓝 x
t : Set ↑s
htc : Set.Countable t
x : α
hx : x ∈ s
htU : ∀ (x : ↑s), ↑x ∈ ⋃ (i : ↑s) (_ : i ∈ t), f ↑i
⊢ x ∈ ⋃ (y : ↑s) (_ : y ∈ t), f ↑y
[PROOFSTEP]
exact htU ⟨x, hx⟩
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
⊢ IsTopologicalBasis (⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i)
[PROOFSTEP]
apply isTopologicalBasis_of_open_of_nhds
[GOAL]
case h_open
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
⊢ ∀ (u : Set ((i : ι) × E i)), u ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i → IsOpen u
[PROOFSTEP]
intro u hu
[GOAL]
case h_open
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
u : Set ((i : ι) × E i)
hu : u ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i
⊢ IsOpen u
[PROOFSTEP]
obtain ⟨i, t, ts, rfl⟩ : ∃ (i : ι) (t : Set (E i)), t ∈ s i ∧ Sigma.mk i '' t = u := by
simpa only [mem_iUnion, mem_image] using hu
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
u : Set ((i : ι) × E i)
hu : u ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i
⊢ ∃ i t, t ∈ s i ∧ Sigma.mk i '' t = u
[PROOFSTEP]
simpa only [mem_iUnion, mem_image] using hu
[GOAL]
case h_open.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
i : ι
t : Set (E i)
ts : t ∈ s i
hu : Sigma.mk i '' t ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i
⊢ IsOpen (Sigma.mk i '' t)
[PROOFSTEP]
exact isOpenMap_sigmaMk _ ((hs i).isOpen ts)
[GOAL]
case h_nhds
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
⊢ ∀ (a : (i : ι) × E i) (u : Set ((i : ι) × E i)),
a ∈ u → IsOpen u → ∃ v, v ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
rintro ⟨i, x⟩ u hxu u_open
[GOAL]
case h_nhds.mk
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
i : ι
x : E i
u : Set ((i : ι) × E i)
hxu : { fst := i, snd := x } ∈ u
u_open : IsOpen u
⊢ ∃ v, v ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i ∧ { fst := i, snd := x } ∈ v ∧ v ⊆ u
[PROOFSTEP]
have hx : x ∈ Sigma.mk i ⁻¹' u := hxu
[GOAL]
case h_nhds.mk
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
i : ι
x : E i
u : Set ((i : ι) × E i)
hxu : { fst := i, snd := x } ∈ u
u_open : IsOpen u
hx : x ∈ Sigma.mk i ⁻¹' u
⊢ ∃ v, v ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i ∧ { fst := i, snd := x } ∈ v ∧ v ⊆ u
[PROOFSTEP]
obtain ⟨v, vs, xv, hv⟩ : ∃ (v : Set (E i)), v ∈ s i ∧ x ∈ v ∧ v ⊆ Sigma.mk i ⁻¹' u :=
(hs i).exists_subset_of_mem_open hx (isOpen_sigma_iff.1 u_open i)
[GOAL]
case h_nhds.mk.intro.intro.intro
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝ : (i : ι) → TopologicalSpace (E i)
s : (i : ι) → Set (Set (E i))
hs : ∀ (i : ι), IsTopologicalBasis (s i)
i : ι
x : E i
u : Set ((i : ι) × E i)
hxu : { fst := i, snd := x } ∈ u
u_open : IsOpen u
hx : x ∈ Sigma.mk i ⁻¹' u
v : Set (E i)
vs : v ∈ s i
xv : x ∈ v
hv : v ⊆ Sigma.mk i ⁻¹' u
⊢ ∃ v, v ∈ ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' s i ∧ { fst := i, snd := x } ∈ v ∧ v ⊆ u
[PROOFSTEP]
exact ⟨Sigma.mk i '' v, mem_iUnion.2 ⟨i, mem_image_of_mem _ vs⟩, mem_image_of_mem _ xv, image_subset_iff.2 hv⟩
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (E i)
inst✝¹ : Countable ι
inst✝ : ∀ (i : ι), SecondCountableTopology (E i)
⊢ SecondCountableTopology ((i : ι) × E i)
[PROOFSTEP]
let b := ⋃ i : ι, (fun u => (Sigma.mk i '' u : Set (Σ i, E i))) '' countableBasis (E i)
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (E i)
inst✝¹ : Countable ι
inst✝ : ∀ (i : ι), SecondCountableTopology (E i)
b : Set (Set ((i : ι) × E i)) := ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' countableBasis (E i)
⊢ SecondCountableTopology ((i : ι) × E i)
[PROOFSTEP]
have A : IsTopologicalBasis b := IsTopologicalBasis.sigma fun i => isBasis_countableBasis _
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (E i)
inst✝¹ : Countable ι
inst✝ : ∀ (i : ι), SecondCountableTopology (E i)
b : Set (Set ((i : ι) × E i)) := ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' countableBasis (E i)
A : IsTopologicalBasis b
⊢ SecondCountableTopology ((i : ι) × E i)
[PROOFSTEP]
have B : b.Countable := countable_iUnion fun i => (countable_countableBasis _).image _
[GOAL]
α : Type u
t : TopologicalSpace α
ι : Type u_1
E : ι → Type u_2
inst✝² : (i : ι) → TopologicalSpace (E i)
inst✝¹ : Countable ι
inst✝ : ∀ (i : ι), SecondCountableTopology (E i)
b : Set (Set ((i : ι) × E i)) := ⋃ (i : ι), (fun u => Sigma.mk i '' u) '' countableBasis (E i)
A : IsTopologicalBasis b
B : Set.Countable b
⊢ SecondCountableTopology ((i : ι) × E i)
[PROOFSTEP]
exact A.secondCountableTopology B
[GOAL]
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
⊢ IsTopologicalBasis ((fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t)
[PROOFSTEP]
apply isTopologicalBasis_of_open_of_nhds
[GOAL]
case h_open
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
⊢ ∀ (u : Set (α ⊕ β)), u ∈ (fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t → IsOpen u
[PROOFSTEP]
rintro u (⟨w, hw, rfl⟩ | ⟨w, hw, rfl⟩)
[GOAL]
case h_open.inl.intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
w : Set α
hw : w ∈ s
⊢ IsOpen ((fun u => Sum.inl '' u) w)
[PROOFSTEP]
exact openEmbedding_inl.isOpenMap w (hs.isOpen hw)
[GOAL]
case h_open.inr.intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
w : Set β
hw : w ∈ t
⊢ IsOpen ((fun u => Sum.inr '' u) w)
[PROOFSTEP]
exact openEmbedding_inr.isOpenMap w (ht.isOpen hw)
[GOAL]
case h_nhds
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
⊢ ∀ (a : α ⊕ β) (u : Set (α ⊕ β)),
a ∈ u → IsOpen u → ∃ v, v ∈ (fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
rintro (x | x) u hxu u_open
[GOAL]
case h_nhds.inl
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
x : α
u : Set (α ⊕ β)
hxu : Sum.inl x ∈ u
u_open : IsOpen u
⊢ ∃ v, v ∈ (fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t ∧ Sum.inl x ∈ v ∧ v ⊆ u
[PROOFSTEP]
obtain ⟨v, vs, xv, vu⟩ : ∃ v ∈ s, x ∈ v ∧ v ⊆ Sum.inl ⁻¹' u :=
hs.exists_subset_of_mem_open hxu (isOpen_sum_iff.1 u_open).1
[GOAL]
case h_nhds.inl.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
x : α
u : Set (α ⊕ β)
hxu : Sum.inl x ∈ u
u_open : IsOpen u
v : Set α
vs : v ∈ s
xv : x ∈ v
vu : v ⊆ Sum.inl ⁻¹' u
⊢ ∃ v, v ∈ (fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t ∧ Sum.inl x ∈ v ∧ v ⊆ u
[PROOFSTEP]
exact ⟨Sum.inl '' v, mem_union_left _ (mem_image_of_mem _ vs), mem_image_of_mem _ xv, image_subset_iff.2 vu⟩
[GOAL]
case h_nhds.inr
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
x : β
u : Set (α ⊕ β)
hxu : Sum.inr x ∈ u
u_open : IsOpen u
⊢ ∃ v, v ∈ (fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t ∧ Sum.inr x ∈ v ∧ v ⊆ u
[PROOFSTEP]
obtain ⟨v, vs, xv, vu⟩ : ∃ v ∈ t, x ∈ v ∧ v ⊆ Sum.inr ⁻¹' u :=
ht.exists_subset_of_mem_open hxu (isOpen_sum_iff.1 u_open).2
[GOAL]
case h_nhds.inr.intro.intro.intro
α : Type u
t✝ : TopologicalSpace α
β : Type u_1
inst✝¹ : TopologicalSpace α
inst✝ : TopologicalSpace β
s : Set (Set α)
hs : IsTopologicalBasis s
t : Set (Set β)
ht : IsTopologicalBasis t
x : β
u : Set (α ⊕ β)
hxu : Sum.inr x ∈ u
u_open : IsOpen u
v : Set β
vs : v ∈ t
xv : x ∈ v
vu : v ⊆ Sum.inr ⁻¹' u
⊢ ∃ v, v ∈ (fun u => Sum.inl '' u) '' s ∪ (fun u => Sum.inr '' u) '' t ∧ Sum.inr x ∈ v ∧ v ⊆ u
[PROOFSTEP]
exact ⟨Sum.inr '' v, mem_union_right _ (mem_image_of_mem _ vs), mem_image_of_mem _ xv, image_subset_iff.2 vu⟩
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : SecondCountableTopology α
inst✝ : SecondCountableTopology β
⊢ SecondCountableTopology (α ⊕ β)
[PROOFSTEP]
let b := (fun u => Sum.inl '' u) '' countableBasis α ∪ (fun u => Sum.inr '' u) '' countableBasis β
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : SecondCountableTopology α
inst✝ : SecondCountableTopology β
b : Set (Set (α ⊕ β)) := (fun u => Sum.inl '' u) '' countableBasis α ∪ (fun u => Sum.inr '' u) '' countableBasis β
⊢ SecondCountableTopology (α ⊕ β)
[PROOFSTEP]
have A : IsTopologicalBasis b := (isBasis_countableBasis α).sum (isBasis_countableBasis β)
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : SecondCountableTopology α
inst✝ : SecondCountableTopology β
b : Set (Set (α ⊕ β)) := (fun u => Sum.inl '' u) '' countableBasis α ∪ (fun u => Sum.inr '' u) '' countableBasis β
A : IsTopologicalBasis b
⊢ SecondCountableTopology (α ⊕ β)
[PROOFSTEP]
have B : b.Countable :=
(Countable.image (countable_countableBasis _) _).union (Countable.image (countable_countableBasis _) _)
[GOAL]
α : Type u
t : TopologicalSpace α
β : Type u_1
inst✝³ : TopologicalSpace α
inst✝² : TopologicalSpace β
inst✝¹ : SecondCountableTopology α
inst✝ : SecondCountableTopology β
b : Set (Set (α ⊕ β)) := (fun u => Sum.inl '' u) '' countableBasis α ∪ (fun u => Sum.inr '' u) '' countableBasis β
A : IsTopologicalBasis b
B : Set.Countable b
⊢ SecondCountableTopology (α ⊕ β)
[PROOFSTEP]
exact A.secondCountableTopology B
[GOAL]
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
⊢ IsTopologicalBasis (image π '' V)
[PROOFSTEP]
apply isTopologicalBasis_of_open_of_nhds
[GOAL]
case h_open
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
⊢ ∀ (u : Set Y), u ∈ image π '' V → IsOpen u
[PROOFSTEP]
rintro - ⟨U, U_in_V, rfl⟩
[GOAL]
case h_open.intro.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set X
U_in_V : U ∈ V
⊢ IsOpen (π '' U)
[PROOFSTEP]
apply h U (hV.isOpen U_in_V)
[GOAL]
case h_nhds
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
⊢ ∀ (a : Y) (u : Set Y), a ∈ u → IsOpen u → ∃ v, v ∈ image π '' V ∧ a ∈ v ∧ v ⊆ u
[PROOFSTEP]
intro y U y_in_U U_open
[GOAL]
case h_nhds
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
y : Y
U : Set Y
y_in_U : y ∈ U
U_open : IsOpen U
⊢ ∃ v, v ∈ image π '' V ∧ y ∈ v ∧ v ⊆ U
[PROOFSTEP]
obtain ⟨x, rfl⟩ := h'.surjective y
[GOAL]
case h_nhds.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set Y
U_open : IsOpen U
x : X
y_in_U : π x ∈ U
⊢ ∃ v, v ∈ image π '' V ∧ π x ∈ v ∧ v ⊆ U
[PROOFSTEP]
let W := π ⁻¹' U
[GOAL]
case h_nhds.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set Y
U_open : IsOpen U
x : X
y_in_U : π x ∈ U
W : Set X := π ⁻¹' U
⊢ ∃ v, v ∈ image π '' V ∧ π x ∈ v ∧ v ⊆ U
[PROOFSTEP]
have x_in_W : x ∈ W := y_in_U
[GOAL]
case h_nhds.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set Y
U_open : IsOpen U
x : X
y_in_U : π x ∈ U
W : Set X := π ⁻¹' U
x_in_W : x ∈ W
⊢ ∃ v, v ∈ image π '' V ∧ π x ∈ v ∧ v ⊆ U
[PROOFSTEP]
have W_open : IsOpen W := U_open.preimage h'.continuous
[GOAL]
case h_nhds.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set Y
U_open : IsOpen U
x : X
y_in_U : π x ∈ U
W : Set X := π ⁻¹' U
x_in_W : x ∈ W
W_open : IsOpen W
⊢ ∃ v, v ∈ image π '' V ∧ π x ∈ v ∧ v ⊆ U
[PROOFSTEP]
obtain ⟨Z, Z_in_V, x_in_Z, Z_in_W⟩ := hV.exists_subset_of_mem_open x_in_W W_open
[GOAL]
case h_nhds.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set Y
U_open : IsOpen U
x : X
y_in_U : π x ∈ U
W : Set X := π ⁻¹' U
x_in_W : x ∈ W
W_open : IsOpen W
Z : Set X
Z_in_V : Z ∈ V
x_in_Z : x ∈ Z
Z_in_W : Z ⊆ W
⊢ ∃ v, v ∈ image π '' V ∧ π x ∈ v ∧ v ⊆ U
[PROOFSTEP]
have πZ_in_U : π '' Z ⊆ U := (Set.image_subset _ Z_in_W).trans (image_preimage_subset π U)
[GOAL]
case h_nhds.intro.intro.intro.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝¹ : TopologicalSpace X
Y : Type u_2
inst✝ : TopologicalSpace Y
π : X → Y
V : Set (Set X)
hV : IsTopologicalBasis V
h' : QuotientMap π
h : IsOpenMap π
U : Set Y
U_open : IsOpen U
x : X
y_in_U : π x ∈ U
W : Set X := π ⁻¹' U
x_in_W : x ∈ W
W_open : IsOpen W
Z : Set X
Z_in_V : Z ∈ V
x_in_Z : x ∈ Z
Z_in_W : Z ⊆ W
πZ_in_U : π '' Z ⊆ U
⊢ ∃ v, v ∈ image π '' V ∧ π x ∈ v ∧ v ⊆ U
[PROOFSTEP]
exact ⟨π '' Z, ⟨Z, Z_in_V, rfl⟩, ⟨x, x_in_Z, rfl⟩, πZ_in_U⟩
[GOAL]
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝² : TopologicalSpace X
Y : Type u_2
inst✝¹ : TopologicalSpace Y
π : X → Y
inst✝ : SecondCountableTopology X
h' : QuotientMap π
h : IsOpenMap π
⊢ ∃ b, Set.Countable b ∧ inst✝¹ = generateFrom b
[PROOFSTEP]
obtain ⟨V, V_countable, -, V_generates⟩ := exists_countable_basis X
[GOAL]
case intro.intro.intro
α : Type u
t : TopologicalSpace α
X : Type u_1
inst✝² : TopologicalSpace X
Y : Type u_2
inst✝¹ : TopologicalSpace Y
π : X → Y
inst✝ : SecondCountableTopology X
h' : QuotientMap π
h : IsOpenMap π
V : Set (Set X)
V_countable : Set.Countable V
V_generates : IsTopologicalBasis V
⊢ ∃ b, Set.Countable b ∧ inst✝¹ = generateFrom b
[PROOFSTEP]
exact ⟨Set.image π '' V, V_countable.image (Set.image π), (V_generates.quotientMap h' h).eq_generateFrom⟩
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
inst✝ : SecondCountableTopology β
hf : Inducing f
⊢ SecondCountableTopology α
[PROOFSTEP]
rw [hf.1]
[GOAL]
α : Type u_1
β : Type u_2
inst✝² : TopologicalSpace α
inst✝¹ : TopologicalSpace β
f : α → β
inst✝ : SecondCountableTopology β
hf : Inducing f
⊢ SecondCountableTopology α
[PROOFSTEP]
exact secondCountableTopology_induced α β f
| {"mathlib_filename": "Mathlib.Topology.Bases", "llama_tokens": 44336} |
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 1 → 2
[GOAL]
case tfae_1_to_2
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
⊢ x ⤳ y → pure x ≤ 𝓝 y
[PROOFSTEP]
exact (pure_le_nhds _).trans
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 2 → 3
[GOAL]
case tfae_2_to_3
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
⊢ pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
[PROOFSTEP]
exact fun h s hso hy => h (hso.mem_nhds hy)
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 3 → 4
[GOAL]
case tfae_3_to_4
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
⊢ (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
[PROOFSTEP]
exact fun h s hsc hx => of_not_not fun hy => h sᶜ hsc.isOpen_compl hy hx
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 4 → 5
[GOAL]
case tfae_4_to_5
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
⊢ (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
[PROOFSTEP]
exact fun h => h _ isClosed_closure (subset_closure <| mem_singleton _)
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 6 ↔ 5
[GOAL]
case tfae_6_iff_5
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
⊢ closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
[PROOFSTEP]
exact isClosed_closure.closure_subset_iff.trans singleton_subset_iff
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 5 ↔ 7
[GOAL]
case tfae_5_iff_7
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
⊢ y ∈ closure {x} ↔ ClusterPt y (pure x)
[PROOFSTEP]
rw [mem_closure_iff_clusterPt, principal_singleton]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
tfae_5_iff_7 : y ∈ closure {x} ↔ ClusterPt y (pure x)
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_have 5 → 1
[GOAL]
case tfae_5_to_1
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
tfae_5_iff_7 : y ∈ closure {x} ↔ ClusterPt y (pure x)
⊢ y ∈ closure {x} → x ⤳ y
[PROOFSTEP]
refine' fun h => (nhds_basis_opens _).ge_iff.2 _
[GOAL]
case tfae_5_to_1
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
tfae_5_iff_7 : y ∈ closure {x} ↔ ClusterPt y (pure x)
h : y ∈ closure {x}
⊢ ∀ (i' : Set X), y ∈ i' ∧ IsOpen i' → i' ∈ 𝓝 x
[PROOFSTEP]
rintro s ⟨hy, ho⟩
[GOAL]
case tfae_5_to_1.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s✝ : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
tfae_5_iff_7 : y ∈ closure {x} ↔ ClusterPt y (pure x)
h : y ∈ closure {x}
s : Set X
hy : y ∈ s
ho : IsOpen s
⊢ s ∈ 𝓝 x
[PROOFSTEP]
rcases mem_closure_iff.1 h s ho hy with ⟨z, hxs, rfl : z = x⟩
[GOAL]
case tfae_5_to_1.intro.intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y✝ z✝ : X
s✝ : Set X
f : X → Y
y : X
s : Set X
hy : y ∈ s
ho : IsOpen s
z : X
hxs : z ∈ s
tfae_1_to_2 : z ⤳ y → pure z ≤ 𝓝 y
tfae_2_to_3 : pure z ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → z ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → z ∈ s) → ∀ (s : Set X), IsClosed s → z ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → z ∈ s → y ∈ s) → y ∈ closure {z}
tfae_6_iff_5 : closure {y} ⊆ closure {z} ↔ y ∈ closure {z}
tfae_5_iff_7 : y ∈ closure {z} ↔ ClusterPt y (pure z)
h : y ∈ closure {z}
⊢ s ∈ 𝓝 z
[PROOFSTEP]
exact ho.mem_nhds hxs
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
x y : X
tfae_1_to_2 : x ⤳ y → pure x ≤ 𝓝 y
tfae_2_to_3 : pure x ≤ 𝓝 y → ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s
tfae_3_to_4 : (∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) → ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s
tfae_4_to_5 : (∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) → y ∈ closure {x}
tfae_6_iff_5 : closure {y} ⊆ closure {x} ↔ y ∈ closure {x}
tfae_5_iff_7 : y ∈ closure {x} ↔ ClusterPt y (pure x)
tfae_5_to_1 : y ∈ closure {x} → x ⤳ y
⊢ TFAE
[x ⤳ y, pure x ≤ 𝓝 y, ∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s, ∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s,
y ∈ closure {x}, closure {y} ⊆ closure {x}, ClusterPt y (pure x)]
[PROOFSTEP]
tfae_finish
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
hf : Inducing f
⊢ f x ⤳ f y ↔ x ⤳ y
[PROOFSTEP]
simp only [specializes_iff_mem_closure, hf.closure_eq_preimage_closure_image, image_singleton, mem_preimage]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
x₁ x₂ : X
y₁ y₂ : Y
⊢ (x₁, y₁) ⤳ (x₂, y₂) ↔ x₁ ⤳ x₂ ∧ y₁ ⤳ y₂
[PROOFSTEP]
simp only [Specializes, nhds_prod_eq, prod_le_prod]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f✝ : X → Y
f g : (i : ι) → π i
⊢ f ⤳ g ↔ ∀ (i : ι), f i ⤳ g i
[PROOFSTEP]
simp only [Specializes, nhds_pi, pi_le_pi]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ ¬x ⤳ y ↔ ∃ S, IsOpen S ∧ y ∈ S ∧ ¬x ∈ S
[PROOFSTEP]
rw [specializes_iff_forall_open]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (¬∀ (s : Set X), IsOpen s → y ∈ s → x ∈ s) ↔ ∃ S, IsOpen S ∧ y ∈ S ∧ ¬x ∈ S
[PROOFSTEP]
push_neg
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (∃ s, IsOpen s ∧ y ∈ s ∧ ¬x ∈ s) ↔ ∃ S, IsOpen S ∧ y ∈ S ∧ ¬x ∈ S
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ ¬x ⤳ y ↔ ∃ S, IsClosed S ∧ x ∈ S ∧ ¬y ∈ S
[PROOFSTEP]
rw [specializes_iff_forall_closed]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (¬∀ (s : Set X), IsClosed s → x ∈ s → y ∈ s) ↔ ∃ S, IsClosed S ∧ x ∈ S ∧ ¬y ∈ S
[PROOFSTEP]
push_neg
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (∃ s, IsClosed s ∧ x ∈ s ∧ ¬y ∈ s) ↔ ∃ S, IsClosed S ∧ x ∈ S ∧ ¬y ∈ S
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (x ~ᵢ y) ↔ ∀ (s : Set X), IsOpen s → (x ∈ s ↔ y ∈ s)
[PROOFSTEP]
simp only [inseparable_iff_specializes_and, specializes_iff_forall_open, ← forall_and, ← iff_def, Iff.comm]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ ¬(x ~ᵢ y) ↔ ∃ s, IsOpen s ∧ Xor' (x ∈ s) (y ∈ s)
[PROOFSTEP]
simp [inseparable_iff_forall_open, ← xor_iff_not_iff]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (x ~ᵢ y) ↔ ∀ (s : Set X), IsClosed s → (x ∈ s ↔ y ∈ s)
[PROOFSTEP]
simp only [inseparable_iff_specializes_and, specializes_iff_forall_closed, ← forall_and, ← iff_def]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ x ⤳ y ∧ y ⤳ x ↔ x ∈ closure {y} ∧ y ∈ closure {x}
[PROOFSTEP]
simp only [specializes_iff_mem_closure, and_comm]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
⊢ (x ~ᵢ y) ↔ closure {x} = closure {y}
[PROOFSTEP]
simp only [inseparable_iff_specializes_and, specializes_iff_closure_subset, ← subset_antisymm_iff, eq_comm]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
hf : Inducing f
⊢ (f x ~ᵢ f y) ↔ (x ~ᵢ y)
[PROOFSTEP]
simp only [inseparable_iff_specializes_and, hf.specializes_iff]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
x₁ x₂ : X
y₁ y₂ : Y
⊢ ((x₁, y₁) ~ᵢ (x₂, y₂)) ↔ (x₁ ~ᵢ x₂) ∧ (y₁ ~ᵢ y₂)
[PROOFSTEP]
simp only [Inseparable, nhds_prod_eq, prod_inj]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f✝ : X → Y
f g : (i : ι) → π i
⊢ (f ~ᵢ g) ↔ ∀ (i : ι), f i ~ᵢ g i
[PROOFSTEP]
simp only [Inseparable, nhds_pi, funext_iff, pi_inj]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
hs : IsOpen s
⊢ mk ⁻¹' (mk '' s) = s
[PROOFSTEP]
refine' Subset.antisymm _ (subset_preimage_image _ _)
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
hs : IsOpen s
⊢ mk ⁻¹' (mk '' s) ⊆ s
[PROOFSTEP]
rintro x ⟨y, hys, hxy⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
hs : IsOpen s
x y : X
hys : y ∈ s
hxy : mk y = mk x
⊢ x ∈ s
[PROOFSTEP]
exact ((mk_eq_mk.1 hxy).mem_open_iff hs).1 hys
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s✝ : Set X
f : X → Y
t : Set (SeparationQuotient X)
s : Set X
hs : IsOpen s
⊢ IsOpen (mk ⁻¹' (mk '' s))
[PROOFSTEP]
rwa [preimage_image_mk_open hs]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
hs : IsClosed s
⊢ mk ⁻¹' (mk '' s) = s
[PROOFSTEP]
refine' Subset.antisymm _ (subset_preimage_image _ _)
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
hs : IsClosed s
⊢ mk ⁻¹' (mk '' s) ⊆ s
[PROOFSTEP]
rintro x ⟨y, hys, hxy⟩
[GOAL]
case intro.intro
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
hs : IsClosed s
x y : X
hys : y ∈ s
hxy : mk y = mk x
⊢ x ∈ s
[PROOFSTEP]
exact ((mk_eq_mk.1 hxy).mem_closed_iff hs).1 hys
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
⊢ IsClosed (Set.range mk)
[PROOFSTEP]
rw [range_mk]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
⊢ IsClosed univ
[PROOFSTEP]
exact isClosed_univ
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
⊢ Filter.map mk (𝓝 x) = 𝓝 (mk x)
[PROOFSTEP]
rw [← comap_mk_nhds_mk, map_comap_of_surjective surjective_mk]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
⊢ Filter.map mk (𝓝ˢ s) = 𝓝ˢ (mk '' s)
[PROOFSTEP]
rw [← comap_mk_nhdsSet_image, map_comap_of_surjective surjective_mk]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
⊢ comap mk (𝓝ˢ t) = 𝓝ˢ (mk ⁻¹' t)
[PROOFSTEP]
conv_lhs => rw [← image_preimage_eq t surjective_mk, comap_mk_nhdsSet_image]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
| comap mk (𝓝ˢ t)
[PROOFSTEP]
rw [← image_preimage_eq t surjective_mk, comap_mk_nhdsSet_image]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
| comap mk (𝓝ˢ t)
[PROOFSTEP]
rw [← image_preimage_eq t surjective_mk, comap_mk_nhdsSet_image]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
| comap mk (𝓝ˢ t)
[PROOFSTEP]
rw [← image_preimage_eq t surjective_mk, comap_mk_nhdsSet_image]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f : X → Y
t : Set (SeparationQuotient X)
x : X
y : Y
⊢ Filter.map (Prod.map mk mk) (𝓝 (x, y)) = 𝓝 (mk x, mk y)
[PROOFSTEP]
rw [nhds_prod_eq, ← prod_map_map_eq', map_mk_nhds, map_mk_nhds, nhds_prod_eq]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y z : X
s✝ : Set X
f : X → Y
t s : Set (SeparationQuotient X)
x : X
⊢ Filter.map mk (𝓝[mk ⁻¹' s] x) = 𝓝[s] mk x
[PROOFSTEP]
rw [nhdsWithin, ← comap_principal, Filter.push_pull, nhdsWithin, map_mk_nhds]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y z : X
s : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → α
hf : ∀ (x y : X), (x ~ᵢ y) → f x = f y
x : X
l : Filter α
⊢ Tendsto (lift f hf) (𝓝 (mk x)) l ↔ Tendsto f (𝓝 x) l
[PROOFSTEP]
simp only [← map_mk_nhds, tendsto_map'_iff, lift_comp_mk]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y z : X
s✝ : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → α
hf : ∀ (x y : X), (x ~ᵢ y) → f x = f y
x : X
s : Set (SeparationQuotient X)
l : Filter α
⊢ Tendsto (lift f hf) (𝓝[s] mk x) l ↔ Tendsto f (𝓝[mk ⁻¹' s] x) l
[PROOFSTEP]
simp only [← map_mk_nhdsWithin_preimage, tendsto_map'_iff, lift_comp_mk]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s✝ : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y
hf : ∀ (x y : X), (x ~ᵢ y) → f x = f y
s : Set (SeparationQuotient X)
⊢ ContinuousOn (lift f hf) s ↔ ContinuousOn f (mk ⁻¹' s)
[PROOFSTEP]
simp only [ContinuousOn, surjective_mk.forall, continuousWithinAt_lift, mem_preimage]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y
hf : ∀ (x y : X), (x ~ᵢ y) → f x = f y
⊢ Continuous (lift f hf) ↔ Continuous f
[PROOFSTEP]
simp only [continuous_iff_continuousOn_univ, continuousOn_lift, preimage_univ]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → α
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
x : X
y : Y
l : Filter α
⊢ Tendsto (uncurry (lift₂ f hf)) (𝓝 (mk x, mk y)) l ↔ Tendsto (uncurry f) (𝓝 (x, y)) l
[PROOFSTEP]
rw [← map_prod_map_mk_nhds, tendsto_map'_iff]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → α
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
x : X
y : Y
l : Filter α
⊢ Tendsto (uncurry (lift₂ f hf) ∘ Prod.map mk mk) (𝓝 (x, y)) l ↔ Tendsto (uncurry f) (𝓝 (x, y)) l
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s✝ : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → α
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
x : X
y : Y
s : Set (SeparationQuotient X × SeparationQuotient Y)
l : Filter α
⊢ Tendsto (uncurry (lift₂ f hf)) (𝓝[s] (mk x, mk y)) l ↔ Tendsto (uncurry f) (𝓝[Prod.map mk mk ⁻¹' s] (x, y)) l
[PROOFSTEP]
rw [nhdsWithin, ← map_prod_map_mk_nhds, ← Filter.push_pull, comap_principal]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x✝ y✝ z : X
s✝ : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → α
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
x : X
y : Y
s : Set (SeparationQuotient X × SeparationQuotient Y)
l : Filter α
⊢ Tendsto (uncurry (lift₂ f hf)) (Filter.map (Prod.map mk mk) (𝓝 (x, y) ⊓ 𝓟 (Prod.map mk mk ⁻¹' s))) l ↔
Tendsto (uncurry f) (𝓝[Prod.map mk mk ⁻¹' s] (x, y)) l
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s✝ : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → Z
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
s : Set (SeparationQuotient X × SeparationQuotient Y)
⊢ ContinuousOn (uncurry (lift₂ f hf)) s ↔ ContinuousOn (uncurry f) (Prod.map mk mk ⁻¹' s)
[PROOFSTEP]
simp_rw [ContinuousOn, (surjective_mk.Prod_map surjective_mk).forall, Prod.forall, Prod.map, continuousWithinAt_lift₂]
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s✝ : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → Z
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
s : Set (SeparationQuotient X × SeparationQuotient Y)
⊢ (∀ (a : X) (b : Y), (mk a, mk b) ∈ s → ContinuousWithinAt (uncurry f) (Prod.map mk mk ⁻¹' s) (a, b)) ↔
∀ (a : X) (b : Y),
(a, b) ∈ (fun x => (mk x.fst, mk x.snd)) ⁻¹' s →
ContinuousWithinAt (uncurry f) ((fun x => (mk x.fst, mk x.snd)) ⁻¹' s) (a, b)
[PROOFSTEP]
rfl
[GOAL]
X : Type u_1
Y : Type u_2
Z : Type u_3
α : Type u_4
ι : Type u_5
π : ι → Type u_6
inst✝³ : TopologicalSpace X
inst✝² : TopologicalSpace Y
inst✝¹ : TopologicalSpace Z
inst✝ : (i : ι) → TopologicalSpace (π i)
x y z : X
s : Set X
f✝ : X → Y
t : Set (SeparationQuotient X)
f : X → Y → Z
hf : ∀ (a : X) (b : Y) (c : X) (d : Y), (a ~ᵢ c) → (b ~ᵢ d) → f a b = f c d
⊢ Continuous (uncurry (lift₂ f hf)) ↔ Continuous (uncurry f)
[PROOFSTEP]
simp only [continuous_iff_continuousOn_univ, continuousOn_lift₂, preimage_univ]
| {"mathlib_filename": "Mathlib.Topology.Inseparable", "llama_tokens": 15960} |