Skip to content
Snippets Groups Projects
Commit 0d0620d5 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Try the ssreflect apply at the place the CI builder fails.

I cannot reproduce the error of the CI builder on my machine with the
same version of Coq (8.5pl2).
parent e46aa078
No related branches found
No related tags found
No related merge requests found
...@@ -94,7 +94,7 @@ Lemma wptp_result n e1 t1 v2 t2 σ1 σ2 φ : ...@@ -94,7 +94,7 @@ Lemma wptp_result n e1 t1 v2 t2 σ1 σ2 φ :
world σ1 WP e1 {{ v, φ v }} wptp t1 world σ1 WP e1 {{ v, φ v }} wptp t1
Nat.iter (S (S n)) (λ P, |=r=> P) ( φ v2). Nat.iter (S (S n)) (λ P, |=r=> P) ( φ v2).
Proof. Proof.
intros. rewrite wptp_steps // (Nat_iter_S_r (S n)); apply rvs_iter_mono. intros. rewrite wptp_steps // (Nat_iter_S_r (S n)); apply: rvs_iter_mono.
iDestruct 1 as (e2 t2') "(% & (Hw & HE & _) & H & _)"; simplify_eq. iDestruct 1 as (e2 t2') "(% & (Hw & HE & _) & H & _)"; simplify_eq.
iDestruct (wp_value_inv with "H") as "H". rewrite pvs_eq /pvs_def. iDestruct (wp_value_inv with "H") as "H". rewrite pvs_eq /pvs_def.
iVs ("H" with "[Hw HE]") as ">(_ & _ & $)"; iFrame; auto. iVs ("H" with "[Hw HE]") as ">(_ & _ & $)"; iFrame; auto.
...@@ -114,7 +114,7 @@ Lemma wptp_safe n e1 e2 t1 t2 σ1 σ2 Φ : ...@@ -114,7 +114,7 @@ Lemma wptp_safe n e1 e2 t1 t2 σ1 σ2 Φ :
world σ1 WP e1 {{ Φ }} wptp t1 world σ1 WP e1 {{ Φ }} wptp t1
Nat.iter (S (S n)) (λ P, |=r=> P) ( (is_Some (to_val e2) reducible e2 σ2)). Nat.iter (S (S n)) (λ P, |=r=> P) ( (is_Some (to_val e2) reducible e2 σ2)).
Proof. Proof.
intros ? He2. rewrite wptp_steps // (Nat_iter_S_r (S n)); apply rvs_iter_mono. intros ? He2. rewrite wptp_steps // (Nat_iter_S_r (S n)); apply: rvs_iter_mono.
iDestruct 1 as (e2' t2') "(% & Hw & H & Htp)"; simplify_eq. iDestruct 1 as (e2' t2') "(% & Hw & H & Htp)"; simplify_eq.
apply elem_of_cons in He2 as [<-|?]; first (iApply wp_safe; by iFrame "Hw H"). apply elem_of_cons in He2 as [<-|?]; first (iApply wp_safe; by iFrame "Hw H").
iApply wp_safe. iFrame "Hw". iApply wp_safe. iFrame "Hw".
......
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