url
stringclasses
147 values
commit
stringclasses
147 values
file_path
stringlengths
7
101
full_name
stringlengths
1
94
start
stringlengths
6
10
end
stringlengths
6
11
tactic
stringlengths
1
11.2k
state_before
stringlengths
3
2.09M
state_after
stringlengths
6
2.09M
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
QuadraticForm.baseChange.Equivalent
[251, 1]
[268, 10]
simp [*]
case intro.val.Cp.intro R M : Type inst✝⁹ : CommRing R inst✝⁸ : AddCommGroup M inst✝⁷ : Module R M M₂ : Type inst✝⁶ : AddCommGroup M₂ inst✝⁵ : Module R M₂ A✝ : Type ?u.496082 inst✝⁴ : Semiring A✝ inst✝³ : Algebra R A✝ inst✝² : Invertible 2 A : Type inst✝¹ : CommRing A inst✝ : Algebra R A Q : QuadraticForm R M S : QuadraticForm R M₂ val : Isometry Q S x✝ y✝ : A ⊗[R] M a✝¹ : ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) = ↑(baseChange A Q) x✝ a✝ : ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) = ↑(baseChange A Q) y✝ B : BilinForm A (A ⊗[R] M₂) hB : ∀ (x y : A ⊗[R] M₂), ↑(baseChange A S) (x + y) = ↑(baseChange A S) x + ↑(baseChange A S) y + BilinForm.bilin B x y ⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) + ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) + BilinForm.bilin B (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) = ↑(baseChange A Q) (x✝ + y✝)
case intro.val.Cp.intro R M : Type inst✝⁹ : CommRing R inst✝⁸ : AddCommGroup M inst✝⁷ : Module R M M₂ : Type inst✝⁶ : AddCommGroup M₂ inst✝⁵ : Module R M₂ A✝ : Type ?u.496082 inst✝⁴ : Semiring A✝ inst✝³ : Algebra R A✝ inst✝² : Invertible 2 A : Type inst✝¹ : CommRing A inst✝ : Algebra R A Q : QuadraticForm R M S : QuadraticForm R M₂ val : Isometry Q S x✝ y✝ : A ⊗[R] M a✝¹ : ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) = ↑(baseChange A Q) x✝ a✝ : ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) = ↑(baseChange A Q) y✝ B : BilinForm A (A ⊗[R] M₂) hB : ∀ (x y : A ⊗[R] M₂), ↑(baseChange A S) (x + y) = ↑(baseChange A S) x + ↑(baseChange A S) y + BilinForm.bilin B x y ⊢ ↑(baseChange A Q) x✝ + ↑(baseChange A Q) y✝ + BilinForm.bilin B (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) = ↑(baseChange A Q) (x✝ + y✝)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
QuadraticForm.baseChange.Equivalent
[251, 1]
[268, 10]
sorry
case intro.val.Cp.intro R M : Type inst✝⁹ : CommRing R inst✝⁸ : AddCommGroup M inst✝⁷ : Module R M M₂ : Type inst✝⁶ : AddCommGroup M₂ inst✝⁵ : Module R M₂ A✝ : Type ?u.496082 inst✝⁴ : Semiring A✝ inst✝³ : Algebra R A✝ inst✝² : Invertible 2 A : Type inst✝¹ : CommRing A inst✝ : Algebra R A Q : QuadraticForm R M S : QuadraticForm R M₂ val : Isometry Q S x✝ y✝ : A ⊗[R] M a✝¹ : ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) = ↑(baseChange A Q) x✝ a✝ : ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) = ↑(baseChange A Q) y✝ B : BilinForm A (A ⊗[R] M₂) hB : ∀ (x y : A ⊗[R] M₂), ↑(baseChange A S) (x + y) = ↑(baseChange A S) x + ↑(baseChange A S) y + BilinForm.bilin B x y ⊢ ↑(baseChange A Q) x✝ + ↑(baseChange A Q) y✝ + BilinForm.bilin B (↑(LinearEquiv.baseChange val.toLinearEquiv) x✝) (↑(LinearEquiv.baseChange val.toLinearEquiv) y✝) = ↑(baseChange A Q) (x✝ + y✝)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
base_change_module_rank_preserved
[282, 1]
[284, 65]
obtain ⟨⟨_, bM⟩⟩ := Module.Free.exists_basis (R := k) (M := M)
k : Type u_3 M : Type (max u_1 u_2) A : Type u_1 inst✝¹⁰ : Field k inst✝⁹ : AddCommGroup M inst✝⁸ : Module k M inst✝⁷ : Ring A inst✝⁶ : Algebra k A inst✝⁵ : Module A M inst✝⁴ : IsScalarTower k A M inst✝³ : StrongRankCondition A inst✝² : Module.Free k M inst✝¹ : Module.Free A M inst✝ : Module.Free k A ⊢ Module.rank k M = Module.rank A (A ⊗[k] M)
case intro.mk k : Type u_3 M : Type (max u_1 u_2) A : Type u_1 inst✝¹⁰ : Field k inst✝⁹ : AddCommGroup M inst✝⁸ : Module k M inst✝⁷ : Ring A inst✝⁶ : Algebra k A inst✝⁵ : Module A M inst✝⁴ : IsScalarTower k A M inst✝³ : StrongRankCondition A inst✝² : Module.Free k M inst✝¹ : Module.Free A M inst✝ : Module.Free k A fst✝ : Type (max u_1 u_2) bM : Basis fst✝ k M ⊢ Module.rank k M = Module.rank A (A ⊗[k] M)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
base_change_module_rank_preserved
[282, 1]
[284, 65]
rw [← bM.mk_eq_rank'', (bM.base_change (A := A)).mk_eq_rank'']
case intro.mk k : Type u_3 M : Type (max u_1 u_2) A : Type u_1 inst✝¹⁰ : Field k inst✝⁹ : AddCommGroup M inst✝⁸ : Module k M inst✝⁷ : Ring A inst✝⁶ : Algebra k A inst✝⁵ : Module A M inst✝⁴ : IsScalarTower k A M inst✝³ : StrongRankCondition A inst✝² : Module.Free k M inst✝¹ : Module.Free A M inst✝ : Module.Free k A fst✝ : Type (max u_1 u_2) bM : Basis fst✝ k M ⊢ Module.rank k M = Module.rank A (A ⊗[k] M)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
simp only [BilinForm.Nondegenerate, not_forall, exists_prop] at *
M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M hB : ¬Nondegenerate B ⊢ ¬Nondegenerate (baseChange A B)
M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M hB : ∃ x, (∀ (n : M), bilin B x n = 0) ∧ ¬x = 0 ⊢ ∃ x, (∀ (n : TensorProduct k A M), bilin (baseChange A B) x n = 0) ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
obtain ⟨x, hn, hx⟩ := hB
M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M hB : ∃ x, (∀ (n : M), bilin B x n = 0) ∧ ¬x = 0 ⊢ ∃ x, (∀ (n : TensorProduct k A M), bilin (baseChange A B) x n = 0) ∧ ¬x = 0
case intro.intro M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ∃ x, (∀ (n : TensorProduct k A M), bilin (baseChange A B) x n = 0) ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
refine ⟨(1 ⊗ₜ x), ?_, ?_⟩
case intro.intro M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ∃ x, (∀ (n : TensorProduct k A M), bilin (baseChange A B) x n = 0) ∧ ¬x = 0
case intro.intro.refine_1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ∀ (n : TensorProduct k A M), bilin (baseChange A B) (1 ⊗ₜ[k] x) n = 0 case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ¬1 ⊗ₜ[k] x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
. intro n induction n using TensorProduct.induction_on . simp . simp [hn] . simp [*]
case intro.intro.refine_1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ∀ (n : TensorProduct k A M), bilin (baseChange A B) (1 ⊗ₜ[k] x) n = 0 case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ¬1 ⊗ₜ[k] x = 0
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ¬1 ⊗ₜ[k] x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
. simp intro h apply hx sorry
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ¬1 ⊗ₜ[k] x = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
intro n
case intro.intro.refine_1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ∀ (n : TensorProduct k A M), bilin (baseChange A B) (1 ⊗ₜ[k] x) n = 0
case intro.intro.refine_1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 n : TensorProduct k A M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) n = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
induction n using TensorProduct.induction_on
case intro.intro.refine_1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 n : TensorProduct k A M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) n = 0
case intro.intro.refine_1.C0 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) 0 = 0 case intro.intro.refine_1.C1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ : A y✝ : M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ ⊗ₜ[k] y✝) = 0 case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
. simp
case intro.intro.refine_1.C0 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) 0 = 0 case intro.intro.refine_1.C1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ : A y✝ : M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ ⊗ₜ[k] y✝) = 0 case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
case intro.intro.refine_1.C1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ : A y✝ : M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ ⊗ₜ[k] y✝) = 0 case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
. simp [hn]
case intro.intro.refine_1.C1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ : A y✝ : M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ ⊗ₜ[k] y✝) = 0 case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
. simp [*]
case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
simp
case intro.intro.refine_1.C0 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) 0 = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
simp [hn]
case intro.intro.refine_1.C1 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ : A y✝ : M ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ ⊗ₜ[k] y✝) = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
simp [*]
case intro.intro.refine_1.Cp M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 x✝ y✝ : TensorProduct k A M a✝¹ : bilin (baseChange A B) (1 ⊗ₜ[k] x) x✝ = 0 a✝ : bilin (baseChange A B) (1 ⊗ₜ[k] x) y✝ = 0 ⊢ bilin (baseChange A B) (1 ⊗ₜ[k] x) (x✝ + y✝) = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
intro h
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 ⊢ ¬1 ⊗ₜ[k] x = 0
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 h : 1 ⊗ₜ[k] x = 0 ⊢ False
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
apply hx
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 h : 1 ⊗ₜ[k] x = 0 ⊢ False
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 h : 1 ⊗ₜ[k] x = 0 ⊢ x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
BilinForm.baseChange_of_degenerate
[307, 1]
[320, 10]
sorry
case intro.intro.refine_2 M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 B : BilinForm k M x : M hn : ∀ (n : M), bilin B x n = 0 hx : ¬x = 0 h : 1 ⊗ₜ[k] x = 0 ⊢ x = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
baseChange_of_degenerate
[323, 1]
[326, 48]
simp only [baseChange_associated]
M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 Q : QuadraticForm k M hQ : ¬BilinForm.Nondegenerate (↑associated Q) ⊢ ¬BilinForm.Nondegenerate (↑associated (baseChange A Q))
M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 Q : QuadraticForm k M hQ : ¬BilinForm.Nondegenerate (↑associated Q) ⊢ ¬BilinForm.Nondegenerate (BilinForm.baseChange A (↑associated Q))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/BaseChange.lean
baseChange_of_degenerate
[323, 1]
[326, 48]
exact BilinForm.baseChange_of_degenerate _ hQ
M k A : Type inst✝¹² : Field k inst✝¹¹ : AddCommGroup M inst✝¹⁰ : Module k M inst✝⁹ : CommRing A inst✝⁸ : Algebra k A inst✝⁷ : Module A M inst✝⁶ : IsScalarTower k A M inst✝⁵ : StrongRankCondition A inst✝⁴ : Module.Free k M inst✝³ : Module.Free A M inst✝² : Module.Free k A inst✝¹ : Invertible 2 inst✝ : Invertible 2 Q : QuadraticForm k M hQ : ¬BilinForm.Nondegenerate (↑associated Q) ⊢ ¬BilinForm.Nondegenerate (BilinForm.baseChange A (↑associated Q))
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
rootsOfUnity.integer_power_of_ringEquiv
[59, 1]
[62, 28]
obtain ⟨m, hm⟩ := MonoidHom.map_cyclic (g.restrictRootsOfUnity n).toMonoidHom
L : Type u inst✝ : Field L n : ℕ+ g : L ≃+* L ⊢ ∃ m, ∀ (t : { x // x ∈ rootsOfUnity n L }), ↑g ↑↑t = ↑↑(t ^ m)
case intro L : Type u inst✝ : Field L n : ℕ+ g : L ≃+* L m : ℤ hm : ∀ (g_1 : { x // x ∈ rootsOfUnity n L }), ↑(MulEquiv.toMonoidHom (RingEquiv.restrictRootsOfUnity g n)) g_1 = g_1 ^ m ⊢ ∃ m, ∀ (t : { x // x ∈ rootsOfUnity n L }), ↑g ↑↑t = ↑↑(t ^ m)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
rootsOfUnity.integer_power_of_ringEquiv
[59, 1]
[62, 28]
exact ⟨m, by simp [← hm]⟩
case intro L : Type u inst✝ : Field L n : ℕ+ g : L ≃+* L m : ℤ hm : ∀ (g_1 : { x // x ∈ rootsOfUnity n L }), ↑(MulEquiv.toMonoidHom (RingEquiv.restrictRootsOfUnity g n)) g_1 = g_1 ^ m ⊢ ∃ m, ∀ (t : { x // x ∈ rootsOfUnity n L }), ↑g ↑↑t = ↑↑(t ^ m)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
rootsOfUnity.integer_power_of_ringEquiv
[59, 1]
[62, 28]
simp [← hm]
L : Type u inst✝ : Field L n : ℕ+ g : L ≃+* L m : ℤ hm : ∀ (g_1 : { x // x ∈ rootsOfUnity n L }), ↑(MulEquiv.toMonoidHom (RingEquiv.restrictRootsOfUnity g n)) g_1 = g_1 ^ m ⊢ ∀ (t : { x // x ∈ rootsOfUnity n L }), ↑g ↑↑t = ↑↑(t ^ m)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
Group.pow_eq_zpow_mod
[83, 1]
[87, 35]
have h2 : x ^ m = x ^ ((n : ℤ) * (m / (n : ℤ)) + m % (n : ℤ)) := congr_arg (fun a => x ^ a) ((Int.add_comm _ _).trans (Int.emod_add_ediv _ _)).symm
L : Type u inst✝¹ : Field L n✝ : ℕ+ G : Type u_1 inst✝ : Group G x : G m : ℤ n : ℕ h : x ^ n = 1 ⊢ x ^ m = x ^ (m % ↑n)
L : Type u inst✝¹ : Field L n✝ : ℕ+ G : Type u_1 inst✝ : Group G x : G m : ℤ n : ℕ h : x ^ n = 1 h2 : x ^ m = x ^ (↑n * (m / ↑n) + m % ↑n) ⊢ x ^ m = x ^ (m % ↑n)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
Group.pow_eq_zpow_mod
[83, 1]
[87, 35]
simp [h, h2, zpow_add, zpow_mul]
L : Type u inst✝¹ : Field L n✝ : ℕ+ G : Type u_1 inst✝ : Group G x : G m : ℤ n : ℕ h : x ^ n = 1 h2 : x ^ m = x ^ (↑n * (m / ↑n) + m % ↑n) ⊢ x ^ m = x ^ (m % ↑n)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.spec
[94, 1]
[98, 67]
rintro t
L : Type u inst✝ : Field L n✝ : ℕ+ g : L ≃+* L n : ℕ+ ⊢ ∀ (t : { x // x ∈ rootsOfUnity n L }), ↑g ↑↑t = ↑↑(t ^ ZMod.val (χ n g))
L : Type u inst✝ : Field L n✝ : ℕ+ g : L ≃+* L n : ℕ+ t : { x // x ∈ rootsOfUnity n L } ⊢ ↑g ↑↑t = ↑↑(t ^ ZMod.val (χ n g))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.spec
[94, 1]
[98, 67]
rw [ModularCyclotomicCharacter_aux_spec g n t, ← zpow_ofNat, ModularCyclotomicCharacter.toFun, ZMod.val_int_cast, ←Group.pow_eq_zpow_mod _ pow_card_eq_one]
L : Type u inst✝ : Field L n✝ : ℕ+ g : L ≃+* L n : ℕ+ t : { x // x ∈ rootsOfUnity n L } ⊢ ↑g ↑↑t = ↑↑(t ^ ZMod.val (χ n g))
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.ext
[100, 1]
[108, 51]
obtain ⟨g, hg⟩ := IsCyclic.exists_generator (α := G)
L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d h : ∀ (t : G), t ^ ZMod.val a = t ^ ZMod.val b ⊢ a = b
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d h : ∀ (t : G), t ^ ZMod.val a = t ^ ZMod.val b g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g ⊢ a = b
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.ext
[100, 1]
[108, 51]
have hgord := orderOf_eq_card_of_forall_mem_zpowers hg
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d h : ∀ (t : G), t ^ ZMod.val a = t ^ ZMod.val b g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g ⊢ a = b
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d h : ∀ (t : G), t ^ ZMod.val a = t ^ ZMod.val b g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G ⊢ a = b
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.ext
[100, 1]
[108, 51]
specialize h g
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d h : ∀ (t : G), t ^ ZMod.val a = t ^ ZMod.val b g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G ⊢ a = b
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G h : g ^ ZMod.val a = g ^ ZMod.val b ⊢ a = b
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.ext
[100, 1]
[108, 51]
rw [pow_eq_pow_iff_modEq, hgord, hGcard, ← ZMod.nat_cast_eq_nat_cast_iff] at h
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G h : g ^ ZMod.val a = g ^ ZMod.val b ⊢ a = b
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G h : ↑(ZMod.val a) = ↑(ZMod.val b) ⊢ a = b
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.ext
[100, 1]
[108, 51]
subst hGcard
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G d : ℕ a b : ZMod d hGcard : Fintype.card G = d g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G h : ↑(ZMod.val a) = ↑(ZMod.val b) ⊢ a = b
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G a b : ZMod (Fintype.card G) h : ↑(ZMod.val a) = ↑(ZMod.val b) ⊢ a = b
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.ext
[100, 1]
[108, 51]
simpa [ZMod.nat_cast_val, ZMod.cast_id'] using h
case intro L : Type u inst✝³ : Field L n : ℕ+ G : Type u_1 inst✝² : Group G inst✝¹ : Fintype G inst✝ : IsCyclic G g : G hg : ∀ (x : G), x ∈ Subgroup.zpowers g hgord : orderOf g = Fintype.card G a b : ZMod (Fintype.card G) h : ↑(ZMod.val a) = ↑(ZMod.val b) ⊢ a = b
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
refine ext (G := rootsOfUnity n L) rfl ?_
L : Type u inst✝ : Field L n : ℕ+ ⊢ χ n (RingEquiv.refl L) = 1
L : Type u inst✝ : Field L n : ℕ+ ⊢ ∀ (t : { x // x ∈ rootsOfUnity n L }), t ^ ZMod.val (χ n (RingEquiv.refl L)) = t ^ ZMod.val 1
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
intro ζ
L : Type u inst✝ : Field L n : ℕ+ ⊢ ∀ (t : { x // x ∈ rootsOfUnity n L }), t ^ ZMod.val (χ n (RingEquiv.refl L)) = t ^ ZMod.val 1
L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } ⊢ ζ ^ ZMod.val (χ n (RingEquiv.refl L)) = ζ ^ ZMod.val 1
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
ext
L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } ⊢ ζ ^ ZMod.val (χ n (RingEquiv.refl L)) = ζ ^ ZMod.val 1
case a.a L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑↑(ζ ^ ZMod.val (χ n (RingEquiv.refl L))) = ↑↑(ζ ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
rw [← spec]
case a.a L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑↑(ζ ^ ZMod.val (χ n (RingEquiv.refl L))) = ↑↑(ζ ^ ZMod.val 1)
case a.a L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
have : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } := Fin.size_positive'
case a.a L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
case a.a L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
obtain (h | h) := this.lt_or_eq
case a.a L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
case a.a.inl L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 < Fintype.card { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1) case a.a.inr L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
have := Fact.mk h
case a.a.inl L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 < Fintype.card { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
case a.a.inl L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 < Fintype.card { x // x ∈ rootsOfUnity n L } this : Fact (1 < Fintype.card { x // x ∈ rootsOfUnity n L }) ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
simp [ZMod.val_one]
case a.a.inl L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 < Fintype.card { x // x ∈ rootsOfUnity n L } this : Fact (1 < Fintype.card { x // x ∈ rootsOfUnity n L }) ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
have := Fintype.card_le_one_iff_subsingleton.mp h.ge
case a.a.inr L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
case a.a.inr L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } this : Subsingleton { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
obtain rfl : ζ = 1 := by apply Subsingleton.elim
case a.a.inr L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } this : Subsingleton { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑ζ = ↑↑(ζ ^ ZMod.val 1)
case a.a.inr L : Type u inst✝ : Field L n : ℕ+ this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } this : Subsingleton { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑1 = ↑↑(1 ^ ZMod.val 1)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
simp
case a.a.inr L : Type u inst✝ : Field L n : ℕ+ this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } this : Subsingleton { x // x ∈ rootsOfUnity n L } ⊢ ↑(RingEquiv.refl L) ↑↑1 = ↑↑(1 ^ ZMod.val 1)
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.id
[110, 1]
[121, 9]
apply Subsingleton.elim
L : Type u inst✝ : Field L n : ℕ+ ζ : { x // x ∈ rootsOfUnity n L } this✝ : 1 ≤ Fintype.card { x // x ∈ rootsOfUnity n L } h : 1 = Fintype.card { x // x ∈ rootsOfUnity n L } this : Subsingleton { x // x ∈ rootsOfUnity n L } ⊢ ζ = 1
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
refine ext (G := rootsOfUnity n L) rfl ?_
L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ⊢ χ n (g * h) = χ n g * χ n h
L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ⊢ ∀ (t : { x // x ∈ rootsOfUnity n L }), t ^ ZMod.val (χ n (g * h)) = t ^ ZMod.val (χ n g * χ n h)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
intro ζ
L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ⊢ ∀ (t : { x // x ∈ rootsOfUnity n L }), t ^ ZMod.val (χ n (g * h)) = t ^ ZMod.val (χ n g * χ n h)
L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ζ ^ ZMod.val (χ n (g * h)) = ζ ^ ZMod.val (χ n g * χ n h)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
ext
L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ζ ^ ZMod.val (χ n (g * h)) = ζ ^ ZMod.val (χ n g * χ n h)
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑↑(ζ ^ ZMod.val (χ n (g * h))) = ↑↑(ζ ^ ZMod.val (χ n g * χ n h))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
rw [← spec]
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑↑(ζ ^ ZMod.val (χ n (g * h))) = ↑↑(ζ ^ ZMod.val (χ n g * χ n h))
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑(g * h) ↑↑ζ = ↑↑(ζ ^ ZMod.val (χ n g * χ n h))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
change g (h (ζ : Lˣ)) = _
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑(g * h) ↑↑ζ = ↑↑(ζ ^ ZMod.val (χ n g * χ n h))
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑g (↑h ↑↑ζ) = ↑↑(ζ ^ ZMod.val (χ n g * χ n h))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
rw [spec, spec, mul_comm, ← pow_mul, eq_comm]
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑g (↑h ↑↑ζ) = ↑↑(ζ ^ ZMod.val (χ n g * χ n h))
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑↑(ζ ^ ZMod.val (χ n h * χ n g)) = ↑↑(ζ ^ (ZMod.val (χ n h) * ZMod.val (χ n g)))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
congr 2
case a.a L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ↑↑(ζ ^ ZMod.val (χ n h * χ n g)) = ↑↑(ζ ^ (ZMod.val (χ n h) * ZMod.val (χ n g)))
case a.a.e_self.e_self L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ζ ^ ZMod.val (χ n h * χ n g) = ζ ^ (ZMod.val (χ n h) * ZMod.val (χ n g))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/CyclotomicCharacter.lean
ModularCyclotomicCharacter.comp
[123, 1]
[133, 91]
simp only [pow_eq_pow_iff_modEq, ← ZMod.nat_cast_eq_nat_cast_iff, SubmonoidClass.coe_pow, ZMod.nat_cast_val, Nat.cast_mul, ZMod.cast_mul (m := orderOf ζ) orderOf_dvd_card_univ]
case a.a.e_self.e_self L : Type u inst✝ : Field L n : ℕ+ g h : L ≃+* L ζ : { x // x ∈ rootsOfUnity n L } ⊢ ζ ^ ZMod.val (χ n h * χ n g) = ζ ^ (ZMod.val (χ n h) * ZMod.val (χ n g))
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
rw [QuadraticForm.Isotropic, QuadraticForm.Anisotropic]
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 ⊢ Isotropic Q
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
have h : ∃ (w : W), w ≠ 0 := by simpa only [ne_eq, rank_zero_iff_forall_zero, not_forall] using h₂
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 h : ∃ w, w ≠ 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
obtain ⟨w, hw⟩ := h
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 h : ∃ w, w ≠ 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
case intro V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
have : Q w = 0 := by rw [h₁] simp only [zero_apply]
case intro V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
case intro V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 this : ↑Q w = 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
tauto
case intro V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 this : ↑Q w = 0 ⊢ ¬∀ (x : W), ↑Q x = 0 → x = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
simpa only [ne_eq, rank_zero_iff_forall_zero, not_forall] using h₂
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 ⊢ ∃ w, w ≠ 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
rw [h₁]
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 ⊢ ↑Q w = 0
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 ⊢ ↑0 w = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.Isotropic_of_zero_quadForm_dim_ge1
[91, 1]
[100, 8]
simp only [zero_apply]
V : Type ?u.12934 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.13476 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h₁ : Q = 0 h₂ : Module.rank k W ≠ 0 w : W hw : w ≠ 0 ⊢ ↑0 w = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
rw [EverywhereLocallyIsotropic]
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : Isotropic F ⊢ EverywhereLocallyIsotropic F
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : Isotropic F ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F)) ∧ Isotropic (baseChange ℝ F)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
simp only [Isotropic, Anisotropic, not_forall, exists_prop] at h ⊢
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : Isotropic F ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F)) ∧ Isotropic (baseChange ℝ F)
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : ∃ x, ↑F x = 0 ∧ ¬x = 0 ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0) ∧ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
push_neg at h
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : ∃ x, ↑F x = 0 ∧ ¬x = 0 ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0) ∧ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : ∃ x, ↑F x = 0 ∧ x ≠ 0 ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0) ∧ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
obtain ⟨x, hx, hne⟩ := h
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V h : ∃ x, ↑F x = 0 ∧ x ≠ 0 ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0) ∧ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
case intro.intro V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0) ∧ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
constructor
case intro.intro V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0) ∧ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0 case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
. intro p hp use (1 ⊗ₜ x) simp only [baseChange_eval, mul_one, hx, _root_.map_zero, mul_zero, true_and] sorry
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0 case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
. use (1 ⊗ₜ x) simp only [baseChange_eval, mul_one, hx, _root_.map_zero, mul_zero, true_and] sorry
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
intro p hp
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 p : ℕ hp : Fact (Nat.Prime p) ⊢ ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
use (1 ⊗ₜ x)
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 p : ℕ hp : Fact (Nat.Prime p) ⊢ ∃ x, ↑(baseChange ℚ_[p] F) x = 0 ∧ ¬x = 0
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 p : ℕ hp : Fact (Nat.Prime p) ⊢ ↑(baseChange ℚ_[p] F) (1 ⊗ₜ[ℚ] x) = 0 ∧ ¬1 ⊗ₜ[ℚ] x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
simp only [baseChange_eval, mul_one, hx, _root_.map_zero, mul_zero, true_and]
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 p : ℕ hp : Fact (Nat.Prime p) ⊢ ↑(baseChange ℚ_[p] F) (1 ⊗ₜ[ℚ] x) = 0 ∧ ¬1 ⊗ₜ[ℚ] x = 0
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 p : ℕ hp : Fact (Nat.Prime p) ⊢ ¬1 ⊗ₜ[ℚ] x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
sorry
case intro.intro.left V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 p : ℕ hp : Fact (Nat.Prime p) ⊢ ¬1 ⊗ₜ[ℚ] x = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
use (1 ⊗ₜ x)
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ∃ x, ↑(baseChange ℝ F) x = 0 ∧ ¬x = 0
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ↑(baseChange ℝ F) (1 ⊗ₜ[ℚ] x) = 0 ∧ ¬1 ⊗ₜ[ℚ] x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
simp only [baseChange_eval, mul_one, hx, _root_.map_zero, mul_zero, true_and]
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ↑(baseChange ℝ F) (1 ⊗ₜ[ℚ] x) = 0 ∧ ¬1 ⊗ₜ[ℚ] x = 0
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ¬1 ⊗ₜ[ℚ] x = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_global_to_local
[103, 1]
[116, 10]
sorry
case intro.intro.right V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.23512 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W F : QuadraticForm ℚ V x : V hx : ↑F x = 0 hne : x ≠ 0 ⊢ ¬1 ⊗ₜ[ℚ] x = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_of_Equivalent
[120, 1]
[127, 74]
simp only [HasseMinkowski, Isotropic, EverywhereLocallyIsotropic] at *
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ HasseMinkowski Q ↔ HasseMinkowski S
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ (¬Anisotropic Q ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] Q)) ∧ ¬Anisotropic (baseChange ℝ Q)) ↔ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] S)) ∧ ¬Anisotropic (baseChange ℝ S))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_of_Equivalent
[120, 1]
[127, 74]
simp only [anisotropic_iff _ _ h]
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ (¬Anisotropic Q ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] Q)) ∧ ¬Anisotropic (baseChange ℝ Q)) ↔ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] S)) ∧ ¬Anisotropic (baseChange ℝ S))
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] Q)) ∧ ¬Anisotropic (baseChange ℝ Q)) ↔ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] S)) ∧ ¬Anisotropic (baseChange ℝ S))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_of_Equivalent
[120, 1]
[127, 74]
rw [anisotropic_iff _ _ (baseChange.Equivalent ℝ _ _ h)]
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] Q)) ∧ ¬Anisotropic (baseChange ℝ Q)) ↔ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] S)) ∧ ¬Anisotropic (baseChange ℝ S))
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] Q)) ∧ ¬Anisotropic (baseChange ℝ S)) ↔ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] S)) ∧ ¬Anisotropic (baseChange ℝ S))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski_of_Equivalent
[120, 1]
[127, 74]
conv in (Anisotropic (baseChange _ Q)) => rw [anisotropic_iff _ _ (baseChange.Equivalent (R := ℚ) ℚ_[p] _ _ h)]
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W Q : QuadraticForm ℚ V S : QuadraticForm ℚ V₂ h : Equivalent Q S ⊢ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] Q)) ∧ ¬Anisotropic (baseChange ℝ S)) ↔ (¬Anisotropic S ↔ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], ¬Anisotropic (baseChange ℚ_[p] S)) ∧ ¬Anisotropic (baseChange ℝ S))
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.anisotropic_of_quadForm_dim_zero
[133, 1]
[137, 12]
intro (w : W) _
V : Type ?u.62236 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.62778 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h : Module.rank k W = 0 ⊢ Anisotropic Q
V : Type ?u.62236 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.62778 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h : Module.rank k W = 0 w : W a✝ : ↑Q w = 0 ⊢ w = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.anisotropic_of_quadForm_dim_zero
[133, 1]
[137, 12]
rw [rank_zero_iff_forall_zero] at h
V : Type ?u.62236 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.62778 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h : Module.rank k W = 0 w : W a✝ : ↑Q w = 0 ⊢ w = 0
V : Type ?u.62236 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.62778 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h : ∀ (x : W), x = 0 w : W a✝ : ↑Q w = 0 ⊢ w = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.anisotropic_of_quadForm_dim_zero
[133, 1]
[137, 12]
exact h w
V : Type ?u.62236 inst✝⁷ : AddCommGroup V inst✝⁶ : Module ℚ V V₂ : Type ?u.62778 inst✝⁵ : AddCommGroup V₂ inst✝⁴ : Module ℚ V₂ inst✝³ : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝² : Field k inst✝¹ : AddCommGroup W inst✝ : Module k W Q : QuadraticForm k W h : ∀ (x : W), x = 0 w : W a✝ : ↑Q w = 0 ⊢ w = 0
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
intro F
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 ⊢ ∀ (F : QuadraticForm ℚ V), HasseMinkowski F
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ HasseMinkowski F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
rw [HasseMinkowski]
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ HasseMinkowski F
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ Isotropic F ↔ EverywhereLocallyIsotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
constructor
V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ Isotropic F ↔ EverywhereLocallyIsotropic F
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ Isotropic F → EverywhereLocallyIsotropic F case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ EverywhereLocallyIsotropic F → Isotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
contrapose
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ Isotropic F → EverywhereLocallyIsotropic F
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ ¬EverywhereLocallyIsotropic F → ¬Isotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
intro
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ ¬EverywhereLocallyIsotropic F → ¬Isotropic F
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬EverywhereLocallyIsotropic F ⊢ ¬Isotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
rw [QuadraticForm.Isotropic]
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬EverywhereLocallyIsotropic F ⊢ ¬Isotropic F
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬EverywhereLocallyIsotropic F ⊢ ¬¬Anisotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
simp only [not_not]
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬EverywhereLocallyIsotropic F ⊢ ¬¬Anisotropic F
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬EverywhereLocallyIsotropic F ⊢ Anisotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
apply anisotropic_of_quadForm_dim_zero _ _ F hV
case mp V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬EverywhereLocallyIsotropic F ⊢ Anisotropic F
no goals
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
contrapose
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ EverywhereLocallyIsotropic F → Isotropic F
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ ¬Isotropic F → ¬EverywhereLocallyIsotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
intro
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V ⊢ ¬Isotropic F → ¬EverywhereLocallyIsotropic F
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F ⊢ ¬EverywhereLocallyIsotropic F
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
rw [QuadraticForm.EverywhereLocallyIsotropic]
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F ⊢ ¬EverywhereLocallyIsotropic F
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F ⊢ ¬((∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F)) ∧ Isotropic (baseChange ℝ F))
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
push_neg
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F ⊢ ¬((∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F)) ∧ Isotropic (baseChange ℝ F))
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F)) → ¬Isotropic (baseChange ℝ F)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
intro
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F ⊢ (∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F)) → ¬Isotropic (baseChange ℝ F)
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F _✝ : ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F) ⊢ ¬Isotropic (baseChange ℝ F)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
simp only [not_not]
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F _✝ : ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F) ⊢ ¬Isotropic (baseChange ℝ F)
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F _✝ : ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F) ⊢ Anisotropic (baseChange ℝ F)
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
apply anisotropic_of_quadForm_dim_zero
case mpr V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F _✝ : ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F) ⊢ Anisotropic (baseChange ℝ F)
case mpr.h V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F _✝ : ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F) ⊢ Module.rank ℝ (TensorProduct ℚ ℝ V) = 0
https://github.com/alexjbest/ant-lorentz.git
1f97add294b2d50f99537c15583666d78b0d7e24
AntLorentz/HasseMinkowski.lean
QuadraticForm.HasseMinkowski0
[140, 1]
[156, 50]
rw [← base_change_module_rank_preserved, hV]
case mpr.h V : Type inst✝⁶ : AddCommGroup V inst✝⁵ : Module ℚ V V₂ : Type ?u.68408 inst✝⁴ : AddCommGroup V₂ inst✝³ : Module ℚ V₂ inst✝² : FiniteDimensional ℚ V F✝ : QuadraticForm ℚ V k W : Type inst✝¹ : Field k inst✝ : AddCommGroup W hV : Module.rank ℚ V = 0 F : QuadraticForm ℚ V a✝ : ¬Isotropic F _✝ : ∀ (p : ℕ) [inst : Fact (Nat.Prime p)], Isotropic (baseChange ℚ_[p] F) ⊢ Module.rank ℝ (TensorProduct ℚ ℝ V) = 0
no goals