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

Notations for X ⊆ Y ⊆ Z.

parent d0131be5
No related branches found
No related tags found
No related merge requests found
...@@ -637,6 +637,11 @@ Notation "(⊄)" := (λ X Y, X ⊄ Y) (only parsing) : C_scope. ...@@ -637,6 +637,11 @@ Notation "(⊄)" := (λ X Y, X ⊄ Y) (only parsing) : C_scope.
Notation "( X ⊄ )" := (λ Y, X Y) (only parsing) : C_scope. Notation "( X ⊄ )" := (λ Y, X Y) (only parsing) : C_scope.
Notation "( ⊄ X )" := (λ Y, Y X) (only parsing) : C_scope. Notation "( ⊄ X )" := (λ Y, Y X) (only parsing) : C_scope.
Notation "X ⊆ Y ⊆ Z" := (X Y Y Z) (at level 70, Y at next level) : C_scope.
Notation "X ⊆ Y ⊂ Z" := (X Y Y Z) (at level 70, Y at next level) : C_scope.
Notation "X ⊂ Y ⊆ Z" := (X Y Y Z) (at level 70, Y at next level) : C_scope.
Notation "X ⊂ Y ⊂ Z" := (X Y Y Z) (at level 70, Y at next level) : C_scope.
(** The class [Lexico A] is used for the lexicographic order on [A]. This order (** The class [Lexico A] is used for the lexicographic order on [A]. This order
is used to create finite maps, finite sets, etc, and is typically different from is used to create finite maps, finite sets, etc, and is typically different from
the order [(⊆)]. *) the order [(⊆)]. *)
......
...@@ -34,7 +34,7 @@ Qed. ...@@ -34,7 +34,7 @@ Qed.
(** Fairly explicit form of opening invariants *) (** Fairly explicit form of opening invariants *)
Lemma inv_open E N P : Lemma inv_open E N P :
nclose N E nclose N E
inv N P E', (E nclose N E' E' E) inv N P E', (E nclose N E' E)
|={E,E'}=> P ( P ={E',E}=★ True). |={E,E'}=> P ( P ={E',E}=★ True).
Proof. Proof.
rewrite /inv. iIntros {?} "Hinv". iDestruct "Hinv" as {i} "[% #Hi]". rewrite /inv. iIntros {?} "Hinv". iDestruct "Hinv" as {i} "[% #Hi]".
......
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