aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asmblock.v
diff options
context:
space:
mode:
Diffstat (limited to 'aarch64/Asmblock.v')
-rw-r--r--aarch64/Asmblock.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/aarch64/Asmblock.v b/aarch64/Asmblock.v
index da45324b..7f94a087 100644
--- a/aarch64/Asmblock.v
+++ b/aarch64/Asmblock.v
@@ -336,12 +336,13 @@ Inductive basic : Type :=
*)
.
+(* Not used in Coq, declared in ocaml directly in PostpassSchedulingOracle.ml
Inductive instruction : Type :=
| PBasic (i: basic)
| PControl (i: control).
Coercion PBasic: basic >-> instruction.
-Coercion PControl: control >-> instruction.
+Coercion PControl: control >-> instruction. *)
(** * Definition of a bblock