diff --git a/iris/bi/internal_eq.v b/iris/bi/internal_eq.v index 65dec0d2847fae830dc5c258c79ac6c291a1ed6c..6dd1a42a78b717e431691b4e8228639d903dcaec 100644 --- a/iris/bi/internal_eq.v +++ b/iris/bi/internal_eq.v @@ -180,7 +180,6 @@ Lemma discrete_fun_equivI {A} {B : A → ofe} (f g : discrete_fun B) : f ≡ g Proof. apply (anti_symm _); auto using fun_extI. apply (internal_eq_rewrite' f g (λ g, ∀ x : A, f x ≡ g x)%I); auto. - intros n h h' Hh; apply forall_ne=> x; apply internal_eq_ne; auto. Qed. Lemma ofe_morO_equivI {A B : ofe} (f g : A -n> B) : f ≡ g ⊣⊢ ∀ x, f x ≡ g x. Proof.