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

move gmap_view_check to tests/algebra.v

parent 8862cf75
No related branches found
No related tags found
No related merge requests found
From iris.algebra Require Import auth excl.
From iris.algebra Require Import auth excl lib.gmap_view.
From iris.base_logic.lib Require Import invariants.
(** Make sure that the same [Equivalence] instance is picked for Leibniz OFEs
......@@ -48,3 +48,9 @@ Section test_prod.
Persistent (PROP:=iPropI Σ) (own γ (((None, None), Some (to_agree true)))).
Proof. apply _. Qed.
End test_prod.
(** Make sure the [auth]/[gmap_view] notation does not mix up its arguments. *)
Definition auth_check {A : ucmraT} :
auth A = authO A := eq_refl.
Definition gmap_view_check {K : Type} `{Countable K} {V : ofeT} :
gmap_view K V = gmap_viewO K V := eq_refl.
......@@ -104,10 +104,6 @@ Definition gmap_viewR (K : Type) `{Countable K} (V : ofeT) : cmraT :=
Definition gmap_viewUR (K : Type) `{Countable K} (V : ofeT) : ucmraT :=
viewUR (gmap_view_rel K V).
(** Make sure the notation does not mix up its arguments. *)
Local Definition gmap_view_check {K : Type} `{Countable K} {V : ofeT} :
gmap_view K V = gmap_viewO K V := eq_refl.
Section definitions.
Context {K : Type} `{Countable K} {V : ofeT}.
......
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