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

Definition

relations.RC

Body

λR. λx. λy. (R x y) ∨ (x = y)

Main Dependencies
Theory

Coq-Jumb
Body

Definition RC : forall (A:Type), (A -> A -> Prop) -> A -> A -> Prop := fun (A:Type) => fun (R:(A -> A -> Prop)) => fun (x:A) => fun (y:A) => connectives.Or (R x y) (logic.eq (A) x y)



Matita-Jumb
Body

definition RC : \forall A : Type[0] . (A -> A -> Prop) -> A -> A -> Prop := \lambda A : Type[0]. \lambda R : A -> A -> Prop. \lambda x : A. \lambda y : A. (Or) (R x y) ((eq) (A) x y)



Lean-jumb
Body

def RC : forall (A : Type) , ((A) -> (A) -> Prop) -> (A) -> (A) -> Prop := fun (A : Type) , fun (R : (A) -> (A) -> Prop) , fun (x : A) , fun (y : A) , (((connectives.Or) ) (((R) (x)) (y))) ((((logic.eq_) (A)) (x)) (y))



PVS-jumb

Body

RC [A:TYPE+] : [[A -> [A -> bool]] -> [A -> [A -> bool]]] = (LAMBDA(R:[A -> [A -> bool]]):(LAMBDA(x:A):(LAMBDA(y:A):connectives_sttfa_th.sttfa_Or(R(x)(y))(logic_sttfa_th.eq[A](x)(y)))))



OpenTheory

Printing for OpenTheory is not working at the moment.