Skip to content

Commit 4d24502

Browse files
committed
Replace record directive "eta-equality" by "no-eta-equality;pattern"
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
1 parent ef9e3d6 commit 4d24502

File tree

2 files changed

+4
-2
lines changed

2 files changed

+4
-2
lines changed

src/Data/Record.agda

+2-1
Original file line numberDiff line numberDiff line change
@@ -63,8 +63,9 @@ mutual
6363
-- inferred from a value of type Record Sig.
6464

6565
record Record {s} (Sig : Signature s) : Set s where
66-
eta-equality
6766
inductive
67+
no-eta-equality
68+
pattern
6869
constructor rec
6970
field fun : Record-fun Sig
7071

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

+2-1
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

0 commit comments

Comments
 (0)