summaryrefslogtreecommitdiff
path: root/tests/examplefiles/test.agda
diff options
context:
space:
mode:
Diffstat (limited to 'tests/examplefiles/test.agda')
-rw-r--r--tests/examplefiles/test.agda7
1 files changed, 7 insertions, 0 deletions
diff --git a/tests/examplefiles/test.agda b/tests/examplefiles/test.agda
index d930a77b..f6cea91c 100644
--- a/tests/examplefiles/test.agda
+++ b/tests/examplefiles/test.agda
@@ -12,11 +12,18 @@ open import Data.List hiding ([_])
open import Data.Vec hiding ([_])
open import Relation.Nullary.Core
open import Relation.Binary.PropositionalEquality using (_≡_; refl; cong; trans; inspect; [_])
+ renaming (setoid to setiod)
open SemiringSolver
{- this is a {- nested -} comment -}
+postulate pierce : {A B : Set} → ((A → B) → A) → A
+
+instance
+ someBool : Bool
+ someBool = true
+
-- Factorial
_! : ℕ → ℕ
0 ! = 1