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

Fix typo siPropC → siPropO.

parent 225cac4f
No related branches found
No related tags found
No related merge requests found
...@@ -33,15 +33,15 @@ Section cofe. ...@@ -33,15 +33,15 @@ Section cofe.
by trans (Q i);[apply HP|apply HQ]. by trans (Q i);[apply HP|apply HQ].
- intros n P Q HPQ; split=> i ?; apply HPQ; auto. - intros n P Q HPQ; split=> i ?; apply HPQ; auto.
Qed. Qed.
Canonical Structure siPropC : ofeT := OfeT siProp siProp_ofe_mixin. Canonical Structure siPropO : ofeT := OfeT siProp siProp_ofe_mixin.
Program Definition siProp_compl : Compl siPropC := λ c, Program Definition siProp_compl : Compl siPropO := λ c,
{| siProp_holds n := c n n |}. {| siProp_holds n := c n n |}.
Next Obligation. Next Obligation.
intros c n1 n2 ??; simpl in *. intros c n1 n2 ??; simpl in *.
apply (chain_cauchy c n2 n1); eauto using siProp_closed. apply (chain_cauchy c n2 n1); eauto using siProp_closed.
Qed. Qed.
Global Program Instance siProp_cofe : Cofe siPropC := {| compl := siProp_compl |}. Global Program Instance siProp_cofe : Cofe siPropO := {| compl := siProp_compl |}.
Next Obligation. Next Obligation.
intros n c; split=>i ?; symmetry; apply (chain_cauchy c i n); auto. intros n c; split=>i ?; symmetry; apply (chain_cauchy c i n); auto.
Qed. Qed.
......
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