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/Data/Fintype/Basic.lean
Function.Embedding.invFun_restrict
[ { "state_after": "case h.mk\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.69537\ninst✝² : Fintype α\ninst✝¹ : DecidableEq β\nf : α ↪ β\nb✝ : ↑(Set.range ↑f)\ninst✝ : Nonempty α\nb : β\nh : b ∈ Set.range ↑f\n⊢ Set.restrict (Set.range ↑f) (invFun ↑f) { val := b, property := h } = invOfMemRange f { val := b, property := h }", "state_before": "α : Type u_1\nβ : Type u_2\nγ : Type ?u.69537\ninst✝² : Fintype α\ninst✝¹ : DecidableEq β\nf : α ↪ β\nb : ↑(Set.range ↑f)\ninst✝ : Nonempty α\n⊢ Set.restrict (Set.range ↑f) (invFun ↑f) = invOfMemRange f", "tactic": "ext ⟨b, h⟩" }, { "state_after": "case h.mk.a\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.69537\ninst✝² : Fintype α\ninst✝¹ : DecidableEq β\nf : α ↪ β\nb✝ : ↑(Set.range ↑f)\ninst✝ : Nonempty α\nb : β\nh : b ∈ Set.range ↑f\n⊢ ↑f (Set.restrict (Set.range ↑f) (invFun ↑f) { val := b, property := h }) =\n ↑f (invOfMemRange f { val := b, property := h })", "state_before": "case h.mk\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.69537\ninst✝² : Fintype α\ninst✝¹ : DecidableEq β\nf : α ↪ β\nb✝ : ↑(Set.range ↑f)\ninst✝ : Nonempty α\nb : β\nh : b ∈ Set.range ↑f\n⊢ Set.restrict (Set.range ↑f) (invFun ↑f) { val := b, property := h } = invOfMemRange f { val := b, property := h }", "tactic": "apply f.injective" }, { "state_after": "no goals", "state_before": "case h.mk.a\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.69537\ninst✝² : Fintype α\ninst✝¹ : DecidableEq β\nf : α ↪ β\nb✝ : ↑(Set.range ↑f)\ninst✝ : Nonempty α\nb : β\nh : b ∈ Set.range ↑f\n⊢ ↑f (Set.restrict (Set.range ↑f) (invFun ↑f) { val := b, property := h }) =\n ↑f (invOfMemRange f { val := b, property := h })", "tactic": "simp [f.left_inv_of_invOfMemRange, @invFun_eq _ _ _ f b (Set.mem_range.mp h)]" } ]
[ 546, 80 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 543, 1 ]
Mathlib/MeasureTheory/Function/EssSup.lean
ae_lt_of_essSup_lt
[]
[ 106, 35 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 103, 1 ]
Mathlib/Computability/Primrec.lean
Primrec.decode
[]
[ 227, 48 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 226, 11 ]
Mathlib/Data/Prod/TProd.lean
List.TProd.ext
[ { "state_after": "case h₁\nι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v.fst = w.fst\n\ncase h₂\nι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v.snd = w.snd", "state_before": "ι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v = w", "tactic": "apply Prod.ext" }, { "state_after": "case h₂\nι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v.snd = w.snd", "state_before": "case h₁\nι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v.fst = w.fst\n\ncase h₂\nι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v.snd = w.snd", "tactic": "rw [← elim_self v, hvw, elim_self]" }, { "state_after": "case h₂\nι : Type u\nα : ι → Type v\ni✝ j✝ : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\nj : ι\nhj : j ∈ is\n⊢ TProd.elim v.snd hj = TProd.elim w.snd hj", "state_before": "case h₂\nι : Type u\nα : ι → Type v\ni✝ j : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\n⊢ v.snd = w.snd", "tactic": "refine' ext (nodup_cons.mp hl).2 fun j hj => _" }, { "state_after": "no goals", "state_before": "case h₂\nι : Type u\nα : ι → Type v\ni✝ j✝ : ι\nl : List ι\nf : (i : ι) → α i\ninst✝ : DecidableEq ι\ni : ι\nis : List ι\nhl : Nodup (i :: is)\nv w : TProd α (i :: is)\nhvw : ∀ (i_1 : ι) (hi : i_1 ∈ i :: is), TProd.elim v hi = TProd.elim w hi\nj : ι\nhj : j ∈ is\n⊢ TProd.elim v.snd hj = TProd.elim w.snd hj", "tactic": "rw [← elim_of_mem hl, hvw, elim_of_mem hl]" } ]
[ 126, 47 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 119, 1 ]
Mathlib/Algebra/Ring/Commute.lean
mul_self_eq_one_iff
[ { "state_after": "no goals", "state_before": "α : Type u\nβ : Type v\nγ : Type w\nR : Type x\ninst✝¹ : NonAssocRing R\ninst✝ : NoZeroDivisors R\na : R\n⊢ a * a = 1 ↔ a = 1 ∨ a = -1", "tactic": "rw [← (Commute.one_right a).mul_self_eq_mul_self_iff, mul_one]" } ]
[ 166, 65 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 164, 1 ]
Mathlib/Algebra/Order/EuclideanAbsoluteValue.lean
AbsoluteValue.IsEuclidean.map_lt_map_iff
[]
[ 55, 20 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 54, 1 ]
Mathlib/Algebra/Homology/HomologicalComplex.lean
HomologicalComplex.Hom.comm_to
[]
[ 551, 13 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 550, 1 ]
Mathlib/Algebra/Free.lean
Magma.AssocQuotient.lift_comp_of'
[]
[ 423, 100 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 423, 1 ]
src/lean/Init/SimpLemmas.lean
Nat.le_zero_eq
[ { "state_after": "no goals", "state_before": "a : Nat\nh : a = 0\n⊢ a ≤ 0", "tactic": "simp [h]" } ]
[ 155, 78 ]
d5348dfac847a56a4595fb6230fd0708dcb4e7e9
https://github.com/leanprover/lean4
[ 154, 9 ]
Mathlib/Analysis/Calculus/FDeriv/Add.lean
DifferentiableWithinAt.add_const
[]
[ 199, 60 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 197, 1 ]
Mathlib/Data/Polynomial/RingDivision.lean
Polynomial.rootSet_maps_to'
[ { "state_after": "R : Type u\nS✝ : Type v\nT : Type w\na b : R\nn : ℕ\ninst✝⁸ : CommRing R\ninst✝⁷ : IsDomain R\np✝ q : R[X]\ninst✝⁶ : CommRing T\np : T[X]\nS : Type u_1\nS' : Type u_2\ninst✝⁵ : CommRing S\ninst✝⁴ : IsDomain S\ninst✝³ : Algebra T S\ninst✝² : CommRing S'\ninst✝¹ : IsDomain S'\ninst✝ : Algebra T S'\nhp : map (algebraMap T S') p = 0 → map (algebraMap T S) p = 0\nf : S →ₐ[T] S'\nx : S\nhx : map (algebraMap T S) p ≠ 0 ∧ ↑(aeval x) p = 0\n⊢ map (algebraMap T S') p ≠ 0 ∧ ↑(aeval (↑f x)) p = 0", "state_before": "R : Type u\nS✝ : Type v\nT : Type w\na b : R\nn : ℕ\ninst✝⁸ : CommRing R\ninst✝⁷ : IsDomain R\np✝ q : R[X]\ninst✝⁶ : CommRing T\np : T[X]\nS : Type u_1\nS' : Type u_2\ninst✝⁵ : CommRing S\ninst✝⁴ : IsDomain S\ninst✝³ : Algebra T S\ninst✝² : CommRing S'\ninst✝¹ : IsDomain S'\ninst✝ : Algebra T S'\nhp : map (algebraMap T S') p = 0 → map (algebraMap T S) p = 0\nf : S →ₐ[T] S'\nx : S\nhx : x ∈ rootSet p S\n⊢ ↑f x ∈ rootSet p S'", "tactic": "rw [mem_rootSet'] at hx⊢" }, { "state_after": "R : Type u\nS✝ : Type v\nT : Type w\na b : R\nn : ℕ\ninst✝⁸ : CommRing R\ninst✝⁷ : IsDomain R\np✝ q : R[X]\ninst✝⁶ : CommRing T\np : T[X]\nS : Type u_1\nS' : Type u_2\ninst✝⁵ : CommRing S\ninst✝⁴ : IsDomain S\ninst✝³ : Algebra T S\ninst✝² : CommRing S'\ninst✝¹ : IsDomain S'\ninst✝ : Algebra T S'\nhp : map (algebraMap T S') p = 0 → map (algebraMap T S) p = 0\nf : S →ₐ[T] S'\nx : S\nhx : map (algebraMap T S) p ≠ 0 ∧ ↑(aeval x) p = 0\n⊢ map (algebraMap T S') p ≠ 0 ∧ 0 = 0", "state_before": "R : Type u\nS✝ : Type v\nT : Type w\na b : R\nn : ℕ\ninst✝⁸ : CommRing R\ninst✝⁷ : IsDomain R\np✝ q : R[X]\ninst✝⁶ : CommRing T\np : T[X]\nS : Type u_1\nS' : Type u_2\ninst✝⁵ : CommRing S\ninst✝⁴ : IsDomain S\ninst✝³ : Algebra T S\ninst✝² : CommRing S'\ninst✝¹ : IsDomain S'\ninst✝ : Algebra T S'\nhp : map (algebraMap T S') p = 0 → map (algebraMap T S) p = 0\nf : S →ₐ[T] S'\nx : S\nhx : map (algebraMap T S) p ≠ 0 ∧ ↑(aeval x) p = 0\n⊢ map (algebraMap T S') p ≠ 0 ∧ ↑(aeval (↑f x)) p = 0", "tactic": "rw [aeval_algHom, AlgHom.comp_apply, hx.2, _root_.map_zero]" }, { "state_after": "no goals", "state_before": "R : Type u\nS✝ : Type v\nT : Type w\na b : R\nn : ℕ\ninst✝⁸ : CommRing R\ninst✝⁷ : IsDomain R\np✝ q : R[X]\ninst✝⁶ : CommRing T\np : T[X]\nS : Type u_1\nS' : Type u_2\ninst✝⁵ : CommRing S\ninst✝⁴ : IsDomain S\ninst✝³ : Algebra T S\ninst✝² : CommRing S'\ninst✝¹ : IsDomain S'\ninst✝ : Algebra T S'\nhp : map (algebraMap T S') p = 0 → map (algebraMap T S) p = 0\nf : S →ₐ[T] S'\nx : S\nhx : map (algebraMap T S) p ≠ 0 ∧ ↑(aeval x) p = 0\n⊢ map (algebraMap T S') p ≠ 0 ∧ 0 = 0", "tactic": "exact ⟨mt hp hx.1, rfl⟩" } ]
[ 958, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 953, 1 ]
Mathlib/Order/SuccPred/Basic.lean
Order.le_pred_iff_of_not_isMin
[]
[ 641, 66 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 640, 1 ]
Mathlib/Algebra/Order/Interval.lean
NonemptyInterval.snd_mul
[]
[ 189, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 188, 1 ]
Mathlib/Analysis/Convex/Side.lean
Function.Injective.wSameSide_map_iff
[ { "state_after": "R : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nh : WSameSide (map f s) (↑f x) (↑f y)\n⊢ WSameSide s x y", "state_before": "R : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\n⊢ WSameSide (map f s) (↑f x) (↑f y) ↔ WSameSide s x y", "tactic": "refine' ⟨fun h => _, fun h => h.map _⟩" }, { "state_after": "case intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nfp₁ : P'\nhfp₁ : fp₁ ∈ map f s\nfp₂ : P'\nhfp₂ : fp₂ ∈ map f s\nh : SameRay R (↑f x -ᵥ fp₁) (↑f y -ᵥ fp₂)\n⊢ WSameSide s x y", "state_before": "R : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nh : WSameSide (map f s) (↑f x) (↑f y)\n⊢ WSameSide s x y", "tactic": "rcases h with ⟨fp₁, hfp₁, fp₂, hfp₂, h⟩" }, { "state_after": "case intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nfp₁ : P'\nhfp₁ : ∃ y, y ∈ s ∧ ↑f y = fp₁\nfp₂ : P'\nhfp₂ : ∃ y, y ∈ s ∧ ↑f y = fp₂\nh : SameRay R (↑f x -ᵥ fp₁) (↑f y -ᵥ fp₂)\n⊢ WSameSide s x y", "state_before": "case intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nfp₁ : P'\nhfp₁ : fp₁ ∈ map f s\nfp₂ : P'\nhfp₂ : fp₂ ∈ map f s\nh : SameRay R (↑f x -ᵥ fp₁) (↑f y -ᵥ fp₂)\n⊢ WSameSide s x y", "tactic": "rw [mem_map] at hfp₁ hfp₂" }, { "state_after": "case intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nfp₂ : P'\nhfp₂ : ∃ y, y ∈ s ∧ ↑f y = fp₂\np₁ : P\nhp₁ : p₁ ∈ s\nh : SameRay R (↑f x -ᵥ ↑f p₁) (↑f y -ᵥ fp₂)\n⊢ WSameSide s x y", "state_before": "case intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nfp₁ : P'\nhfp₁ : ∃ y, y ∈ s ∧ ↑f y = fp₁\nfp₂ : P'\nhfp₂ : ∃ y, y ∈ s ∧ ↑f y = fp₂\nh : SameRay R (↑f x -ᵥ fp₁) (↑f y -ᵥ fp₂)\n⊢ WSameSide s x y", "tactic": "rcases hfp₁ with ⟨p₁, hp₁, rfl⟩" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\np₁ : P\nhp₁ : p₁ ∈ s\np₂ : P\nhp₂ : p₂ ∈ s\nh : SameRay R (↑f x -ᵥ ↑f p₁) (↑f y -ᵥ ↑f p₂)\n⊢ WSameSide s x y", "state_before": "case intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\nfp₂ : P'\nhfp₂ : ∃ y, y ∈ s ∧ ↑f y = fp₂\np₁ : P\nhp₁ : p₁ ∈ s\nh : SameRay R (↑f x -ᵥ ↑f p₁) (↑f y -ᵥ fp₂)\n⊢ WSameSide s x y", "tactic": "rcases hfp₂ with ⟨p₂, hp₂, rfl⟩" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\np₁ : P\nhp₁ : p₁ ∈ s\np₂ : P\nhp₂ : p₂ ∈ s\nh : SameRay R (↑f x -ᵥ ↑f p₁) (↑f y -ᵥ ↑f p₂)\n⊢ SameRay R (x -ᵥ p₁) (y -ᵥ p₂)", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\np₁ : P\nhp₁ : p₁ ∈ s\np₂ : P\nhp₂ : p₂ ∈ s\nh : SameRay R (↑f x -ᵥ ↑f p₁) (↑f y -ᵥ ↑f p₂)\n⊢ WSameSide s x y", "tactic": "refine' ⟨p₁, hp₁, p₂, hp₂, _⟩" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\np₁ : P\nhp₁ : p₁ ∈ s\np₂ : P\nhp₂ : p₂ ∈ s\nh : SameRay R (x -ᵥ p₁) (y -ᵥ p₂)\n⊢ SameRay R (x -ᵥ p₁) (y -ᵥ p₂)", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\np₁ : P\nhp₁ : p₁ ∈ s\np₂ : P\nhp₂ : p₂ ∈ s\nh : SameRay R (↑f x -ᵥ ↑f p₁) (↑f y -ᵥ ↑f p₂)\n⊢ SameRay R (x -ᵥ p₁) (y -ᵥ p₂)", "tactic": "simp_rw [← linearMap_vsub, (f.linear_injective_iff.2 hf).sameRay_map_iff] at h" }, { "state_after": "no goals", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nR : Type u_1\nV : Type u_2\nV' : Type u_4\nP : Type u_3\nP' : Type u_5\ninst✝⁶ : StrictOrderedCommRing R\ninst✝⁵ : AddCommGroup V\ninst✝⁴ : Module R V\ninst✝³ : AddTorsor V P\ninst✝² : AddCommGroup V'\ninst✝¹ : Module R V'\ninst✝ : AddTorsor V' P'\ns : AffineSubspace R P\nx y : P\nf : P →ᵃ[R] P'\nhf : Function.Injective ↑f\np₁ : P\nhp₁ : p₁ ∈ s\np₂ : P\nhp₂ : p₂ ∈ s\nh : SameRay R (x -ᵥ p₁) (y -ᵥ p₂)\n⊢ SameRay R (x -ᵥ p₁) (y -ᵥ p₂)", "tactic": "exact h" } ]
[ 84, 10 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 74, 1 ]
Mathlib/Analysis/SpecialFunctions/Pow/Real.lean
Real.one_lt_rpow_iff
[ { "state_after": "case inl\ny z : ℝ\nhx : 0 ≤ 0\n⊢ 1 < 0 ^ y ↔ 1 < 0 ∧ 0 < y ∨ 0 < 0 ∧ 0 < 1 ∧ y < 0\n\ncase inr\nx y z : ℝ\nhx✝ : 0 ≤ x\nhx : 0 < x\n⊢ 1 < x ^ y ↔ 1 < x ∧ 0 < y ∨ 0 < x ∧ x < 1 ∧ y < 0", "state_before": "x y z : ℝ\nhx : 0 ≤ x\n⊢ 1 < x ^ y ↔ 1 < x ∧ 0 < y ∨ 0 < x ∧ x < 1 ∧ y < 0", "tactic": "rcases hx.eq_or_lt with (rfl | hx)" }, { "state_after": "no goals", "state_before": "case inl\ny z : ℝ\nhx : 0 ≤ 0\n⊢ 1 < 0 ^ y ↔ 1 < 0 ∧ 0 < y ∨ 0 < 0 ∧ 0 < 1 ∧ y < 0", "tactic": "rcases _root_.em (y = 0) with (rfl | hy) <;> simp [*, lt_irrefl, (zero_lt_one' ℝ).not_lt]" }, { "state_after": "no goals", "state_before": "case inr\nx y z : ℝ\nhx✝ : 0 ≤ x\nhx : 0 < x\n⊢ 1 < x ^ y ↔ 1 < x ∧ 0 < y ∨ 0 < x ∧ x < 1 ∧ y < 0", "tactic": "simp [one_lt_rpow_iff_of_pos hx, hx]" } ]
[ 574, 41 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 571, 1 ]
Mathlib/GroupTheory/GroupAction/Defs.lean
AddMonoid.End.smul_def
[]
[ 1133, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1132, 1 ]
Mathlib/Topology/UniformSpace/Basic.lean
Filter.HasBasis.biInter_biUnion_ball
[ { "state_after": "case h\nα : Type ua\nβ : Type ub\nγ : Type uc\nδ : Type ud\nι : Sort u_1\ninst✝ : UniformSpace α\np : ι → Prop\nU : ι → Set (α × α)\nh : HasBasis (𝓤 α) p U\ns : Set α\nx : α\n⊢ (x ∈ ⋂ (i : ι) (_ : p i), ⋃ (x : α) (_ : x ∈ s), ball x (U i)) ↔ x ∈ closure s", "state_before": "α : Type ua\nβ : Type ub\nγ : Type uc\nδ : Type ud\nι : Sort u_1\ninst✝ : UniformSpace α\np : ι → Prop\nU : ι → Set (α × α)\nh : HasBasis (𝓤 α) p U\ns : Set α\n⊢ (⋂ (i : ι) (_ : p i), ⋃ (x : α) (_ : x ∈ s), ball x (U i)) = closure s", "tactic": "ext x" }, { "state_after": "no goals", "state_before": "case h\nα : Type ua\nβ : Type ub\nγ : Type uc\nδ : Type ud\nι : Sort u_1\ninst✝ : UniformSpace α\np : ι → Prop\nU : ι → Set (α × α)\nh : HasBasis (𝓤 α) p U\ns : Set α\nx : α\n⊢ (x ∈ ⋂ (i : ι) (_ : p i), ⋃ (x : α) (_ : x ∈ s), ball x (U i)) ↔ x ∈ closure s", "tactic": "simp [mem_closure_iff_nhds_basis (nhds_basis_uniformity h), ball]" } ]
[ 1079, 68 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1075, 1 ]
src/lean/Init/Data/Nat/Basic.lean
Nat.lt_eq
[]
[ 87, 52 ]
d5348dfac847a56a4595fb6230fd0708dcb4e7e9
https://github.com/leanprover/lean4
[ 87, 9 ]
Mathlib/Data/Fintype/Basic.lean
Set.filter_mem_univ_eq_toFinset
[ { "state_after": "case a\nα : Type u_1\nβ : Type ?u.98777\nγ : Type ?u.98780\ns✝ t : Set α\ninst✝² : Fintype α\ns : Set α\ninst✝¹ : Fintype ↑s\ninst✝ : DecidablePred fun x => x ∈ s\na✝ : α\n⊢ a✝ ∈ filter (fun x => x ∈ s) Finset.univ ↔ a✝ ∈ toFinset s", "state_before": "α : Type u_1\nβ : Type ?u.98777\nγ : Type ?u.98780\ns✝ t : Set α\ninst✝² : Fintype α\ns : Set α\ninst✝¹ : Fintype ↑s\ninst✝ : DecidablePred fun x => x ∈ s\n⊢ filter (fun x => x ∈ s) Finset.univ = toFinset s", "tactic": "ext" }, { "state_after": "no goals", "state_before": "case a\nα : Type u_1\nβ : Type ?u.98777\nγ : Type ?u.98780\ns✝ t : Set α\ninst✝² : Fintype α\ns : Set α\ninst✝¹ : Fintype ↑s\ninst✝ : DecidablePred fun x => x ∈ s\na✝ : α\n⊢ a✝ ∈ filter (fun x => x ∈ s) Finset.univ ↔ a✝ ∈ toFinset s", "tactic": "simp only [Finset.mem_univ, decide_eq_true_eq, forall_true_left, mem_filter,\n true_and, mem_toFinset]" } ]
[ 797, 28 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 793, 1 ]
Mathlib/Data/Multiset/Sort.lean
Multiset.sort_eq
[]
[ 49, 63 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 48, 1 ]
Mathlib/Data/Real/Irrational.lean
Irrational.of_int_mul
[ { "state_after": "no goals", "state_before": "q : ℚ\nx y : ℝ\nm : ℤ\nh : Irrational (↑m * x)\n⊢ Irrational (↑↑m * x)", "tactic": "rwa [cast_coe_int]" } ]
[ 360, 40 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 359, 1 ]
Mathlib/Data/Set/Intervals/OrdConnectedComponent.lean
Set.ordConnectedComponent_ordConnectedProj
[]
[ 125, 77 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 123, 1 ]
Mathlib/Data/Set/Intervals/SurjOn.lean
surjOn_Ioi_of_monotone_surjective
[ { "state_after": "α : Type u_1\nβ : Type u_2\ninst✝¹ : LinearOrder α\ninst✝ : PartialOrder β\nf : α → β\nh_mono : Monotone f\nh_surj : Surjective f\na : α\n⊢ SurjOn f (Iic aᶜ) (Ioi (f a)ᶜᶜ)", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝¹ : LinearOrder α\ninst✝ : PartialOrder β\nf : α → β\nh_mono : Monotone f\nh_surj : Surjective f\na : α\n⊢ SurjOn f (Ioi a) (Ioi (f a))", "tactic": "rw [← compl_Iic, ← compl_compl (Ioi (f a))]" }, { "state_after": "α : Type u_1\nβ : Type u_2\ninst✝¹ : LinearOrder α\ninst✝ : PartialOrder β\nf : α → β\nh_mono : Monotone f\nh_surj : Surjective f\na : α\n⊢ MapsTo f (Iic a) (Ioi (f a)ᶜ)", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝¹ : LinearOrder α\ninst✝ : PartialOrder β\nf : α → β\nh_mono : Monotone f\nh_surj : Surjective f\na : α\n⊢ SurjOn f (Iic aᶜ) (Ioi (f a)ᶜᶜ)", "tactic": "refine' MapsTo.surjOn_compl _ h_surj" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type u_2\ninst✝¹ : LinearOrder α\ninst✝ : PartialOrder β\nf : α → β\nh_mono : Monotone f\nh_surj : Surjective f\na : α\n⊢ MapsTo f (Iic a) (Ioi (f a)ᶜ)", "tactic": "exact fun x hx => (h_mono hx).not_lt" } ]
[ 71, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 67, 1 ]
Mathlib/CategoryTheory/Limits/Shapes/Diagonal.lean
CategoryTheory.Limits.diagonalObjPullbackFstIso_inv_snd_snd
[ { "state_after": "C : Type u_2\ninst✝⁵ : Category C\nX✝ Y✝ Z✝ : C\ninst✝⁴ : HasPullbacks C\nS T : C\nf✝ : X✝ ⟶ T\ng✝ : Y✝ ⟶ T\ni : T ⟶ S\ninst✝³ : HasPullback i i\ninst✝² : HasPullback f✝ g✝\ninst✝¹ : HasPullback (f✝ ≫ i) (g✝ ≫ i)\ninst✝ :\n HasPullback (diagonal i)\n (map (f✝ ≫ i) (g✝ ≫ i) i i f✝ g✝ (𝟙 S) (_ : (f✝ ≫ i) ≫ 𝟙 S = f✝ ≫ i) (_ : (g✝ ≫ i) ≫ 𝟙 S = g✝ ≫ i))\nX Y Z : C\nf : X ⟶ Z\ng : Y ⟶ Z\n⊢ (pullbackRightPullbackFstIso f g fst ≪≫\n congrHom (_ : fst ≫ f = snd ≫ g) (_ : g = g) ≪≫\n pullbackAssoc f g g g ≪≫ pullbackSymmetry f (fst ≫ g) ≪≫ congrHom (_ : fst ≫ g = snd ≫ g) (_ : f = f)).inv ≫\n snd ≫ snd =\n fst ≫ snd", "state_before": "C : Type u_2\ninst✝⁵ : Category C\nX✝ Y✝ Z✝ : C\ninst✝⁴ : HasPullbacks C\nS T : C\nf✝ : X✝ ⟶ T\ng✝ : Y✝ ⟶ T\ni : T ⟶ S\ninst✝³ : HasPullback i i\ninst✝² : HasPullback f✝ g✝\ninst✝¹ : HasPullback (f✝ ≫ i) (g✝ ≫ i)\ninst✝ :\n HasPullback (diagonal i)\n (map (f✝ ≫ i) (g✝ ≫ i) i i f✝ g✝ (𝟙 S) (_ : (f✝ ≫ i) ≫ 𝟙 S = f✝ ≫ i) (_ : (g✝ ≫ i) ≫ 𝟙 S = g✝ ≫ i))\nX Y Z : C\nf : X ⟶ Z\ng : Y ⟶ Z\n⊢ (diagonalObjPullbackFstIso f g).inv ≫ snd ≫ snd = fst ≫ snd", "tactic": "delta diagonalObjPullbackFstIso" }, { "state_after": "no goals", "state_before": "C : Type u_2\ninst✝⁵ : Category C\nX✝ Y✝ Z✝ : C\ninst✝⁴ : HasPullbacks C\nS T : C\nf✝ : X✝ ⟶ T\ng✝ : Y✝ ⟶ T\ni : T ⟶ S\ninst✝³ : HasPullback i i\ninst✝² : HasPullback f✝ g✝\ninst✝¹ : HasPullback (f✝ ≫ i) (g✝ ≫ i)\ninst✝ :\n HasPullback (diagonal i)\n (map (f✝ ≫ i) (g✝ ≫ i) i i f✝ g✝ (𝟙 S) (_ : (f✝ ≫ i) ≫ 𝟙 S = f✝ ≫ i) (_ : (g✝ ≫ i) ≫ 𝟙 S = g✝ ≫ i))\nX Y Z : C\nf : X ⟶ Z\ng : Y ⟶ Z\n⊢ (pullbackRightPullbackFstIso f g fst ≪≫\n congrHom (_ : fst ≫ f = snd ≫ g) (_ : g = g) ≪≫\n pullbackAssoc f g g g ≪≫ pullbackSymmetry f (fst ≫ g) ≪≫ congrHom (_ : fst ≫ g = snd ≫ g) (_ : f = f)).inv ≫\n snd ≫ snd =\n fst ≫ snd", "tactic": "simp" } ]
[ 354, 7 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 350, 1 ]
Mathlib/Algebra/ModEq.lean
AddCommGroup.ModEq.add_iff_right
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : AddCommGroup α\np a a₁ a₂ b b₁ b₂ c : α\nn : ℕ\nz : ℤ\nx✝ : a₂ ≡ b₂ [PMOD p]\nm : ℤ\nhm : b₂ - a₂ = m • p\n⊢ (∃ b, b₁ + b₂ - (a₁ + a₂) = ↑(Equiv.addRight m).symm.symm b • p) ↔ a₁ ≡ b₁ [PMOD p]", "tactic": "simp [add_sub_add_comm, hm, add_smul, ModEq]" } ]
[ 198, 101 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 196, 11 ]
Mathlib/Data/Dfinsupp/Multiset.lean
Multiset.toDfinsupp_singleton
[ { "state_after": "no goals", "state_before": "α : Type u_1\nβ : α → Type ?u.43713\ninst✝ : DecidableEq α\na : α\n⊢ ↑toDfinsupp {a} = Dfinsupp.single a 1", "tactic": "rw [← replicate_one, toDfinsupp_replicate]" } ]
[ 80, 45 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 79, 1 ]
Mathlib/MeasureTheory/Integral/PeakFunction.lean
tendsto_set_integral_pow_smul_of_unique_maximum_of_isCompact_of_measure_nhdsWithin_pos
[ { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "let φ : ℕ → α → ℝ := fun n x => (∫ x in s, c x ^ n ∂μ)⁻¹ * c x ^ n" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "have hnφ : ∀ n, ∀ x ∈ s, 0 ≤ φ n x := by\n intro n x hx\n apply mul_nonneg (inv_nonneg.2 _) (pow_nonneg (hnc x hx) _)\n exact set_integral_nonneg hs.measurableSet fun x hx => pow_nonneg (hnc x hx) _" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "have I : ∀ n, IntegrableOn (fun x => c x ^ n) s μ := fun n =>\n ContinuousOn.integrableOn_compact hs (hc.pow n)" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "have J : ∀ n, 0 ≤ᵐ[μ.restrict s] fun x : α => c x ^ n := by\n intro n\n filter_upwards [ae_restrict_mem hs.measurableSet] with x hx\n exact pow_nonneg (hnc x hx) n" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "have P : ∀ n, (0 : ℝ) < ∫ x in s, c x ^ n ∂μ := by\n intro n\n refine' (set_integral_pos_iff_support_of_nonneg_ae (J n) (I n)).2 _\n obtain ⟨u, u_open, x₀_u, hu⟩ : ∃ u : Set α, IsOpen u ∧ x₀ ∈ u ∧ u ∩ s ⊆ c ⁻¹' Ioi 0 :=\n _root_.continuousOn_iff.1 hc x₀ h₀ (Ioi (0 : ℝ)) isOpen_Ioi hnc₀\n apply (hμ u u_open x₀_u).trans_le\n exact measure_mono fun x hx => ⟨ne_of_gt (pow_pos (a := c x) (hu hx) _), hx.2⟩" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "have hiφ : ∀ n, (∫ x in s, φ n x ∂μ) = 1 := fun n => by\n rw [integral_mul_left, inv_mul_cancel (P n).ne']" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nA : ∀ (u : Set α), IsOpen u → x₀ ∈ u → TendstoUniformlyOn φ 0 atTop (s \\ u)\nthis : Tendsto (fun i => ∫ (x : α) in s, φ i x • g x ∂μ) atTop (𝓝 (g x₀))\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nA : ∀ (u : Set α), IsOpen u → x₀ ∈ u → TendstoUniformlyOn φ 0 atTop (s \\ u)\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "have : Tendsto (fun i : ℕ => ∫ x : α in s, φ i x • g x ∂μ) atTop (𝓝 (g x₀)) :=\n tendsto_set_integral_peak_smul_of_integrableOn_of_continuousWithinAt hs.measurableSet\n hs.measure_lt_top.ne (eventually_of_forall hnφ) A (eventually_of_forall hiφ) hmg hcg" }, { "state_after": "case h.e'_3.h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nA : ∀ (u : Set α), IsOpen u → x₀ ∈ u → TendstoUniformlyOn φ 0 atTop (s \\ u)\nthis : Tendsto (fun i => ∫ (x : α) in s, φ i x • g x ∂μ) atTop (𝓝 (g x₀))\nx✝ : ℕ\n⊢ ((∫ (x : α) in s, c x ^ x✝ ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ x✝ • g x ∂μ) = ∫ (x : α) in s, φ x✝ x • g x ∂μ", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nA : ∀ (u : Set α), IsOpen u → x₀ ∈ u → TendstoUniformlyOn φ 0 atTop (s \\ u)\nthis : Tendsto (fun i => ∫ (x : α) in s, φ i x • g x ∂μ) atTop (𝓝 (g x₀))\n⊢ Tendsto (fun n => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ n • g x ∂μ) atTop (𝓝 (g x₀))", "tactic": "convert this" }, { "state_after": "no goals", "state_before": "case h.e'_3.h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nA : ∀ (u : Set α), IsOpen u → x₀ ∈ u → TendstoUniformlyOn φ 0 atTop (s \\ u)\nthis : Tendsto (fun i => ∫ (x : α) in s, φ i x • g x ∂μ) atTop (𝓝 (g x₀))\nx✝ : ℕ\n⊢ ((∫ (x : α) in s, c x ^ x✝ ∂μ)⁻¹ • ∫ (x : α) in s, c x ^ x✝ • g x ∂μ) = ∫ (x : α) in s, φ x✝ x • g x ∂μ", "tactic": "simp_rw [← smul_smul, integral_smul]" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nn : ℕ\nx : α\nhx : x ∈ s\n⊢ 0 ≤ φ n x", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\n⊢ ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x", "tactic": "intro n x hx" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nn : ℕ\nx : α\nhx : x ∈ s\n⊢ 0 ≤ ∫ (x : α) in s, c x ^ n ∂μ", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nn : ℕ\nx : α\nhx : x ∈ s\n⊢ 0 ≤ φ n x", "tactic": "apply mul_nonneg (inv_nonneg.2 _) (pow_nonneg (hnc x hx) _)" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nn : ℕ\nx : α\nhx : x ∈ s\n⊢ 0 ≤ ∫ (x : α) in s, c x ^ n ∂μ", "tactic": "exact set_integral_nonneg hs.measurableSet fun x hx => pow_nonneg (hnc x hx) _" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nn : ℕ\n⊢ 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\n⊢ ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n", "tactic": "intro n" }, { "state_after": "case h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nn : ℕ\nx : α\nhx : x ∈ s\n⊢ OfNat.ofNat 0 x ≤ c x ^ n", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nn : ℕ\n⊢ 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n", "tactic": "filter_upwards [ae_restrict_mem hs.measurableSet] with x hx" }, { "state_after": "no goals", "state_before": "case h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nn : ℕ\nx : α\nhx : x ∈ s\n⊢ OfNat.ofNat 0 x ≤ c x ^ n", "tactic": "exact pow_nonneg (hnc x hx) n" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\n⊢ 0 < ∫ (x : α) in s, c x ^ n ∂μ", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\n⊢ ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ", "tactic": "intro n" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\n⊢ 0 < ↑↑μ ((Function.support fun x => c x ^ n) ∩ s)", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\n⊢ 0 < ∫ (x : α) in s, c x ^ n ∂μ", "tactic": "refine' (set_integral_pos_iff_support_of_nonneg_ae (J n) (I n)).2 _" }, { "state_after": "case intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\nu : Set α\nu_open : IsOpen u\nx₀_u : x₀ ∈ u\nhu : u ∩ s ⊆ c ⁻¹' Ioi 0\n⊢ 0 < ↑↑μ ((Function.support fun x => c x ^ n) ∩ s)", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\n⊢ 0 < ↑↑μ ((Function.support fun x => c x ^ n) ∩ s)", "tactic": "obtain ⟨u, u_open, x₀_u, hu⟩ : ∃ u : Set α, IsOpen u ∧ x₀ ∈ u ∧ u ∩ s ⊆ c ⁻¹' Ioi 0 :=\n _root_.continuousOn_iff.1 hc x₀ h₀ (Ioi (0 : ℝ)) isOpen_Ioi hnc₀" }, { "state_after": "case intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\nu : Set α\nu_open : IsOpen u\nx₀_u : x₀ ∈ u\nhu : u ∩ s ⊆ c ⁻¹' Ioi 0\n⊢ ↑↑μ (u ∩ s) ≤ ↑↑μ ((Function.support fun x => c x ^ n) ∩ s)", "state_before": "case intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\nu : Set α\nu_open : IsOpen u\nx₀_u : x₀ ∈ u\nhu : u ∩ s ⊆ c ⁻¹' Ioi 0\n⊢ 0 < ↑↑μ ((Function.support fun x => c x ^ n) ∩ s)", "tactic": "apply (hμ u u_open x₀_u).trans_le" }, { "state_after": "no goals", "state_before": "case intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nn : ℕ\nu : Set α\nu_open : IsOpen u\nx₀_u : x₀ ∈ u\nhu : u ∩ s ⊆ c ⁻¹' Ioi 0\n⊢ ↑↑μ (u ∩ s) ≤ ↑↑μ ((Function.support fun x => c x ^ n) ∩ s)", "tactic": "exact measure_mono fun x hx => ⟨ne_of_gt (pow_pos (a := c x) (hu hx) _), hx.2⟩" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nn : ℕ\n⊢ (∫ (x : α) in s, φ n x ∂μ) = 1", "tactic": "rw [integral_mul_left, inv_mul_cancel (P n).ne']" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\n⊢ ∀ (u : Set α), IsOpen u → x₀ ∈ u → TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "intro u u_open x₀u" }, { "state_after": "case intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "state_before": "case intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "obtain ⟨t', tt', t'x₀⟩ : ∃ t', t < t' ∧ t' < c x₀ := exists_between tx₀" }, { "state_after": "case intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "state_before": "case intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "have t'_pos : 0 < t' := t_pos.trans_lt tt'" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "state_before": "case intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "obtain ⟨v, v_open, x₀_v, hv⟩ : ∃ v : Set α, IsOpen v ∧ x₀ ∈ v ∧ v ∩ s ⊆ c ⁻¹' Ioi t' :=\n _root_.continuousOn_iff.1 hc x₀ h₀ (Ioi t') isOpen_Ioi t'x₀" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 ((ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * 0))\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "have N :\n Tendsto (fun n => (μ (v ∩ s)).toReal⁻¹ * (t / t') ^ n) atTop\n (𝓝 ((μ (v ∩ s)).toReal⁻¹ * 0)) := by\n apply Tendsto.mul tendsto_const_nhds _\n apply tendsto_pow_atTop_nhds_0_of_lt_1 (div_nonneg t_pos t'_pos.le)\n exact (div_lt_one t'_pos).2 tt'" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 ((ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * 0))\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "rw [MulZeroClass.mul_zero] at N" }, { "state_after": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\nε : ℝ\nεpos : ε > 0\n⊢ ∀ᶠ (n : ℕ) in atTop, ∀ (x : α), x ∈ s \\ u → dist (OfNat.ofNat 0 x) (φ n x) < ε", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\n⊢ TendstoUniformlyOn φ 0 atTop (s \\ u)", "tactic": "refine' tendstoUniformlyOn_iff.2 fun ε εpos => _" }, { "state_after": "case h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\nε : ℝ\nεpos : ε > 0\nn : ℕ\nhn : (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n < ε\nx : α\nhx : x ∈ s \\ u\n⊢ dist (OfNat.ofNat 0 x) ((∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n) < ε", "state_before": "case intro.intro.intro.intro.intro.intro.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\nε : ℝ\nεpos : ε > 0\n⊢ ∀ᶠ (n : ℕ) in atTop, ∀ (x : α), x ∈ s \\ u → dist (OfNat.ofNat 0 x) (φ n x) < ε", "tactic": "filter_upwards [(tendsto_order.1 N).2 ε εpos] with n hn x hx" }, { "state_after": "case h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\nε : ℝ\nεpos : ε > 0\nn : ℕ\nhn : (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n < ε\nx : α\nhx : x ∈ s \\ u\n⊢ (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n < ε", "state_before": "case h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\nε : ℝ\nεpos : ε > 0\nn : ℕ\nhn : (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n < ε\nx : α\nhx : x ∈ s \\ u\n⊢ dist (OfNat.ofNat 0 x) ((∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n) < ε", "tactic": "simp only [Pi.zero_apply, dist_zero_left, Real.norm_of_nonneg (hnφ n x hx.1)]" }, { "state_after": "no goals", "state_before": "case h\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\nN : Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 0)\nε : ℝ\nεpos : ε > 0\nn : ℕ\nhn : (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n < ε\nx : α\nhx : x ∈ s \\ u\n⊢ (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n < ε", "tactic": "exact (M n x hx).trans_lt hn" }, { "state_after": "case inl\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : s \\ u = ∅\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t\n\ncase inr\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : Set.Nonempty (s \\ u)\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t", "tactic": "rcases eq_empty_or_nonempty (s \\ u) with (h | h)" }, { "state_after": "case inr.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : Set.Nonempty (s \\ u)\nx : α\nhx : x ∈ s \\ u\nh'x : ∀ (y : α), y ∈ s \\ u → c y ≤ c x\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t", "state_before": "case inr\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : Set.Nonempty (s \\ u)\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t", "tactic": "obtain ⟨x, hx, h'x⟩ : ∃ x ∈ s \\ u, ∀ y ∈ s \\ u, c y ≤ c x :=\n IsCompact.exists_isMaxOn (hs.diff u_open) h (hc.mono (diff_subset _ _))" }, { "state_after": "case inr.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : Set.Nonempty (s \\ u)\nx : α\nhx : x ∈ s \\ u\nh'x : ∀ (y : α), y ∈ s \\ u → c y ≤ c x\n⊢ x ≠ x₀", "state_before": "case inr.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : Set.Nonempty (s \\ u)\nx : α\nhx : x ∈ s \\ u\nh'x : ∀ (y : α), y ∈ s \\ u → c y ≤ c x\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t", "tactic": "refine' ⟨c x, hnc x hx.1, h'c x hx.1 _, h'x⟩" }, { "state_after": "case inr.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nc : α → ℝ\nhc : ContinuousOn c s\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhmg : IntegrableOn g s\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nh : Set.Nonempty (s \\ u)\nx : α\nhx : x ∈ s \\ u\nh'x : ∀ (y : α), y ∈ s \\ u → c y ≤ c x\nhμ : ∀ (u : Set α), IsOpen u → x ∈ u → 0 < ↑↑μ (u ∩ s)\nh'c : ∀ (y : α), y ∈ s → y ≠ x → c y < c x\nhnc₀ : 0 < c x\nh₀ : x ∈ s\nhcg : ContinuousWithinAt g s x\nx₀u : x ∈ u\n⊢ False", "state_before": "case inr.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : Set.Nonempty (s \\ u)\nx : α\nhx : x ∈ s \\ u\nh'x : ∀ (y : α), y ∈ s \\ u → c y ≤ c x\n⊢ x ≠ x₀", "tactic": "rintro rfl" }, { "state_after": "no goals", "state_before": "case inr.intro.intro\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nc : α → ℝ\nhc : ContinuousOn c s\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhmg : IntegrableOn g s\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nh : Set.Nonempty (s \\ u)\nx : α\nhx : x ∈ s \\ u\nh'x : ∀ (y : α), y ∈ s \\ u → c y ≤ c x\nhμ : ∀ (u : Set α), IsOpen u → x ∈ u → 0 < ↑↑μ (u ∩ s)\nh'c : ∀ (y : α), y ∈ s → y ≠ x → c y < c x\nhnc₀ : 0 < c x\nh₀ : x ∈ s\nhcg : ContinuousWithinAt g s x\nx₀u : x ∈ u\n⊢ False", "tactic": "exact hx.2 x₀u" }, { "state_after": "no goals", "state_before": "case inl\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : s \\ u = ∅\n⊢ ∃ t, 0 ≤ t ∧ t < c x₀ ∧ ∀ (x : α), x ∈ s \\ u → c x ≤ t", "tactic": "exact\n ⟨0, le_rfl, hnc₀, by simp only [h, mem_empty_iff_false, IsEmpty.forall_iff, imp_true_iff]⟩" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nh : s \\ u = ∅\n⊢ ∀ (x : α), x ∈ s \\ u → c x ≤ 0", "tactic": "simp only [h, mem_empty_iff_false, IsEmpty.forall_iff, imp_true_iff]" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\n⊢ ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n", "tactic": "intro n x hx" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ (c x ^ n / ∫ (x : α) in s, c x ^ n ∂μ) ≤ t ^ n / (t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n", "tactic": "simp_rw [← div_eq_inv_mul, div_pow, div_div]" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ c x ^ n ≤ t ^ n\n\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ 0 < t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s))", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ (c x ^ n / ∫ (x : α) in s, c x ^ n ∂μ) ≤ t ^ n / (t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)))", "tactic": "apply div_le_div (pow_nonneg t_pos n) _ _ B" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) = ∫ (x : α) in v ∩ s, t' ^ n ∂μ", "tactic": "simp only [integral_const, Measure.restrict_apply, MeasurableSet.univ, univ_inter,\n Algebra.id.smul_eq_mul, mul_comm]" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ IntegrableOn (fun a => t' ^ n) (v ∩ s)\n\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ IntegrableOn (fun a => c a ^ n) (v ∩ s)\n\nα : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ ∀ (x : α), x ∈ v ∩ s → t' ^ n ≤ c x ^ n", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ (∫ (x : α) in v ∩ s, t' ^ n ∂μ) ≤ ∫ (y : α) in v ∩ s, c y ^ n ∂μ", "tactic": "apply set_integral_mono_on _ _ (v_open.measurableSet.inter hs.measurableSet) _" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ ↑↑μ (v ∩ s) < ⊤", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ IntegrableOn (fun a => t' ^ n) (v ∩ s)", "tactic": "apply integrableOn_const.2 (Or.inr _)" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ ↑↑μ (v ∩ s) < ⊤", "tactic": "exact lt_of_le_of_lt (measure_mono (inter_subset_right _ _)) hs.measure_lt_top" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ IntegrableOn (fun a => c a ^ n) (v ∩ s)", "tactic": "exact (I n).mono (inter_subset_right _ _) le_rfl" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx✝ : α\nhx✝ : x✝ ∈ s \\ u\nx : α\nhx : x ∈ v ∩ s\n⊢ t' ^ n ≤ c x ^ n", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\n⊢ ∀ (x : α), x ∈ v ∩ s → t' ^ n ≤ c x ^ n", "tactic": "intro x hx" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx✝ : α\nhx✝ : x✝ ∈ s \\ u\nx : α\nhx : x ∈ v ∩ s\n⊢ t' ^ n ≤ c x ^ n", "tactic": "exact pow_le_pow_of_le_left t'_pos.le (le_of_lt (hv hx)) _" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ c x ^ n ≤ t ^ n", "tactic": "exact pow_le_pow_of_le_left (hnc _ hx.1) (ht x hx) _" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ ↑↑μ (v ∩ s) ≠ ⊤", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ 0 < t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s))", "tactic": "apply mul_pos (pow_pos (t_pos.trans_lt tt') _) (ENNReal.toReal_pos (hμ v v_open x₀_v).ne' _)" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\nthis : ↑↑μ (v ∩ s) ≤ ↑↑μ s\n⊢ ↑↑μ (v ∩ s) ≠ ⊤", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\n⊢ ↑↑μ (v ∩ s) ≠ ⊤", "tactic": "have : μ (v ∩ s) ≤ μ s := measure_mono (inter_subset_right _ _)" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nn : ℕ\nx : α\nhx : x ∈ s \\ u\nB : t' ^ n * ENNReal.toReal (↑↑μ (v ∩ s)) ≤ ∫ (y : α) in s, c y ^ n ∂μ\nthis : ↑↑μ (v ∩ s) ≤ ↑↑μ s\n⊢ ↑↑μ (v ∩ s) ≠ ⊤", "tactic": "exact ne_of_lt (lt_of_le_of_lt this hs.measure_lt_top)" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\n⊢ Tendsto (fun x => (t / t') ^ x) atTop (𝓝 0)", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\n⊢ Tendsto (fun n => (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n) atTop (𝓝 ((ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * 0))", "tactic": "apply Tendsto.mul tendsto_const_nhds _" }, { "state_after": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\n⊢ t / t' < 1", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\n⊢ Tendsto (fun x => (t / t') ^ x) atTop (𝓝 0)", "tactic": "apply tendsto_pow_atTop_nhds_0_of_lt_1 (div_nonneg t_pos t'_pos.le)" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type u_2\nι : Type ?u.628948\nhm : MeasurableSpace α\nμ : MeasureTheory.Measure α\ninst✝⁶ : TopologicalSpace α\ninst✝⁵ : BorelSpace α\ninst✝⁴ : NormedAddCommGroup E\ninst✝³ : NormedSpace ℝ E\ng : α → E\nl : Filter ι\nx₀ : α\ns : Set α\nφ✝ : ι → α → ℝ\ninst✝² : CompleteSpace E\ninst✝¹ : MetrizableSpace α\ninst✝ : IsLocallyFiniteMeasure μ\nhs : IsCompact s\nhμ : ∀ (u : Set α), IsOpen u → x₀ ∈ u → 0 < ↑↑μ (u ∩ s)\nc : α → ℝ\nhc : ContinuousOn c s\nh'c : ∀ (y : α), y ∈ s → y ≠ x₀ → c y < c x₀\nhnc : ∀ (x : α), x ∈ s → 0 ≤ c x\nhnc₀ : 0 < c x₀\nh₀ : x₀ ∈ s\nhmg : IntegrableOn g s\nhcg : ContinuousWithinAt g s x₀\nφ : ℕ → α → ℝ := fun n x => (∫ (x : α) in s, c x ^ n ∂μ)⁻¹ * c x ^ n\nhnφ : ∀ (n : ℕ) (x : α), x ∈ s → 0 ≤ φ n x\nI : ∀ (n : ℕ), IntegrableOn (fun x => c x ^ n) s\nJ : ∀ (n : ℕ), 0 ≤ᶠ[ae (Measure.restrict μ s)] fun x => c x ^ n\nP : ∀ (n : ℕ), 0 < ∫ (x : α) in s, c x ^ n ∂μ\nhiφ : ∀ (n : ℕ), (∫ (x : α) in s, φ n x ∂μ) = 1\nu : Set α\nu_open : IsOpen u\nx₀u : x₀ ∈ u\nt : ℝ\nt_pos : 0 ≤ t\ntx₀ : t < c x₀\nht : ∀ (x : α), x ∈ s \\ u → c x ≤ t\nt' : ℝ\ntt' : t < t'\nt'x₀ : t' < c x₀\nt'_pos : 0 < t'\nv : Set α\nv_open : IsOpen v\nx₀_v : x₀ ∈ v\nhv : v ∩ s ⊆ c ⁻¹' Ioi t'\nM : ∀ (n : ℕ) (x : α), x ∈ s \\ u → φ n x ≤ (ENNReal.toReal (↑↑μ (v ∩ s)))⁻¹ * (t / t') ^ n\n⊢ t / t' < 1", "tactic": "exact (div_lt_one t'_pos).2 tt'" } ]
[ 285, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 198, 1 ]
Mathlib/Algebra/Order/Hom/Basic.lean
map_eq_zero_iff_eq_one
[ { "state_after": "ι : Type ?u.52007\nF : Type u_2\nα : Type u_3\nβ : Type u_1\nγ : Type ?u.52019\nδ : Type ?u.52022\ninst✝² : Group α\ninst✝¹ : OrderedAddCommMonoid β\ninst✝ : GroupNormClass F α β\nf : F\n⊢ ↑f 1 = 0", "state_before": "ι : Type ?u.52007\nF : Type u_2\nα : Type u_3\nβ : Type u_1\nγ : Type ?u.52019\nδ : Type ?u.52022\ninst✝² : Group α\ninst✝¹ : OrderedAddCommMonoid β\ninst✝ : GroupNormClass F α β\nf : F\nx : α\n⊢ x = 1 → ↑f x = 0", "tactic": "rintro rfl" }, { "state_after": "no goals", "state_before": "ι : Type ?u.52007\nF : Type u_2\nα : Type u_3\nβ : Type u_1\nγ : Type ?u.52019\nδ : Type ?u.52022\ninst✝² : Group α\ninst✝¹ : OrderedAddCommMonoid β\ninst✝ : GroupNormClass F α β\nf : F\n⊢ ↑f 1 = 0", "tactic": "exact map_one_eq_zero _" } ]
[ 296, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 293, 1 ]
Mathlib/ModelTheory/FinitelyGenerated.lean
FirstOrder.Language.Substructure.cg_closure
[]
[ 146, 15 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 145, 1 ]
Mathlib/Topology/MetricSpace/Infsep.lean
Finset.coe_infsep_of_offDiag_empty
[ { "state_after": "α : Type u_1\nβ : Type ?u.77060\ninst✝¹ : PseudoMetricSpace α\nx y z : α\ns✝ t : Set α\ninst✝ : DecidableEq α\ns : Finset α\nhs : ¬Finset.Nonempty (Finset.offDiag s)\n⊢ infsep ↑s = 0", "state_before": "α : Type u_1\nβ : Type ?u.77060\ninst✝¹ : PseudoMetricSpace α\nx y z : α\ns✝ t : Set α\ninst✝ : DecidableEq α\ns : Finset α\nhs : Finset.offDiag s = ∅\n⊢ infsep ↑s = 0", "tactic": "rw [← Finset.not_nonempty_iff_eq_empty] at hs" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type ?u.77060\ninst✝¹ : PseudoMetricSpace α\nx y z : α\ns✝ t : Set α\ninst✝ : DecidableEq α\ns : Finset α\nhs : ¬Finset.Nonempty (Finset.offDiag s)\n⊢ infsep ↑s = 0", "tactic": "rw [Finset.coe_infsep, dif_neg hs]" } ]
[ 517, 37 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 514, 1 ]
Mathlib/Algebra/Quaternion.lean
QuaternionAlgebra.eq_re_iff_mem_range_coe
[]
[ 688, 66 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 686, 1 ]
Mathlib/LinearAlgebra/Matrix/Charpoly/Basic.lean
charmatrix_apply_eq
[ { "state_after": "no goals", "state_before": "R : Type u\ninst✝² : CommRing R\nn : Type w\ninst✝¹ : DecidableEq n\ninst✝ : Fintype n\nM : Matrix n n R\ni : n\n⊢ charmatrix M i i = X - ↑C (M i i)", "tactic": "simp only [charmatrix, RingHom.mapMatrix_apply, sub_apply, scalar_apply_eq, map_apply]" } ]
[ 62, 89 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 60, 1 ]
Mathlib/Data/Real/EReal.lean
EReal.bot_sub
[]
[ 841, 12 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 840, 1 ]
Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean
MeasureTheory.integral_Ioi_of_hasDerivAt_of_nonpos'
[]
[ 793, 7 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 790, 1 ]
Mathlib/Init/Algebra/Order.lean
le_antisymm_iff
[]
[ 197, 78 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 196, 1 ]
Mathlib/Analysis/BoxIntegral/Partition/Basic.lean
BoxIntegral.Prepartition.filter_of_true
[ { "state_after": "case h\nι : Type u_1\nI J✝ J₁ J₂ : Box ι\nπ π₁ π₂ : Prepartition I\nx : ι → ℝ\nπi πi₁ πi₂ : (J : Box ι) → Prepartition J\np : Box ι → Prop\nhp : ∀ (J : Box ι), J ∈ π → p J\nJ : Box ι\n⊢ J ∈ filter π p ↔ J ∈ π", "state_before": "ι : Type u_1\nI J J₁ J₂ : Box ι\nπ π₁ π₂ : Prepartition I\nx : ι → ℝ\nπi πi₁ πi₂ : (J : Box ι) → Prepartition J\np : Box ι → Prop\nhp : ∀ (J : Box ι), J ∈ π → p J\n⊢ filter π p = π", "tactic": "ext J" }, { "state_after": "no goals", "state_before": "case h\nι : Type u_1\nI J✝ J₁ J₂ : Box ι\nπ π₁ π₂ : Prepartition I\nx : ι → ℝ\nπi πi₁ πi₂ : (J : Box ι) → Prepartition J\np : Box ι → Prop\nhp : ∀ (J : Box ι), J ∈ π → p J\nJ : Box ι\n⊢ J ∈ filter π p ↔ J ∈ π", "tactic": "simpa using hp J" } ]
[ 612, 19 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 610, 1 ]
Mathlib/NumberTheory/Padics/PadicIntegers.lean
PadicInt.pow_p_dvd_int_iff
[ { "state_after": "no goals", "state_before": "p : ℕ\nhp : Fact (Nat.Prime p)\nn : ℕ\na : ℤ\n⊢ ↑p ^ n ∣ ↑a ↔ ↑(p ^ n) ∣ a", "tactic": "rw [← Nat.cast_pow, ← norm_int_le_pow_iff_dvd, norm_le_pow_iff_mem_span_pow,\n Ideal.mem_span_singleton, Nat.cast_pow]" } ]
[ 581, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 579, 1 ]
Mathlib/Logic/Basic.lean
forall_apply_eq_imp_iff
[ { "state_after": "no goals", "state_before": "ι : Sort ?u.18610\nα : Sort ?u.18615\nκ : ι → Sort ?u.18612\np✝ q : α → Prop\nβ : Sort u_1\nf : α → β\np : β → Prop\n⊢ (∀ (a : α) (b : β), f a = b → p b) ↔ ∀ (a : α), p (f a)", "tactic": "simp" } ]
[ 803, 53 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 802, 1 ]
Mathlib/Algebra/Module/LocalizedModule.lean
LocalizedModule.add_smul'
[ { "state_after": "case H\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\ny : Localization S\nz : LocalizedModule S M\ndatax : R × { x // x ∈ S }\n⊢ (Localization.mk datax.fst datax.snd + y) • z = Localization.mk datax.fst datax.snd • z + y • z", "state_before": "R : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nx y : Localization S\nz : LocalizedModule S M\n⊢ (x + y) • z = x • z + y • z", "tactic": "induction' x using Localization.induction_on with datax" }, { "state_after": "case H.H\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nz : LocalizedModule S M\ndatax datay : R × { x // x ∈ S }\n⊢ (Localization.mk datax.fst datax.snd + Localization.mk datay.fst datay.snd) • z =\n Localization.mk datax.fst datax.snd • z + Localization.mk datay.fst datay.snd • z", "state_before": "case H\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\ny : Localization S\nz : LocalizedModule S M\ndatax : R × { x // x ∈ S }\n⊢ (Localization.mk datax.fst datax.snd + y) • z = Localization.mk datax.fst datax.snd • z + y • z", "tactic": "induction' y using Localization.induction_on with datay" }, { "state_after": "case H.H.h\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\ndatax datay : R × { x // x ∈ S }\nm : M\nt : { x // x ∈ S }\n⊢ (Localization.mk datax.fst datax.snd + Localization.mk datay.fst datay.snd) • mk m t =\n Localization.mk datax.fst datax.snd • mk m t + Localization.mk datay.fst datay.snd • mk m t", "state_before": "case H.H\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nz : LocalizedModule S M\ndatax datay : R × { x // x ∈ S }\n⊢ (Localization.mk datax.fst datax.snd + Localization.mk datay.fst datay.snd) • z =\n Localization.mk datax.fst datax.snd • z + Localization.mk datay.fst datay.snd • z", "tactic": "induction' z using LocalizedModule.induction_on with m t" }, { "state_after": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ (Localization.mk (r, s).fst (r, s).snd + Localization.mk (r', s').fst (r', s').snd) • mk m t =\n Localization.mk (r, s).fst (r, s).snd • mk m t + Localization.mk (r', s').fst (r', s').snd • mk m t", "state_before": "case H.H.h\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\ndatax datay : R × { x // x ∈ S }\nm : M\nt : { x // x ∈ S }\n⊢ (Localization.mk datax.fst datax.snd + Localization.mk datay.fst datay.snd) • mk m t =\n Localization.mk datax.fst datax.snd • mk m t + Localization.mk datay.fst datay.snd • mk m t", "tactic": "rcases datax, datay with ⟨⟨r, s⟩, ⟨r', s'⟩⟩" }, { "state_after": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ ∃ u,\n u • ((r, s).snd * t * ((r', s').snd * t)) • (↑(r, s).snd * (r', s').fst + ↑(r', s').snd * (r, s).fst) • m =\n u • ((r, s).snd * (r', s').snd * t) • (((r', s').snd * t) • (r, s).fst • m + ((r, s).snd * t) • (r', s').fst • m)", "state_before": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ (Localization.mk (r, s).fst (r, s).snd + Localization.mk (r', s').fst (r', s').snd) • mk m t =\n Localization.mk (r, s).fst (r, s).snd • mk m t + Localization.mk (r', s').fst (r', s').snd • mk m t", "tactic": "rw [Localization.add_mk, mk_smul_mk, mk_smul_mk, mk_smul_mk, mk_add_mk, mk_eq]" }, { "state_after": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ 1 • ((r, s).snd * t * ((r', s').snd * t)) • (↑(r, s).snd * (r', s').fst + ↑(r', s').snd * (r, s).fst) • m =\n 1 • ((r, s).snd * (r', s').snd * t) • (((r', s').snd * t) • (r, s).fst • m + ((r, s).snd * t) • (r', s').fst • m)", "state_before": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ ∃ u,\n u • ((r, s).snd * t * ((r', s').snd * t)) • (↑(r, s).snd * (r', s').fst + ↑(r', s').snd * (r, s).fst) • m =\n u • ((r, s).snd * (r', s').snd * t) • (((r', s').snd * t) • (r, s).fst • m + ((r, s).snd * t) • (r', s').fst • m)", "tactic": "use 1" }, { "state_after": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ (↑s * ↑t * (↑s' * ↑t) * (↑s * r')) • m + (↑s * ↑t * (↑s' * ↑t) * (↑s' * r)) • m =\n (↑s * ↑s' * ↑t * (↑s' * ↑t * r)) • m + (↑s * ↑s' * ↑t * (↑s * ↑t * r')) • m", "state_before": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ 1 • ((r, s).snd * t * ((r', s').snd * t)) • (↑(r, s).snd * (r', s').fst + ↑(r', s').snd * (r, s).fst) • m =\n 1 • ((r, s).snd * (r', s').snd * t) • (((r', s').snd * t) • (r, s).fst • m + ((r, s).snd * t) • (r', s').fst • m)", "tactic": "simp only [one_smul, add_smul, smul_add, ← mul_smul, Submonoid.smul_def, Submonoid.coe_mul,\n Submonoid.coe_one]" }, { "state_after": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ (↑s * ↑t * (↑s' * ↑t) * (↑s' * r)) • m + (↑s * ↑t * (↑s' * ↑t) * (↑s * r')) • m =\n (↑s * ↑s' * ↑t * (↑s' * ↑t * r)) • m + (↑s * ↑s' * ↑t * (↑s * ↑t * r')) • m", "state_before": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ (↑s * ↑t * (↑s' * ↑t) * (↑s * r')) • m + (↑s * ↑t * (↑s' * ↑t) * (↑s' * r)) • m =\n (↑s * ↑s' * ↑t * (↑s' * ↑t * r)) • m + (↑s * ↑s' * ↑t * (↑s * ↑t * r')) • m", "tactic": "rw [add_comm]" }, { "state_after": "no goals", "state_before": "case H.H.h.mk.mk\nR : Type u\ninst✝² : CommSemiring R\nS : Submonoid R\nM : Type v\ninst✝¹ : AddCommMonoid M\ninst✝ : Module R M\nm : M\nt : { x // x ∈ S }\nr : R\ns : { x // x ∈ S }\nr' : R\ns' : { x // x ∈ S }\n⊢ (↑s * ↑t * (↑s' * ↑t) * (↑s' * r)) • m + (↑s * ↑t * (↑s' * ↑t) * (↑s * r')) • m =\n (↑s * ↑s' * ↑t * (↑s' * ↑t * r)) • m + (↑s * ↑s' * ↑t * (↑s * ↑t * r')) • m", "tactic": "ring_nf" } ]
[ 381, 10 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 369, 9 ]
Mathlib/RingTheory/Subring/Basic.lean
Subring.sInf_toAddSubgroup
[]
[ 753, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 751, 1 ]
Mathlib/Data/Set/Basic.lean
Set.mem_insert
[]
[ 1113, 13 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1112, 1 ]
Mathlib/Data/Polynomial/Div.lean
Polynomial.div_wf_lemma
[ { "state_after": "R : Type u\nS : Type v\nT : Type w\nA : Type z\na b : R\nn : ℕ\ninst✝ : Ring R\np q : R[X]\nh : degree q ≤ degree p ∧ p ≠ 0\nhq : Monic q\nhp : leadingCoeff p ≠ 0\nhq0 : q ≠ 0\n⊢ degree q ≤ degree p", "state_before": "R : Type u\nS : Type v\nT : Type w\nA : Type z\na b : R\nn : ℕ\ninst✝ : Ring R\np q : R[X]\nh : degree q ≤ degree p ∧ p ≠ 0\nhq : Monic q\nhp : leadingCoeff p ≠ 0\nhq0 : q ≠ 0\n⊢ ↑(natDegree q) ≤ ↑(natDegree p)", "tactic": "rw [← Nat.cast_withBot, ← Nat.cast_withBot, ← degree_eq_natDegree h.2,\n← degree_eq_natDegree hq0]" }, { "state_after": "no goals", "state_before": "R : Type u\nS : Type v\nT : Type w\nA : Type z\na b : R\nn : ℕ\ninst✝ : Ring R\np q : R[X]\nh : degree q ≤ degree p ∧ p ≠ 0\nhq : Monic q\nhp : leadingCoeff p ≠ 0\nhq0 : q ≠ 0\n⊢ degree q ≤ degree p", "tactic": "exact h.1" }, { "state_after": "no goals", "state_before": "R : Type u\nS : Type v\nT : Type w\nA : Type z\na b : R\nn : ℕ\ninst✝ : Ring R\np q : R[X]\nh : degree q ≤ degree p ∧ p ≠ 0\nhq : Monic q\nhp : leadingCoeff p ≠ 0\nhq0 : q ≠ 0\nhlt : natDegree q ≤ natDegree p\n⊢ degree p = degree (↑C (leadingCoeff p) * X ^ (natDegree p - natDegree q) * q)", "tactic": "rw [hq.degree_mul, degree_C_mul_X_pow _ hp, degree_eq_natDegree h.2,\n degree_eq_natDegree hq0, ← Nat.cast_add, tsub_add_cancel_of_le hlt]" }, { "state_after": "no goals", "state_before": "R : Type u\nS : Type v\nT : Type w\nA : Type z\na b : R\nn : ℕ\ninst✝ : Ring R\np q : R[X]\nh : degree q ≤ degree p ∧ p ≠ 0\nhq : Monic q\nhp : leadingCoeff p ≠ 0\nhq0 : q ≠ 0\nhlt : natDegree q ≤ natDegree p\n⊢ leadingCoeff p = leadingCoeff (↑C (leadingCoeff p) * X ^ (natDegree p - natDegree q) * q)", "tactic": "rw [leadingCoeff_mul_monic hq, leadingCoeff_mul_X_pow, leadingCoeff_C]" } ]
[ 111, 84 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 99, 1 ]
Mathlib/Algebra/Module/Bimodule.lean
Subbimodule.smul_mem
[ { "state_after": "R : Type u_4\nA : Type u_2\nB : Type u_1\nM : Type u_3\ninst✝¹¹ : CommSemiring R\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : Module R M\ninst✝⁸ : Semiring A\ninst✝⁷ : Semiring B\ninst✝⁶ : Module A M\ninst✝⁵ : Module B M\ninst✝⁴ : Algebra R A\ninst✝³ : Algebra R B\ninst✝² : IsScalarTower R A M\ninst✝¹ : IsScalarTower R B M\ninst✝ : SMulCommClass A B M\np : Submodule (A ⊗[R] B) M\na : A\nm : M\nhm : m ∈ p\n⊢ a • m = a ⊗ₜ[R] 1 • m", "state_before": "R : Type u_4\nA : Type u_2\nB : Type u_1\nM : Type u_3\ninst✝¹¹ : CommSemiring R\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : Module R M\ninst✝⁸ : Semiring A\ninst✝⁷ : Semiring B\ninst✝⁶ : Module A M\ninst✝⁵ : Module B M\ninst✝⁴ : Algebra R A\ninst✝³ : Algebra R B\ninst✝² : IsScalarTower R A M\ninst✝¹ : IsScalarTower R B M\ninst✝ : SMulCommClass A B M\np : Submodule (A ⊗[R] B) M\na : A\nm : M\nhm : m ∈ p\n⊢ a • m ∈ p", "tactic": "suffices a • m = a ⊗ₜ[R] (1 : B) • m by exact this.symm ▸ p.smul_mem _ hm" }, { "state_after": "no goals", "state_before": "R : Type u_4\nA : Type u_2\nB : Type u_1\nM : Type u_3\ninst✝¹¹ : CommSemiring R\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : Module R M\ninst✝⁸ : Semiring A\ninst✝⁷ : Semiring B\ninst✝⁶ : Module A M\ninst✝⁵ : Module B M\ninst✝⁴ : Algebra R A\ninst✝³ : Algebra R B\ninst✝² : IsScalarTower R A M\ninst✝¹ : IsScalarTower R B M\ninst✝ : SMulCommClass A B M\np : Submodule (A ⊗[R] B) M\na : A\nm : M\nhm : m ∈ p\n⊢ a • m = a ⊗ₜ[R] 1 • m", "tactic": "simp [TensorProduct.Algebra.smul_def]" }, { "state_after": "no goals", "state_before": "R : Type u_4\nA : Type u_2\nB : Type u_1\nM : Type u_3\ninst✝¹¹ : CommSemiring R\ninst✝¹⁰ : AddCommMonoid M\ninst✝⁹ : Module R M\ninst✝⁸ : Semiring A\ninst✝⁷ : Semiring B\ninst✝⁶ : Module A M\ninst✝⁵ : Module B M\ninst✝⁴ : Algebra R A\ninst✝³ : Algebra R B\ninst✝² : IsScalarTower R A M\ninst✝¹ : IsScalarTower R B M\ninst✝ : SMulCommClass A B M\np : Submodule (A ⊗[R] B) M\na : A\nm : M\nhm : m ∈ p\nthis : a • m = a ⊗ₜ[R] 1 • m\n⊢ a • m ∈ p", "tactic": "exact this.symm ▸ p.smul_mem _ hm" } ]
[ 100, 40 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 98, 1 ]
Mathlib/SetTheory/Ordinal/FixedPoint.lean
Ordinal.derivFamily_eq_enumOrd
[ { "state_after": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ StrictMono (derivFamily f) ∧ Set.range (derivFamily f) = ⋂ (i : ι), fixedPoints (f i)", "state_before": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ derivFamily f = enumOrd (⋂ (i : ι), fixedPoints (f i))", "tactic": "rw [← eq_enumOrd _ (fp_family_unbounded.{u, v} H)]" }, { "state_after": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ Set.range (derivFamily f) = ⋂ (i : ι), fixedPoints (f i)", "state_before": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ StrictMono (derivFamily f) ∧ Set.range (derivFamily f) = ⋂ (i : ι), fixedPoints (f i)", "tactic": "use (derivFamily_isNormal f).strictMono" }, { "state_after": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ (∀ (a : Ordinal), derivFamily f a ∈ ⋂ (i : ι), fixedPoints (f i)) ∧\n ∀ (b : Ordinal), (b ∈ ⋂ (i : ι), fixedPoints (f i)) → ∃ a, derivFamily f a = b", "state_before": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ Set.range (derivFamily f) = ⋂ (i : ι), fixedPoints (f i)", "tactic": "rw [Set.range_eq_iff]" }, { "state_after": "case refine'_1\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ ∀ (a : Ordinal), derivFamily f a ∈ ⋂ (i : ι), fixedPoints (f i)\n\ncase refine'_2\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nha : a ∈ ⋂ (i : ι), fixedPoints (f i)\n⊢ ∃ a_1, derivFamily f a_1 = a", "state_before": "ι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ (∀ (a : Ordinal), derivFamily f a ∈ ⋂ (i : ι), fixedPoints (f i)) ∧\n ∀ (b : Ordinal), (b ∈ ⋂ (i : ι), fixedPoints (f i)) → ∃ a, derivFamily f a = b", "tactic": "refine' ⟨_, fun a ha => _⟩" }, { "state_after": "case refine'_2\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nha : ∀ (i : ι), a ∈ fixedPoints (f i)\n⊢ ∃ a_1, derivFamily f a_1 = a", "state_before": "case refine'_2\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nha : a ∈ ⋂ (i : ι), fixedPoints (f i)\n⊢ ∃ a_1, derivFamily f a_1 = a", "tactic": "rw [Set.mem_iInter] at ha" }, { "state_after": "no goals", "state_before": "case refine'_2\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nha : ∀ (i : ι), a ∈ fixedPoints (f i)\n⊢ ∃ a_1, derivFamily f a_1 = a", "tactic": "rwa [← fp_iff_derivFamily H]" }, { "state_after": "case refine'_1.intro\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nS : Set Ordinal\ni : ι\nhi : (fun i => fixedPoints (f i)) i = S\n⊢ derivFamily f a ∈ S", "state_before": "case refine'_1\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\n⊢ ∀ (a : Ordinal), derivFamily f a ∈ ⋂ (i : ι), fixedPoints (f i)", "tactic": "rintro a S ⟨i, hi⟩" }, { "state_after": "case refine'_1.intro\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nS : Set Ordinal\ni : ι\nhi : (fun i => fixedPoints (f i)) i = S\n⊢ derivFamily f a ∈ (fun i => fixedPoints (f i)) i", "state_before": "case refine'_1.intro\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nS : Set Ordinal\ni : ι\nhi : (fun i => fixedPoints (f i)) i = S\n⊢ derivFamily f a ∈ S", "tactic": "rw [← hi]" }, { "state_after": "no goals", "state_before": "case refine'_1.intro\nι : Type u\nf : ι → Ordinal → Ordinal\nH : ∀ (i : ι), IsNormal (f i)\na : Ordinal\nS : Set Ordinal\ni : ι\nhi : (fun i => fixedPoints (f i)) i = S\n⊢ derivFamily f a ∈ (fun i => fixedPoints (f i)) i", "tactic": "exact derivFamily_fp (H i) a" } ]
[ 242, 31 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 232, 1 ]
Mathlib/Data/Set/Pointwise/Interval.lean
Set.image_mul_left_Ioo
[ { "state_after": "no goals", "state_before": "α : Type u_1\ninst✝ : LinearOrderedField α\na✝ a : α\nh : 0 < a\nb c : α\n⊢ (fun x x_1 => x * x_1) a '' Ioo b c = Ioo (a * b) (a * c)", "tactic": "convert image_mul_right_Ioo b c h using 1 <;> simp only [mul_comm _ a]" } ]
[ 759, 73 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 757, 1 ]
Mathlib/SetTheory/Game/PGame.lean
PGame.le_trans_aux
[]
[ 512, 77 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 507, 9 ]
Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean
ContinuousAffineMap.toConstProdContinuousLinearMap_fst
[]
[ 277, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 275, 1 ]
Mathlib/Order/Filter/Basic.lean
Filter.eventuallyLE_bind
[]
[ 2731, 10 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2729, 1 ]
Mathlib/Algebra/IndicatorFunction.lean
Set.mulIndicator_le
[]
[ 875, 43 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 873, 1 ]
Mathlib/Topology/Algebra/Monoid.lean
nhds_one_mul_nhds
[]
[ 154, 45 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 151, 1 ]
Mathlib/MeasureTheory/Function/LpSeminorm.lean
MeasureTheory.Memℒp.restrict
[]
[ 600, 43 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 599, 1 ]
Mathlib/LinearAlgebra/AnnihilatingPolynomial.lean
Polynomial.monic_annIdealGenerator
[]
[ 129, 55 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 127, 1 ]
Mathlib/MeasureTheory/Constructions/Prod/Integral.lean
MeasureTheory.integrable_prod_mul
[ { "state_after": "case refine'_1\nα : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ AEStronglyMeasurable (fun z => f z.fst * g z.snd) (Measure.prod μ ν)\n\ncase refine'_2\nα : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ ∀ᵐ (x : α) ∂μ, Integrable fun y => f (x, y).fst * g (x, y).snd\n\ncase refine'_3\nα : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ Integrable fun x => ∫ (y : β), ‖f (x, y).fst * g (x, y).snd‖ ∂ν", "state_before": "α : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ Integrable fun z => f z.fst * g z.snd", "tactic": "refine' (integrable_prod_iff _).2 ⟨_, _⟩" }, { "state_after": "no goals", "state_before": "case refine'_1\nα : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ AEStronglyMeasurable (fun z => f z.fst * g z.snd) (Measure.prod μ ν)", "tactic": "exact hf.1.fst.mul hg.1.snd" }, { "state_after": "no goals", "state_before": "case refine'_2\nα : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ ∀ᵐ (x : α) ∂μ, Integrable fun y => f (x, y).fst * g (x, y).snd", "tactic": "exact eventually_of_forall fun x => hg.const_mul (f x)" }, { "state_after": "no goals", "state_before": "case refine'_3\nα : Type u_2\nα' : Type ?u.2408961\nβ : Type u_3\nβ' : Type ?u.2408967\nγ : Type ?u.2408970\nE : Type ?u.2408973\ninst✝⁷ : MeasurableSpace α\ninst✝⁶ : MeasurableSpace α'\ninst✝⁵ : MeasurableSpace β\ninst✝⁴ : MeasurableSpace β'\ninst✝³ : MeasurableSpace γ\nμ μ' : Measure α\nν ν' : Measure β\nτ : Measure γ\ninst✝² : NormedAddCommGroup E\ninst✝¹ : SigmaFinite ν\nL : Type u_1\ninst✝ : IsROrC L\nf : α → L\ng : β → L\nhf : Integrable f\nhg : Integrable g\n⊢ Integrable fun x => ∫ (y : β), ‖f (x, y).fst * g (x, y).snd‖ ∂ν", "tactic": "simpa only [norm_mul, integral_mul_left] using hf.norm.mul_const _" } ]
[ 318, 71 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 313, 1 ]
Mathlib/LinearAlgebra/Matrix/Reindex.lean
Matrix.reindexAlgEquiv_refl
[]
[ 147, 28 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 146, 1 ]
Mathlib/Algebra/Group/Units.lean
Units.val_inv_eq_inv_val
[]
[ 407, 50 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 406, 1 ]
Mathlib/Data/Part.lean
Part.left_dom_of_union_dom
[]
[ 847, 92 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 847, 1 ]
Mathlib/Order/Circular.lean
Set.mem_cIoo
[]
[ 355, 10 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 354, 1 ]
Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean
Complex.arg_neg_eq_arg_sub_pi_iff
[ { "state_after": "case inl\nx : ℂ\nhi : x.im < 0\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0\n\ncase inr.inl\nx : ℂ\nhi : x.im = 0\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0\n\ncase inr.inr\nx : ℂ\nhi : 0 < x.im\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0", "state_before": "x : ℂ\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0", "tactic": "rcases lt_trichotomy x.im 0 with (hi | hi | hi)" }, { "state_after": "no goals", "state_before": "case inl\nx : ℂ\nhi : x.im < 0\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0", "tactic": "simp [hi, hi.ne, hi.not_lt, arg_neg_eq_arg_add_pi_of_im_neg, sub_eq_add_neg, ←\n add_eq_zero_iff_eq_neg, Real.pi_ne_zero]" }, { "state_after": "case inr.inl\nx : ℂ\nhi : x.im = 0\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "state_before": "case inr.inl\nx : ℂ\nhi : x.im = 0\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0", "tactic": "rw [(ext rfl hi : x = x.re)]" }, { "state_after": "case inr.inl.inl\nx : ℂ\nhi : x.im = 0\nhr : x.re < 0\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0\n\ncase inr.inl.inr.inl\nx : ℂ\nhi : x.im = 0\nhr : x.re = 0\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0\n\ncase inr.inl.inr.inr\nx : ℂ\nhi : x.im = 0\nhr : 0 < x.re\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "state_before": "case inr.inl\nx : ℂ\nhi : x.im = 0\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "tactic": "rcases lt_trichotomy x.re 0 with (hr | hr | hr)" }, { "state_after": "case inr.inl.inl\nx : ℂ\nhi : x.im = 0\nhr : x.re < 0\n⊢ 0 = π - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "state_before": "case inr.inl.inl\nx : ℂ\nhi : x.im = 0\nhr : x.re < 0\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "tactic": "rw [arg_ofReal_of_neg hr, ← ofReal_neg, arg_ofReal_of_nonneg (Left.neg_pos_iff.2 hr).le]" }, { "state_after": "no goals", "state_before": "case inr.inl.inl\nx : ℂ\nhi : x.im = 0\nhr : x.re < 0\n⊢ 0 = π - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "tactic": "simp [hr]" }, { "state_after": "no goals", "state_before": "case inr.inl.inr.inl\nx : ℂ\nhi : x.im = 0\nhr : x.re = 0\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "tactic": "simp [hr, hi, Real.pi_ne_zero]" }, { "state_after": "case inr.inl.inr.inr\nx : ℂ\nhi : x.im = 0\nhr : 0 < x.re\n⊢ π = 0 - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "state_before": "case inr.inl.inr.inr\nx : ℂ\nhi : x.im = 0\nhr : 0 < x.re\n⊢ arg (-↑x.re) = arg ↑x.re - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "tactic": "rw [arg_ofReal_of_nonneg hr.le, ← ofReal_neg, arg_ofReal_of_neg (Left.neg_neg_iff.2 hr)]" }, { "state_after": "no goals", "state_before": "case inr.inl.inr.inr\nx : ℂ\nhi : x.im = 0\nhr : 0 < x.re\n⊢ π = 0 - π ↔ 0 < (↑x.re).im ∨ (↑x.re).im = 0 ∧ (↑x.re).re < 0", "tactic": "simp [hr.not_lt, ← add_eq_zero_iff_eq_neg, Real.pi_ne_zero]" }, { "state_after": "no goals", "state_before": "case inr.inr\nx : ℂ\nhi : 0 < x.im\n⊢ arg (-x) = arg x - π ↔ 0 < x.im ∨ x.im = 0 ∧ x.re < 0", "tactic": "simp [hi, arg_neg_eq_arg_sub_pi_of_im_pos]" } ]
[ 398, 47 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 385, 1 ]
Mathlib/Data/Polynomial/Expand.lean
Polynomial.coe_expand
[]
[ 44, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 43, 1 ]
Mathlib/MeasureTheory/Decomposition/Lebesgue.lean
MeasureTheory.SignedMeasure.singularPart_smul_nnreal
[ { "state_after": "α : Type u_1\nβ : Type ?u.623899\nm : MeasurableSpace α\nμ✝ ν : Measure α\ns✝ t s : SignedMeasure α\nμ : Measure α\nr : ℝ≥0\n⊢ toSignedMeasure (Measure.singularPart (toJordanDecomposition (r • s)).posPart μ) -\n toSignedMeasure (Measure.singularPart (toJordanDecomposition (r • s)).negPart μ) =\n toSignedMeasure (r • Measure.singularPart (toJordanDecomposition s).posPart μ) -\n toSignedMeasure (r • Measure.singularPart (toJordanDecomposition s).negPart μ)", "state_before": "α : Type u_1\nβ : Type ?u.623899\nm : MeasurableSpace α\nμ✝ ν : Measure α\ns✝ t s : SignedMeasure α\nμ : Measure α\nr : ℝ≥0\n⊢ singularPart (r • s) μ = r • singularPart s μ", "tactic": "rw [singularPart, singularPart, smul_sub, ← toSignedMeasure_smul, ← toSignedMeasure_smul]" } ]
[ 1089, 91 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1081, 1 ]
Mathlib/Topology/Instances/ENNReal.lean
Real.diam_Ico
[ { "state_after": "no goals", "state_before": "α : Type ?u.562585\nβ : Type ?u.562588\nγ : Type ?u.562591\ninst✝ : PseudoEMetricSpace α\na b : ℝ\nh : a ≤ b\n⊢ Metric.diam (Ico a b) = b - a", "tactic": "simp [Metric.diam, ENNReal.toReal_ofReal (sub_nonneg.2 h)]" } ]
[ 1560, 61 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1559, 1 ]
Mathlib/CategoryTheory/Subobject/Lattice.lean
CategoryTheory.Subobject.top_eq_id
[]
[ 233, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 232, 1 ]
Mathlib/Order/Interval.lean
Interval.coe_sSubset_coe
[]
[ 483, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 482, 1 ]
Mathlib/Topology/Bases.lean
TopologicalSpace.isSeparable_univ_iff
[ { "state_after": "case mp\nα : Type u\nt : TopologicalSpace α\n⊢ IsSeparable univ → SeparableSpace α\n\ncase mpr\nα : Type u\nt : TopologicalSpace α\n⊢ SeparableSpace α → IsSeparable univ", "state_before": "α : Type u\nt : TopologicalSpace α\n⊢ IsSeparable univ ↔ SeparableSpace α", "tactic": "constructor" }, { "state_after": "case mp.intro.intro\nα : Type u\nt : TopologicalSpace α\nc : Set α\nc_count : Set.Countable c\nhc : univ ⊆ closure c\n⊢ SeparableSpace α", "state_before": "case mp\nα : Type u\nt : TopologicalSpace α\n⊢ IsSeparable univ → SeparableSpace α", "tactic": "rintro ⟨c, c_count, hc⟩" }, { "state_after": "no goals", "state_before": "case mp.intro.intro\nα : Type u\nt : TopologicalSpace α\nc : Set α\nc_count : Set.Countable c\nhc : univ ⊆ closure c\n⊢ SeparableSpace α", "tactic": "refine' ⟨⟨c, c_count, by rwa [dense_iff_closure_eq, ← univ_subset_iff]⟩⟩" }, { "state_after": "no goals", "state_before": "α : Type u\nt : TopologicalSpace α\nc : Set α\nc_count : Set.Countable c\nhc : univ ⊆ closure c\n⊢ Dense c", "tactic": "rwa [dense_iff_closure_eq, ← univ_subset_iff]" }, { "state_after": "case mpr\nα : Type u\nt : TopologicalSpace α\nh : SeparableSpace α\n⊢ IsSeparable univ", "state_before": "case mpr\nα : Type u\nt : TopologicalSpace α\n⊢ SeparableSpace α → IsSeparable univ", "tactic": "intro h" }, { "state_after": "case mpr.intro.intro\nα : Type u\nt : TopologicalSpace α\nh : SeparableSpace α\nc : Set α\nc_count : Set.Countable c\nhc : Dense c\n⊢ IsSeparable univ", "state_before": "case mpr\nα : Type u\nt : TopologicalSpace α\nh : SeparableSpace α\n⊢ IsSeparable univ", "tactic": "rcases exists_countable_dense α with ⟨c, c_count, hc⟩" }, { "state_after": "no goals", "state_before": "case mpr.intro.intro\nα : Type u\nt : TopologicalSpace α\nh : SeparableSpace α\nc : Set α\nc_count : Set.Countable c\nhc : Dense c\n⊢ IsSeparable univ", "tactic": "exact ⟨c, c_count, by rwa [univ_subset_iff, ← dense_iff_closure_eq]⟩" }, { "state_after": "no goals", "state_before": "α : Type u\nt : TopologicalSpace α\nh : SeparableSpace α\nc : Set α\nc_count : Set.Countable c\nhc : Dense c\n⊢ univ ⊆ closure c", "tactic": "rwa [univ_subset_iff, ← dense_iff_closure_eq]" } ]
[ 426, 73 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 420, 1 ]
Mathlib/RingTheory/PowerSeries/Basic.lean
PowerSeries.constantCoeff_comp_C
[]
[ 1544, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1543, 1 ]
Mathlib/Data/Real/ENNReal.lean
ENNReal.coe_zpow
[ { "state_after": "case ofNat\nα : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℕ\n⊢ ↑(r ^ Int.ofNat n) = ↑r ^ Int.ofNat n\n\ncase negSucc\nα : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℕ\n⊢ ↑(r ^ Int.negSucc n) = ↑r ^ Int.negSucc n", "state_before": "α : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℤ\n⊢ ↑(r ^ n) = ↑r ^ n", "tactic": "cases' n with n n" }, { "state_after": "no goals", "state_before": "case ofNat\nα : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℕ\n⊢ ↑(r ^ Int.ofNat n) = ↑r ^ Int.ofNat n", "tactic": "simp only [Int.ofNat_eq_coe, coe_pow, zpow_ofNat]" }, { "state_after": "case negSucc\nα : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℕ\nthis : r ^ Nat.succ n ≠ 0\n⊢ ↑(r ^ Int.negSucc n) = ↑r ^ Int.negSucc n", "state_before": "case negSucc\nα : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℕ\n⊢ ↑(r ^ Int.negSucc n) = ↑r ^ Int.negSucc n", "tactic": "have : r ^ n.succ ≠ 0 := pow_ne_zero (n + 1) hr" }, { "state_after": "no goals", "state_before": "case negSucc\nα : Type ?u.359170\nβ : Type ?u.359173\na b c d : ℝ≥0∞\nr p q : ℝ≥0\nhr : r ≠ 0\nn : ℕ\nthis : r ^ Nat.succ n ≠ 0\n⊢ ↑(r ^ Int.negSucc n) = ↑r ^ Int.negSucc n", "tactic": "simp only [zpow_negSucc, coe_inv this, coe_pow]" } ]
[ 1859, 52 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1855, 1 ]
Mathlib/MeasureTheory/Integral/Bochner.lean
MeasureTheory.snorm_one_le_of_le'
[ { "state_after": "α : Type u_1\nE : Type ?u.1760021\nF : Type ?u.1760024\n𝕜 : Type ?u.1760027\ninst✝⁸ : NormedAddCommGroup E\ninst✝⁷ : NormedSpace ℝ E\ninst✝⁶ : CompleteSpace E\ninst✝⁵ : NontriviallyNormedField 𝕜\ninst✝⁴ : NormedSpace 𝕜 E\ninst✝³ : SMulCommClass ℝ 𝕜 E\ninst✝² : NormedAddCommGroup F\ninst✝¹ : NormedSpace ℝ F\ninst✝ : CompleteSpace F\nm0 : MeasurableSpace α\nμ : Measure α\nr : ℝ\nf : α → ℝ\nhfint : Integrable f\nhfint' : 0 ≤ ∫ (x : α), f x ∂μ\nhf : ∀ᵐ (ω : α) ∂μ, f ω ≤ r\n⊢ ∀ᵐ (ω : α) ∂μ, f ω ≤ ↑(Real.toNNReal r)", "state_before": "α : Type u_1\nE : Type ?u.1760021\nF : Type ?u.1760024\n𝕜 : Type ?u.1760027\ninst✝⁸ : NormedAddCommGroup E\ninst✝⁷ : NormedSpace ℝ E\ninst✝⁶ : CompleteSpace E\ninst✝⁵ : NontriviallyNormedField 𝕜\ninst✝⁴ : NormedSpace 𝕜 E\ninst✝³ : SMulCommClass ℝ 𝕜 E\ninst✝² : NormedAddCommGroup F\ninst✝¹ : NormedSpace ℝ F\ninst✝ : CompleteSpace F\nm0 : MeasurableSpace α\nμ : Measure α\nr : ℝ\nf : α → ℝ\nhfint : Integrable f\nhfint' : 0 ≤ ∫ (x : α), f x ∂μ\nhf : ∀ᵐ (ω : α) ∂μ, f ω ≤ r\n⊢ snorm f 1 μ ≤ 2 * ↑↑μ univ * ENNReal.ofReal r", "tactic": "refine' snorm_one_le_of_le hfint hfint' _" }, { "state_after": "α : Type u_1\nE : Type ?u.1760021\nF : Type ?u.1760024\n𝕜 : Type ?u.1760027\ninst✝⁸ : NormedAddCommGroup E\ninst✝⁷ : NormedSpace ℝ E\ninst✝⁶ : CompleteSpace E\ninst✝⁵ : NontriviallyNormedField 𝕜\ninst✝⁴ : NormedSpace 𝕜 E\ninst✝³ : SMulCommClass ℝ 𝕜 E\ninst✝² : NormedAddCommGroup F\ninst✝¹ : NormedSpace ℝ F\ninst✝ : CompleteSpace F\nm0 : MeasurableSpace α\nμ : Measure α\nr : ℝ\nf : α → ℝ\nhfint : Integrable f\nhfint' : 0 ≤ ∫ (x : α), f x ∂μ\nhf : ∀ᵐ (ω : α) ∂μ, f ω ≤ r\n⊢ ∀ᵐ (ω : α) ∂μ, f ω ≤ r ∨ f ω ≤ 0", "state_before": "α : Type u_1\nE : Type ?u.1760021\nF : Type ?u.1760024\n𝕜 : Type ?u.1760027\ninst✝⁸ : NormedAddCommGroup E\ninst✝⁷ : NormedSpace ℝ E\ninst✝⁶ : CompleteSpace E\ninst✝⁵ : NontriviallyNormedField 𝕜\ninst✝⁴ : NormedSpace 𝕜 E\ninst✝³ : SMulCommClass ℝ 𝕜 E\ninst✝² : NormedAddCommGroup F\ninst✝¹ : NormedSpace ℝ F\ninst✝ : CompleteSpace F\nm0 : MeasurableSpace α\nμ : Measure α\nr : ℝ\nf : α → ℝ\nhfint : Integrable f\nhfint' : 0 ≤ ∫ (x : α), f x ∂μ\nhf : ∀ᵐ (ω : α) ∂μ, f ω ≤ r\n⊢ ∀ᵐ (ω : α) ∂μ, f ω ≤ ↑(Real.toNNReal r)", "tactic": "simp only [Real.coe_toNNReal', le_max_iff]" }, { "state_after": "no goals", "state_before": "α : Type u_1\nE : Type ?u.1760021\nF : Type ?u.1760024\n𝕜 : Type ?u.1760027\ninst✝⁸ : NormedAddCommGroup E\ninst✝⁷ : NormedSpace ℝ E\ninst✝⁶ : CompleteSpace E\ninst✝⁵ : NontriviallyNormedField 𝕜\ninst✝⁴ : NormedSpace 𝕜 E\ninst✝³ : SMulCommClass ℝ 𝕜 E\ninst✝² : NormedAddCommGroup F\ninst✝¹ : NormedSpace ℝ F\ninst✝ : CompleteSpace F\nm0 : MeasurableSpace α\nμ : Measure α\nr : ℝ\nf : α → ℝ\nhfint : Integrable f\nhfint' : 0 ≤ ∫ (x : α), f x ∂μ\nhf : ∀ᵐ (ω : α) ∂μ, f ω ≤ r\n⊢ ∀ᵐ (ω : α) ∂μ, f ω ≤ r ∨ f ω ≤ 0", "tactic": "filter_upwards [hf]with ω hω using Or.inl hω" } ]
[ 1881, 47 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1877, 1 ]
Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean
CategoryTheory.Limits.parallelPair_map_left
[]
[ 235, 85 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 235, 1 ]
Mathlib/MeasureTheory/Integral/FundThmCalculus.lean
Continuous.integral_hasStrictDerivAt
[]
[ 685, 20 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 682, 1 ]
Mathlib/Algebra/GradedMonoid.lean
GradedMonoid.mk_pow
[ { "state_after": "no goals", "state_before": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn : ℕ\n⊢ mk i a ^ n = mk (n • i) (GMonoid.gnpow n a)", "tactic": "match n with\n| 0 =>\n rw [pow_zero]\n exact (GMonoid.gnpow_zero' ⟨_, a⟩).symm\n| n+1 =>\n rw [pow_succ, mk_pow a n, mk_mul_mk]\n exact (GMonoid.gnpow_succ' n ⟨_, a⟩).symm" }, { "state_after": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn : ℕ\n⊢ 1 = mk (0 • i) (GMonoid.gnpow 0 a)", "state_before": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn : ℕ\n⊢ mk i a ^ 0 = mk (0 • i) (GMonoid.gnpow 0 a)", "tactic": "rw [pow_zero]" }, { "state_after": "no goals", "state_before": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn : ℕ\n⊢ 1 = mk (0 • i) (GMonoid.gnpow 0 a)", "tactic": "exact (GMonoid.gnpow_zero' ⟨_, a⟩).symm" }, { "state_after": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn✝ n : ℕ\n⊢ mk (i + n • i) (GMul.mul a (GMonoid.gnpow n a)) = mk ((n + 1) • i) (GMonoid.gnpow (n + 1) a)", "state_before": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn✝ n : ℕ\n⊢ mk i a ^ (n + 1) = mk ((n + 1) • i) (GMonoid.gnpow (n + 1) a)", "tactic": "rw [pow_succ, mk_pow a n, mk_mul_mk]" }, { "state_after": "no goals", "state_before": "ι : Type u_1\nA : ι → Type u_2\ninst✝¹ : AddMonoid ι\ninst✝ : GMonoid A\ni : ι\na : A i\nn✝ n : ℕ\n⊢ mk (i + n • i) (GMul.mul a (GMonoid.gnpow n a)) = mk ((n + 1) • i) (GMonoid.gnpow (n + 1) a)", "tactic": "exact (GMonoid.gnpow_succ' n ⟨_, a⟩).symm" } ]
[ 222, 46 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 214, 1 ]
Mathlib/Data/Real/ENNReal.lean
ENNReal.toReal_mul
[]
[ 2239, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 2238, 1 ]
Mathlib/GroupTheory/GroupAction/Pi.lean
Set.piecewise_smul
[]
[ 262, 51 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 260, 1 ]
Mathlib/GroupTheory/Subgroup/ZPowers.lean
Subgroup.center_eq_infi'
[ { "state_after": "no goals", "state_before": "G : Type u_1\ninst✝² : Group G\nA : Type ?u.41951\ninst✝¹ : AddGroup A\nN : Type ?u.41957\ninst✝ : Group N\ns : Set G\ng : G\nS : Set G\nhS : closure S = ⊤\n⊢ center G = ⨅ (g : ↑S), centralizer (zpowers ↑g)", "tactic": "rw [center_eq_iInf S hS, ← iInf_subtype'']" } ]
[ 250, 48 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 248, 1 ]
Mathlib/MeasureTheory/Integral/SetIntegral.lean
MeasureTheory.integral_union_eq_left_of_forall
[]
[ 331, 63 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 329, 1 ]
Mathlib/Topology/DenseEmbedding.lean
DenseEmbedding.subtype
[ { "state_after": "case h.mk\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.33913\nδ : Type ?u.33916\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\ne : α → β\nde : DenseEmbedding e\np : α → Prop\nx : β\nhx : x ∈ closure (e '' {x | p x})\n⊢ { val := x, property := hx } ∈ closure (range (subtypeEmb p e)) ↔ { val := x, property := hx } ∈ univ", "state_before": "α : Type u_1\nβ : Type u_2\nγ : Type ?u.33913\nδ : Type ?u.33916\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\ne : α → β\nde : DenseEmbedding e\np : α → Prop\n⊢ closure (range (subtypeEmb p e)) = univ", "tactic": "ext ⟨x, hx⟩" }, { "state_after": "case h.mk\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.33913\nδ : Type ?u.33916\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\ne : α → β\nde : DenseEmbedding e\np : α → Prop\nx : β\nhx✝ : x ∈ closure (e '' {x | p x})\nhx : x ∈ closure (range fun x => e ↑x)\n⊢ { val := x, property := hx✝ } ∈ closure (range (subtypeEmb p e)) ↔ { val := x, property := hx✝ } ∈ univ", "state_before": "case h.mk\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.33913\nδ : Type ?u.33916\ninst✝³ : TopologicalSpace α\ninst✝² : TopologicalSpace β\ninst✝¹ : TopologicalSpace γ\ninst✝ : TopologicalSpace δ\ne : α → β\nde : DenseEmbedding e\np : α → Prop\nx : β\nhx : x ∈ closure (e '' {x | p x})\n⊢ { val := x, property := hx } ∈ closure (range (subtypeEmb p e)) ↔ { val := x, property := hx } ∈ univ", "tactic": "rw [image_eq_range] at hx" } ]
[ 292, 21 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 282, 11 ]
Mathlib/MeasureTheory/Function/AEEqFun.lean
MeasureTheory.AEEqFun.zpow_toGerm
[]
[ 792, 20 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 791, 1 ]
Mathlib/CategoryTheory/Closed/Cartesian.lean
CategoryTheory.CartesianClosed.uncurry_id_eq_ev
[ { "state_after": "no goals", "state_before": "C : Type u\ninst✝³ : Category C\nA✝ B X✝ X' Y Y' Z : C\ninst✝² : HasFiniteProducts C\ninst✝¹ : Exponentiable A✝\nA X : C\ninst✝ : Exponentiable A\n⊢ uncurry (𝟙 (A ⟹ X)) = (exp.ev A).app X", "tactic": "rw [uncurry_eq, prod.map_id_id, id_comp]" } ]
[ 233, 43 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 232, 1 ]
Mathlib/Order/Hom/CompleteLattice.lean
map_iInf₂
[ { "state_after": "no goals", "state_before": "F : Type u_3\nα : Type u_1\nβ : Type u_2\nγ : Type ?u.8713\nδ : Type ?u.8716\nι : Sort u_4\nκ : ι → Sort u_5\ninst✝² : InfSet α\ninst✝¹ : InfSet β\ninst✝ : sInfHomClass F α β\nf : F\ng : (i : ι) → κ i → α\n⊢ ↑f (⨅ (i : ι) (j : κ i), g i j) = ⨅ (i : ι) (j : κ i), ↑f (g i j)", "tactic": "simp_rw [map_iInf]" } ]
[ 144, 73 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 143, 1 ]
Mathlib/LinearAlgebra/LinearIndependent.lean
linearIndependent_empty
[ { "state_after": "no goals", "state_before": "ι : Type u'\nι' : Type ?u.212015\nR : Type u_2\nK : Type ?u.212021\nM : Type u_1\nM' : Type ?u.212027\nM'' : Type ?u.212030\nV : Type u\nV' : Type ?u.212035\nv : ι → M\ninst✝⁶ : Semiring R\ninst✝⁵ : AddCommMonoid M\ninst✝⁴ : AddCommMonoid M'\ninst✝³ : AddCommMonoid M''\ninst✝² : Module R M\ninst✝¹ : Module R M'\ninst✝ : Module R M''\na b : R\nx y : M\n⊢ LinearIndependent R fun x => ↑x", "tactic": "simp [linearIndependent_subtype_disjoint]" } ]
[ 415, 44 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 414, 1 ]
Mathlib/Data/Fintype/Option.lean
univ_option
[]
[ 33, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 32, 1 ]
Mathlib/Data/List/Pairwise.lean
List.rel_of_pairwise_cons
[]
[ 49, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 48, 1 ]
Mathlib/MeasureTheory/Function/UniformIntegrable.lean
MeasureTheory.tendsto_Lp_of_tendsto_ae
[ { "state_after": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ Tendsto (fun n => snorm (f n - g) p μ) atTop (𝓝 0)", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\n⊢ Tendsto (fun n => snorm (f n - g) p μ) atTop (𝓝 0)", "tactic": "have : ∀ n, snorm (f n - g) p μ = snorm ((hf n).mk (f n) - hg.1.mk g) p μ :=\n fun n => snorm_congr_ae ((hf n).ae_eq_mk.sub hg.1.ae_eq_mk)" }, { "state_after": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ Tendsto\n (fun n =>\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ)\n atTop (𝓝 0)", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ Tendsto (fun n => snorm (f n - g) p μ) atTop (𝓝 0)", "tactic": "simp_rw [this]" }, { "state_after": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ ∀ᵐ (x : α) ∂μ,\n Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop\n (𝓝 (AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x))", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ Tendsto\n (fun n =>\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ)\n atTop (𝓝 0)", "tactic": "refine' tendsto_Lp_of_tendsto_ae_of_meas μ hp hp' (fun n => (hf n).stronglyMeasurable_mk)\n hg.1.stronglyMeasurable_mk (hg.ae_eq hg.1.ae_eq_mk) (hui.ae_eq fun n => (hf n).ae_eq_mk) _" }, { "state_after": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\n⊢ ∀ᵐ (x : α) ∂μ,\n Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop\n (𝓝 (AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x))", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ ∀ᵐ (x : α) ∂μ,\n Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop\n (𝓝 (AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x))", "tactic": "have h_ae_forall_eq : ∀ᵐ x ∂μ, ∀ n, f n x = (hf n).mk (f n) x := by\n rw [ae_all_iff]\n exact fun n => (hf n).ae_eq_mk" }, { "state_after": "case h\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\n⊢ Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop\n (𝓝 (AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x))", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\n⊢ ∀ᵐ (x : α) ∂μ,\n Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop\n (𝓝 (AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x))", "tactic": "filter_upwards [hfg, h_ae_forall_eq, hg.1.ae_eq_mk] with x hx_tendsto hxf_eq hxg_eq" }, { "state_after": "case h\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\n⊢ Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop (𝓝 (g x))", "state_before": "case h\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\n⊢ Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop\n (𝓝 (AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x))", "tactic": "rw [← hxg_eq]" }, { "state_after": "case h.e'_3\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\n⊢ (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) = fun n => f n x", "state_before": "case h\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\n⊢ Tendsto (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) atTop (𝓝 (g x))", "tactic": "convert hx_tendsto using 1" }, { "state_after": "case h.e'_3.h\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\nn : ℕ\n⊢ AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x = f n x", "state_before": "case h.e'_3\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\n⊢ (fun n => AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x) = fun n => f n x", "tactic": "ext1 n" }, { "state_after": "no goals", "state_before": "case h.e'_3.h\nα : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\nh_ae_forall_eq : ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nx : α\nhx_tendsto : Tendsto (fun n => f n x) atTop (𝓝 (g x))\nhxf_eq : ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x\nhxg_eq : g x = AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ) x\nn : ℕ\n⊢ AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x = f n x", "tactic": "exact (hxf_eq n).symm" }, { "state_after": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ ∀ (i : ℕ), ∀ᵐ (a : α) ∂μ, f i a = AEStronglyMeasurable.mk (f i) (_ : AEStronglyMeasurable (f i) μ) a", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ ∀ᵐ (x : α) ∂μ, ∀ (n : ℕ), f n x = AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) x", "tactic": "rw [ae_all_iff]" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type u_2\nι : Type ?u.487716\nm : MeasurableSpace α\nμ : Measure α\ninst✝¹ : NormedAddCommGroup β\np : ℝ≥0∞\ninst✝ : IsFiniteMeasure μ\nhp : 1 ≤ p\nhp' : p ≠ ⊤\nf : ℕ → α → β\ng : α → β\nhf : ∀ (n : ℕ), AEStronglyMeasurable (f n) μ\nhg : Memℒp g p\nhui : UnifIntegrable f p μ\nhfg : ∀ᵐ (x : α) ∂μ, Tendsto (fun n => f n x) atTop (𝓝 (g x))\nthis :\n ∀ (n : ℕ),\n snorm (f n - g) p μ =\n snorm\n (AEStronglyMeasurable.mk (f n) (_ : AEStronglyMeasurable (f n) μ) -\n AEStronglyMeasurable.mk g (_ : AEStronglyMeasurable g μ))\n p μ\n⊢ ∀ (i : ℕ), ∀ᵐ (a : α) ∂μ, f i a = AEStronglyMeasurable.mk (f i) (_ : AEStronglyMeasurable (f i) μ) a", "tactic": "exact fun n => (hf n).ae_eq_mk" } ]
[ 574, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 558, 1 ]
Mathlib/Topology/Sheaves/SheafCondition/PairwiseIntersections.lean
TopCat.Sheaf.objSupIsoProdEqLocus_hom_snd
[]
[ 484, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 479, 1 ]
Mathlib/CategoryTheory/WithTerminal.lean
CategoryTheory.WithTerminal.lift_map_liftStar
[ { "state_after": "C : Type u\ninst✝¹ : Category C\nD : Type u_1\ninst✝ : Category D\nZ : D\nF : C ⥤ D\nM : (x : C) → F.obj x ⟶ Z\nhM : ∀ (x y : C) (f : x ⟶ y), F.map f ≫ M y = M x\nx : C\n⊢ (lift F M hM).map (Limits.IsTerminal.from starTerminal (incl.obj x)) = M x", "state_before": "C : Type u\ninst✝¹ : Category C\nD : Type u_1\ninst✝ : Category D\nZ : D\nF : C ⥤ D\nM : (x : C) → F.obj x ⟶ Z\nhM : ∀ (x y : C) (f : x ⟶ y), F.map f ≫ M y = M x\nx : C\n⊢ (lift F M hM).map (Limits.IsTerminal.from starTerminal (incl.obj x)) ≫ (liftStar F M hM).hom =\n (inclLift F M hM).hom.app x ≫ M x", "tactic": "erw [Category.id_comp, Category.comp_id]" }, { "state_after": "no goals", "state_before": "C : Type u\ninst✝¹ : Category C\nD : Type u_1\ninst✝ : Category D\nZ : D\nF : C ⥤ D\nM : (x : C) → F.obj x ⟶ Z\nhM : ∀ (x y : C) (f : x ⟶ y), F.map f ≫ M y = M x\nx : C\n⊢ (lift F M hM).map (Limits.IsTerminal.from starTerminal (incl.obj x)) = M x", "tactic": "rfl" } ]
[ 191, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 186, 1 ]
Mathlib/Data/Matrix/Basic.lean
Matrix.one_apply_ne'
[]
[ 550, 23 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 549, 1 ]
Mathlib/Topology/Homotopy/Contractible.lean
contractible_iff_id_nullhomotopic
[ { "state_after": "case mp\nY : Type u_1\ninst✝ : TopologicalSpace Y\n⊢ ContractibleSpace Y → Nullhomotopic (ContinuousMap.id Y)\n\ncase mpr\nY : Type u_1\ninst✝ : TopologicalSpace Y\n⊢ Nullhomotopic (ContinuousMap.id Y) → ContractibleSpace Y", "state_before": "Y : Type u_1\ninst✝ : TopologicalSpace Y\n⊢ ContractibleSpace Y ↔ Nullhomotopic (ContinuousMap.id Y)", "tactic": "constructor" }, { "state_after": "case mpr.intro\nY : Type u_1\ninst✝ : TopologicalSpace Y\np : Y\nh : Homotopic (ContinuousMap.id Y) (const Y p)\n⊢ ContractibleSpace Y", "state_before": "case mpr\nY : Type u_1\ninst✝ : TopologicalSpace Y\n⊢ Nullhomotopic (ContinuousMap.id Y) → ContractibleSpace Y", "tactic": "rintro ⟨p, h⟩" }, { "state_after": "case mpr.intro.refine_1\nY : Type u_1\ninst✝ : TopologicalSpace Y\np : Y\nh : Homotopic (ContinuousMap.id Y) (const Y p)\n⊢ Homotopic (comp (const Unit p) (const Y ())) (ContinuousMap.id Y)\n\ncase mpr.intro.refine_2\nY : Type u_1\ninst✝ : TopologicalSpace Y\np : Y\nh : Homotopic (ContinuousMap.id Y) (const Y p)\n⊢ Homotopic (comp (const Y ()) (const Unit p)) (ContinuousMap.id Unit)", "state_before": "case mpr.intro\nY : Type u_1\ninst✝ : TopologicalSpace Y\np : Y\nh : Homotopic (ContinuousMap.id Y) (const Y p)\n⊢ ContractibleSpace Y", "tactic": "refine\n { hequiv_unit' :=\n ⟨{ toFun := ContinuousMap.const _ ()\n invFun := ContinuousMap.const _ p\n left_inv := ?_\n right_inv := ?_ }⟩ }" }, { "state_after": "case mp\nY : Type u_1\ninst✝ : TopologicalSpace Y\na✝ : ContractibleSpace Y\n⊢ Nullhomotopic (ContinuousMap.id Y)", "state_before": "case mp\nY : Type u_1\ninst✝ : TopologicalSpace Y\n⊢ ContractibleSpace Y → Nullhomotopic (ContinuousMap.id Y)", "tactic": "intro" }, { "state_after": "no goals", "state_before": "case mp\nY : Type u_1\ninst✝ : TopologicalSpace Y\na✝ : ContractibleSpace Y\n⊢ Nullhomotopic (ContinuousMap.id Y)", "tactic": "apply id_nullhomotopic" }, { "state_after": "no goals", "state_before": "case mpr.intro.refine_1\nY : Type u_1\ninst✝ : TopologicalSpace Y\np : Y\nh : Homotopic (ContinuousMap.id Y) (const Y p)\n⊢ Homotopic (comp (const Unit p) (const Y ())) (ContinuousMap.id Y)", "tactic": "exact h.symm" }, { "state_after": "no goals", "state_before": "case mpr.intro.refine_2\nY : Type u_1\ninst✝ : TopologicalSpace Y\np : Y\nh : Homotopic (ContinuousMap.id Y) (const Y p)\n⊢ Homotopic (comp (const Y ()) (const Unit p)) (ContinuousMap.id Unit)", "tactic": "convert Homotopic.refl (ContinuousMap.id Unit)" } ]
[ 85, 51 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 72, 1 ]
Mathlib/Data/Set/Pointwise/SMul.lean
Set.mul_subset_iff_right
[]
[ 438, 26 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 437, 1 ]
Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean
Complex.sin_sub_int_mul_two_pi
[]
[ 1189, 32 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1188, 1 ]
Mathlib/LinearAlgebra/Basis.lean
Basis.map_equivFun
[]
[ 924, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 923, 1 ]
src/lean/Init/Core.lean
HEq.elim
[]
[ 619, 20 ]
d5348dfac847a56a4595fb6230fd0708dcb4e7e9
https://github.com/leanprover/lean4
[ 618, 1 ]
Mathlib/Algebra/Lie/IdealOperations.lean
LieSubmodule.lie_comm
[ { "state_after": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nI J : LieIdeal R L\nN₂ : LieSubmodule R L M₂\n⊢ ∀ (I J : LieIdeal R L), ⁅I, J⁆ ≤ ⁅J, I⁆", "state_before": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nI J : LieIdeal R L\nN₂ : LieSubmodule R L M₂\n⊢ ⁅I, J⁆ = ⁅J, I⁆", "tactic": "suffices ∀ I J : LieIdeal R L, ⁅I, J⁆ ≤ ⁅J, I⁆ by exact le_antisymm (this I J) (this J I)" }, { "state_after": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\n⊢ ∀ (I J : LieIdeal R L), ⁅I, J⁆ ≤ ⁅J, I⁆", "state_before": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nI J : LieIdeal R L\nN₂ : LieSubmodule R L M₂\n⊢ ∀ (I J : LieIdeal R L), ⁅I, J⁆ ≤ ⁅J, I⁆", "tactic": "clear! I J" }, { "state_after": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\n⊢ ⁅I, J⁆ ≤ ⁅J, I⁆", "state_before": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\n⊢ ∀ (I J : LieIdeal R L), ⁅I, J⁆ ≤ ⁅J, I⁆", "tactic": "intro I J" }, { "state_after": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\n⊢ {m | ∃ x n, ⁅↑x, ↑n⁆ = m} ⊆ ↑⁅J, I⁆", "state_before": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\n⊢ ⁅I, J⁆ ≤ ⁅J, I⁆", "tactic": "rw [lieIdeal_oper_eq_span, lieSpan_le]" }, { "state_after": "case intro.intro\nR : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\nx : L\ny : { x // x ∈ I }\nz : { x // x ∈ J }\nh : ⁅↑y, ↑z⁆ = x\n⊢ x ∈ ↑⁅J, I⁆", "state_before": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\n⊢ {m | ∃ x n, ⁅↑x, ↑n⁆ = m} ⊆ ↑⁅J, I⁆", "tactic": "rintro x ⟨y, z, h⟩" }, { "state_after": "case intro.intro\nR : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\nx : L\ny : { x // x ∈ I }\nz : { x // x ∈ J }\nh : ⁅↑y, ↑z⁆ = x\n⊢ ⁅↑y, ↑z⁆ ∈ ↑⁅J, I⁆", "state_before": "case intro.intro\nR : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\nx : L\ny : { x // x ∈ I }\nz : { x // x ∈ J }\nh : ⁅↑y, ↑z⁆ = x\n⊢ x ∈ ↑⁅J, I⁆", "tactic": "rw [← h]" }, { "state_after": "case intro.intro\nR : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\nx : L\ny : { x // x ∈ I }\nz : { x // x ∈ J }\nh : ⁅↑y, ↑z⁆ = x\n⊢ ⁅↑z, ↑(-y)⁆ ∈ ↑⁅J, I⁆", "state_before": "case intro.intro\nR : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\nx : L\ny : { x // x ∈ I }\nz : { x // x ∈ J }\nh : ⁅↑y, ↑z⁆ = x\n⊢ ⁅↑y, ↑z⁆ ∈ ↑⁅J, I⁆", "tactic": "rw [← lie_skew, ← lie_neg, ← LieSubmodule.coe_neg]" }, { "state_after": "no goals", "state_before": "case intro.intro\nR : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nN₂ : LieSubmodule R L M₂\nI J : LieIdeal R L\nx : L\ny : { x // x ∈ I }\nz : { x // x ∈ J }\nh : ⁅↑y, ↑z⁆ = x\n⊢ ⁅↑z, ↑(-y)⁆ ∈ ↑⁅J, I⁆", "tactic": "apply lie_coe_mem_lie" }, { "state_after": "no goals", "state_before": "R : Type u\nL : Type v\nM : Type w\nM₂ : Type w₁\ninst✝¹⁰ : CommRing R\ninst✝⁹ : LieRing L\ninst✝⁸ : LieAlgebra R L\ninst✝⁷ : AddCommGroup M\ninst✝⁶ : Module R M\ninst✝⁵ : LieRingModule L M\ninst✝⁴ : LieModule R L M\ninst✝³ : AddCommGroup M₂\ninst✝² : Module R M₂\ninst✝¹ : LieRingModule L M₂\ninst✝ : LieModule R L M₂\nN N' : LieSubmodule R L M\nI J : LieIdeal R L\nN₂ : LieSubmodule R L M₂\nthis : ∀ (I J : LieIdeal R L), ⁅I, J⁆ ≤ ⁅J, I⁆\n⊢ ⁅I, J⁆ = ⁅J, I⁆", "tactic": "exact le_antisymm (this I J) (this J I)" } ]
[ 123, 24 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 118, 1 ]
Mathlib/Analysis/SpecificLimits/Normed.lean
NormedRing.tsum_geometric_of_norm_lt_1
[ { "state_after": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖x ^ 0 + ∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖∑' (n : ℕ), x ^ n‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "tactic": "rw [tsum_eq_zero_add (NormedRing.summable_geometric_of_norm_lt_1 x h)]" }, { "state_after": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖1 + ∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖x ^ 0 + ∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "tactic": "simp only [_root_.pow_zero]" }, { "state_after": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖1‖ + ‖∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖1 + ∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "tactic": "refine' le_trans (norm_add_le _ _) _" }, { "state_after": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\nthis : ‖∑' (b : ℕ), (fun n => x ^ (n + 1)) b‖ ≤ (1 - ‖x‖)⁻¹ - 1\n⊢ ‖1‖ + ‖∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖1‖ + ‖∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "tactic": "have : ‖∑' b : ℕ, (fun n ↦ x ^ (n + 1)) b‖ ≤ (1 - ‖x‖)⁻¹ - 1 := by\n refine' tsum_of_norm_bounded _ fun b ↦ norm_pow_le' _ (Nat.succ_pos b)\n convert (hasSum_nat_add_iff' 1).mpr (hasSum_geometric_of_lt_1 (norm_nonneg x) h)\n simp" }, { "state_after": "no goals", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\nthis : ‖∑' (b : ℕ), (fun n => x ^ (n + 1)) b‖ ≤ (1 - ‖x‖)⁻¹ - 1\n⊢ ‖1‖ + ‖∑' (b : ℕ), x ^ (b + 1)‖ ≤ ‖1‖ - 1 + (1 - ‖x‖)⁻¹", "tactic": "linarith" }, { "state_after": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ HasSum (fun b => ‖x‖ ^ (b + 1)) ((1 - ‖x‖)⁻¹ - 1)", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ ‖∑' (b : ℕ), (fun n => x ^ (n + 1)) b‖ ≤ (1 - ‖x‖)⁻¹ - 1", "tactic": "refine' tsum_of_norm_bounded _ fun b ↦ norm_pow_le' _ (Nat.succ_pos b)" }, { "state_after": "case h.e'_6.h.e'_6\nα : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ 1 = ∑ i in Finset.range 1, ‖x‖ ^ i", "state_before": "α : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ HasSum (fun b => ‖x‖ ^ (b + 1)) ((1 - ‖x‖)⁻¹ - 1)", "tactic": "convert (hasSum_nat_add_iff' 1).mpr (hasSum_geometric_of_lt_1 (norm_nonneg x) h)" }, { "state_after": "no goals", "state_before": "case h.e'_6.h.e'_6\nα : Type ?u.1234446\nβ : Type ?u.1234449\nι : Type ?u.1234452\nR : Type u_1\ninst✝¹ : NormedRing R\ninst✝ : CompleteSpace R\nx : R\nh : ‖x‖ < 1\n⊢ 1 = ∑ i in Finset.range 1, ‖x‖ ^ i", "tactic": "simp" } ]
[ 480, 11 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 471, 1 ]
Mathlib/Algebra/BigOperators/Basic.lean
Finset.prod_ite_index
[]
[ 1106, 43 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1104, 1 ]
Mathlib/Data/Real/ENNReal.lean
ENNReal.ofReal_sum_of_nonneg
[ { "state_after": "α : Type u_1\nβ : Type ?u.204043\na b c d : ℝ≥0∞\nr p q : ℝ≥0\ns : Finset α\nf : α → ℝ\nhf : ∀ (i : α), i ∈ s → 0 ≤ f i\n⊢ Real.toNNReal (∑ i in s, f i) = ∑ a in s, Real.toNNReal (f a)", "state_before": "α : Type u_1\nβ : Type ?u.204043\na b c d : ℝ≥0∞\nr p q : ℝ≥0\ns : Finset α\nf : α → ℝ\nhf : ∀ (i : α), i ∈ s → 0 ≤ f i\n⊢ ENNReal.ofReal (∑ i in s, f i) = ∑ i in s, ENNReal.ofReal (f i)", "tactic": "simp_rw [ENNReal.ofReal, ← coe_finset_sum, coe_eq_coe]" }, { "state_after": "no goals", "state_before": "α : Type u_1\nβ : Type ?u.204043\na b c d : ℝ≥0∞\nr p q : ℝ≥0\ns : Finset α\nf : α → ℝ\nhf : ∀ (i : α), i ∈ s → 0 ≤ f i\n⊢ Real.toNNReal (∑ i in s, f i) = ∑ a in s, Real.toNNReal (f a)", "tactic": "exact Real.toNNReal_sum_of_nonneg hf" } ]
[ 1260, 39 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1257, 1 ]
Mathlib/SetTheory/Ordinal/Arithmetic.lean
Ordinal.isLimit_add_iff
[ { "state_after": "case mp\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a\n\ncase mpr\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit b ∨ b = 0 ∧ IsLimit a\n⊢ IsLimit (a + b)", "state_before": "α : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\n⊢ IsLimit (a + b) ↔ IsLimit b ∨ b = 0 ∧ IsLimit a", "tactic": "constructor <;> intro h" }, { "state_after": "case mpr.inl\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit b\n⊢ IsLimit (a + b)\n\ncase mpr.inr.intro\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na : Ordinal\nh : IsLimit a\n⊢ IsLimit (a + 0)", "state_before": "case mpr\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit b ∨ b = 0 ∧ IsLimit a\n⊢ IsLimit (a + b)", "tactic": "rcases h with (h | ⟨rfl, h⟩)" }, { "state_after": "case mpr.inr.intro\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na : Ordinal\nh : IsLimit a\n⊢ IsLimit (a + 0)", "state_before": "case mpr.inl\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit b\n⊢ IsLimit (a + b)\n\ncase mpr.inr.intro\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na : Ordinal\nh : IsLimit a\n⊢ IsLimit (a + 0)", "tactic": "exact add_isLimit a h" }, { "state_after": "no goals", "state_before": "case mpr.inr.intro\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na : Ordinal\nh : IsLimit a\n⊢ IsLimit (a + 0)", "tactic": "simpa only [add_zero]" }, { "state_after": "case pos\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : b = 0\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a\n\ncase neg\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a", "state_before": "case mp\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a", "tactic": "by_cases h' : b = 0" }, { "state_after": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ IsLimit b", "state_before": "case neg\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a", "tactic": "left" }, { "state_after": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ IsLimit (a + b - a)", "state_before": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ IsLimit b", "tactic": "rw [← add_sub_cancel a b]" }, { "state_after": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ a < a + b", "state_before": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ IsLimit (a + b - a)", "tactic": "apply sub_isLimit h" }, { "state_after": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\nthis : a + 0 < a + b\n⊢ a < a + b\n\ncase this\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ a + 0 < a + b", "state_before": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ a < a + b", "tactic": "suffices : a + 0 < a + b" }, { "state_after": "case this\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ a + 0 < a + b", "state_before": "case neg.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\nthis : a + 0 < a + b\n⊢ a < a + b\n\ncase this\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ a + 0 < a + b", "tactic": "simpa only [add_zero] using this" }, { "state_after": "no goals", "state_before": "case this\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : ¬b = 0\n⊢ a + 0 < a + b", "tactic": "rwa [add_lt_add_iff_left, Ordinal.pos_iff_ne_zero]" }, { "state_after": "case pos\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit a\nh' : b = 0\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a", "state_before": "case pos\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit (a + b)\nh' : b = 0\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a", "tactic": "rw [h', add_zero] at h" }, { "state_after": "case pos.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit a\nh' : b = 0\n⊢ b = 0 ∧ IsLimit a", "state_before": "case pos\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit a\nh' : b = 0\n⊢ IsLimit b ∨ b = 0 ∧ IsLimit a", "tactic": "right" }, { "state_after": "no goals", "state_before": "case pos.h\nα : Type ?u.248176\nβ : Type ?u.248179\nγ : Type ?u.248182\nr : α → α → Prop\ns : β → β → Prop\nt : γ → γ → Prop\na b : Ordinal\nh : IsLimit a\nh' : b = 0\n⊢ b = 0 ∧ IsLimit a", "tactic": "exact ⟨h', h⟩" } ]
[ 988, 77 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 976, 1 ]
Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean
Matrix.det_smul_inv_vecMul_eq_cramer_transpose
[ { "state_after": "no goals", "state_before": "l : Type ?u.364914\nm : Type u\nn : Type u'\nα : Type v\ninst✝² : Fintype n\ninst✝¹ : DecidableEq n\ninst✝ : CommRing α\nA✝ B A : Matrix n n α\nb : n → α\nh : IsUnit (det A)\n⊢ det A • vecMul b A⁻¹ = ↑(cramer Aᵀ) b", "tactic": "rw [← A⁻¹.transpose_transpose, vecMul_transpose, transpose_nonsing_inv, ← det_transpose,\n Aᵀ.det_smul_inv_mulVec_eq_cramer _ (isUnit_det_transpose A h)]" } ]
[ 615, 67 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 612, 1 ]
Mathlib/Data/Num/Lemmas.lean
Num.succ_to_nat
[]
[ 299, 17 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 298, 1 ]
Mathlib/LinearAlgebra/BilinearForm.lean
BilinForm.Nondegenerate.congr
[]
[ 1301, 85 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 1298, 1 ]
Mathlib/RingTheory/Ideal/QuotientOperations.lean
DoubleQuot.coe_quotLeftToQuotSupₐ
[]
[ 690, 6 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 689, 1 ]
Mathlib/Topology/SubsetProperties.lean
IsCompact.ne_univ
[]
[ 757, 29 ]
5a919533f110b7d76410134a237ee374f24eaaad
https://github.com/leanprover-community/mathlib4
[ 756, 1 ]