aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Program
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2016-08-19 15:04:04 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2016-08-19 15:04:04 +0200
commit05f3192fedc354eb34ac10813bd7f1ffadfd4405 (patch)
tree67f1c62bf665d76ddc46aba734100e43132ddec4 /theories/Program
parentdd9ee0c788556640f47a797814ffddba76ae540f (diff)
parent4c0c4b46993aeb31786d60cb278cfb317dea454e (diff)
Merge remote-tracking branch 'origin/pr/246' into v8.6
Diffstat (limited to 'theories/Program')
-rw-r--r--theories/Program/Equality.v5
-rw-r--r--theories/Program/Subset.v1
2 files changed, 3 insertions, 3 deletions
diff --git a/theories/Program/Equality.v b/theories/Program/Equality.v
index a349eb908..d6f9bb9df 100644
--- a/theories/Program/Equality.v
+++ b/theories/Program/Equality.v
@@ -8,7 +8,6 @@
(** Tactics related to (dependent) equality and proof irrelevance. *)
-Require Export ProofIrrelevance.
Require Export JMeq.
Require Import Coq.Program.Tactics.
@@ -143,7 +142,7 @@ Ltac pi_eq_proof_hyp p :=
| [ H : X = Y |- _ ] =>
match p with
| H => fail 2
- | _ => rewrite (proof_irrelevance (X = Y) p H)
+ | _ => rewrite (UIP _ X Y p H)
end
| _ => fail " No hypothesis with same type "
end
@@ -166,7 +165,7 @@ Hint Rewrite <- eq_rect_eq : refl_id.
[coerce_* t eq_refl = t]. *)
Lemma JMeq_eq_refl {A} (x : A) : JMeq_eq (@JMeq_refl _ x) = eq_refl.
-Proof. apply proof_irrelevance. Qed.
+Proof. apply UIP. Qed.
Lemma UIP_refl_refl A (x : A) :
Eqdep.EqdepTheory.UIP_refl A x eq_refl = eq_refl.
diff --git a/theories/Program/Subset.v b/theories/Program/Subset.v
index c8f37318d..2a3ec926b 100644
--- a/theories/Program/Subset.v
+++ b/theories/Program/Subset.v
@@ -9,6 +9,7 @@
Require Import Coq.Program.Utils.
Require Import Coq.Program.Equality.
+Require Export ProofIrrelevance.
Local Open Scope program_scope.