Skip to content

Commit

Permalink
bump to nightly-2023-07-04-19
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Jul 4, 2023
1 parent 0dba3a1 commit 4217d5f
Show file tree
Hide file tree
Showing 23 changed files with 210 additions and 205 deletions.
8 changes: 4 additions & 4 deletions Mathbin/Algebra/BigOperators/Fin.lean
Expand Up @@ -227,7 +227,7 @@ theorem prod_Ioi_succ {M : Type _} [CommMonoid M] {n : ℕ} (i : Fin n) (v : Fin
#print Fin.prod_congr' /-
@[to_additive]
theorem prod_congr' {M : Type _} [CommMonoid M] {a b : ℕ} (f : Fin b → M) (h : a = b) :
∏ i : Fin a, f (cast h i) = ∏ i : Fin b, f i := by subst h; congr; ext; congr; ext;
∏ i : Fin a, f (castIso h i) = ∏ i : Fin b, f i := by subst h; congr; ext; congr; ext;
rw [coe_cast]
#align fin.prod_congr' Fin.prod_congr'
#align fin.sum_congr' Fin.sum_congr'
Expand Down Expand Up @@ -385,7 +385,7 @@ def finFunctionFinEquiv {m n : ℕ} : (Fin n → Fin m) ≃ Fin (m ^ n) :=
fun a => by
dsimp
induction' n with n ih generalizing a
· haveI : Subsingleton (Fin (m ^ 0)) := (Fin.cast <| pow_zero _).toEquiv.Subsingleton
· haveI : Subsingleton (Fin (m ^ 0)) := (Fin.castIso <| pow_zero _).toEquiv.Subsingleton
exact Subsingleton.elim _ _
simp_rw [Fin.forall_iff, Fin.ext_iff, Fin.val_mk] at ih
ext
Expand Down Expand Up @@ -451,14 +451,14 @@ def finPiFinEquiv {m : ℕ} {n : Fin m → ℕ} : (∀ i : Fin m, Fin (n i)) ≃
refine' Fin.consInduction _ _ n
· intro a
haveI : Subsingleton (Fin (∏ i : Fin 0, i.elim0ₓ)) :=
(Fin.cast <| prod_empty).toEquiv.Subsingleton
(Fin.castIso <| prod_empty).toEquiv.Subsingleton
exact Subsingleton.elim _ _
· intro n x xs ih a
simp_rw [Fin.forall_iff, Fin.ext_iff, Fin.val_mk] at ih
ext
simp_rw [Fin.val_mk, Fin.sum_univ_succ, Fin.cons_succ]
have := fun i : Fin n =>
Fintype.prod_equiv (Fin.cast <| Fin.val_succ i).toEquiv
Fintype.prod_equiv (Fin.castIso <| Fin.val_succ i).toEquiv
(fun j => (Fin.cons x xs : _ → ℕ) (Fin.castLE (Fin.is_lt _).le j))
(fun j => (Fin.cons x xs : _ → ℕ) (Fin.castLE (Nat.succ_le_succ (Fin.is_lt _).le) j))
fun j => rfl
Expand Down
10 changes: 5 additions & 5 deletions Mathbin/AlgebraicTopology/DoldKan/Faces.lean
Expand Up @@ -114,7 +114,7 @@ theorem comp_Hσ_eq {Y : C} {n a q : ℕ} {φ : Y ⟶ X _[n + 1]} (v : HigherFac
swap
· rintro ⟨k, hk⟩
suffices φ ≫ X.δ (⟨a + 2 + k, by linarith⟩ : Fin (n + 2)) = 0 by
simp only [this, Fin.natAdd_mk, Fin.cast_mk, zero_comp, smul_zero]
simp only [this, Fin.natAdd_mk, Fin.castIso_mk, zero_comp, smul_zero]
convert v ⟨a + k + 1, by linarith⟩ (by rw [Fin.val_mk]; linarith)
rw [Nat.succ_eq_add_one]
linarith
Expand All @@ -138,7 +138,7 @@ theorem comp_Hσ_eq {Y : C} {n a q : ℕ} {φ : Y ⟶ X _[n + 1]} (v : HigherFac
skip
rw [Fin.sum_univ_castSucc, Fin.sum_univ_castSucc]
rw [Fin.sum_univ_castSucc]
simp only [Fin.last, Fin.castLE_mk, Fin.coe_cast, Fin.cast_mk, Fin.coe_castLE, Fin.val_mk,
simp only [Fin.last, Fin.castLE_mk, Fin.coe_castIso, Fin.castIso_mk, Fin.coe_castLE, Fin.val_mk,
Fin.castSucc_mk, Fin.coe_castSucc]
/- the purpose of the following `simplif` is to create three subgoals in order
to finish the proof -/
Expand All @@ -162,7 +162,7 @@ theorem comp_Hσ_eq {Y : C} {n a q : ℕ} {φ : Y ⟶ X _[n + 1]} (v : HigherFac
rintro ⟨i, hi⟩ h₀
have hia : (⟨i, by linarith⟩ : Fin (n + 2)) ≤ Fin.castSucc (⟨a, by linarith⟩ : Fin (n + 1)) :=
by simpa only [Fin.le_iff_val_le_val, Fin.val_mk, Fin.castSucc_mk, ← lt_succ_iff] using hi
simp only [Fin.val_mk, Fin.castLE_mk, Fin.castSucc_mk, Fin.succ_mk, assoc, Fin.cast_mk, ←
simp only [Fin.val_mk, Fin.castLE_mk, Fin.castSucc_mk, Fin.succ_mk, assoc, Fin.castIso_mk, ←
δ_comp_σ_of_le X hia, add_eq_zero_iff_eq_neg, ← neg_zsmul]
congr
ring
Expand All @@ -182,7 +182,7 @@ theorem comp_Hσ_eq_zero {Y : C} {n q : ℕ} {φ : Y ⟶ X _[n + 1]} (v : Higher
alternating_face_map_complex.obj_d_eq]
rw [← Fin.sum_congr' _ (show 2 + (n + 1) = n + 1 + 2 by linarith), Fin.sum_trunc]
· simp only [Fin.sum_univ_castSucc, Fin.sum_univ_zero, zero_add, Fin.last, Fin.castLE_mk,
Fin.cast_mk, Fin.castSucc_mk]
Fin.castIso_mk, Fin.castSucc_mk]
simp only [Fin.mk_zero, Fin.val_zero, pow_zero, one_zsmul, Fin.mk_one, Fin.val_one, pow_one,
neg_smul, comp_neg]
erw [δ_comp_σ_self, δ_comp_σ_succ, add_right_neg]
Expand All @@ -193,7 +193,7 @@ theorem comp_Hσ_eq_zero {Y : C} {n q : ℕ} {φ : Y ⟶ X _[n + 1]} (v : Higher
dsimp at h
linarith
· dsimp
simp only [Fin.cast_natAdd, Fin.coe_pred, Fin.coe_addNat, add_succ_sub_one]
simp only [Fin.castIso_natAdd, Fin.coe_pred, Fin.coe_addNat, add_succ_sub_one]
linarith
· rw [Fin.lt_iff_val_lt_val]
dsimp
Expand Down
11 changes: 6 additions & 5 deletions Mathbin/Analysis/Analytic/Basic.lean
Expand Up @@ -1394,7 +1394,8 @@ def changeOriginIndexEquiv :
invFun s :=
⟨s.1 - s.2.card, s.2.card,
⟨s.2.map
(Fin.cast <| (tsub_add_cancel_of_le <| card_finset_fin_le s.2).symm).toEquiv.toEmbedding,
(Fin.castIso <|
(tsub_add_cancel_of_le <| card_finset_fin_le s.2).symm).toEquiv.toEmbedding,
Finset.card_map _⟩⟩
left_inv := by
rintro ⟨k, l, ⟨s : Finset (Fin <| k + l), hs : s.card = l⟩⟩
Expand All @@ -1406,16 +1407,16 @@ def changeOriginIndexEquiv :
k' = k →
l' = l →
∀ (hkl : k + l = k' + l') (hs'),
(⟨k', l', ⟨Finset.map (Fin.cast hkl).toEquiv.toEmbedding s, hs'⟩⟩ :
(⟨k', l', ⟨Finset.map (Fin.castIso hkl).toEquiv.toEmbedding s, hs'⟩⟩ :
Σ k l : ℕ, { s : Finset (Fin (k + l)) // s.card = l }) =
⟨k, l, ⟨s, hs⟩⟩
by apply this <;> simp only [hs, add_tsub_cancel_right]
rintro _ _ rfl rfl hkl hs'
simp only [Equiv.refl_toEmbedding, Fin.cast_refl, Finset.map_refl, eq_self_iff_true,
simp only [Equiv.refl_toEmbedding, Fin.castIso_refl, Finset.map_refl, eq_self_iff_true,
OrderIso.refl_toEquiv, and_self_iff, heq_iff_eq]
right_inv := by
rintro ⟨n, s⟩
simp [tsub_add_cancel_of_le (card_finset_fin_le s), Fin.cast_to_equiv]
simp [tsub_add_cancel_of_le (card_finset_fin_le s), Fin.castIso_to_equiv]
#align formal_multilinear_series.change_origin_index_equiv FormalMultilinearSeries.changeOriginIndexEquiv
-/

Expand Down Expand Up @@ -1574,7 +1575,7 @@ theorem changeOrigin_eval (h : (‖x‖₊ + ‖y‖₊ : ℝ≥0∞) < p.radius
have :
∀ (m) (hm : n = m),
p n (s.piecewise (fun _ => x) fun _ => y) =
p m ((s.map (Fin.cast hm).toEquiv.toEmbedding).piecewise (fun _ => x) fun _ => y) :=
p m ((s.map (Fin.castIso hm).toEquiv.toEmbedding).piecewise (fun _ => x) fun _ => y) :=
by rintro m rfl; simp
apply this
#align formal_multilinear_series.change_origin_eval FormalMultilinearSeries.changeOrigin_eval
Expand Down

0 comments on commit 4217d5f

Please sign in to comment.