Skip to content

Commit afea968

Browse files
committed
[ cleanup ] Use So and All from base in tests
1 parent 3b58e1c commit afea968

File tree

2 files changed

+5
-20
lines changed

2 files changed

+5
-20
lines changed

tests/idris2/with/with012/WithProof0ElabFail.idr

Lines changed: 2 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,7 @@
11
module WithProof0ElabFail
22

3+
import Data.So
4+
import Data.List.Quantifiers
35
import Language.Reflection
46

57
%default total
@@ -8,16 +10,6 @@ import Language.Reflection
810

911
%hide List.filter
1012

11-
data So : Bool -> Type where
12-
Oh : So True
13-
14-
eqToSo : b = True -> So b
15-
eqToSo Refl = Oh
16-
17-
data All : (0 p : a -> Type) -> List a -> Type where
18-
Nil : All p Nil
19-
(::) : {0 xs : List a} -> p x -> All p xs -> All p (x :: xs)
20-
2113
filter : (p : a -> Bool) -> (xs : List a) -> List a
2214
filter p [] = []
2315
filter p (x :: xs) with (p x)

tests/idris2/with/with012/WithProof0Fail.idr

Lines changed: 3 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -1,19 +1,12 @@
11
module WithProof0Fail
22

3+
import Data.So
4+
import Data.List.Quantifiers
5+
36
%default total
47

58
%hide List.filter
69

7-
data So : Bool -> Type where
8-
Oh : So True
9-
10-
eqToSo : b = True -> So b
11-
eqToSo Refl = Oh
12-
13-
data All : (0 p : a -> Type) -> List a -> Type where
14-
Nil : All p Nil
15-
(::) : {0 xs : List a} -> p x -> All p xs -> All p (x :: xs)
16-
1710
filter : (p : a -> Bool) -> (xs : List a) -> List a
1811
filter p [] = []
1912
filter p (x :: xs) with (p x)

0 commit comments

Comments
 (0)