File tree 2 files changed +14
-2
lines changed
2 files changed +14
-2
lines changed Original file line number Diff line number Diff line change @@ -3812,6 +3812,15 @@ This is a full list of proofs that have changed form to use irrelevant instance
3812
3812
WellFounded _<_ → Irreflexive _≈_ _<_
3813
3813
```
3814
3814
3815
+ * Added new types and operations to ` Reflection.TCM ` :
3816
+ ```
3817
+ Blocker : Set
3818
+ blockerMeta : Meta → Blocker
3819
+ blockerAny : List Blocker → Blocker
3820
+ blockerAll : List Blocker → Blocker
3821
+ blockTC : Blocker → TC A
3822
+ ```
3823
+
3815
3824
* Added new file ` Relation.Binary.Reasoning.Base.Apartness `
3816
3825
3817
3826
This is how to use it:
Original file line number Diff line number Diff line change 8
8
9
9
module Reflection.TCM where
10
10
11
- open import Reflection.AST.Term
12
11
import Agda.Builtin.Reflection as Builtin
12
+
13
+ open import Reflection.AST.Term
13
14
import Reflection.TCM.Format as Format
14
15
15
16
------------------------------------------------------------------------
@@ -29,7 +30,9 @@ open Builtin public
29
30
; getContext; extendContext; inContext; freshName
30
31
; declareDef; declarePostulate; defineFun; getType; getDefinition
31
32
; blockOnMeta; commitTC; isMacro; withNormalisation
32
- ; debugPrint; noConstraints; runSpeculative)
33
+ ; debugPrint; noConstraints; runSpeculative
34
+ ; Blocker; blockerMeta; blockerAny; blockerAll; blockTC
35
+ )
33
36
renaming (returnTC to pure)
34
37
35
38
open Format public
You can’t perform that action at this time.
0 commit comments