summaryrefslogtreecommitdiff
path: root/cfrontend/Clight.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-08-18 10:06:03 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-08-18 10:06:03 +0000
commit0438984dece5f028bea55322d80aa4f363a782cb (patch)
tree31537550fde324ff49a883d53ed30640ff4442fc /cfrontend/Clight.v
parent6f9b68c8de22fe540bfe85c2fabec4b967c6a80d (diff)
Nettoyages pour doc
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1471 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend/Clight.v')
-rw-r--r--cfrontend/Clight.v18
1 files changed, 6 insertions, 12 deletions
diff --git a/cfrontend/Clight.v b/cfrontend/Clight.v
index 4f4123e..f183ade 100644
--- a/cfrontend/Clight.v
+++ b/cfrontend/Clight.v
@@ -320,18 +320,12 @@ End EXPR.
Inductive cont: Type :=
| Kstop: cont
- | Kseq: statement -> cont -> cont
- (**r [Kseq s2 k] = after [s1] in [s1;s2] *)
- | Kwhile: expr -> statement -> cont -> cont
- (**r [Kwhile e s k] = after [s] in [while (e) s] *)
- | Kdowhile: expr -> statement -> cont -> cont
- (**r [Kdowhile e s k] = after [s] in [do s while (e)] *)
- | Kfor2: expr -> statement -> statement -> cont -> cont
- (**r [Kfor2 e2 e3 s k] = after [s] in [for'(e2;e3) s] *)
- | Kfor3: expr -> statement -> statement -> cont -> cont
- (**r [Kfor3 e2 e3 s k] = after [e3] in [for'(e2;e3) s] *)
- | Kswitch: cont -> cont
- (**r catches [break] statements arising out of [switch] *)
+ | Kseq: statement -> cont -> cont (**r [Kseq s2 k] = after [s1] in [s1;s2] *)
+ | Kwhile: expr -> statement -> cont -> cont (**r [Kwhile e s k] = after [s] in [while (e) s] *)
+ | Kdowhile: expr -> statement -> cont -> cont (**r [Kdowhile e s k] = after [s] in [do s while (e)] *)
+ | Kfor2: expr -> statement -> statement -> cont -> cont (**r [Kfor2 e2 e3 s k] = after [s] in [for'(e2;e3) s] *)
+ | Kfor3: expr -> statement -> statement -> cont -> cont (**r [Kfor3 e2 e3 s k] = after [e3] in [for'(e2;e3) s] *)
+ | Kswitch: cont -> cont (**r catches [break] statements arising out of [switch] *)
| Kcall: option ident -> (**r where to store result *)
function -> (**r calling function *)
env -> (**r local env of calling function *)