Skip to content

Commit 0c4d96e

Browse files
committed
fix: add DecidableEq to two lemmas (#11376)
1 parent 415f214 commit 0c4d96e

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

Mathlib/Analysis/Calculus/ContDiff/Basic.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1230,7 +1230,8 @@ theorem contDiff_pi : ContDiff 𝕜 n Φ ↔ ∀ i, ContDiff 𝕜 n fun x => Φ
12301230
simp only [← contDiffOn_univ, contDiffOn_pi]
12311231
#align cont_diff_pi contDiff_pi
12321232

1233-
theorem contDiff_update (k : ℕ∞) (x : ∀ i, F' i) (i : ι) : ContDiff 𝕜 k (update x i) := by
1233+
theorem contDiff_update [DecidableEq ι] (k : ℕ∞) (x : ∀ i, F' i) (i : ι) :
1234+
ContDiff 𝕜 k (update x i) := by
12341235
rw [contDiff_pi]
12351236
intro j
12361237
dsimp [Function.update]
@@ -1240,7 +1241,8 @@ theorem contDiff_update (k : ℕ∞) (x : ∀ i, F' i) (i : ι) : ContDiff 𝕜
12401241
· exact contDiff_const
12411242

12421243
variable (F') in
1243-
theorem contDiff_single (k : ℕ∞) (i : ι) : ContDiff 𝕜 k (Pi.single i : F' i → ∀ i, F' i) :=
1244+
theorem contDiff_single [DecidableEq ι] (k : ℕ∞) (i : ι) :
1245+
ContDiff 𝕜 k (Pi.single i : F' i → ∀ i, F' i) :=
12441246
contDiff_update k 0 i
12451247

12461248
variable (𝕜 E)

0 commit comments

Comments
 (0)