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/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_non_zero_square_non_square | [25, 1] | [53, 9] | exact mem_univ _ | F : Type u_1
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
this : filter (fun x => ¬IsSquare x) univ = filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ
cf :
Finset.card (filter (fun a => ¬a = 0 ∧ IsSquare a) univ) = Finset.card (filter (fun a => ¬a = 0 ∧ ¬IsSquare a) univ)
⊢ 0 ∈ univ | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_non_zero_square_non_square | [25, 1] | [53, 9] | rw [← h', Nat.bit1_div_two] | F : Type u_1
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
this✝ : filter (fun x => ¬IsSquare x) univ = filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ
cf :
Finset.card (filter (fun a => ¬a = 0 ∧ IsSquare a) univ) = Finset.card (filter (fun a => ¬a = 0 ∧ ¬IsSquare a) univ)
this : filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ ∪ {0} = univ
h' : bit1 (Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ)) = Fintype.card F
⊢ Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ) = Fintype.card F / 2 | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_non_zero_square_non_square | [25, 1] | [53, 9] | rw [Finset.disjoint_left] | F : Type u_1
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
this✝ : filter (fun x => ¬IsSquare x) univ = filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ
cf :
Finset.card (filter (fun a => ¬a = 0 ∧ IsSquare a) univ) = Finset.card (filter (fun a => ¬a = 0 ∧ ¬IsSquare a) univ)
this : filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ ∪ {0} = univ
h' :
Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ) +
Finset.card {0} =
Finset.card univ
⊢ Disjoint (filter (fun x => x ≠ 0 ∧ IsSquare x) univ) (filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ) | F : Type u_1
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
this✝ : filter (fun x => ¬IsSquare x) univ = filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ
cf :
Finset.card (filter (fun a => ¬a = 0 ∧ IsSquare a) univ) = Finset.card (filter (fun a => ¬a = 0 ∧ ¬IsSquare a) univ)
this : filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ ∪ {0} = univ
h' :
Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ) +
Finset.card {0} =
Finset.card univ
⊢ ∀ ⦃a : F⦄, a ∈ filter (fun x => x ≠ 0 ∧ IsSquare x) univ → a ∉ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_non_zero_square_non_square | [25, 1] | [53, 9] | simp (config := { contextual := true }) | F : Type u_1
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
this✝ : filter (fun x => ¬IsSquare x) univ = filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ
cf :
Finset.card (filter (fun a => ¬a = 0 ∧ IsSquare a) univ) = Finset.card (filter (fun a => ¬a = 0 ∧ ¬IsSquare a) univ)
this : filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ ∪ {0} = univ
h' :
Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ) +
Finset.card {0} =
Finset.card univ
⊢ ∀ ⦃a : F⦄, a ∈ filter (fun x => x ≠ 0 ∧ IsSquare x) univ → a ∉ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_non_zero_square_non_square | [25, 1] | [53, 9] | simp | F : Type u_1
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
this✝ : filter (fun x => ¬IsSquare x) univ = filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ
cf :
Finset.card (filter (fun a => ¬a = 0 ∧ IsSquare a) univ) = Finset.card (filter (fun a => ¬a = 0 ∧ ¬IsSquare a) univ)
this : filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ ∪ {0} = univ
h' :
Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ ∪ {0}) =
Finset.card univ
⊢ Disjoint (filter (fun x => x ≠ 0 ∧ IsSquare x) univ ∪ filter (fun x => x ≠ 0 ∧ ¬IsSquare x) univ) {0} | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_square | [55, 1] | [61, 7] | rw [← (card_non_zero_square_non_square hF).1] | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ Finset.card (filter IsSquare univ) = Fintype.card F / 2 + 1 | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ Finset.card (filter IsSquare univ) = Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ) + 1 |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_square | [55, 1] | [61, 7] | simp only [and_comm, ← filter_filter, filter_ne'] | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ Finset.card (filter IsSquare univ) = Finset.card (filter (fun x => x ≠ 0 ∧ IsSquare x) univ) + 1 | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ Finset.card (filter IsSquare univ) = Finset.card (erase (filter (fun a => IsSquare a) univ) 0) + 1 |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_square | [55, 1] | [61, 7] | rw [card_erase_add_one] | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ Finset.card (filter IsSquare univ) = Finset.card (erase (filter (fun a => IsSquare a) univ) 0) + 1 | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ 0 ∈ filter (fun a => IsSquare a) univ |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean | card_square | [55, 1] | [61, 7] | simp | F✝ : Type u_1
inst✝⁴ : Fintype F✝
inst✝³ : Field F✝
F : Type u_2
inst✝² : Fintype F
inst✝¹ : Field F
inst✝ : DecidableEq F
hF : ringChar F ≠ 2
⊢ 0 ∈ filter (fun a => IsSquare a) univ | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.hMul | [16, 1] | [21, 18] | intro x y h | α : Type u_1
inst✝¹ : LE α
inst✝ : Semigroup α
a b : α
ha : MulLECancellable a
hb : MulLECancellable b
⊢ MulLECancellable (a * b) | α : Type u_1
inst✝¹ : LE α
inst✝ : Semigroup α
a b : α
ha : MulLECancellable a
hb : MulLECancellable b
x y : α
h : a * b * x ≤ a * b * y
⊢ x ≤ y |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.hMul | [16, 1] | [21, 18] | rw [mul_assoc, mul_assoc] at h | α : Type u_1
inst✝¹ : LE α
inst✝ : Semigroup α
a b : α
ha : MulLECancellable a
hb : MulLECancellable b
x y : α
h : a * b * x ≤ a * b * y
⊢ x ≤ y | α : Type u_1
inst✝¹ : LE α
inst✝ : Semigroup α
a b : α
ha : MulLECancellable a
hb : MulLECancellable b
x y : α
h : a * (b * x) ≤ a * (b * y)
⊢ x ≤ y |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.hMul | [16, 1] | [21, 18] | exact hb (ha h) | α : Type u_1
inst✝¹ : LE α
inst✝ : Semigroup α
a b : α
ha : MulLECancellable a
hb : MulLECancellable b
x y : α
h : a * (b * x) ≤ a * (b * y)
⊢ x ≤ y | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.of_hMul_left | [24, 1] | [30, 29] | intro x y h | α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
⊢ MulLECancellable b | α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
x y : α
h : b * x ≤ b * y
⊢ x ≤ y |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.of_hMul_left | [24, 1] | [30, 29] | apply hab | α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
x y : α
h : b * x ≤ b * y
⊢ x ≤ y | case a
α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
x y : α
h : b * x ≤ b * y
⊢ a * b * x ≤ a * b * y |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.of_hMul_left | [24, 1] | [30, 29] | rw [mul_assoc, mul_assoc] | case a
α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
x y : α
h : b * x ≤ b * y
⊢ a * b * x ≤ a * b * y | case a
α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
x y : α
h : b * x ≤ b * y
⊢ a * (b * x) ≤ a * (b * y) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Algebra/Order/Monoid/Lemmas.lean | MulLECancellable.of_hMul_left | [24, 1] | [30, 29] | exact mul_le_mul_left' h a | case a
α : Type u_1
inst✝² : LE α
inst✝¹ : Semigroup α
inst✝ : CovariantClass α α (fun x x_1 => x * x_1) fun x x_1 => x ≤ x_1
a b : α
hab : MulLECancellable (a * b)
x y : α
h : b * x ≤ b * y
⊢ a * (b * x) ≤ a * (b * y) | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_head | [21, 1] | [27, 23] | rw [funext_iff, Fin.forall_fin_succ] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ update (vecCons x t) 0 y = vecCons y t | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ update (vecCons x t) 0 y 0 = vecCons y t 0 ∧
∀ (i_1 : Fin i), update (vecCons x t) 0 y (succ i_1) = vecCons y t (succ i_1) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_head | [21, 1] | [27, 23] | refine' ⟨rfl, fun j => _⟩ | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ update (vecCons x t) 0 y 0 = vecCons y t 0 ∧
∀ (i_1 : Fin i), update (vecCons x t) 0 y (succ i_1) = vecCons y t (succ i_1) | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ update (vecCons x t) 0 y (succ j) = vecCons y t (succ j) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_head | [21, 1] | [27, 23] | rw [update_noteq] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ update (vecCons x t) 0 y (succ j) = vecCons y t (succ j) | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ vecCons x t (succ j) = vecCons y t (succ j)
case h
α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ succ j ≠ 0 |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_head | [21, 1] | [27, 23] | exact succ_ne_zero j | case h
α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ succ j ≠ 0 | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_head | [21, 1] | [27, 23] | simp only [vecCons, Fin.cons_succ] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ vecCons x t (succ j) = vecCons y t (succ j) | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_one | [29, 1] | [36, 51] | simp only [funext_iff, forall_fin_succ] | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
⊢ update (vecCons x (vecCons y t)) 1 z = vecCons x (vecCons z t) | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
⊢ update (vecCons x (vecCons y t)) 1 z 0 = vecCons x (vecCons z t) 0 ∧
update (vecCons x (vecCons y t)) 1 z (succ 0) = vecCons x (vecCons z t) (succ 0) ∧
∀ (i_1 : Fin i),
update (vecCons x (vecCons y t)) 1 z (succ (succ i_1)) = vecCons x (vecCons z t) (succ (succ i_1)) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_one | [29, 1] | [36, 51] | refine' ⟨rfl, rfl, fun j => _⟩ | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
⊢ update (vecCons x (vecCons y t)) 1 z 0 = vecCons x (vecCons z t) 0 ∧
update (vecCons x (vecCons y t)) 1 z (succ 0) = vecCons x (vecCons z t) (succ 0) ∧
∀ (i_1 : Fin i),
update (vecCons x (vecCons y t)) 1 z (succ (succ i_1)) = vecCons x (vecCons z t) (succ (succ i_1)) | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
j : Fin i
⊢ update (vecCons x (vecCons y t)) 1 z (succ (succ j)) = vecCons x (vecCons z t) (succ (succ j)) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_one | [29, 1] | [36, 51] | rw [update_noteq] | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
j : Fin i
⊢ update (vecCons x (vecCons y t)) 1 z (succ (succ j)) = vecCons x (vecCons z t) (succ (succ j)) | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
j : Fin i
⊢ vecCons x (vecCons y t) (succ (succ j)) = vecCons x (vecCons z t) (succ (succ j))
case h
α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
j : Fin i
⊢ succ (succ j) ≠ 1 |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_one | [29, 1] | [36, 51] | exact (succ_injective _).ne (Fin.succ_ne_zero _) | case h
α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
j : Fin i
⊢ succ (succ j) ≠ 1 | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_one | [29, 1] | [36, 51] | simp only [vecCons, cons_succ] | α : Type u_1
i : ℕ
x y z : α
t : Fin i → α
j : Fin i
⊢ vecCons x (vecCons y t) (succ (succ j)) = vecCons x (vecCons z t) (succ (succ j)) | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_two | [38, 1] | [45, 71] | simp only [funext_iff, forall_fin_succ] | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
⊢ update (vecCons w (vecCons x (vecCons y t))) 2 z = vecCons w (vecCons x (vecCons z t)) | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
⊢ update (vecCons w (vecCons x (vecCons y t))) 2 z 0 = vecCons w (vecCons x (vecCons z t)) 0 ∧
update (vecCons w (vecCons x (vecCons y t))) 2 z (succ 0) = vecCons w (vecCons x (vecCons z t)) (succ 0) ∧
update (vecCons w (vecCons x (vecCons y t))) 2 z (succ (succ 0)) =
vecCons w (vecCons x (vecCons z t)) (succ (succ 0)) ∧
∀ (i_1 : Fin i),
update (vecCons w (vecCons x (vecCons y t))) 2 z (succ (succ (succ i_1))) =
vecCons w (vecCons x (vecCons z t)) (succ (succ (succ i_1))) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_two | [38, 1] | [45, 71] | refine' ⟨rfl, rfl, rfl, fun j => _⟩ | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
⊢ update (vecCons w (vecCons x (vecCons y t))) 2 z 0 = vecCons w (vecCons x (vecCons z t)) 0 ∧
update (vecCons w (vecCons x (vecCons y t))) 2 z (succ 0) = vecCons w (vecCons x (vecCons z t)) (succ 0) ∧
update (vecCons w (vecCons x (vecCons y t))) 2 z (succ (succ 0)) =
vecCons w (vecCons x (vecCons z t)) (succ (succ 0)) ∧
∀ (i_1 : Fin i),
update (vecCons w (vecCons x (vecCons y t))) 2 z (succ (succ (succ i_1))) =
vecCons w (vecCons x (vecCons z t)) (succ (succ (succ i_1))) | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
j : Fin i
⊢ update (vecCons w (vecCons x (vecCons y t))) 2 z (succ (succ (succ j))) =
vecCons w (vecCons x (vecCons z t)) (succ (succ (succ j))) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_two | [38, 1] | [45, 71] | rw [update_noteq] | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
j : Fin i
⊢ update (vecCons w (vecCons x (vecCons y t))) 2 z (succ (succ (succ j))) =
vecCons w (vecCons x (vecCons z t)) (succ (succ (succ j))) | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
j : Fin i
⊢ vecCons w (vecCons x (vecCons y t)) (succ (succ (succ j))) =
vecCons w (vecCons x (vecCons z t)) (succ (succ (succ j)))
case h
α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
j : Fin i
⊢ succ (succ (succ j)) ≠ 2 |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_two | [38, 1] | [45, 71] | exact (succ_injective _).ne ((succ_injective _).ne (succ_ne_zero _)) | case h
α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
j : Fin i
⊢ succ (succ (succ j)) ≠ 2 | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.update_cons_two | [38, 1] | [45, 71] | simp only [vecCons, cons_succ] | α : Type u_1
i : ℕ
w x y z : α
t : Fin i → α
j : Fin i
⊢ vecCons w (vecCons x (vecCons y t)) (succ (succ (succ j))) =
vecCons w (vecCons x (vecCons z t)) (succ (succ (succ j))) | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | rw [funext_iff] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1) = vecCons y (vecCons x t) | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ ∀ (a : Fin (Nat.succ (Nat.succ i))), (vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) a = vecCons y (vecCons x t) a |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | simp only [forall_fin_succ] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ ∀ (a : Fin (Nat.succ (Nat.succ i))), (vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) a = vecCons y (vecCons x t) a | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ (vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) 0 = vecCons y (vecCons x t) 0 ∧
(vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) (succ 0) = vecCons y (vecCons x t) (succ 0) ∧
∀ (i_1 : Fin i),
(vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) (succ (succ i_1)) = vecCons y (vecCons x t) (succ (succ i_1)) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | refine' ⟨rfl, rfl, fun j => _⟩ | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
⊢ (vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) 0 = vecCons y (vecCons x t) 0 ∧
(vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) (succ 0) = vecCons y (vecCons x t) (succ 0) ∧
∀ (i_1 : Fin i),
(vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) (succ (succ i_1)) = vecCons y (vecCons x t) (succ (succ i_1)) | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ (vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) (succ (succ j)) = vecCons y (vecCons x t) (succ (succ j)) |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | simp only [vecCons, cons_succ, comp_apply] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ (vecCons x (vecCons y t) ∘ ↑(Equiv.swap 0 1)) (succ (succ j)) = vecCons y (vecCons x t) (succ (succ j)) | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ cons x (cons y t) (↑(Equiv.swap 0 1) (succ (succ j))) = t j |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | rw [Equiv.swap_apply_of_ne_of_ne, cons_succ, cons_succ] | α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ cons x (cons y t) (↑(Equiv.swap 0 1) (succ (succ j))) = t j | case a
α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ succ (succ j) ≠ 0
case a
α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ succ (succ j) ≠ 1 |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | exact (succ_injective _).ne (succ_ne_zero _) | case a
α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ succ (succ j) ≠ 1 | no goals |
https://github.com/b-mehta/ExponentialRamsey.git | 7e17b629a915a082869f494c8afa56a3e1c7a88d | ExponentialRamsey/Prereq/Mathlib/Data/Fin/VecNotation.lean | Function.swap_cons | [47, 1] | [56, 47] | exact succ_ne_zero _ | case a
α : Type u_1
i : ℕ
x y : α
t : Fin i → α
j : Fin i
⊢ succ (succ j) ≠ 0 | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChange_eval | [93, 1] | [100, 8] | unfold baseChange | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ bilin (baseChange A F) (a ⊗ₜ[R] m) (b ⊗ₜ[R] n) = a * b * ↑(algebraMap R A) (bilin F m n) | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ bilin
(let L := ↑(toLinHom R) F;
let L' := LinearMap.baseChange A L;
↑LinearMap.toBilin
(LinearMap.comp
(LinearMap.baseChangeLeft R A (M →ₗ[R] R) (A ⊗[R] M →ₗ[A] A)
(LinearMap.comp (↑R (↑(LinearMap.llcomp A (A ⊗[R] M) (A ⊗[R] R) A) (AlgebraTensorModule.lift (boop A))))
(LinearMap.baseChangeHom R A M R)))
L'))
(a ⊗ₜ[R] m) (b ⊗ₜ[R] n) =
a * b * ↑(algebraMap R A) (bilin F m n) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChange_eval | [93, 1] | [100, 8] | dsimp | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ bilin
(let L := ↑(toLinHom R) F;
let L' := LinearMap.baseChange A L;
↑LinearMap.toBilin
(LinearMap.comp
(LinearMap.baseChangeLeft R A (M →ₗ[R] R) (A ⊗[R] M →ₗ[A] A)
(LinearMap.comp (↑R (↑(LinearMap.llcomp A (A ⊗[R] M) (A ⊗[R] R) A) (AlgebraTensorModule.lift (boop A))))
(LinearMap.baseChangeHom R A M R)))
L'))
(a ⊗ₜ[R] m) (b ⊗ₜ[R] n) =
a * b * ↑(algebraMap R A) (bilin F m n) | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ bilin
(↑LinearMap.toBilin
(LinearMap.comp
(LinearMap.baseChangeLeft R A (M →ₗ[R] R) (A ⊗[R] M →ₗ[A] A)
(LinearMap.comp (↑R (↑(LinearMap.llcomp A (A ⊗[R] M) (A ⊗[R] R) A) (AlgebraTensorModule.lift (boop A))))
(LinearMap.baseChangeHom R A M R)))
(LinearMap.baseChange A (↑(toLinHom R) F))))
(a ⊗ₜ[R] m) (b ⊗ₜ[R] n) =
a * b * ↑(algebraMap R A) (bilin F m n) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChange_eval | [93, 1] | [100, 8] | unfold bilin | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ bilin
(↑LinearMap.toBilin
(LinearMap.comp
(LinearMap.baseChangeLeft R A (M →ₗ[R] R) (A ⊗[R] M →ₗ[A] A)
(LinearMap.comp (↑R (↑(LinearMap.llcomp A (A ⊗[R] M) (A ⊗[R] R) A) (AlgebraTensorModule.lift (boop A))))
(LinearMap.baseChangeHom R A M R)))
(LinearMap.baseChange A (↑(toLinHom R) F))))
(a ⊗ₜ[R] m) (b ⊗ₜ[R] n) =
a * b * ↑(algebraMap R A) (bilin F m n) | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ (↑LinearMap.toBilin
(LinearMap.comp
(LinearMap.baseChangeLeft R A (M →ₗ[R] R) (A ⊗[R] M →ₗ[A] A)
(LinearMap.comp (↑R (↑(LinearMap.llcomp A (A ⊗[R] M) (A ⊗[R] R) A) (AlgebraTensorModule.lift (boop A))))
(LinearMap.baseChangeHom R A M R)))
(LinearMap.baseChange A (↑(toLinHom R) F)))).1
(a ⊗ₜ[R] m) (b ⊗ₜ[R] n) =
a * b * ↑(algebraMap R A) (F.1 m n) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChange_eval | [93, 1] | [100, 8] | sorry | R✝ : Type ?u.164095
M✝ : Type ?u.164098
A✝ : Type ?u.164322
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
a b : A
m n : M
⊢ (↑LinearMap.toBilin
(LinearMap.comp
(LinearMap.baseChangeLeft R A (M →ₗ[R] R) (A ⊗[R] M →ₗ[A] A)
(LinearMap.comp (↑R (↑(LinearMap.llcomp A (A ⊗[R] M) (A ⊗[R] R) A) (AlgebraTensorModule.lift (boop A))))
(LinearMap.baseChangeHom R A M R)))
(LinearMap.baseChange A (↑(toLinHom R) F)))).1
(a ⊗ₜ[R] m) (b ⊗ₜ[R] n) =
a * b * ↑(algebraMap R A) (F.1 m n) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_eval | [103, 1] | [111, 7] | rw [baseChange, BilinForm.toQuadraticForm_apply, BilinForm.baseChange_eval, associated_apply,
← two_smul R m, QuadraticForm.map_smul] | R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ ↑(baseChange A F) (a ⊗ₜ[R] m) = a * a * ↑(algebraMap R A) (↑F m) | R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ a * a * ↑(algebraMap R A) (⅟2 * (2 * 2 * ↑F m - ↑F m - ↑F m)) = a * a * ↑(algebraMap R A) (↑F m) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_eval | [103, 1] | [111, 7] | congr | R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ a * a * ↑(algebraMap R A) (⅟2 * (2 * 2 * ↑F m - ↑F m - ↑F m)) = a * a * ↑(algebraMap R A) (↑F m) | case e_a.h.e_6.h
R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ ⅟2 * (2 * 2 * ↑F m - ↑F m - ↑F m) = ↑F m |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_eval | [103, 1] | [111, 7] | rw [mul_assoc, invOf_mul_eq_iff_eq_mul_left] | case e_a.h.e_6.h
R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ ⅟2 * (2 * 2 * ↑F m - ↑F m - ↑F m) = ↑F m | case e_a.h.e_6.h
R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ 2 * (2 * ↑F m) - ↑F m - ↑F m = 2 * ↑F m |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_eval | [103, 1] | [111, 7] | ring | case e_a.h.e_6.h
R✝ : Type ?u.206610
M✝ : Type ?u.206613
A✝ : Type ?u.206837
inst✝¹⁷ : CommSemiring R✝
inst✝¹⁶ : AddCommMonoid M✝
inst✝¹⁵ : Module R✝ M✝
inst✝¹⁴ : CommSemiring A✝
inst✝¹³ : Algebra R✝ A✝
inst✝¹² : Invertible 2
R A M N T : Type
inst✝¹¹ : CommRing R
inst✝¹⁰ : CommRing A
inst✝⁹ : Algebra R A
inst✝⁸ : AddCommGroup M
inst✝⁷ : AddCommGroup N
inst✝⁶ : Module R M
inst✝⁵ : Module R N
inst✝⁴ : AddCommGroup T
inst✝³ : Module A T
inst✝² : Module R T
inst✝¹ : IsScalarTower R A T
a : A
F : QuadraticForm R M
m : M
inst✝ : Invertible 2
⊢ 2 * (2 * ↑F m) - ↑F m - ↑F m = 2 * ↑F m | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp [IsSymm] at * | R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : IsSymm F
⊢ IsSymm (baseChange A F) | R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
⊢ ∀ (x y : A ⊗[R] M), bilin (baseChange A F) x y = bilin (baseChange A F) y x |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | intros x y | R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
⊢ ∀ (x y : A ⊗[R] M), bilin (baseChange A F) x y = bilin (baseChange A F) y x | R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x y : A ⊗[R] M
⊢ bilin (baseChange A F) x y = bilin (baseChange A F) y x |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | induction x using TensorProduct.induction_on generalizing y | R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x y : A ⊗[R] M
⊢ bilin (baseChange A F) x y = bilin (baseChange A F) y x | case C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
y : A ⊗[R] M
⊢ bilin (baseChange A F) 0 y = bilin (baseChange A F) y 0
case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ : A
y✝ : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) y = bilin (baseChange A F) y (x✝ ⊗ₜ[R] y✝)
case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . simp | case C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
y : A ⊗[R] M
⊢ bilin (baseChange A F) 0 y = bilin (baseChange A F) y 0
case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ : A
y✝ : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) y = bilin (baseChange A F) y (x✝ ⊗ₜ[R] y✝)
case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) | case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ : A
y✝ : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) y = bilin (baseChange A F) y (x✝ ⊗ₜ[R] y✝)
case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . rename_i t z
induction y using TensorProduct.induction_on
. simp
. rename_i e r
simp [hF, mul_comm t]
. rename_i e r he hr
simp [*] | case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ : A
y✝ : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) y = bilin (baseChange A F) y (x✝ ⊗ₜ[R] y✝)
case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) | case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . rename_i t z ht hz
induction y using TensorProduct.induction_on
. simp
. rename_i e r
simp [*]
. rename_i e r _ _
simp only [add_right, add_left, *]
ac_rfl | case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp | case C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
y : A ⊗[R] M
⊢ bilin (baseChange A F) 0 y = bilin (baseChange A F) y 0 | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | rename_i t z | case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ : A
y✝ : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) y = bilin (baseChange A F) y (x✝ ⊗ₜ[R] y✝) | case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) y = bilin (baseChange A F) y (t ⊗ₜ[R] z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | induction y using TensorProduct.induction_on | case C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
y : A ⊗[R] M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) y = bilin (baseChange A F) y (t ⊗ₜ[R] z) | case C1.C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) 0 = bilin (baseChange A F) 0 (t ⊗ₜ[R] z)
case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t ⊗ₜ[R] z)
case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . simp | case C1.C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) 0 = bilin (baseChange A F) 0 (t ⊗ₜ[R] z)
case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t ⊗ₜ[R] z)
case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) | case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t ⊗ₜ[R] z)
case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . rename_i e r
simp [hF, mul_comm t] | case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t ⊗ₜ[R] z)
case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) | case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . rename_i e r he hr
simp [*] | case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp | case C1.C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) 0 = bilin (baseChange A F) 0 (t ⊗ₜ[R] z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | rename_i e r | case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t ⊗ₜ[R] z) | case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
e : A
r : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (e ⊗ₜ[R] r) = bilin (baseChange A F) (e ⊗ₜ[R] r) (t ⊗ₜ[R] z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp [hF, mul_comm t] | case C1.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
e : A
r : M
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (e ⊗ₜ[R] r) = bilin (baseChange A F) (e ⊗ₜ[R] r) (t ⊗ₜ[R] z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | rename_i e r he hr | case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t ⊗ₜ[R] z) x✝ = bilin (baseChange A F) x✝ (t ⊗ₜ[R] z)
a✝ : bilin (baseChange A F) (t ⊗ₜ[R] z) y✝ = bilin (baseChange A F) y✝ (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t ⊗ₜ[R] z) | case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
e r : A ⊗[R] M
he : bilin (baseChange A F) (t ⊗ₜ[R] z) e = bilin (baseChange A F) e (t ⊗ₜ[R] z)
hr : bilin (baseChange A F) (t ⊗ₜ[R] z) r = bilin (baseChange A F) r (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (e + r) = bilin (baseChange A F) (e + r) (t ⊗ₜ[R] z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp [*] | case C1.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t : A
z : M
e r : A ⊗[R] M
he : bilin (baseChange A F) (t ⊗ₜ[R] z) e = bilin (baseChange A F) e (t ⊗ₜ[R] z)
hr : bilin (baseChange A F) (t ⊗ₜ[R] z) r = bilin (baseChange A F) r (t ⊗ₜ[R] z)
⊢ bilin (baseChange A F) (t ⊗ₜ[R] z) (e + r) = bilin (baseChange A F) (e + r) (t ⊗ₜ[R] z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | rename_i t z ht hz | case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
x✝ y✝ : A ⊗[R] M
a✝¹ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) x✝ y = bilin (baseChange A F) y x✝
a✝ : ∀ (y : A ⊗[R] M), bilin (baseChange A F) y✝ y = bilin (baseChange A F) y y✝
y : A ⊗[R] M
⊢ bilin (baseChange A F) (x✝ + y✝) y = bilin (baseChange A F) y (x✝ + y✝) | case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
y : A ⊗[R] M
⊢ bilin (baseChange A F) (t + z) y = bilin (baseChange A F) y (t + z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | induction y using TensorProduct.induction_on | case Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
y : A ⊗[R] M
⊢ bilin (baseChange A F) (t + z) y = bilin (baseChange A F) y (t + z) | case Cp.C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
⊢ bilin (baseChange A F) (t + z) 0 = bilin (baseChange A F) 0 (t + z)
case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t + z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t + z)
case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . simp | case Cp.C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
⊢ bilin (baseChange A F) (t + z) 0 = bilin (baseChange A F) 0 (t + z)
case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t + z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t + z)
case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) | case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t + z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t + z)
case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . rename_i e r
simp [*] | case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t + z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t + z)
case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | . rename_i e r _ _
simp only [add_right, add_left, *]
ac_rfl | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp | case Cp.C0
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
⊢ bilin (baseChange A F) (t + z) 0 = bilin (baseChange A F) 0 (t + z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | rename_i e r | case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ : A
y✝ : M
⊢ bilin (baseChange A F) (t + z) (x✝ ⊗ₜ[R] y✝) = bilin (baseChange A F) (x✝ ⊗ₜ[R] y✝) (t + z) | case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
e : A
r : M
⊢ bilin (baseChange A F) (t + z) (e ⊗ₜ[R] r) = bilin (baseChange A F) (e ⊗ₜ[R] r) (t + z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp [*] | case Cp.C1
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
e : A
r : M
⊢ bilin (baseChange A F) (t + z) (e ⊗ₜ[R] r) = bilin (baseChange A F) (e ⊗ₜ[R] r) (t + z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | rename_i e r _ _ | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
x✝ y✝ : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) x✝ = bilin (baseChange A F) x✝ (t + z)
a✝ : bilin (baseChange A F) (t + z) y✝ = bilin (baseChange A F) y✝ (t + z)
⊢ bilin (baseChange A F) (t + z) (x✝ + y✝) = bilin (baseChange A F) (x✝ + y✝) (t + z) | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
e r : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) e = bilin (baseChange A F) e (t + z)
a✝ : bilin (baseChange A F) (t + z) r = bilin (baseChange A F) r (t + z)
⊢ bilin (baseChange A F) (t + z) (e + r) = bilin (baseChange A F) (e + r) (t + z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | simp only [add_right, add_left, *] | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
e r : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) e = bilin (baseChange A F) e (t + z)
a✝ : bilin (baseChange A F) (t + z) r = bilin (baseChange A F) r (t + z)
⊢ bilin (baseChange A F) (t + z) (e + r) = bilin (baseChange A F) (e + r) (t + z) | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
e r : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) e = bilin (baseChange A F) e (t + z)
a✝ : bilin (baseChange A F) (t + z) r = bilin (baseChange A F) r (t + z)
⊢ bilin (baseChange A F) e t + bilin (baseChange A F) e z + (bilin (baseChange A F) r t + bilin (baseChange A F) r z) =
bilin (baseChange A F) e t + bilin (baseChange A F) r t + (bilin (baseChange A F) e z + bilin (baseChange A F) r z) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | BilinForm.baseChangeSymm | [113, 1] | [133, 13] | ac_rfl | case Cp.Cp
R✝ : Type ?u.255543
M✝ : Type ?u.255546
A✝ : Type ?u.255770
inst✝¹⁶ : CommSemiring R✝
inst✝¹⁵ : AddCommMonoid M✝
inst✝¹⁴ : Module R✝ M✝
inst✝¹³ : CommSemiring A✝
inst✝¹² : Algebra R✝ A✝
inst✝¹¹ : Invertible 2
R A M N T : Type
inst✝¹⁰ : CommRing R
inst✝⁹ : CommRing A
inst✝⁸ : Algebra R A
inst✝⁷ : AddCommGroup M
inst✝⁶ : AddCommGroup N
inst✝⁵ : Module R M
inst✝⁴ : Module R N
inst✝³ : AddCommGroup T
inst✝² : Module A T
inst✝¹ : Module R T
inst✝ : IsScalarTower R A T
F : BilinForm R M
hF : ∀ (x y : M), bilin F x y = bilin F y x
t z : A ⊗[R] M
ht : ∀ (y : A ⊗[R] M), bilin (baseChange A F) t y = bilin (baseChange A F) y t
hz : ∀ (y : A ⊗[R] M), bilin (baseChange A F) z y = bilin (baseChange A F) y z
e r : A ⊗[R] M
a✝¹ : bilin (baseChange A F) (t + z) e = bilin (baseChange A F) e (t + z)
a✝ : bilin (baseChange A F) (t + z) r = bilin (baseChange A F) r (t + z)
⊢ bilin (baseChange A F) e t + bilin (baseChange A F) e z + (bilin (baseChange A F) r t + bilin (baseChange A F) r z) =
bilin (baseChange A F) e t + bilin (baseChange A F) r t + (bilin (baseChange A F) e z + bilin (baseChange A F) r z) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associatedHom | [135, 1] | [141, 30] | simp only [baseChange] | R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ ↑(associatedHom R) (baseChange A F) = BilinForm.baseChange A (↑(associatedHom R) F) | R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ ↑(associatedHom R) (BilinForm.toQuadraticForm (BilinForm.baseChange A (↑(associatedHom R) F))) =
BilinForm.baseChange A (↑(associatedHom R) F) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associatedHom | [135, 1] | [141, 30] | apply associated_left_inverse | R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ ↑(associatedHom R) (BilinForm.toQuadraticForm (BilinForm.baseChange A (↑(associatedHom R) F))) =
BilinForm.baseChange A (↑(associatedHom R) F) | case h
R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ BilinForm.IsSymm (BilinForm.baseChange A (↑(associatedHom R) F)) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associatedHom | [135, 1] | [141, 30] | apply BilinForm.baseChangeSymm | case h
R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ BilinForm.IsSymm (BilinForm.baseChange A (↑(associatedHom R) F)) | case h.hF
R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ BilinForm.IsSymm (↑(associatedHom R) F) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associatedHom | [135, 1] | [141, 30] | exact associated_isSymm R F | case h.hF
R✝ : Type ?u.271123
M✝ : Type ?u.271126
A✝ : Type ?u.271350
inst✝¹⁸ : CommSemiring R✝
inst✝¹⁷ : AddCommMonoid M✝
inst✝¹⁶ : Module R✝ M✝
inst✝¹⁵ : CommSemiring A✝
inst✝¹⁴ : Algebra R✝ A✝
inst✝¹³ : Invertible 2
R A M N T : Type
inst✝¹² : CommRing R
inst✝¹¹ : CommRing A
inst✝¹⁰ : Algebra R A
inst✝⁹ : AddCommGroup M
inst✝⁸ : AddCommGroup N
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : AddCommGroup T
inst✝⁴ : Module A T
inst✝³ : Module R T
inst✝² : IsScalarTower R A T
F : QuadraticForm R M
inst✝¹ : Invertible 2
inst✝ : Invertible 2
⊢ BilinForm.IsSymm (↑(associatedHom R) F) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associated | [150, 1] | [157, 31] | simp only [baseChange] | R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ ↑associated (baseChange A F) = BilinForm.baseChange A (↑associated F) | R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ ↑associated (BilinForm.toQuadraticForm (BilinForm.baseChange A (↑(associatedHom R₁) F))) =
BilinForm.baseChange A (↑associated F) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associated | [150, 1] | [157, 31] | apply associated_left_inverse | R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ ↑associated (BilinForm.toQuadraticForm (BilinForm.baseChange A (↑(associatedHom R₁) F))) =
BilinForm.baseChange A (↑associated F) | case h
R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ BilinForm.IsSymm (BilinForm.baseChange A (↑(associatedHom R₁) F)) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associated | [150, 1] | [157, 31] | apply BilinForm.baseChangeSymm | case h
R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ BilinForm.IsSymm (BilinForm.baseChange A (↑(associatedHom R₁) F)) | case h.hF
R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ BilinForm.IsSymm (↑(associatedHom R₁) F) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange_associated | [150, 1] | [157, 31] | exact associated_isSymm R₁ F | case h.hF
R✝ : Type ?u.346845
M✝ : Type ?u.346848
A✝¹ : Type ?u.347072
R₁ : Type
inst✝²³ : CommSemiring R✝
inst✝²² : AddCommMonoid M✝
inst✝²¹ : Module R✝ M✝
inst✝²⁰ : CommSemiring A✝¹
inst✝¹⁹ : Algebra R✝ A✝¹
inst✝¹⁸ : Invertible 2
R A✝ M N T : Type
inst✝¹⁷ : CommRing R
inst✝¹⁶ : CommRing A✝
inst✝¹⁵ : Algebra R A✝
inst✝¹⁴ : AddCommGroup M
inst✝¹³ : AddCommGroup N
inst✝¹² : Module R M
inst✝¹¹ : Module R N
inst✝¹⁰ : AddCommGroup T
inst✝⁹ : Module A✝ T
inst✝⁸ : Module R T
inst✝⁷ : IsScalarTower R A✝ T
inst✝⁶ : CommRing R₁
inst✝⁵ : AddCommGroup M
inst✝⁴ : Module R₁ M
inst✝³ : Invertible 2
A : Type
inst✝² : CommRing A
inst✝¹ : Algebra R₁ A
inst✝ : Invertible 2
F✝ F : QuadraticForm R₁ M
⊢ BilinForm.IsSymm (↑(associatedHom R₁) F) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | LinearMap.baseChange_id | [212, 1] | [218, 112] | ext | R✝ : Type ?u.384027
M✝ : Type ?u.384030
inst✝¹² : CommRing R✝
inst✝¹¹ : AddCommGroup M✝
inst✝¹⁰ : Module R✝ M✝
M₂ : Type ?u.384791
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R✝ M₂
A✝ : Type ?u.385494
inst✝⁷ : Semiring A✝
inst✝⁶ : Algebra R✝ A✝
inst✝⁵ : Invertible 2
R : Type u_1
A : Type u_2
M : Type u_3
inst✝⁴ : CommRing R
inst✝³ : Ring A
inst✝² : Algebra R A
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
⊢ baseChange A id = id | case a.h.h
R✝ : Type ?u.384027
M✝ : Type ?u.384030
inst✝¹² : CommRing R✝
inst✝¹¹ : AddCommGroup M✝
inst✝¹⁰ : Module R✝ M✝
M₂ : Type ?u.384791
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R✝ M₂
A✝ : Type ?u.385494
inst✝⁷ : Semiring A✝
inst✝⁶ : Algebra R✝ A✝
inst✝⁵ : Invertible 2
R : Type u_1
A : Type u_2
M : Type u_3
inst✝⁴ : CommRing R
inst✝³ : Ring A
inst✝² : Algebra R A
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x✝ : M
⊢ ↑(↑(AlgebraTensorModule.curry (baseChange A id)) 1) x✝ = ↑(↑(AlgebraTensorModule.curry id) 1) x✝ |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | LinearMap.baseChange_id | [212, 1] | [218, 112] | simp only [AlgebraTensorModule.curry_apply, curry_apply, coe_restrictScalars, baseChange_tmul, id_coe, id_eq] | case a.h.h
R✝ : Type ?u.384027
M✝ : Type ?u.384030
inst✝¹² : CommRing R✝
inst✝¹¹ : AddCommGroup M✝
inst✝¹⁰ : Module R✝ M✝
M₂ : Type ?u.384791
inst✝⁹ : AddCommGroup M₂
inst✝⁸ : Module R✝ M₂
A✝ : Type ?u.385494
inst✝⁷ : Semiring A✝
inst✝⁶ : Algebra R✝ A✝
inst✝⁵ : Invertible 2
R : Type u_1
A : Type u_2
M : Type u_3
inst✝⁴ : CommRing R
inst✝³ : Ring A
inst✝² : Algebra R A
inst✝¹ : AddCommMonoid M
inst✝ : Module R M
x✝ : M
⊢ ↑(↑(AlgebraTensorModule.curry (baseChange A id)) 1) x✝ = ↑(↑(AlgebraTensorModule.curry id) 1) x✝ | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | LinearMap.baseChange_comp | [221, 1] | [227, 7] | ext | R✝ : Type ?u.401799
M✝ : Type ?u.401802
inst✝¹⁶ : CommRing R✝
inst✝¹⁵ : AddCommGroup M✝
inst✝¹⁴ : Module R✝ M✝
M₂ : Type ?u.402563
inst✝¹³ : AddCommGroup M₂
inst✝¹² : Module R✝ M₂
A✝ : Type ?u.403266
inst✝¹¹ : Semiring A✝
inst✝¹⁰ : Algebra R✝ A✝
inst✝⁹ : Invertible 2
B : Type u_1
R : Type u_2
A : Type u_3
M : Type u_4
N : Type u_5
inst✝⁸ : CommRing R
inst✝⁷ : Ring A
inst✝⁶ : Algebra R A
inst✝⁵ : AddCommMonoid M
inst✝⁴ : AddCommMonoid N
inst✝³ : AddCommMonoid B
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : Module R B
f : M →ₗ[R] N
g : N →ₗ[R] B
⊢ comp (baseChange A g) (baseChange A f) = baseChange A (comp g f) | case a.h.h
R✝ : Type ?u.401799
M✝ : Type ?u.401802
inst✝¹⁶ : CommRing R✝
inst✝¹⁵ : AddCommGroup M✝
inst✝¹⁴ : Module R✝ M✝
M₂ : Type ?u.402563
inst✝¹³ : AddCommGroup M₂
inst✝¹² : Module R✝ M₂
A✝ : Type ?u.403266
inst✝¹¹ : Semiring A✝
inst✝¹⁰ : Algebra R✝ A✝
inst✝⁹ : Invertible 2
B : Type u_1
R : Type u_2
A : Type u_3
M : Type u_4
N : Type u_5
inst✝⁸ : CommRing R
inst✝⁷ : Ring A
inst✝⁶ : Algebra R A
inst✝⁵ : AddCommMonoid M
inst✝⁴ : AddCommMonoid N
inst✝³ : AddCommMonoid B
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : Module R B
f : M →ₗ[R] N
g : N →ₗ[R] B
x✝ : M
⊢ ↑(↑(AlgebraTensorModule.curry (comp (baseChange A g) (baseChange A f))) 1) x✝ =
↑(↑(AlgebraTensorModule.curry (baseChange A (comp g f))) 1) x✝ |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | LinearMap.baseChange_comp | [221, 1] | [227, 7] | simp | case a.h.h
R✝ : Type ?u.401799
M✝ : Type ?u.401802
inst✝¹⁶ : CommRing R✝
inst✝¹⁵ : AddCommGroup M✝
inst✝¹⁴ : Module R✝ M✝
M₂ : Type ?u.402563
inst✝¹³ : AddCommGroup M₂
inst✝¹² : Module R✝ M₂
A✝ : Type ?u.403266
inst✝¹¹ : Semiring A✝
inst✝¹⁰ : Algebra R✝ A✝
inst✝⁹ : Invertible 2
B : Type u_1
R : Type u_2
A : Type u_3
M : Type u_4
N : Type u_5
inst✝⁸ : CommRing R
inst✝⁷ : Ring A
inst✝⁶ : Algebra R A
inst✝⁵ : AddCommMonoid M
inst✝⁴ : AddCommMonoid N
inst✝³ : AddCommMonoid B
inst✝² : Module R M
inst✝¹ : Module R N
inst✝ : Module R B
f : M →ₗ[R] N
g : N →ₗ[R] B
x✝ : M
⊢ ↑(↑(AlgebraTensorModule.curry (comp (baseChange A g) (baseChange A f))) 1) x✝ =
↑(↑(AlgebraTensorModule.curry (baseChange A (comp g f))) 1) x✝ | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | cases' h with val | 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₂
h : QuadraticForm.Equivalent Q S
⊢ QuadraticForm.Equivalent (baseChange A Q) (baseChange A S) | case 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
⊢ QuadraticForm.Equivalent (baseChange A Q) (baseChange A S) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | constructor | case 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
⊢ QuadraticForm.Equivalent (baseChange A Q) (baseChange A S) | case intro.val
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
⊢ Isometry (baseChange A Q) (baseChange A S) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | use (LinearEquiv.baseChange val.toLinearEquiv) | case intro.val
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
⊢ Isometry (baseChange A Q) (baseChange A S) | case intro.val
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
⊢ ∀ (m : A ⊗[R] M),
↑(baseChange A S) (AddHom.toFun (↑(LinearEquiv.baseChange val.toLinearEquiv)).toAddHom m) = ↑(baseChange A Q) m |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | intro m | case intro.val
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
⊢ ∀ (m : A ⊗[R] M),
↑(baseChange A S) (AddHom.toFun (↑(LinearEquiv.baseChange val.toLinearEquiv)).toAddHom m) = ↑(baseChange A Q) m | case intro.val
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
m : A ⊗[R] M
⊢ ↑(baseChange A S) (AddHom.toFun (↑(LinearEquiv.baseChange val.toLinearEquiv)).toAddHom m) = ↑(baseChange A Q) m |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | simp | case intro.val
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
m : A ⊗[R] M
⊢ ↑(baseChange A S) (AddHom.toFun (↑(LinearEquiv.baseChange val.toLinearEquiv)).toAddHom m) = ↑(baseChange A Q) m | case intro.val
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
m : A ⊗[R] M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) m) = ↑(baseChange A Q) m |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | induction m using TensorProduct.induction_on | case intro.val
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
m : A ⊗[R] M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) m) = ↑(baseChange A Q) m | case intro.val.C0
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
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) 0) = ↑(baseChange A Q) 0
case intro.val.C1
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✝ : A
y✝ : M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ ⊗ₜ[R] y✝)) = ↑(baseChange A Q) (x✝ ⊗ₜ[R] y✝)
case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | . simp | case intro.val.C0
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
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) 0) = ↑(baseChange A Q) 0
case intro.val.C1
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✝ : A
y✝ : M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ ⊗ₜ[R] y✝)) = ↑(baseChange A Q) (x✝ ⊗ₜ[R] y✝)
case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) | case intro.val.C1
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✝ : A
y✝ : M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ ⊗ₜ[R] y✝)) = ↑(baseChange A Q) (x✝ ⊗ₜ[R] y✝)
case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | . simp | case intro.val.C1
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✝ : A
y✝ : M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ ⊗ₜ[R] y✝)) = ↑(baseChange A Q) (x✝ ⊗ₜ[R] y✝)
case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) | case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | . simp [map_add, *]
obtain ⟨B, hB⟩ := (baseChange A S).exists_companion
rw [hB] at *
simp [*]
sorry | case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | simp | case intro.val.C0
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
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) 0) = ↑(baseChange A Q) 0 | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | simp | case intro.val.C1
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✝ : A
y✝ : M
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ ⊗ₜ[R] y✝)) = ↑(baseChange A Q) (x✝ ⊗ₜ[R] y✝) | no goals |
https://github.com/alexjbest/ant-lorentz.git | 1f97add294b2d50f99537c15583666d78b0d7e24 | AntLorentz/BaseChange.lean | QuadraticForm.baseChange.Equivalent | [251, 1] | [268, 10] | simp [map_add, *] | case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(LinearEquiv.baseChange val.toLinearEquiv) (x✝ + y✝)) = ↑(baseChange A Q) (x✝ + y✝) | case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(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] | obtain ⟨B, hB⟩ := (baseChange A S).exists_companion | case intro.val.Cp
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✝
⊢ ↑(baseChange A S) (↑(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 S) (↑(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] | rw [hB] at * | 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✝ + ↑(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 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✝) |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.