From f5bb397acd12292f6b41438778f2df7391d6f2fe Mon Sep 17 00:00:00 2001 From: Michael Schmidt Date: Wed, 14 Oct 2015 15:26:56 +0200 Subject: bug 17392: remove trailing whitespace in source files --- powerpc/CombineOp.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'powerpc/CombineOp.v') diff --git a/powerpc/CombineOp.v b/powerpc/CombineOp.v index 6ad6987d..15ddb76f 100644 --- a/powerpc/CombineOp.v +++ b/powerpc/CombineOp.v @@ -10,7 +10,7 @@ (* *) (* *********************************************************************) -(** Recognition of combined operations, addressing modes and conditions +(** Recognition of combined operations, addressing modes and conditions during the [CSE] phase. *) Require Import Coqlib. @@ -95,7 +95,7 @@ Function combine_op (op: operation) (args: list valnum) : option(operation * lis end | Oandimm n, x :: nil => match get x with - | Some(Op (Oandimm m) ys) => + | Some(Op (Oandimm m) ys) => Some(let p := Int.and m n in if Int.eq p m then (Omove, x :: nil) else (Oandimm p, ys)) | Some(Op (Orolm amount m) ys) => -- cgit