full_name
stringlengths 3
121
| state
stringlengths 7
9.32k
| tactic
stringlengths 3
5.35k
| target_state
stringlengths 7
19k
| url
stringclasses 1
value | commit
stringclasses 1
value | file_path
stringlengths 21
79
|
---|---|---|---|---|---|---|
ChainComplex.isIso_descOpcycles_iff
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ : K.d 1 0 ≫ φ = 0
⊢ ∀ (i : ℕ) (hx : (ComplexShape.down ℕ).prev 0 = i) (hφ : K.d i 0 ≫ φ = 0),
IsIso (HomologicalComplex.descOpcycles K φ i hx hφ) ↔ (ShortComplex.mk (K.d i 0) φ hφ).Exact ∧ Epi φ
|
rintro _ rfl hφ
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ✝ : K.d 1 0 ≫ φ = 0
hφ : K.d ((ComplexShape.down ℕ).prev 0) 0 ≫ φ = 0
⊢ IsIso (HomologicalComplex.descOpcycles K φ ((ComplexShape.down ℕ).prev 0) ⋯ hφ) ↔
(ShortComplex.mk (K.d ((ComplexShape.down ℕ).prev 0) 0) φ hφ).Exact ∧ Epi φ
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean
|
ChainComplex.isIso_descOpcycles_iff
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ✝ : K.d 1 0 ≫ φ = 0
hφ : K.d ((ComplexShape.down ℕ).prev 0) 0 ≫ φ = 0
⊢ IsIso (HomologicalComplex.descOpcycles K φ ((ComplexShape.down ℕ).prev 0) ⋯ hφ) ↔
(ShortComplex.mk (K.d ((ComplexShape.down ℕ).prev 0) 0) φ hφ).Exact ∧ Epi φ
|
let α : K.sc 0 ⟶ <a>CategoryTheory.ShortComplex.mk</a> (0 : X ⟶ X) (0 : X ⟶ X) (by simp) := { τ₁ := 0 τ₂ := φ τ₃ := 0 }
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ✝ : K.d 1 0 ≫ φ = 0
hφ : K.d ((ComplexShape.down ℕ).prev 0) 0 ≫ φ = 0
α : HomologicalComplex.sc K 0 ⟶ ShortComplex.mk 0 0 ⋯ := { τ₁ := 0, τ₂ := φ, τ₃ := 0, comm₁₂ := ⋯, comm₂₃ := ⋯ }
⊢ IsIso (HomologicalComplex.descOpcycles K φ ((ComplexShape.down ℕ).prev 0) ⋯ hφ) ↔
(ShortComplex.mk (K.d ((ComplexShape.down ℕ).prev 0) 0) φ hφ).Exact ∧ Epi φ
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean
|
ChainComplex.isIso_descOpcycles_iff
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ✝ : K.d 1 0 ≫ φ = 0
hφ : K.d ((ComplexShape.down ℕ).prev 0) 0 ≫ φ = 0
α : HomologicalComplex.sc K 0 ⟶ ShortComplex.mk 0 0 ⋯ := { τ₁ := 0, τ₂ := φ, τ₃ := 0, comm₁₂ := ⋯, comm₂₃ := ⋯ }
⊢ IsIso (HomologicalComplex.descOpcycles K φ ((ComplexShape.down ℕ).prev 0) ⋯ hφ) ↔
(ShortComplex.mk (K.d ((ComplexShape.down ℕ).prev 0) 0) φ hφ).Exact ∧ Epi φ
|
exact (<a>CategoryTheory.ShortComplex.quasiIso_iff_isIso_descOpcycles</a> α (by simp) <a>rfl</a> <a>rfl</a>).symm.trans (<a>CategoryTheory.ShortComplex.quasiIso_iff_of_zeros'</a> α (by simp) <a>rfl</a> <a>rfl</a>)
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean
|
ChainComplex.isIso_descOpcycles_iff
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ : K.d 1 0 ≫ φ = 0
this :
∀ (i : ℕ) (hx : (ComplexShape.down ℕ).prev 0 = i) (hφ : K.d i 0 ≫ φ = 0),
IsIso (HomologicalComplex.descOpcycles K φ i hx hφ) ↔ (ShortComplex.mk (K.d i 0) φ hφ).Exact ∧ Epi φ
⊢ (ComplexShape.down ℕ).prev 0 = 1
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean
|
ChainComplex.isIso_descOpcycles_iff
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ✝ : K.d 1 0 ≫ φ = 0
hφ : K.d ((ComplexShape.down ℕ).prev 0) 0 ≫ φ = 0
⊢ 0 ≫ 0 = 0
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean
|
ChainComplex.isIso_descOpcycles_iff
|
C : Type u_1
inst✝² : Category.{u_2, u_1} C
inst✝¹ : Abelian C
K : ChainComplex C ℕ
X : C
φ : K.X 0 ⟶ X
inst✝ : HomologicalComplex.HasHomology K 0
hφ✝ : K.d 1 0 ≫ φ = 0
hφ : K.d ((ComplexShape.down ℕ).prev 0) 0 ≫ φ = 0
α : HomologicalComplex.sc K 0 ⟶ ShortComplex.mk 0 0 ⋯ := { τ₁ := 0, τ₂ := φ, τ₃ := 0, comm₁₂ := ⋯, comm₂₃ := ⋯ }
⊢ (HomologicalComplex.sc K 0).g = 0
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean
|
Sum.liftRel_inl_inl
|
α✝ : Type u_1
γ✝ : Type u_2
r : α✝ → γ✝ → Prop
β✝ : Type u_3
δ✝ : Type u_4
s : β✝ → δ✝ → Prop
a : α✝
c : γ✝
h : LiftRel r s (inl a) (inl c)
⊢ r a c
|
cases h
|
case inl
α✝ : Type u_1
γ✝ : Type u_2
r : α✝ → γ✝ → Prop
β✝ : Type u_3
δ✝ : Type u_4
s : β✝ → δ✝ → Prop
a : α✝
c : γ✝
a✝ : r a c
⊢ r a c
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
.lake/packages/batteries/Batteries/Data/Sum/Basic.lean
|
Sum.liftRel_inl_inl
|
case inl
α✝ : Type u_1
γ✝ : Type u_2
r : α✝ → γ✝ → Prop
β✝ : Type u_3
δ✝ : Type u_4
s : β✝ → δ✝ → Prop
a : α✝
c : γ✝
a✝ : r a c
⊢ r a c
|
assumption
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
.lake/packages/batteries/Batteries/Data/Sum/Basic.lean
|
SetTheory.PGame.short_birthday
|
case mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
⊢ ∀ [inst : (mk xl xr xL xR).Short], (mk xl xr xL xR).birthday < Ordinal.omega
|
intro hs
|
case mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
hs : (mk xl xr xL xR).Short
⊢ (mk xl xr xL xR).birthday < Ordinal.omega
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
hs : (mk xl xr xL xR).Short
⊢ (mk xl xr xL xR).birthday < Ordinal.omega
|
rcases hs with ⟨sL, sR⟩
|
case mk.mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (mk xl xr xL xR).birthday < Ordinal.omega
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (mk xl xr xL xR).birthday < Ordinal.omega
|
rw [<a>SetTheory.PGame.birthday</a>, <a>max_lt_iff</a>]
|
case mk.mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xL i).birthday) < Ordinal.omega ∧ (Ordinal.lsub fun i => (xR i).birthday) < Ordinal.omega
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xL i).birthday) < Ordinal.omega ∧ (Ordinal.lsub fun i => (xR i).birthday) < Ordinal.omega
|
constructor
|
case mk.mk.left
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xL i).birthday) < Ordinal.omega
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xR i).birthday) < Ordinal.omega
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk.left
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xL i).birthday) < Ordinal.omega
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xR i).birthday) < Ordinal.omega
|
all_goals rw [← <a>Cardinal.ord_aleph0</a>] refine <a>Cardinal.lsub_lt_ord_of_isRegular</a>.{u, u} <a>Cardinal.isRegular_aleph0</a> (<a>Cardinal.lt_aleph0_of_finite</a> _) fun i => ?_ rw [<a>Cardinal.ord_aleph0</a>]
|
case mk.mk.left
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xl
⊢ (xL i).birthday < Ordinal.omega
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xr
⊢ (xR i).birthday < Ordinal.omega
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xR i).birthday) < Ordinal.omega
|
rw [← <a>Cardinal.ord_aleph0</a>]
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xR i).birthday) < Cardinal.aleph0.ord
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
⊢ (Ordinal.lsub fun i => (xR i).birthday) < Cardinal.aleph0.ord
|
refine <a>Cardinal.lsub_lt_ord_of_isRegular</a>.{u, u} <a>Cardinal.isRegular_aleph0</a> (<a>Cardinal.lt_aleph0_of_finite</a> _) fun i => ?_
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xr
⊢ (xR i).birthday < Cardinal.aleph0.ord
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xr
⊢ (xR i).birthday < Cardinal.aleph0.ord
|
rw [<a>Cardinal.ord_aleph0</a>]
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xr
⊢ (xR i).birthday < Ordinal.omega
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk.left
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xl
⊢ (xL i).birthday < Ordinal.omega
|
apply ihl
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
SetTheory.PGame.short_birthday
|
case mk.mk.right
xl xr : Type u
xL : xl → PGame
xR : xr → PGame
ihl : ∀ (a : xl) [inst : (xL a).Short], (xL a).birthday < Ordinal.omega
ihr : ∀ (a : xr) [inst : (xR a).Short], (xR a).birthday < Ordinal.omega
inst✝¹ : Fintype xl
inst✝ : Fintype xr
sL : (i : xl) → (xL i).Short
sR : (j : xr) → (xR j).Short
i : xr
⊢ (xR i).birthday < Ordinal.omega
|
apply ihr
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Game/Short.lean
|
Cardinal.two_le_iff'
|
α β : Type u
c : Cardinal.{?u.235324}
x : α
⊢ 2 ≤ #α ↔ ∃ y, y ≠ x
|
rw [<a>Cardinal.two_le_iff</a>, ← <a>nontrivial_iff</a>, <a>nontrivial_iff_exists_ne</a> x]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Cardinal/Basic.lean
|
Submonoid.LocalizationMap.map_map
|
M : Type u_1
inst✝⁵ : CommMonoid M
S : Submonoid M
N : Type u_2
inst✝⁴ : CommMonoid N
P : Type u_3
inst✝³ : CommMonoid P
f : S.LocalizationMap N
g : M →* P
hg : ∀ (y : ↥S), IsUnit (g ↑y)
T : Submonoid P
hy : ∀ (y : ↥S), g ↑y ∈ T
Q : Type u_4
inst✝² : CommMonoid Q
k : T.LocalizationMap Q
A : Type u_5
inst✝¹ : CommMonoid A
U : Submonoid A
R : Type u_6
inst✝ : CommMonoid R
j : U.LocalizationMap R
l : P →* A
hl : ∀ (w : ↥T), l ↑w ∈ U
x : N
⊢ (k.map hl j) ((f.map hy k) x) = (f.map ⋯ j) x
|
rw [← @<a>Submonoid.LocalizationMap.map_comp_map</a> M _ S N _ P _ f g T hy Q _ k A _ U R _ j l hl]
|
M : Type u_1
inst✝⁵ : CommMonoid M
S : Submonoid M
N : Type u_2
inst✝⁴ : CommMonoid N
P : Type u_3
inst✝³ : CommMonoid P
f : S.LocalizationMap N
g : M →* P
hg : ∀ (y : ↥S), IsUnit (g ↑y)
T : Submonoid P
hy : ∀ (y : ↥S), g ↑y ∈ T
Q : Type u_4
inst✝² : CommMonoid Q
k : T.LocalizationMap Q
A : Type u_5
inst✝¹ : CommMonoid A
U : Submonoid A
R : Type u_6
inst✝ : CommMonoid R
j : U.LocalizationMap R
l : P →* A
hl : ∀ (w : ↥T), l ↑w ∈ U
x : N
⊢ (k.map hl j) ((f.map hy k) x) = ((k.map hl j).comp (f.map hy k)) x
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/GroupTheory/MonoidLocalization.lean
|
Submonoid.LocalizationMap.map_map
|
M : Type u_1
inst✝⁵ : CommMonoid M
S : Submonoid M
N : Type u_2
inst✝⁴ : CommMonoid N
P : Type u_3
inst✝³ : CommMonoid P
f : S.LocalizationMap N
g : M →* P
hg : ∀ (y : ↥S), IsUnit (g ↑y)
T : Submonoid P
hy : ∀ (y : ↥S), g ↑y ∈ T
Q : Type u_4
inst✝² : CommMonoid Q
k : T.LocalizationMap Q
A : Type u_5
inst✝¹ : CommMonoid A
U : Submonoid A
R : Type u_6
inst✝ : CommMonoid R
j : U.LocalizationMap R
l : P →* A
hl : ∀ (w : ↥T), l ↑w ∈ U
x : N
⊢ (k.map hl j) ((f.map hy k) x) = ((k.map hl j).comp (f.map hy k)) x
|
simp only [<a>MonoidHom.coe_comp</a>, <a>Function.comp_apply</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/GroupTheory/MonoidLocalization.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q
inst✝ : Module S Q
e : M ≃ₗ[R] N
⊢ IsBaseChange R ↑e
|
apply <a>IsBaseChange.of_lift_unique</a>
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q
inst✝ : Module S Q
e : M ≃ₗ[R] N
⊢ ∀ (Q : Type (max v₁ v₂ u_1)) [inst : AddCommMonoid Q] [inst_1 : Module R Q] [inst_2 : Module R Q]
[inst_3 : IsScalarTower R R Q] (g : M →ₗ[R] Q), ∃! g', ↑R g' ∘ₗ ↑e = g
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q
inst✝ : Module S Q
e : M ≃ₗ[R] N
⊢ ∀ (Q : Type (max v₁ v₂ u_1)) [inst : AddCommMonoid Q] [inst_1 : Module R Q] [inst_2 : Module R Q]
[inst_3 : IsScalarTower R R Q] (g : M →ₗ[R] Q), ∃! g', ↑R g' ∘ₗ ↑e = g
|
intro Q I₁ I₂ I₃ I₄ g
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
⊢ ∃! g', ↑R g' ∘ₗ ↑e = g
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
⊢ ∃! g', ↑R g' ∘ₗ ↑e = g
|
have : I₂ = I₃ := by ext r q show (by let _ := I₂; exact r • q) = (by let _ := I₃; exact r • q) dsimp rw [← <a>one_smul</a> R q, <a>smul_smul</a>, ← @<a>smul_assoc</a> _ _ _ (<a>id</a> _) (<a>id</a> _) (<a>id</a> _) I₄, <a>smul_eq_mul</a>]
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
this : I₂ = I₃
⊢ ∃! g', ↑R g' ∘ₗ ↑e = g
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
this : I₂ = I₃
⊢ ∃! g', ↑R g' ∘ₗ ↑e = g
|
cases this
|
case h.refl
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
⊢ ∃! g', ↑R g' ∘ₗ ↑e = g
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h.refl
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
⊢ ∃! g', ↑R g' ∘ₗ ↑e = g
|
refine ⟨g.comp e.symm.toLinearMap, by ext simp, ?_⟩
|
case h.refl
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
⊢ ∀ (y : N →ₗ[R] Q), (fun g' => ↑R g' ∘ₗ ↑e = g) y → y = g ∘ₗ ↑e.symm
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h.refl
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
⊢ ∀ (y : N →ₗ[R] Q), (fun g' => ↑R g' ∘ₗ ↑e = g) y → y = g ∘ₗ ↑e.symm
|
rintro y (rfl : _ = _)
|
case h.refl
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
I₄ : IsScalarTower R R Q
y : N →ₗ[R] Q
⊢ y = (↑R y ∘ₗ ↑e) ∘ₗ ↑e.symm
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h.refl
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
I₄ : IsScalarTower R R Q
y : N →ₗ[R] Q
⊢ y = (↑R y ∘ₗ ↑e) ∘ₗ ↑e.symm
|
ext
|
case h.refl.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
I₄ : IsScalarTower R R Q
y : N →ₗ[R] Q
x✝ : N
⊢ y x✝ = ((↑R y ∘ₗ ↑e) ∘ₗ ↑e.symm) x✝
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h.refl.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
I₄ : IsScalarTower R R Q
y : N →ₗ[R] Q
x✝ : N
⊢ y x✝ = ((↑R y ∘ₗ ↑e) ∘ₗ ↑e.symm) x✝
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
⊢ I₂ = I₃
|
ext r q
|
case smul.h.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ SMul.smul r q = SMul.smul r q
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case smul.h.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ SMul.smul r q = SMul.smul r q
|
show (by let _ := I₂; exact r • q) = (by let _ := I₃; exact r • q)
|
case smul.h.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ (let x := I₂;
r • q) =
let x := I₃;
r • q
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case smul.h.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ (let x := I₂;
r • q) =
let x := I₃;
r • q
|
dsimp
|
case smul.h.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ r • q = r • q
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case smul.h.h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ r • q = r • q
|
rw [← <a>one_smul</a> R q, <a>smul_smul</a>, ← @<a>smul_assoc</a> _ _ _ (<a>id</a> _) (<a>id</a> _) (<a>id</a> _) I₄, <a>smul_eq_mul</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ ?m.349239
|
let _ := I₂
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
x✝ : Module R Q := I₂
⊢ ?m.349239
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
x✝ : Module R Q := I₂
⊢ ?m.349239
|
exact r • q
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
⊢ Q
|
let _ := I₃
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
x✝ : Module R Q := I₃
⊢ Q
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ I₃ : Module R Q
I₄ : IsScalarTower R R Q
g : M →ₗ[R] Q
r : R
q : Q
x✝ : Module R Q := I₃
⊢ Q
|
exact r • q
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
⊢ (fun g' => ↑R g' ∘ₗ ↑e = g) (g ∘ₗ ↑e.symm)
|
ext
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
x✝ : M
⊢ (↑R (g ∘ₗ ↑e.symm) ∘ₗ ↑e) x✝ = g x✝
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
IsBaseChange.ofEquiv
|
case h
R : Type u_1
M : Type v₁
N : Type v₂
S : Type v₃
inst✝¹² : AddCommMonoid M
inst✝¹¹ : AddCommMonoid N
inst✝¹⁰ : CommSemiring R
inst✝⁹ : CommSemiring S
inst✝⁸ : Algebra R S
inst✝⁷ : Module R M
inst✝⁶ : Module R N
inst✝⁵ : Module S N
inst✝⁴ : IsScalarTower R S N
f : M →ₗ[R] N
h : IsBaseChange S f
P : Type u_2
Q✝ : Type u_3
inst✝³ : AddCommMonoid P
inst✝² : Module R P
inst✝¹ : AddCommMonoid Q✝
inst✝ : Module S Q✝
e : M ≃ₗ[R] N
Q : Type (max v₁ v₂ u_1)
I₁ : AddCommMonoid Q
I₂ : Module R Q
g : M →ₗ[R] Q
I₄ : IsScalarTower R R Q
x✝ : M
⊢ (↑R (g ∘ₗ ↑e.symm) ∘ₗ ↑e) x✝ = g x✝
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/RingTheory/IsTensorProduct.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
⊢ IsIdempotentComplete C
|
refine ⟨?_⟩
|
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
⊢ ∀ (X : C) (p : X ⟶ X), p ≫ p = p → ∃ Y i e, i ≫ e = 𝟙 Y ∧ e ≫ i = p
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
⊢ ∀ (X : C) (p : X ⟶ X), p ≫ p = p → ∃ Y i e, i ≫ e = 𝟙 Y ∧ e ≫ i = p
|
intro X p hp
|
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
⊢ ∃ Y i e, i ≫ e = 𝟙 Y ∧ e ≫ i = p
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
⊢ ∃ Y i e, i ≫ e = 𝟙 Y ∧ e ≫ i = p
|
rcases <a>CategoryTheory.IsIdempotentComplete.idempotents_split</a> (<a>Opposite.op</a> X) p.op (by rw [← <a>CategoryTheory.op_comp</a>, hp]) with ⟨Y, i, e, ⟨h₁, h₂⟩⟩
|
case intro.intro.intro.intro
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ ∃ Y i e, i ≫ e = 𝟙 Y ∧ e ≫ i = p
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
case intro.intro.intro.intro
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ ∃ Y i e, i ≫ e = 𝟙 Y ∧ e ≫ i = p
|
use Y.unop, e.unop, i.unop
|
case h
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ e.unop ≫ i.unop = 𝟙 Y.unop ∧ i.unop ≫ e.unop = p
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
case h
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ e.unop ≫ i.unop = 𝟙 Y.unop ∧ i.unop ≫ e.unop = p
|
constructor
|
case h.left
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ e.unop ≫ i.unop = 𝟙 Y.unop
case h.right
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ i.unop ≫ e.unop = p
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
⊢ p.op ≫ p.op = p.op
|
rw [← <a>CategoryTheory.op_comp</a>, hp]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
case h.left
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ e.unop ≫ i.unop = 𝟙 Y.unop
|
simp only [← <a>CategoryTheory.unop_comp</a>, h₁]
|
case h.left
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ (𝟙 Y).unop = 𝟙 Y.unop
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
case h.left
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ (𝟙 Y).unop = 𝟙 Y.unop
|
rfl
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
case h.right
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ i.unop ≫ e.unop = p
|
simp only [← <a>CategoryTheory.unop_comp</a>, h₂]
|
case h.right
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ p.op.unop = p
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
CategoryTheory.Idempotents.isIdempotentComplete_of_isIdempotentComplete_opposite
|
case h.right
C : Type u_1
inst✝ : Category.{u_2, u_1} C
h : IsIdempotentComplete Cᵒᵖ
X : C
p : X ⟶ X
hp : p ≫ p = p
Y : Cᵒᵖ
i : Y ⟶ { unop := X }
e : { unop := X } ⟶ Y
h₁ : i ≫ e = 𝟙 Y
h₂ : e ≫ i = p.op
⊢ p.op.unop = p
|
rfl
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Idempotents/Basic.lean
|
Mathlib.Meta.NormNum.isRat_inv_zero
|
α : Type u_1
inst✝ : DivisionRing α
⊢ (↑0)⁻¹ = ↑0
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Tactic/NormNum/Inv.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ ↑(approx i f n) a = (Finset.range n).sup fun k => if i k ≤ f a then i k else 0
|
dsimp only [<a>MeasureTheory.SimpleFunc.approx</a>]
|
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ ↑((Finset.range n).sup fun k => (const α (i k)).restrict {a | i k ≤ f a}) a =
(Finset.range n).sup fun k => if i k ≤ f a then i k else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ ↑((Finset.range n).sup fun k => (const α (i k)).restrict {a | i k ≤ f a}) a =
(Finset.range n).sup fun k => if i k ≤ f a then i k else 0
|
rw [<a>MeasureTheory.SimpleFunc.finset_sup_apply</a>]
|
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ ((Finset.range n).sup fun c => ↑((const α (i c)).restrict {a | i c ≤ f a}) a) =
(Finset.range n).sup fun k => if i k ≤ f a then i k else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ ((Finset.range n).sup fun c => ↑((const α (i c)).restrict {a | i c ≤ f a}) a) =
(Finset.range n).sup fun k => if i k ≤ f a then i k else 0
|
congr
|
case e_f
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ (fun c => ↑((const α (i c)).restrict {a | i c ≤ f a}) a) = fun k => if i k ≤ f a then i k else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
case e_f
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
⊢ (fun c => ↑((const α (i c)).restrict {a | i c ≤ f a}) a) = fun k => if i k ≤ f a then i k else 0
|
funext k
|
case e_f.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
k : ℕ
⊢ ↑((const α (i k)).restrict {a | i k ≤ f a}) a = if i k ≤ f a then i k else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
case e_f.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
k : ℕ
⊢ ↑((const α (i k)).restrict {a | i k ≤ f a}) a = if i k ≤ f a then i k else 0
|
rw [<a>MeasureTheory.SimpleFunc.restrict_apply</a>]
|
case e_f.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
k : ℕ
⊢ {a | i k ≤ f a}.indicator (↑(const α (i k))) a = if i k ≤ f a then i k else 0
case e_f.h.hs
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
k : ℕ
⊢ MeasurableSet {a | i k ≤ f a}
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
case e_f.h
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
k : ℕ
⊢ {a | i k ≤ f a}.indicator (↑(const α (i k))) a = if i k ≤ f a then i k else 0
|
simp only [<a>MeasureTheory.SimpleFunc.coe_const</a>, <a>Set.mem_setOf_eq</a>, <a>Set.indicator_apply</a>, <a>Function.const_apply</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
MeasureTheory.SimpleFunc.approx_apply
|
case e_f.h.hs
α : Type u_1
β : Type u_2
γ : Type u_3
δ : Type u_4
inst✝⁷ : MeasurableSpace α
K : Type u_5
inst✝⁶ : SemilatticeSup β
inst✝⁵ : OrderBot β
inst✝⁴ : Zero β
inst✝³ : TopologicalSpace β
inst✝² : OrderClosedTopology β
inst✝¹ : MeasurableSpace β
inst✝ : OpensMeasurableSpace β
i : ℕ → β
f : α → β
n : ℕ
a : α
hf : Measurable f
k : ℕ
⊢ MeasurableSet {a | i k ≤ f a}
|
exact hf <a>measurableSet_Ici</a>
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Function/SimpleFunc.lean
|
InnerProductSpace.Core.inner_self_im
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝² : _root_.RCLike 𝕜
inst✝¹ : AddCommGroup F
inst✝ : Module 𝕜 F
c : Core 𝕜 F
x : F
⊢ im ⟪x, x⟫_𝕜 = 0
|
rw [← @<a>RCLike.ofReal_inj</a> 𝕜, <a>RCLike.im_eq_conj_sub</a>]
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝² : _root_.RCLike 𝕜
inst✝¹ : AddCommGroup F
inst✝ : Module 𝕜 F
c : Core 𝕜 F
x : F
⊢ I * ((starRingEnd 𝕜) ⟪x, x⟫_𝕜 - ⟪x, x⟫_𝕜) / 2 = ↑0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Analysis/InnerProductSpace/Basic.lean
|
InnerProductSpace.Core.inner_self_im
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝² : _root_.RCLike 𝕜
inst✝¹ : AddCommGroup F
inst✝ : Module 𝕜 F
c : Core 𝕜 F
x : F
⊢ I * ((starRingEnd 𝕜) ⟪x, x⟫_𝕜 - ⟪x, x⟫_𝕜) / 2 = ↑0
|
simp [<a>InnerProductSpace.Core.inner_conj_symm</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Analysis/InnerProductSpace/Basic.lean
|
zpow_neg_mul_zpow_self
|
α : Type u_1
M₀ : Type u_2
G₀ : Type u_3
M₀' : Type u_4
G₀' : Type u_5
F : Type u_6
F' : Type u_7
inst✝¹ : MonoidWithZero M₀
inst✝ : GroupWithZero G₀
a b c d : G₀
m n✝ : ℕ
n : ℤ
ha : a ≠ 0
⊢ a ^ (-n) * a ^ n = 1
|
rw [<a>zpow_neg</a>]
|
α : Type u_1
M₀ : Type u_2
G₀ : Type u_3
M₀' : Type u_4
G₀' : Type u_5
F : Type u_6
F' : Type u_7
inst✝¹ : MonoidWithZero M₀
inst✝ : GroupWithZero G₀
a b c d : G₀
m n✝ : ℕ
n : ℤ
ha : a ≠ 0
⊢ (a ^ n)⁻¹ * a ^ n = 1
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/GroupWithZero/Units/Basic.lean
|
zpow_neg_mul_zpow_self
|
α : Type u_1
M₀ : Type u_2
G₀ : Type u_3
M₀' : Type u_4
G₀' : Type u_5
F : Type u_6
F' : Type u_7
inst✝¹ : MonoidWithZero M₀
inst✝ : GroupWithZero G₀
a b c d : G₀
m n✝ : ℕ
n : ℤ
ha : a ≠ 0
⊢ (a ^ n)⁻¹ * a ^ n = 1
|
exact <a>inv_mul_cancel</a> (<a>zpow_ne_zero</a> n ha)
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Algebra/GroupWithZero/Units/Basic.lean
|
OrthogonalFamily.inner_right_fintype
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝⁷ : _root_.RCLike 𝕜
inst✝⁶ : NormedAddCommGroup E
inst✝⁵ : InnerProductSpace 𝕜 E
inst✝⁴ : NormedAddCommGroup F
inst✝³ : InnerProductSpace ℝ F
ι : Type u_4
G : ι → Type u_5
inst✝² : (i : ι) → NormedAddCommGroup (G i)
inst✝¹ : (i : ι) → InnerProductSpace 𝕜 (G i)
V : (i : ι) → G i →ₗᵢ[𝕜] E
hV : OrthogonalFamily 𝕜 G V
dec_V : (i : ι) → (x : G i) → Decidable (x ≠ 0)
inst✝ : Fintype ι
l : (i : ι) → G i
i : ι
v : G i
⊢ ⟪(V i) v, ∑ j : ι, (V j) (l j)⟫_𝕜 = ⟪v, l i⟫_𝕜
|
classical calc ⟪V i v, ∑ j : ι, V j (l j)⟫ = ∑ j : ι, ⟪V i v, V j (l j)⟫ := by rw [<a>inner_sum</a>] _ = ∑ <a>Finset.univ</a>, <a>ite</a> (i = j) ⟪V i v, V j (l j)⟫ 0 := (<a>congr_arg</a> (<a>Finset.sum</a> <a>Finset.univ</a>) <| <a>funext</a> fun j => hV.eq_ite v (l j)) _ = ⟪v, l i⟫ := by simp only [<a>Finset.sum_ite_eq</a>, <a>Finset.mem_univ</a>, (V i).<a>LinearIsometry.inner_map_map</a>, <a>if_true</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Analysis/InnerProductSpace/Basic.lean
|
OrthogonalFamily.inner_right_fintype
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝⁷ : _root_.RCLike 𝕜
inst✝⁶ : NormedAddCommGroup E
inst✝⁵ : InnerProductSpace 𝕜 E
inst✝⁴ : NormedAddCommGroup F
inst✝³ : InnerProductSpace ℝ F
ι : Type u_4
G : ι → Type u_5
inst✝² : (i : ι) → NormedAddCommGroup (G i)
inst✝¹ : (i : ι) → InnerProductSpace 𝕜 (G i)
V : (i : ι) → G i →ₗᵢ[𝕜] E
hV : OrthogonalFamily 𝕜 G V
dec_V : (i : ι) → (x : G i) → Decidable (x ≠ 0)
inst✝ : Fintype ι
l : (i : ι) → G i
i : ι
v : G i
⊢ ⟪(V i) v, ∑ j : ι, (V j) (l j)⟫_𝕜 = ⟪v, l i⟫_𝕜
|
calc ⟪V i v, ∑ j : ι, V j (l j)⟫ = ∑ j : ι, ⟪V i v, V j (l j)⟫ := by rw [<a>inner_sum</a>] _ = ∑ <a>Finset.univ</a>, <a>ite</a> (i = j) ⟪V i v, V j (l j)⟫ 0 := (<a>congr_arg</a> (<a>Finset.sum</a> <a>Finset.univ</a>) <| <a>funext</a> fun j => hV.eq_ite v (l j)) _ = ⟪v, l i⟫ := by simp only [<a>Finset.sum_ite_eq</a>, <a>Finset.mem_univ</a>, (V i).<a>LinearIsometry.inner_map_map</a>, <a>if_true</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Analysis/InnerProductSpace/Basic.lean
|
OrthogonalFamily.inner_right_fintype
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝⁷ : _root_.RCLike 𝕜
inst✝⁶ : NormedAddCommGroup E
inst✝⁵ : InnerProductSpace 𝕜 E
inst✝⁴ : NormedAddCommGroup F
inst✝³ : InnerProductSpace ℝ F
ι : Type u_4
G : ι → Type u_5
inst✝² : (i : ι) → NormedAddCommGroup (G i)
inst✝¹ : (i : ι) → InnerProductSpace 𝕜 (G i)
V : (i : ι) → G i →ₗᵢ[𝕜] E
hV : OrthogonalFamily 𝕜 G V
dec_V : (i : ι) → (x : G i) → Decidable (x ≠ 0)
inst✝ : Fintype ι
l : (i : ι) → G i
i : ι
v : G i
⊢ ⟪(V i) v, ∑ j : ι, (V j) (l j)⟫_𝕜 = ∑ j : ι, ⟪(V i) v, (V j) (l j)⟫_𝕜
|
rw [<a>inner_sum</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Analysis/InnerProductSpace/Basic.lean
|
OrthogonalFamily.inner_right_fintype
|
𝕜 : Type u_1
E : Type u_2
F : Type u_3
inst✝⁷ : _root_.RCLike 𝕜
inst✝⁶ : NormedAddCommGroup E
inst✝⁵ : InnerProductSpace 𝕜 E
inst✝⁴ : NormedAddCommGroup F
inst✝³ : InnerProductSpace ℝ F
ι : Type u_4
G : ι → Type u_5
inst✝² : (i : ι) → NormedAddCommGroup (G i)
inst✝¹ : (i : ι) → InnerProductSpace 𝕜 (G i)
V : (i : ι) → G i →ₗᵢ[𝕜] E
hV : OrthogonalFamily 𝕜 G V
dec_V : (i : ι) → (x : G i) → Decidable (x ≠ 0)
inst✝ : Fintype ι
l : (i : ι) → G i
i : ι
v : G i
⊢ (∑ j : ι, if i = j then ⟪(V i) v, (V j) (l j)⟫_𝕜 else 0) = ⟪v, l i⟫_𝕜
|
simp only [<a>Finset.sum_ite_eq</a>, <a>Finset.mem_univ</a>, (V i).<a>LinearIsometry.inner_map_map</a>, <a>if_true</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Analysis/InnerProductSpace/Basic.lean
|
Filter.image_mem_of_mem_comap
|
α : Type u
β : Type v
γ : Type w
δ : Type u_1
ι : Sort x
l f✝ f₁ f₂ : Filter α
g g₁ g₂ : Filter β
m : α → β
m' : β → γ
s : Set α
t : Set β
f : Filter α
c : β → α
h : range c ∈ f
W : Set β
W_in : W ∈ comap c f
⊢ c '' W ∈ f
|
rw [← <a>Filter.map_comap_of_mem</a> h]
|
α : Type u
β : Type v
γ : Type w
δ : Type u_1
ι : Sort x
l f✝ f₁ f₂ : Filter α
g g₁ g₂ : Filter β
m : α → β
m' : β → γ
s : Set α
t : Set β
f : Filter α
c : β → α
h : range c ∈ f
W : Set β
W_in : W ∈ comap c f
⊢ c '' W ∈ map c (comap c f)
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Order/Filter/Basic.lean
|
Filter.image_mem_of_mem_comap
|
α : Type u
β : Type v
γ : Type w
δ : Type u_1
ι : Sort x
l f✝ f₁ f₂ : Filter α
g g₁ g₂ : Filter β
m : α → β
m' : β → γ
s : Set α
t : Set β
f : Filter α
c : β → α
h : range c ∈ f
W : Set β
W_in : W ∈ comap c f
⊢ c '' W ∈ map c (comap c f)
|
exact <a>Filter.image_mem_map</a> W_in
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Order/Filter/Basic.lean
|
CategoryTheory.Subobject.factors_left_of_factors_add
|
C : Type u₁
inst✝² : Category.{v₁, u₁} C
X✝ Y✝ Z : C
D : Type u₂
inst✝¹ : Category.{v₂, u₂} D
inst✝ : Preadditive C
X Y : C
P : Subobject Y
f g : X ⟶ Y
w : P.Factors (f + g)
wg : P.Factors g
⊢ (P.factorThru (f + g) w - P.factorThru g wg) ≫ (representative.obj P).arrow = f
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Subobject/FactorThru.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h : d₁ ≤ d₂
s : Set X
⊢ μH[d₂] s ≤ μH[d₁] s
|
rcases h.eq_or_lt with (rfl | h)
|
case inl
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ : ℝ
s : Set X
h : d₁ ≤ d₁
⊢ μH[d₁] s ≤ μH[d₁] s
case inr
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
⊢ μH[d₂] s ≤ μH[d₁] s
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
case inr
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
⊢ μH[d₂] s ≤ μH[d₁] s
|
cases' <a>MeasureTheory.Measure.hausdorffMeasure_zero_or_top</a> h s with hs hs
|
case inr.inl
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₂] s = 0
⊢ μH[d₂] s ≤ μH[d₁] s
case inr.inr
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₁] s = ⊤
⊢ μH[d₂] s ≤ μH[d₁] s
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
case inl
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ : ℝ
s : Set X
h : d₁ ≤ d₁
⊢ μH[d₁] s ≤ μH[d₁] s
|
exact <a>le_rfl</a>
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
case inr.inl
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₂] s = 0
⊢ μH[d₂] s ≤ μH[d₁] s
|
rw [hs]
|
case inr.inl
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₂] s = 0
⊢ 0 ≤ μH[d₁] s
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
case inr.inl
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₂] s = 0
⊢ 0 ≤ μH[d₁] s
|
exact <a>zero_le</a> _
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
case inr.inr
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₁] s = ⊤
⊢ μH[d₂] s ≤ μH[d₁] s
|
rw [hs]
|
case inr.inr
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₁] s = ⊤
⊢ μH[d₂] s ≤ ⊤
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
MeasureTheory.Measure.hausdorffMeasure_mono
|
case inr.inr
ι : Type u_1
X : Type u_2
Y : Type u_3
inst✝³ : EMetricSpace X
inst✝² : EMetricSpace Y
inst✝¹ : MeasurableSpace X
inst✝ : BorelSpace X
d₁ d₂ : ℝ
h✝ : d₁ ≤ d₂
s : Set X
h : d₁ < d₂
hs : μH[d₁] s = ⊤
⊢ μH[d₂] s ≤ ⊤
|
exact <a>le_top</a>
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/MeasureTheory/Measure/Hausdorff.lean
|
Multiset.mem_sup
|
F : Type u_1
α✝ : Type u_2
β✝ : Type u_3
γ : Type u_4
ι : Type u_5
κ : Type u_6
α : Type u_7
β : Type u_8
inst✝ : DecidableEq β
s : Finset α
f : α → Multiset β
x : β
⊢ x ∈ s.sup f ↔ ∃ v ∈ s, x ∈ f v
|
induction s using <a>Finset.cons_induction</a> <;> simp [*]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/Data/Finset/Lattice.lean
|
eval_minpolyDiv_of_aeval_eq_zero
|
R : Type u_2
K : Type ?u.52975
L : Type ?u.52978
S : Type u_1
inst✝⁷ : CommRing R
inst✝⁶ : Field K
inst✝⁵ : Field L
inst✝⁴ : CommRing S
inst✝³ : Algebra R S
inst✝² : Algebra K L
x : S
hx : IsIntegral R x
inst✝¹ : IsDomain S
inst✝ : DecidableEq S
y : S
hy : (aeval y) (minpoly R x) = 0
⊢ eval y (minpolyDiv R x) = if x = y then (aeval x) (derivative (minpoly R x)) else 0
|
rw [<a>Polynomial.eval</a>, <a>eval₂_minpolyDiv_of_eval₂_eq_zero</a>, <a>RingHom.id_apply</a>, <a>RingHom.id_apply</a>]
|
case hy
R : Type u_2
K : Type ?u.52975
L : Type ?u.52978
S : Type u_1
inst✝⁷ : CommRing R
inst✝⁶ : Field K
inst✝⁵ : Field L
inst✝⁴ : CommRing S
inst✝³ : Algebra R S
inst✝² : Algebra K L
x : S
hx : IsIntegral R x
inst✝¹ : IsDomain S
inst✝ : DecidableEq S
y : S
hy : (aeval y) (minpoly R x) = 0
⊢ eval₂ ((RingHom.id S).comp (algebraMap R S)) y (minpoly R x) = 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/FieldTheory/Minpoly/MinpolyDiv.lean
|
eval_minpolyDiv_of_aeval_eq_zero
|
case hy
R : Type u_2
K : Type ?u.52975
L : Type ?u.52978
S : Type u_1
inst✝⁷ : CommRing R
inst✝⁶ : Field K
inst✝⁵ : Field L
inst✝⁴ : CommRing S
inst✝³ : Algebra R S
inst✝² : Algebra K L
x : S
hx : IsIntegral R x
inst✝¹ : IsDomain S
inst✝ : DecidableEq S
y : S
hy : (aeval y) (minpoly R x) = 0
⊢ eval₂ ((RingHom.id S).comp (algebraMap R S)) y (minpoly R x) = 0
|
simpa [<a>Polynomial.aeval_def</a>] using hy
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/FieldTheory/Minpoly/MinpolyDiv.lean
|
sum_bernoulli
|
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ k ∈ range n, ↑(n.choose k) * bernoulli k = if n = 1 then 1 else 0
|
cases' n with n n
|
case zero
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
⊢ ∑ k ∈ range 0, ↑(Nat.choose 0 k) * bernoulli k = if 0 = 1 then 1 else 0
case succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ k ∈ range (n + 1), ↑((n + 1).choose k) * bernoulli k = if n + 1 = 1 then 1 else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ k ∈ range (n + 1), ↑((n + 1).choose k) * bernoulli k = if n + 1 = 1 then 1 else 0
|
cases' n with n n
|
case succ.zero
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
⊢ ∑ k ∈ range (0 + 1), ↑((0 + 1).choose k) * bernoulli k = if 0 + 1 = 1 then 1 else 0
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ k ∈ range (n + 1 + 1), ↑((n + 1 + 1).choose k) * bernoulli k = if n + 1 + 1 = 1 then 1 else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ k ∈ range (n + 1 + 1), ↑((n + 1 + 1).choose k) * bernoulli k = if n + 1 + 1 = 1 then 1 else 0
|
suffices (∑ i ∈ <a>Finset.range</a> n, ↑((n + 2).<a>Nat.choose</a> (i + 2)) * <a>bernoulli</a> (i + 2)) = n / 2 by simp only [this, <a>Finset.sum_range_succ'</a>, <a>Nat.cast_succ</a>, <a>bernoulli_one</a>, <a>bernoulli_zero</a>, <a>Nat.choose_one_right</a>, <a>mul_one</a>, <a>Nat.choose_zero_right</a>, <a>Nat.cast_zero</a>, <a>if_false</a>, <a>zero_add</a>, <a>Nat.succ_succ_ne_one</a>] ring
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
|
have f := <a>sum_bernoulli'</a> n.succ.succ
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f : ∑ k ∈ range n.succ.succ, ↑(n.succ.succ.choose k) * bernoulli' k = ↑n.succ.succ
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f : ∑ k ∈ range n.succ.succ, ↑(n.succ.succ.choose k) * bernoulli' k = ↑n.succ.succ
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
|
simp_rw [<a>Finset.sum_range_succ'</a>, <a>Nat.cast_succ</a>, ← <a>eq_sub_iff_add_eq</a>] at f
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
|
refine <a>Eq.trans</a> ?_ (<a>Eq.trans</a> f ?_)
|
case succ.succ.refine_1
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) =
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1)
case succ.succ.refine_2
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1) = ↑n / 2
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case zero
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
⊢ ∑ k ∈ range 0, ↑(Nat.choose 0 k) * bernoulli k = if 0 = 1 then 1 else 0
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.zero
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
⊢ ∑ k ∈ range (0 + 1), ↑((0 + 1).choose k) * bernoulli k = if 0 + 1 = 1 then 1 else 0
|
rw [<a>Finset.sum_range_one</a>]
|
case succ.zero
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
⊢ ↑((0 + 1).choose 0) * bernoulli 0 = if 0 + 1 = 1 then 1 else 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.zero
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
⊢ ↑((0 + 1).choose 0) * bernoulli 0 = if 0 + 1 = 1 then 1 else 0
|
simp
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
this : ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
⊢ ∑ k ∈ range (n + 1 + 1), ↑((n + 1 + 1).choose k) * bernoulli k = if n + 1 + 1 = 1 then 1 else 0
|
simp only [this, <a>Finset.sum_range_succ'</a>, <a>Nat.cast_succ</a>, <a>bernoulli_one</a>, <a>bernoulli_zero</a>, <a>Nat.choose_one_right</a>, <a>mul_one</a>, <a>Nat.choose_zero_right</a>, <a>Nat.cast_zero</a>, <a>if_false</a>, <a>zero_add</a>, <a>Nat.succ_succ_ne_one</a>]
|
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
this : ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
⊢ ↑n / 2 + (↑n + 1 + 1) * (-1 / 2) + 1 = 0
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
this : ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) = ↑n / 2
⊢ ↑n / 2 + (↑n + 1 + 1) * (-1 / 2) + 1 = 0
|
ring
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ.refine_1
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ∑ i ∈ range n, ↑((n + 2).choose (i + 2)) * bernoulli (i + 2) =
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1)
|
congr
|
case succ.succ.refine_1.e_f
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ (fun i => ↑((n + 2).choose (i + 2)) * bernoulli (i + 2)) = fun k =>
↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1)
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ.refine_1.e_f
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ (fun i => ↑((n + 2).choose (i + 2)) * bernoulli (i + 2)) = fun k =>
↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1)
|
funext x
|
case succ.succ.refine_1.e_f.h
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
x : ℕ
⊢ ↑((n + 2).choose (x + 2)) * bernoulli (x + 2) = ↑(n.succ.succ.choose (x + 1 + 1)) * bernoulli' (x + 1 + 1)
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ.refine_1.e_f.h
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
x : ℕ
⊢ ↑((n + 2).choose (x + 2)) * bernoulli (x + 2) = ↑(n.succ.succ.choose (x + 1 + 1)) * bernoulli' (x + 1 + 1)
|
rw [<a>bernoulli_eq_bernoulli'_of_ne_one</a> (<a>Nat.succ_ne_zero</a> x ∘ <a>Nat.succ.inj</a>)]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ.refine_2
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1) = ↑n / 2
|
simp only [<a>one_div</a>, <a>mul_one</a>, <a>bernoulli'_zero</a>, <a>Nat.cast_one</a>, <a>Nat.choose_zero_right</a>, <a>add_sub_cancel_right</a>, <a>zero_add</a>, <a>Nat.choose_one_right</a>, <a>Nat.cast_succ</a>, <a>Nat.cast_add</a>, <a>Nat.cast_one</a>, <a>bernoulli'_one</a>, <a>one_div</a>]
|
case succ.succ.refine_2
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ↑n + 1 + 1 - (↑0 + 1) - (↑n + 1 + 1) * 2⁻¹ = ↑n / 2
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
sum_bernoulli
|
case succ.succ.refine_2
A : Type u_1
inst✝¹ : CommRing A
inst✝ : Algebra ℚ A
n : ℕ
f :
∑ k ∈ range n, ↑(n.succ.succ.choose (k + 1 + 1)) * bernoulli' (k + 1 + 1) =
↑n + 1 + 1 - ↑(n.succ.succ.choose 0) * bernoulli' 0 - ↑(n.succ.succ.choose (0 + 1)) * bernoulli' (0 + 1)
⊢ ↑n + 1 + 1 - (↑0 + 1) - (↑n + 1 + 1) * 2⁻¹ = ↑n / 2
|
ring
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/NumberTheory/Bernoulli.lean
|
CategoryTheory.braiding_rightUnitor
|
C : Type u₁
inst✝² : Category.{v₁, u₁} C
inst✝¹ : MonoidalCategory C
inst✝ : BraidedCategory C
X : C
⊢ (β_ (𝟙_ C) X).hom ≫ (ρ_ X).hom = (λ_ X).hom
|
rw [← <a>CategoryTheory.MonoidalCategory.whiskerLeft_iff</a>, <a>CategoryTheory.MonoidalCategory.whiskerLeft_comp</a>, <a>CategoryTheory.braiding_rightUnitor_aux₂</a>]
|
no goals
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean
|
Ordinal.exists_fundamental_sequence
|
α : Type u_1
r : α → α → Prop
a : Ordinal.{u}
⊢ ∃ f, a.IsFundamentalSequence a.cof.ord f
|
suffices h : ∃ o f, <a>Ordinal.IsFundamentalSequence</a> a o f by rcases h with ⟨o, f, hf⟩ exact ⟨_, hf.ord_cof⟩
|
α : Type u_1
r : α → α → Prop
a : Ordinal.{u}
⊢ ∃ o f, a.IsFundamentalSequence o f
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Cardinal/Cofinality.lean
|
Ordinal.exists_fundamental_sequence
|
α : Type u_1
r : α → α → Prop
a : Ordinal.{u}
⊢ ∃ o f, a.IsFundamentalSequence o f
|
rcases <a>Ordinal.exists_lsub_cof</a> a with ⟨ι, f, hf, hι⟩
|
case intro.intro.intro
α : Type u_1
r : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
⊢ ∃ o f, a.IsFundamentalSequence o f
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Cardinal/Cofinality.lean
|
Ordinal.exists_fundamental_sequence
|
case intro.intro.intro
α : Type u_1
r : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
⊢ ∃ o f, a.IsFundamentalSequence o f
|
rcases <a>Cardinal.ord_eq</a> ι with ⟨r, wo, hr⟩
|
case intro.intro.intro.intro.intro
α : Type u_1
r✝ : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
r : ι → ι → Prop
wo : IsWellOrder ι r
hr : (#ι).ord = type r
⊢ ∃ o f, a.IsFundamentalSequence o f
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Cardinal/Cofinality.lean
|
Ordinal.exists_fundamental_sequence
|
case intro.intro.intro.intro.intro
α : Type u_1
r✝ : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
r : ι → ι → Prop
wo : IsWellOrder ι r
hr : (#ι).ord = type r
⊢ ∃ o f, a.IsFundamentalSequence o f
|
haveI := wo
|
case intro.intro.intro.intro.intro
α : Type u_1
r✝ : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
r : ι → ι → Prop
wo : IsWellOrder ι r
hr : (#ι).ord = type r
this : IsWellOrder ι r
⊢ ∃ o f, a.IsFundamentalSequence o f
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Cardinal/Cofinality.lean
|
Ordinal.exists_fundamental_sequence
|
case intro.intro.intro.intro.intro
α : Type u_1
r✝ : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
r : ι → ι → Prop
wo : IsWellOrder ι r
hr : (#ι).ord = type r
this : IsWellOrder ι r
⊢ ∃ o f, a.IsFundamentalSequence o f
|
let r' := <a>Subrel</a> r { i | ∀ j, r j i → f j < f i }
|
case intro.intro.intro.intro.intro
α : Type u_1
r✝ : α → α → Prop
a : Ordinal.{u}
ι : Type u
f : ι → Ordinal.{u}
hf : lsub f = a
hι : #ι = a.cof
r : ι → ι → Prop
wo : IsWellOrder ι r
hr : (#ι).ord = type r
this : IsWellOrder ι r
r' : ↑{i | ∀ (j : ι), r j i → f j < f i} → ↑{i | ∀ (j : ι), r j i → f j < f i} → Prop :=
Subrel r {i | ∀ (j : ι), r j i → f j < f i}
⊢ ∃ o f, a.IsFundamentalSequence o f
|
https://github.com/leanprover-community/mathlib4
|
29dcec074de168ac2bf835a77ef68bbe069194c5
|
Mathlib/SetTheory/Cardinal/Cofinality.lean
|
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.