From a00d9bd814bc97622b2e9cf86c0a78e300680f70 Mon Sep 17 00:00:00 2001 From: "Paolo G. Giarrusso" <p.giarrusso@gmail.com> Date: Mon, 30 Mar 2020 01:03:30 +0200 Subject: [PATCH] Replace explicit use of Inj instances by inj This was inconsistent and not explained before. --- theories/namespaces.v | 2 +- theories/option.v | 4 ++-- 2 files changed, 3 insertions(+), 3 deletions(-) diff --git a/theories/namespaces.v b/theories/namespaces.v index c135f3bb..2d5038c0 100644 --- a/theories/namespaces.v +++ b/theories/namespaces.v @@ -58,7 +58,7 @@ Section namespace. intros Hxy a. unfold up_close. rewrite !nclose_eq, !ndot_eq. unfold nclose_def, ndot_def; rewrite !elem_coPset_suffixes. intros [qx ->] [qy Hqy]. - revert Hqy. by intros [= ?%encode_inj]%positives_flatten_suffix_eq. + revert Hqy. by intros [= ?%(inj _)]%positives_flatten_suffix_eq. Qed. Lemma ndot_preserve_disjoint_l N E x : ↑N ## E → ↑N.@x ## E. diff --git a/theories/option.v b/theories/option.v index 9ba258be..f658505e 100644 --- a/theories/option.v +++ b/theories/option.v @@ -189,8 +189,8 @@ Lemma fmap_Some_equiv {A B} `{Equiv B} `{!Equivalence (≡@{B})} (f : A → B) m f <$> mx ≡ Some y ↔ ∃ x, mx = Some x ∧ y ≡ f x. Proof. destruct mx; simpl; split. - - intros ?%Some_equiv_inj. eauto. - - intros (? & ->%Some_inj & ?). constructor. done. + - intros ?%(inj _). eauto. + - intros (? & ->%(inj _) & ?). constructor. done. - intros ?%symmetry%equiv_None. done. - intros (? & ? & ?). done. Qed. -- GitLab