aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Wfsimpl.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-10-20 13:32:18 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-10-20 13:32:18 +0200
commit4d542bc7eafadb16b845cf05d1eb4988eb55ed0f (patch)
tree1961b41815fc6e392cc0bd2beeb0fb504bc160ce /lib/Wfsimpl.v
parent7a6bb90048db7a254e959b1e3c308bac5fe6c418 (diff)
downloadcompcert-kvx-4d542bc7eafadb16b845cf05d1eb4988eb55ed0f.tar.gz
compcert-kvx-4d542bc7eafadb16b845cf05d1eb4988eb55ed0f.zip
Updated PR by removing whitespaces. Bug 17450.
Diffstat (limited to 'lib/Wfsimpl.v')
-rw-r--r--lib/Wfsimpl.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/lib/Wfsimpl.v b/lib/Wfsimpl.v
index 1ed6326a..4f80822e 100644
--- a/lib/Wfsimpl.v
+++ b/lib/Wfsimpl.v
@@ -35,9 +35,9 @@ Definition Fix (x: A) : B := Wf.Fix Rwf (fun (x: A) => B) F x.
Theorem unroll_Fix:
forall x, Fix x = F (fun (y: A) (P: R y x) => Fix y).
Proof.
- unfold Fix; intros. apply Wf.Fix_eq with (P := fun (x: A) => B).
+ unfold Fix; intros. apply Wf.Fix_eq with (P := fun (x: A) => B).
intros. assert (f = g). apply functional_extensionality_dep; intros.
- apply functional_extensionality; intros. auto.
+ apply functional_extensionality; intros. auto.
subst g; auto.
Qed.
@@ -56,9 +56,9 @@ Definition Fixm (x: A) : B := Wf.Fix (well_founded_ltof A measure) (fun (x: A) =
Theorem unroll_Fixm:
forall x, Fixm x = F (fun (y: A) (P: measure y < measure x) => Fixm y).
Proof.
- unfold Fixm; intros. apply Wf.Fix_eq with (P := fun (x: A) => B).
+ unfold Fixm; intros. apply Wf.Fix_eq with (P := fun (x: A) => B).
intros. assert (f = g). apply functional_extensionality_dep; intros.
- apply functional_extensionality; intros. auto.
+ apply functional_extensionality; intros. auto.
subst g; auto.
Qed.