Skip to content
Snippets Groups Projects
Commit b3eb5903 authored by David Swasey's avatar David Swasey
Browse files

Hoist type `pbit` to `language`.

parent 2a11f08f
No related branches found
No related tags found
No related merge requests found
...@@ -43,6 +43,8 @@ Class LanguageCtx (Λ : language) (K : expr Λ → expr Λ) := { ...@@ -43,6 +43,8 @@ Class LanguageCtx (Λ : language) (K : expr Λ → expr Λ) := {
Instance language_ctx_id Λ : LanguageCtx Λ id. Instance language_ctx_id Λ : LanguageCtx Λ id.
Proof. constructor; naive_solver. Qed. Proof. constructor; naive_solver. Qed.
Variant pbit := progress | noprogress.
Section language. Section language.
Context {Λ : language}. Context {Λ : language}.
Implicit Types v : val Λ. Implicit Types v : val Λ.
......
...@@ -11,8 +11,6 @@ Class irisG' (Λstate : Type) (Σ : gFunctors) := IrisG { ...@@ -11,8 +11,6 @@ Class irisG' (Λstate : Type) (Σ : gFunctors) := IrisG {
}. }.
Notation irisG Λ Σ := (irisG' (state Λ) Σ). Notation irisG Λ Σ := (irisG' (state Λ) Σ).
CoInductive pbit := progress | noprogress.
Definition wp_pre `{irisG Λ Σ} (p : pbit) Definition wp_pre `{irisG Λ Σ} (p : pbit)
(wp : coPset -c> expr Λ -c> (val Λ -c> iProp Σ) -c> iProp Σ) : (wp : coPset -c> expr Λ -c> (val Λ -c> iProp Σ) -c> iProp Σ) :
coPset -c> expr Λ -c> (val Λ -c> iProp Σ) -c> iProp Σ := λ E e1 Φ, coPset -c> expr Λ -c> (val Λ -c> iProp Σ) -c> iProp Σ := λ E e1 Φ,
......
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