Skip to content

Commit

Permalink
mention a limitation
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Feb 7, 2024
1 parent d6cf2a4 commit 036ada4
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 1 deletion.
7 changes: 7 additions & 0 deletions Cubical/Tactics/CommRingSolver/Examples.agda
Original file line number Diff line number Diff line change
Expand Up @@ -35,8 +35,15 @@ module TestErrors (R : CommRing ℓ) where
module TestWithℤ where
open CommRingStr (ℤCommRing .snd)

{-
the following is not possible yet: the ring solver normalises the goal
and expands some of the definitions of the operations. A possible fix could be
to not normalize - but then one has to (at least) translate every use of a binary
minus. (#1101)
ex13 : (x y : ℤ) → (x · y) · 1r ≡ 1r · (y · x)
ex13 x y = solve! ℤCommRing
-}

ex0 : (a b : fst ℤCommRing) a + b ≡ b + a
ex0 a b = solve! ℤCommRing
Expand Down
2 changes: 1 addition & 1 deletion Cubical/Tactics/CommRingSolver/Reflection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -13,7 +13,7 @@ open import Cubical.Data.Maybe
open import Cubical.Data.Sigma
open import Cubical.Data.List
open import Cubical.Data.Nat.Literals
open import Cubical.Data.Int.Base hiding (abs)
open import Cubical.Data.Int.Base hiding (abs; _-_)
open import Cubical.Data.Int using (fromNegℤ; fromNatℤ)
open import Cubical.Data.Nat using (ℕ; discreteℕ) renaming (_+_ to _+ℕ_)
open import Cubical.Data.Bool
Expand Down

0 comments on commit 036ada4

Please sign in to comment.