Skip to content

Commit

Permalink
Replace record directive "eta-equality" by "no-eta-equality;pattern"
Browse files Browse the repository at this point in the history
Future Agda might not allow unguarded record types with eta-equality
in the safe mode anymore.

So we switch eta off here, but make the constructor a pattern so that
it can still be matched on.

Re: agda/agda#7470
  • Loading branch information
andreasabel committed Sep 6, 2024
1 parent ef9e3d6 commit 4d24502
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 2 deletions.
3 changes: 2 additions & 1 deletion src/Data/Record.agda
Original file line number Diff line number Diff line change
Expand Up @@ -63,8 +63,9 @@ mutual
-- inferred from a value of type Record Sig.

record Record {s} (Sig : Signature s) : Set s where
eta-equality
inductive
no-eta-equality
pattern
constructor rec
field fun : Record-fun Sig

Expand Down
3 changes: 2 additions & 1 deletion src/Tactic/RingSolver/Core/Polynomial/Base.agda
Original file line number Diff line number Diff line change
Expand Up @@ -130,8 +130,9 @@ Normalised : ∀ {i} → Coeff i + → Set
infixl 6 _⊐_
record Poly n where
inductive
no-eta-equality
pattern -- To allow matching on constructor
constructor _⊐_
eta-equality -- To allow matching on constructor
field
{i} :
flat : FlatPoly i
Expand Down

0 comments on commit 4d24502

Please sign in to comment.