aboutsummaryrefslogtreecommitdiffstats
path: root/common/Determinism.v
diff options
context:
space:
mode:
Diffstat (limited to 'common/Determinism.v')
-rw-r--r--common/Determinism.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/common/Determinism.v b/common/Determinism.v
index d0099ba9..7ea19663 100644
--- a/common/Determinism.v
+++ b/common/Determinism.v
@@ -36,7 +36,7 @@ Require Import Behaviors.
that this external call succeeds, has result [r], and changes
the world to [w]. *)
-Inductive world: Type :=
+CoInductive world: Type :=
World (io: ident -> list eventval -> option (eventval * world))
(vload: memory_chunk -> ident -> int -> option (eventval * world))
(vstore: memory_chunk -> ident -> int -> eventval -> option world).