Skip to content
Snippets Groups Projects
Commit d72f8214 authored by Ralf Jung's avatar Ralf Jung
Browse files

fix for f_equiv improvements

parent 467fa48b
No related branches found
No related tags found
No related merge requests found
......@@ -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.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment