Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2021-05-15 14:21 738c19f5

View on Github →

refactor(linear_algebra/matrix): split matrix.lean into multiple files (#7593) The file linear_algebra/matrix.lean used to be very big and contain a lot of parts that did not depend on each other, so I split each of those parts into its own little file. Most of the new files ended up in linear_algebra/matrix/, except for linear_algebra/trace.lean and linear_algebra/determinant.lean which did not contain anything matrix-specific. Apart from the local improvement in matrix.lean itself, the import graph is now also a bit cleaner. Renames:

  • linear_algebra/determinant.lean -> linear_algebra/matrix/determinant.lean
  • linear_algebra/nonsingular_inverse.lean -> linear_algebra/matrix/nonsingular_inverse.lean Split off from linear_algebra/matrix.lean:
  • linear_algebra/matrix/basis.lean
  • linear_algebra/matrix/block.lean
  • linear_algebra/matrix/diagonal.lean
  • linear_algebra/matrix/dot_product.lean
  • linear_algebra/matrix/dual.lean
  • linear_algebra/matrix/finite_dimensional.lean
  • linear_algebra/matrix/reindex.lean
  • linear_algebra/matrix/to_lin.lean
  • linear_algebra/matrix/to_linear_equiv.lean
  • linear_algebra/matrix/trace.lean
  • linear_algebra/determinant.lean (Unfortunately, I could not persuade git to remember that I moved the original determinant.lean to matrix/determinant.lean)
  • linear_algebra/trace.lean

Estimated changes

added def basis.det
added theorem basis.det_apply
added theorem basis.det_self
added theorem is_basis.iff_det
deleted theorem matrix.alg_hom.map_det
deleted def matrix.det
deleted theorem matrix.det_apply'
deleted theorem matrix.det_apply
deleted theorem matrix.det_block_diagonal
deleted theorem matrix.det_diagonal
deleted theorem matrix.det_fin_zero
deleted theorem matrix.det_mul
deleted theorem matrix.det_mul_aux
deleted theorem matrix.det_mul_column
deleted theorem matrix.det_mul_row
deleted theorem matrix.det_one
deleted theorem matrix.det_permutation
deleted theorem matrix.det_permute
deleted theorem matrix.det_reindex_self
deleted theorem matrix.det_smul
deleted theorem matrix.det_succ_column
deleted theorem matrix.det_succ_row
deleted theorem matrix.det_succ_row_zero
deleted theorem matrix.det_transpose
deleted theorem matrix.det_unique
deleted theorem matrix.det_update_row_add
deleted theorem matrix.det_zero
deleted theorem matrix.det_zero_of_row_eq
deleted theorem matrix.ring_hom.map_det
deleted def alg_equiv_matrix'
deleted def alg_equiv_matrix
deleted theorem algebra.to_matrix_lmul'
deleted theorem algebra.to_matrix_lmul_eq
deleted theorem algebra.to_matrix_lsmul
deleted def basis.det
deleted theorem basis.det_apply
deleted theorem basis.det_self
deleted theorem basis.to_lin_to_matrix
deleted def basis.to_matrix
deleted theorem basis.to_matrix_apply
deleted theorem basis.to_matrix_self
deleted theorem basis.to_matrix_update
deleted theorem is_basis.iff_det
deleted theorem linear_equiv.is_unit_det
deleted theorem linear_map.to_matrix'_id
deleted theorem linear_map.to_matrix'_mul
deleted theorem linear_map.to_matrix_comp
deleted theorem linear_map.to_matrix_id
deleted theorem linear_map.to_matrix_mul
deleted theorem linear_map.to_matrix_one
deleted theorem linear_map.to_matrix_symm
deleted def linear_map.trace
deleted theorem linear_map.trace_aux_def
deleted theorem linear_map.trace_aux_eq
deleted theorem linear_map.trace_mul_comm
deleted theorem matrix.det_to_block
deleted def matrix.diag
deleted theorem matrix.diag_apply
deleted theorem matrix.diag_one
deleted theorem matrix.diag_transpose
deleted theorem matrix.diagonal_to_lin'
deleted theorem matrix.dot_product_eq
deleted theorem matrix.dot_product_eq_iff
deleted theorem matrix.equiv_block_det
deleted theorem matrix.finrank_matrix
deleted theorem matrix.ker_to_lin_eq_bot
deleted def matrix.mul_vec_lin
deleted theorem matrix.mul_vec_lin_apply
deleted theorem matrix.mul_vec_std_basis
deleted theorem matrix.proj_diagonal
deleted theorem matrix.range_diagonal
deleted theorem matrix.rank_diagonal
deleted theorem matrix.rank_vec_mul_vec
deleted def matrix.to_lin'
deleted theorem matrix.to_lin'_apply
deleted theorem matrix.to_lin'_mul
deleted theorem matrix.to_lin'_one
deleted theorem matrix.to_lin'_symm
deleted theorem matrix.to_lin'_to_matrix'
deleted def matrix.to_lin
deleted theorem matrix.to_lin_apply
deleted theorem matrix.to_lin_mul
deleted theorem matrix.to_lin_one
deleted theorem matrix.to_lin_self
deleted theorem matrix.to_lin_symm
deleted theorem matrix.to_lin_to_matrix
deleted theorem matrix.to_lin_transpose
deleted def matrix.trace
deleted theorem matrix.trace_apply
deleted theorem matrix.trace_diag
deleted theorem matrix.trace_mul_comm
deleted theorem matrix.trace_one
deleted theorem matrix.trace_transpose
added theorem matrix.alg_hom.map_det
added def matrix.det
added theorem matrix.det_apply'
added theorem matrix.det_apply
added theorem matrix.det_diagonal
added theorem matrix.det_fin_zero
added theorem matrix.det_mul
added theorem matrix.det_mul_aux
added theorem matrix.det_mul_column
added theorem matrix.det_mul_row
added theorem matrix.det_one
added theorem matrix.det_permutation
added theorem matrix.det_permute
added theorem matrix.det_smul
added theorem matrix.det_succ_column
added theorem matrix.det_succ_row
added theorem matrix.det_transpose
added theorem matrix.det_unique
added theorem matrix.det_zero
added def alg_equiv_matrix
added def matrix.to_lin'
added theorem matrix.to_lin'_apply
added theorem matrix.to_lin'_mul
added theorem matrix.to_lin'_one
added theorem matrix.to_lin'_symm
added def matrix.to_lin
added theorem matrix.to_lin_apply
added theorem matrix.to_lin_mul
added theorem matrix.to_lin_one
added theorem matrix.to_lin_self
added theorem matrix.to_lin_symm