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

some minor changes for better 8.5-compatibility

parent 024e8089
No related branches found
No related tags found
No related merge requests found
Require Import ssreflect. Require Import Ssreflect.ssreflect.
Require Import world_prop core_lang lang iris_core iris_plog iris_vs_rules iris_ht_rules. Require Import world_prop core_lang lang iris_core iris_plog iris_vs_rules iris_ht_rules.
Require Import ModuRes.RA ModuRes.SPred ModuRes.BI ModuRes.PreoMet ModuRes.Finmap ModuRes.CMRA ModuRes.DecEnsemble. Require Import ModuRes.RA ModuRes.SPred ModuRes.BI ModuRes.PreoMet ModuRes.Finmap ModuRes.CMRA ModuRes.DecEnsemble.
......
...@@ -248,7 +248,8 @@ Module Type IRIS_PLOG (RL : VIRA_T) (C : CORE_LANG) (R: IRIS_RES RL C) (WP: WORL ...@@ -248,7 +248,8 @@ Module Type IRIS_PLOG (RL : VIRA_T) (C : CORE_LANG) (R: IRIS_RES RL C) (WP: WORL
exists w', P w' (S (S k)) exists w', P w' (S (S k))
/\ wsat σ (m2 mf) (w' · wf) (S (S k)))]. /\ wsat σ (m2 mf) (w' · wf) (S (S k)))].
Next Obligation. Next Obligation.
inversion HLe. repeat intro.
by inversion HLe.
Qed. Qed.
Next Obligation. Next Obligation.
intros n1 n2 HLe HP wf; intros. intros n1 n2 HLe HP wf; intros.
......
...@@ -165,7 +165,7 @@ Module Type IRIS_VS_RULES (RL : VIRA_T) (C : CORE_LANG) (R: IRIS_RES RL C) (WP: ...@@ -165,7 +165,7 @@ Module Type IRIS_VS_RULES (RL : VIRA_T) (C : CORE_LANG) (R: IRIS_RES RL C) (WP:
- exists (w2, wq). split; last split. - exists (w2, wq). split; last split.
+ rewrite [ra_op]lock. simpl. reflexivity. + rewrite [ra_op]lock. simpl. reflexivity.
+ assumption. + assumption.
+ apply propsMN, HQ. omega. + eapply propsMN, HQ. omega.
- now rewrite -assoc. - now rewrite -assoc.
Qed. Qed.
......
Require Import ssreflect. Require Import Ssreflect.ssreflect Omega.
Require Import Arith Min Max List ListSet Lists.
Require Import MetricCore. Require Import MetricCore.
Require Import PreoMet. Require Import PreoMet.
Require Import RA CMRA SPred. Require Import RA CMRA SPred.
Require Import Arith Min Max List ListSet Lists.
Set Bullet Behavior "Strict Subproofs". Set Bullet Behavior "Strict Subproofs".
...@@ -548,11 +548,11 @@ Section FinDom. ...@@ -548,11 +548,11 @@ Section FinDom.
refine (fix F (l: list K) := refine (fix F (l: list K) :=
match l as l return (forall f, dom f = l -> T f) with match l as l return (forall f, dom f = l -> T f) with
| [] => fun f Hdom => Text fdEmpty f _ Temp | [] => fun f Hdom => Text fdEmpty f _ Temp
| k::l => fun f Hdom => let f' := f \ k in | k::l' => fun f Hdom => let f' := f \ k in
let Hindom: k dom f := _ in let Hindom: k dom f := _ in
let v' := fdLookup_indom f k Hindom in let v' := fdLookup_indom f k Hindom in
Text (fdStrongUpdate k (Some v') f') f _ Text (fdStrongUpdate k (Some v') f') f _
(Tstep k v' f' _ (F l f' _)) (Tstep k v' f' _ (F l' f' _))
end); clear F. end); clear F.
- split. - split.
+ move=>k /=. symmetry. apply fdLookup_notin_strong. rewrite Hdom. tauto. + move=>k /=. symmetry. apply fdLookup_notin_strong. rewrite Hdom. tauto.
...@@ -566,7 +566,7 @@ Section FinDom. ...@@ -566,7 +566,7 @@ Section FinDom.
+ rewrite Hdom /dom /=. f_equal. rewrite /dom /= Hdom. + rewrite Hdom /dom /=. f_equal. rewrite /dom /= Hdom.
rewrite DecEq_refl. rewrite DecEq_refl.
assert (Hnod := dom_nodup f). rewrite Hdom in Hnod. assert (Hnod := dom_nodup f). rewrite Hdom in Hnod.
assert (Hfilt1: (filter_dupes [] l0) = l0). assert (Hfilt1: (filter_dupes [] l') = l').
{ apply filter_dupes_id. simpl. inversion Hnod; subst. assumption. } { apply filter_dupes_id. simpl. inversion Hnod; subst. assumption. }
rewrite Hfilt1. apply filter_dupes_id. assumption. rewrite Hfilt1. apply filter_dupes_id. assumption.
- subst f'. apply fdLookup_notin. rewrite fdStrongUpdate_eq. reflexivity. - subst f'. apply fdLookup_notin. rewrite fdStrongUpdate_eq. reflexivity.
...@@ -581,20 +581,6 @@ Section FinDom. ...@@ -581,20 +581,6 @@ Section FinDom.
fun f => fdRectInner (dom f) f eq_refl. fun f => fdRectInner (dom f) f eq_refl.
End Recursion. End Recursion.
(* No need to restrict this Lemma to fdRectInner - that just messes up the details. *)
(* Lemma fdRectInner_eqL l l' f (Heq: dom f = l) (Heq': dom f = l')
(T: (K -f> V) -> Type) (F: forall l (f: K -f> V), dom f = l -> T f) :
F l f Heq = F l' f Heq'.
Proof.
assert (Heql: l = l').
{ transitivity (dom f); first symmetry; assumption. }
revert Heq'.
refine (match Heql in eq _ l'' return (forall Heq' : dom f = l'', F l f Heq = F l'' f Heq') with
| eq_refl => _
end).
move=>Heq'. reflexivity.
Qed. *)
Section Fold. Section Fold.
Context {T: Type}. Context {T: Type}.
Context (Temp: T) (Tstep: K -> V -> T -> T). Context (Temp: T) (Tstep: K -> V -> T -> T).
......
...@@ -71,5 +71,3 @@ Ltac contradiction_eq := match goal with ...@@ -71,5 +71,3 @@ Ltac contradiction_eq := match goal with
(* Well-founded induction. *) (* Well-founded induction. *)
Definition wf_nat_ind := well_founded_induction Wf_nat.lt_wf. Definition wf_nat_ind := well_founded_induction Wf_nat.lt_wf.
\ No newline at end of file
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