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/Algebra/ModEq.lean
AddCommGroup.not_modEq_iff_ne_add_zsmul
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : AddCommGroup α\np a a₁ a₂ b b₁ b₂ c : α\nn : ℕ\nz : ℤ\n⊢ ¬a ≡ b [PMOD p] ↔ ∀ (z : ℤ), b ≠ a + z • p", "tactic": "rw [modEq_iff_eq_add_zsmul, not_exists]" } ]
[ 297, 42 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 296, 1 ]
Mathlib/NumberTheory/Padics/RingHoms.lean
PadicInt.limNthHom_zero
[ { "state_after": "p : ℕ\nhp_prime : Fact (Nat.Prime p)\nR : Type u_1\ninst✝ : NonAssocSemiring R\nf : (k : ℕ) → R →+* ZMod (p ^ k)\nf_compat : ∀ (k1 k2 : ℕ) (hk : k1 ≤ k2), RingHom.comp (ZMod.castHom (_ : p ^ k1 ∣ p ^ k2) (ZMod (p ^ k1))) (f k2) = f k1\n⊢ ofIntSeq 0 (_ : IsCauSeq (padicNorm p) fun n => ↑(OfNat.ofNat 0 n)) = 0", "state_before": "p : ℕ\nhp_prime : Fact (Nat.Prime p)\nR : Type u_1\ninst✝ : NonAssocSemiring R\nf : (k : ℕ) → R →+* ZMod (p ^ k)\nf_compat : ∀ (k1 k2 : ℕ) (hk : k1 ≤ k2), RingHom.comp (ZMod.castHom (_ : p ^ k1 ∣ p ^ k2) (ZMod (p ^ k1))) (f k2) = f k1\n⊢ limNthHom f_compat 0 = 0", "tactic": "simp [limNthHom]" }, { "state_after": "no goals", "state_before": "p : ℕ\nhp_prime : Fact (Nat.Prime p)\nR : Type u_1\ninst✝ : NonAssocSemiring R\nf : (k : ℕ) → R →+* ZMod (p ^ k)\nf_compat : ∀ (k1 k2 : ℕ) (hk : k1 ≤ k2), RingHom.comp (ZMod.castHom (_ : p ^ k1 ∣ p ^ k2) (ZMod (p ^ k1))) (f k2) = f k1\n⊢ ofIntSeq 0 (_ : IsCauSeq (padicNorm p) fun n => ↑(OfNat.ofNat 0 n)) = 0", "tactic": "rfl" } ]
[ 592, 78 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 592, 1 ]
Mathlib/Algebra/Ring/Equiv.lean
RingEquiv.coe_toNonUnitalRingHom
[]
[ 619, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 618, 1 ]
Mathlib/Data/Set/Pointwise/BigOperators.lean
Set.image_multiset_prod
[ { "state_after": "no goals", "state_before": "ι : Type ?u.19659\nα : Type u_1\nβ : Type u_2\nF : Type u_3\ninst✝² : CommMonoid α\ninst✝¹ : CommMonoid β\ninst✝ : MonoidHomClass F α β\nf : F\n⊢ ∀ (a : List (Set α)),\n ↑f '' Multiset.prod (Quotient.mk (List.isSetoid (Set α)) a) =\n Multiset.prod (Multiset.map (fun s => ↑f '' s) (Quotient.mk (List.isSetoid (Set α)) a))", "tactic": "simpa only [Multiset.quot_mk_to_coe, Multiset.coe_prod, Multiset.coe_map] using\n image_list_prod f" } ]
[ 50, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 46, 1 ]
Mathlib/Data/Nat/Factorization/Basic.lean
Nat.ord_compl_of_not_prime
[ { "state_after": "no goals", "state_before": "n p : ℕ\nhp : ¬Prime p\n⊢ n / p ^ ↑(factorization n) p = n", "tactic": "simp [factorization_eq_zero_of_non_prime n hp]" } ]
[ 365, 49 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 364, 1 ]
Mathlib/Data/Multiset/Basic.lean
Multiset.attach_map_val'
[]
[ 1535, 70 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1534, 1 ]
Mathlib/GroupTheory/PGroup.lean
IsPGroup.iff_orderOf
[ { "state_after": "no goals", "state_before": "p : ℕ\nG : Type u_1\ninst✝ : Group G\nhp : Fact (Nat.Prime p)\ng : G\nk : ℕ\nhk : orderOf g = p ^ k\n⊢ g ^ p ^ k = 1", "tactic": "rw [← hk, pow_orderOf_eq_one]" } ]
[ 48, 63 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 43, 1 ]
Std/Logic.lean
or_or_or_comm
[ { "state_after": "no goals", "state_before": "a b c d : Prop\n⊢ (a ∨ b) ∨ c ∨ d ↔ (a ∨ c) ∨ b ∨ d", "tactic": "rw [← or_assoc, @or_right_comm a, or_assoc]" } ]
[ 281, 46 ]
e68aa8f5fe47aad78987df45f99094afbcb5e936
https://github.com/leanprover/std4
[ 280, 1 ]
Mathlib/GroupTheory/NielsenSchreier.lean
IsFreeGroupoid.SpanningTree.loopOfHom_eq_id
[ { "state_after": "G : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : e ∈ wideSubquiverSymmetrify T a b\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n treeHom T b", "state_before": "G : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : e ∈ wideSubquiverSymmetrify T a b\n⊢ loopOfHom T (of e) = 𝟙 (IsFreeGroupoid.SpanningTree.root' T)", "tactic": "rw [loopOfHom, ← Category.assoc, IsIso.comp_inv_eq, Category.id_comp]" }, { "state_after": "case inl\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T a b (Sum.inl e)\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n treeHom T b\n\ncase inr\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T b a (Sum.inr e)\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n treeHom T b", "state_before": "G : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : e ∈ wideSubquiverSymmetrify T a b\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n treeHom T b", "tactic": "cases' H with H H" }, { "state_after": "case inl\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T a b (Sum.inl e)\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n homOfPath T default ≫ Sum.recOn (↑{ val := Sum.inl e, property := H }) (fun e => of e) fun e => inv (of e)", "state_before": "case inl\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T a b (Sum.inl e)\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n treeHom T b", "tactic": "rw [treeHom_eq T (Path.cons default ⟨Sum.inl e, H⟩), homOfPath]" }, { "state_after": "no goals", "state_before": "case inl\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T a b (Sum.inl e)\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n homOfPath T default ≫ Sum.recOn (↑{ val := Sum.inl e, property := H }) (fun e => of e) fun e => inv (of e)", "tactic": "rfl" }, { "state_after": "case inr\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T b a (Sum.inr e)\n⊢ (homOfPath T default ≫ Sum.recOn (↑{ val := Sum.inr e, property := H }) (fun e => of e) fun e => inv (of e)) ≫ of e =\n treeHom T b", "state_before": "case inr\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T b a (Sum.inr e)\n⊢ treeHom T\n (let_fun this := a;\n this) ≫\n of e =\n treeHom T b", "tactic": "rw [treeHom_eq T (Path.cons default ⟨Sum.inr e, H⟩), homOfPath]" }, { "state_after": "no goals", "state_before": "case inr\nG : Type u\ninst✝² : Groupoid G\ninst✝¹ : IsFreeGroupoid G\nT : WideSubquiver (Symmetrify (Generators G))\ninst✝ : Arborescence (WideSubquiver.toType (Symmetrify (Generators G)) T)\na b : Generators G\ne : a ⟶ b\nH : T b a (Sum.inr e)\n⊢ (homOfPath T default ≫ Sum.recOn (↑{ val := Sum.inr e, property := H }) (fun e => of e) fun e => inv (of e)) ≫ of e =\n treeHom T b", "tactic": "simp only [IsIso.inv_hom_id, Category.comp_id, Category.assoc, treeHom]" } ]
[ 205, 76 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 198, 1 ]
Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean
uniformCauchySeqOn_ball_of_fderiv
[ { "state_after": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "tactic": "letI : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 _" }, { "state_after": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "tactic": "have : NeBot l := (cauchy_map_iff.1 hfg).1" }, { "state_after": "case inl\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : r ≤ 0\n⊢ UniformCauchySeqOn f l (Metric.ball x r)\n\ncase inr\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "tactic": "rcases le_or_lt r 0 with (hr | hr)" }, { "state_after": "case inr\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "state_before": "case inr\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "tactic": "rw [SeminormedAddGroup.uniformCauchySeqOn_iff_tendstoUniformlyOn_zero] at hf' ⊢" }, { "state_after": "case inr\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)", "state_before": "case inr\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "suffices\n TendstoUniformlyOn (fun (n : ι × ι) (z : E) => f n.1 z - f n.2 z - (f n.1 x - f n.2 x)) 0\n (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun (n : ι × ι) (_ : E) => f n.1 x - f n.2 x) 0\n (l ×ˢ l) (Metric.ball x r) by\n have := this.1.add this.2\n rw [add_zero] at this\n refine' this.congr _\n apply eventually_of_forall\n intro n z _\n simp" }, { "state_after": "case inr.left\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r)\n\ncase inr.right\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)", "state_before": "case inr\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "constructor" }, { "state_after": "no goals", "state_before": "case inl\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : UniformCauchySeqOn f' l (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : r ≤ 0\n⊢ UniformCauchySeqOn f l (Metric.ball x r)", "tactic": "simp only [Metric.ball_eq_empty.2 hr, UniformCauchySeqOn, Set.mem_empty_iff_false,\n IsEmpty.forall_iff, eventually_const, imp_true_iff]" }, { "state_after": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n (0 + 0) (l ×ˢ l) (Metric.ball x r)\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝¹ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝ : NeBot l\nhr : 0 < r\nthis :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "have := this.1.add this.2" }, { "state_after": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n (0 + 0) (l ×ˢ l) (Metric.ball x r)\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "rw [add_zero] at this" }, { "state_after": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l,\n Set.EqOn (((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x) n)\n (fun z => f n.fst z - f n.snd z) (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "refine' this.congr _" }, { "state_after": "case hp\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\n⊢ ∀ (x_1 : ι × ι),\n Set.EqOn (((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_2 => f n.fst x - f n.snd x) x_1)\n (fun z => f x_1.fst z - f x_1.snd z) (Metric.ball x r)", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l,\n Set.EqOn (((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x) n)\n (fun z => f n.fst z - f n.snd z) (Metric.ball x r)", "tactic": "apply eventually_of_forall" }, { "state_after": "case hp\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\nn : ι × ι\nz : E\na✝ : z ∈ Metric.ball x r\n⊢ ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x) n z =\n (fun z => f n.fst z - f n.snd z) z", "state_before": "case hp\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\n⊢ ∀ (x_1 : ι × ι),\n Set.EqOn (((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_2 => f n.fst x - f n.snd x) x_1)\n (fun z => f x_1.fst z - f x_1.snd z) (Metric.ball x r)", "tactic": "intro n z _" }, { "state_after": "no goals", "state_before": "case hp\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝² : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝¹ : NeBot l\nhr : 0 < r\nthis✝ :\n TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r) ∧\n TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)\nthis :\n TendstoUniformlyOn ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x)\n 0 (l ×ˢ l) (Metric.ball x r)\nn : ι × ι\nz : E\na✝ : z ∈ Metric.ball x r\n⊢ ((fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) + fun n x_1 => f n.fst x - f n.snd x) n z =\n (fun z => f n.fst z - f n.snd z) z", "tactic": "simp" }, { "state_after": "case inr.left\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E),\n x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x_1 - f n.snd x_1 - (f n.fst x - f n.snd x)) < ε", "state_before": "case inr.left\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n z => f n.fst z - f n.snd z - (f n.fst x - f n.snd x)) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "rw [Metric.tendstoUniformlyOn_iff] at hf' ⊢" }, { "state_after": "case inr.left\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E),\n x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x_1 - f n.snd x_1 - (f n.fst x - f n.snd x)) < ε", "state_before": "case inr.left\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E),\n x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x_1 - f n.snd x_1 - (f n.fst x - f n.snd x)) < ε", "tactic": "intro ε hε" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E),\n x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x_1 - f n.snd x_1 - (f n.fst x - f n.snd x)) < ε", "state_before": "case inr.left\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E),\n x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x_1 - f n.snd x_1 - (f n.fst x - f n.snd x)) < ε", "tactic": "obtain ⟨q, hqpos, hq⟩ : ∃ q : ℝ, 0 < q ∧ q * r < ε := by\n simp_rw [mul_comm]\n exact exists_pos_mul_lt hε.lt r" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\n⊢ ∀ (x_1 : ι × ι),\n (∀ (x_2 : E), x_2 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_2) (f' x_1.fst x_2 - f' x_1.snd x_2) < q) →\n ∀ (x_2 : E),\n x_2 ∈ Metric.ball x r →\n dist (OfNat.ofNat 0 x_2) (f x_1.fst x_2 - f x_1.snd x_2 - (f x_1.fst x - f x_1.snd x)) < ε", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E),\n x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x_1 - f n.snd x_1 - (f n.fst x - f n.snd x)) < ε", "tactic": "apply (hf' q hqpos.gt).mono" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < q\ny : E\nhy : y ∈ Metric.ball x r\n⊢ dist (OfNat.ofNat 0 y) (f n.fst y - f n.snd y - (f n.fst x - f n.snd x)) < ε", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\n⊢ ∀ (x_1 : ι × ι),\n (∀ (x_2 : E), x_2 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_2) (f' x_1.fst x_2 - f' x_1.snd x_2) < q) →\n ∀ (x_2 : E),\n x_2 ∈ Metric.ball x r →\n dist (OfNat.ofNat 0 x_2) (f x_1.fst x_2 - f x_1.snd x_2 - (f x_1.fst x - f x_1.snd x)) < ε", "tactic": "intro n hn y hy" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\n⊢ ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ < ε", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < q\ny : E\nhy : y ∈ Metric.ball x r\n⊢ dist (OfNat.ofNat 0 y) (f n.fst y - f n.snd y - (f n.fst x - f n.snd x)) < ε", "tactic": "simp_rw [dist_eq_norm, Pi.zero_apply, zero_sub, norm_neg] at hn ⊢" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\n⊢ ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ < ε", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\n⊢ ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ < ε", "tactic": "have mvt :=\n Convex.norm_image_sub_le_of_norm_hasFDerivWithin_le\n (fun z hz => ((hf n.1 z hz).sub (hf n.2 z hz)).hasFDerivWithinAt) (fun z hz => (hn z hz).le)\n (convex_ball x r) (Metric.mem_ball_self hr) hy" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\n⊢ q * ‖y - x‖ < ε", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\n⊢ ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ < ε", "tactic": "refine' lt_of_le_of_lt mvt _" }, { "state_after": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝¹ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝ : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\nthis : q * ‖y - x‖ < q * r\n⊢ q * ‖y - x‖ < ε", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\n⊢ q * ‖y - x‖ < ε", "tactic": "have : q * ‖y - x‖ < q * r :=\n mul_lt_mul' rfl.le (by simpa only [dist_eq_norm] using Metric.mem_ball.mp hy) (norm_nonneg _)\n hqpos" }, { "state_after": "no goals", "state_before": "case inr.left.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝¹ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis✝ : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\nthis : q * ‖y - x‖ < q * r\n⊢ q * ‖y - x‖ < ε", "tactic": "exact this.trans hq" }, { "state_after": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∃ q, 0 < q ∧ r * q < ε", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∃ q, 0 < q ∧ q * r < ε", "tactic": "simp_rw [mul_comm]" }, { "state_after": "no goals", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∃ q, 0 < q ∧ r * q < ε", "tactic": "exact exists_pos_mul_lt hε.lt r" }, { "state_after": "no goals", "state_before": "ι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' :\n ∀ (ε : ℝ),\n ε > 0 →\n ∀ᶠ (n : ι × ι) in l ×ˢ l,\n ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f' n.fst x_1 - f' n.snd x_1) < ε\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nq : ℝ\nhqpos : 0 < q\nhq : q * r < ε\nn : ι × ι\ny : E\nhy : y ∈ Metric.ball x r\nhn : ∀ (x_1 : E), x_1 ∈ Metric.ball x r → ‖f' n.fst x_1 - f' n.snd x_1‖ < q\nmvt : ‖f n.fst y - f n.snd y - (f n.fst x - f n.snd x)‖ ≤ q * ‖y - x‖\n⊢ ‖y - x‖ < r", "tactic": "simpa only [dist_eq_norm] using Metric.mem_ball.mp hy" }, { "state_after": "case inr.right\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l, ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x - f n.snd x) < ε", "state_before": "case inr.right\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\n⊢ TendstoUniformlyOn (fun n x_1 => f n.fst x - f n.snd x) 0 (l ×ˢ l) (Metric.ball x r)", "tactic": "refine' Metric.tendstoUniformlyOn_iff.mpr fun ε hε => _" }, { "state_after": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l, ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x - f n.snd x) < ε", "state_before": "case inr.right\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l, ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x - f n.snd x) < ε", "tactic": "obtain ⟨t, ht, ht'⟩ := (Metric.cauchy_iff.mp hfg).2 ε hε" }, { "state_after": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\n⊢ ∃ pa,\n (∀ᶠ (x : ι) in l, pa x) ∧\n ∃ pb,\n (∀ᶠ (y : ι) in l, pb y) ∧\n ∀ {x_1 : ι},\n pa x_1 →\n ∀ {y : ι},\n pb y →\n ∀ (x_2 : E),\n x_2 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_2) (f (x_1, y).fst x - f (x_1, y).snd x) < ε", "state_before": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\n⊢ ∀ᶠ (n : ι × ι) in l ×ˢ l, ∀ (x_1 : E), x_1 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_1) (f n.fst x - f n.snd x) < ε", "tactic": "rw [eventually_prod_iff]" }, { "state_after": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\n⊢ ∀ {x_1 : ι},\n (fun n => f n x ∈ t) x_1 →\n ∀ {y : ι},\n (fun n => f n x ∈ t) y →\n ∀ (x_2 : E), x_2 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_2) (f (x_1, y).fst x - f (x_1, y).snd x) < ε", "state_before": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\n⊢ ∃ pa,\n (∀ᶠ (x : ι) in l, pa x) ∧\n ∃ pb,\n (∀ᶠ (y : ι) in l, pb y) ∧\n ∀ {x_1 : ι},\n pa x_1 →\n ∀ {y : ι},\n pb y →\n ∀ (x_2 : E),\n x_2 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_2) (f (x_1, y).fst x - f (x_1, y).snd x) < ε", "tactic": "refine' ⟨fun n => f n x ∈ t, ht, fun n => f n x ∈ t, ht, _⟩" }, { "state_after": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\nn : ι\nhn : f n x ∈ t\nn' : ι\nhn' : f n' x ∈ t\nz : E\na✝ : z ∈ Metric.ball x r\n⊢ dist (OfNat.ofNat 0 z) (f (n, n').fst x - f (n, n').snd x) < ε", "state_before": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\n⊢ ∀ {x_1 : ι},\n (fun n => f n x ∈ t) x_1 →\n ∀ {y : ι},\n (fun n => f n x ∈ t) y →\n ∀ (x_2 : E), x_2 ∈ Metric.ball x r → dist (OfNat.ofNat 0 x_2) (f (x_1, y).fst x - f (x_1, y).snd x) < ε", "tactic": "intro n hn n' hn' z _" }, { "state_after": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\nn : ι\nhn : f n x ∈ t\nn' : ι\nhn' : f n' x ∈ t\nz : E\na✝ : z ∈ Metric.ball x r\n⊢ dist (f (n, n').fst x) (f (n, n').snd x) < ε", "state_before": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\nn : ι\nhn : f n x ∈ t\nn' : ι\nhn' : f n' x ∈ t\nz : E\na✝ : z ∈ Metric.ball x r\n⊢ dist (OfNat.ofNat 0 z) (f (n, n').fst x - f (n, n').snd x) < ε", "tactic": "rw [dist_eq_norm, Pi.zero_apply, zero_sub, norm_neg, ← dist_eq_norm]" }, { "state_after": "no goals", "state_before": "case inr.right.intro.intro\nι : Type u_3\nl : Filter ι\nE : Type u_1\ninst✝⁴ : NormedAddCommGroup E\n𝕜 : Type u_4\ninst✝³ : IsROrC 𝕜\ninst✝² : NormedSpace 𝕜 E\nG : Type u_2\ninst✝¹ : NormedAddCommGroup G\ninst✝ : NormedSpace 𝕜 G\nf : ι → E → G\ng : E → G\nf' : ι → E → E →L[𝕜] G\ng' : E → E →L[𝕜] G\nx : E\nr : ℝ\nhf' : TendstoUniformlyOn (fun n z => f' n.fst z - f' n.snd z) 0 (l ×ˢ l) (Metric.ball x r)\nhf : ∀ (n : ι) (y : E), y ∈ Metric.ball x r → HasFDerivAt (f n) (f' n y) y\nhfg : Cauchy (map (fun n => f n x) l)\nthis✝ : NormedSpace ℝ E := NormedSpace.restrictScalars ℝ 𝕜 E\nthis : NeBot l\nhr : 0 < r\nε : ℝ\nhε : ε > 0\nt : Set G\nht : t ∈ map (fun n => f n x) l\nht' : ∀ (x : G), x ∈ t → ∀ (y : G), y ∈ t → dist x y < ε\nn : ι\nhn : f n x ∈ t\nn' : ι\nhn' : f n' x ∈ t\nz : E\na✝ : z ∈ Metric.ball x r\n⊢ dist (f (n, n').fst x) (f (n, n').snd x) < ε", "tactic": "exact ht' _ hn _ hn'" } ]
[ 225, 25 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 179, 1 ]
Mathlib/Order/Bounds/Basic.lean
BddBelow.image2_bddAbove
[ { "state_after": "case intro.intro\nα : Type u\nβ : Type v\nγ : Type w\nι : Sort x\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : Preorder γ\nf : α → β → γ\ns : Set α\nt : Set β\na✝ : α\nb✝ : β\nh₀ : ∀ (b : β), Antitone (swap f b)\nh₁ : ∀ (a : α), Antitone (f a)\na : α\nha : a ∈ lowerBounds s\nb : β\nhb : b ∈ lowerBounds t\n⊢ BddAbove (Set.image2 f s t)", "state_before": "α : Type u\nβ : Type v\nγ : Type w\nι : Sort x\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : Preorder γ\nf : α → β → γ\ns : Set α\nt : Set β\na : α\nb : β\nh₀ : ∀ (b : β), Antitone (swap f b)\nh₁ : ∀ (a : α), Antitone (f a)\n⊢ BddBelow s → BddBelow t → BddAbove (Set.image2 f s t)", "tactic": "rintro ⟨a, ha⟩ ⟨b, hb⟩" }, { "state_after": "no goals", "state_before": "case intro.intro\nα : Type u\nβ : Type v\nγ : Type w\nι : Sort x\ninst✝² : Preorder α\ninst✝¹ : Preorder β\ninst✝ : Preorder γ\nf : α → β → γ\ns : Set α\nt : Set β\na✝ : α\nb✝ : β\nh₀ : ∀ (b : β), Antitone (swap f b)\nh₁ : ∀ (a : α), Antitone (f a)\na : α\nha : a ∈ lowerBounds s\nb : β\nhb : b ∈ lowerBounds t\n⊢ BddAbove (Set.image2 f s t)", "tactic": "exact ⟨f a b, mem_upperBounds_image2_of_mem_lowerBounds h₀ h₁ ha hb⟩" } ]
[ 1481, 71 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1479, 1 ]
Mathlib/Algebra/Quaternion.lean
QuaternionAlgebra.sub_self_im
[]
[ 303, 80 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 302, 1 ]
Mathlib/Data/Fin/Tuple/Basic.lean
Fin.insertNth_zero'
[ { "state_after": "no goals", "state_before": "m n : ℕ\nα : Fin (n + 1) → Type u\nβ : Type v\nx : β\np : Fin n → β\n⊢ insertNth 0 x p = cons x p", "tactic": "simp [insertNth_zero]" } ]
[ 732, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 731, 1 ]
Mathlib/Logic/Equiv/List.lean
Encodable.mem_sortedUniv
[]
[ 208, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 207, 1 ]
Mathlib/Analysis/Normed/Group/Hom.lean
NormedAddGroupHom.NormNoninc.id
[]
[ 838, 51 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 838, 1 ]
Mathlib/Order/CompleteLattice.lean
iSup_nat_gt_zero_eq
[]
[ 1682, 31 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1681, 1 ]
Mathlib/Topology/Order/Basic.lean
csSup_mem_closure
[]
[ 2776, 36 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2775, 1 ]
Mathlib/Topology/CompactOpen.lean
ContinuousMap.continuous_comp_left
[ { "state_after": "α : Type u_3\nβ : Type u_1\nγ : Type u_2\ninst✝² : TopologicalSpace α\ninst✝¹ : TopologicalSpace β\ninst✝ : TopologicalSpace γ\ng : C(β, γ)\nf : C(α, β)\nm : Set C(α, γ)\nx✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}\ns : Set α\nhs : IsCompact s\nu : Set γ\nhu : IsOpen u\nhm : m = CompactOpen.gen s u\n⊢ IsOpen (CompactOpen.gen (↑f '' s) u)", "state_before": "α : Type u_3\nβ : Type u_1\nγ : Type u_2\ninst✝² : TopologicalSpace α\ninst✝¹ : TopologicalSpace β\ninst✝ : TopologicalSpace γ\ng : C(β, γ)\nf : C(α, β)\nm : Set C(α, γ)\nx✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}\ns : Set α\nhs : IsCompact s\nu : Set γ\nhu : IsOpen u\nhm : m = CompactOpen.gen s u\n⊢ IsOpen ((fun g => comp g f) ⁻¹' m)", "tactic": "rw [hm, image_gen f hs hu]" }, { "state_after": "no goals", "state_before": "α : Type u_3\nβ : Type u_1\nγ : Type u_2\ninst✝² : TopologicalSpace α\ninst✝¹ : TopologicalSpace β\ninst✝ : TopologicalSpace γ\ng : C(β, γ)\nf : C(α, β)\nm : Set C(α, γ)\nx✝ : m ∈ {m | ∃ s x u x, m = CompactOpen.gen s u}\ns : Set α\nhs : IsCompact s\nu : Set γ\nhu : IsOpen u\nhm : m = CompactOpen.gen s u\n⊢ IsOpen (CompactOpen.gen (↑f '' s) u)", "tactic": "exact ContinuousMap.isOpen_gen (hs.image f.2) hu" } ]
[ 125, 53 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 122, 1 ]
Mathlib/Order/SuccPred/Basic.lean
Order.Ioo_succ_right_eq_insert_of_not_isMax
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝¹ : PartialOrder α\ninst✝ : SuccOrder α\na b : α\nh₁ : a < b\nh₂ : ¬IsMax b\n⊢ Ioo a (succ b) = insert b (Ioo a b)", "tactic": "simp_rw [← Iio_inter_Ioi, Iio_succ_eq_insert_of_not_isMax h₂, insert_inter_of_mem (mem_Ioi.2 h₁)]" } ]
[ 471, 100 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 469, 1 ]
Mathlib/GroupTheory/Submonoid/Basic.lean
Submonoid.closure_iUnion
[]
[ 536, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 535, 1 ]
Mathlib/Data/Set/Intervals/Basic.lean
Set.Iio_subset_Iio_union_Ico
[]
[ 1374, 74 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1373, 1 ]
Mathlib/Topology/Algebra/Nonarchimedean/Basic.lean
NonarchimedeanRing.left_mul_subset
[]
[ 143, 98 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 141, 1 ]
Mathlib/CategoryTheory/Category/Basic.lean
CategoryTheory.ite_comp
[ { "state_after": "no goals", "state_before": "C : Type u\ninst✝¹ : Category C\nX✝ Y✝ Z✝ : C\nP : Prop\ninst✝ : Decidable P\nX Y Z : C\nf f' : X ⟶ Y\ng : Y ⟶ Z\n⊢ (if P then f else f') ≫ g = if P then f ≫ g else f' ≫ g", "tactic": "aesop" } ]
[ 247, 72 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 246, 1 ]
Mathlib/Algebra/Order/Floor.lean
Nat.le_floor_iff
[]
[ 134, 28 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 133, 1 ]
Mathlib/Data/Num/Lemmas.lean
ZNum.cast_mul
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : Ring α\nm n : ZNum\n⊢ ↑(m * n) = ↑m * ↑n", "tactic": "rw [← cast_to_int, mul_to_int, Int.cast_mul, cast_to_int, cast_to_int]" } ]
[ 1355, 73 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1354, 1 ]
Mathlib/RingTheory/Subsemiring/Basic.lean
Subsemiring.top_prod
[ { "state_after": "no goals", "state_before": "R : Type u\nS : Type v\nT : Type w\ninst✝² : NonAssocSemiring R\nM : Submonoid R\ninst✝¹ : NonAssocSemiring S\ninst✝ : NonAssocSemiring T\ns : Subsemiring S\nx : R × S\n⊢ x ∈ prod ⊤ s ↔ x ∈ comap (RingHom.snd R S) s", "tactic": "simp [mem_prod, MonoidHom.coe_snd]" } ]
[ 1074, 53 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1073, 1 ]
Mathlib/Topology/Connected.lean
connectedComponent_nonempty
[]
[ 605, 30 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 604, 1 ]
Mathlib/Analysis/Calculus/Inverse.lean
HasStrictFDerivAt.map_nhds_eq_of_surj
[ { "state_after": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\n⊢ map f (𝓝 a) = 𝓝 (f a)", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\n⊢ map f (𝓝 a) = 𝓝 (f a)", "tactic": "let f'symm := f'.nonlinearRightInverseOfSurjective h" }, { "state_after": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\n⊢ map f (𝓝 a) = 𝓝 (f a)", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\n⊢ map f (𝓝 a) = 𝓝 (f a)", "tactic": "set c : ℝ≥0 := f'symm.nnnorm⁻¹ / 2 with hc" }, { "state_after": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\n⊢ map f (𝓝 a) = 𝓝 (f a)", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\n⊢ map f (𝓝 a) = 𝓝 (f a)", "tactic": "have f'symm_pos : 0 < f'symm.nnnorm := f'.nonlinearRightInverseOfSurjective_nnnorm_pos h" }, { "state_after": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\ncpos : 0 < c\n⊢ map f (𝓝 a) = 𝓝 (f a)", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\n⊢ map f (𝓝 a) = 𝓝 (f a)", "tactic": "have cpos : 0 < c := by simp [hc, half_pos, inv_pos, f'symm_pos]" }, { "state_after": "case intro.intro\n𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\ncpos : 0 < c\ns : Set E\ns_nhds : s ∈ 𝓝 a\nhs : ApproximatesLinearOn f f' s c\n⊢ map f (𝓝 a) = 𝓝 (f a)", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\ncpos : 0 < c\n⊢ map f (𝓝 a) = 𝓝 (f a)", "tactic": "obtain ⟨s, s_nhds, hs⟩ : ∃ s ∈ 𝓝 a, ApproximatesLinearOn f f' s c :=\n hf.approximates_deriv_on_nhds (Or.inr cpos)" }, { "state_after": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\ncpos : 0 < c\ns : Set E\ns_nhds : s ∈ 𝓝 a\nhs : ApproximatesLinearOn f f' s c\n⊢ f'symm.nnnorm⁻¹ ≠ 0", "state_before": "case intro.intro\n𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\ncpos : 0 < c\ns : Set E\ns_nhds : s ∈ 𝓝 a\nhs : ApproximatesLinearOn f f' s c\n⊢ map f (𝓝 a) = 𝓝 (f a)", "tactic": "apply hs.map_nhds_eq f'symm s_nhds (Or.inr (NNReal.half_lt_self _))" }, { "state_after": "no goals", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\ncpos : 0 < c\ns : Set E\ns_nhds : s ∈ 𝓝 a\nhs : ApproximatesLinearOn f f' s c\n⊢ f'symm.nnnorm⁻¹ ≠ 0", "tactic": "simp [ne_of_gt f'symm_pos]" }, { "state_after": "no goals", "state_before": "𝕜 : Type u_3\ninst✝¹⁰ : NontriviallyNormedField 𝕜\nE : Type u_1\ninst✝⁹ : NormedAddCommGroup E\ninst✝⁸ : NormedSpace 𝕜 E\nF : Type u_2\ninst✝⁷ : NormedAddCommGroup F\ninst✝⁶ : NormedSpace 𝕜 F\nG : Type ?u.515211\ninst✝⁵ : NormedAddCommGroup G\ninst✝⁴ : NormedSpace 𝕜 G\nG' : Type ?u.515314\ninst✝³ : NormedAddCommGroup G'\ninst✝² : NormedSpace 𝕜 G'\nε : ℝ\ninst✝¹ : CompleteSpace E\ninst✝ : CompleteSpace F\nf : E → F\nf' : E →L[𝕜] F\na : E\nhf : HasStrictFDerivAt f f' a\nh : LinearMap.range f' = ⊤\nf'symm : ContinuousLinearMap.NonlinearRightInverse f' := ContinuousLinearMap.nonlinearRightInverseOfSurjective f' h\nc : ℝ≥0 := f'symm.nnnorm⁻¹ / 2\nhc : c = f'symm.nnnorm⁻¹ / 2\nf'symm_pos : 0 < f'symm.nnnorm\n⊢ 0 < c", "tactic": "simp [hc, half_pos, inv_pos, f'symm_pos]" } ]
[ 562, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 552, 1 ]
Mathlib/Algebra/Parity.lean
IsSquare.pow
[ { "state_after": "case intro\nF : Type ?u.8146\nα : Type u_1\nβ : Type ?u.8152\nR : Type ?u.8155\ninst✝ : Monoid α\nn✝ n : ℕ\na : α\n⊢ IsSquare ((a * a) ^ n)", "state_before": "F : Type ?u.8146\nα : Type u_1\nβ : Type ?u.8152\nR : Type ?u.8155\ninst✝ : Monoid α\nn✝ : ℕ\na : α\nn : ℕ\n⊢ IsSquare a → IsSquare (a ^ n)", "tactic": "rintro ⟨a, rfl⟩" }, { "state_after": "no goals", "state_before": "case intro\nF : Type ?u.8146\nα : Type u_1\nβ : Type ?u.8152\nR : Type ?u.8155\ninst✝ : Monoid α\nn✝ n : ℕ\na : α\n⊢ IsSquare ((a * a) ^ n)", "tactic": "exact ⟨a ^ n, (Commute.refl _).mul_pow _⟩" } ]
[ 108, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 106, 1 ]
Mathlib/Data/Set/Image.lean
Set.mem_range_self
[]
[ 657, 11 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 656, 1 ]
Mathlib/Algebra/Group/Units.lean
IsUnit.mul_right_cancel
[]
[ 788, 19 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 787, 11 ]
Mathlib/GroupTheory/MonoidLocalization.lean
Submonoid.LocalizationMap.lift_left_inverse
[ { "state_after": "M : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\n⊢ ↑(toMap f) (sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst =\n ↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * z", "state_before": "M : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\n⊢ ↑(lift k (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap f) ↑y)))\n (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z) =\n z", "tactic": "rw [lift_spec]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst =\n ↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * z", "state_before": "M : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\n⊢ ↑(toMap f) (sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst =\n ↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * z", "tactic": "cases' f.surj z with x hx" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst =\n ↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * mk' f x.fst x.snd", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst =\n ↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * z", "tactic": "conv_rhs =>\n congr\n next => skip\n rw [f.eq_mk'_iff_mul_eq.2 hx]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) ((sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst * ↑x.snd) =\n ↑(toMap f) (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst)", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst =\n ↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * mk' f x.fst x.snd", "tactic": "rw [mk', ← mul_assoc, mul_inv_right f.map_units, ← f.toMap.map_mul, ← f.toMap.map_mul]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k) ((sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst * ↑x.snd) =\n ↑(toMap k) (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst)", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) ((sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst * ↑x.snd) =\n ↑(toMap f) (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst)", "tactic": "apply k.eq_of_eq f.map_units" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k) (sec f z).fst *\n (↑(toMap k) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap k) ↑x.snd) =\n ↑(toMap k) ↑(sec f z).snd *\n (↑(toMap k) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap k) x.fst)", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k) ((sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).fst * ↑x.snd) =\n ↑(toMap k) (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst)", "tactic": "rw [k.toMap.map_mul, k.toMap.map_mul, ← sec_spec, mul_assoc, lift_spec_mul]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k)\n ((sec f z).fst * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑x.snd)) =\n ↑(toMap k)\n (↑(sec f z).snd * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst))", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k) (sec f z).fst *\n (↑(toMap k) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap k) ↑x.snd) =\n ↑(toMap k) ↑(sec f z).snd *\n (↑(toMap k) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap k) x.fst)", "tactic": "repeat' rw [← k.toMap.map_mul]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f)\n ((sec f z).fst * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑x.snd)) =\n ↑(toMap f)\n (↑(sec f z).snd * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst))", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k)\n ((sec f z).fst * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑x.snd)) =\n ↑(toMap k)\n (↑(sec f z).snd * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst))", "tactic": "apply f.eq_of_eq k.map_units" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec f z).fst *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) ↑x.snd) =\n ↑(toMap f) ↑(sec f z).snd *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) x.fst)", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f)\n ((sec f z).fst * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑x.snd)) =\n ↑(toMap f)\n (↑(sec f z).snd * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst))", "tactic": "repeat' rw [f.toMap.map_mul]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) ↑(sec f z).snd * z *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) ↑x.snd) =\n ↑(toMap f) ↑(sec f z).snd *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd *\n (z * ↑(toMap f) ↑x.snd))", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec f z).fst *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) ↑x.snd) =\n ↑(toMap f) ↑(sec f z).snd *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) x.fst)", "tactic": "rw [sec_spec', ← hx]" }, { "state_after": "no goals", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) ↑(sec f z).snd * z *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) ↑x.snd) =\n ↑(toMap f) ↑(sec f z).snd *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd *\n (z * ↑(toMap f) ↑x.snd))", "tactic": "ac_rfl" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k)\n ((sec f z).fst * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑x.snd)) =\n ↑(toMap k)\n (↑(sec f z).snd * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst))", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap k)\n ((sec f z).fst * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑x.snd)) =\n ↑(toMap k)\n (↑(sec f z).snd * (↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * x.fst))", "tactic": "rw [← k.toMap.map_mul]" }, { "state_after": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec f z).fst *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) ↑x.snd) =\n ↑(toMap f) ↑(sec f z).snd *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) x.fst)", "state_before": "case intro\nM : Type u_1\ninst✝² : CommMonoid M\nS : Submonoid M\nN : Type u_3\ninst✝¹ : CommMonoid N\nP : Type u_2\ninst✝ : CommMonoid P\nf : LocalizationMap S N\ng : M →* P\nhg : ∀ (y : { x // x ∈ S }), IsUnit (↑g ↑y)\nk : LocalizationMap S P\nz : N\nx : M × { x // x ∈ S }\nhx : z * ↑(toMap f) ↑x.snd = ↑(toMap f) x.fst\n⊢ ↑(toMap f) (sec f z).fst *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) ↑x.snd) =\n ↑(toMap f) ↑(sec f z).snd *\n (↑(toMap f) ↑(sec k (↑(lift f (_ : ∀ (y : { x // x ∈ S }), IsUnit (↑(toMap k) ↑y))) z)).snd * ↑(toMap f) x.fst)", "tactic": "rw [f.toMap.map_mul]" } ]
[ 1079, 9 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1064, 1 ]
Mathlib/FieldTheory/Fixed.lean
finrank_algHom
[]
[ 342, 86 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 340, 1 ]
Mathlib/Algebra/Module/LinearMap.lean
LinearMap.restrictScalars_inj
[]
[ 476, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 474, 1 ]
Mathlib/Data/PFunctor/Multivariate/M.lean
MvPFunctor.M.dest_corec
[ { "state_after": "n : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ dest P (corec P g x) = ?m.38931\n\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ ?m.38931 = (TypeVec.id ::: corec P g) <$$> g x\n\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ Obj P (α ::: M P α)", "state_before": "n : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ dest P (corec P g x) = (TypeVec.id ::: corec P g) <$$> g x", "tactic": "trans" }, { "state_after": "n : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ { fst := (g x).fst,\n snd :=\n splitFun (dropFun (g x).snd)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘\n lastFun (g x).snd) } =\n (TypeVec.id ::: corec P g) <$$> g x", "state_before": "n : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ dest P (corec P g x) = ?m.38931\n\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ ?m.38931 = (TypeVec.id ::: corec P g) <$$> g x\n\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ Obj P (α ::: M P α)", "tactic": "apply M.dest_corec'" }, { "state_after": "case mk\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ { fst := { fst := a, snd := f }.fst,\n snd :=\n splitFun (dropFun { fst := a, snd := f }.snd)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘\n lastFun { fst := a, snd := f }.snd) } =\n (TypeVec.id ::: corec P g) <$$> { fst := a, snd := f }", "state_before": "n : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\n⊢ { fst := (g x).fst,\n snd :=\n splitFun (dropFun (g x).snd)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘\n lastFun (g x).snd) } =\n (TypeVec.id ::: corec P g) <$$> g x", "tactic": "cases' g x with a f" }, { "state_after": "case mk\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ { fst := a,\n snd :=\n splitFun (dropFun f)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘ lastFun f) } =\n (TypeVec.id ::: corec P g) <$$> { fst := a, snd := f }", "state_before": "case mk\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ { fst := { fst := a, snd := f }.fst,\n snd :=\n splitFun (dropFun { fst := a, snd := f }.snd)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘\n lastFun { fst := a, snd := f }.snd) } =\n (TypeVec.id ::: corec P g) <$$> { fst := a, snd := f }", "tactic": "dsimp" }, { "state_after": "case mk\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ { fst := a,\n snd :=\n splitFun (dropFun f)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘ lastFun f) } =\n { fst := a, snd := (TypeVec.id ::: corec P g) ⊚ f }", "state_before": "case mk\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ { fst := a,\n snd :=\n splitFun (dropFun f)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘ lastFun f) } =\n (TypeVec.id ::: corec P g) <$$> { fst := a, snd := f }", "tactic": "rw [MvPFunctor.map_eq]" }, { "state_after": "case mk.e_snd\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ splitFun (dropFun f)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘ lastFun f) =\n (TypeVec.id ::: corec P g) ⊚ f", "state_before": "case mk\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ { fst := a,\n snd :=\n splitFun (dropFun f)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘ lastFun f) } =\n { fst := a, snd := (TypeVec.id ::: corec P g) ⊚ f }", "tactic": "congr" }, { "state_after": "no goals", "state_before": "case mk.e_snd\nn : ℕ\nP : MvPFunctor (n + 1)\nα : TypeVec n\nβ : Type u\ng : β → Obj P (α ::: β)\nx : β\na : P.A\nf : B P a ⟹ α ::: β\n⊢ splitFun (dropFun f)\n ((corec' P (fun b => (g b).fst) (fun b => dropFun (g b).snd) fun b => lastFun (g b).snd) ∘ lastFun f) =\n (TypeVec.id ::: corec P g) ⊚ f", "tactic": "conv =>\n rhs\n rw [← split_dropFun_lastFun f, appendFun_comp_splitFun]" } ]
[ 262, 60 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 254, 1 ]
Mathlib/Topology/Category/TopCat/Limits/Cofiltered.lean
TopCat.isTopologicalBasis_cofiltered_limit
[ { "state_after": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "tactic": "let D := limitConeInfi F" }, { "state_after": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "tactic": "let E : C.pt ≅ D.pt := hC.conePointUniqueUpToIso (limitConeInfiIsLimit _)" }, { "state_after": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "tactic": "have hE : Inducing E.hom := (TopCat.homeoOfIso E).inducing" }, { "state_after": "case h.e'_3\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\n⊢ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} =\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "convert isTopologicalBasis_iInf hT fun j (x : D.pt) => D.π.app j x using 1" }, { "state_after": "case h.e'_3.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} ↔\n U0 ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "state_before": "case h.e'_3\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\n⊢ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} =\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "tactic": "ext U0" }, { "state_after": "case h.e'_3.h.mp\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} →\n U0 ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}\n\ncase h.e'_3.h.mpr\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\n⊢ U0 ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i} →\n U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} ↔\n U0 ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "tactic": "constructor" }, { "state_after": "case h.e'_3.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\n⊢ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V} =\n Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\n⊢ IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "tactic": "convert this.inducing hE" }, { "state_after": "case h.e'_3.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nU0 : Set ↑C.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V} ↔\n U0 ∈ Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\n⊢ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V} =\n Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "ext U0" }, { "state_after": "case h.e'_3.h.h.mp\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nU0 : Set ↑C.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V} →\n U0 ∈ Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\n\ncase h.e'_3.h.h.mpr\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nU0 : Set ↑C.pt\n⊢ U0 ∈ Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} →\n U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nU0 : Set ↑C.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V} ↔\n U0 ∈ Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "constructor" }, { "state_after": "case h.e'_3.h.h.mp.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\n⊢ (forget TopCat).map (C.π.app j) ⁻¹' V ∈\n Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.h.mp\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nU0 : Set ↑C.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V} →\n U0 ∈ Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "rintro ⟨j, V, hV, rfl⟩" }, { "state_after": "no goals", "state_before": "case h.e'_3.h.h.mp.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\n⊢ (forget TopCat).map (C.π.app j) ⁻¹' V ∈\n Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "refine' ⟨D.π.app j ⁻¹' V, ⟨j, V, hV, rfl⟩, rfl⟩" }, { "state_after": "case h.e'_3.h.h.mpr.intro.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\n⊢ (forget TopCat).map E.hom ⁻¹' ((forget TopCat).map (D.π.app j) ⁻¹' V) ∈\n {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.h.mpr\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nU0 : Set ↑C.pt\n⊢ U0 ∈ Set.preimage ((forget TopCat).map E.hom) '' {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} →\n U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "tactic": "rintro ⟨W, ⟨j, V, hV, rfl⟩, rfl⟩" }, { "state_after": "no goals", "state_before": "case h.e'_3.h.h.mpr.intro.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nthis : IsTopologicalBasis {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}\ne_1✝ : ↑C.pt = (forget TopCat).obj C.pt\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\n⊢ (forget TopCat).map E.hom ⁻¹' ((forget TopCat).map (D.π.app j) ⁻¹' V) ∈\n {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (C.π.app j) ⁻¹' V}", "tactic": "refine' ⟨j, V, hV, rfl⟩" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\n⊢ (forget TopCat).map (D.π.app j) ⁻¹' V ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "state_before": "case h.e'_3.h.mp\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V} →\n U0 ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "tactic": "rintro ⟨j, V, hV, rfl⟩" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ (forget TopCat).map (D.π.app j) ⁻¹' V ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "state_before": "case h.e'_3.h.mp.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\n⊢ (forget TopCat).map (D.π.app j) ⁻¹' V ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "tactic": "let U : ∀ i, Set (F.obj i) := fun i =>\n if h : i = j then by\n rw [h]\n exact V\n else Set.univ" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ ∀ (i : J), i ∈ {j} → U i ∈ T i\n\ncase h.e'_3.h.mp.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ (forget TopCat).map (D.π.app j) ⁻¹' V = ⋂ (i : J) (_ : i ∈ {j}), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i", "state_before": "case h.e'_3.h.mp.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ (forget TopCat).map (D.π.app j) ⁻¹' V ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i}", "tactic": "refine' ⟨U, {j}, _, _⟩" }, { "state_after": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\ni : J\nh : i = j\n⊢ Set ↑(F.obj j)", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\ni : J\nh : i = j\n⊢ Set ↑(F.obj i)", "tactic": "rw [h]" }, { "state_after": "no goals", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\ni : J\nh : i = j\n⊢ Set ↑(F.obj j)", "tactic": "exact V" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i ∈ {j}\n⊢ U i ∈ T i", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ ∀ (i : J), i ∈ {j} → U i ∈ T i", "tactic": "rintro i h" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i = j\n⊢ U i ∈ T i", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i ∈ {j}\n⊢ U i ∈ T i", "tactic": "rw [Finset.mem_singleton] at h" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i = j\n⊢ (if h : i = j then cast (_ : Set ↑(F.obj j) = Set ↑(F.obj i)) V else Set.univ) ∈ T i", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i = j\n⊢ U i ∈ T i", "tactic": "dsimp" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i = j\n⊢ cast (_ : Set ↑(F.obj j) = Set ↑(F.obj i)) V ∈ T i", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i = j\n⊢ (if h : i = j then cast (_ : Set ↑(F.obj j) = Set ↑(F.obj i)) V else Set.univ) ∈ T i", "tactic": "rw [dif_pos h]" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\ni : J\nV : Set ↑(F.obj i)\nhV : V ∈ T i\nU : (i : J) → Set ↑(F.obj i) :=\n fun i_1 => if h : i_1 = i then Eq.mpr (_ : Set ↑(F.obj i_1) = Set ↑(F.obj i)) V else Set.univ\n⊢ cast (_ : Set ↑(F.obj i) = Set ↑(F.obj i)) V ∈ T i", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\ni : J\nh : i = j\n⊢ cast (_ : Set ↑(F.obj j) = Set ↑(F.obj i)) V ∈ T i", "tactic": "subst h" }, { "state_after": "no goals", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\ni : J\nV : Set ↑(F.obj i)\nhV : V ∈ T i\nU : (i : J) → Set ↑(F.obj i) :=\n fun i_1 => if h : i_1 = i then Eq.mpr (_ : Set ↑(F.obj i_1) = Set ↑(F.obj i)) V else Set.univ\n⊢ cast (_ : Set ↑(F.obj i) = Set ↑(F.obj i)) V ∈ T i", "tactic": "exact hV" }, { "state_after": "case h.e'_3.h.mp.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ (forget TopCat).map ((limitConeInfi F).π.app j) ⁻¹' V =\n ⋂ (i : J) (_ : i ∈ {j}),\n (fun x => (forget TopCat).map ((limitConeInfi F).π.app i) x) ⁻¹'\n if h : i = j then cast (_ : Set ↑(F.obj j) = Set ↑(F.obj i)) V else Set.univ", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ (forget TopCat).map (D.π.app j) ⁻¹' V = ⋂ (i : J) (_ : i ∈ {j}), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i", "tactic": "dsimp" }, { "state_after": "no goals", "state_before": "case h.e'_3.h.mp.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nj : J\nV : Set ↑(F.obj j)\nhV : V ∈ T j\nU : (i : J) → Set ↑(F.obj i) := fun i => if h : i = j then Eq.mpr (_ : Set ↑(F.obj i) = Set ↑(F.obj j)) V else Set.univ\n⊢ (forget TopCat).map ((limitConeInfi F).π.app j) ⁻¹' V =\n ⋂ (i : J) (_ : i ∈ {j}),\n (fun x => (forget TopCat).map ((limitConeInfi F).π.app i) x) ⁻¹'\n if h : i = j then cast (_ : Set ↑(F.obj j) = Set ↑(F.obj i)) V else Set.univ", "tactic": "simp" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.mpr\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\n⊢ U0 ∈\n {S |\n ∃ U F_1,\n (∀ (i : J), i ∈ F_1 → U i ∈ T i) ∧\n S = ⋂ (i : J) (_ : i ∈ F_1), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i} →\n U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "rintro ⟨U, G, h1, h2⟩" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.mpr.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "obtain ⟨j, hj⟩ := IsCofiltered.inf_objs_exists G" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "let g : ∀ (e) (_he : e ∈ G), j ⟶ e := fun _ he => (hj he).some" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "let Vs : J → Set (F.obj j) := fun e => if h : e ∈ G then F.map (g e h) ⁻¹' U e else Set.univ" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "let V : Set (F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ V ∈ T j\n\ncase h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ U0 = (forget TopCat).map (D.π.app j) ⁻¹' V", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ U0 ∈ {U | ∃ j V, V ∈ T j ∧ U = (forget TopCat).map (D.π.app j) ⁻¹' V}", "tactic": "refine' ⟨j, V, _, _⟩" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\n⊢ ∀ (e : J), e ∈ G → Vs e ∈ T j", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\n⊢ V ∈ T j", "tactic": "refine' this _ _ _ (univ _) (inter _) _" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\ne : J\nhe : e ∈ G\n⊢ Vs e ∈ T j", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\n⊢ ∀ (e : J), e ∈ G → Vs e ∈ T j", "tactic": "intro e he" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\ne : J\nhe : e ∈ G\n⊢ (if h : e ∈ G then (forget TopCat).map (F.map (Nonempty.some (_ : Nonempty (j ⟶ e)))) ⁻¹' U e else Set.univ) ∈ T j", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\ne : J\nhe : e ∈ G\n⊢ Vs e ∈ T j", "tactic": "dsimp" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (F.map (Nonempty.some (_ : Nonempty (j ⟶ e)))) ⁻¹' U e ∈ T j", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\ne : J\nhe : e ∈ G\n⊢ (if h : e ∈ G then (forget TopCat).map (F.map (Nonempty.some (_ : Nonempty (j ⟶ e)))) ⁻¹' U e else Set.univ) ∈ T j", "tactic": "rw [dif_pos he]" }, { "state_after": "no goals", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_1\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nthis :\n ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (F.map (Nonempty.some (_ : Nonempty (j ⟶ e)))) ⁻¹' U e ∈ T j", "tactic": "exact compat j e (g e he) (U e) (h1 e he)" }, { "state_after": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\nE : Finset J\n⊢ ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ ∀ (S : Set (Set ↑(F.obj j))) (E : Finset J) (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S", "tactic": "intro S E" }, { "state_after": "case empty\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\n⊢ ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ ∅ → P e ∈ S) → (⋂ (e : J) (_ : e ∈ ∅), P e) ∈ S\n\ncase insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\n⊢ ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ insert a E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ insert a E), P e) ∈ S", "state_before": "J : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\nE : Finset J\n⊢ ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S", "tactic": "induction' E using Finset.induction_on with a E _ hh1" }, { "state_after": "case empty\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\nP : J → Set ↑(F.obj j)\nhe : Set.univ ∈ S\nx✝ : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\n⊢ (∀ (e : J), e ∈ ∅ → P e ∈ S) → (⋂ (e : J) (_ : e ∈ ∅), P e) ∈ S", "state_before": "case empty\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\n⊢ ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ ∅ → P e ∈ S) → (⋂ (e : J) (_ : e ∈ ∅), P e) ∈ S", "tactic": "intro P he _" }, { "state_after": "no goals", "state_before": "case empty\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\nP : J → Set ↑(F.obj j)\nhe : Set.univ ∈ S\nx✝ : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\n⊢ (∀ (e : J), e ∈ ∅ → P e ∈ S) → (⋂ (e : J) (_ : e ∈ ∅), P e) ∈ S", "tactic": "simpa" }, { "state_after": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\n⊢ (⋂ (e : J) (_ : e ∈ insert a E), hh2 e) ∈ S", "state_before": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\n⊢ ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ insert a E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ insert a E), P e) ∈ S", "tactic": "intro hh2 hh3 hh4 hh5" }, { "state_after": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\n⊢ (hh2 a ∩ ⋂ (x : J) (_ : x ∈ E), hh2 x) ∈ S", "state_before": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\n⊢ (⋂ (e : J) (_ : e ∈ insert a E), hh2 e) ∈ S", "tactic": "rw [Finset.set_biInter_insert]" }, { "state_after": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\n⊢ ∀ (e : J), e ∈ E → hh2 e ∈ S", "state_before": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\n⊢ (hh2 a ∩ ⋂ (x : J) (_ : x ∈ E), hh2 x) ∈ S", "tactic": "refine' hh4 _ _ (hh5 _ (Finset.mem_insert_self _ _)) (hh1 _ hh3 hh4 _)" }, { "state_after": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\ne : J\nhe : e ∈ E\n⊢ hh2 e ∈ S", "state_before": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\n⊢ ∀ (e : J), e ∈ E → hh2 e ∈ S", "tactic": "intro e he" }, { "state_after": "no goals", "state_before": "case insert\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE✝ : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E✝.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\nS : Set (Set ↑(F.obj j))\na : J\nE : Finset J\na✝ : ¬a ∈ E\nhh1 :\n ∀ (P : J → Set ↑(F.obj j)),\n Set.univ ∈ S →\n (∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S) →\n (∀ (e : J), e ∈ E → P e ∈ S) → (⋂ (e : J) (_ : e ∈ E), P e) ∈ S\nhh2 : J → Set ↑(F.obj j)\nhh3 : Set.univ ∈ S\nhh4 : ∀ (A B : Set ↑(F.obj j)), A ∈ S → B ∈ S → A ∩ B ∈ S\nhh5 : ∀ (e : J), e ∈ insert a E → hh2 e ∈ S\ne : J\nhe : e ∈ E\n⊢ hh2 e ∈ S", "tactic": "exact hh5 e (Finset.mem_insert_of_mem he)" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) = (forget TopCat).map (D.π.app j) ⁻¹' V", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ U0 = (forget TopCat).map (D.π.app j) ⁻¹' V", "tactic": "rw [h2]" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) =\n (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (e : J) (_ : e ∈ G), Vs e", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) = (forget TopCat).map (D.π.app j) ⁻¹' V", "tactic": "change _ = (D.π.app j)⁻¹' ⋂ (e : J) (_ : e ∈ G), Vs e" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) =\n ⋂ (i : J), (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (_ : i ∈ G), Vs i", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) =\n (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (e : J) (_ : e ∈ G), Vs e", "tactic": "rw [Set.preimage_iInter]" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (fun i => ⋂ (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) = fun i =>\n (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (_ : i ∈ G), Vs i", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) =\n ⋂ (i : J), (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (_ : i ∈ G), Vs i", "tactic": "apply congrArg" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\n⊢ (⋂ (_ : e ∈ G), (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e) =\n (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (_ : e ∈ G), Vs e", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\n⊢ (fun i => ⋂ (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i) = fun i =>\n (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (_ : i ∈ G), Vs i", "tactic": "ext1 e" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\n⊢ (⋂ (_ : e ∈ G), (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e) =\n ⋂ (_ : e ∈ G), (forget TopCat).map (D.π.app j) ⁻¹' Vs e", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\n⊢ (⋂ (_ : e ∈ G), (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e) =\n (forget TopCat).map (D.π.app j) ⁻¹' ⋂ (_ : e ∈ G), Vs e", "tactic": "erw [Set.preimage_iInter]" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\n⊢ (fun x => (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e) = fun i => (forget TopCat).map (D.π.app j) ⁻¹' Vs e", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\n⊢ (⋂ (_ : e ∈ G), (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e) =\n ⋂ (_ : e ∈ G), (forget TopCat).map (D.π.app j) ⁻¹' Vs e", "tactic": "apply congrArg" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e = (forget TopCat).map (D.π.app j) ⁻¹' Vs e", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\n⊢ (fun x => (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e) = fun i => (forget TopCat).map (D.π.app j) ⁻¹' Vs e", "tactic": "ext1 he" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (D.π.app e) ⁻¹' U e =\n (forget TopCat).map (D.π.app j) ⁻¹' if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (fun x => (forget TopCat).map (D.π.app e) x) ⁻¹' U e = (forget TopCat).map (D.π.app j) ⁻¹' Vs e", "tactic": "change (forget TopCat).map (D.π.app e)⁻¹' U e =\n (forget TopCat).map (D.π.app j) ⁻¹' if h : e ∈ G then F.map (g e h) ⁻¹' U e else Set.univ" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (D.π.app e) ⁻¹' U e =\n (forget TopCat).map (F.map (g e he)) ∘ (forget TopCat).map (D.π.app j) ⁻¹' U e", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (D.π.app e) ⁻¹' U e =\n (forget TopCat).map (D.π.app j) ⁻¹' if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ", "tactic": "rw [dif_pos he, ← Set.preimage_comp]" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ Set.preimage ((forget TopCat).map (D.π.app e)) =\n Set.preimage ((forget TopCat).map (F.map (g e he)) ∘ (forget TopCat).map (D.π.app j))", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (D.π.app e) ⁻¹' U e =\n (forget TopCat).map (F.map (g e he)) ∘ (forget TopCat).map (D.π.app j) ⁻¹' U e", "tactic": "apply congrFun" }, { "state_after": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (D.π.app e) = (forget TopCat).map (F.map (g e he)) ∘ (forget TopCat).map (D.π.app j)", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ Set.preimage ((forget TopCat).map (D.π.app e)) =\n Set.preimage ((forget TopCat).map (F.map (g e he)) ∘ (forget TopCat).map (D.π.app j))", "tactic": "apply congrArg" }, { "state_after": "no goals", "state_before": "case h.e'_3.h.mpr.intro.intro.intro.intro.refine'_2.h.h.h.h.h.h\nJ : Type v\ninst✝¹ : SmallCategory J\ninst✝ : IsCofiltered J\nF : J ⥤ TopCatMax\nC : Cone F\nhC : IsLimit C\nT : (j : J) → Set (Set ↑(F.obj j))\nhT : ∀ (j : J), IsTopologicalBasis (T j)\nuniv : ∀ (i : J), Set.univ ∈ T i\ninter : ∀ (i : J) (U1 U2 : Set ↑(F.obj i)), U1 ∈ T i → U2 ∈ T i → U1 ∩ U2 ∈ T i\ncompat : ∀ (i j : J) (f : i ⟶ j) (V : Set ↑(F.obj j)), V ∈ T j → (forget TopCat).map (F.map f) ⁻¹' V ∈ T i\nD : Cone F := limitConeInfi F\nE : C.pt ≅ D.pt := IsLimit.conePointUniqueUpToIso hC (limitConeInfiIsLimit F)\nhE : Inducing ((forget TopCat).map E.hom)\nU0 : Set ↑D.pt\nU : (i : J) → Set ↑(F.obj i)\nG : Finset J\nh1 : ∀ (i : J), i ∈ G → U i ∈ T i\nh2 : U0 = ⋂ (i : J) (_ : i ∈ G), (fun x => (forget TopCat).map (D.π.app i) x) ⁻¹' U i\nj : J\nhj : ∀ {X : J}, X ∈ G → Nonempty (j ⟶ X)\ng : (e : J) → e ∈ G → (j ⟶ e) := fun x he => Nonempty.some (_ : Nonempty (j ⟶ x))\nVs : J → Set ↑(F.obj j) := fun e => if h : e ∈ G then (forget TopCat).map (F.map (g e h)) ⁻¹' U e else Set.univ\nV : Set ↑(F.obj j) := ⋂ (e : J) (_ : e ∈ G), Vs e\ne : J\nhe : e ∈ G\n⊢ (forget TopCat).map (D.π.app e) = (forget TopCat).map (F.map (g e he)) ∘ (forget TopCat).map (D.π.app j)", "tactic": "rw [←coe_comp, D.w]" } ]
[ 129, 28 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 45, 1 ]
Mathlib/Analysis/Convex/Hull.lean
convexHull_subset_affineSpan
[]
[ 218, 65 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 217, 1 ]
Mathlib/Algebra/Associated.lean
associated_unit_mul_left_iff
[]
[ 504, 42 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 502, 1 ]
Mathlib/MeasureTheory/Constructions/Pi.lean
MeasureTheory.Measure.pi_pi
[ { "state_after": "ι : Type u_2\nι' : Type ?u.3051144\nα : ι → Type u_1\ninst✝² : Fintype ι\nm : (i : ι) → OuterMeasure (α i)\ninst✝¹ : (i : ι) → MeasurableSpace (α i)\nμ : (i : ι) → Measure (α i)\ninst✝ : ∀ (i : ι), SigmaFinite (μ i)\ns : (i : ι) → Set (α i)\nthis : Encodable ι\n⊢ ↑↑(Measure.pi μ) (Set.pi univ s) = ∏ i : ι, ↑↑(μ i) (s i)", "state_before": "ι : Type u_2\nι' : Type ?u.3051144\nα : ι → Type u_1\ninst✝² : Fintype ι\nm : (i : ι) → OuterMeasure (α i)\ninst✝¹ : (i : ι) → MeasurableSpace (α i)\nμ : (i : ι) → Measure (α i)\ninst✝ : ∀ (i : ι), SigmaFinite (μ i)\ns : (i : ι) → Set (α i)\n⊢ ↑↑(Measure.pi μ) (Set.pi univ s) = ∏ i : ι, ↑↑(μ i) (s i)", "tactic": "haveI : Encodable ι := Fintype.toEncodable ι" }, { "state_after": "no goals", "state_before": "ι : Type u_2\nι' : Type ?u.3051144\nα : ι → Type u_1\ninst✝² : Fintype ι\nm : (i : ι) → OuterMeasure (α i)\ninst✝¹ : (i : ι) → MeasurableSpace (α i)\nμ : (i : ι) → Measure (α i)\ninst✝ : ∀ (i : ι), SigmaFinite (μ i)\ns : (i : ι) → Set (α i)\nthis : Encodable ι\n⊢ ↑↑(Measure.pi μ) (Set.pi univ s) = ∏ i : ι, ↑↑(μ i) (s i)", "tactic": "rw [← pi'_eq_pi, pi'_pi]" } ]
[ 400, 27 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 398, 1 ]
Mathlib/Topology/UniformSpace/Separation.lean
separated_def'
[ { "state_after": "α✝ : Type u\nβ : Type v\nγ : Type w\ninst✝³ : UniformSpace α✝\ninst✝² : UniformSpace β\ninst✝¹ : UniformSpace γ\nα : Type u\ninst✝ : UniformSpace α\nx y : α\n⊢ (¬x = y → ¬∀ (r : Set (α × α)), r ∈ 𝓤 α → (x, y) ∈ r) ↔ x ≠ y → ∃ r, r ∈ 𝓤 α ∧ ¬(x, y) ∈ r", "state_before": "α✝ : Type u\nβ : Type v\nγ : Type w\ninst✝³ : UniformSpace α✝\ninst✝² : UniformSpace β\ninst✝¹ : UniformSpace γ\nα : Type u\ninst✝ : UniformSpace α\nx y : α\n⊢ (∀ (r : Set (α × α)), r ∈ 𝓤 α → (x, y) ∈ r) → x = y ↔ x ≠ y → ∃ r, r ∈ 𝓤 α ∧ ¬(x, y) ∈ r", "tactic": "rw [← not_imp_not]" }, { "state_after": "no goals", "state_before": "α✝ : Type u\nβ : Type v\nγ : Type w\ninst✝³ : UniformSpace α✝\ninst✝² : UniformSpace β\ninst✝¹ : UniformSpace γ\nα : Type u\ninst✝ : UniformSpace α\nx y : α\n⊢ (¬x = y → ¬∀ (r : Set (α × α)), r ∈ 𝓤 α → (x, y) ∈ r) ↔ x ≠ y → ∃ r, r ∈ 𝓤 α ∧ ¬(x, y) ∈ r", "tactic": "simp [not_forall]" } ]
[ 144, 91 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 142, 1 ]
Mathlib/Topology/Constructions.lean
continuousAt_fst
[]
[ 341, 30 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 340, 1 ]
Mathlib/CategoryTheory/Preadditive/Injective.lean
CategoryTheory.Adjunction.map_injective
[ { "state_after": "C : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\n⊢ ∃ h, g ≫ h = f", "state_before": "C : Type u₁\ninst✝² : Category C\nD : Type u_2\ninst✝¹ : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\n⊢ ∀ [inst : Mono g], ∃ h, g ≫ h = f", "tactic": "intro" }, { "state_after": "case intro\nC : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\nw : F.obj Y ⟶ I\nh : F.map g ≫ w = F.map f ≫ adj.counit.app I\n⊢ ∃ h, g ≫ h = f", "state_before": "C : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\n⊢ ∃ h, g ≫ h = f", "tactic": "rcases hI.factors (F.map f ≫ adj.counit.app _) (F.map g) with ⟨w,h⟩" }, { "state_after": "case intro\nC : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\nw : F.obj Y ⟶ I\nh : F.map g ≫ w = F.map f ≫ adj.counit.app I\n⊢ g ≫ adj.unit.app Y ≫ G.map w = f", "state_before": "case intro\nC : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\nw : F.obj Y ⟶ I\nh : F.map g ≫ w = F.map f ≫ adj.counit.app I\n⊢ ∃ h, g ≫ h = f", "tactic": "use adj.unit.app Y ≫ G.map w" }, { "state_after": "case intro\nC : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\nw : F.obj Y ⟶ I\nh : F.map g ≫ w = F.map f ≫ adj.counit.app I\n⊢ adj.unit.app X ≫ G.map (F.map f ≫ adj.counit.app I) = f", "state_before": "case intro\nC : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\nw : F.obj Y ⟶ I\nh : F.map g ≫ w = F.map f ≫ adj.counit.app I\n⊢ g ≫ adj.unit.app Y ≫ G.map w = f", "tactic": "rw [← unit_naturality_assoc, ← G.map_comp, h]" }, { "state_after": "no goals", "state_before": "case intro\nC : Type u₁\ninst✝³ : Category C\nD : Type u_2\ninst✝² : Category D\nF : C ⥤ D\nG : D ⥤ C\nadj : F ⊣ G\ninst✝¹ : Functor.PreservesMonomorphisms F\nI : D\nhI : Injective I\nX Y : C\nf : X ⟶ G.obj I\ng : X ⟶ Y\ninst✝ : Mono g\nw : F.obj Y ⟶ I\nh : F.map g ≫ w = F.map f ≫ adj.counit.app I\n⊢ adj.unit.app X ≫ G.map (F.map f ≫ adj.counit.app I) = f", "tactic": "simp" } ]
[ 324, 10 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 317, 1 ]
Mathlib/RingTheory/HahnSeries.lean
HahnSeries.support_nonempty_iff
[ { "state_after": "no goals", "state_before": "Γ : Type u_1\nR : Type u_2\ninst✝¹ : PartialOrder Γ\ninst✝ : Zero R\nx : HahnSeries Γ R\n⊢ Set.Nonempty (support x) ↔ x ≠ 0", "tactic": "rw [support, support_nonempty_iff, Ne.def, coeff_fun_eq_zero_iff]" } ]
[ 141, 68 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 140, 8 ]
Mathlib/Topology/ContinuousOn.lean
continuousOn_open_iff
[ { "state_after": "α : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ (∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) ↔ ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)", "state_before": "α : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ ContinuousOn f s ↔ ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)", "tactic": "rw [continuousOn_iff']" }, { "state_after": "case mp\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ (∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) → ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)\n\ncase mpr\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ (∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)) → ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s", "state_before": "α : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ (∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) ↔ ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)", "tactic": "constructor" }, { "state_after": "case mp\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s\nt : Set β\nht : IsOpen t\n⊢ IsOpen (s ∩ f ⁻¹' t)", "state_before": "case mp\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ (∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s) → ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)", "tactic": "intro h t ht" }, { "state_after": "case mp.intro.intro\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s\nt : Set β\nht : IsOpen t\nu : Set α\nu_open : IsOpen u\nhu : f ⁻¹' t ∩ s = u ∩ s\n⊢ IsOpen (s ∩ f ⁻¹' t)", "state_before": "case mp\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s\nt : Set β\nht : IsOpen t\n⊢ IsOpen (s ∩ f ⁻¹' t)", "tactic": "rcases h t ht with ⟨u, u_open, hu⟩" }, { "state_after": "case mp.intro.intro\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s\nt : Set β\nht : IsOpen t\nu : Set α\nu_open : IsOpen u\nhu : f ⁻¹' t ∩ s = u ∩ s\n⊢ IsOpen (u ∩ s)", "state_before": "case mp.intro.intro\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s\nt : Set β\nht : IsOpen t\nu : Set α\nu_open : IsOpen u\nhu : f ⁻¹' t ∩ s = u ∩ s\n⊢ IsOpen (s ∩ f ⁻¹' t)", "tactic": "rw [inter_comm, hu]" }, { "state_after": "no goals", "state_before": "case mp.intro.intro\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s\nt : Set β\nht : IsOpen t\nu : Set α\nu_open : IsOpen u\nhu : f ⁻¹' t ∩ s = u ∩ s\n⊢ IsOpen (u ∩ s)", "tactic": "apply IsOpen.inter u_open hs" }, { "state_after": "case mpr\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)\nt : Set β\nht : IsOpen t\n⊢ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s", "state_before": "case mpr\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\n⊢ (∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)) → ∀ (t : Set β), IsOpen t → ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s", "tactic": "intro h t ht" }, { "state_after": "case mpr\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)\nt : Set β\nht : IsOpen t\n⊢ f ⁻¹' t ∩ s = s ∩ f ⁻¹' t ∩ s", "state_before": "case mpr\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)\nt : Set β\nht : IsOpen t\n⊢ ∃ u, IsOpen u ∧ f ⁻¹' t ∩ s = u ∩ s", "tactic": "refine' ⟨s ∩ f ⁻¹' t, h t ht, _⟩" }, { "state_after": "no goals", "state_before": "case mpr\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.342559\nδ : Type ?u.342562\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\nf : α → β\ns : Set α\nhs : IsOpen s\nh : ∀ (t : Set β), IsOpen t → IsOpen (s ∩ f ⁻¹' t)\nt : Set β\nht : IsOpen t\n⊢ f ⁻¹' t ∩ s = s ∩ f ⁻¹' t ∩ s", "tactic": "rw [@inter_comm _ s (f ⁻¹' t), inter_assoc, inter_self]" } ]
[ 1004, 60 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 994, 1 ]
Mathlib/Topology/Instances/Real.lean
Real.continuous_inv
[]
[ 116, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 115, 1 ]
Mathlib/Topology/ContinuousFunction/Basic.lean
ContinuousMap.restrict_apply
[]
[ 372, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 371, 1 ]
Mathlib/Data/Nat/PartENat.lean
PartENat.dom_natCast
[]
[ 121, 10 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 120, 1 ]
Mathlib/Analysis/Calculus/Deriv/Mul.lean
derivWithin_mul_const
[]
[ 226, 52 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 224, 1 ]
Mathlib/GroupTheory/Subgroup/Basic.lean
Subgroup.inf_subgroupOf_inf_normal_of_left
[]
[ 3584, 58 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 3579, 1 ]
Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean
ContDiffAt.cexp
[]
[ 164, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 162, 1 ]
Mathlib/Analysis/InnerProductSpace/Calculus.lean
DifferentiableWithinAt.norm_sq
[]
[ 262, 87 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 260, 1 ]
Mathlib/Data/List/Perm.lean
List.Subperm.countp_le
[]
[ 479, 50 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 477, 1 ]
Mathlib/Data/Fintype/Sum.lean
Finset.exists_equiv_extend_of_card_eq
[ { "state_after": "case empty\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\n⊢ ∃ g, ∀ (i : α), i ∈ ∅ → ↑(↑g i) = f i\n\ncase insert\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf : α → β\nhfst : image f s ⊆ t\nhfs : Set.InjOn f ↑s\n⊢ ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i", "tactic": "induction' s using Finset.induction with a s has H generalizing f" }, { "state_after": "case insert\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "state_before": "case insert\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "tactic": "have hfst' : Finset.image f s ⊆ t := (Finset.image_mono _ (s.subset_insert a)).trans hfst" }, { "state_after": "case insert\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "state_before": "case insert\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "tactic": "have hfs' : Set.InjOn f s := hfs.mono (s.subset_insert a)" }, { "state_after": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "state_before": "case insert\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "tactic": "obtain ⟨g', hg'⟩ := H hfst' hfs'" }, { "state_after": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "state_before": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "tactic": "have hfat : f a ∈ t := hfst (mem_image_of_mem _ (s.mem_insert_self a))" }, { "state_after": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\n⊢ ∀ (i : α), i ∈ insert a s → ↑(↑(g'.trans (Equiv.swap { val := f a, property := hfat } (↑g' a))) i) = f i", "state_before": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\n⊢ ∃ g, ∀ (i : α), i ∈ insert a s → ↑(↑g i) = f i", "tactic": "use g'.trans (Equiv.swap (⟨f a, hfat⟩ : t) (g' a))" }, { "state_after": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\n⊢ ∀ (i : α), i = a ∨ i ∈ s → ↑(↑(g'.trans (Equiv.swap { val := f a, property := hfat } (↑g' a))) i) = f i", "state_before": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\n⊢ ∀ (i : α), i ∈ insert a s → ↑(↑(g'.trans (Equiv.swap { val := f a, property := hfat } (↑g' a))) i) = f i", "tactic": "simp_rw [mem_insert]" }, { "state_after": "case insert.intro.inl\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\ns : Finset α\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\ni : α\nhas : ¬i ∈ s\nhfst : image f (insert i s) ⊆ t\nhfs : Set.InjOn f ↑(insert i s)\nhfat : f i ∈ t\n⊢ ↑(↑(g'.trans (Equiv.swap { val := f i, property := hfat } (↑g' i))) i) = f i\n\ncase insert.intro.inr\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\ni : α\nhi : i ∈ s\n⊢ ↑(↑(g'.trans (Equiv.swap { val := f a, property := hfat } (↑g' a))) i) = f i", "state_before": "case insert.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\n⊢ ∀ (i : α), i = a ∨ i ∈ s → ↑(↑(g'.trans (Equiv.swap { val := f a, property := hfat } (↑g' a))) i) = f i", "tactic": "rintro i (rfl | hi)" }, { "state_after": "case insert.intro.inr.a\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\ni : α\nhi : i ∈ s\n⊢ ↑g' i ≠ { val := f a, property := hfat }\n\ncase insert.intro.inr.a\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\ni : α\nhi : i ∈ s\n⊢ ↑g' i ≠ ↑g' a", "state_before": "case insert.intro.inr\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\ni : α\nhi : i ∈ s\n⊢ ↑(↑(g'.trans (Equiv.swap { val := f a, property := hfat } (↑g' a))) i) = f i", "tactic": "rw [Equiv.trans_apply, Equiv.swap_apply_of_ne_of_ne, hg' _ hi]" }, { "state_after": "case empty.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\ne : α ≃ { x // x ∈ t }\n⊢ ∃ g, ∀ (i : α), i ∈ ∅ → ↑(↑g i) = f i", "state_before": "case empty\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\n⊢ ∃ g, ∀ (i : α), i ∈ ∅ → ↑(↑g i) = f i", "tactic": "obtain ⟨e⟩ : Nonempty (α ≃ ↥t) := by rwa [← Fintype.card_eq, Fintype.card_coe]" }, { "state_after": "case empty.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\ne : α ≃ { x // x ∈ t }\n⊢ ∀ (i : α), i ∈ ∅ → ↑(↑e i) = f i", "state_before": "case empty.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\ne : α ≃ { x // x ∈ t }\n⊢ ∃ g, ∀ (i : α), i ∈ ∅ → ↑(↑g i) = f i", "tactic": "use e" }, { "state_after": "no goals", "state_before": "case empty.intro\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\ne : α ≃ { x // x ∈ t }\n⊢ ∀ (i : α), i ∈ ∅ → ↑(↑e i) = f i", "tactic": "simp" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s\nf : α → β\nhfst : image f ∅ ⊆ t\nhfs : Set.InjOn f ↑∅\n⊢ Nonempty (α ≃ { x // x ∈ t })", "tactic": "rwa [← Fintype.card_eq, Fintype.card_coe]" }, { "state_after": "no goals", "state_before": "case insert.intro.inl\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\ns : Finset α\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\ni : α\nhas : ¬i ∈ s\nhfst : image f (insert i s) ⊆ t\nhfs : Set.InjOn f ↑(insert i s)\nhfat : f i ∈ t\n⊢ ↑(↑(g'.trans (Equiv.swap { val := f i, property := hfat } (↑g' i))) i) = f i", "tactic": "simp" }, { "state_after": "no goals", "state_before": "case insert.intro.inr.a\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\ni : α\nhi : i ∈ s\n⊢ ↑g' i ≠ { val := f a, property := hfat }", "tactic": "exact\n ne_of_apply_ne Subtype.val\n (ne_of_eq_of_ne (hg' _ hi) <|\n hfs.ne (subset_insert _ _ hi) (mem_insert_self _ _) <| ne_of_mem_of_not_mem hi has)" }, { "state_after": "no goals", "state_before": "case insert.intro.inr.a\nα : Type u_1\nβ : Type u_2\ninst✝¹ : Fintype α\ninst✝ : DecidableEq β\nt : Finset β\nhαt : Fintype.card α = card t\ns✝ : Finset α\nf✝ : α → β\nhfst✝ : image f✝ s✝ ⊆ t\nhfs✝ : Set.InjOn f✝ ↑s✝\na : α\ns : Finset α\nhas : ¬a ∈ s\nH : ∀ {f : α → β}, image f s ⊆ t → Set.InjOn f ↑s → ∃ g, ∀ (i : α), i ∈ s → ↑(↑g i) = f i\nf : α → β\nhfst : image f (insert a s) ⊆ t\nhfs : Set.InjOn f ↑(insert a s)\nhfst' : image f s ⊆ t\nhfs' : Set.InjOn f ↑s\ng' : α ≃ { x // x ∈ t }\nhg' : ∀ (i : α), i ∈ s → ↑(↑g' i) = f i\nhfat : f a ∈ t\ni : α\nhi : i ∈ s\n⊢ ↑g' i ≠ ↑g' a", "tactic": "exact g'.injective.ne (ne_of_mem_of_not_mem hi has)" } ]
[ 103, 58 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 82, 1 ]
Mathlib/Data/List/Sort.lean
List.Sorted.merge
[ { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\nx✝¹ x✝ : Sorted r []\n⊢ Sorted r (List.merge r [] [])", "tactic": "simp [List.merge]" }, { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\nb : α\nl' : List α\nx✝ : Sorted r []\nh₂ : Sorted r (b :: l')\n⊢ Sorted r (List.merge r [] (b :: l'))", "tactic": "simpa [List.merge] using h₂" }, { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nh₁ : Sorted r (a :: l)\nx✝ : Sorted r []\n⊢ Sorted r (List.merge r (a :: l) [])", "tactic": "simpa [List.merge] using h₁" }, { "state_after": "case pos\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))\n\ncase neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))", "tactic": "by_cases h : a ≼ b" }, { "state_after": "case pos\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\n⊢ ∀ (b' : α), b' ∈ List.merge r l (b :: l') → r a b'", "state_before": "case pos\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))", "tactic": "suffices ∀ (b' : α) (_ : b' ∈ List.merge r l (b :: l')), r a b' by\n simpa [List.merge, h, h₁.of_cons.merge h₂]" }, { "state_after": "case pos\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\n⊢ r a b'", "state_before": "case pos\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\n⊢ ∀ (b' : α), b' ∈ List.merge r l (b :: l') → r a b'", "tactic": "intro b' bm" }, { "state_after": "case pos.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\nbe : b' = b\n⊢ r a b'\n\ncase pos.inr.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\nbl : b' ∈ l\n⊢ r a b'\n\ncase pos.inr.inr\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\nbl' : b' ∈ l'\n⊢ r a b'", "state_before": "case pos\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\n⊢ r a b'", "tactic": "rcases show b' = b ∨ b' ∈ l ∨ b' ∈ l' by\n simpa [or_left_comm] using (perm_merge _ _ _).subset bm with\n (be | bl | bl')" }, { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nthis : ∀ (b' : α), b' ∈ List.merge r l (b :: l') → r a b'\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))", "tactic": "simpa [List.merge, h, h₁.of_cons.merge h₂]" }, { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\n⊢ b' = b ∨ b' ∈ l ∨ b' ∈ l'", "tactic": "simpa [or_left_comm] using (perm_merge _ _ _).subset bm" }, { "state_after": "case pos.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nbm : b ∈ List.merge r l (b :: l')\n⊢ r a b", "state_before": "case pos.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\nbe : b' = b\n⊢ r a b'", "tactic": "subst b'" }, { "state_after": "no goals", "state_before": "case pos.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nbm : b ∈ List.merge r l (b :: l')\n⊢ r a b", "tactic": "assumption" }, { "state_after": "no goals", "state_before": "case pos.inr.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\nbl : b' ∈ l\n⊢ r a b'", "tactic": "exact rel_of_sorted_cons h₁ _ bl" }, { "state_after": "no goals", "state_before": "case pos.inr.inr\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : r a b\nb' : α\nbm : b' ∈ List.merge r l (b :: l')\nbl' : b' ∈ l'\n⊢ r a b'", "tactic": "exact _root_.trans h (rel_of_sorted_cons h₂ _ bl')" }, { "state_after": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\n⊢ ∀ (b' : α), b' ∈ List.merge r (a :: l) l' → r b b'", "state_before": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))", "tactic": "suffices ∀ (b' : α) (_ : b' ∈ List.merge r (a :: l) l'), r b b' by\n simpa [List.merge, h, h₁.merge h₂.of_cons]" }, { "state_after": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\n⊢ r b b'", "state_before": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\n⊢ ∀ (b' : α), b' ∈ List.merge r (a :: l) l' → r b b'", "tactic": "intro b' bm" }, { "state_after": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\n⊢ r b b'", "state_before": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\n⊢ r b b'", "tactic": "have ba : b ≼ a := (total_of r _ _).resolve_left h" }, { "state_after": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nthis : b' = a ∨ b' ∈ l ∨ b' ∈ l'\n⊢ r b b'", "state_before": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\n⊢ r b b'", "tactic": "have : b' = a ∨ b' ∈ l ∨ b' ∈ l' := by simpa using (perm_merge _ _ _).subset bm" }, { "state_after": "case neg.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nbe : b' = a\n⊢ r b b'\n\ncase neg.inr.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nbl : b' ∈ l\n⊢ r b b'\n\ncase neg.inr.inr\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nbl' : b' ∈ l'\n⊢ r b b'", "state_before": "case neg\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nthis : b' = a ∨ b' ∈ l ∨ b' ∈ l'\n⊢ r b b'", "tactic": "rcases this with (be | bl | bl')" }, { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nthis : ∀ (b' : α), b' ∈ List.merge r (a :: l) l' → r b b'\n⊢ Sorted r (List.merge r (a :: l) (b :: l'))", "tactic": "simpa [List.merge, h, h₁.merge h₂.of_cons]" }, { "state_after": "no goals", "state_before": "α : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\n⊢ b' = a ∨ b' ∈ l ∨ b' ∈ l'", "tactic": "simpa using (perm_merge _ _ _).subset bm" }, { "state_after": "case neg.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nba : r b a\nbm : a ∈ List.merge r (a :: l) l'\n⊢ r b a", "state_before": "case neg.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nbe : b' = a\n⊢ r b b'", "tactic": "subst b'" }, { "state_after": "no goals", "state_before": "case neg.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nba : r b a\nbm : a ∈ List.merge r (a :: l) l'\n⊢ r b a", "tactic": "assumption" }, { "state_after": "no goals", "state_before": "case neg.inr.inl\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nbl : b' ∈ l\n⊢ r b b'", "tactic": "exact _root_.trans ba (rel_of_sorted_cons h₁ _ bl)" }, { "state_after": "no goals", "state_before": "case neg.inr.inr\nα : Type uu\nr : α → α → Prop\ninst✝² : DecidableRel r\ninst✝¹ : IsTotal α r\ninst✝ : IsTrans α r\na : α\nl : List α\nb : α\nl' : List α\nh₁ : Sorted r (a :: l)\nh₂ : Sorted r (b :: l')\nh : ¬r a b\nb' : α\nbm : b' ∈ List.merge r (a :: l) l'\nba : r b a\nbl' : b' ∈ l'\n⊢ r b b'", "tactic": "exact rel_of_sorted_cons h₂ _ bl'" } ]
[ 437, 65 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 411, 1 ]
Mathlib/GroupTheory/SpecificGroups/Cyclic.lean
IsCyclic.card_orderOf_eq_totient
[ { "state_after": "no goals", "state_before": "α : Type u\na : α\ninst✝² : Group α\ninst✝¹ : IsCyclic α\ninst✝ : Fintype α\nd : ℕ\nhd : d ∣ Fintype.card α\n⊢ card (filter (fun a => orderOf a = d) univ) = φ d", "tactic": "classical apply card_orderOf_eq_totient_aux₂ (fun n => IsCyclic.card_pow_eq_one_le) hd" }, { "state_after": "no goals", "state_before": "α : Type u\na : α\ninst✝² : Group α\ninst✝¹ : IsCyclic α\ninst✝ : Fintype α\nd : ℕ\nhd : d ∣ Fintype.card α\n⊢ card (filter (fun a => orderOf a = d) univ) = φ d", "tactic": "apply card_orderOf_eq_totient_aux₂ (fun n => IsCyclic.card_pow_eq_one_le) hd" } ]
[ 419, 89 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 417, 1 ]
Mathlib/Data/Dfinsupp/Interval.lean
Dfinsupp.support_rangeIcc_subset
[ { "state_after": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\n⊢ x ∈ support f ∪ support g", "state_before": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\n⊢ support (rangeIcc f g) ⊆ support f ∪ support g", "tactic": "refine' fun x hx => _" }, { "state_after": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\nh : ¬x ∈ support f ∪ support g\n⊢ False", "state_before": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\n⊢ x ∈ support f ∪ support g", "tactic": "by_contra h" }, { "state_after": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\nh : ¬x ∈ support f ∪ support g\n⊢ ↑(rangeIcc f g) x = 0", "state_before": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\nh : ¬x ∈ support f ∪ support g\n⊢ False", "tactic": "refine' not_mem_support_iff.2 _ hx" }, { "state_after": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\nh : ¬x ∈ support f ∪ support g\n⊢ Icc 0 0 = 0", "state_before": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\nh : ¬x ∈ support f ∪ support g\n⊢ ↑(rangeIcc f g) x = 0", "tactic": "rw [rangeIcc_apply, not_mem_support_iff.1 (not_mem_mono (subset_union_left _ _) h),\n not_mem_support_iff.1 (not_mem_mono (subset_union_right _ _) h)]" }, { "state_after": "no goals", "state_before": "ι : Type u_1\nα : ι → Type u_2\ninst✝⁴ : (i : ι) → Zero (α i)\ninst✝³ : (i : ι) → PartialOrder (α i)\ninst✝² : (i : ι) → LocallyFiniteOrder (α i)\nf g : Π₀ (i : ι), α i\ni : ι\na : α i\ninst✝¹ : DecidableEq ι\ninst✝ : (i : ι) → DecidableEq (α i)\nx : ι\nhx : x ∈ support (rangeIcc f g)\nh : ¬x ∈ support f ∪ support g\n⊢ Icc 0 0 = 0", "tactic": "exact Icc_self _" } ]
[ 135, 19 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 128, 1 ]
Mathlib/FieldTheory/IsAlgClosed/Basic.lean
IsAlgClosure.equivOfEquiv_symm_comp_algebraMap
[]
[ 530, 59 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 527, 1 ]
Mathlib/Algebra/Order/Ring/Lemmas.lean
neg_of_mul_pos_left
[]
[ 576, 84 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 575, 1 ]
Mathlib/RingTheory/Polynomial/Basic.lean
Ideal.isPrime_map_C_of_isPrime
[]
[ 728, 38 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 726, 1 ]
Mathlib/Analysis/NormedSpace/MazurUlam.lean
IsometryEquiv.coeFn_toRealAffineIsometryEquiv
[]
[ 159, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 158, 1 ]
Mathlib/Analysis/Calculus/ContDiffDef.lean
contDiffOn_succ_iff_hasFDerivWithinAt
[ { "state_after": "case mp\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\n⊢ ContDiffOn 𝕜 (↑(n + 1)) f s →\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\n\ncase mpr\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\n⊢ (∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u) →\n ContDiffOn 𝕜 (↑(n + 1)) f s", "state_before": "𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\n⊢ ContDiffOn 𝕜 (↑(n + 1)) f s ↔\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u", "tactic": "constructor" }, { "state_after": "case mp\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u", "state_before": "case mp\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\n⊢ ContDiffOn 𝕜 (↑(n + 1)) f s →\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u", "tactic": "intro h x hx" }, { "state_after": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp : HasFTaylorSeriesUpToOn (↑(Nat.succ n)) f p u\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u", "state_before": "case mp\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u", "tactic": "rcases(h x hx) n.succ le_rfl with ⟨u, hu, p, Hp⟩" }, { "state_after": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp : HasFTaylorSeriesUpToOn (↑(Nat.succ n)) f p u\n⊢ ContDiffOn 𝕜 (↑n) (fun y => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p y 1)) u", "state_before": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp : HasFTaylorSeriesUpToOn (↑(Nat.succ n)) f p u\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u", "tactic": "refine'\n ⟨u, hu, fun y => (continuousMultilinearCurryFin1 𝕜 E F) (p y 1), fun y hy =>\n Hp.hasFDerivWithinAt (WithTop.coe_le_coe.2 (Nat.le_add_left 1 n)) hy, _⟩" }, { "state_after": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\n⊢ ContDiffOn 𝕜 (↑n) (fun y => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p y 1)) u", "state_before": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp : HasFTaylorSeriesUpToOn (↑(Nat.succ n)) f p u\n⊢ ContDiffOn 𝕜 (↑n) (fun y => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p y 1)) u", "tactic": "rw [hasFTaylorSeriesUpToOn_succ_iff_right] at Hp" }, { "state_after": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm✝ n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\nz : E\nhz : z ∈ u\nm : ℕ\nhm : ↑m ≤ ↑n\n⊢ ∃ u_1,\n u_1 ∈ 𝓝[insert z u] z ∧\n ∃ p_1, HasFTaylorSeriesUpToOn (↑m) (fun y => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p y 1)) p_1 u_1", "state_before": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\n⊢ ContDiffOn 𝕜 (↑n) (fun y => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p y 1)) u", "tactic": "intro z hz m hm" }, { "state_after": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm✝ n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\nz : E\nhz : z ∈ u\nm : ℕ\nhm : ↑m ≤ ↑n\n⊢ u ∈ 𝓝[insert z u] z", "state_before": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm✝ n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\nz : E\nhz : z ∈ u\nm : ℕ\nhm : ↑m ≤ ↑n\n⊢ ∃ u_1,\n u_1 ∈ 𝓝[insert z u] z ∧\n ∃ p_1, HasFTaylorSeriesUpToOn (↑m) (fun y => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p y 1)) p_1 u_1", "tactic": "refine' ⟨u, _, fun x : E => (p x).shift, Hp.2.2.of_le hm⟩" }, { "state_after": "case h.e'_5.h.e'_4\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm✝ n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\nz : E\nhz : z ∈ u\nm : ℕ\nhm : ↑m ≤ ↑n\n⊢ insert z u = u", "state_before": "case mp.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm✝ n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\nz : E\nhz : z ∈ u\nm : ℕ\nhm : ↑m ≤ ↑n\n⊢ u ∈ 𝓝[insert z u] z", "tactic": "convert @self_mem_nhdsWithin _ _ z u" }, { "state_after": "no goals", "state_before": "case h.e'_5.h.e'_4\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm✝ n✝ : ℕ∞\np✝ : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh : ContDiffOn 𝕜 (↑(n + 1)) f s\nx : E\nhx : x ∈ s\nu : Set E\nhu : u ∈ 𝓝[insert x s] x\np : E → FormalMultilinearSeries 𝕜 E F\nHp :\n (∀ (x : E), x ∈ u → ContinuousMultilinearMap.uncurry0 (p x 0) = f x) ∧\n (∀ (x : E), x ∈ u → HasFDerivWithinAt (fun y => p y 0) (ContinuousMultilinearMap.curryLeft (p x 1)) u x) ∧\n HasFTaylorSeriesUpToOn (↑n) (fun x => ↑(continuousMultilinearCurryFin1 𝕜 E F) (p x 1))\n (fun x => FormalMultilinearSeries.shift (p x)) u\nz : E\nhz : z ∈ u\nm : ℕ\nhm : ↑m ≤ ↑n\n⊢ insert z u = u", "tactic": "exact insert_eq_of_mem hz" }, { "state_after": "case mpr\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\n⊢ ContDiffWithinAt 𝕜 (↑(n + 1)) f s x", "state_before": "case mpr\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\n⊢ (∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u) →\n ContDiffOn 𝕜 (↑(n + 1)) f s", "tactic": "intro h x hx" }, { "state_after": "case mpr\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffWithinAt 𝕜 (↑n) f' u x", "state_before": "case mpr\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\n⊢ ContDiffWithinAt 𝕜 (↑(n + 1)) f s x", "tactic": "rw [contDiffWithinAt_succ_iff_hasFDerivWithinAt]" }, { "state_after": "case mpr.intro.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\nu : Set E\nu_nhbd : u ∈ 𝓝[insert x s] x\nf' : E → E →L[𝕜] F\nhu : ∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x\nhf' : ContDiffOn 𝕜 (↑n) f' u\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffWithinAt 𝕜 (↑n) f' u x", "state_before": "case mpr\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffWithinAt 𝕜 (↑n) f' u x", "tactic": "rcases h x hx with ⟨u, u_nhbd, f', hu, hf'⟩" }, { "state_after": "case mpr.intro.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\nu : Set E\nu_nhbd : u ∈ 𝓝[insert x s] x\nf' : E → E →L[𝕜] F\nhu : ∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x\nhf' : ContDiffOn 𝕜 (↑n) f' u\nthis : x ∈ u\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffWithinAt 𝕜 (↑n) f' u x", "state_before": "case mpr.intro.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\nu : Set E\nu_nhbd : u ∈ 𝓝[insert x s] x\nf' : E → E →L[𝕜] F\nhu : ∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x\nhf' : ContDiffOn 𝕜 (↑n) f' u\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffWithinAt 𝕜 (↑n) f' u x", "tactic": "have : x ∈ u := mem_of_mem_nhdsWithin (mem_insert _ _) u_nhbd" }, { "state_after": "no goals", "state_before": "case mpr.intro.intro.intro.intro\n𝕜 : Type u\ninst✝⁸ : NontriviallyNormedField 𝕜\nE : Type uE\ninst✝⁷ : NormedAddCommGroup E\ninst✝⁶ : NormedSpace 𝕜 E\nF : Type uF\ninst✝⁵ : NormedAddCommGroup F\ninst✝⁴ : NormedSpace 𝕜 F\nG : Type uG\ninst✝³ : NormedAddCommGroup G\ninst✝² : NormedSpace 𝕜 G\nX : Type uX\ninst✝¹ : NormedAddCommGroup X\ninst✝ : NormedSpace 𝕜 X\ns s₁ t u✝ : Set E\nf f₁ : E → F\ng : F → G\nx✝ x₀ : E\nc : F\nm n✝ : ℕ∞\np : E → FormalMultilinearSeries 𝕜 E F\nn : ℕ\nh :\n ∀ (x : E),\n x ∈ s →\n ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffOn 𝕜 (↑n) f' u\nx : E\nhx : x ∈ s\nu : Set E\nu_nhbd : u ∈ 𝓝[insert x s] x\nf' : E → E →L[𝕜] F\nhu : ∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x\nhf' : ContDiffOn 𝕜 (↑n) f' u\nthis : x ∈ u\n⊢ ∃ u, u ∈ 𝓝[insert x s] x ∧ ∃ f', (∀ (x : E), x ∈ u → HasFDerivWithinAt f (f' x) u x) ∧ ContDiffWithinAt 𝕜 (↑n) f' u x", "tactic": "exact ⟨u, u_nhbd, f', hu, hf' x this⟩" } ]
[ 755, 42 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 735, 1 ]
Mathlib/SetTheory/Cardinal/Basic.lean
Cardinal.power_ne_zero
[]
[ 585, 34 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 582, 1 ]
Mathlib/Data/Finset/Interval.lean
Finset.card_Ico_finset
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : DecidableEq α\ns t : Finset α\nh : s ⊆ t\n⊢ card (Ico s t) = 2 ^ (card t - card s) - 1", "tactic": "rw [card_Ico_eq_card_Icc_sub_one, card_Icc_finset h]" } ]
[ 109, 55 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 108, 1 ]
Mathlib/Data/List/Chain.lean
List.Chain'.take
[]
[ 331, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 330, 1 ]
Mathlib/Data/Bool/Basic.lean
Bool.or_inr
[ { "state_after": "no goals", "state_before": "a b : Bool\nH : b = true\n⊢ (a || b) = true", "tactic": "cases a <;> simp [H]" } ]
[ 162, 72 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 162, 1 ]
Mathlib/Algebra/AddTorsor.lean
vsub_self
[ { "state_after": "no goals", "state_before": "G : Type u_1\nP : Type u_2\ninst✝ : AddGroup G\nT : AddTorsor G P\np : P\n⊢ p -ᵥ p = 0", "tactic": "rw [← zero_add (p -ᵥ p), ← vadd_vsub_assoc, vadd_vsub]" } ]
[ 128, 57 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 127, 1 ]
Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean
Asymptotics.IsLittleO.add_isEquivalent
[]
[ 177, 37 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 176, 1 ]
Mathlib/Data/Real/EReal.lean
EReal.coe_lt_coe_iff
[]
[ 108, 27 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 107, 11 ]
Mathlib/Data/Finite/Card.lean
Finite.card_le_of_injective
[ { "state_after": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.2279\ninst✝ : Finite β\nf : α → β\nhf : Function.Injective f\nthis : Fintype β\n⊢ Nat.card α ≤ Nat.card β", "state_before": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.2279\ninst✝ : Finite β\nf : α → β\nhf : Function.Injective f\n⊢ Nat.card α ≤ Nat.card β", "tactic": "haveI := Fintype.ofFinite β" }, { "state_after": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.2279\ninst✝ : Finite β\nf : α → β\nhf : Function.Injective f\nthis✝ : Fintype β\nthis : Fintype α\n⊢ Nat.card α ≤ Nat.card β", "state_before": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.2279\ninst✝ : Finite β\nf : α → β\nhf : Function.Injective f\nthis : Fintype β\n⊢ Nat.card α ≤ Nat.card β", "tactic": "haveI := Fintype.ofInjective f hf" }, { "state_after": "no goals", "state_before": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.2279\ninst✝ : Finite β\nf : α → β\nhf : Function.Injective f\nthis✝ : Fintype β\nthis : Fintype α\n⊢ Nat.card α ≤ Nat.card β", "tactic": "simpa only [Nat.card_eq_fintype_card, ge_iff_le] using Fintype.card_le_of_injective f hf" } ]
[ 105, 91 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 101, 1 ]
Mathlib/Data/Set/Pointwise/Finite.lean
Set.infinite_smul_set
[]
[ 155, 56 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 154, 1 ]
Mathlib/MeasureTheory/Measure/MeasureSpace.lean
MeasureTheory.Measure.count_injective_image'
[ { "state_after": "case pos\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : Set.Finite s\n⊢ ↑↑count (f '' s) = ↑↑count s\n\ncase neg\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : ¬Set.Finite s\n⊢ ↑↑count (f '' s) = ↑↑count s", "state_before": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\n⊢ ↑↑count (f '' s) = ↑↑count s", "tactic": "by_cases hs : s.Finite" }, { "state_after": "case pos.intro\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Finset β\ns_mble : MeasurableSet ↑s\nfs_mble : MeasurableSet (f '' ↑s)\n⊢ ↑↑count (f '' ↑s) = ↑↑count ↑s", "state_before": "case pos\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : Set.Finite s\n⊢ ↑↑count (f '' s) = ↑↑count s", "tactic": "lift s to Finset β using hs" }, { "state_after": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Finset β\ns_mble : MeasurableSet ↑s\nfs_mble : MeasurableSet (f '' ↑s)\n⊢ MeasurableSet ↑(Finset.image f s)", "state_before": "case pos.intro\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Finset β\ns_mble : MeasurableSet ↑s\nfs_mble : MeasurableSet (f '' ↑s)\n⊢ ↑↑count (f '' ↑s) = ↑↑count ↑s", "tactic": "rw [← Finset.coe_image, count_apply_finset' _, count_apply_finset' s_mble,\n s.card_image_of_injective hf]" }, { "state_after": "no goals", "state_before": "α : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Finset β\ns_mble : MeasurableSet ↑s\nfs_mble : MeasurableSet (f '' ↑s)\n⊢ MeasurableSet ↑(Finset.image f s)", "tactic": "simpa only [Finset.coe_image] using fs_mble" }, { "state_after": "case neg\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : ¬Set.Finite s\n⊢ ↑↑count (f '' s) = ⊤", "state_before": "case neg\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : ¬Set.Finite s\n⊢ ↑↑count (f '' s) = ↑↑count s", "tactic": "rw [count_apply_infinite hs]" }, { "state_after": "case neg\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : ¬Set.Finite (f '' s)\n⊢ ↑↑count (f '' s) = ⊤", "state_before": "case neg\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : ¬Set.Finite s\n⊢ ↑↑count (f '' s) = ⊤", "tactic": "rw [← finite_image_iff <| hf.injOn _] at hs" }, { "state_after": "no goals", "state_before": "case neg\nα : Type u_2\nβ : Type u_1\nγ : Type ?u.386958\nδ : Type ?u.386961\nι : Type ?u.386964\nR : Type ?u.386967\nR' : Type ?u.386970\nm0 : MeasurableSpace α\ninst✝² : MeasurableSpace β\ninst✝¹ : MeasurableSpace γ\nμ μ₁ μ₂ μ₃ ν ν' ν₁ ν₂ : Measure α\ns✝ s' t : Set α\ninst✝ : MeasurableSpace α\nf : β → α\nhf : Injective f\ns : Set β\ns_mble : MeasurableSet s\nfs_mble : MeasurableSet (f '' s)\nhs : ¬Set.Finite (f '' s)\n⊢ ↑↑count (f '' s) = ⊤", "tactic": "rw [count_apply_infinite hs]" } ]
[ 2330, 33 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2321, 1 ]
Mathlib/LinearAlgebra/AffineSpace/Combination.lean
Finset.weightedVSubOfPoint_eq_of_sum_eq_zero
[ { "state_after": "case h\nk : Type u_1\nV : Type u_3\nP : Type u_4\ninst✝² : Ring k\ninst✝¹ : AddCommGroup V\ninst✝ : Module k V\nS : AffineSpace V P\nι : Type u_2\ns : Finset ι\nι₂ : Type ?u.31556\ns₂ : Finset ι₂\nw : ι → k\np : ι → P\nh : ∑ i in s, w i = 0\nb₁ b₂ : P\n⊢ ↑(weightedVSubOfPoint s p b₁) w - ↑(weightedVSubOfPoint s p b₂) w = 0", "state_before": "k : Type u_1\nV : Type u_3\nP : Type u_4\ninst✝² : Ring k\ninst✝¹ : AddCommGroup V\ninst✝ : Module k V\nS : AffineSpace V P\nι : Type u_2\ns : Finset ι\nι₂ : Type ?u.31556\ns₂ : Finset ι₂\nw : ι → k\np : ι → P\nh : ∑ i in s, w i = 0\nb₁ b₂ : P\n⊢ ↑(weightedVSubOfPoint s p b₁) w = ↑(weightedVSubOfPoint s p b₂) w", "tactic": "apply eq_of_sub_eq_zero" }, { "state_after": "case h\nk : Type u_1\nV : Type u_3\nP : Type u_4\ninst✝² : Ring k\ninst✝¹ : AddCommGroup V\ninst✝ : Module k V\nS : AffineSpace V P\nι : Type u_2\ns : Finset ι\nι₂ : Type ?u.31556\ns₂ : Finset ι₂\nw : ι → k\np : ι → P\nh : ∑ i in s, w i = 0\nb₁ b₂ : P\n⊢ ∑ x in s, (w x • (p x -ᵥ b₁) - w x • (p x -ᵥ b₂)) = 0", "state_before": "case h\nk : Type u_1\nV : Type u_3\nP : Type u_4\ninst✝² : Ring k\ninst✝¹ : AddCommGroup V\ninst✝ : Module k V\nS : AffineSpace V P\nι : Type u_2\ns : Finset ι\nι₂ : Type ?u.31556\ns₂ : Finset ι₂\nw : ι → k\np : ι → P\nh : ∑ i in s, w i = 0\nb₁ b₂ : P\n⊢ ↑(weightedVSubOfPoint s p b₁) w - ↑(weightedVSubOfPoint s p b₂) w = 0", "tactic": "rw [weightedVSubOfPoint_apply, weightedVSubOfPoint_apply, ← sum_sub_distrib]" }, { "state_after": "no goals", "state_before": "case h\nk : Type u_1\nV : Type u_3\nP : Type u_4\ninst✝² : Ring k\ninst✝¹ : AddCommGroup V\ninst✝ : Module k V\nS : AffineSpace V P\nι : Type u_2\ns : Finset ι\nι₂ : Type ?u.31556\ns₂ : Finset ι₂\nw : ι → k\np : ι → P\nh : ∑ i in s, w i = 0\nb₁ b₂ : P\n⊢ ∑ x in s, w x • (b₂ -ᵥ b₁) = 0", "tactic": "rw [← sum_smul, h, zero_smul]" } ]
[ 127, 32 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 118, 1 ]
Mathlib/Analysis/InnerProductSpace/Projection.lean
orthogonalProjectionFn_eq
[]
[ 476, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 474, 1 ]
Mathlib/Algebra/Parity.lean
Even.mul_left
[]
[ 282, 34 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 281, 1 ]
Mathlib/Data/List/Basic.lean
List.take_cons
[]
[ 1926, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1925, 1 ]
Mathlib/Analysis/InnerProductSpace/PiL2.lean
EuclideanSpace.edist_eq
[]
[ 143, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 141, 1 ]
Mathlib/Data/Set/Finite.lean
Finset.bddBelow
[]
[ 1646, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1645, 11 ]
Mathlib/Topology/Algebra/Module/Basic.lean
ContinuousLinearMap.to_ring_inverse
[ { "state_after": "case pos\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ∃ e', ↑e' = f\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)\n\ncase neg\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ¬∃ e', ↑e' = f\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "state_before": "R : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "tactic": "by_cases h₁ : ∃ e' : M ≃L[R] M₂, e' = f" }, { "state_after": "case pos.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "state_before": "case pos\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ∃ e', ↑e' = f\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "tactic": "obtain ⟨e', he'⟩ := h₁" }, { "state_after": "case pos.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\n⊢ inverse ↑e' = comp (Ring.inverse (comp ↑(ContinuousLinearEquiv.symm e) ↑e')) ↑(ContinuousLinearEquiv.symm e)", "state_before": "case pos.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "tactic": "rw [← he']" }, { "state_after": "case pos.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\n⊢ inverse ↑e' =\n comp (Ring.inverse ↑(ContinuousLinearEquiv.trans e' (ContinuousLinearEquiv.symm e))) ↑(ContinuousLinearEquiv.symm e)", "state_before": "case pos.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\n⊢ inverse ↑e' = comp (Ring.inverse (comp ↑(ContinuousLinearEquiv.symm e) ↑e')) ↑(ContinuousLinearEquiv.symm e)", "tactic": "change _ = Ring.inverse (e'.trans e.symm : M →L[R] M) ∘L (e.symm : M₂ →L[R] M)" }, { "state_after": "case pos.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\nx✝ : M₂\n⊢ ↑(inverse ↑e') x✝ =\n ↑(comp (Ring.inverse ↑(ContinuousLinearEquiv.trans e' (ContinuousLinearEquiv.symm e)))\n ↑(ContinuousLinearEquiv.symm e))\n x✝", "state_before": "case pos.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\n⊢ inverse ↑e' =\n comp (Ring.inverse ↑(ContinuousLinearEquiv.trans e' (ContinuousLinearEquiv.symm e))) ↑(ContinuousLinearEquiv.symm e)", "tactic": "ext" }, { "state_after": "no goals", "state_before": "case pos.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\ne' : M ≃L[R] M₂\nhe' : ↑e' = f\nx✝ : M₂\n⊢ ↑(inverse ↑e') x✝ =\n ↑(comp (Ring.inverse ↑(ContinuousLinearEquiv.trans e' (ContinuousLinearEquiv.symm e)))\n ↑(ContinuousLinearEquiv.symm e))\n x✝", "tactic": "simp" }, { "state_after": "case neg\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ¬∃ e', ↑e' = f\n⊢ ¬IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f)", "state_before": "case neg\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ¬∃ e', ↑e' = f\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "tactic": "suffices ¬IsUnit ((e.symm : M₂ →L[R] M).comp f) by simp [this, h₁]" }, { "state_after": "case neg\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f)\n⊢ ∃ e', ↑e' = f", "state_before": "case neg\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ¬∃ e', ↑e' = f\n⊢ ¬IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f)", "tactic": "contrapose! h₁" }, { "state_after": "case neg.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\n⊢ ∃ e', ↑e' = f", "state_before": "case neg\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f)\n⊢ ∃ e', ↑e' = f", "tactic": "rcases h₁ with ⟨F, hF⟩" }, { "state_after": "case neg.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\n⊢ ↑(ContinuousLinearEquiv.trans (↑(ContinuousLinearEquiv.unitsEquiv R M) F) e) = f", "state_before": "case neg.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\n⊢ ∃ e', ↑e' = f", "tactic": "use (ContinuousLinearEquiv.unitsEquiv _ _ F).trans e" }, { "state_after": "case neg.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\nx✝ : M\n⊢ ↑↑(ContinuousLinearEquiv.trans (↑(ContinuousLinearEquiv.unitsEquiv R M) F) e) x✝ = ↑f x✝", "state_before": "case neg.intro\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\n⊢ ↑(ContinuousLinearEquiv.trans (↑(ContinuousLinearEquiv.unitsEquiv R M) F) e) = f", "tactic": "ext" }, { "state_after": "case neg.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\nx✝ : M\n⊢ ↑e (↑↑F x✝) = ↑f x✝", "state_before": "case neg.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\nx✝ : M\n⊢ ↑↑(ContinuousLinearEquiv.trans (↑(ContinuousLinearEquiv.unitsEquiv R M) F) e) x✝ = ↑f x✝", "tactic": "dsimp" }, { "state_after": "case neg.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\nx✝ : M\n⊢ ↑e (↑(comp (↑(ContinuousLinearEquiv.symm e)) f) x✝) = ↑f x✝", "state_before": "case neg.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\nx✝ : M\n⊢ ↑e (↑↑F x✝) = ↑f x✝", "tactic": "rw [hF]" }, { "state_after": "no goals", "state_before": "case neg.intro.h\nR : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nF : (M →L[R] M)ˣ\nhF : ↑F = comp (↑(ContinuousLinearEquiv.symm e)) f\nx✝ : M\n⊢ ↑e (↑(comp (↑(ContinuousLinearEquiv.symm e)) f) x✝) = ↑f x✝", "tactic": "simp" }, { "state_after": "no goals", "state_before": "R : Type u_1\nM : Type u_2\nM₂ : Type u_3\ninst✝⁷ : TopologicalSpace M\ninst✝⁶ : TopologicalSpace M₂\ninst✝⁵ : Ring R\ninst✝⁴ : AddCommGroup M\ninst✝³ : TopologicalAddGroup M\ninst✝² : Module R M\ninst✝¹ : AddCommGroup M₂\ninst✝ : Module R M₂\ne : M ≃L[R] M₂\nf : M →L[R] M₂\nh₁ : ¬∃ e', ↑e' = f\nthis : ¬IsUnit (comp (↑(ContinuousLinearEquiv.symm e)) f)\n⊢ inverse f = comp (Ring.inverse (comp (↑(ContinuousLinearEquiv.symm e)) f)) ↑(ContinuousLinearEquiv.symm e)", "tactic": "simp [this, h₁]" } ]
[ 2545, 9 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2530, 1 ]
Mathlib/Algebra/Algebra/Operations.lean
Submodule.pow_toAddSubmonoid
[ { "state_after": "case zero\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝ : A\nn : ℕ\nh✝ : n ≠ 0\nh : Nat.zero ≠ 0\n⊢ (M ^ Nat.zero).toAddSubmonoid = M.toAddSubmonoid ^ Nat.zero\n\ncase succ\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝¹ : A\nn✝ : ℕ\nh✝ : n✝ ≠ 0\nn : ℕ\nih : n ≠ 0 → (M ^ n).toAddSubmonoid = M.toAddSubmonoid ^ n\nh : Nat.succ n ≠ 0\n⊢ (M ^ Nat.succ n).toAddSubmonoid = M.toAddSubmonoid ^ Nat.succ n", "state_before": "ι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝ : A\nn : ℕ\nh : n ≠ 0\n⊢ (M ^ n).toAddSubmonoid = M.toAddSubmonoid ^ n", "tactic": "induction' n with n ih" }, { "state_after": "no goals", "state_before": "case zero\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝ : A\nn : ℕ\nh✝ : n ≠ 0\nh : Nat.zero ≠ 0\n⊢ (M ^ Nat.zero).toAddSubmonoid = M.toAddSubmonoid ^ Nat.zero", "tactic": "exact (h rfl).elim" }, { "state_after": "case succ\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝¹ : A\nn✝ : ℕ\nh✝ : n✝ ≠ 0\nn : ℕ\nih : n ≠ 0 → (M ^ n).toAddSubmonoid = M.toAddSubmonoid ^ n\nh : Nat.succ n ≠ 0\n⊢ M.toAddSubmonoid * (M ^ n).toAddSubmonoid = M.toAddSubmonoid * M.toAddSubmonoid ^ n", "state_before": "case succ\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝¹ : A\nn✝ : ℕ\nh✝ : n✝ ≠ 0\nn : ℕ\nih : n ≠ 0 → (M ^ n).toAddSubmonoid = M.toAddSubmonoid ^ n\nh : Nat.succ n ≠ 0\n⊢ (M ^ Nat.succ n).toAddSubmonoid = M.toAddSubmonoid ^ Nat.succ n", "tactic": "rw [pow_succ, pow_succ, mul_toAddSubmonoid]" }, { "state_after": "no goals", "state_before": "case succ\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝¹ : A\nn✝ : ℕ\nh✝ : n✝ ≠ 0\nn : ℕ\nih : n ≠ 0 → (M ^ n).toAddSubmonoid = M.toAddSubmonoid ^ n\nh : Nat.succ n ≠ 0\n⊢ M.toAddSubmonoid * (M ^ n).toAddSubmonoid = M.toAddSubmonoid * M.toAddSubmonoid ^ n", "tactic": "cases n with\n| zero => rw [pow_zero, pow_zero, mul_one, ← mul_toAddSubmonoid, mul_one]\n| succ n => rw [ih n.succ_ne_zero]" }, { "state_after": "no goals", "state_before": "case succ.zero\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝ : A\nn : ℕ\nh✝ : n ≠ 0\nih : Nat.zero ≠ 0 → (M ^ Nat.zero).toAddSubmonoid = M.toAddSubmonoid ^ Nat.zero\nh : Nat.succ Nat.zero ≠ 0\n⊢ M.toAddSubmonoid * (M ^ Nat.zero).toAddSubmonoid = M.toAddSubmonoid * M.toAddSubmonoid ^ Nat.zero", "tactic": "rw [pow_zero, pow_zero, mul_one, ← mul_toAddSubmonoid, mul_one]" }, { "state_after": "no goals", "state_before": "case succ.succ\nι : Sort uι\nR : Type u\ninst✝² : CommSemiring R\nA : Type v\ninst✝¹ : Semiring A\ninst✝ : Algebra R A\nS T : Set A\nM N P Q : Submodule R A\nm n✝¹ : A\nn✝ : ℕ\nh✝ : n✝ ≠ 0\nn : ℕ\nih : Nat.succ n ≠ 0 → (M ^ Nat.succ n).toAddSubmonoid = M.toAddSubmonoid ^ Nat.succ n\nh : Nat.succ (Nat.succ n) ≠ 0\n⊢ M.toAddSubmonoid * (M ^ Nat.succ n).toAddSubmonoid = M.toAddSubmonoid * M.toAddSubmonoid ^ Nat.succ n", "tactic": "rw [ih n.succ_ne_zero]" } ]
[ 425, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 419, 1 ]
Mathlib/SetTheory/ZFC/Basic.lean
ZFSet.toSet_subset_iff
[ { "state_after": "no goals", "state_before": "x y : ZFSet\n⊢ toSet x ⊆ toSet y ↔ x ⊆ y", "tactic": "simp [subset_def, Set.subset_def]" } ]
[ 792, 36 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 791, 1 ]
Mathlib/Algebra/Group/Pi.lean
Pi.mulSingle_inf
[]
[ 486, 30 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 484, 1 ]
Mathlib/Combinatorics/Hindman.lean
Hindman.FP.singleton
[ { "state_after": "case zero\nM : Type u_1\ninst✝ : Semigroup M\na✝ a : Stream' M\n⊢ Stream'.nth a Nat.zero ∈ FP a\n\ncase succ\nM : Type u_1\ninst✝ : Semigroup M\na✝ : Stream' M\ni : ℕ\nih : ∀ (a : Stream' M), Stream'.nth a i ∈ FP a\na : Stream' M\n⊢ Stream'.nth a (Nat.succ i) ∈ FP a", "state_before": "M : Type u_1\ninst✝ : Semigroup M\na : Stream' M\ni : ℕ\n⊢ Stream'.nth a i ∈ FP a", "tactic": "induction' i with i ih generalizing a" }, { "state_after": "no goals", "state_before": "case zero\nM : Type u_1\ninst✝ : Semigroup M\na✝ a : Stream' M\n⊢ Stream'.nth a Nat.zero ∈ FP a", "tactic": "apply FP.head" }, { "state_after": "case succ.h\nM : Type u_1\ninst✝ : Semigroup M\na✝ : Stream' M\ni : ℕ\nih : ∀ (a : Stream' M), Stream'.nth a i ∈ FP a\na : Stream' M\n⊢ FP (Stream'.tail a) (Stream'.nth a (Nat.succ i))", "state_before": "case succ\nM : Type u_1\ninst✝ : Semigroup M\na✝ : Stream' M\ni : ℕ\nih : ∀ (a : Stream' M), Stream'.nth a i ∈ FP a\na : Stream' M\n⊢ Stream'.nth a (Nat.succ i) ∈ FP a", "tactic": "apply FP.tail" }, { "state_after": "no goals", "state_before": "case succ.h\nM : Type u_1\ninst✝ : Semigroup M\na✝ : Stream' M\ni : ℕ\nih : ∀ (a : Stream' M), Stream'.nth a i ∈ FP a\na : Stream' M\n⊢ FP (Stream'.tail a) (Stream'.nth a (Nat.succ i))", "tactic": "apply ih" } ]
[ 262, 13 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 258, 1 ]
Mathlib/CategoryTheory/Monoidal/Rigid/Basic.lean
CategoryTheory.rightAdjointMate_comp_evaluation
[ { "state_after": "C : Type u₁\ninst✝³ : Category C\ninst✝² : MonoidalCategory C\nX Y : C\ninst✝¹ : HasRightDual X\ninst✝ : HasRightDual Y\nf : X ⟶ Y\n⊢ ↑(tensorRightHomEquiv Yᘁ X Xᘁ (𝟙_ C)) ((fᘁ ⊗ 𝟙 X) ≫ ε_ X Xᘁ) =\n ↑(tensorRightHomEquiv Yᘁ X Xᘁ (𝟙_ C)) ((𝟙 Yᘁ ⊗ f) ≫ ε_ Y Yᘁ)", "state_before": "C : Type u₁\ninst✝³ : Category C\ninst✝² : MonoidalCategory C\nX Y : C\ninst✝¹ : HasRightDual X\ninst✝ : HasRightDual Y\nf : X ⟶ Y\n⊢ (fᘁ ⊗ 𝟙 X) ≫ ε_ X Xᘁ = (𝟙 Yᘁ ⊗ f) ≫ ε_ Y Yᘁ", "tactic": "apply_fun tensorRightHomEquiv _ X (Xᘁ) _" }, { "state_after": "no goals", "state_before": "C : Type u₁\ninst✝³ : Category C\ninst✝² : MonoidalCategory C\nX Y : C\ninst✝¹ : HasRightDual X\ninst✝ : HasRightDual Y\nf : X ⟶ Y\n⊢ ↑(tensorRightHomEquiv Yᘁ X Xᘁ (𝟙_ C)) ((fᘁ ⊗ 𝟙 X) ≫ ε_ X Xᘁ) =\n ↑(tensorRightHomEquiv Yᘁ X Xᘁ (𝟙_ C)) ((𝟙 Yᘁ ⊗ f) ≫ ε_ Y Yᘁ)", "tactic": "simp" } ]
[ 566, 7 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 563, 1 ]
Mathlib/CategoryTheory/Limits/Shapes/ZeroObjects.lean
CategoryTheory.Limits.IsZero.unop
[]
[ 138, 95 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 136, 1 ]
Mathlib/Topology/Separation.lean
t0Space_of_injective_of_continuous
[]
[ 326, 38 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 324, 1 ]
Mathlib/NumberTheory/Padics/PadicVal.lean
range_pow_padicValNat_subset_divisors
[ { "state_after": "p n : ℕ\nhn : n ≠ 0\nt : ℕ\nht : t ∈ Finset.image (fun x => p ^ x) (Finset.range (padicValNat p n + 1))\n⊢ t ∈ divisors n", "state_before": "p n : ℕ\nhn : n ≠ 0\n⊢ Finset.image (fun x => p ^ x) (Finset.range (padicValNat p n + 1)) ⊆ divisors n", "tactic": "intro t ht" }, { "state_after": "p n : ℕ\nhn : n ≠ 0\nt : ℕ\nht : ∃ a, a < padicValNat p n + 1 ∧ p ^ a = t\n⊢ t ∈ divisors n", "state_before": "p n : ℕ\nhn : n ≠ 0\nt : ℕ\nht : t ∈ Finset.image (fun x => p ^ x) (Finset.range (padicValNat p n + 1))\n⊢ t ∈ divisors n", "tactic": "simp only [exists_prop, Finset.mem_image, Finset.mem_range] at ht" }, { "state_after": "case intro.intro\np n : ℕ\nhn : n ≠ 0\nk : ℕ\nhk : k < padicValNat p n + 1\n⊢ p ^ k ∈ divisors n", "state_before": "p n : ℕ\nhn : n ≠ 0\nt : ℕ\nht : ∃ a, a < padicValNat p n + 1 ∧ p ^ a = t\n⊢ t ∈ divisors n", "tactic": "obtain ⟨k, hk, rfl⟩ := ht" }, { "state_after": "case intro.intro\np n : ℕ\nhn : n ≠ 0\nk : ℕ\nhk : k < padicValNat p n + 1\n⊢ p ^ k ∣ n ∧ n ≠ 0", "state_before": "case intro.intro\np n : ℕ\nhn : n ≠ 0\nk : ℕ\nhk : k < padicValNat p n + 1\n⊢ p ^ k ∈ divisors n", "tactic": "rw [Nat.mem_divisors]" }, { "state_after": "no goals", "state_before": "case intro.intro\np n : ℕ\nhn : n ≠ 0\nk : ℕ\nhk : k < padicValNat p n + 1\n⊢ p ^ k ∣ n ∧ n ≠ 0", "tactic": "exact ⟨(pow_dvd_pow p <| by linarith).trans pow_padicValNat_dvd, hn⟩" }, { "state_after": "no goals", "state_before": "p n : ℕ\nhn : n ≠ 0\nk : ℕ\nhk : k < padicValNat p n + 1\n⊢ k ≤ padicValNat p n", "tactic": "linarith" } ]
[ 495, 71 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 489, 1 ]
Mathlib/Data/Polynomial/Degree/Definitions.lean
Polynomial.natDegree_C
[ { "state_after": "case pos\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\n⊢ natDegree (↑C a) = 0\n\ncase neg\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : ¬a = 0\n⊢ natDegree (↑C a) = 0", "state_before": "R : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\n⊢ natDegree (↑C a) = 0", "tactic": "by_cases ha : a = 0" }, { "state_after": "case pos\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\nthis : ↑C a = 0\n⊢ natDegree (↑C a) = 0", "state_before": "case pos\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\n⊢ natDegree (↑C a) = 0", "tactic": "have : C a = 0 := by rw [ha, C_0]" }, { "state_after": "case pos\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\nthis : ↑C a = 0\n⊢ WithBot.unbot' 0 ⊥ = 0", "state_before": "case pos\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\nthis : ↑C a = 0\n⊢ natDegree (↑C a) = 0", "tactic": "rw [natDegree, degree_eq_bot.2 this]" }, { "state_after": "no goals", "state_before": "case pos\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\nthis : ↑C a = 0\n⊢ WithBot.unbot' 0 ⊥ = 0", "tactic": "rfl" }, { "state_after": "no goals", "state_before": "R : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : a = 0\n⊢ ↑C a = 0", "tactic": "rw [ha, C_0]" }, { "state_after": "case neg\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : ¬a = 0\n⊢ WithBot.unbot' 0 0 = 0", "state_before": "case neg\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : ¬a = 0\n⊢ natDegree (↑C a) = 0", "tactic": "rw [natDegree, degree_C ha]" }, { "state_after": "no goals", "state_before": "case neg\nR : Type u\nS : Type v\na✝ b c d : R\nn m : ℕ\ninst✝ : Semiring R\np q r : R[X]\na : R\nha : ¬a = 0\n⊢ WithBot.unbot' 0 0 = 0", "tactic": "rfl" } ]
[ 275, 8 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 269, 1 ]
Mathlib/Data/Multiset/Lattice.lean
Multiset.sup_le
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝¹ : SemilatticeSup α\ninst✝ : OrderBot α\ns : Multiset α\na : α\n⊢ sup 0 ≤ a ↔ ∀ (b : α), b ∈ 0 → b ≤ a", "tactic": "simp" }, { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝¹ : SemilatticeSup α\ninst✝ : OrderBot α\ns : Multiset α\na : α\n⊢ ∀ ⦃a_1 : α⦄ {s : Multiset α},\n (sup s ≤ a ↔ ∀ (b : α), b ∈ s → b ≤ a) → (sup (a_1 ::ₘ s) ≤ a ↔ ∀ (b : α), b ∈ a_1 ::ₘ s → b ≤ a)", "tactic": "simp (config := { contextual := true }) [or_imp, forall_and]" } ]
[ 63, 70 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 61, 1 ]
Mathlib/Data/Nat/Digits.lean
Nat.lt_base_pow_length_digits
[ { "state_after": "case succ.succ\nn m b : ℕ\n⊢ m < succ (succ b) ^ List.length (digits (succ (succ b)) m)", "state_before": "n b m : ℕ\nhb : 1 < b\n⊢ m < b ^ List.length (digits b m)", "tactic": "rcases b with (_ | _ | b) <;> try simp_all" }, { "state_after": "no goals", "state_before": "case succ.succ\nn m b : ℕ\n⊢ m < succ (succ b) ^ List.length (digits (succ (succ b)) m)", "tactic": "exact lt_base_pow_length_digits'" }, { "state_after": "case succ.succ\nn m b : ℕ\n⊢ m < succ (succ b) ^ List.length (digits (succ (succ b)) m)", "state_before": "case succ.succ\nn m b : ℕ\nhb : 1 < succ (succ b)\n⊢ m < succ (succ b) ^ List.length (digits (succ (succ b)) m)", "tactic": "simp_all" } ]
[ 424, 35 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 422, 1 ]
Mathlib/Data/Polynomial/Degree/Definitions.lean
Polynomial.degree_C_mul_X_pow_le
[ { "state_after": "R : Type u\nS : Type v\na✝ b c d : R\nn✝ m : ℕ\ninst✝ : Semiring R\np q r : R[X]\nn : ℕ\na : R\n⊢ degree (↑(monomial n) a) ≤ ↑n", "state_before": "R : Type u\nS : Type v\na✝ b c d : R\nn✝ m : ℕ\ninst✝ : Semiring R\np q r : R[X]\nn : ℕ\na : R\n⊢ degree (↑C a * X ^ n) ≤ ↑n", "tactic": "rw [C_mul_X_pow_eq_monomial]" }, { "state_after": "no goals", "state_before": "R : Type u\nS : Type v\na✝ b c d : R\nn✝ m : ℕ\ninst✝ : Semiring R\np q r : R[X]\nn : ℕ\na : R\n⊢ degree (↑(monomial n) a) ≤ ↑n", "tactic": "apply degree_monomial_le" } ]
[ 309, 27 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 307, 1 ]
Mathlib/AlgebraicTopology/SimplexCategory.lean
SimplexCategory.skeletalFunctor.coe_map
[]
[ 365, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 363, 1 ]
src/lean/Init/Data/Char/Basic.lean
Char.isValidUInt32
[ { "state_after": "no goals", "state_before": "n : Nat\nh : isValidCharNat n\n⊢ n < UInt32.size", "tactic": "match h with\n| Or.inl h =>\n apply Nat.lt_trans h\n decide\n| Or.inr ⟨_, h₂⟩ =>\n apply Nat.lt_trans h₂\n decide" }, { "state_after": "n : Nat\nh✝ : isValidCharNat n\nh : n < 55296\n⊢ 55296 < UInt32.size", "state_before": "n : Nat\nh✝ : isValidCharNat n\nh : n < 55296\n⊢ n < UInt32.size", "tactic": "apply Nat.lt_trans h" }, { "state_after": "no goals", "state_before": "n : Nat\nh✝ : isValidCharNat n\nh : n < 55296\n⊢ 55296 < UInt32.size", "tactic": "decide" }, { "state_after": "n : Nat\nh : isValidCharNat n\nleft✝ : 57343 < n\nh₂ : n < 1114112\n⊢ 1114112 < UInt32.size", "state_before": "n : Nat\nh : isValidCharNat n\nleft✝ : 57343 < n\nh₂ : n < 1114112\n⊢ n < UInt32.size", "tactic": "apply Nat.lt_trans h₂" }, { "state_after": "no goals", "state_before": "n : Nat\nh : isValidCharNat n\nleft✝ : 57343 < n\nh₂ : n < 1114112\n⊢ 1114112 < UInt32.size", "tactic": "decide" } ]
[ 41, 11 ]
d5348dfac847a56a4595fb6230fd0708dcb4e7e9
https://github.com/leanprover/lean4
[ 34, 1 ]
Mathlib/Analysis/Convex/Function.lean
LinearMap.concaveOn
[ { "state_after": "no goals", "state_before": "𝕜 : Type u_1\nE : Type u_2\nF : Type ?u.183332\nα : Type ?u.183335\nβ : Type u_3\nι : Type ?u.183341\ninst✝⁶ : OrderedSemiring 𝕜\ninst✝⁵ : AddCommMonoid E\ninst✝⁴ : AddCommMonoid F\ninst✝³ : OrderedAddCommMonoid α\ninst✝² : OrderedAddCommMonoid β\ninst✝¹ : Module 𝕜 E\ninst✝ : Module 𝕜 β\nf : E →ₗ[𝕜] β\ns : Set E\nhs : Convex 𝕜 s\nx✝⁸ : E\nx✝⁷ : x✝⁸ ∈ s\nx✝⁶ : E\nx✝⁵ : x✝⁶ ∈ s\nx✝⁴ x✝³ : 𝕜\nx✝² : 0 ≤ x✝⁴\nx✝¹ : 0 ≤ x✝³\nx✝ : x✝⁴ + x✝³ = 1\n⊢ x✝⁴ • ↑f x✝⁸ + x✝³ • ↑f x✝⁶ ≤ ↑f (x✝⁴ • x✝⁸ + x✝³ • x✝⁶)", "tactic": "rw [f.map_add, f.map_smul, f.map_smul]" } ]
[ 366, 75 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 365, 1 ]
Std/Data/List/Init/Lemmas.lean
List.drop_length_le
[]
[ 141, 62 ]
e68aa8f5fe47aad78987df45f99094afbcb5e936
https://github.com/leanprover/std4
[ 140, 1 ]
Mathlib/Analysis/NormedSpace/Basic.lean
frontier_closedBall
[ { "state_after": "no goals", "state_before": "α : Type ?u.89099\nβ : Type ?u.89102\nγ : Type ?u.89105\nι : Type ?u.89108\ninst✝⁶ : NormedField α\ninst✝⁵ : SeminormedAddCommGroup β\nE : Type u_1\ninst✝⁴ : SeminormedAddCommGroup E\ninst✝³ : NormedSpace α E\nF : Type ?u.89139\ninst✝² : SeminormedAddCommGroup F\ninst✝¹ : NormedSpace α F\ninst✝ : NormedSpace ℝ E\nx : E\nr : ℝ\nhr : r ≠ 0\n⊢ frontier (closedBall x r) = sphere x r", "tactic": "rw [frontier, closure_closedBall, interior_closedBall x hr, closedBall_diff_ball]" } ]
[ 155, 84 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 153, 1 ]
Mathlib/SetTheory/Ordinal/Arithmetic.lean
Ordinal.IsLimit.pos
[]
[ 288, 46 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 287, 1 ]
Mathlib/RingTheory/UniqueFactorizationDomain.lean
UniqueFactorizationMonoid.dvd_iff_normalizedFactors_le_normalizedFactors
[ { "state_after": "case mp\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ x ∣ y → normalizedFactors x ≤ normalizedFactors y\n\ncase mpr\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ normalizedFactors x ≤ normalizedFactors y → x ∣ y", "state_before": "α : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ x ∣ y ↔ normalizedFactors x ≤ normalizedFactors y", "tactic": "constructor" }, { "state_after": "case mp.intro\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx : α\nhx : x ≠ 0\nc : α\nhy : x * c ≠ 0\n⊢ normalizedFactors x ≤ normalizedFactors (x * c)", "state_before": "case mp\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ x ∣ y → normalizedFactors x ≤ normalizedFactors y", "tactic": "rintro ⟨c, rfl⟩" }, { "state_after": "no goals", "state_before": "case mp.intro\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx : α\nhx : x ≠ 0\nc : α\nhy : x * c ≠ 0\n⊢ normalizedFactors x ≤ normalizedFactors (x * c)", "tactic": "simp [hx, right_ne_zero_of_mul hy]" }, { "state_after": "case mpr\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ normalizedFactors x ≤ normalizedFactors y → Multiset.prod (normalizedFactors x) ∣ Multiset.prod (normalizedFactors y)", "state_before": "case mpr\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ normalizedFactors x ≤ normalizedFactors y → x ∣ y", "tactic": "rw [← (normalizedFactors_prod hx).dvd_iff_dvd_left, ←\n (normalizedFactors_prod hy).dvd_iff_dvd_right]" }, { "state_after": "no goals", "state_before": "case mpr\nα : Type u_1\ninst✝³ : CancelCommMonoidWithZero α\ninst✝² : DecidableEq α\ninst✝¹ : NormalizationMonoid α\ninst✝ : UniqueFactorizationMonoid α\nx y : α\nhx : x ≠ 0\nhy : y ≠ 0\n⊢ normalizedFactors x ≤ normalizedFactors y → Multiset.prod (normalizedFactors x) ∣ Multiset.prod (normalizedFactors y)", "tactic": "apply Multiset.prod_dvd_prod_of_le" } ]
[ 728, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 721, 1 ]
Mathlib/Analysis/NormedSpace/ContinuousLinearMap.lean
ContinuousLinearEquiv.toSpanNonzeroSingleton_homothety
[]
[ 276, 54 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 274, 1 ]
Mathlib/RingTheory/Polynomial/Bernstein.lean
bernsteinPolynomial.iterate_derivative_at_1
[ { "state_after": "R : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\n⊢ eval 1 ((↑derivative^[n - ν]) (comp (bernsteinPolynomial R n (n - ν)) (1 - X))) =\n (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "state_before": "R : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\n⊢ eval 1 ((↑derivative^[n - ν]) (bernsteinPolynomial R n ν)) = (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "tactic": "rw [flip' _ _ _ h]" }, { "state_after": "R : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\n⊢ (-1) ^ (n - ν) * eval (↑(n - (n - ν - 1))) (pochhammer R (n - ν)) =\n (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "state_before": "R : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\n⊢ eval 1 ((↑derivative^[n - ν]) (comp (bernsteinPolynomial R n (n - ν)) (1 - X))) =\n (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "tactic": "simp [Polynomial.eval_comp, h]" }, { "state_after": "case inl\nR : Type u_1\ninst✝ : CommRing R\nν : ℕ\nh : ν ≤ ν\n⊢ (-1) ^ (ν - ν) * eval (↑(ν - (ν - ν - 1))) (pochhammer R (ν - ν)) =\n (-1) ^ (ν - ν) * eval (↑ν + 1) (pochhammer R (ν - ν))\n\ncase inr\nR : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\nh' : ν < n\n⊢ (-1) ^ (n - ν) * eval (↑(n - (n - ν - 1))) (pochhammer R (n - ν)) =\n (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "state_before": "R : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\n⊢ (-1) ^ (n - ν) * eval (↑(n - (n - ν - 1))) (pochhammer R (n - ν)) =\n (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "tactic": "obtain rfl | h' := h.eq_or_lt" }, { "state_after": "no goals", "state_before": "case inl\nR : Type u_1\ninst✝ : CommRing R\nν : ℕ\nh : ν ≤ ν\n⊢ (-1) ^ (ν - ν) * eval (↑(ν - (ν - ν - 1))) (pochhammer R (ν - ν)) =\n (-1) ^ (ν - ν) * eval (↑ν + 1) (pochhammer R (ν - ν))", "tactic": "simp" }, { "state_after": "case inr.e_a.e_a\nR : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\nh' : ν < n\n⊢ ↑(n - (n - ν - 1)) = ↑ν + 1", "state_before": "case inr\nR : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\nh' : ν < n\n⊢ (-1) ^ (n - ν) * eval (↑(n - (n - ν - 1))) (pochhammer R (n - ν)) =\n (-1) ^ (n - ν) * eval (↑ν + 1) (pochhammer R (n - ν))", "tactic": "congr" }, { "state_after": "case inr.e_a.e_a\nR : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\nh' : ν < n\n⊢ ↑(n - (n - ν - 1)) = ↑(ν + 1)", "state_before": "case inr.e_a.e_a\nR : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\nh' : ν < n\n⊢ ↑(n - (n - ν - 1)) = ↑ν + 1", "tactic": "norm_cast" }, { "state_after": "no goals", "state_before": "case inr.e_a.e_a\nR : Type u_1\ninst✝ : CommRing R\nn ν : ℕ\nh : ν ≤ n\nh' : ν < n\n⊢ ↑(n - (n - ν - 1)) = ↑(ν + 1)", "tactic": "rw [← tsub_add_eq_tsub_tsub, tsub_tsub_cancel_of_le (Nat.succ_le_iff.mpr h')]" } ]
[ 238, 82 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 229, 1 ]
Mathlib/LinearAlgebra/StdBasis.lean
Pi.basis_repr
[]
[ 268, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 266, 1 ]