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

Tweak.

parent 0d55d5de
No related branches found
No related tags found
No related merge requests found
...@@ -3,7 +3,6 @@ From osiris.channel Require Import proto_channel proofmode. ...@@ -3,7 +3,6 @@ From osiris.channel Require Import proto_channel proofmode.
From iris.heap_lang Require Import proofmode notation. From iris.heap_lang Require Import proofmode notation.
From iris.heap_lang Require Import assert. From iris.heap_lang Require Import assert.
From osiris.utils Require Import list compare spin_lock contribution. From osiris.utils Require Import list compare spin_lock contribution.
From osiris.examples Require Import sort_elem.
From iris.algebra Require Import gmultiset. From iris.algebra Require Import gmultiset.
Definition mapper : val := Definition mapper : val :=
...@@ -47,14 +46,14 @@ Definition mapper_service : val := λ: "n" "f" "xs", ...@@ -47,14 +46,14 @@ Definition mapper_service : val := λ: "n" "f" "xs",
start_mappers "n" "f" "l" "c") in start_mappers "n" "f" "l" "c") in
mapper_service_loop "n" "c" "xs" (lnil #()). mapper_service_loop "n" "c" "xs" (lnil #()).
Class map_sortG Σ A `{Countable A} := { Class mapperG Σ A `{Countable A} := {
map_sort_contributionG :> contributionG Σ (gmultisetUR A); mapper_contributionG :> contributionG Σ (gmultisetUR A);
map_sort_lockG :> lockG Σ; mapper_lockG :> lockG Σ;
}. }.
Section mapper. Section mapper.
Context `{Countable A, Countable B}. Context `{Countable A, Countable B}.
Context `{!heapG Σ, !proto_chanG Σ, map_sortG Σ A} (N : namespace). Context `{!heapG Σ, !proto_chanG Σ, mapperG Σ A} (N : namespace).
Context (IA : A val iProp Σ) (IB : B val iProp Σ) (f : A B). Context (IA : A val iProp Σ) (IB : B val iProp Σ) (f : A B).
Local Open Scope nat_scope. Local Open Scope nat_scope.
......
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