File tree Expand file tree Collapse file tree 1 file changed +5
-0
lines changed Expand file tree Collapse file tree 1 file changed +5
-0
lines changed Original file line number Diff line number Diff line change @@ -24,6 +24,7 @@ open import Relation.Nullary.Decidable.Core using (yes; no)
24
24
25
25
open import Reflection.AST.Abstraction hiding (map)
26
26
open import Reflection.AST.Argument hiding (map)
27
+ open import Reflection.AST.Argument.Quantity
27
28
open import Reflection.AST.Argument.Relevance
28
29
open import Reflection.AST.Argument.Visibility
29
30
open import Reflection.AST.Argument.Modality
@@ -58,6 +59,10 @@ showVisibility visible = "visible"
58
59
showVisibility hidden = "hidden"
59
60
showVisibility instance′ = "instance"
60
61
62
+ showQuantity : Quantity → String
63
+ showQuantity quantity-0 = "quantity-0"
64
+ showQuantity quantity-ω = "quantity-ω"
65
+
61
66
showLiteral : Literal → String
62
67
showLiteral (nat x) = ℕ.show x
63
68
showLiteral (word64 x) = ℕ.show (Word64.toℕ x)
You can’t perform that action at this time.
0 commit comments