Skip to content

Commit

Permalink
docs: Matrix.IsTotallyUnimodular docstring (#19338)
Browse files Browse the repository at this point in the history
  • Loading branch information
madvorak committed Nov 21, 2024
1 parent e2d0dfc commit d1c99f2
Showing 1 changed file with 2 additions and 1 deletion.
Original file line number Diff line number Diff line change
Expand Up @@ -28,7 +28,8 @@ namespace Matrix

variable {m n R : Type*} [CommRing R]

/-- Is the matrix `A` totally unimodular? -/
/-- `A.IsTotallyUnimodular` means that every square submatrix of `A` (not necessarily contiguous)
has determinant `0` or `1` or `-1`. -/
def IsTotallyUnimodular (A : Matrix m n R) : Prop :=
∀ k : ℕ, ∀ f : Fin k → m, ∀ g : Fin k → n, f.Injective → g.Injective →
(A.submatrix f g).det = 0
Expand Down

0 comments on commit d1c99f2

Please sign in to comment.