@@ -4,40 +4,39 @@ module Reflection.Syntax where
4
4
5
5
open import Meta.Prelude
6
6
7
- open import Reflection.AST.Argument public
8
- hiding (map)
9
- open import Reflection.AST.Term public
10
- hiding (_≟_; getName)
11
- open import Reflection.AST.Name public
12
- hiding (_≟_; _≡ᵇ_; _≈_; _≈?_)
13
7
open import Reflection.AST.Definition public
14
- hiding (_≟_)
15
- open import Reflection.AST.Meta public
16
- hiding (_≟_; _≡ᵇ_; _≈_; _≈?_)
8
+ using (Definition; function; data-type; axiom; record′; constructor′; primitive′)
9
+ open import Reflection.AST.Pattern public
10
+ using (Pattern; con; dot; var; lit; proj; absurd)
11
+ open import Reflection.AST.Term public
12
+ using ( Term; pi; var; con; def; lam; pat-lam; sort; lit; meta; unknown
13
+ ; vLam; hLam; iLam; Π[_∶_]_; vΠ[_∶_]_; hΠ[_∶_]_; iΠ[_∶_]_
14
+ ; Type; Telescope
15
+ ; Sort; set; prop; propLit; inf
16
+ ; Clause; Clauses; clause; absurd-clause
17
+ )
17
18
open import Reflection.AST.Abstraction public
18
- using (unAbs)
19
-
20
- open import Agda.Builtin.Reflection public
21
- using (ArgInfo; Modality; Visibility; Literal; Meta)
22
-
19
+ using (Abs; abs; unAbs)
23
20
open import Reflection.AST.Argument public
24
- using (Arg; arg)
21
+ using (Arg; Args; arg; vArg; hArg; iArg; unArg; _⟨∷⟩_; map-Args)
22
+ open import Reflection.AST.Literal public
23
+ using (Literal)
24
+ open import Reflection.AST.Meta public
25
+ using (Meta)
26
+ open import Reflection.AST.Name public
27
+ using (Name)
25
28
open import Reflection.AST.Argument.Visibility public
26
29
using (Visibility; visible; hidden; instance′)
27
30
open import Reflection.AST.Argument.Information public
28
31
using (ArgInfo; arg-info)
29
- open import Reflection.AST.Abstraction public
30
- using (Abs; abs; unAbs )
31
- open import Reflection.AST.Argument public
32
- using (vArg; hArg; iArg; unArg; _⟨∷⟩_; map-Args )
32
+ open import Reflection.AST.Argument.Modality public
33
+ using (Modality; modality )
34
+ open import Reflection.AST.Argument.Relevance public
35
+ using (Relevance; relevant; irrelevant )
33
36
open import Reflection public
34
- using ( Name; Meta; Literal; Pattern; Clause
35
- ; ErrorPart; strErr
36
- ; Term; Type; pi; var; con; def; lam; pat-lam; agda-sort; lit; meta; unknown
37
- ; Definition; data-cons; data-type; record-type
38
- )
37
+ using (ErrorPart; strErr)
39
38
40
- open import Reflection using (hidden; instance′; TC)
39
+ open import Reflection using (TC)
41
40
42
41
-- ** Smart constructors
43
42
@@ -103,7 +102,7 @@ pattern _◇ n = Pattern.con n []
103
102
pattern _◇⟦_⟧ n x = Pattern.con n (vArg x ∷ [])
104
103
pattern _◇⟦_∣_⟧ n x y = Pattern.con n (vArg x ∷ vArg y ∷ [])
105
104
106
- pattern `Set = agda- sort (set (quote 0ℓ ∙))
105
+ pattern `Set = sort (set (quote 0ℓ ∙))
107
106
108
107
-- ** useful type aliases
109
108
PatTelescope = Telescope
0 commit comments