aboutsummaryrefslogtreecommitdiffstats
path: root/common/Determinism.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2015-06-07 09:25:53 +0200
committerXavier Leroy <xavier.leroy@inria.fr>2015-06-07 09:25:53 +0200
commit584eac7027cd4d29c5ca8744453ffeea8f18b501 (patch)
tree374cd5c593eae420ff4e14e73de4c73709a6a87e /common/Determinism.v
parent9f30d4984863ec655a03996646805202dc2a07c9 (diff)
downloadcompcert-kvx-584eac7027cd4d29c5ca8744453ffeea8f18b501.tar.gz
compcert-kvx-584eac7027cd4d29c5ca8744453ffeea8f18b501.zip
Represent external worlds by a coinductive type rather than an inductive type.
As noticed by R. Krebbers, an inductive type for external worlds implies that all sequences of program-world interactions are finite, which is not the case.
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).