Idris2Doc : Decidable.Order.Strict
Index
Default
Alternative
Black & White
Definitions interface Irreflexive : (ty : Type ) -> (ty -> ty -> Type ) -> Type Parameters : ty, relMethods : irreflexive : Not (rel x x ) Implementation : Irreflexive Nat LT irreflexive : Irreflexive ty rel => Not (rel x x ) Totality : total Visibility : public export interface StrictPreorder : (ty : Type ) -> (ty -> ty -> Type ) -> Type Parameters : ty, relConstraints : Transitive ty rel, Irreflexive ty relImplementation : StrictPreorder Nat LT interface Asymmetric : (ty : Type ) -> (ty -> ty -> Type ) -> Type Parameters : ty, relMethods : asymmetric : rel x y -> Not (rel y x ) asymmetric : Asymmetric ty rel => rel x y -> Not (rel y x ) Totality : total Visibility : public export record EqOr : Rel t -> t -> t -> Type Totality : total Visibility : public export Constructor : MkEqOr : Either (a = b ) (spo a b ) -> EqOr spo a b Projection : .runEqOr : EqOr spo a b -> Either (a = b ) (spo a b ) Hints : (Irreflexive ty rel , Asymmetric ty rel ) => Antisymmetric ty (EqOr rel ) Connex ty rel => Connex ty (EqOr rel ) (Irreflexive ty rel , (Asymmetric ty rel , Transitive ty rel )) => PartialOrder ty (EqOr rel ) Transitive ty rel => Preorder ty (EqOr rel ) Reflexive ty (EqOr rel ) (Connex ty rel , DecEq ty ) => StronglyConnex ty (EqOr rel ) Transitive ty rel => Transitive ty (EqOr rel ) .runEqOr : EqOr spo a b -> Either (a = b ) (spo a b ) Totality : total Visibility : public export runEqOr : EqOr spo a b -> Either (a = b ) (spo a b ) Totality : total Visibility : public export data DecOrdering : t -> t -> Type Totality : total Visibility : public export Constructors : DecLT : lt a b -> DecOrdering a b DecEQ : a = b -> DecOrdering a b DecGT : lt b a -> DecOrdering a b interface StrictOrdered : (t : Type ) -> (t -> t -> Type ) -> Type Parameters : t, spoConstraints : StrictPreorder t spoMethods : order : (a : t ) -> (b : t ) -> DecOrdering a b Implementation : StrictOrdered Nat LT order : StrictOrdered t spo => (a : t ) -> (b : t ) -> DecOrdering a b Totality : total Visibility : public export Produced by Idris 2 version 0.8.0-8c970f1ba