Skip to content

Commit

Permalink
simplify test
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Oct 17, 2024
1 parent 679e195 commit 7e6041c
Showing 1 changed file with 8 additions and 9 deletions.
17 changes: 8 additions & 9 deletions test/DFinsuppMultiLinear.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,12 +2,11 @@ import Mathlib.Data.DFinsupp.Multilinear
import Mathlib.Data.DFinsupp.Notation

/--
info:
fun₀
| !["hello", "complicated", "world"] => 231
| !["hello", "complicated", "test file"] => 273
| !["goodbye", "complicated", "world"] => 385
| !["goodbye", "complicated", "test file"] => 455
info: fun₀
| !["hello", "complicated", "world"] => 20
| !["hello", "complicated", "test file"] => 30
| !["goodbye", "complicated", "world"] => -20
| !["goodbye", "complicated", "test file"] => -30
-/
#guard_msgs in
#eval DFinsupp.piMultilinear
Expand All @@ -16,7 +15,7 @@ fun₀
(N := fun _ => ℤ)
(R := ℤ)
(f := fun _ => MultilinearMap.mkPiAlgebra ℤ (Fin 3) ℤ) <|
Fin.cons (fun₀ | "hello" => 3 | "goodbye" => 5) <|
Fin.cons (fun₀ | "complicated" => 7) <|
Fin.cons (fun₀ | "world" => 11 | "test file" => 13) <|
Fin.cons (fun₀ | "hello" => 1 | "goodbye" => -1) <|
Fin.cons (fun₀ | "complicated" => 10) <|
Fin.cons (fun₀ | "world" => 2 | "test file" => 3) <|
IsEmpty.elim inferInstance

0 comments on commit 7e6041c

Please sign in to comment.