Skip to content

Commit

Permalink
matrix notation
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Oct 23, 2023
1 parent bca61be commit 798574a
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion src/exercises_sources/thursday/linear_algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -133,7 +133,7 @@ Hints:
* Use the `simp` tactic to simplify `(x + y) i` to `x i + y i` and `(s • x) i` to `s * x i`.
* To deal with equalities containing many `+` and `*` symbols, use the `ring` tactic.
-/
def A : matrix (fin 2) (fin 2) R := ![![1, 0], ![-2, 1]]
def A : matrix (fin 2) (fin 2) R := !![1, 0; -2, 1]
def your_bilin_form : bilin_form R (fin 2 → R) :=
sorry

Expand Down
2 changes: 1 addition & 1 deletion src/solutions/thursday/linear_algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -196,7 +196,7 @@ Hints:
* Use the `simp` tactic to simplify `(x + y) i` to `x i + y i` and `(s • x) i` to `s * x i`.
* To deal with equalities containing many `+` and `*` symbols, use the `ring` tactic.
-/
def A : matrix (fin 2) (fin 2) R := ![![1, 0], ![-2, 1]]
def A : matrix (fin 2) (fin 2) R := !![1, 0; -2, 1]
def your_bilin_form : bilin_form R (fin 2 → R) :=
-- sorry
{ bilin := λ v w, v 0 * w 0 + v 1 * w 1 - 2 * v 1 * w 0,
Expand Down

0 comments on commit 798574a

Please sign in to comment.