24 lines
372 B
Coq
Executable file
24 lines
372 B
Coq
Executable file
Require Import Naturelle.
|
|
Section Session1_2019_Logique_Exercice_1.
|
|
|
|
Variable A B C : Prop.
|
|
|
|
Theorem Exercice_1_Coq : (A -> B -> C) -> ((A /\ B) -> C).
|
|
intros.
|
|
cut B.
|
|
cut A.
|
|
exact H.
|
|
destruct H0.
|
|
exact H0.
|
|
destruct H0.
|
|
exact H1.
|
|
Qed.
|
|
|
|
Theorem Exercice_1_Naturelle : (A -> B -> C) -> ((A /\ B) -> C).
|
|
Proof.
|
|
(* A COMPLETER *)
|
|
Qed.
|
|
|
|
End Session1_2019_Logique_Exercice_1.
|
|
|