Skip to content
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
9 changes: 9 additions & 0 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -3801,6 +3801,15 @@ This is a full list of proofs that have changed form to use irrelevant instance
WellFounded _<_ → Irreflexive _≈_ _<_
```

* Added new types and operations to `Reflection.TCM`:
```
Blocker : Set
blockerMeta : Meta → Blocker
blockerAny : List Blocker → Blocker
blockerAll : List Blocker → Blocker
blockTC : Blocker → TC A
```

* Added new file `Relation.Binary.Reasoning.Base.Apartness`

This is how to use it:
Expand Down
7 changes: 5 additions & 2 deletions src/Reflection/TCM.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,8 +8,9 @@

module Reflection.TCM where

open import Reflection.AST.Term
import Agda.Builtin.Reflection as Builtin

open import Reflection.AST.Term
import Reflection.TCM.Format as Format

------------------------------------------------------------------------
Expand All @@ -29,7 +30,9 @@ open Builtin public
; getContext; extendContext; inContext; freshName
; declareDef; declarePostulate; defineFun; getType; getDefinition
; blockOnMeta; commitTC; isMacro; withNormalisation
; debugPrint; noConstraints; runSpeculative)
; debugPrint; noConstraints; runSpeculative
; Blocker; blockerMeta; blockerAny; blockerAll; blockTC
)
renaming (returnTC to pure)

open Format public
Expand Down