summaryrefslogtreecommitdiff
path: root/powerpc/Constprop.v
diff options
context:
space:
mode:
Diffstat (limited to 'powerpc/Constprop.v')
-rw-r--r--powerpc/Constprop.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/powerpc/Constprop.v b/powerpc/Constprop.v
index 6ec27a3..76ea153 100644
--- a/powerpc/Constprop.v
+++ b/powerpc/Constprop.v
@@ -32,7 +32,7 @@ Require Import Kildall.
(** To each pseudo-register at each program point, the static analysis
associates a compile-time approximation taken from the following set. *)
-Inductive approx : Set :=
+Inductive approx : Type :=
| Novalue: approx (** No value possible, code is unreachable. *)
| Unknown: approx (** All values are possible,
no compile-time information is available. *)
@@ -139,7 +139,7 @@ Definition eval_static_condition (cond: condition) (vl: list approx) :=
end.
*)
-Inductive eval_static_condition_cases: forall (cond: condition) (vl: list approx), Set :=
+Inductive eval_static_condition_cases: forall (cond: condition) (vl: list approx), Type :=
| eval_static_condition_case1:
forall c n1 n2,
eval_static_condition_cases (Ccomp c) (I n1 :: I n2 :: nil)
@@ -271,7 +271,7 @@ Definition eval_static_operation (op: operation) (vl: list approx) :=
end.
*)
-Inductive eval_static_operation_cases: forall (op: operation) (vl: list approx), Set :=
+Inductive eval_static_operation_cases: forall (op: operation) (vl: list approx), Type :=
| eval_static_operation_case1:
forall v1,
eval_static_operation_cases (Omove) (v1::nil)
@@ -696,7 +696,7 @@ Variable approx: D.t.
Definition intval (r: reg) : option int :=
match D.get r approx with I n => Some n | _ => None end.
-Inductive cond_strength_reduction_cases: condition -> list reg -> Set :=
+Inductive cond_strength_reduction_cases: condition -> list reg -> Type :=
| csr_case1:
forall c r1 r2,
cond_strength_reduction_cases (Ccomp c) (r1 :: r2 :: nil)
@@ -789,7 +789,7 @@ Definition make_xorimm (n: int) (r: reg) :=
then (Omove, r :: nil)
else (Oxorimm n, r :: nil).
-Inductive op_strength_reduction_cases: operation -> list reg -> Set :=
+Inductive op_strength_reduction_cases: operation -> list reg -> Type :=
| op_strength_reduction_case1:
forall (r1: reg) (r2: reg),
op_strength_reduction_cases Oadd (r1 :: r2 :: nil)
@@ -949,7 +949,7 @@ Definition op_strength_reduction (op: operation) (args: list reg) :=
(op, args)
end.
-Inductive addr_strength_reduction_cases: forall (addr: addressing) (args: list reg), Set :=
+Inductive addr_strength_reduction_cases: forall (addr: addressing) (args: list reg), Type :=
| addr_strength_reduction_case1:
forall (r1: reg) (r2: reg),
addr_strength_reduction_cases (Aindexed2) (r1 :: r2 :: nil)