aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-02 22:11:54 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-02 22:23:20 +0100
commit844431761eaaf0c42d7daf3ae21de731aa230eee (patch)
tree1ad54331eb08d2b860bfaa1ae95e6a08ecec2771 /theories/Logic
parent4df1ddc6d6bd0707396337869b663b4c8f930f60 (diff)
Improving elimination with indices, getting rid of intrusive residual
local definitions...
Diffstat (limited to 'theories/Logic')
-rw-r--r--theories/Logic/EqdepFacts.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Logic/EqdepFacts.v b/theories/Logic/EqdepFacts.v
index 939fbe408..1cef233d6 100644
--- a/theories/Logic/EqdepFacts.v
+++ b/theories/Logic/EqdepFacts.v
@@ -374,13 +374,13 @@ Proof.
symmetry. apply UIP_refl. }
transitivity (eq_trans (eq_trans (UIP (eq_refl x) (eq_refl x)) z)
(eq_sym (UIP (eq_refl x) (eq_refl x)))).
- - destruct z. unfold e. destruct (UIP _ _). reflexivity.
+ - destruct z. destruct (UIP _ _). reflexivity.
- change
(match eq_refl x as y' in _ = x' return y' = y' -> Prop with
| eq_refl => fun z => z = (eq_refl (eq_refl x))
end (eq_trans (eq_trans (UIP (eq_refl x) (eq_refl x)) z)
(eq_sym (UIP (eq_refl x) (eq_refl x))))).
- destruct z. unfold e. destruct (UIP _ _). reflexivity.
+ destruct z. destruct (UIP _ _). reflexivity.
Qed.
Theorem UIP_shift : forall U, UIP_refl_ U -> forall x:U, UIP_refl_ (x = x).
Proof (fun U UIP_refl x =>