Skip to content
Snippets Groups Projects
Commit 5c33aedd authored by David Swasey's avatar David Swasey
Browse files

Weaken res_sat: We'll always keep a physical state around.

parent c2d5b157
No related branches found
No related tags found
No related merge requests found
......@@ -102,11 +102,7 @@ Module Type IRIS_PLOG (RL : RA_T) (C : CORE_LANG) (R: IRIS_RES RL C) (WP: WORLD_
Qed.
(* When is a resource okay with a state? *)
Definition res_sat (r: res) σ: Prop := r /\
match fst r with
| ex_own s => s = σ
| _ => True (* We don't care. Note that validity is ensured by the first conjunct. *)
end.
Definition res_sat (r: res) σ: Prop := r /\ fst r == ex_own state σ.
Global Instance res_sat_dist : Proper (equiv ==> equiv ==> iff) res_sat.
Proof.
......
(** Resource algebras: Commutative monoids with a decidable validity predicate. *)
(** Resource algebras: Commutative monoids with a validity predicate. *)
Require Import Bool.
Require Import Predom.
......
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