aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/Pipeline.v
diff options
context:
space:
mode:
authorGravatar Robert Sloan <varomodt@gmail.com>2016-06-23 17:10:32 -0400
committerGravatar Robert Sloan <varomodt@gmail.com>2016-06-23 17:10:32 -0400
commite153f32401bc9e5ce108a41349e5a28055a56f70 (patch)
tree87c8f619d880930cd84ca35cc8426edc4ad0d668 /src/Assembly/Pipeline.v
parent75543f3bd0d74406de85796b6ce9b6cd54b93053 (diff)
QhasmUtil.v: Remove 8.4-incompatible intro name
Diffstat (limited to 'src/Assembly/Pipeline.v')
-rw-r--r--src/Assembly/Pipeline.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Assembly/Pipeline.v b/src/Assembly/Pipeline.v
index 67e39a804..ceb98a3a2 100644
--- a/src/Assembly/Pipeline.v
+++ b/src/Assembly/Pipeline.v
@@ -68,7 +68,7 @@ Module PipelineExamples.
plet b := v[[0]] in
([b ^& a; a ^+ b])).
pseudo_solve.
- Admitted. (*TODO (rsloan): eapply unification *)
+ Admitted. (* TODO (rsloan): eapply unification *)
Definition comb_ex_str :=
(Pipeline.toString (proj1_sig comb_example)).