Open
Description
I've been using the monoid solver and found that the following example doesn't work:
module _ {a} {A : Set a} where
open import Data.List.Properties using (++-monoid)
open import Tactic.MonoidSolver using (solve)
test : ∀ (xs ys zs : List A) (x : A) → (xs ++ x ∷ ys) ++ zs ≡ xs ++ x ∷ (ys ++ zs)
test _ _ _ _ = solve (++-monoid A)
Metadata
Metadata
Assignees
Labels
No labels