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

Definition

relations.injective

Body

λf. ∀ x y, (f x) = (f y) ⇒ x = y

Main Dependencies
constant
Theory
constant

Coq-Jumb
Body

Definition injective : forall (A:Type), forall (B:Type), (A -> B) -> Prop := fun (A:Type) => fun (B:Type) => fun (f:(A -> B)) => forall (x:A), forall (y:A), (logic.eq (B) (f x) (f y)) -> logic.eq (A) x y



Matita-Jumb
Body

definition injective : \forall A : Type[0] . \forall B : Type[0] . (A -> B) -> Prop := \lambda A : Type[0]. \lambda B : Type[0]. \lambda f : A -> B. \forall (x:A). \forall (y:A). ((eq) (B) (f x) (f y)) -> (eq) (A) x y



Lean-jumb
Body

def injective : forall (A : Type) , forall (B : Type) , ((A) -> B) -> Prop := fun (A : Type) , fun (B : Type) , fun (f : (A) -> B) , forall (x:A) , forall (y:A) , ((((logic.eq_) (B)) ((f) (x))) ((f) (y))) -> (((logic.eq_) (A)) (x)) (y)



PVS-jumb

Body

injective [A:TYPE+,B:TYPE+] : [[A -> B] -> bool] = (LAMBDA(f:[A -> B]):(FORALL(x:A):(FORALL(y:A):(logic_sttfa_th.eq[B](f(x))(f(y)) => logic_sttfa_th.eq[A](x)(y)))))



OpenTheory

Printing for OpenTheory is not working at the moment.