Skip to content

Commit

Permalink
Add iff versions of two stdlib bool lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
JasonGross committed Sep 18, 2023
1 parent b881f18 commit 3105f39
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions theories/Bool/Bool.v
Original file line number Diff line number Diff line change
Expand Up @@ -739,11 +739,21 @@ Qed.

Notation bool_3 := eq_true_negb_classical (only parsing). (* Compatibility *)

Lemma eq_true_negb_classical_iff : forall b:bool, negb b <> true <-> b = true.
Proof.
destr_bool; intuition.
Qed.

Lemma eq_true_not_negb : forall b:bool, b <> true -> negb b = true.
Proof.
destr_bool; intuition.
Qed.

Lemma eq_true_not_negb_iff : forall b:bool, b <> true <-> negb b = true.
Proof.
destr_bool; intuition.
Qed.

Notation bool_6 := eq_true_not_negb (only parsing). (* Compatibility *)

#[global]
Expand Down

0 comments on commit 3105f39

Please sign in to comment.