Skip to content

Commit

Permalink
Add simple test for implicit binding around quotes
Browse files Browse the repository at this point in the history
  • Loading branch information
mb64 committed Aug 7, 2020
1 parent 8f54466 commit e73fdac
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions tests/idris2/reflection004/refdecl.idr
Expand Up @@ -4,6 +4,12 @@ import Language.Reflection

%language ElabReflection

fc : FC
fc = EmptyFC

quoteTest : TTImp -> TTImp -> List Decl
quoteTest f arg = `[ myFunc : ~(IApp fc f arg) ]

axes : (n : Nat) -> {auto gt : GT n 0} -> {auto lte : LTE n 4} -> Vect n String
axes 1 = ["x"]
axes 2 = "y" :: axes 1
Expand Down

0 comments on commit e73fdac

Please sign in to comment.