Skip to content

Commit aaff5ad

Browse files
committed
chore(Data/Fin/Tuple): generalize Type to Sort (#17161)
Generalize definitions and theorems in `Data/Fin/Tuple/Basic` to take in `Sort` by default instead of `Type`. The exceptions are theorems that interact with existing type classes such as `Preorder`, `Prod`, and `Set`, which expect `Type`. For instance, the following is added specifically for some theorems about `Preorder`: ```lean4 variable {α : Fin (n + 1) → Type*} -- instead of variable {α : Fin (n + 1) → Sort*} ``` Co-authored-by: Quang Dao <quangdao@umich.edu>
1 parent c76e7c6 commit aaff5ad

File tree

2 files changed

+67
-56
lines changed

2 files changed

+67
-56
lines changed

Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -302,7 +302,7 @@ noncomputable def fslope (p : FormalMultilinearSeries 𝕜 𝕜 E) : FormalMulti
302302
theorem coeff_fslope : p.fslope.coeff n = p.coeff (n + 1) := by
303303
simp only [fslope, coeff, ContinuousMultilinearMap.curryLeft_apply]
304304
congr 1
305-
exact Fin.cons_self_tail 1
305+
exact Fin.cons_self_tail (fun _ => (1 : 𝕜))
306306

307307
@[simp]
308308
theorem coeff_iterate_fslope (k n : ℕ) : (fslope^[k] p).coeff n = p.coeff (n + k) := by

0 commit comments

Comments
 (0)