Intuitionistic Propositional Logic

Prove the following theorems ( without using tauto !).
Lemma and_assoc : forall A B C:Prop, A /\ (B /\ C) -> (A /\ B) /\ C.

Lemma and_imp_dist : forall A B C D:Prop,
                     (A -> B) /\ (C -> D) -> A /\ C -> B /\ D.

Lemma not_contrad : forall A : Prop, ~(A /\ ~A).

Lemma or_and_not : forall A B : Prop, (A\/B)/\~A -> B.

Solution

Look at this file

Note

Each of these proofs can be replaced by a simple call to tauto.


Going home
Pierre Castéran