aboutsummaryrefslogtreecommitdiffstats
path: root/backend/PPC.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/PPC.v')
-rw-r--r--backend/PPC.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/backend/PPC.v b/backend/PPC.v
index 66d96c29..5cd5e9f5 100644
--- a/backend/PPC.v
+++ b/backend/PPC.v
@@ -793,6 +793,8 @@ Inductive step: state -> trace -> state -> Prop :=
End RELSEM.
+(** Execution of whole programs. *)
+
Inductive initial_state (p: program): state -> Prop :=
| initial_state_intro:
let ge := Genv.globalenv p in
@@ -812,3 +814,4 @@ Inductive final_state: state -> int -> Prop :=
Definition exec_program (p: program) (beh: program_behavior) : Prop :=
program_behaves step (initial_state p) final_state (Genv.globalenv p) beh.
+