TP-modelisation/TP2-3/enigme/enigme_Predicats_Thm01_1.v
2023-06-10 20:56:24 +02:00

28 lines
443 B
Coq

(* This file is generated by Why3's Coq driver *)
(* Beware! Only edit allowed sections below *)
Require Import BuiltIn.
Require BuiltIn.
Parameter a: Prop.
Parameter b: Prop.
Parameter c: Prop.
(* Why3 assumption *)
Definition da : Prop := b /\ ~ c.
(* Why3 assumption *)
Definition db : Prop := a -> c.
(* Why3 assumption *)
Definition dc : Prop := ~ c /\ (a \/ b).
(* Why3 goal *)
Theorem Thm01 : da /\ (db /\ dc).
Proof.
Qed.