aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/Init/Logic.v3
1 files changed, 0 insertions, 3 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index 4bed42a0b..17d712246 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -318,19 +318,16 @@ Section Logic_lemmas.
Proof.
destruct 1; trivial.
Defined.
- Opaque eq_sym.
Theorem eq_trans : x = y -> y = z -> x = z.
Proof.
destruct 2; trivial.
Defined.
- Opaque eq_trans.
Theorem f_equal : x = y -> f x = f y.
Proof.
destruct 1; trivial.
Defined.
- Opaque f_equal.
Theorem not_eq_sym : x <> y -> y <> x.
Proof.