summaryrefslogtreecommitdiff
path: root/backend/Cminor.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Cminor.v')
-rw-r--r--backend/Cminor.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/backend/Cminor.v b/backend/Cminor.v
index c12c6fc..aaf7510 100644
--- a/backend/Cminor.v
+++ b/backend/Cminor.v
@@ -103,9 +103,8 @@ Inductive binary_operation : Type :=
| Ocmpl: comparison -> binary_operation (**r long signed comparison *)
| Ocmplu: comparison -> binary_operation. (**r long unsigned comparison *)
-(** Expressions include reading local variables, constants and
- arithmetic operations, reading store locations, and conditional
- expressions (similar to [e1 ? e2 : e3] in C). *)
+(** Expressions include reading local variables, constants,
+ arithmetic operations, and memory loads. *)
Inductive expr : Type :=
| Evar : ident -> expr