aboutsummaryrefslogtreecommitdiffstats
path: root/driver
diff options
context:
space:
mode:
authorMichael Schmidt <github@mschmidt.me>2015-10-14 15:26:56 +0200
committerMichael Schmidt <github@mschmidt.me>2015-10-14 15:26:56 +0200
commitf5bb397acd12292f6b41438778f2df7391d6f2fe (patch)
treeb5964ca4c395b0db639565d0d0fddc9c44e34cf1 /driver
parentfd83d08d27057754202c575ed8a42d01b1af54c5 (diff)
downloadcompcert-f5bb397acd12292f6b41438778f2df7391d6f2fe.tar.gz
compcert-f5bb397acd12292f6b41438778f2df7391d6f2fe.zip
bug 17392: remove trailing whitespace in source files
Diffstat (limited to 'driver')
-rw-r--r--driver/Compiler.v48
-rw-r--r--driver/Complements.v24
2 files changed, 36 insertions, 36 deletions
diff --git a/driver/Compiler.v b/driver/Compiler.v
index 3920665e..ea5849ec 100644
--- a/driver/Compiler.v
+++ b/driver/Compiler.v
@@ -159,7 +159,7 @@ Definition transf_cminor_program (p: Cminor.program) : res Asm.program :=
@@@ transf_rtl_program.
Definition transf_clight_program (p: Clight.program) : res Asm.program :=
- OK p
+ OK p
@@ print print_Clight
@@@ time "Simplification of locals" SimplLocals.transf_program
@@@ time "C#minor generation" Cshmgen.transl_program
@@ -167,7 +167,7 @@ Definition transf_clight_program (p: Clight.program) : res Asm.program :=
@@@ transf_cminor_program.
Definition transf_c_program (p: Csyntax.program) : res Asm.program :=
- OK p
+ OK p
@@@ time "Clight generation" SimplExpr.transl_program
@@@ transf_clight_program.
@@ -182,14 +182,14 @@ Lemma print_identity:
forall (A: Type) (printer: A -> unit) (prog: A),
print printer prog = prog.
Proof.
- intros; unfold print. destruct (printer prog); auto.
+ intros; unfold print. destruct (printer prog); auto.
Qed.
Lemma compose_print_identity:
- forall (A: Type) (x: res A) (f: A -> unit),
+ forall (A: Type) (x: res A) (f: A -> unit),
x @@ print f = x.
Proof.
- intros. destruct x; simpl. rewrite print_identity. auto. auto.
+ intros. destruct x; simpl. rewrite print_identity. auto. auto.
Qed.
Remark forward_simulation_identity:
@@ -199,8 +199,8 @@ Proof.
- auto.
- exists s1; auto.
- subst s2; auto.
-- subst s2. exists s1'; auto.
-Qed.
+- subst s2. exists s1'; auto.
+Qed.
Lemma total_if_simulation:
forall (A: Type) (sem: A -> semantics) (flag: unit -> bool) (f: A -> A) (prog: A),
@@ -259,15 +259,15 @@ Proof.
destruct (partial_if debug Debugvar.transf_program p7) as [p71|] eqn:?; simpl in H; try discriminate.
destruct (Stacking.transf_program p71) as [p8|] eqn:?; simpl in H; try discriminate.
apply compose_forward_simulation with (RTL.semantics p1).
- apply total_if_simulation. apply Tailcallproof.transf_program_correct.
+ apply total_if_simulation. apply Tailcallproof.transf_program_correct.
apply compose_forward_simulation with (RTL.semantics p11).
apply Inliningproof.transf_program_correct; auto.
apply compose_forward_simulation with (RTL.semantics p12).
- apply Renumberproof.transf_program_correct.
+ apply Renumberproof.transf_program_correct.
apply compose_forward_simulation with (RTL.semantics p2).
apply total_if_simulation. apply Constpropproof.transf_program_correct.
apply compose_forward_simulation with (RTL.semantics p21).
- apply total_if_simulation. apply Renumberproof.transf_program_correct.
+ apply total_if_simulation. apply Renumberproof.transf_program_correct.
apply compose_forward_simulation with (RTL.semantics p3).
eapply partial_if_simulation; eauto. apply CSEproof.transf_program_correct.
apply compose_forward_simulation with (RTL.semantics p31).
@@ -281,7 +281,7 @@ Proof.
apply compose_forward_simulation with (Linear.semantics p6).
apply Linearizeproof.transf_program_correct; auto.
apply compose_forward_simulation with (Linear.semantics p7).
- apply CleanupLabelsproof.transf_program_correct.
+ apply CleanupLabelsproof.transf_program_correct.
apply compose_forward_simulation with (Linear.semantics p71).
eapply partial_if_simulation; eauto. apply Debugvarproof.transf_program_correct.
apply compose_forward_simulation with (Mach.semantics Asmgenproof0.return_address_offset p8).
@@ -289,8 +289,8 @@ Proof.
exact Asmgenproof.return_address_exists.
auto.
apply Asmgenproof.transf_program_correct; eauto.
- split. auto.
- apply forward_to_backward_simulation. auto.
+ split. auto.
+ apply forward_to_backward_simulation. auto.
apply RTL.semantics_receptive.
apply Asm.semantics_determinate.
Qed.
@@ -305,15 +305,15 @@ Proof.
assert (F: forward_simulation (Cminor.semantics p) (Asm.semantics tp)).
unfold transf_cminor_program, time in H.
repeat rewrite compose_print_identity in H.
- simpl in H.
+ simpl in H.
destruct (Selection.sel_program p) as [p1|] eqn:?; simpl in H; try discriminate.
destruct (RTLgen.transl_program p1) as [p2|] eqn:?; simpl in H; try discriminate.
eapply compose_forward_simulation. apply Selectionproof.transf_program_correct. eauto.
eapply compose_forward_simulation. apply RTLgenproof.transf_program_correct. eassumption.
exact (fst (transf_rtl_program_correct _ _ H)).
- split. auto.
- apply forward_to_backward_simulation. auto.
+ split. auto.
+ apply forward_to_backward_simulation. auto.
apply Cminor.semantics_receptive.
apply Asm.semantics_determinate.
Qed.
@@ -324,7 +324,7 @@ Theorem transf_clight_program_correct:
forward_simulation (Clight.semantics1 p) (Asm.semantics tp)
* backward_simulation (Clight.semantics1 p) (Asm.semantics tp).
Proof.
- intros.
+ intros.
assert (F: forward_simulation (Clight.semantics1 p) (Asm.semantics tp)).
revert H; unfold transf_clight_program, time; simpl.
rewrite print_identity.
@@ -335,10 +335,10 @@ Proof.
eapply compose_forward_simulation. apply SimplLocalsproof.transf_program_correct. eauto.
eapply compose_forward_simulation. apply Cshmgenproof.transl_program_correct. eauto.
eapply compose_forward_simulation. apply Cminorgenproof.transl_program_correct. eauto.
- exact (fst (transf_cminor_program_correct _ _ EQ3)).
+ exact (fst (transf_cminor_program_correct _ _ EQ3)).
- split. auto.
- apply forward_to_backward_simulation. auto.
+ split. auto.
+ apply forward_to_backward_simulation. auto.
apply Clight.semantics_receptive.
apply Asm.semantics_determinate.
Qed.
@@ -355,9 +355,9 @@ Proof.
caseEq (SimplExpr.transl_program p); simpl; try congruence; intros p0 EQ0.
intros EQ1.
eapply compose_forward_simulation. apply SimplExprproof.transl_program_correct. eauto.
- exact (fst (transf_clight_program_correct _ _ EQ1)).
+ exact (fst (transf_clight_program_correct _ _ EQ1)).
- split. auto.
+ split. auto.
apply forward_to_backward_simulation.
apply factor_forward_simulation. auto. eapply sd_traces. eapply Asm.semantics_determinate.
apply atomic_receptive. apply Cstrategy.semantics_strongly_receptive.
@@ -369,10 +369,10 @@ Theorem transf_c_program_correct:
transf_c_program p = OK tp ->
backward_simulation (Csem.semantics p) (Asm.semantics tp).
Proof.
- intros.
+ intros.
apply compose_backward_simulation with (atomic (Cstrategy.semantics p)).
eapply sd_traces; eapply Asm.semantics_determinate.
- apply factor_backward_simulation.
+ apply factor_backward_simulation.
apply Cstrategy.strategy_simulation.
apply Csem.semantics_single_events.
eapply ssr_well_behaved; eapply Cstrategy.semantics_strongly_receptive.
diff --git a/driver/Complements.v b/driver/Complements.v
index 57351a2a..8651f2ff 100644
--- a/driver/Complements.v
+++ b/driver/Complements.v
@@ -44,7 +44,7 @@ Theorem transf_c_program_preservation:
program_behaves (Asm.semantics tp) beh ->
exists beh', program_behaves (Csem.semantics p) beh' /\ behavior_improves beh' beh.
Proof.
- intros. eapply backward_simulation_behavior_improves; eauto.
+ intros. eapply backward_simulation_behavior_improves; eauto.
apply transf_c_program_correct; auto.
Qed.
@@ -81,7 +81,7 @@ Proof.
assert (WBT: forall p, well_behaved_traces (Cstrategy.semantics p)).
intros. eapply ssr_well_behaved. apply Cstrategy.semantics_strongly_receptive.
intros. intuition.
- eapply forward_simulation_behavior_improves; eauto.
+ eapply forward_simulation_behavior_improves; eauto.
apply (fst (transf_cstrategy_program_correct _ _ H)).
exploit backward_simulation_behavior_improves.
apply (snd (transf_cstrategy_program_correct _ _ H)).
@@ -92,7 +92,7 @@ Proof.
exploit backward_simulation_same_safe_behavior.
apply (snd (transf_cstrategy_program_correct _ _ H)).
intros. rewrite <- atomic_behaviors in H2; eauto. eauto.
- intros. rewrite atomic_behaviors; auto.
+ intros. rewrite atomic_behaviors; auto.
Qed.
(** We can also use the alternate big-step semantics for [Cstrategy]
@@ -114,7 +114,7 @@ Proof.
apply behavior_bigstep_terminates with (Cstrategy.bigstep_semantics p); auto.
apply Cstrategy.bigstep_semantics_sound.
exploit (behavior_bigstep_diverges (Cstrategy.bigstep_semantics_sound p)). eassumption.
- intros [A | [t [A B]]].
+ intros [A | [t [A B]]].
left. apply transf_cstrategy_program_preservation with p; auto. red; auto.
right; exists t; split; auto. apply transf_cstrategy_program_preservation with p; auto. red; auto.
Qed.
@@ -125,10 +125,10 @@ Qed.
of the source C program satisfies a given specification
(a predicate on the observable behavior of the program),
then all executions of the produced Asm program satisfy
- this specification as well.
+ this specification as well.
We first show this result for specifications that are stable
- under the [behavior_improves] relation. *)
+ under the [behavior_improves] relation. *)
Section SPECS_PRESERVED.
@@ -145,7 +145,7 @@ Theorem transf_c_program_preserves_spec:
Proof.
intros.
exploit transf_c_program_preservation; eauto. intros [beh' [A B]].
- apply spec_stable with beh'; auto.
+ apply spec_stable with beh'; auto.
Qed.
End SPECS_PRESERVED.
@@ -166,9 +166,9 @@ Theorem transf_c_program_preserves_safety_spec:
(forall beh, program_behaves (Csem.semantics p) beh -> spec beh) ->
(forall beh, program_behaves (Asm.semantics tp) beh -> spec beh).
Proof.
- intros. eapply transf_c_program_preserves_spec; eauto.
- intros. destruct H2. congruence. destruct H2 as [t [EQ1 EQ2]].
- subst beh1. elim (spec_safety _ H3).
+ intros. eapply transf_c_program_preserves_spec; eauto.
+ intros. destruct H2. congruence. destruct H2 as [t [EQ1 EQ2]].
+ subst beh1. elim (spec_safety _ H3).
Qed.
End SAFETY_PRESERVED.
@@ -196,8 +196,8 @@ Proof.
destruct H2 as [t [C D]]. subst.
destruct A as [b1 E]. destruct D as [b2 F].
destruct b1; simpl in E; inv E.
- exists t1; split; auto.
- exists (behavior_app t0 b2); apply behavior_app_assoc.
+ exists t1; split; auto.
+ exists (behavior_app t0 b2); apply behavior_app_assoc.
Qed.
End LIVENESS_PRESERVED.