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

Theorem

cong.transitive_congruent

Statement

∀ p, transitive (λn. λm. n ≡ m [p])

Main Dependencies
Theory

Coq-Jumb
Statement

Theorem transitive_congruent : forall (p:nat.nat), relations.transitive (nat.nat) (fun (n:nat.nat) => fun (m:nat.nat) => congruent n m p).



Matita-Jumb
Statement

theorem transitive_congruent : \forall (p:nat). (transitive) (nat) (\lambda n : nat. \lambda m : nat. (congruent) n m p).



Lean-jumb
Statement

theorem transitive_congruent : forall (p:nat.nat) , ((relations.transitive) (nat.nat)) (fun (n : nat.nat) , fun (m : nat.nat) , ((((cong.congruent) ) (n)) (m)) (p)).



PVS-jumb

Statement

transitive_congruent : LEMMA (FORALL(p:nat_sttfa_th.sttfa_nat):relations_sttfa_th.transitive[nat_sttfa_th.sttfa_nat]((LAMBDA(n:nat_sttfa_th.sttfa_nat):(LAMBDA(m:nat_sttfa_th.sttfa_nat):cong_sttfa.congruent(n)(m)(p)))))



OpenTheory

Printing for OpenTheory is not working at the moment.