You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
import Data.Vect
%defaulttotaldataNumber=N1|N2|N3|N4EqNumberwhereN1==N1=TrueN2==N2=TrueN3==N3=TrueN4==N4=True_==_=False
namespace All
public export
dataAll: (p : a -> Type) -> (xs : Vect n a) ->TypewhereNil: All p []
(::) : {x : a} -> p x -> All p xs -> All p (x :: xs)
namespace AllDifferent
public export
dataAllDifferent:Vect n Number ->TypewhereNil: AllDifferent []
(::) :All (\y => x == y =False) xs
->AllDifferent xs
->AllDifferent (x :: xs)
bug: AllDifferent [N1, N1, N1]
bug =%search
Issue by ziman
Wednesday May 06, 2020 at 20:03 GMT
Originally opened as edwinb/Idris2-boot#355
Steps to Reproduce
Expected Behavior
%search
fails to find the valueObserved Behavior
When I lift the lambda from the definition of
AllDifferent.(::)
, the program is correctly rejected.The text was updated successfully, but these errors were encountered: