@@ -193,7 +193,7 @@ begin
193
193
rcases i with ⟨i, _⟩,
194
194
rcases j with ⟨j, _⟩,
195
195
rcases k with ⟨k, _⟩,
196
- simp only [subtype .mk_le_mk, fin.cast_succ_mk] at H,
196
+ simp only [fin .mk_le_mk, fin.cast_succ_mk] at H,
197
197
dsimp,
198
198
split_ifs,
199
199
-- Most of the goals can now be handled by `linarith`,
@@ -241,28 +241,28 @@ begin
241
241
rcases i with ⟨i, _⟩,
242
242
rcases j with ⟨j, _⟩,
243
243
rcases k with ⟨k, _⟩,
244
- simp only [subtype .mk_lt_mk, fin.cast_succ_mk] at H,
244
+ simp only [fin .mk_lt_mk, fin.cast_succ_mk] at H,
245
245
suffices : ite (_ < ite (k < i + 1 ) _ _) _ _ =
246
246
ite _ (ite (j < k) (k - 1 ) k) (ite (j < k) (k - 1 ) k + 1 ),
247
247
{ simpa [apply_dite fin.cast_succ, fin.pred_above] with push_cast, },
248
248
split_ifs,
249
249
-- Most of the goals can now be handled by `linarith`,
250
250
-- but we have to deal with three of them by hand.
251
251
swap 2 ,
252
- { simp only [subtype .mk_lt_mk] at h_1,
252
+ { simp only [fin .mk_lt_mk] at h_1,
253
253
simp only [not_lt] at h_2,
254
254
simp only [self_eq_add_right, one_ne_zero],
255
255
exact lt_irrefl (k - 1 ) (lt_of_lt_of_le
256
256
(nat.pred_lt (ne_of_lt (lt_of_le_of_lt (zero_le _) h_1)).symm)
257
257
(le_trans (nat.le_of_lt_succ h) h_2)) },
258
258
swap 4 ,
259
- { simp only [subtype .mk_lt_mk] at h_1,
259
+ { simp only [fin .mk_lt_mk] at h_1,
260
260
simp only [not_lt] at h,
261
261
simp only [nat.add_succ_sub_one, add_zero],
262
262
exfalso,
263
263
exact lt_irrefl _ (lt_of_le_of_lt (nat.le_pred_of_lt (nat.lt_of_succ_le h)) h_3), },
264
264
swap 4 ,
265
- { simp only [subtype .mk_lt_mk] at h_1,
265
+ { simp only [fin .mk_lt_mk] at h_1,
266
266
simp only [not_lt] at h_3,
267
267
simp only [nat.add_succ_sub_one, add_zero],
268
268
exact (nat.succ_pred_eq_of_pos (lt_of_le_of_lt (zero_le _) h_2)).symm, },
@@ -281,7 +281,7 @@ begin
281
281
rcases i with ⟨i, _⟩,
282
282
rcases j with ⟨j, _⟩,
283
283
rcases k with ⟨k, _⟩,
284
- simp only [subtype .mk_le_mk] at H,
284
+ simp only [fin .mk_le_mk] at H,
285
285
-- At this point `simp with push_cast` makes good progress, but neither `simp?` nor `squeeze_simp`
286
286
-- return usable sets of lemmas.
287
287
-- To avoid using a non-terminal simp, we make a `suffices` statement indicating the shape
0 commit comments