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

Theorem

logic.not_to_not

Statement

∀ A B, A ⇒ B ⇒ ¬B ⇒ ¬A

Main Dependencies
Theory

Coq-Jumb
Statement

Theorem not_to_not : forall (A:Prop), forall (B:Prop), (A -> B) -> (connectives.Not B) -> connectives.Not A.



Matita-Jumb
Statement

theorem not_to_not : \forall (A:Prop). \forall (B:Prop). ((A) -> B) -> ((Not) B) -> (Not) A.



Lean-jumb
Statement

theorem not_to_not : forall (A:Prop) , forall (B:Prop) , ((A) -> B) -> (((connectives.Not) ) (B)) -> ((connectives.Not) ) (A).



PVS-jumb

Statement

not_to_not : LEMMA (FORALL(A:bool):(FORALL(B:bool):((A => B) => (connectives_sttfa_th.sttfa_Not(B) => connectives_sttfa_th.sttfa_Not(A)))))



OpenTheory

Printing for OpenTheory is not working at the moment.