Skip to content

Commit 2baf4c4

Browse files
committed
Tactic.RingSolver.Core.Polynomial: drop eta-equality for constructor _⊐_
Future Agda versions might no longer support eta for unguarded records in `--safe` mode. Dropping eta-equality for constructor _⊐_ only requires changing the order of clauses in ⊞-inj. Re: agda/agda#7470
1 parent ef9e3d6 commit 2baf4c4

File tree

1 file changed

+3
-2
lines changed
  • src/Tactic/RingSolver/Core/Polynomial

1 file changed

+3
-2
lines changed

src/Tactic/RingSolver/Core/Polynomial/Base.agda

+3-2
Original file line numberDiff line numberDiff line change
@@ -130,8 +130,9 @@ Normalised : ∀ {i} → Coeff i + → Set
130130
infixl 6 _⊐_
131131
record Poly n where
132132
inductive
133+
no-eta-equality
134+
pattern -- To allow matching on constructor
133135
constructor _⊐_
134-
eta-equality -- To allow matching on constructor
135136
field
136137
{i} :
137138
flat : FlatPoly i
@@ -285,8 +286,8 @@ mutual
285286
FlatPoly i
286287
Coeff k +
287288
Coeff k *
288-
⊞-inj i≤k xs (y ⊐ j≤k ≠0 Δ zero & ys) = ⊞-match (inj-compare j≤k i≤k) y xs Δ zero ∷↓ ys
289289
⊞-inj i≤k xs (y Δ suc j & ys) = xs ⊐ i≤k Δ zero ∷↓ ∹ y Δ j & ys
290+
⊞-inj i≤k xs (y ⊐ j≤k ≠0 Δ zero & ys) = ⊞-match (inj-compare j≤k i≤k) y xs Δ zero ∷↓ ys
290291

291292
⊞-coeffs : {n} Coeff n * Coeff n * Coeff n *
292293
⊞-coeffs (∹ x Δ i & xs) ys = ⊞-zip-r x i xs ys

0 commit comments

Comments
 (0)