Skip to content

Commit 9a68858

Browse files
plt-amyandreasabel
authored andcommitted
Add new blocking primitives to Reflection.TCM (#1972)
1 parent dac1b2b commit 9a68858

File tree

2 files changed

+14
-2
lines changed

2 files changed

+14
-2
lines changed

CHANGELOG.md

+9
Original file line numberDiff line numberDiff line change
@@ -3801,6 +3801,15 @@ This is a full list of proofs that have changed form to use irrelevant instance
38013801
WellFounded _<_ → Irreflexive _≈_ _<_
38023802
```
38033803

3804+
* Added new types and operations to `Reflection.TCM`:
3805+
```
3806+
Blocker : Set
3807+
blockerMeta : Meta → Blocker
3808+
blockerAny : List Blocker → Blocker
3809+
blockerAll : List Blocker → Blocker
3810+
blockTC : Blocker → TC A
3811+
```
3812+
38043813
* Added new file `Relation.Binary.Reasoning.Base.Apartness`
38053814

38063815
This is how to use it:

src/Reflection/TCM.agda

+5-2
Original file line numberDiff line numberDiff line change
@@ -8,8 +8,9 @@
88

99
module Reflection.TCM where
1010

11-
open import Reflection.AST.Term
1211
import Agda.Builtin.Reflection as Builtin
12+
13+
open import Reflection.AST.Term
1314
import Reflection.TCM.Format as Format
1415

1516
------------------------------------------------------------------------
@@ -29,7 +30,9 @@ open Builtin public
2930
; getContext; extendContext; inContext; freshName
3031
; declareDef; declarePostulate; defineFun; getType; getDefinition
3132
; blockOnMeta; commitTC; isMacro; withNormalisation
32-
; debugPrint; noConstraints; runSpeculative)
33+
; debugPrint; noConstraints; runSpeculative
34+
; Blocker; blockerMeta; blockerAny; blockerAll; blockTC
35+
)
3336
renaming (returnTC to pure)
3437

3538
open Format public

0 commit comments

Comments
 (0)