TP-modelisation/BE2020/coq_exercice_2.v
2023-06-10 20:56:24 +02:00

18 lines
298 B
Coq
Executable file

Require Import Naturelle.
Section Session1_2020_Logique_Exercice_2.
Variable A B : Prop.
Theorem Exercice_2_Naturelle : (A -> B) -> ((~A) \/ B).
Proof.
(* A COMPLETER *)
Qed.
Theorem Exercice_2_Coq : (A -> B) -> ((~A) \/ B).
Proof.
(* A COMPLETER *)
Qed.
End Session1_2020_Logique_Exercice_2.