// This prints the left floatting menu
Dedukti    Load Matita      Load Coq         Load Lean        Load PVS         Load OpenTheory Load
Dedukti-jumb

Definition

relations.reflexive

Body

λR. ∀ x, R x x

Main Dependencies
Theory

Coq-Jumb
Body

Definition reflexive : forall (A:Type), (A -> A -> Prop) -> Prop := fun (A:Type) => fun (R:(A -> A -> Prop)) => forall (x:A), R x x



Matita-Jumb
Body

definition reflexive : \forall A : Type[0] . (A -> A -> Prop) -> Prop := \lambda A : Type[0]. \lambda R : A -> A -> Prop. \forall (x:A). R x x



Lean-jumb
Body

def reflexive : forall (A : Type) , ((A) -> (A) -> Prop) -> Prop := fun (A : Type) , fun (R : (A) -> (A) -> Prop) , forall (x:A) , ((R) (x)) (x)



PVS-jumb

Body

reflexive [A:TYPE+] : [[A -> [A -> bool]] -> bool] = (LAMBDA(R:[A -> [A -> bool]]):(FORALL(x:A):R(x)(x)))



OpenTheory

Printing for OpenTheory is not working at the moment.