Skip to content

Commit beaa3f2

Browse files
authored
Hide n argument in Tactic.RingSolver.NonReflective._⊜_ (#1149)
1 parent 912c3b9 commit beaa3f2

File tree

3 files changed

+5
-3
lines changed

3 files changed

+5
-3
lines changed

CHANGELOG.md

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -21,6 +21,8 @@ Bug-fixes
2121
Non-backwards compatible changes
2222
--------------------------------
2323

24+
* The `n` argument to `_⊜_` in `Tactic.RingSolver.NonReflective` has been made implict rather than explicit.
25+
2426
* `Data.Empty.Polymorphic` and `Data.Unit.Polymorphic` were rewritten
2527
to explicitly use `Lift` rather that defining new types. This means
2628
that these are now compatible with `` and `` from the rest of the

src/Tactic/RingSolver.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -154,7 +154,7 @@ private
154154
callSolver : Vec String numVars Term Term Args Type
155155
callSolver nms lhs rhs =
156156
2 ⋯⟅∷⟆ ring ⟨∷⟩ toTerm numVars ⟨∷⟩
157-
vlams nms (quote _⊜_ $ʳ (toTerm numVars ⟨∷⟩ E lhs ⟨∷⟩ E rhs ⟨∷⟩ [])) ⟨∷⟩
157+
vlams nms (quote _⊜_ $ʳ (toTerm numVars ⟅∷⟆ E lhs ⟨∷⟩ E rhs ⟨∷⟩ [])) ⟨∷⟩
158158
hlams nms (quote refl $ʳ (1 ⋯⟅∷⟆ [])) ⟨∷⟩
159159
[]
160160
where

src/Tactic/RingSolver/NonReflective.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -93,9 +93,9 @@ solve : ∀ (n : ℕ) →
9393
solve = Ops.solve
9494
{-# INLINE solve #-}
9595

96-
_⊜_ : (n :)
96+
_⊜_ : {n :}
9797
Expr Carrier n
9898
Expr Carrier n
9999
Expr Carrier n × Expr Carrier n
100-
_⊜_ _ = _,_
100+
_⊜_ = _,_
101101
{-# INLINE _⊜_ #-}

0 commit comments

Comments
 (0)