aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/Eqdep_dec.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Logic/Eqdep_dec.v')
-rw-r--r--theories/Logic/Eqdep_dec.v11
1 files changed, 5 insertions, 6 deletions
diff --git a/theories/Logic/Eqdep_dec.v b/theories/Logic/Eqdep_dec.v
index 0758bd1f9..e4adc8cf1 100644
--- a/theories/Logic/Eqdep_dec.v
+++ b/theories/Logic/Eqdep_dec.v
@@ -63,10 +63,10 @@ Section EqdepDec.
Let nu_constant : forall (y:A) (u v:x = y), nu u = nu v.
intros.
unfold nu.
- case (eq_dec y); intros.
+ destruct (eq_dec y) as [Heq|Hneq].
reflexivity.
- case n; trivial.
+ case Hneq; trivial.
Qed.
@@ -117,12 +117,11 @@ Section EqdepDec.
intros.
cut (proj (ex_intro P x y) y = proj (ex_intro P x y') y).
simpl.
- case (eq_dec x).
- intro e.
- elim e using K_dec_one_var; trivial.
+ destruct (eq_dec x) as [Heq|Hneq].
+ elim Heq using K_dec_one_var; trivial.
intros.
- case n; trivial.
+ case Hneq; trivial.
case H.
reflexivity.