Skip to content

Commit

Permalink
Fix conflicts with latest mathlib
Browse files Browse the repository at this point in the history
  • Loading branch information
Vierkantor committed Jan 27, 2020
1 parent 9dc30e9 commit 3a44403
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/linear_algebra/nonsingular_inverse.lean
Original file line number Diff line number Diff line change
Expand Up @@ -297,11 +297,18 @@ lemma nonsing_inv_val (A : matrix n n α) (i j : n) :
lemma transpose_nonsing_inv (A : matrix n n α) : (A.nonsing_inv)ᵀ = (Aᵀ).nonsing_inv :=
by {ext, simp [transpose_val, nonsing_inv_val, det_transpose, (adjugate_transpose A).symm]}

section

-- Increase max depth to allow inference of `mul_action α (matrix n n α)`.
set_option class.instance_max_depth 60

/-- The `nonsing_inv` of `A` is a right inverse. -/
theorem mul_nonsing_inv (A : matrix n n α) (inv_mul_cancel : A.det⁻¹ * A.det = 1) :
A ⬝ nonsing_inv A = 1 :=
by erw [mul_smul, mul_adjugate, smul_smul, inv_mul_cancel, @one_smul _ _ _ (pi.mul_action _)]

end

/-- The `nonsing_inv` of `A` is a left inverse. -/
theorem nonsing_inv_mul (A : matrix n n α) (inv_mul_cancel : A.det⁻¹ * A.det = 1) :
nonsing_inv A ⬝ A = 1 :=
Expand Down

0 comments on commit 3a44403

Please sign in to comment.