Skip to content
Snippets Groups Projects
Commit 803e091e authored by Gregory Malecha's avatar Gregory Malecha
Browse files

adding fixme

parent c1a30c58
No related branches found
No related tags found
No related merge requests found
...@@ -150,10 +150,10 @@ s/\blist_singletonM_included\b/list_singleton_included/g ...@@ -150,10 +150,10 @@ s/\blist_singletonM_included\b/list_singleton_included/g
* New ASCII versions of Iris notations. These are marked printing only and * New ASCII versions of Iris notations. These are marked printing only and
can be made available using `Require Import iris.bi.ascii`. The new can be made available using `Require Import iris.bi.ascii`. The new
notation is († disambiguated using notation scopes): notations are (notations marked [†] are disambiguated using notation scopes):
- entailment: `|--` for `⊢` and `-|-` for `⊣⊢` - entailment: `|--` for `⊢` and `-|-` for `⊣⊢`
- logic: `->` for `→`, `/\\` for `∧`, `\\/` for `∨`, and `<->` for `↔` - logic[†]: `->` for `→`, `/\\` for `∧`, `\\/` for `∨`, and `<->` for `↔`
- quantifiers: `forall` for `∀` and `exists` for `∃` - quantifiers[†]: `forall` for `∀` and `exists` for `∃`
- separation logic: `**` for `∗`, `-*` for `-∗`, and `*-*` for `∗-∗` - separation logic: `**` for `∗`, `-*` for `-∗`, and `*-*` for `∗-∗`
- step indexing: `|>` for `▷` - step indexing: `|>` for `▷`
- modalities: `<intuit>` for `□` and `<except_0>` for `◇` - modalities: `<intuit>` for `□` and `<except_0>` for `◇`
...@@ -165,8 +165,8 @@ s/\blist_singletonM_included\b/list_singleton_included/g ...@@ -165,8 +165,8 @@ s/\blist_singletonM_included\b/list_singleton_included/g
- `P ={E1,E2}=* Q` for `P ={E1,E2}=∗ Q` - `P ={E1,E2}=* Q` for `P ={E1,E2}=∗ Q`
- `|={E1,E2,E3}|>=> Q` for `|={E1,E2,E3}▷=> Q` - `|={E1,E2,E3}|>=> Q` for `|={E1,E2,E3}▷=> Q`
- `|={E1,E2}|>=>^n Q` for `|={E1,E2}▷=>^n Q` - `|={E1,E2}|>=>^n Q` for `|={E1,E2}▷=>^n Q`
The full list can be found in [theories/bi/ascii.v](theories/bi/ascii.v), where the ASCII notations The full list can be found in [theories/bi/ascii.v](theories/bi/ascii.v),
are defined in terms of the unicode notations. where the ASCII notations are defined in terms of the unicode notations.
**Changes in heap_lang:** **Changes in heap_lang:**
......
...@@ -2,22 +2,24 @@ From iris.bi Require Import interface derived_connectives updates. ...@@ -2,22 +2,24 @@ From iris.bi Require Import interface derived_connectives updates.
From iris.algebra Require Export ofe. From iris.algebra Require Export ofe.
(** note: we use [|--] instead of [|-] because the latter is used by (** note: we use [|--] instead of [|-] because the latter is used by
Ltac's [match goal] construct Ltac's [match goal] construct.
*) *)
Notation "P |-- Q" := (P Q) Notation "P |-- Q" := (P Q)
(at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope. (at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope.
Notation "P '|--@{' PROP } Q" := (P ⊢@{PROP} Q) (at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope. Notation "P '|--@{' PROP } Q" := (P ⊢@{PROP} Q) (at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope.
Notation "(|--)" := () (only parsing) : stdpp_scope. Notation "(|--)" := () (only parsing) : stdpp_scope.
(* FIXME: fix notation *)
Notation "('|--@{' PROP } )" := (bi_entails (PROP:=PROP)) (only parsing) : stdpp_scope. Notation "('|--@{' PROP } )" := (bi_entails (PROP:=PROP)) (only parsing) : stdpp_scope.
Notation "|-- Q" := ( Q%I) (at level 20, Q at level 200, only parsing) : stdpp_scope.
Notation "'|--@{' PROP } Q" := (⊢@{PROP} Q) (at level 20, Q at level 200, only parsing) : stdpp_scope.
Notation "P -|- Q" := (P ⊣⊢ Q) (at level 95, no associativity, only parsing) : stdpp_scope. Notation "P -|- Q" := (P ⊣⊢ Q) (at level 95, no associativity, only parsing) : stdpp_scope.
Notation "P '-|-@{' PROP } Q" := (P ⊣⊢@{PROP} Q) (at level 95, no associativity, only parsing) : stdpp_scope. Notation "P '-|-@{' PROP } Q" := (P ⊣⊢@{PROP} Q) (at level 95, no associativity, only parsing) : stdpp_scope.
Notation "(-|-)" := (⊣⊢) (only parsing) : stdpp_scope. Notation "(-|-)" := (⊣⊢) (only parsing) : stdpp_scope.
(* FIXME: fix notation *)
Notation "('-|-@{' PROP } )" := (equiv (A:=bi_car PROP)) (only parsing) : stdpp_scope. Notation "('-|-@{' PROP } )" := (equiv (A:=bi_car PROP)) (only parsing) : stdpp_scope.
Notation "|-- Q" := ( Q%I) (at level 20, Q at level 200, only parsing) : stdpp_scope.
Notation "'|--@{' PROP } Q" := (⊢@{PROP} Q) (at level 20, Q at level 200, only parsing) : stdpp_scope.
Notation "P -* Q" := (P Q)%stdpp (at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope. Notation "P -* Q" := (P Q)%stdpp (at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope.
(* FIXME: Notation "'⌜' φ '⌝'" := (bi_pure φ%type%stdpp) : bi_scope. *) (* FIXME: Notation "'⌜' φ '⌝'" := (bi_pure φ%type%stdpp) : bi_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