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

Theorem

logic.proj1

Statement

∀ A B, A ∧ B ⇒ A

Main Dependencies
Theory

Coq-Jumb
Statement

Theorem proj1 : forall (A:Prop), forall (B:Prop), (connectives.And A B) -> A.



Matita-Jumb
Statement

theorem proj1 : \forall (A:Prop). \forall (B:Prop). ((And) A B) -> A.



Lean-jumb
Statement

theorem proj1 : forall (A:Prop) , forall (B:Prop) , ((((connectives.And) ) (A)) (B)) -> A.



PVS-jumb

Statement

proj1 : LEMMA (FORALL(A:bool):(FORALL(B:bool):(connectives_sttfa_th.sttfa_And(A)(B) => A)))



OpenTheory

Printing for OpenTheory is not working at the moment.