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
module WF
Pred:Type->TypePred a = a ->TypeSubset: Pred a -> Pred a ->TypeSubset {a} P1P2= {x: a} -> P1 x -> P2 x
subsetBuild: (a : Type) -> (Q : Pred a) -> (Rec : Pred a -> Pred a) ->
((P : Pred a) -> Rec P `Subset` P -> Q `Subset` Rec P) ->
((P : Pred a) -> Rec P `Subset` P -> Q `Subset` P)
subsetBuild a QRec builder P f x q = f x (builder P f x q)
The text was updated successfully, but these errors were encountered:
Rel: (a : Type) ->TypeRel a = a -> a ->Type||| Take the transitive closure of a relationdataTC: Rel t -> Rel t whereTCIncl: r x y -> TC r x y
TCTrans: TC r x y -> TC r y z -> TC r x z
class Transitive (rel : Rel a) wheretrans: x `rel` y -> y `rel` z -> x `rel` z
TransitiveR: Rel a ->TypeTransitiveR {a} rel = {x,y,z:a} -> x `rel` y -> y `rel` z -> x `rel` z
instance Transitive (TC rel) where
trans xRy yRz =TCTrans xRy yRz
Type checking ./test.idr
test.idr:12:13:When checking left hand side of subsetBuild:
subsetBuild a QRec builder P f x x does not have a function type (P x)
Holes: WF.subsetBuild
The error message is rather short:
The code producing it is also reasonably short:
The text was updated successfully, but these errors were encountered: