file_path
stringlengths
11
79
full_name
stringlengths
2
100
traced_tactics
list
end
list
commit
stringclasses
4 values
url
stringclasses
4 values
start
list
Mathlib/Order/Filter/Ultrafilter.lean
Ultrafilter.le_sup_iff
[ { "state_after": "no goals", "state_before": "α : Type u\nβ : Type v\nγ : Type ?u.10908\nf✝ g✝ : Ultrafilter α\ns t : Set α\np q : α → Prop\nu : Ultrafilter α\nf g : Filter α\n⊢ ¬↑u ≤ f ⊔ g ↔ ¬(↑u ≤ f ∨ ↑u ≤ g)", "tactic": "simp only [← disjoint_iff_not_le, not_or, disjoint_sup_right]" } ]
[ 174, 84 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 173, 1 ]
Mathlib/Data/Polynomial/Eval.lean
Polynomial.eval₂_mul_C'
[ { "state_after": "case hf\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\n⊢ ∀ (k : ℕ), Commute (↑f (coeff (↑C a) k)) x", "state_before": "R : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\n⊢ eval₂ f x (p * ↑C a) = eval₂ f x p * ↑f a", "tactic": "rw [eval₂_mul_noncomm, eval₂_C]" }, { "state_after": "case hf\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\nk : ℕ\n⊢ Commute (↑f (coeff (↑C a) k)) x", "state_before": "case hf\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\n⊢ ∀ (k : ℕ), Commute (↑f (coeff (↑C a) k)) x", "tactic": "intro k" }, { "state_after": "case pos\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\nk : ℕ\nhk : k = 0\n⊢ Commute (↑f (coeff (↑C a) k)) x\n\ncase neg\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\nk : ℕ\nhk : ¬k = 0\n⊢ Commute (↑f (coeff (↑C a) k)) x", "state_before": "case hf\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\nk : ℕ\n⊢ Commute (↑f (coeff (↑C a) k)) x", "tactic": "by_cases hk : k = 0" }, { "state_after": "no goals", "state_before": "case pos\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\nk : ℕ\nhk : k = 0\n⊢ Commute (↑f (coeff (↑C a) k)) x", "tactic": "simp only [hk, h, coeff_C_zero, coeff_C_ne_zero]" }, { "state_after": "no goals", "state_before": "case neg\nR : Type u\nS : Type v\nT : Type w\nι : Type y\na b : R\nm n : ℕ\ninst✝² : Semiring R\np q r : R[X]\ninst✝¹ : Semiring S\nf : R →+* S\nx : S\ninst✝ : Semiring T\nh : Commute (↑f a) x\nk : ℕ\nhk : ¬k = 0\n⊢ Commute (↑f (coeff (↑C a) k)) x", "tactic": "simp only [coeff_C_ne_zero hk, RingHom.map_zero, Commute.zero_left]" } ]
[ 204, 72 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 199, 1 ]
Mathlib/Order/WellFoundedSet.lean
Set.PartiallyWellOrderedOn.prod
[ { "state_after": "ι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf✝ : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\nf : ℕ → α × β\nhf : ∀ (n : ℕ), f n ∈ s ×ˢ t\n⊢ ∃ m n, m < n ∧ (fun x y => r x.fst y.fst ∧ r' x.snd y.snd) (f m) (f n)", "state_before": "ι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\n⊢ PartiallyWellOrderedOn (s ×ˢ t) fun x y => r x.fst y.fst ∧ r' x.snd y.snd", "tactic": "intro f hf" }, { "state_after": "case intro\nι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf✝ : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\nf : ℕ → α × β\nhf : ∀ (n : ℕ), f n ∈ s ×ˢ t\ng₁ : ℕ ↪o ℕ\nh₁ : ∀ (m n : ℕ), m ≤ n → r ((Prod.fst ∘ f) (↑g₁ m)) ((Prod.fst ∘ f) (↑g₁ n))\n⊢ ∃ m n, m < n ∧ (fun x y => r x.fst y.fst ∧ r' x.snd y.snd) (f m) (f n)", "state_before": "ι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf✝ : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\nf : ℕ → α × β\nhf : ∀ (n : ℕ), f n ∈ s ×ˢ t\n⊢ ∃ m n, m < n ∧ (fun x y => r x.fst y.fst ∧ r' x.snd y.snd) (f m) (f n)", "tactic": "obtain ⟨g₁, h₁⟩ := hs.exists_monotone_subseq (Prod.fst ∘ f) fun n => (hf n).1" }, { "state_after": "case intro.intro.intro.intro\nι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf✝ : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\nf : ℕ → α × β\nhf : ∀ (n : ℕ), f n ∈ s ×ˢ t\ng₁ : ℕ ↪o ℕ\nh₁ : ∀ (m n : ℕ), m ≤ n → r ((Prod.fst ∘ f) (↑g₁ m)) ((Prod.fst ∘ f) (↑g₁ n))\nm n : ℕ\nhlt : m < n\nhle : r' ((Prod.snd ∘ f ∘ ↑g₁) m) ((Prod.snd ∘ f ∘ ↑g₁) n)\n⊢ ∃ m n, m < n ∧ (fun x y => r x.fst y.fst ∧ r' x.snd y.snd) (f m) (f n)", "state_before": "case intro\nι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf✝ : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\nf : ℕ → α × β\nhf : ∀ (n : ℕ), f n ∈ s ×ˢ t\ng₁ : ℕ ↪o ℕ\nh₁ : ∀ (m n : ℕ), m ≤ n → r ((Prod.fst ∘ f) (↑g₁ m)) ((Prod.fst ∘ f) (↑g₁ n))\n⊢ ∃ m n, m < n ∧ (fun x y => r x.fst y.fst ∧ r' x.snd y.snd) (f m) (f n)", "tactic": "obtain ⟨m, n, hlt, hle⟩ := ht (Prod.snd ∘ f ∘ g₁) fun n => (hf _).2" }, { "state_after": "no goals", "state_before": "case intro.intro.intro.intro\nι : Type ?u.91578\nα : Type u_2\nβ : Type u_1\nr : α → α → Prop\nr' : β → β → Prop\nf✝ : α → β\ns t✝ : Set α\na : α\ninst✝¹ : IsRefl α r\ninst✝ : IsTrans α r\nt : Set β\nhs : PartiallyWellOrderedOn s r\nht : PartiallyWellOrderedOn t r'\nf : ℕ → α × β\nhf : ∀ (n : ℕ), f n ∈ s ×ˢ t\ng₁ : ℕ ↪o ℕ\nh₁ : ∀ (m n : ℕ), m ≤ n → r ((Prod.fst ∘ f) (↑g₁ m)) ((Prod.fst ∘ f) (↑g₁ n))\nm n : ℕ\nhlt : m < n\nhle : r' ((Prod.snd ∘ f ∘ ↑g₁) m) ((Prod.snd ∘ f ∘ ↑g₁) n)\n⊢ ∃ m n, m < n ∧ (fun x y => r x.fst y.fst ∧ r' x.snd y.snd) (f m) (f n)", "tactic": "exact ⟨g₁ m, g₁ n, g₁.strictMono hlt, h₁ _ _ hlt.le, hle⟩" } ]
[ 374, 60 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 368, 11 ]
Mathlib/Algebra/BigOperators/Finsupp.lean
Finsupp.sum_ite_self_eq_aux
[ { "state_after": "α : Type u_1\nι : Type ?u.64782\nγ : Type ?u.64785\nA : Type ?u.64788\nB : Type ?u.64791\nC : Type ?u.64794\ninst✝⁷ : AddCommMonoid A\ninst✝⁶ : AddCommMonoid B\ninst✝⁵ : AddCommMonoid C\nt : ι → A → C\nh0 : ∀ (i : ι), t i 0 = 0\nh1 : ∀ (i : ι) (x y : A), t i (x + y) = t i x + t i y\ns : Finset α\nf✝ : α → ι →₀ A\ni : ι\ng : ι →₀ A\nk : ι → A → γ → B\nx : γ\nβ : Type ?u.67924\nM : Type ?u.67927\nM' : Type ?u.67930\nN✝ : Type ?u.67933\nP : Type ?u.67936\nG : Type ?u.67939\nH : Type ?u.67942\nR : Type ?u.67945\nS : Type ?u.67948\ninst✝⁴ : Zero M\ninst✝³ : Zero M'\ninst✝² : CommMonoid N✝\ninst✝¹ : DecidableEq α\nN : Type u_2\ninst✝ : AddCommMonoid N\nf : α →₀ N\na : α\n⊢ ↑f a = 0 → 0 = ↑f a", "state_before": "α : Type u_1\nι : Type ?u.64782\nγ : Type ?u.64785\nA : Type ?u.64788\nB : Type ?u.64791\nC : Type ?u.64794\ninst✝⁷ : AddCommMonoid A\ninst✝⁶ : AddCommMonoid B\ninst✝⁵ : AddCommMonoid C\nt : ι → A → C\nh0 : ∀ (i : ι), t i 0 = 0\nh1 : ∀ (i : ι) (x y : A), t i (x + y) = t i x + t i y\ns : Finset α\nf✝ : α → ι →₀ A\ni : ι\ng : ι →₀ A\nk : ι → A → γ → B\nx : γ\nβ : Type ?u.67924\nM : Type ?u.67927\nM' : Type ?u.67930\nN✝ : Type ?u.67933\nP : Type ?u.67936\nG : Type ?u.67939\nH : Type ?u.67942\nR : Type ?u.67945\nS : Type ?u.67948\ninst✝⁴ : Zero M\ninst✝³ : Zero M'\ninst✝² : CommMonoid N✝\ninst✝¹ : DecidableEq α\nN : Type u_2\ninst✝ : AddCommMonoid N\nf : α →₀ N\na : α\n⊢ (if a ∈ f.support then ↑f a else 0) = ↑f a", "tactic": "simp only [mem_support_iff, ne_eq, ite_eq_left_iff, not_not]" }, { "state_after": "no goals", "state_before": "α : Type u_1\nι : Type ?u.64782\nγ : Type ?u.64785\nA : Type ?u.64788\nB : Type ?u.64791\nC : Type ?u.64794\ninst✝⁷ : AddCommMonoid A\ninst✝⁶ : AddCommMonoid B\ninst✝⁵ : AddCommMonoid C\nt : ι → A → C\nh0 : ∀ (i : ι), t i 0 = 0\nh1 : ∀ (i : ι) (x y : A), t i (x + y) = t i x + t i y\ns : Finset α\nf✝ : α → ι →₀ A\ni : ι\ng : ι →₀ A\nk : ι → A → γ → B\nx : γ\nβ : Type ?u.67924\nM : Type ?u.67927\nM' : Type ?u.67930\nN✝ : Type ?u.67933\nP : Type ?u.67936\nG : Type ?u.67939\nH : Type ?u.67942\nR : Type ?u.67945\nS : Type ?u.67948\ninst✝⁴ : Zero M\ninst✝³ : Zero M'\ninst✝² : CommMonoid N✝\ninst✝¹ : DecidableEq α\nN : Type u_2\ninst✝ : AddCommMonoid N\nf : α →₀ N\na : α\n⊢ ↑f a = 0 → 0 = ↑f a", "tactic": "exact fun h ↦ h.symm" } ]
[ 134, 23 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 131, 1 ]
Mathlib/Algebra/DirectSum/Basic.lean
DirectSum.addHom_ext'
[]
[ 187, 47 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 185, 1 ]
Mathlib/Data/Multiset/Antidiagonal.lean
Multiset.prod_map_add
[ { "state_after": "case refine'_1\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns : Multiset α\nf g : α → β\n⊢ prod (map (fun a => f a + g a) 0) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal 0))\n\ncase refine'_2\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns : Multiset α\nf g : α → β\n⊢ ∀ ⦃a : α⦄ {s : Multiset α},\n prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s)) →\n prod (map (fun a => f a + g a) (a ::ₘ s)) =\n sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal (a ::ₘ s)))", "state_before": "α : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns : Multiset α\nf g : α → β\n⊢ prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s))", "tactic": "refine' s.induction_on _ _" }, { "state_after": "no goals", "state_before": "case refine'_1\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns : Multiset α\nf g : α → β\n⊢ prod (map (fun a => f a + g a) 0) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal 0))", "tactic": "simp only [map_zero, prod_zero, antidiagonal_zero, map_singleton, mul_one, sum_singleton]" }, { "state_after": "case refine'_2\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns✝ : Multiset α\nf g : α → β\na : α\ns : Multiset α\nih : prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s))\n⊢ prod (map (fun a => f a + g a) (a ::ₘ s)) =\n sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal (a ::ₘ s)))", "state_before": "case refine'_2\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns : Multiset α\nf g : α → β\n⊢ ∀ ⦃a : α⦄ {s : Multiset α},\n prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s)) →\n prod (map (fun a => f a + g a) (a ::ₘ s)) =\n sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal (a ::ₘ s)))", "tactic": "intro a s ih" }, { "state_after": "case refine'_2\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns✝ : Multiset α\nf g : α → β\na : α\ns : Multiset α\nih : prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s))\n⊢ sum (map (fun i => prod (map f i.fst) * (f a * prod (map g i.snd))) (antidiagonal s)) +\n sum (map (fun i => prod (map f i.fst) * (g a * prod (map g i.snd))) (antidiagonal s)) =\n sum (map (fun x => prod (map f x.fst) * (g a * prod (map g x.snd))) (antidiagonal s)) +\n sum (map (fun i => prod (map f i.fst) * (f a * prod (map g i.snd))) (antidiagonal s))", "state_before": "case refine'_2\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns✝ : Multiset α\nf g : α → β\na : α\ns : Multiset α\nih : prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s))\n⊢ prod (map (fun a => f a + g a) (a ::ₘ s)) =\n sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal (a ::ₘ s)))", "tactic": "simp only [map_cons, prod_cons, ih, sum_map_mul_left.symm, add_mul, mul_left_comm (f a),\n mul_left_comm (g a), sum_map_add, antidiagonal_cons, Prod_map, id_eq, map_add, map_map,\n Function.comp_apply, mul_assoc, sum_add]" }, { "state_after": "no goals", "state_before": "case refine'_2\nα : Type u_2\nβ : Type u_1\ninst✝ : CommSemiring β\ns✝ : Multiset α\nf g : α → β\na : α\ns : Multiset α\nih : prod (map (fun a => f a + g a) s) = sum (map (fun p => prod (map f p.fst) * prod (map g p.snd)) (antidiagonal s))\n⊢ sum (map (fun i => prod (map f i.fst) * (f a * prod (map g i.snd))) (antidiagonal s)) +\n sum (map (fun i => prod (map f i.fst) * (g a * prod (map g i.snd))) (antidiagonal s)) =\n sum (map (fun x => prod (map f x.fst) * (g a * prod (map g x.snd))) (antidiagonal s)) +\n sum (map (fun i => prod (map f i.fst) * (f a * prod (map g i.snd))) (antidiagonal s))", "tactic": "exact add_comm _ _" } ]
[ 118, 23 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 109, 1 ]
Mathlib/Computability/Partrec.lean
Computable.ofOption
[ { "state_after": "case some\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.37095\nσ : Type ?u.37098\ninst✝³ : Primcodable α\ninst✝² : Primcodable β\ninst✝¹ : Primcodable γ\ninst✝ : Primcodable σ\nf : α → Option β\nhf : Computable f\nn : ℕ\na : α\n⊢ ↑(Nat.ppred (encode (f a))) = map encode ↑(f a)", "state_before": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.37095\nσ : Type ?u.37098\ninst✝³ : Primcodable α\ninst✝² : Primcodable β\ninst✝¹ : Primcodable γ\ninst✝ : Primcodable σ\nf : α → Option β\nhf : Computable f\nn : ℕ\n⊢ (do\n let n ← Part.bind ↑(decode n) fun a => map encode (↑f a)\n ↑(Nat.ppred n)) =\n Part.bind ↑(decode n) fun a => map encode ((fun a => ↑(f a)) a)", "tactic": "cases' decode (α := α) n with a <;> simp" }, { "state_after": "no goals", "state_before": "case some\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.37095\nσ : Type ?u.37098\ninst✝³ : Primcodable α\ninst✝² : Primcodable β\ninst✝¹ : Primcodable γ\ninst✝ : Primcodable σ\nf : α → Option β\nhf : Computable f\nn : ℕ\na : α\n⊢ ↑(Nat.ppred (encode (f a))) = map encode ↑(f a)", "tactic": "cases' f a with b <;> simp" } ]
[ 293, 31 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 290, 1 ]
Mathlib/LinearAlgebra/Alternating.lean
AlternatingMap.domCoprod.summand_eq_zero_of_smul_invariant
[ { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\nσ : Perm (ιa ⊕ ιb)\n⊢ swap i j • Quotient.mk'' σ = Quotient.mk'' σ → ↑(summand a b (Quotient.mk'' σ)) v = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\n⊢ swap i j • σ = σ → ↑(summand a b σ) v = 0", "tactic": "refine Quotient.inductionOn' σ fun σ => ?_" }, { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\nσ : Perm (ιa ⊕ ιb)\n⊢ swap i j • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\nσ : Perm (ιa ⊕ ιb)\n⊢ swap i j • Quotient.mk'' σ = Quotient.mk'' σ → ↑(summand a b (Quotient.mk'' σ)) v = 0", "tactic": "dsimp only [Quotient.liftOn'_mk'', Quotient.map'_mk'', MultilinearMap.smul_apply,\n MultilinearMap.domDomCongr_apply, MultilinearMap.domCoprod_apply, domCoprod.summand]" }, { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\nσ : Perm (ιa ⊕ ιb)\nhσ : swap i j • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\nσ : Perm (ιa ⊕ ιb)\n⊢ swap i j • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "intro hσ" }, { "state_after": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inl.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιa) (val_1 : ιb),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιb) (val_1 : ιa),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\ni j : ιa ⊕ ιb\nhv : v i = v j\nhij : i ≠ j\nσ : Perm (ιa ⊕ ιb)\nhσ : swap i j • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "cases' hi : σ⁻¹ i with val val <;> cases' hj : σ⁻¹ j with val_1 val_1 <;>\n rw [Perm.inv_eq_iff_eq] at hi hj <;> substs hi hj <;> revert val val_1" }, { "state_after": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιb) (val_1 : ιa),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inl.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιa) (val_1 : ιb),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιb) (val_1 : ιa),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "case inl.inr =>\n intro i' j' _ _ hσ\n obtain ⟨⟨sl, sr⟩, hσ⟩ := QuotientGroup.leftRel_apply.mp (Quotient.exact' hσ)\n replace hσ := Equiv.congr_fun hσ (Sum.inl i')\n dsimp only at hσ\n rw [smul_eq_mul, ← mul_swap_eq_swap_mul, mul_inv_rev, swap_inv, inv_mul_cancel_right] at hσ\n simp at hσ" }, { "state_after": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιb) (val_1 : ιa),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "case inr.inl =>\n intro i' j' _ _ hσ\n obtain ⟨⟨sl, sr⟩, hσ⟩ := QuotientGroup.leftRel_apply.mp (Quotient.exact' hσ)\n replace hσ := Equiv.congr_fun hσ (Sum.inr i')\n dsimp only at hσ\n rw [smul_eq_mul, ← mul_swap_eq_swap_mul, mul_inv_rev, swap_inv, inv_mul_cancel_right] at hσ\n simp at hσ" }, { "state_after": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0\n\ncase inr.inr\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "case inr.inr =>\n intro i' j' hv hij _\n convert smul_zero (M := ℤˣ) (A := N₁ ⊗[R'] N₂) _\n convert TensorProduct.tmul_zero (R := R') (M := N₁) N₂ _\n exact AlternatingMap.map_eq_zero_of_eq _ _ hv fun hij' => hij (hij' ▸ rfl)" }, { "state_after": "no goals", "state_before": "case inl.inl\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "case inl.inl =>\n intro i' j' hv hij _\n convert smul_zero (M := ℤˣ) (A := N₁ ⊗[R'] N₂) _\n convert TensorProduct.zero_tmul (R := R') N₁ (N := N₂) _\n exact AlternatingMap.map_eq_zero_of_eq _ _ hv fun hij' => hij (hij' ▸ rfl)" }, { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιa) (val_1 : ιb),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "intro i' j' _ _ hσ" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(Perm.sumCongrHom ιa ιb) (sl, sr) = ((fun x x_1 => x • x_1) (swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j'))) σ)⁻¹ * σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "obtain ⟨⟨sl, sr⟩, hσ⟩ := QuotientGroup.leftRel_apply.mp (Quotient.exact' hσ)" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inl i') =\n ↑(((fun x x_1 => x • x_1) (swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j'))) σ)⁻¹ * σ) (Sum.inl i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(Perm.sumCongrHom ιa ιb) (sl, sr) = ((fun x x_1 => x • x_1) (swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j'))) σ)⁻¹ * σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "replace hσ := Equiv.congr_fun hσ (Sum.inl i')" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inl i') =\n ↑((swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • σ)⁻¹ * σ) (Sum.inl i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inl i') =\n ↑(((fun x x_1 => x • x_1) (swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j'))) σ)⁻¹ * σ) (Sum.inl i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "dsimp only at hσ" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inl i') = ↑(swap (Sum.inl i') (Sum.inr j')) (Sum.inl i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inl i') =\n ↑((swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • σ)⁻¹ * σ) (Sum.inl i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "rw [smul_eq_mul, ← mul_swap_eq_swap_mul, mul_inv_rev, swap_inv, inv_mul_cancel_right] at hσ" }, { "state_after": "no goals", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιa\nj' : ιb\nhv✝ : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inr j'))\nhij✝ : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inl i') = ↑(swap (Sum.inl i') (Sum.inr j')) (Sum.inl i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "simp at hσ" }, { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val : ιb) (val_1 : ιa),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "intro i' j' _ _ hσ" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(Perm.sumCongrHom ιa ιb) (sl, sr) = ((fun x x_1 => x • x_1) (swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j'))) σ)⁻¹ * σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "obtain ⟨⟨sl, sr⟩, hσ⟩ := QuotientGroup.leftRel_apply.mp (Quotient.exact' hσ)" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inr i') =\n ↑(((fun x x_1 => x • x_1) (swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j'))) σ)⁻¹ * σ) (Sum.inr i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(Perm.sumCongrHom ιa ιb) (sl, sr) = ((fun x x_1 => x • x_1) (swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j'))) σ)⁻¹ * σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "replace hσ := Equiv.congr_fun hσ (Sum.inr i')" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inr i') =\n ↑((swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • σ)⁻¹ * σ) (Sum.inr i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inr i') =\n ↑(((fun x x_1 => x • x_1) (swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j'))) σ)⁻¹ * σ) (Sum.inr i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "dsimp only at hσ" }, { "state_after": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inr i') = ↑(swap (Sum.inr i') (Sum.inl j')) (Sum.inr i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ :\n ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inr i') =\n ↑((swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • σ)⁻¹ * σ) (Sum.inr i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "rw [smul_eq_mul, ← mul_swap_eq_swap_mul, mul_inv_rev, swap_inv, inv_mul_cancel_right] at hσ" }, { "state_after": "no goals", "state_before": "case intro.mk\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' : ιb\nj' : ιa\nhv✝ : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inl j'))\nhij✝ : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\nsl : Perm ιa\nsr : Perm ιb\nhσ : ↑(↑(Perm.sumCongrHom ιa ιb) (sl, sr)) (Sum.inr i') = ↑(swap (Sum.inr i') (Sum.inl j')) (Sum.inr i')\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "simp at hσ" }, { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιb\nhv : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inr j'))\nhij : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιb),\n v (↑σ (Sum.inr val)) = v (↑σ (Sum.inr val_1)) →\n ↑σ (Sum.inr val) ≠ ↑σ (Sum.inr val_1) →\n swap (↑σ (Sum.inr val)) (↑σ (Sum.inr val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "intro i' j' hv hij _" }, { "state_after": "case h.e'_2.h.e'_6\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιb\nhv : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inr j'))\nhij : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ ((↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιb\nhv : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inr j'))\nhij : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "convert smul_zero (M := ℤˣ) (A := N₁ ⊗[R'] N₂) _" }, { "state_after": "case h.e'_2.h.e'_10\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιb\nhv : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inr j'))\nhij : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "case h.e'_2.h.e'_6\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιb\nhv : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inr j'))\nhij : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ ((↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "convert TensorProduct.tmul_zero (R := R') (M := N₁) N₂ _" }, { "state_after": "no goals", "state_before": "case h.e'_2.h.e'_10\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιb\nhv : v (↑σ (Sum.inr i')) = v (↑σ (Sum.inr j'))\nhij : ↑σ (Sum.inr i') ≠ ↑σ (Sum.inr j')\nhσ✝ : swap (↑σ (Sum.inr i')) (↑σ (Sum.inr j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "exact AlternatingMap.map_eq_zero_of_eq _ _ hv fun hij' => hij (hij' ▸ rfl)" }, { "state_after": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιa\nhv : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inl j'))\nhij : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\n⊢ ∀ (val val_1 : ιa),\n v (↑σ (Sum.inl val)) = v (↑σ (Sum.inl val_1)) →\n ↑σ (Sum.inl val) ≠ ↑σ (Sum.inl val_1) →\n swap (↑σ (Sum.inl val)) (↑σ (Sum.inl val_1)) • Quotient.mk'' σ = Quotient.mk'' σ →\n (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "intro i' j' hv hij _" }, { "state_after": "case h.e'_2.h.e'_6\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιa\nhv : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inl j'))\nhij : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ ((↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "state_before": "R : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιa\nhv : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inl j'))\nhij : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑Perm.sign σ • (↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "convert smul_zero (M := ℤˣ) (A := N₁ ⊗[R'] N₂) _" }, { "state_after": "case h.e'_2.h.e'_9\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιa\nhv : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inl j'))\nhij : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑↑a fun i => v (↑σ (Sum.inl i))) = 0", "state_before": "case h.e'_2.h.e'_6\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιa\nhv : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inl j'))\nhij : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ ((↑↑a fun i => v (↑σ (Sum.inl i))) ⊗ₜ[R'] ↑↑b fun i => v (↑σ (Sum.inr i))) = 0", "tactic": "convert TensorProduct.zero_tmul (R := R') N₁ (N := N₂) _" }, { "state_after": "no goals", "state_before": "case h.e'_2.h.e'_9\nR : Type ?u.948464\ninst✝²¹ : Semiring R\nM : Type ?u.948470\ninst✝²⁰ : AddCommMonoid M\ninst✝¹⁹ : Module R M\nN : Type ?u.948502\ninst✝¹⁸ : AddCommMonoid N\ninst✝¹⁷ : Module R N\nP : Type ?u.948532\ninst✝¹⁶ : AddCommMonoid P\ninst✝¹⁵ : Module R P\nM' : Type ?u.948562\ninst✝¹⁴ : AddCommGroup M'\ninst✝¹³ : Module R M'\nN' : Type ?u.948950\ninst✝¹² : AddCommGroup N'\ninst✝¹¹ : Module R N'\nι : Type ?u.949338\nι' : Type ?u.949341\nι'' : Type ?u.949344\nιa : Type u_4\nιb : Type u_6\ninst✝¹⁰ : Fintype ιa\ninst✝⁹ : Fintype ιb\nR' : Type u_1\nMᵢ : Type u_2\nN₁ : Type u_3\nN₂ : Type u_5\ninst✝⁸ : CommSemiring R'\ninst✝⁷ : AddCommGroup N₁\ninst✝⁶ : Module R' N₁\ninst✝⁵ : AddCommGroup N₂\ninst✝⁴ : Module R' N₂\ninst✝³ : AddCommMonoid Mᵢ\ninst✝² : Module R' Mᵢ\ninst✝¹ : DecidableEq ιa\ninst✝ : DecidableEq ιb\na : AlternatingMap R' Mᵢ N₁ ιa\nb : AlternatingMap R' Mᵢ N₂ ιb\nσ✝ : Perm.ModSumCongr ιa ιb\nv : ιa ⊕ ιb → Mᵢ\nσ : Perm (ιa ⊕ ιb)\ni' j' : ιa\nhv : v (↑σ (Sum.inl i')) = v (↑σ (Sum.inl j'))\nhij : ↑σ (Sum.inl i') ≠ ↑σ (Sum.inl j')\nhσ✝ : swap (↑σ (Sum.inl i')) (↑σ (Sum.inl j')) • Quotient.mk'' σ = Quotient.mk'' σ\n⊢ (↑↑a fun i => v (↑σ (Sum.inl i))) = 0", "tactic": "exact AlternatingMap.map_eq_zero_of_eq _ _ hv fun hij' => hij (hij' ▸ rfl)" } ]
[ 1047, 79 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1011, 1 ]
Mathlib/Order/GaloisConnection.lean
GaloisConnection.u_comm_of_l_comm
[]
[ 362, 49 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 356, 1 ]
Mathlib/Data/Nat/Log.lean
Nat.log_zero_right
[]
[ 77, 35 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 76, 1 ]
Mathlib/Algebra/BigOperators/Finsupp.lean
Finsupp.prod_sum_index
[]
[ 535, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 531, 1 ]
Mathlib/RingTheory/Subsemiring/Basic.lean
RingHom.restrict_apply
[]
[ 1137, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1136, 1 ]
Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean
Real.continuousAt_rpow_const
[ { "state_after": "x q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt ((fun p => p.fst ^ p.snd) ∘ fun y => (y, q)) x", "state_before": "x q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt (fun x => x ^ q) x", "tactic": "change ContinuousAt ((fun p : ℝ × ℝ => p.1 ^ p.2) ∘ fun y : ℝ => (y, q)) x" }, { "state_after": "case hg\nx q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt (fun p => p.fst ^ p.snd) (x, q)\n\ncase hf\nx q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt (fun y => (y, q)) x", "state_before": "x q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt ((fun p => p.fst ^ p.snd) ∘ fun y => (y, q)) x", "tactic": "apply ContinuousAt.comp" }, { "state_after": "no goals", "state_before": "case hg\nx q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt (fun p => p.fst ^ p.snd) (x, q)", "tactic": "exact continuousAt_rpow (x, q) h" }, { "state_after": "no goals", "state_before": "case hf\nx q : ℝ\nh : x ≠ 0 ∨ 0 < q\n⊢ ContinuousAt (fun y => (y, q)) x", "tactic": "exact (continuous_id'.prod_mk continuous_const).continuousAt" } ]
[ 268, 65 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 263, 1 ]
Std/Data/Array/Lemmas.lean
Array.back_eq_back?
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : Inhabited α\na : Array α\n⊢ back a = Option.getD (back? a) default", "tactic": "simp [back, back?]" } ]
[ 71, 21 ]
e68aa8f5fe47aad78987df45f99094afbcb5e936
https://github.com/leanprover/std4
[ 70, 9 ]
Mathlib/Data/Set/Pairwise/Basic.lean
Set.PairwiseDisjoint.mono
[]
[ 258, 28 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 257, 1 ]
Mathlib/Combinatorics/SetFamily/Shadow.lean
Finset.upShadow_empty
[]
[ 197, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 196, 1 ]
Mathlib/Topology/Algebra/Order/Field.lean
Filter.Tendsto.atTop_mul_neg
[ { "state_after": "𝕜 : Type u_1\nα : Type u_2\ninst✝² : LinearOrderedField 𝕜\ninst✝¹ : TopologicalSpace 𝕜\ninst✝ : OrderTopology 𝕜\nl : Filter α\nf g : α → 𝕜\nC : 𝕜\nhC : C < 0\nhf : Tendsto f l atTop\nhg : Tendsto g l (𝓝 C)\nthis : Tendsto (fun x => f x * -g x) l atTop\n⊢ Tendsto (fun x => f x * g x) l atBot", "state_before": "𝕜 : Type u_1\nα : Type u_2\ninst✝² : LinearOrderedField 𝕜\ninst✝¹ : TopologicalSpace 𝕜\ninst✝ : OrderTopology 𝕜\nl : Filter α\nf g : α → 𝕜\nC : 𝕜\nhC : C < 0\nhf : Tendsto f l atTop\nhg : Tendsto g l (𝓝 C)\n⊢ Tendsto (fun x => f x * g x) l atBot", "tactic": "have := hf.atTop_mul (neg_pos.2 hC) hg.neg" } ]
[ 83, 92 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 80, 1 ]
Mathlib/Analysis/Calculus/Deriv/Add.lean
hasDerivAtFilter_neg
[]
[ 243, 50 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 242, 1 ]
Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean
UniformFun.hasBasis_uniformity
[]
[ 313, 46 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 311, 11 ]
Mathlib/Data/Pi/Algebra.lean
Pi.prod_snd_fst
[]
[ 352, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 351, 1 ]
Mathlib/Data/Complex/Exponential.lean
Real.expNear_zero
[ { "state_after": "no goals", "state_before": "x r : ℝ\n⊢ expNear 0 x r = r", "tactic": "simp [expNear]" } ]
[ 1752, 68 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1752, 1 ]
Mathlib/Analysis/Normed/Group/Hom.lean
NormedAddGroupHom.antilipschitz_of_norm_ge
[ { "state_after": "no goals", "state_before": "V : Type ?u.211727\nV₁ : Type u_1\nV₂ : Type u_2\nV₃ : Type ?u.211736\ninst✝³ : SeminormedAddCommGroup V\ninst✝² : SeminormedAddCommGroup V₁\ninst✝¹ : SeminormedAddCommGroup V₂\ninst✝ : SeminormedAddCommGroup V₃\nf g : NormedAddGroupHom V₁ V₂\nK : ℝ≥0\nh : ∀ (x : V₁), ‖x‖ ≤ ↑K * ‖↑f x‖\nx y : V₁\n⊢ dist x y ≤ ↑K * dist (↑f x) (↑f y)", "tactic": "simpa only [dist_eq_norm, map_sub] using h (x - y)" } ]
[ 174, 100 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 173, 1 ]
Mathlib/LinearAlgebra/SesquilinearForm.lean
LinearMap.ortho_smul_right
[ { "state_after": "R : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\n⊢ ↑(↑B x) y = 0 ↔ ↑(↑B x) (a • y) = 0", "state_before": "R : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\n⊢ IsOrtho B x y ↔ IsOrtho B x (a • y)", "tactic": "dsimp only [IsOrtho]" }, { "state_after": "case mp\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑(↑B x) y = 0\n⊢ ↑(↑B x) (a • y) = 0\n\ncase mpr\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑(↑B x) (a • y) = 0\n⊢ ↑(↑B x) y = 0", "state_before": "R : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\n⊢ ↑(↑B x) y = 0 ↔ ↑(↑B x) (a • y) = 0", "tactic": "constructor <;> intro H" }, { "state_after": "no goals", "state_before": "case mp\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑(↑B x) y = 0\n⊢ ↑(↑B x) (a • y) = 0", "tactic": "rw [map_smulₛₗ, H, smul_zero]" }, { "state_after": "case mpr\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑I₂ a = 0 ∨ ↑(↑B x) y = 0\n⊢ ↑(↑B x) y = 0", "state_before": "case mpr\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑(↑B x) (a • y) = 0\n⊢ ↑(↑B x) y = 0", "tactic": "rw [map_smulₛₗ, smul_eq_zero] at H" }, { "state_after": "case mpr.inl\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑I₂ a = 0\n⊢ ↑(↑B x) y = 0\n\ncase mpr.inr\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑(↑B x) y = 0\n⊢ ↑(↑B x) y = 0", "state_before": "case mpr\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑I₂ a = 0 ∨ ↑(↑B x) y = 0\n⊢ ↑(↑B x) y = 0", "tactic": "cases' H with H H" }, { "state_after": "case mpr.inl\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : a = 0\n⊢ ↑(↑B x) y = 0", "state_before": "case mpr.inl\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑I₂ a = 0\n⊢ ↑(↑B x) y = 0", "tactic": "simp at H" }, { "state_after": "case mpr.inl.h\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : a = 0\n⊢ False", "state_before": "case mpr.inl\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : a = 0\n⊢ ↑(↑B x) y = 0", "tactic": "exfalso" }, { "state_after": "no goals", "state_before": "case mpr.inl.h\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : a = 0\n⊢ False", "tactic": "exact ha H" }, { "state_after": "no goals", "state_before": "case mpr.inr\nR : Type ?u.48188\nR₁ : Type ?u.48191\nR₂ : Type ?u.48194\nR₃ : Type ?u.48197\nM : Type ?u.48200\nM₁ : Type ?u.48203\nM₂ : Type ?u.48206\nMₗ₁ : Type ?u.48209\nMₗ₁' : Type ?u.48212\nMₗ₂ : Type ?u.48215\nMₗ₂' : Type ?u.48218\nK : Type u_2\nK₁ : Type u_1\nK₂ : Type u_5\nV : Type ?u.48230\nV₁ : Type u_3\nV₂ : Type u_4\nn : Type ?u.48239\ninst✝⁶ : Field K\ninst✝⁵ : Field K₁\ninst✝⁴ : AddCommGroup V₁\ninst✝³ : Module K₁ V₁\ninst✝² : Field K₂\ninst✝¹ : AddCommGroup V₂\ninst✝ : Module K₂ V₂\nI₁ : K₁ →+* K\nI₂ : K₂ →+* K\nI₁' : K₁ →+* K\nJ₁ J₂ : K →+* K\nB : V₁ →ₛₗ[I₁] V₂ →ₛₗ[I₂] K\nx : V₁\ny : V₂\na : K₂\nha : a ≠ 0\nH : ↑(↑B x) y = 0\n⊢ ↑(↑B x) y = 0", "tactic": "exact H" } ]
[ 138, 14 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 128, 1 ]
Mathlib/Algebra/Hom/Group.lean
MonoidHom.mk_coe
[]
[ 791, 56 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 790, 1 ]
Mathlib/Data/List/Perm.lean
List.subset_cons_diff
[]
[ 831, 27 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 830, 1 ]
Mathlib/Algebra/BigOperators/Finsupp.lean
MonoidHom.finsupp_prod_apply
[]
[ 270, 36 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 268, 1 ]
Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean
AffineEquiv.trans_assoc
[]
[ 356, 19 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 354, 1 ]
Mathlib/Algebra/Hom/Centroid.lean
CentroidHom.coe_toAddMonoidHom
[]
[ 123, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 122, 1 ]
Mathlib/Order/Filter/Bases.lean
Filter.HasBasis.inf_principal
[ { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type ?u.43930\nγ : Type ?u.43933\nι : Sort u_2\nι' : Sort ?u.43939\nl l' : Filter α\np : ι → Prop\ns : ι → Set α\nt✝ : Set α\ni : ι\np' : ι' → Prop\ns'✝ : ι' → Set α\ni' : ι'\nhl : HasBasis l p s\ns' t : Set α\n⊢ t ∈ l ⊓ 𝓟 s' ↔ ∃ i, p i ∧ s i ∩ s' ⊆ t", "tactic": "simp only [mem_inf_principal, hl.mem_iff, subset_def, mem_setOf_eq, mem_inter_iff, and_imp]" } ]
[ 623, 97 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 620, 1 ]
Mathlib/Algebra/Order/Pi.lean
Function.const_lt_one
[]
[ 157, 30 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 156, 1 ]
Mathlib/Order/Interval.lean
Interval.coe_top
[]
[ 503, 14 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 502, 1 ]
Mathlib/RingTheory/DedekindDomain/PID.lean
IsDedekindDomain.isPrincipalIdealRing_localization_over_prime
[ { "state_after": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\n⊢ IsPrincipalIdealRing Sₚ", "state_before": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\n⊢ IsPrincipalIdealRing Sₚ", "tactic": "letI := Classical.decEq (Ideal Sₚ)" }, { "state_after": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis✝ : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\nthis : DecidablePred fun P => IsPrime P := Classical.decPred fun P => IsPrime P\n⊢ IsPrincipalIdealRing Sₚ", "state_before": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\n⊢ IsPrincipalIdealRing Sₚ", "tactic": "letI := Classical.decPred fun P : Ideal Sₚ => P.IsPrime" }, { "state_after": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis✝ : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\nthis : DecidablePred fun P => IsPrime P := Classical.decPred fun P => IsPrime P\nP : Ideal Sₚ\n⊢ P ∈ Finset.filter (fun P => IsPrime P) ({⊥} ∪ Multiset.toFinset (normalizedFactors (map (algebraMap R Sₚ) p))) ↔\n P ∈ {I | IsPrime I}", "state_before": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis✝ : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\nthis : DecidablePred fun P => IsPrime P := Classical.decPred fun P => IsPrime P\n⊢ IsPrincipalIdealRing Sₚ", "tactic": "refine'\n IsPrincipalIdealRing.of_finite_primes\n (Set.Finite.ofFinset\n (Finset.filter (fun P => P.IsPrime)\n ({⊥} ∪ (normalizedFactors (Ideal.map (algebraMap R Sₚ) p)).toFinset))\n fun P => _)" }, { "state_after": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis✝ : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\nthis : DecidablePred fun P => IsPrime P := Classical.decPred fun P => IsPrime P\nP : Ideal Sₚ\n⊢ (P = ⊥ ∨ P ∈ normalizedFactors (map (algebraMap R Sₚ) p)) ∧ IsPrime P ↔ IsPrime P", "state_before": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis✝ : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\nthis : DecidablePred fun P => IsPrime P := Classical.decPred fun P => IsPrime P\nP : Ideal Sₚ\n⊢ P ∈ Finset.filter (fun P => IsPrime P) ({⊥} ∪ Multiset.toFinset (normalizedFactors (map (algebraMap R Sₚ) p))) ↔\n P ∈ {I | IsPrime I}", "tactic": "rw [Finset.mem_filter, Finset.mem_union, Finset.mem_singleton, Set.mem_setOf,\n Multiset.mem_toFinset]" }, { "state_after": "no goals", "state_before": "R : Type ?u.282964\ninst✝¹⁵ : CommRing R\ninst✝¹⁴ : IsDomain R\ninst✝¹³ : IsDedekindDomain R\nS : Type ?u.283172\ninst✝¹² : CommRing S\ninst✝¹¹ : IsDomain S\ninst✝¹⁰ : Algebra R S\ninst✝⁹ : Module.Free R S\ninst✝⁸ : Module.Finite R S\np : Ideal R\nhp0 : p ≠ ⊥\ninst✝⁷ : IsPrime p\nSₚ : Type u_1\ninst✝⁶ : CommRing Sₚ\ninst✝⁵ : Algebra S Sₚ\ninst✝⁴ : IsLocalization (Algebra.algebraMapSubmonoid S (primeCompl p)) Sₚ\ninst✝³ : Algebra R Sₚ\ninst✝² : IsScalarTower R S Sₚ\ninst✝¹ : IsDomain Sₚ\ninst✝ : IsDedekindDomain Sₚ\nthis✝ : DecidableEq (Ideal Sₚ) := Classical.decEq (Ideal Sₚ)\nthis : DecidablePred fun P => IsPrime P := Classical.decPred fun P => IsPrime P\nP : Ideal Sₚ\n⊢ (P = ⊥ ∨ P ∈ normalizedFactors (map (algebraMap R Sₚ) p)) ∧ IsPrime P ↔ IsPrime P", "tactic": "exact\n and_iff_right_of_imp fun hP =>\n or_iff_not_imp_left.mpr (IsLocalization.OverPrime.mem_normalizedFactors_of_isPrime S p hp0 hP)" } ]
[ 273, 101 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 259, 1 ]
Mathlib/Data/List/Rotate.lean
List.rotate_rotate
[ { "state_after": "no goals", "state_before": "α : Type u\nl : List α\nn m : ℕ\n⊢ rotate (rotate l n) m = rotate l (n + m)", "tactic": "rw [rotate_eq_rotate', rotate_eq_rotate', rotate_eq_rotate', rotate'_rotate']" } ]
[ 163, 80 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 162, 1 ]
Mathlib/Algebra/Free.lean
FreeSemigroup.head_mul
[]
[ 475, 66 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 475, 1 ]
Mathlib/Order/Filter/Lift.lean
Filter.lift'_pure
[ { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type u_2\nγ : Type ?u.36150\nι : Sort ?u.36153\nf f₁ f₂ : Filter α\nh h₁ h₂ : Set α → Set β\na : α\nhh : Monotone h\n⊢ Filter.lift' (pure a) h = 𝓟 (h {a})", "tactic": "rw [← principal_singleton, lift'_principal hh]" } ]
[ 324, 49 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 323, 1 ]
Mathlib/Logic/Embedding/Basic.lean
Function.Embedding.toFun_eq_coe
[]
[ 112, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 111, 1 ]
Mathlib/Order/Filter/Basic.lean
Filter.seq_eq_filter_seq
[]
[ 2695, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2693, 1 ]
Mathlib/Dynamics/OmegaLimit.lean
mem_omegaLimit_singleton_iff_map_cluster_point
[ { "state_after": "no goals", "state_before": "τ : Type u_2\nα : Type u_3\nβ : Type u_1\nι : Type ?u.31315\ninst✝ : TopologicalSpace β\nf : Filter τ\nϕ : τ → α → β\ns s₁ s₂ : Set α\nx : α\ny : β\n⊢ y ∈ ω f ϕ {x} ↔ MapClusterPt y f fun t => ϕ t x", "tactic": "simp_rw [mem_omegaLimit_iff_frequently, mapClusterPt_iff, singleton_inter_nonempty, mem_preimage]" } ]
[ 160, 100 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 158, 1 ]
Mathlib/RepresentationTheory/Action.lean
Action.id_hom
[]
[ 153, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 152, 1 ]
Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean
measurable_cInf
[]
[ 1364, 55 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1361, 1 ]
Mathlib/Order/Basic.lean
lt_of_eq_of_lt'
[]
[ 203, 22 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 202, 1 ]
Mathlib/Data/Set/Pairwise/Basic.lean
Set.pairwise_insert_of_symmetric_of_not_mem
[ { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type ?u.11936\nγ : Type ?u.11939\nι : Type ?u.11942\nι' : Type ?u.11945\nr p q : α → α → Prop\nf g : ι → α\ns t u : Set α\na b : α\nhr : Symmetric r\nha : ¬a ∈ s\n⊢ Set.Pairwise (insert a s) r ↔ Set.Pairwise s r ∧ ∀ (b : α), b ∈ s → r a b", "tactic": "simp only [pairwise_insert_of_not_mem ha, hr.iff a, and_self_iff]" } ]
[ 183, 68 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 181, 1 ]
Mathlib/RingTheory/IntegralClosure.lean
IsIntegral.multiset_prod
[]
[ 647, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 645, 1 ]
Mathlib/Algebra/Star/Basic.lean
star_eq_zero
[]
[ 287, 31 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 286, 1 ]
Mathlib/Algebra/Hom/Centroid.lean
CentroidHom.nsmul_apply
[]
[ 341, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 340, 1 ]
Mathlib/Control/Functor/Multivariate.lean
MvFunctor.id_map
[]
[ 110, 27 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 109, 1 ]
Mathlib/SetTheory/Ordinal/Arithmetic.lean
Ordinal.omega_pos
[]
[ 2413, 17 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2412, 1 ]
Mathlib/Order/Atoms.lean
GaloisCoinsertion.isCoatom_of_l_top
[]
[ 771, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 769, 1 ]
Mathlib/Data/List/Sort.lean
List.Sorted.lt_of_le
[]
[ 54, 42 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 52, 11 ]
Mathlib/Topology/Constructions.lean
embedding_sigma_map
[ { "state_after": "no goals", "state_before": "α : Type u\nβ : Type v\nγ : Type ?u.534439\nδ : Type ?u.534442\nε : Type ?u.534445\nζ : Type ?u.534448\nι : Type u_1\nκ : Type u_2\nσ : ι → Type u_3\nτ : κ → Type u_4\ninst✝² : (i : ι) → TopologicalSpace (σ i)\ninst✝¹ : (k : κ) → TopologicalSpace (τ k)\ninst✝ : TopologicalSpace α\nf₁ : ι → κ\nf₂ : (i : ι) → σ i → τ (f₁ i)\nh : Injective f₁\n⊢ _root_.Embedding (Sigma.map f₁ f₂) ↔ ∀ (i : ι), _root_.Embedding (f₂ i)", "tactic": "simp only [embedding_iff, Injective.sigma_map, inducing_sigma_map h, forall_and, h.sigma_map_iff]" } ]
[ 1566, 100 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1564, 1 ]
Mathlib/Analysis/Calculus/FDeriv/Basic.lean
fderivWithin_univ
[]
[ 649, 52 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 648, 1 ]
Mathlib/Algebra/Hom/GroupAction.lean
MulSemiringActionHom.map_sub
[]
[ 525, 16 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 524, 11 ]
Mathlib/GroupTheory/Perm/Fin.lean
Fin.cycleRange_last
[ { "state_after": "case H.h\nn : ℕ\ni : Fin (n + 1)\n⊢ ↑(↑(cycleRange (last n)) i) = ↑(↑(finRotate (n + 1)) i)", "state_before": "n : ℕ\n⊢ cycleRange (last n) = finRotate (n + 1)", "tactic": "ext i" }, { "state_after": "no goals", "state_before": "case H.h\nn : ℕ\ni : Fin (n + 1)\n⊢ ↑(↑(cycleRange (last n)) i) = ↑(↑(finRotate (n + 1)) i)", "tactic": "rw [coe_cycleRange_of_le (le_last _), coe_finRotate]" } ]
[ 238, 55 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 236, 1 ]
Mathlib/Data/Nat/Factors.lean
Nat.factors_subset_of_dvd
[]
[ 238, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 237, 1 ]
Mathlib/Combinatorics/SimpleGraph/Connectivity.lean
SimpleGraph.Walk.tail_support_append
[ { "state_after": "no goals", "state_before": "V : Type u\nV' : Type v\nV'' : Type w\nG : SimpleGraph V\nG' : SimpleGraph V'\nG'' : SimpleGraph V''\nu v w : V\np : Walk G u v\np' : Walk G v w\n⊢ List.tail (support (append p p')) = List.tail (support p) ++ List.tail (support p')", "tactic": "rw [support_append, List.tail_append_of_ne_nil _ _ (support_ne_nil _)]" } ]
[ 567, 73 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 565, 1 ]
Mathlib/Geometry/Manifold/LocalInvariantProperties.lean
StructureGroupoid.LocalInvariantProp.liftPropOn_chart_symm
[]
[ 529, 73 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 527, 1 ]
Mathlib/Data/Set/Intervals/Monotone.lean
MonotoneOn.Ici
[]
[ 45, 34 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 44, 11 ]
Mathlib/RingTheory/NonZeroDivisors.lean
le_nonZeroDivisors_of_noZeroDivisors
[]
[ 143, 37 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 140, 1 ]
Mathlib/Data/Rat/NNRat.lean
NNRat.coe_mk
[]
[ 95, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 94, 1 ]
Mathlib/LinearAlgebra/AffineSpace/Ordered.lean
lineMap_lt_map_iff_slope_lt_slope_left
[]
[ 239, 66 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 237, 1 ]
Mathlib/Data/Set/Countable.lean
Set.Countable.union
[]
[ 220, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 219, 1 ]
Mathlib/Algebra/Group/Pi.lean
Pi.single_mul_right_apply
[]
[ 523, 91 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 521, 1 ]
Mathlib/Topology/StoneCech.lean
denseInducing_pure
[]
[ 146, 50 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 144, 1 ]
Mathlib/GroupTheory/FreeGroup.lean
FreeGroup.Red.exact
[]
[ 668, 51 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 665, 1 ]
Mathlib/Order/JordanHolder.lean
CompositionSeries.toList_injective
[ { "state_after": "X : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₁ s₂ : CompositionSeries X\nh : List.ofFn s₁.series = List.ofFn s₂.series\nh₁ : s₁.length = s₂.length\n⊢ s₁ = s₂", "state_before": "X : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₁ s₂ : CompositionSeries X\nh : List.ofFn s₁.series = List.ofFn s₂.series\n⊢ s₁ = s₂", "tactic": "have h₁ : s₁.length = s₂.length :=\n Nat.succ_injective\n ((List.length_ofFn s₁).symm.trans <| (congr_arg List.length h).trans <| List.length_ofFn s₂)" }, { "state_after": "X : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₁ s₂ : CompositionSeries X\nh : List.ofFn s₁.series = List.ofFn s₂.series\nh₁ : s₁.length = s₂.length\nh₂ :\n ∀ (i : Fin (Nat.succ s₁.length)),\n series s₁ i = series s₂ (↑(Fin.cast (_ : Nat.succ s₁.length = Nat.succ s₂.length)) i)\n⊢ s₁ = s₂", "state_before": "X : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₁ s₂ : CompositionSeries X\nh : List.ofFn s₁.series = List.ofFn s₂.series\nh₁ : s₁.length = s₂.length\n⊢ s₁ = s₂", "tactic": "have h₂ : ∀ i : Fin s₁.length.succ, s₁ i = s₂ (Fin.cast (congr_arg Nat.succ h₁) i) :=\n congr_fun <| List.ofFn_injective <| h.trans <| List.ofFn_congr (congr_arg Nat.succ h₁).symm _" }, { "state_after": "case mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₂ : CompositionSeries X\nlength✝ : ℕ\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn { length := length✝, series := series✝, step' := step'✝ }.series = List.ofFn s₂.series\nh₁ : { length := length✝, series := series✝, step' := step'✝ }.length = s₂.length\nh₂ :\n ∀ (i : Fin (Nat.succ { length := length✝, series := series✝, step' := step'✝ }.length)),\n series { length := length✝, series := series✝, step' := step'✝ } i =\n series s₂\n (↑(Fin.cast\n (_ : Nat.succ { length := length✝, series := series✝, step' := step'✝ }.length = Nat.succ s₂.length))\n i)\n⊢ { length := length✝, series := series✝, step' := step'✝ } = s₂", "state_before": "X : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₁ s₂ : CompositionSeries X\nh : List.ofFn s₁.series = List.ofFn s₂.series\nh₁ : s₁.length = s₂.length\nh₂ :\n ∀ (i : Fin (Nat.succ s₁.length)),\n series s₁ i = series s₂ (↑(Fin.cast (_ : Nat.succ s₁.length = Nat.succ s₂.length)) i)\n⊢ s₁ = s₂", "tactic": "cases s₁" }, { "state_after": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝¹ : ℕ\nseries✝¹ : Fin (length✝¹ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝¹), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nlength✝ : ℕ\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh :\n List.ofFn { length := length✝¹, series := series✝¹, step' := step'✝¹ }.series =\n List.ofFn { length := length✝, series := series✝, step' := step'✝ }.series\nh₁ :\n { length := length✝¹, series := series✝¹, step' := step'✝¹ }.length =\n { length := length✝, series := series✝, step' := step'✝ }.length\nh₂ :\n ∀ (i : Fin (Nat.succ { length := length✝¹, series := series✝¹, step' := step'✝¹ }.length)),\n series { length := length✝¹, series := series✝¹, step' := step'✝¹ } i =\n series { length := length✝, series := series✝, step' := step'✝ }\n (↑(Fin.cast\n (_ :\n Nat.succ { length := length✝¹, series := series✝¹, step' := step'✝¹ }.length =\n Nat.succ { length := length✝, series := series✝, step' := step'✝ }.length))\n i)\n⊢ { length := length✝¹, series := series✝¹, step' := step'✝¹ } =\n { length := length✝, series := series✝, step' := step'✝ }", "state_before": "case mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\ns₂ : CompositionSeries X\nlength✝ : ℕ\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn { length := length✝, series := series✝, step' := step'✝ }.series = List.ofFn s₂.series\nh₁ : { length := length✝, series := series✝, step' := step'✝ }.length = s₂.length\nh₂ :\n ∀ (i : Fin (Nat.succ { length := length✝, series := series✝, step' := step'✝ }.length)),\n series { length := length✝, series := series✝, step' := step'✝ } i =\n series s₂\n (↑(Fin.cast\n (_ : Nat.succ { length := length✝, series := series✝, step' := step'✝ }.length = Nat.succ s₂.length))\n i)\n⊢ { length := length✝, series := series✝, step' := step'✝ } = s₂", "tactic": "cases s₂" }, { "state_after": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝¹ : ℕ\nseries✝¹ : Fin (length✝¹ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝¹), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nlength✝ : ℕ\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₁ : length✝¹ = length✝\nh₂ : ∀ (i : Fin (Nat.succ length✝¹)), series✝¹ i = series✝ (↑(Fin.cast (_ : Nat.succ length✝¹ = Nat.succ length✝)) i)\n⊢ { length := length✝¹, series := series✝¹, step' := step'✝¹ } =\n { length := length✝, series := series✝, step' := step'✝ }", "state_before": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝¹ : ℕ\nseries✝¹ : Fin (length✝¹ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝¹), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nlength✝ : ℕ\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh :\n List.ofFn { length := length✝¹, series := series✝¹, step' := step'✝¹ }.series =\n List.ofFn { length := length✝, series := series✝, step' := step'✝ }.series\nh₁ :\n { length := length✝¹, series := series✝¹, step' := step'✝¹ }.length =\n { length := length✝, series := series✝, step' := step'✝ }.length\nh₂ :\n ∀ (i : Fin (Nat.succ { length := length✝¹, series := series✝¹, step' := step'✝¹ }.length)),\n series { length := length✝¹, series := series✝¹, step' := step'✝¹ } i =\n series { length := length✝, series := series✝, step' := step'✝ }\n (↑(Fin.cast\n (_ :\n Nat.succ { length := length✝¹, series := series✝¹, step' := step'✝¹ }.length =\n Nat.succ { length := length✝, series := series✝, step' := step'✝ }.length))\n i)\n⊢ { length := length✝¹, series := series✝¹, step' := step'✝¹ } =\n { length := length✝, series := series✝, step' := step'✝ }", "tactic": "dsimp at h h₁ h₂" }, { "state_after": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝ : ℕ\nseries✝¹ : Fin (length✝ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₂ : ∀ (i : Fin (Nat.succ length✝)), series✝¹ i = series✝ (↑(Fin.cast (_ : Nat.succ length✝ = Nat.succ length✝)) i)\n⊢ { length := length✝, series := series✝¹, step' := step'✝¹ } =\n { length := length✝, series := series✝, step' := step'✝ }", "state_before": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝¹ : ℕ\nseries✝¹ : Fin (length✝¹ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝¹), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nlength✝ : ℕ\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₁ : length✝¹ = length✝\nh₂ : ∀ (i : Fin (Nat.succ length✝¹)), series✝¹ i = series✝ (↑(Fin.cast (_ : Nat.succ length✝¹ = Nat.succ length✝)) i)\n⊢ { length := length✝¹, series := series✝¹, step' := step'✝¹ } =\n { length := length✝, series := series✝, step' := step'✝ }", "tactic": "subst h₁" }, { "state_after": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝ : ℕ\nseries✝¹ : Fin (length✝ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₂ : ∀ (i : Fin (Nat.succ length✝)), series✝¹ i = series✝ (↑(Fin.cast (_ : Nat.succ length✝ = Nat.succ length✝)) i)\n⊢ series✝¹ = series✝", "state_before": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝ : ℕ\nseries✝¹ : Fin (length✝ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₂ : ∀ (i : Fin (Nat.succ length✝)), series✝¹ i = series✝ (↑(Fin.cast (_ : Nat.succ length✝ = Nat.succ length✝)) i)\n⊢ { length := length✝, series := series✝¹, step' := step'✝¹ } =\n { length := length✝, series := series✝, step' := step'✝ }", "tactic": "simp only [mk.injEq, heq_eq_eq, true_and]" }, { "state_after": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝ : ℕ\nseries✝¹ : Fin (length✝ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₂ : ∀ (i : Fin (Nat.succ length✝)), series✝¹ i = series✝ (↑(OrderIso.refl (Fin (Nat.succ length✝))) i)\n⊢ series✝¹ = series✝", "state_before": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝ : ℕ\nseries✝¹ : Fin (length✝ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₂ : ∀ (i : Fin (Nat.succ length✝)), series✝¹ i = series✝ (↑(Fin.cast (_ : Nat.succ length✝ = Nat.succ length✝)) i)\n⊢ series✝¹ = series✝", "tactic": "simp only [Fin.cast_refl] at h₂" }, { "state_after": "no goals", "state_before": "case mk.mk\nX : Type u\ninst✝¹ : Lattice X\ninst✝ : JordanHolderLattice X\nlength✝ : ℕ\nseries✝¹ : Fin (length✝ + 1) → X\nstep'✝¹ : ∀ (i : Fin length✝), IsMaximal (series✝¹ (↑Fin.castSucc i)) (series✝¹ (Fin.succ i))\nseries✝ : Fin (length✝ + 1) → X\nstep'✝ : ∀ (i : Fin length✝), IsMaximal (series✝ (↑Fin.castSucc i)) (series✝ (Fin.succ i))\nh : List.ofFn series✝¹ = List.ofFn series✝\nh₂ : ∀ (i : Fin (Nat.succ length✝)), series✝¹ i = series✝ (↑(OrderIso.refl (Fin (Nat.succ length✝))) i)\n⊢ series✝¹ = series✝", "tactic": "exact funext h₂" } ]
[ 245, 18 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 227, 1 ]
Mathlib/CategoryTheory/MorphismProperty.lean
CategoryTheory.MorphismProperty.isomorphisms.iff
[ { "state_after": "no goals", "state_before": "C : Type u\ninst✝¹ : Category C\nD : Type ?u.59249\ninst✝ : Category D\nX Y : C\nf : X ⟶ Y\n⊢ isomorphisms C f ↔ IsIso f", "tactic": "rfl" } ]
[ 404, 66 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 404, 1 ]
Mathlib/Analysis/ODE/PicardLindelof.lean
PicardLindelof.proj_of_mem
[ { "state_after": "no goals", "state_before": "E : Type u_1\ninst✝¹ : NormedAddCommGroup E\ninst✝ : NormedSpace ℝ E\nv : PicardLindelof E\nt : ℝ\nht : t ∈ Icc v.tMin v.tMax\n⊢ ↑(proj v t) = t", "tactic": "simp only [proj, projIcc_of_mem v.tMin_le_tMax ht]" } ]
[ 152, 53 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 151, 1 ]
Std/Data/List/Lemmas.lean
List.isPrefix.filter
[ { "state_after": "case intro\nα : Type u_1\np : α → Bool\nl₁ xs : List α\n⊢ List.filter p l₁ <+: List.filter p (l₁ ++ xs)", "state_before": "α : Type u_1\np : α → Bool\nl₁ l₂ : List α\nh : l₁ <+: l₂\n⊢ List.filter p l₁ <+: List.filter p l₂", "tactic": "obtain ⟨xs, rfl⟩ := h" }, { "state_after": "case intro\nα : Type u_1\np : α → Bool\nl₁ xs : List α\n⊢ List.filter p l₁ <+: List.filter p l₁ ++ List.filter p xs", "state_before": "case intro\nα : Type u_1\np : α → Bool\nl₁ xs : List α\n⊢ List.filter p l₁ <+: List.filter p (l₁ ++ xs)", "tactic": "rw [filter_append]" }, { "state_after": "no goals", "state_before": "case intro\nα : Type u_1\np : α → Bool\nl₁ xs : List α\n⊢ List.filter p l₁ <+: List.filter p l₁ ++ List.filter p xs", "tactic": "apply prefix_append" } ]
[ 1739, 42 ]
e68aa8f5fe47aad78987df45f99094afbcb5e936
https://github.com/leanprover/std4
[ 1736, 1 ]
Mathlib/Algebra/Group/Semiconj.lean
SemiconjBy.units_val_iff
[]
[ 165, 28 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 164, 1 ]
Mathlib/Order/LocallyFinite.lean
Ico_toDual
[ { "state_after": "α : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\n⊢ Ico (↑toDual a) (↑toDual b) = Ioc b a", "state_before": "α : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\n⊢ Ico (↑toDual a) (↑toDual b) = map (Equiv.toEmbedding toDual) (Ioc b a)", "tactic": "refine' Eq.trans _ map_refl.symm" }, { "state_after": "case a\nα : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\nc : (fun x => αᵒᵈ) a\n⊢ c ∈ Ico (↑toDual a) (↑toDual b) ↔ c ∈ Ioc b a", "state_before": "α : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\n⊢ Ico (↑toDual a) (↑toDual b) = Ioc b a", "tactic": "ext c" }, { "state_after": "case a\nα : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\nc : (fun x => αᵒᵈ) a\n⊢ ↑toDual a ≤ c ∧ c < ↑toDual b ↔ b < c ∧ c ≤ a", "state_before": "case a\nα : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\nc : (fun x => αᵒᵈ) a\n⊢ c ∈ Ico (↑toDual a) (↑toDual b) ↔ c ∈ Ioc b a", "tactic": "rw [mem_Ico, mem_Ioc (α := α)]" }, { "state_after": "no goals", "state_before": "case a\nα : Type u_1\nβ : Type ?u.112926\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : LocallyFiniteOrder α\na b : α\nc : (fun x => αᵒᵈ) a\n⊢ ↑toDual a ≤ c ∧ c < ↑toDual b ↔ b < c ∧ c ≤ a", "tactic": "exact and_comm" } ]
[ 838, 17 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 834, 1 ]
Mathlib/Logic/Equiv/Fin.lean
Fin.snoc_eq_cons_rotate
[ { "state_after": "case h.mk\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "state_before": "m n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\n⊢ snoc v a = fun i => cons a v (↑(finRotate (n + 1)) i)", "tactic": "ext ⟨i, h⟩" }, { "state_after": "case pos\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : i < n\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })\n\ncase neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : ¬i < n\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "state_before": "case h.mk\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "tactic": "by_cases h' : i < n" }, { "state_after": "case pos\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : i < n\n⊢ _root_.cast (_ : α = α) (v (castLT { val := i, isLt := h } h')) =\n cases a v { val := i + 1, isLt := (_ : Nat.succ i < Nat.succ n) }", "state_before": "case pos\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : i < n\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "tactic": "rw [finRotate_of_lt h', Fin.snoc, Fin.cons, dif_pos h']" }, { "state_after": "no goals", "state_before": "case pos\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : i < n\n⊢ _root_.cast (_ : α = α) (v (castLT { val := i, isLt := h } h')) =\n cases a v { val := i + 1, isLt := (_ : Nat.succ i < Nat.succ n) }", "tactic": "rfl" }, { "state_after": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : ¬i < n\nh'' : n = i\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "state_before": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : ¬i < n\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "tactic": "have h'' : n = i := by\n simp only [not_lt] at h'\n exact (Nat.eq_of_le_of_lt_succ h' h).symm" }, { "state_after": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\nh : n < n + 1\nh' : ¬n < n\n⊢ snoc v a { val := n, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := n, isLt := h })", "state_before": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : ¬i < n\nh'' : n = i\n⊢ snoc v a { val := i, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := i, isLt := h })", "tactic": "subst h''" }, { "state_after": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\nh : n < n + 1\nh' : ¬n < n\n⊢ _root_.cast (_ : α = α) a = cases a v { val := 0, isLt := (_ : 0 < Nat.succ n) }", "state_before": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\nh : n < n + 1\nh' : ¬n < n\n⊢ snoc v a { val := n, isLt := h } = cons a v (↑(finRotate (n + 1)) { val := n, isLt := h })", "tactic": "rw [finRotate_last', Fin.snoc, Fin.cons, dif_neg (lt_irrefl _)]" }, { "state_after": "no goals", "state_before": "case neg\nm n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\nh : n < n + 1\nh' : ¬n < n\n⊢ _root_.cast (_ : α = α) a = cases a v { val := 0, isLt := (_ : 0 < Nat.succ n) }", "tactic": "rfl" }, { "state_after": "m n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : n ≤ i\n⊢ n = i", "state_before": "m n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : ¬i < n\n⊢ n = i", "tactic": "simp only [not_lt] at h'" }, { "state_after": "no goals", "state_before": "m n : ℕ\nα : Type u_1\nv : Fin n → α\na : α\ni : ℕ\nh : i < n + 1\nh' : n ≤ i\n⊢ n = i", "tactic": "exact (Nat.eq_of_le_of_lt_succ h' h).symm" } ]
[ 427, 8 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 416, 1 ]
Mathlib/LinearAlgebra/Basic.lean
Submodule.subtype_comp_ofLe
[ { "state_after": "case h.mk\nR : Type u_1\nR₁ : Type ?u.394963\nR₂ : Type ?u.394966\nR₃ : Type ?u.394969\nR₄ : Type ?u.394972\nS : Type ?u.394975\nK : Type ?u.394978\nK₂ : Type ?u.394981\nM : Type u_2\nM' : Type ?u.394987\nM₁ : Type ?u.394990\nM₂ : Type ?u.394993\nM₃ : Type ?u.394996\nM₄ : Type ?u.394999\nN : Type ?u.395002\nN₂ : Type ?u.395005\nι : Type ?u.395008\nV : Type ?u.395011\nV₂ : Type ?u.395014\ninst✝¹³ : Semiring R\ninst✝¹² : Semiring R₂\ninst✝¹¹ : Semiring R₃\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : AddCommMonoid M₂\ninst✝⁸ : AddCommMonoid M₃\ninst✝⁷ : AddCommMonoid M'\ninst✝⁶ : Module R M\ninst✝⁵ : Module R M'\ninst✝⁴ : Module R₂ M₂\ninst✝³ : Module R₃ M₃\nσ₁₂ : R →+* R₂\nσ₂₃ : R₂ →+* R₃\nσ₁₃ : R →+* R₃\nσ₂₁ : R₂ →+* R\ninst✝² : RingHomInvPair σ₁₂ σ₂₁\ninst✝¹ : RingHomInvPair σ₂₁ σ₁₂\ninst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃\np✝ p' : Submodule R M\nq✝ q' : Submodule R₂ M₂\nq₁ q₁' : Submodule R M'\nr : R\nx y : M\np q : Submodule R M\nh : p ≤ q\nb : M\nhb : b ∈ p\n⊢ ↑(LinearMap.comp (Submodule.subtype q) (ofLe h)) { val := b, property := hb } =\n ↑(Submodule.subtype p) { val := b, property := hb }", "state_before": "R : Type u_1\nR₁ : Type ?u.394963\nR₂ : Type ?u.394966\nR₃ : Type ?u.394969\nR₄ : Type ?u.394972\nS : Type ?u.394975\nK : Type ?u.394978\nK₂ : Type ?u.394981\nM : Type u_2\nM' : Type ?u.394987\nM₁ : Type ?u.394990\nM₂ : Type ?u.394993\nM₃ : Type ?u.394996\nM₄ : Type ?u.394999\nN : Type ?u.395002\nN₂ : Type ?u.395005\nι : Type ?u.395008\nV : Type ?u.395011\nV₂ : Type ?u.395014\ninst✝¹³ : Semiring R\ninst✝¹² : Semiring R₂\ninst✝¹¹ : Semiring R₃\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : AddCommMonoid M₂\ninst✝⁸ : AddCommMonoid M₃\ninst✝⁷ : AddCommMonoid M'\ninst✝⁶ : Module R M\ninst✝⁵ : Module R M'\ninst✝⁴ : Module R₂ M₂\ninst✝³ : Module R₃ M₃\nσ₁₂ : R →+* R₂\nσ₂₃ : R₂ →+* R₃\nσ₁₃ : R →+* R₃\nσ₂₁ : R₂ →+* R\ninst✝² : RingHomInvPair σ₁₂ σ₂₁\ninst✝¹ : RingHomInvPair σ₂₁ σ₁₂\ninst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃\np✝ p' : Submodule R M\nq✝ q' : Submodule R₂ M₂\nq₁ q₁' : Submodule R M'\nr : R\nx y : M\np q : Submodule R M\nh : p ≤ q\n⊢ LinearMap.comp (Submodule.subtype q) (ofLe h) = Submodule.subtype p", "tactic": "ext ⟨b, hb⟩" }, { "state_after": "no goals", "state_before": "case h.mk\nR : Type u_1\nR₁ : Type ?u.394963\nR₂ : Type ?u.394966\nR₃ : Type ?u.394969\nR₄ : Type ?u.394972\nS : Type ?u.394975\nK : Type ?u.394978\nK₂ : Type ?u.394981\nM : Type u_2\nM' : Type ?u.394987\nM₁ : Type ?u.394990\nM₂ : Type ?u.394993\nM₃ : Type ?u.394996\nM₄ : Type ?u.394999\nN : Type ?u.395002\nN₂ : Type ?u.395005\nι : Type ?u.395008\nV : Type ?u.395011\nV₂ : Type ?u.395014\ninst✝¹³ : Semiring R\ninst✝¹² : Semiring R₂\ninst✝¹¹ : Semiring R₃\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : AddCommMonoid M₂\ninst✝⁸ : AddCommMonoid M₃\ninst✝⁷ : AddCommMonoid M'\ninst✝⁶ : Module R M\ninst✝⁵ : Module R M'\ninst✝⁴ : Module R₂ M₂\ninst✝³ : Module R₃ M₃\nσ₁₂ : R →+* R₂\nσ₂₃ : R₂ →+* R₃\nσ₁₃ : R →+* R₃\nσ₂₁ : R₂ →+* R\ninst✝² : RingHomInvPair σ₁₂ σ₂₁\ninst✝¹ : RingHomInvPair σ₂₁ σ₁₂\ninst✝ : RingHomCompTriple σ₁₂ σ₂₃ σ₁₃\np✝ p' : Submodule R M\nq✝ q' : Submodule R₂ M₂\nq₁ q₁' : Submodule R M'\nr : R\nx y : M\np q : Submodule R M\nh : p ≤ q\nb : M\nhb : b ∈ p\n⊢ ↑(LinearMap.comp (Submodule.subtype q) (ofLe h)) { val := b, property := hb } =\n ↑(Submodule.subtype p) { val := b, property := hb }", "tactic": "rfl" } ]
[ 641, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 638, 1 ]
Mathlib/Data/Polynomial/Splits.lean
Polynomial.adjoin_rootSet_eq_range
[ { "state_after": "F : Type u\nK : Type v\nL : Type w\ninst✝⁴ : Field K\ninst✝³ : Field L\ninst✝² : Field F\ni : K →+* L\ninst✝¹ : Algebra F K\ninst✝ : Algebra F L\np : F[X]\nh : Splits (algebraMap F K) p\nf : K →ₐ[F] L\n⊢ Subalgebra.map f (Algebra.adjoin F (rootSet p K)) = Subalgebra.map f ⊤ ↔ Algebra.adjoin F (rootSet p K) = ⊤", "state_before": "F : Type u\nK : Type v\nL : Type w\ninst✝⁴ : Field K\ninst✝³ : Field L\ninst✝² : Field F\ni : K →+* L\ninst✝¹ : Algebra F K\ninst✝ : Algebra F L\np : F[X]\nh : Splits (algebraMap F K) p\nf : K →ₐ[F] L\n⊢ Algebra.adjoin F (rootSet p L) = AlgHom.range f ↔ Algebra.adjoin F (rootSet p K) = ⊤", "tactic": "rw [← image_rootSet h f, Algebra.adjoin_image, ← Algebra.map_top]" }, { "state_after": "no goals", "state_before": "F : Type u\nK : Type v\nL : Type w\ninst✝⁴ : Field K\ninst✝³ : Field L\ninst✝² : Field F\ni : K →+* L\ninst✝¹ : Algebra F K\ninst✝ : Algebra F L\np : F[X]\nh : Splits (algebraMap F K) p\nf : K →ₐ[F] L\n⊢ Subalgebra.map f (Algebra.adjoin F (rootSet p K)) = Subalgebra.map f ⊤ ↔ Algebra.adjoin F (rootSet p K) = ⊤", "tactic": "exact (Subalgebra.map_injective f.toRingHom.injective).eq_iff" } ]
[ 348, 64 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 344, 1 ]
Mathlib/Algebra/Group/Commute.lean
Commute.mul_mul_mul_comm
[ { "state_after": "no goals", "state_before": "G : Type ?u.3529\nS : Type u_1\ninst✝ : Semigroup S\na✝ b c : S\nhbc : Commute b c\na d : S\n⊢ a * b * (c * d) = a * c * (b * d)", "tactic": "simp only [hbc.left_comm, mul_assoc]" } ]
[ 132, 81 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 131, 11 ]
Mathlib/Data/Set/Intervals/Disjoint.lean
Set.biUnion_Ioc_eq_Ioi_self_iff
[ { "state_after": "no goals", "state_before": "ι : Sort u\nα : Type v\nβ : Type w\ninst✝ : LinearOrder α\na₁ a₂ b₁ b₂ : α\np : ι → Prop\nf : (i : ι) → p i → α\na : α\n⊢ (⋃ (i : ι) (hi : p i), Ioc a (f i hi)) = Ioi a ↔ ∀ (x : α), a < x → ∃ i hi, x ≤ f i hi", "tactic": "simp [← Ioi_inter_Iic, ← inter_iUnion, subset_def]" } ]
[ 174, 53 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 172, 1 ]
Mathlib/MeasureTheory/Measure/MeasureSpace.lean
MeasureTheory.ae_restrict_of_ae_restrict_of_subset
[]
[ 2845, 67 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2843, 1 ]
Mathlib/Data/PFunctor/Multivariate/M.lean
MvPFunctor.M.bisim'
[ { "state_after": "case refine_3\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\nthis : ∀ (x y : M P α), EqvGen R x y → x = y\n⊢ x = y\n\ncase refine_1\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\n⊢ Equivalence (EqvGen R)\n\ncase refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\n⊢ ∀ (x y : M P α),\n EqvGen R x y → (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "state_before": "n : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\n⊢ x = y", "tactic": "have := M.bisim₀ P (EqvGen R) ?_ ?_" }, { "state_after": "no goals", "state_before": "case refine_3\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\nthis : ∀ (x y : M P α), EqvGen R x y → x = y\n⊢ x = y", "tactic": "solve_by_elim [EqvGen.rel]" }, { "state_after": "no goals", "state_before": "case refine_1\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\n⊢ Equivalence (EqvGen R)", "tactic": "apply EqvGen.is_equivalence" }, { "state_after": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\n⊢ ∀ (x y : M P α),\n EqvGen R x y → (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "state_before": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nr : R x y\n⊢ ∀ (x y : M P α),\n EqvGen R x y → (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "tactic": "clear r x y" }, { "state_after": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nHr : EqvGen R x y\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "state_before": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\n⊢ ∀ (x y : M P α),\n EqvGen R x y → (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "tactic": "introv Hr" }, { "state_after": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nHr : EqvGen R x y\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "state_before": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nHr : EqvGen R x y\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "tactic": "have : ∀ x y, R x y → EqvGen R x y := @EqvGen.rel _ R" }, { "state_after": "case refine_2.rel\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ : M P α\na✝ : R x✝ y✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝\n\ncase refine_2.refl\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ : M P α\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝\n\ncase refine_2.symm\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ : M P α\na✝ : EqvGen R x✝ y✝\na_ih✝ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝\n\ncase refine_2.trans\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ z✝ : M P α\na✝¹ : EqvGen R x✝ y✝\na✝ : EqvGen R y✝ z✝\na_ih✝¹ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝\na_ih✝ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P z✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P z✝", "state_before": "case refine_2\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nHr : EqvGen R x y\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y", "tactic": "induction Hr" }, { "state_after": "no goals", "state_before": "case refine_2.refl\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ : M P α\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝\n\ncase refine_2.symm\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ : M P α\na✝ : EqvGen R x✝ y✝\na_ih✝ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝\n\ncase refine_2.trans\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ z✝ : M P α\na✝¹ : EqvGen R x✝ y✝\na✝ : EqvGen R y✝ z✝\na_ih✝¹ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝\na_ih✝ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P z✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P z✝", "tactic": "all_goals aesop" }, { "state_after": "case refine_2.rel\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ : M P α\na✝ : R x✝ y✝\n⊢ (TypeVec.id ::: Quot.factor R (EqvGen R) this ∘ Quot.mk R) <$$> dest P x✝ =\n (TypeVec.id ::: Quot.factor R (EqvGen R) this ∘ Quot.mk R) <$$> dest P y✝", "state_before": "case refine_2.rel\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ : M P α\na✝ : R x✝ y✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝", "tactic": "rw [← Quot.factor_mk_eq R (EqvGen R) this]" }, { "state_after": "no goals", "state_before": "case refine_2.rel\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ : M P α\na✝ : R x✝ y✝\n⊢ (TypeVec.id ::: Quot.factor R (EqvGen R) this ∘ Quot.mk R) <$$> dest P x✝ =\n (TypeVec.id ::: Quot.factor R (EqvGen R) this ∘ Quot.mk R) <$$> dest P y✝", "tactic": "rwa [appendFun_comp_id, ← MvFunctor.map_map, ← MvFunctor.map_map, h]" }, { "state_after": "no goals", "state_before": "case refine_2.trans\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nR : M P α → M P α → Prop\nh : ∀ (x y : M P α), R x y → (TypeVec.id ::: Quot.mk R) <$$> dest P x = (TypeVec.id ::: Quot.mk R) <$$> dest P y\nx y : M P α\nthis : ∀ (x y : M P α), R x y → EqvGen R x y\nx✝ y✝ z✝ : M P α\na✝¹ : EqvGen R x✝ y✝\na✝ : EqvGen R y✝ z✝\na_ih✝¹ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝\na_ih✝ : (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P y✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P z✝\n⊢ (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P x✝ = (TypeVec.id ::: Quot.mk (EqvGen R)) <$$> dest P z✝", "tactic": "aesop" } ]
[ 365, 20 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 352, 1 ]
Mathlib/Data/Vector/Basic.lean
Vector.toList_scanl
[]
[ 348, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 347, 1 ]
Mathlib/Data/Finset/Pointwise.lean
Finset.Nonempty.smul
[]
[ 1329, 18 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1328, 1 ]
Mathlib/Data/Set/Pointwise/SMul.lean
Set.smul_iInter₂_subset
[]
[ 290, 36 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 288, 1 ]
Mathlib/Algebra/Divisibility/Basic.lean
dvd_of_mul_right_dvd
[]
[ 91, 30 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 90, 1 ]
Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean
CircleDeg1Lift.iterate_pos_eq_iff
[ { "state_after": "no goals", "state_before": "f g : CircleDeg1Lift\nx : ℝ\nm : ℤ\nn : ℕ\nhn : 0 < n\n⊢ (↑f^[n]) x = x + ↑n * ↑m ↔ ↑f x = x + ↑m", "tactic": "simpa only [nsmul_eq_mul, add_right_iterate] using\n (f.commute_add_int m).iterate_pos_eq_iff_map_eq f.monotone (strictMono_id.add_const (m : ℝ)) hn" } ]
[ 603, 100 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 600, 1 ]
Mathlib/FieldTheory/Finite/Basic.lean
FiniteField.sum_pow_lt_card_sub_one
[ { "state_after": "case pos\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : i = 0\n⊢ ∑ x : K, x ^ i = 0\n\ncase neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\n⊢ ∑ x : K, x ^ i = 0", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\n⊢ ∑ x : K, x ^ i = 0", "tactic": "by_cases hi : i = 0" }, { "state_after": "no goals", "state_before": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\n⊢ ∑ x : K, x ^ i = 0", "tactic": "classical\n have hiq : ¬q - 1 ∣ i := by contrapose! h; exact Nat.le_of_dvd (Nat.pos_of_ne_zero hi) h\n let φ : Kˣ ↪ K := ⟨fun x ↦ x, Units.ext⟩\n have : univ.map φ = univ \\ {0} := by\n ext x\n simp only [true_and_iff, Function.Embedding.coeFn_mk, mem_sdiff, Units.exists_iff_ne_zero,\n mem_univ, mem_map, exists_prop_of_true, mem_singleton]\n calc\n (∑ x : K, x ^ i) = ∑ x in univ \\ {(0 : K)}, x ^ i := by\n rw [← sum_sdiff ({0} : Finset K).subset_univ, sum_singleton,\n zero_pow (Nat.pos_of_ne_zero hi), add_zero]\n _ = ∑ x : Kˣ, (x ^ i : K) := by simp [← this, univ.sum_map φ]\n _ = 0 := by rw [sum_pow_units K i, if_neg]; exact hiq" }, { "state_after": "no goals", "state_before": "case pos\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : i = 0\n⊢ ∑ x : K, x ^ i = 0", "tactic": "simp only [hi, nsmul_one, sum_const, pow_zero, card_univ, cast_card_eq_zero]" }, { "state_after": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\n⊢ ∑ x : K, x ^ i = 0", "state_before": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\n⊢ ∑ x : K, x ^ i = 0", "tactic": "have hiq : ¬q - 1 ∣ i := by contrapose! h; exact Nat.le_of_dvd (Nat.pos_of_ne_zero hi) h" }, { "state_after": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\n⊢ ∑ x : K, x ^ i = 0", "state_before": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\n⊢ ∑ x : K, x ^ i = 0", "tactic": "let φ : Kˣ ↪ K := ⟨fun x ↦ x, Units.ext⟩" }, { "state_after": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ∑ x : K, x ^ i = 0", "state_before": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\n⊢ ∑ x : K, x ^ i = 0", "tactic": "have : univ.map φ = univ \\ {0} := by\n ext x\n simp only [true_and_iff, Function.Embedding.coeFn_mk, mem_sdiff, Units.exists_iff_ne_zero,\n mem_univ, mem_map, exists_prop_of_true, mem_singleton]" }, { "state_after": "no goals", "state_before": "case neg\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ∑ x : K, x ^ i = 0", "tactic": "calc\n (∑ x : K, x ^ i) = ∑ x in univ \\ {(0 : K)}, x ^ i := by\n rw [← sum_sdiff ({0} : Finset K).subset_univ, sum_singleton,\n zero_pow (Nat.pos_of_ne_zero hi), add_zero]\n _ = ∑ x : Kˣ, (x ^ i : K) := by simp [← this, univ.sum_map φ]\n _ = 0 := by rw [sum_pow_units K i, if_neg]; exact hiq" }, { "state_after": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nhi : ¬i = 0\nh : q - 1 ∣ i\n⊢ q - 1 ≤ i", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\n⊢ ¬q - 1 ∣ i", "tactic": "contrapose! h" }, { "state_after": "no goals", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nhi : ¬i = 0\nh : q - 1 ∣ i\n⊢ q - 1 ≤ i", "tactic": "exact Nat.le_of_dvd (Nat.pos_of_ne_zero hi) h" }, { "state_after": "case a\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nx : K\n⊢ x ∈ map φ univ ↔ x ∈ univ \\ {0}", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\n⊢ map φ univ = univ \\ {0}", "tactic": "ext x" }, { "state_after": "no goals", "state_before": "case a\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nx : K\n⊢ x ∈ map φ univ ↔ x ∈ univ \\ {0}", "tactic": "simp only [true_and_iff, Function.Embedding.coeFn_mk, mem_sdiff, Units.exists_iff_ne_zero,\n mem_univ, mem_map, exists_prop_of_true, mem_singleton]" }, { "state_after": "no goals", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ∑ x : K, x ^ i = ∑ x in univ \\ {0}, x ^ i", "tactic": "rw [← sum_sdiff ({0} : Finset K).subset_univ, sum_singleton,\n zero_pow (Nat.pos_of_ne_zero hi), add_zero]" }, { "state_after": "no goals", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ∑ x in univ \\ {0}, x ^ i = ∑ x : Kˣ, ↑(x ^ i)", "tactic": "simp [← this, univ.sum_map φ]" }, { "state_after": "case hnc\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ¬q - 1 ∣ i", "state_before": "K : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ∑ x : Kˣ, ↑(x ^ i) = 0", "tactic": "rw [sum_pow_units K i, if_neg]" }, { "state_after": "no goals", "state_before": "case hnc\nK : Type u_1\nR : Type ?u.640358\ninst✝¹ : Field K\ninst✝ : Fintype K\ni : ℕ\nh : i < q - 1\nhi : ¬i = 0\nhiq : ¬q - 1 ∣ i\nφ : Kˣ ↪ K := { toFun := fun x => ↑x, inj' := (_ : Function.Injective Units.val) }\nthis : map φ univ = univ \\ {0}\n⊢ ¬q - 1 ∣ i", "tactic": "exact hiq" } ]
[ 224, 60 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 209, 1 ]
Mathlib/Data/Fintype/Card.lean
Fintype.card_of_subtype
[ { "state_after": "α : Type u_1\nβ : Type ?u.3349\nγ : Type ?u.3352\np : α → Prop\ns : Finset α\nH : ∀ (x : α), x ∈ s ↔ p x\ninst✝ : Fintype { x // p x }\n⊢ card { x // p x } = card { x // p x }", "state_before": "α : Type u_1\nβ : Type ?u.3349\nγ : Type ?u.3352\np : α → Prop\ns : Finset α\nH : ∀ (x : α), x ∈ s ↔ p x\ninst✝ : Fintype { x // p x }\n⊢ card { x // p x } = Finset.card s", "tactic": "rw [← subtype_card s H]" }, { "state_after": "case h.e_2.h\nα : Type u_1\nβ : Type ?u.3349\nγ : Type ?u.3352\np : α → Prop\ns : Finset α\nH : ∀ (x : α), x ∈ s ↔ p x\ninst✝ : Fintype { x // p x }\n⊢ inst✝ = Fintype.subtype s H", "state_before": "α : Type u_1\nβ : Type ?u.3349\nγ : Type ?u.3352\np : α → Prop\ns : Finset α\nH : ∀ (x : α), x ∈ s ↔ p x\ninst✝ : Fintype { x // p x }\n⊢ card { x // p x } = card { x // p x }", "tactic": "congr" }, { "state_after": "no goals", "state_before": "case h.e_2.h\nα : Type u_1\nβ : Type ?u.3349\nγ : Type ?u.3352\np : α → Prop\ns : Finset α\nH : ∀ (x : α), x ∈ s ↔ p x\ninst✝ : Fintype { x // p x }\n⊢ inst✝ = Fintype.subtype s H", "tactic": "apply Subsingleton.elim" } ]
[ 131, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 127, 1 ]
Std/Data/Nat/Lemmas.lean
Nat.mul_dvd_mul
[ { "state_after": "no goals", "state_before": "a b c d e : Nat\nhe : b = a * e\nf : Nat\nhf : d = c * f\n⊢ b * d = a * c * (e * f)", "tactic": "simp [he, hf, Nat.mul_assoc, Nat.mul_left_comm, Nat.mul_comm]" } ]
[ 684, 78 ]
e68aa8f5fe47aad78987df45f99094afbcb5e936
https://github.com/leanprover/std4
[ 682, 11 ]
Mathlib/Order/Hom/CompleteLattice.lean
FrameHom.coe_copy
[]
[ 579, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 578, 1 ]
Mathlib/Data/Set/Intervals/Monotone.lean
MonotoneOn.Ioi
[]
[ 77, 34 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 76, 11 ]
Mathlib/Data/Multiset/Fintype.lean
Multiset.coe_mk
[]
[ 87, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 86, 1 ]
Mathlib/Data/Semiquot.lean
Semiquot.isPure_iff
[]
[ 237, 66 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 236, 1 ]
Mathlib/MeasureTheory/Integral/SetToL1.lean
MeasureTheory.DominatedFinMeasAdditive.eq_zero
[ { "state_after": "no goals", "state_before": "α : Type u_2\nE : Type ?u.102358\nF : Type ?u.102361\nF' : Type ?u.102364\nG : Type ?u.102367\n𝕜 : Type ?u.102370\np : ℝ≥0∞\ninst✝⁸ : NormedAddCommGroup E\ninst✝⁷ : NormedSpace ℝ E\ninst✝⁶ : NormedAddCommGroup F\ninst✝⁵ : NormedSpace ℝ F\ninst✝⁴ : NormedAddCommGroup F'\ninst✝³ : NormedSpace ℝ F'\ninst✝² : NormedAddCommGroup G\nm✝ : MeasurableSpace α\nμ : Measure α\nβ✝ : Type ?u.102670\ninst✝¹ : SeminormedAddCommGroup β✝\nT✝ T' : Set α → β✝\nC✝ C' : ℝ\nβ : Type u_1\ninst✝ : NormedAddCommGroup β\nT : Set α → β\nC : ℝ\nm : MeasurableSpace α\nhT : DominatedFinMeasAdditive 0 T C\ns : Set α\nhs : MeasurableSet s\n⊢ ↑↑0 s = 0", "tactic": "simp only [Measure.coe_zero, Pi.zero_apply]" } ]
[ 217, 81 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 214, 1 ]
Mathlib/Data/Set/Pointwise/Interval.lean
Set.image_sub_const_Ico
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : OrderedAddCommGroup α\na b c : α\n⊢ (fun x => x - a) '' Ico b c = Ico (b - a) (c - a)", "tactic": "simp [sub_eq_neg_add]" } ]
[ 396, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 395, 1 ]
Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean
CategoryTheory.Limits.coprod.inr_desc
[]
[ 651, 21 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 649, 1 ]
Mathlib/Analysis/NormedSpace/Multilinear.lean
ContinuousMultilinearMap.norm_ofSubsingleton
[ { "state_after": "case a\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\n⊢ ‖ofSubsingleton 𝕜 G i'‖ ≤ 1\n\ncase a\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "state_before": "𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\n⊢ ‖ofSubsingleton 𝕜 G i'‖ = 1", "tactic": "apply le_antisymm" }, { "state_after": "case a\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm✝ : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\nm : ι → G\n⊢ ‖↑(ofSubsingleton 𝕜 G i') m‖ ≤ 1 * ∏ i : ι, ‖m i‖", "state_before": "case a\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\n⊢ ‖ofSubsingleton 𝕜 G i'‖ ≤ 1", "tactic": "refine' op_norm_le_bound _ zero_le_one fun m => _" }, { "state_after": "no goals", "state_before": "case a\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm✝ : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\nm : ι → G\n⊢ ‖↑(ofSubsingleton 𝕜 G i') m‖ ≤ 1 * ∏ i : ι, ‖m i‖", "tactic": "rw [Fintype.prod_subsingleton _ i', one_mul, ofSubsingleton_apply]" }, { "state_after": "case a.intro\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g✝ : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\ng : G\nhg : g ≠ 0\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "state_before": "case a\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "tactic": "obtain ⟨g, hg⟩ := exists_ne (0 : G)" }, { "state_after": "case a.intro\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g✝ : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\ng : G\nhg : ‖g‖ ≠ 0\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "state_before": "case a.intro\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g✝ : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\ng : G\nhg : g ≠ 0\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "tactic": "rw [← norm_ne_zero_iff] at hg" }, { "state_after": "case a.intro\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g✝ : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\ng : G\nhg : ‖g‖ ≠ 0\nthis : ‖↑(ofSubsingleton 𝕜 G i') fun x => g‖ / ∏ i : ι, ‖g‖ ≤ ‖ofSubsingleton 𝕜 G i'‖\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "state_before": "case a.intro\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g✝ : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\ng : G\nhg : ‖g‖ ≠ 0\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "tactic": "have := (ofSubsingleton 𝕜 G i').ratio_le_op_norm fun _ => g" }, { "state_after": "no goals", "state_before": "case a.intro\n𝕜 : Type u\nι : Type v\nι' : Type v'\nn : ℕ\nE : ι → Type wE\nE₁ : ι → Type wE₁\nE' : ι' → Type wE'\nEi : Fin (Nat.succ n) → Type wEi\nG : Type wG\nG' : Type wG'\ninst✝¹⁹ : Fintype ι\ninst✝¹⁸ : Fintype ι'\ninst✝¹⁷ : NontriviallyNormedField 𝕜\ninst✝¹⁶ : (i : ι) → NormedAddCommGroup (E i)\ninst✝¹⁵ : (i : ι) → NormedSpace 𝕜 (E i)\ninst✝¹⁴ : (i : ι) → NormedAddCommGroup (E₁ i)\ninst✝¹³ : (i : ι) → NormedSpace 𝕜 (E₁ i)\ninst✝¹² : (i : ι') → NormedAddCommGroup (E' i)\ninst✝¹¹ : (i : ι') → NormedSpace 𝕜 (E' i)\ninst✝¹⁰ : (i : Fin (Nat.succ n)) → NormedAddCommGroup (Ei i)\ninst✝⁹ : (i : Fin (Nat.succ n)) → NormedSpace 𝕜 (Ei i)\ninst✝⁸ : NormedAddCommGroup G\ninst✝⁷ : NormedSpace 𝕜 G\ninst✝⁶ : NormedAddCommGroup G'\ninst✝⁵ : NormedSpace 𝕜 G'\nc : 𝕜\nf g✝ : ContinuousMultilinearMap 𝕜 E G\nm : (i : ι) → E i\n𝕜' : Type ?u.600696\ninst✝⁴ : NormedField 𝕜'\ninst✝³ : NormedSpace 𝕜' G\ninst✝² : SMulCommClass 𝕜 𝕜' G\ninst✝¹ : Subsingleton ι\ninst✝ : Nontrivial G\ni' : ι\ng : G\nhg : ‖g‖ ≠ 0\nthis : ‖↑(ofSubsingleton 𝕜 G i') fun x => g‖ / ∏ i : ι, ‖g‖ ≤ ‖ofSubsingleton 𝕜 G i'‖\n⊢ 1 ≤ ‖ofSubsingleton 𝕜 G i'‖", "tactic": "rwa [Fintype.prod_subsingleton _ i', ofSubsingleton_apply, div_self hg] at this" } ]
[ 518, 84 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 510, 1 ]
Mathlib/RingTheory/Localization/Integer.lean
IsLocalization.exist_integer_multiples_of_finite
[ { "state_after": "case intro\nR : Type u_2\ninst✝⁵ : CommRing R\nM : Submonoid R\nS : Type u_3\ninst✝⁴ : CommRing S\ninst✝³ : Algebra R S\nP : Type ?u.28129\ninst✝² : CommRing P\ninst✝¹ : IsLocalization M S\nι : Type u_1\ninst✝ : Finite ι\nf : ι → S\nval✝ : Fintype ι\n⊢ ∃ b, ∀ (i : ι), IsInteger R (↑b • f i)", "state_before": "R : Type u_2\ninst✝⁵ : CommRing R\nM : Submonoid R\nS : Type u_3\ninst✝⁴ : CommRing S\ninst✝³ : Algebra R S\nP : Type ?u.28129\ninst✝² : CommRing P\ninst✝¹ : IsLocalization M S\nι : Type u_1\ninst✝ : Finite ι\nf : ι → S\n⊢ ∃ b, ∀ (i : ι), IsInteger R (↑b • f i)", "tactic": "cases nonempty_fintype ι" }, { "state_after": "case intro.intro\nR : Type u_2\ninst✝⁵ : CommRing R\nM : Submonoid R\nS : Type u_3\ninst✝⁴ : CommRing S\ninst✝³ : Algebra R S\nP : Type ?u.28129\ninst✝² : CommRing P\ninst✝¹ : IsLocalization M S\nι : Type u_1\ninst✝ : Finite ι\nf : ι → S\nval✝ : Fintype ι\nb : { x // x ∈ M }\nhb : ∀ (i : ι), i ∈ Finset.univ → IsInteger R (↑b • f i)\n⊢ ∃ b, ∀ (i : ι), IsInteger R (↑b • f i)", "state_before": "case intro\nR : Type u_2\ninst✝⁵ : CommRing R\nM : Submonoid R\nS : Type u_3\ninst✝⁴ : CommRing S\ninst✝³ : Algebra R S\nP : Type ?u.28129\ninst✝² : CommRing P\ninst✝¹ : IsLocalization M S\nι : Type u_1\ninst✝ : Finite ι\nf : ι → S\nval✝ : Fintype ι\n⊢ ∃ b, ∀ (i : ι), IsInteger R (↑b • f i)", "tactic": "obtain ⟨b, hb⟩ := exist_integer_multiples M Finset.univ f" }, { "state_after": "no goals", "state_before": "case intro.intro\nR : Type u_2\ninst✝⁵ : CommRing R\nM : Submonoid R\nS : Type u_3\ninst✝⁴ : CommRing S\ninst✝³ : Algebra R S\nP : Type ?u.28129\ninst✝² : CommRing P\ninst✝¹ : IsLocalization M S\nι : Type u_1\ninst✝ : Finite ι\nf : ι → S\nval✝ : Fintype ι\nb : { x // x ∈ M }\nhb : ∀ (i : ι), i ∈ Finset.univ → IsInteger R (↑b • f i)\n⊢ ∃ b, ∀ (i : ι), IsInteger R (↑b • f i)", "tactic": "exact ⟨b, fun i => hb i (Finset.mem_univ _)⟩" } ]
[ 117, 47 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 113, 1 ]
Mathlib/LinearAlgebra/Span.lean
Submodule.disjoint_span_singleton'
[]
[ 469, 85 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 467, 1 ]
Mathlib/ModelTheory/Semantics.lean
FirstOrder.Language.LHom.realize_onBoundedFormula
[ { "state_after": "case falsum\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ falsum) v xs ↔ Realize falsum v xs\n\ncase equal\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nt₁✝ t₂✝ : Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (equal t₁✝ t₂✝)) v xs ↔ Realize (equal t₁✝ t₂✝) v xs\n\ncase rel\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ l✝ : ℕ\nR✝ : Relations L l✝\nts✝ : Fin l✝ → Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (rel R✝ ts✝)) v xs ↔ Realize (rel R✝ ts✝) v xs\n\ncase imp\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nf₁✝ f₂✝ : BoundedFormula L α n✝\nih1 : ∀ {xs : Fin n✝ → M}, Realize (onBoundedFormula φ f₁✝) v xs ↔ Realize f₁✝ v xs\nih2 : ∀ {xs : Fin n✝ → M}, Realize (onBoundedFormula φ f₂✝) v xs ↔ Realize f₂✝ v xs\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (f₁✝ ⟹ f₂✝)) v xs ↔ Realize (f₁✝ ⟹ f₂✝) v xs\n\ncase all\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nf✝ : BoundedFormula L α (n✝ + 1)\nih3 : ∀ {xs : Fin (n✝ + 1) → M}, Realize (onBoundedFormula φ f✝) v xs ↔ Realize f✝ v xs\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (∀'f✝)) v xs ↔ Realize (∀'f✝) v xs", "state_before": "L : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nψ : BoundedFormula L α n\nv : α → M\nxs : Fin n → M\n⊢ Realize (onBoundedFormula φ ψ) v xs ↔ Realize ψ v xs", "tactic": "induction' ψ with _ _ _ _ _ _ _ _ _ _ _ ih1 ih2 _ _ ih3" }, { "state_after": "no goals", "state_before": "case falsum\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ falsum) v xs ↔ Realize falsum v xs", "tactic": "rfl" }, { "state_after": "case equal\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nt₁✝ t₂✝ : Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ Term.realize (Sum.elim v xs) t₁✝ = Term.realize (Sum.elim v xs) t₂✝ ↔ Realize (equal t₁✝ t₂✝) v xs", "state_before": "case equal\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nt₁✝ t₂✝ : Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (equal t₁✝ t₂✝)) v xs ↔ Realize (equal t₁✝ t₂✝) v xs", "tactic": "simp only [onBoundedFormula, realize_bdEqual, realize_onTerm]" }, { "state_after": "no goals", "state_before": "case equal\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nt₁✝ t₂✝ : Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ Term.realize (Sum.elim v xs) t₁✝ = Term.realize (Sum.elim v xs) t₂✝ ↔ Realize (equal t₁✝ t₂✝) v xs", "tactic": "rfl" }, { "state_after": "case rel\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ l✝ : ℕ\nR✝ : Relations L l✝\nts✝ : Fin l✝ → Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ (RelMap R✝ fun i => Term.realize (Sum.elim v xs) (ts✝ i)) ↔ Realize (rel R✝ ts✝) v xs", "state_before": "case rel\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ l✝ : ℕ\nR✝ : Relations L l✝\nts✝ : Fin l✝ → Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (rel R✝ ts✝)) v xs ↔ Realize (rel R✝ ts✝) v xs", "tactic": "simp only [onBoundedFormula, realize_rel, LHom.map_onRelation,\n Function.comp_apply, realize_onTerm]" }, { "state_after": "no goals", "state_before": "case rel\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ l✝ : ℕ\nR✝ : Relations L l✝\nts✝ : Fin l✝ → Term L (α ⊕ Fin n✝)\nxs : Fin n✝ → M\n⊢ (RelMap R✝ fun i => Term.realize (Sum.elim v xs) (ts✝ i)) ↔ Realize (rel R✝ ts✝) v xs", "tactic": "rfl" }, { "state_after": "no goals", "state_before": "case imp\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nf₁✝ f₂✝ : BoundedFormula L α n✝\nih1 : ∀ {xs : Fin n✝ → M}, Realize (onBoundedFormula φ f₁✝) v xs ↔ Realize f₁✝ v xs\nih2 : ∀ {xs : Fin n✝ → M}, Realize (onBoundedFormula φ f₂✝) v xs ↔ Realize f₂✝ v xs\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (f₁✝ ⟹ f₂✝)) v xs ↔ Realize (f₁✝ ⟹ f₂✝) v xs", "tactic": "simp only [onBoundedFormula, ih1, ih2, realize_imp]" }, { "state_after": "no goals", "state_before": "case all\nL : Language\nL' : Language\nM : Type w\nN : Type ?u.231167\nP : Type ?u.231170\ninst✝⁴ : Structure L M\ninst✝³ : Structure L N\ninst✝² : Structure L P\nα : Type u'\nβ : Type v'\nn✝¹ : ℕ\ninst✝¹ : Structure L' M\nφ : L →ᴸ L'\ninst✝ : IsExpansionOn φ M\nn : ℕ\nv : α → M\nxs✝ : Fin n → M\nn✝ : ℕ\nf✝ : BoundedFormula L α (n✝ + 1)\nih3 : ∀ {xs : Fin (n✝ + 1) → M}, Realize (onBoundedFormula φ f✝) v xs ↔ Realize f✝ v xs\nxs : Fin n✝ → M\n⊢ Realize (onBoundedFormula φ (∀'f✝)) v xs ↔ Realize (∀'f✝) v xs", "tactic": "simp only [onBoundedFormula, ih3, realize_all]" } ]
[ 595, 51 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 584, 1 ]
Mathlib/LinearAlgebra/Matrix/IsDiag.lean
Matrix.IsDiag.diagonal_diag
[ { "state_after": "case inl\nα : Type u_1\nβ : Type ?u.560\nR : Type ?u.563\nn : Type u_2\nm : Type ?u.569\ninst✝¹ : Zero α\ninst✝ : DecidableEq n\nA : Matrix n n α\nh : IsDiag A\ni : n\n⊢ diagonal (diag A) i i = A i i\n\ncase inr\nα : Type u_1\nβ : Type ?u.560\nR : Type ?u.563\nn : Type u_2\nm : Type ?u.569\ninst✝¹ : Zero α\ninst✝ : DecidableEq n\nA : Matrix n n α\nh : IsDiag A\ni j : n\nhij : i ≠ j\n⊢ diagonal (diag A) i j = A i j", "state_before": "α : Type u_1\nβ : Type ?u.560\nR : Type ?u.563\nn : Type u_2\nm : Type ?u.569\ninst✝¹ : Zero α\ninst✝ : DecidableEq n\nA : Matrix n n α\nh : IsDiag A\ni j : n\n⊢ diagonal (diag A) i j = A i j", "tactic": "obtain rfl | hij := Decidable.eq_or_ne i j" }, { "state_after": "no goals", "state_before": "case inl\nα : Type u_1\nβ : Type ?u.560\nR : Type ?u.563\nn : Type u_2\nm : Type ?u.569\ninst✝¹ : Zero α\ninst✝ : DecidableEq n\nA : Matrix n n α\nh : IsDiag A\ni : n\n⊢ diagonal (diag A) i i = A i i", "tactic": "rw [diagonal_apply_eq, diag]" }, { "state_after": "no goals", "state_before": "case inr\nα : Type u_1\nβ : Type ?u.560\nR : Type ?u.563\nn : Type u_2\nm : Type ?u.569\ninst✝¹ : Zero α\ninst✝ : DecidableEq n\nA : Matrix n n α\nh : IsDiag A\ni j : n\nhij : i ≠ j\n⊢ diagonal (diag A) i j = A i j", "tactic": "rw [diagonal_apply_ne _ hij, h hij]" } ]
[ 54, 42 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 49, 1 ]
Mathlib/MeasureTheory/Measure/GiryMonad.lean
MeasureTheory.Measure.bind_zero_left
[ { "state_after": "no goals", "state_before": "α : Type u_2\nβ : Type u_1\ninst✝¹ : MeasurableSpace α\ninst✝ : MeasurableSpace β\nf : α → Measure β\n⊢ bind 0 f = 0", "tactic": "simp [bind]" } ]
[ 160, 76 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 160, 1 ]
Mathlib/Logic/Encodable/Lattice.lean
Encodable.iUnion_decode₂_disjoint_on
[ { "state_after": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\n⊢ (Disjoint on fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) i j", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\n⊢ Pairwise (Disjoint on fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b)", "tactic": "rintro i j ij" }, { "state_after": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\nx : α\n⊢ x ∈ (fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) i → ¬x ∈ (fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) j", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\n⊢ (Disjoint on fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) i j", "tactic": "refine' disjoint_left.mpr fun x => _" }, { "state_after": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\nx : α\n⊢ ∀ (a : β), encode a = i → x ∈ f a → ∀ (b : β), encode b = j → ¬x ∈ f b", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\nx : α\n⊢ x ∈ (fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) i → ¬x ∈ (fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) j", "tactic": "suffices ∀ a, encode a = i → x ∈ f a → ∀ b, encode b = j → x ∉ f b by simpa [decode₂_eq_some]" }, { "state_after": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\nx : α\na : β\nha : x ∈ f a\nb : β\nij : encode a ≠ encode b\nhb : x ∈ f b\n⊢ False", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\nx : α\n⊢ ∀ (a : β), encode a = i → x ∈ f a → ∀ (b : β), encode b = j → ¬x ∈ f b", "tactic": "rintro a rfl ha b rfl hb" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\nx : α\na : β\nha : x ∈ f a\nb : β\nij : encode a ≠ encode b\nhb : x ∈ f b\n⊢ False", "tactic": "exact (hd (mt (congr_arg encode) ij)).le_bot ⟨ha, hb⟩" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝ : Encodable β\nf : β → Set α\nhd : Pairwise (Disjoint on f)\ni j : ℕ\nij : i ≠ j\nx : α\nthis : ∀ (a : β), encode a = i → x ∈ f a → ∀ (b : β), encode b = j → ¬x ∈ f b\n⊢ x ∈ (fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) i → ¬x ∈ (fun i => ⋃ (b : β) (_ : b ∈ decode₂ β i), f b) j", "tactic": "simpa [decode₂_eq_some]" } ]
[ 61, 56 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 55, 1 ]
Mathlib/Data/Finmap.lean
Finmap.insert_toFinmap
[ { "state_after": "no goals", "state_before": "α : Type u\nβ : α → Type v\ninst✝ : DecidableEq α\na : α\nb : β a\ns : AList β\n⊢ insert a b ⟦s⟧ = ⟦AList.insert a b s⟧", "tactic": "simp [insert]" } ]
[ 485, 16 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 483, 1 ]