Skip to content

Commit

Permalink
make one example more meaningful
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Aug 2, 2024
1 parent 1e251b8 commit 49ab241
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Cubical/Tactics/CommRingSolver/Examples.agda
Original file line number Diff line number Diff line change
Expand Up @@ -65,7 +65,7 @@ module Test (R : CommRing ℓ) (x y z : fst R) where
ex1 : x ≡ x
ex1 = solve! R

ex2 : x ≡ x
ex2 : (0r - 1r) · x ≡ 0r - x
ex2 = solve! R

ex3 : x + y ≡ y + x
Expand Down

0 comments on commit 49ab241

Please sign in to comment.