blob: 10c988fc02b1ea210b60cec15861d8f633ed92e6 (
plain)
1
2
3
4
5
6
7
8
9
10
|
Require Export Bool.
Lemma neg2xor : forall b, xorb true b = negb b.
Proof. auto. Qed.
Goal forall b1 b2, (negb b1 = b2) -> xorb true b1 = b2.
Proof.
intros b1 b2.
Fail rewrite neg2xor.
Abort.
|