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

bump std++; fix for f_equiv improvements

parent 467fa48b
No related branches found
No related tags found
No related merge requests found
...@@ -15,7 +15,7 @@ iris.prelude, iris.algebra, iris.si_logic, iris.bi, iris.proofmode, iris.base_lo ...@@ -15,7 +15,7 @@ iris.prelude, iris.algebra, iris.si_logic, iris.bi, iris.proofmode, iris.base_lo
depends: [ depends: [
"coq" { (>= "8.12" & < "8.15~") | (= "dev") } "coq" { (>= "8.12" & < "8.15~") | (= "dev") }
"coq-stdpp" { (= "dev.2021-09-06.1.64419715") | (= "dev") } "coq-stdpp" { (= "dev.2021-09-27.0.7d5f3593") | (= "dev") }
] ]
build: ["./make-package" "iris" "-j%{jobs}%"] build: ["./make-package" "iris" "-j%{jobs}%"]
......
...@@ -180,7 +180,6 @@ Lemma discrete_fun_equivI {A} {B : A → ofe} (f g : discrete_fun B) : f ≡ g ...@@ -180,7 +180,6 @@ Lemma discrete_fun_equivI {A} {B : A → ofe} (f g : discrete_fun B) : f ≡ g
Proof. Proof.
apply (anti_symm _); auto using fun_extI. apply (anti_symm _); auto using fun_extI.
apply (internal_eq_rewrite' f g (λ g, x : A, f x g x)%I); auto. 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. Qed.
Lemma ofe_morO_equivI {A B : ofe} (f g : A -n> B) : f g ⊣⊢ x, f x g x. Lemma ofe_morO_equivI {A B : ofe} (f g : A -n> B) : f g ⊣⊢ x, f x g x.
Proof. Proof.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment