|
8 | 8 |
|
9 | 9 | module Reflection.AST.AlphaEquality where
|
10 | 10 |
|
11 |
| -open import Data.Bool.Base using (Bool; true; false; _∧_) |
12 |
| -open import Data.List.Base using ([]; _∷_) |
13 |
| -open import Data.Nat.Base as ℕ using (ℕ; zero; suc; _≡ᵇ_) |
14 |
| -open import Data.Product.Base using (_,_) |
15 |
| -open import Relation.Nullary.Decidable.Core using (⌊_⌋) |
16 |
| -open import Relation.Binary.Definitions using (DecidableEquality) |
17 |
| - |
18 |
| -open import Reflection.AST.Abstraction |
19 |
| -open import Reflection.AST.Argument |
20 |
| -open import Reflection.AST.Argument.Information as ArgInfo |
21 |
| -open import Reflection.AST.Argument.Modality as Modality |
22 |
| -open import Reflection.AST.Argument.Visibility as Visibility |
23 |
| -open import Reflection.AST.Meta as Meta |
24 |
| -open import Reflection.AST.Name as Name |
25 |
| -open import Reflection.AST.Literal as Literal |
| 11 | +open import Data.Bool.Base using (Bool; true; false; _∧_) |
| 12 | +open import Data.List.Base using ([]; _∷_) |
| 13 | +open import Data.Nat.Base as ℕ using (ℕ; zero; suc; _≡ᵇ_) |
| 14 | +open import Data.Product.Base using (_,_) |
| 15 | +open import Relation.Nullary.Decidable.Core using (⌊_⌋) |
| 16 | +open import Relation.Binary.Definitions using (DecidableEquality) |
| 17 | +open import Reflection.AST.Abstraction using (Abs; abs) |
| 18 | +open import Reflection.AST.Argument using (Arg; arg; Args) |
| 19 | +open import Reflection.AST.Argument.Information as ArgInfo using (ArgInfo) |
| 20 | +open import Reflection.AST.Argument.Modality as Modality using (Modality) |
| 21 | +open import Reflection.AST.Argument.Visibility as Visibility using (Visibility) |
| 22 | +open import Reflection.AST.Meta as Meta using (Meta) |
| 23 | +open import Reflection.AST.Name as Name using (Name) |
| 24 | +open import Reflection.AST.Literal as Literal using (Literal) |
26 | 25 | open import Reflection.AST.Term
|
27 | 26 | open import Level using (Level)
|
28 | 27 |
|
|
0 commit comments