Skip to content

Commit a43b3f1

Browse files
maxwell-thumqawbecrdteyjcommelinRuben-VandeVelde
committed
feat: port Data.Fin.Tuple.Basic (#1516)
Co-authored-by: qawbecrdtey <40463813+qawbecrdtey@users.noreply.github.com> Co-authored-by: Johan Commelin <johan@commelin.net> Co-authored-by: Ruben Van de Velde <65514131+Ruben-VandeVelde@users.noreply.github.com>
1 parent 5f2b48d commit a43b3f1

File tree

3 files changed

+841
-1
lines changed

3 files changed

+841
-1
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -227,6 +227,7 @@ import Mathlib.Data.Erased
227227
import Mathlib.Data.Fin.Basic
228228
import Mathlib.Data.Fin.Fin2
229229
import Mathlib.Data.Fin.SuccPred
230+
import Mathlib.Data.Fin.Tuple.Basic
230231
import Mathlib.Data.Finite.Defs
231232
import Mathlib.Data.Finset.Basic
232233
import Mathlib.Data.Finset.Card

Mathlib/Data/Fin/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -501,7 +501,7 @@ theorem revOrderIso_symm_apply (i : Fin n) : revOrderIso.symm i = OrderDual.toDu
501501

502502
/-- The greatest value of `Fin (n+1)` -/
503503
def last (n : ℕ) : Fin (n + 1) :=
504-
_, n.lt_succ_self⟩
504+
n, n.lt_succ_self⟩
505505
#align fin.last Fin.last
506506

507507
@[simp, norm_cast]

0 commit comments

Comments
 (0)