]> git.lizzy.rs Git - rust.git/blob - src/libsyntax/ext/expand.rs
Auto merge of #30469 - nagisa:mir-gv-prettify, r=luqmana
[rust.git] / src / libsyntax / ext / expand.rs
1 // Copyright 2012-2014 The Rust Project Developers. See the COPYRIGHT
2 // file at the top-level directory of this distribution and at
3 // http://rust-lang.org/COPYRIGHT.
4 //
5 // Licensed under the Apache License, Version 2.0 <LICENSE-APACHE or
6 // http://www.apache.org/licenses/LICENSE-2.0> or the MIT license
7 // <LICENSE-MIT or http://opensource.org/licenses/MIT>, at your
8 // option. This file may not be copied, modified, or distributed
9 // except according to those terms.
10
11 use ast::{Block, Crate, DeclLocal, PatMac};
12 use ast::{Local, Ident, Mac_, Name};
13 use ast::{ItemMac, MacStmtWithSemicolon, Mrk, Stmt, StmtDecl, StmtMac};
14 use ast::{StmtExpr, StmtSemi};
15 use ast::TokenTree;
16 use ast;
17 use ext::mtwt;
18 use ext::build::AstBuilder;
19 use attr;
20 use attr::{AttrMetaMethods, WithAttrs};
21 use codemap;
22 use codemap::{Span, Spanned, ExpnInfo, NameAndSpan, MacroBang, MacroAttribute};
23 use ext::base::*;
24 use feature_gate::{self, Features};
25 use fold;
26 use fold::*;
27 use util::move_map::MoveMap;
28 use parse;
29 use parse::token::{fresh_mark, fresh_name, intern};
30 use ptr::P;
31 use util::small_vector::SmallVector;
32 use visit;
33 use visit::Visitor;
34 use std_inject;
35
36 use std::collections::HashSet;
37
38
39 pub fn expand_expr(e: P<ast::Expr>, fld: &mut MacroExpander) -> P<ast::Expr> {
40     let expr_span = e.span;
41     return e.and_then(|ast::Expr {id, node, span, attrs}| match node {
42
43         // expr_mac should really be expr_ext or something; it's the
44         // entry-point for all syntax extensions.
45         ast::ExprMac(mac) => {
46
47             // Assert that we drop any macro attributes on the floor here
48             drop(attrs);
49
50             let expanded_expr = match expand_mac_invoc(mac, span,
51                                                        |r| r.make_expr(),
52                                                        mark_expr, fld) {
53                 Some(expr) => expr,
54                 None => {
55                     return DummyResult::raw_expr(span);
56                 }
57             };
58
59             // Keep going, outside-in.
60             let fully_expanded = fld.fold_expr(expanded_expr);
61             let span = fld.new_span(span);
62             fld.cx.bt_pop();
63
64             fully_expanded.map(|e| ast::Expr {
65                 id: ast::DUMMY_NODE_ID,
66                 node: e.node,
67                 span: span,
68                 attrs: e.attrs,
69             })
70         }
71
72         ast::ExprInPlace(placer, value_expr) => {
73             // Ensure feature-gate is enabled
74             feature_gate::check_for_placement_in(
75                 fld.cx.ecfg.features,
76                 &fld.cx.parse_sess.span_diagnostic,
77                 expr_span);
78
79             let placer = fld.fold_expr(placer);
80             let value_expr = fld.fold_expr(value_expr);
81             fld.cx.expr(span, ast::ExprInPlace(placer, value_expr))
82                 .with_attrs(fold_thin_attrs(attrs, fld))
83         }
84
85         ast::ExprWhile(cond, body, opt_ident) => {
86             let cond = fld.fold_expr(cond);
87             let (body, opt_ident) = expand_loop_block(body, opt_ident, fld);
88             fld.cx.expr(span, ast::ExprWhile(cond, body, opt_ident))
89                 .with_attrs(fold_thin_attrs(attrs, fld))
90         }
91
92         ast::ExprWhileLet(pat, expr, body, opt_ident) => {
93             let pat = fld.fold_pat(pat);
94             let expr = fld.fold_expr(expr);
95
96             // Hygienic renaming of the body.
97             let ((body, opt_ident), mut rewritten_pats) =
98                 rename_in_scope(vec![pat],
99                                 fld,
100                                 (body, opt_ident),
101                                 |rename_fld, fld, (body, opt_ident)| {
102                 expand_loop_block(rename_fld.fold_block(body), opt_ident, fld)
103             });
104             assert!(rewritten_pats.len() == 1);
105
106             fld.cx.expr(span, ast::ExprWhileLet(rewritten_pats.remove(0), expr, body, opt_ident))
107                 .with_attrs(fold_thin_attrs(attrs, fld))
108         }
109
110         ast::ExprLoop(loop_block, opt_ident) => {
111             let (loop_block, opt_ident) = expand_loop_block(loop_block, opt_ident, fld);
112             fld.cx.expr(span, ast::ExprLoop(loop_block, opt_ident))
113                 .with_attrs(fold_thin_attrs(attrs, fld))
114         }
115
116         ast::ExprForLoop(pat, head, body, opt_ident) => {
117             let pat = fld.fold_pat(pat);
118
119             // Hygienic renaming of the for loop body (for loop binds its pattern).
120             let ((body, opt_ident), mut rewritten_pats) =
121                 rename_in_scope(vec![pat],
122                                 fld,
123                                 (body, opt_ident),
124                                 |rename_fld, fld, (body, opt_ident)| {
125                 expand_loop_block(rename_fld.fold_block(body), opt_ident, fld)
126             });
127             assert!(rewritten_pats.len() == 1);
128
129             let head = fld.fold_expr(head);
130             fld.cx.expr(span, ast::ExprForLoop(rewritten_pats.remove(0), head, body, opt_ident))
131                 .with_attrs(fold_thin_attrs(attrs, fld))
132         }
133
134         ast::ExprIfLet(pat, sub_expr, body, else_opt) => {
135             let pat = fld.fold_pat(pat);
136
137             // Hygienic renaming of the body.
138             let (body, mut rewritten_pats) =
139                 rename_in_scope(vec![pat],
140                                 fld,
141                                 body,
142                                 |rename_fld, fld, body| {
143                 fld.fold_block(rename_fld.fold_block(body))
144             });
145             assert!(rewritten_pats.len() == 1);
146
147             let else_opt = else_opt.map(|else_opt| fld.fold_expr(else_opt));
148             let sub_expr = fld.fold_expr(sub_expr);
149             fld.cx.expr(span, ast::ExprIfLet(rewritten_pats.remove(0), sub_expr, body, else_opt))
150                 .with_attrs(fold_thin_attrs(attrs, fld))
151         }
152
153         ast::ExprClosure(capture_clause, fn_decl, block) => {
154             let (rewritten_fn_decl, rewritten_block)
155                 = expand_and_rename_fn_decl_and_block(fn_decl, block, fld);
156             let new_node = ast::ExprClosure(capture_clause,
157                                             rewritten_fn_decl,
158                                             rewritten_block);
159             P(ast::Expr{id:id, node: new_node, span: fld.new_span(span),
160                         attrs: fold_thin_attrs(attrs, fld)})
161         }
162
163         _ => {
164             P(noop_fold_expr(ast::Expr {
165                 id: id,
166                 node: node,
167                 span: span,
168                 attrs: attrs
169             }, fld))
170         }
171     });
172 }
173
174 /// Expand a (not-ident-style) macro invocation. Returns the result
175 /// of expansion and the mark which must be applied to the result.
176 /// Our current interface doesn't allow us to apply the mark to the
177 /// result until after calling make_expr, make_items, etc.
178 fn expand_mac_invoc<T, F, G>(mac: ast::Mac,
179                              span: codemap::Span,
180                              parse_thunk: F,
181                              mark_thunk: G,
182                              fld: &mut MacroExpander)
183                              -> Option<T> where
184     F: for<'a> FnOnce(Box<MacResult+'a>) -> Option<T>,
185     G: FnOnce(T, Mrk) -> T,
186 {
187     // it would almost certainly be cleaner to pass the whole
188     // macro invocation in, rather than pulling it apart and
189     // marking the tts and the ctxt separately. This also goes
190     // for the other three macro invocation chunks of code
191     // in this file.
192
193     let Mac_ { path: pth, tts, .. } = mac.node;
194     if pth.segments.len() > 1 {
195         fld.cx.span_err(pth.span,
196                         "expected macro name without module \
197                         separators");
198         // let compilation continue
199         return None;
200     }
201     let extname = pth.segments[0].identifier.name;
202     match fld.cx.syntax_env.find(extname) {
203         None => {
204             fld.cx.span_err(
205                 pth.span,
206                 &format!("macro undefined: '{}!'",
207                         &extname));
208             fld.cx.suggest_macro_name(&extname.as_str(), pth.span);
209
210             // let compilation continue
211             None
212         }
213         Some(rc) => match *rc {
214             NormalTT(ref expandfun, exp_span, allow_internal_unstable) => {
215                 fld.cx.bt_push(ExpnInfo {
216                         call_site: span,
217                         callee: NameAndSpan {
218                             format: MacroBang(extname),
219                             span: exp_span,
220                             allow_internal_unstable: allow_internal_unstable,
221                         },
222                     });
223                 let fm = fresh_mark();
224                 let marked_before = mark_tts(&tts[..], fm);
225
226                 // The span that we pass to the expanders we want to
227                 // be the root of the call stack. That's the most
228                 // relevant span and it's the actual invocation of
229                 // the macro.
230                 let mac_span = fld.cx.original_span();
231
232                 let opt_parsed = {
233                     let expanded = expandfun.expand(fld.cx,
234                                                     mac_span,
235                                                     &marked_before[..]);
236                     parse_thunk(expanded)
237                 };
238                 let parsed = match opt_parsed {
239                     Some(e) => e,
240                     None => {
241                         fld.cx.span_err(
242                             pth.span,
243                             &format!("non-expression macro in expression position: {}",
244                                     extname
245                                     ));
246                         return None;
247                     }
248                 };
249                 Some(mark_thunk(parsed,fm))
250             }
251             _ => {
252                 fld.cx.span_err(
253                     pth.span,
254                     &format!("'{}' is not a tt-style macro",
255                             extname));
256                 None
257             }
258         }
259     }
260 }
261
262 /// Rename loop label and expand its loop body
263 ///
264 /// The renaming procedure for loop is different in the sense that the loop
265 /// body is in a block enclosed by loop head so the renaming of loop label
266 /// must be propagated to the enclosed context.
267 fn expand_loop_block(loop_block: P<Block>,
268                      opt_ident: Option<Ident>,
269                      fld: &mut MacroExpander) -> (P<Block>, Option<Ident>) {
270     match opt_ident {
271         Some(label) => {
272             let new_label = fresh_name(label);
273             let rename = (label, new_label);
274
275             // The rename *must not* be added to the pending list of current
276             // syntax context otherwise an unrelated `break` or `continue` in
277             // the same context will pick that up in the deferred renaming pass
278             // and be renamed incorrectly.
279             let mut rename_list = vec!(rename);
280             let mut rename_fld = IdentRenamer{renames: &mut rename_list};
281             let renamed_ident = rename_fld.fold_ident(label);
282
283             // The rename *must* be added to the enclosed syntax context for
284             // `break` or `continue` to pick up because by definition they are
285             // in a block enclosed by loop head.
286             fld.cx.syntax_env.push_frame();
287             fld.cx.syntax_env.info().pending_renames.push(rename);
288             let expanded_block = expand_block_elts(loop_block, fld);
289             fld.cx.syntax_env.pop_frame();
290
291             (expanded_block, Some(renamed_ident))
292         }
293         None => (fld.fold_block(loop_block), opt_ident)
294     }
295 }
296
297 // eval $e with a new exts frame.
298 // must be a macro so that $e isn't evaluated too early.
299 macro_rules! with_exts_frame {
300     ($extsboxexpr:expr,$macros_escape:expr,$e:expr) =>
301     ({$extsboxexpr.push_frame();
302       $extsboxexpr.info().macros_escape = $macros_escape;
303       let result = $e;
304       $extsboxexpr.pop_frame();
305       result
306      })
307 }
308
309 // When we enter a module, record it, for the sake of `module!`
310 pub fn expand_item(it: P<ast::Item>, fld: &mut MacroExpander)
311                    -> SmallVector<P<ast::Item>> {
312     let it = expand_item_multi_modifier(Annotatable::Item(it), fld);
313
314     expand_annotatable(it, fld)
315         .into_iter().map(|i| i.expect_item()).collect()
316 }
317
318 /// Expand item_underscore
319 fn expand_item_underscore(item: ast::Item_, fld: &mut MacroExpander) -> ast::Item_ {
320     match item {
321         ast::ItemFn(decl, unsafety, constness, abi, generics, body) => {
322             let (rewritten_fn_decl, rewritten_body)
323                 = expand_and_rename_fn_decl_and_block(decl, body, fld);
324             let expanded_generics = fold::noop_fold_generics(generics,fld);
325             ast::ItemFn(rewritten_fn_decl, unsafety, constness, abi,
326                         expanded_generics, rewritten_body)
327         }
328         _ => noop_fold_item_underscore(item, fld)
329     }
330 }
331
332 // does this attribute list contain "macro_use" ?
333 fn contains_macro_use(fld: &mut MacroExpander, attrs: &[ast::Attribute]) -> bool {
334     for attr in attrs {
335         let mut is_use = attr.check_name("macro_use");
336         if attr.check_name("macro_escape") {
337             fld.cx.span_warn(attr.span, "macro_escape is a deprecated synonym for macro_use");
338             is_use = true;
339             if let ast::AttrStyle::Inner = attr.node.style {
340                 fld.cx.fileline_help(attr.span, "consider an outer attribute, \
341                                              #[macro_use] mod ...");
342             }
343         };
344
345         if is_use {
346             match attr.node.value.node {
347                 ast::MetaWord(..) => (),
348                 _ => fld.cx.span_err(attr.span, "arguments to macro_use are not allowed here"),
349             }
350             return true;
351         }
352     }
353     false
354 }
355
356 // Support for item-position macro invocations, exactly the same
357 // logic as for expression-position macro invocations.
358 pub fn expand_item_mac(it: P<ast::Item>,
359                        fld: &mut MacroExpander) -> SmallVector<P<ast::Item>> {
360     let (extname, path_span, tts, span, attrs, ident) = it.and_then(|it| match it.node {
361         ItemMac(codemap::Spanned { node: Mac_ { path, tts, .. }, .. }) =>
362             (path.segments[0].identifier.name, path.span, tts, it.span, it.attrs, it.ident),
363         _ => fld.cx.span_bug(it.span, "invalid item macro invocation")
364     });
365
366     let fm = fresh_mark();
367     let items = {
368         let expanded = match fld.cx.syntax_env.find(extname) {
369             None => {
370                 fld.cx.span_err(path_span,
371                                 &format!("macro undefined: '{}!'",
372                                         extname));
373                 // let compilation continue
374                 return SmallVector::zero();
375             }
376
377             Some(rc) => match *rc {
378                 NormalTT(ref expander, tt_span, allow_internal_unstable) => {
379                     if ident.name != parse::token::special_idents::invalid.name {
380                         fld.cx
381                             .span_err(path_span,
382                                       &format!("macro {}! expects no ident argument, given '{}'",
383                                                extname,
384                                                ident));
385                         return SmallVector::zero();
386                     }
387                     fld.cx.bt_push(ExpnInfo {
388                         call_site: span,
389                         callee: NameAndSpan {
390                             format: MacroBang(extname),
391                             span: tt_span,
392                             allow_internal_unstable: allow_internal_unstable,
393                         }
394                     });
395                     // mark before expansion:
396                     let marked_before = mark_tts(&tts[..], fm);
397                     expander.expand(fld.cx, span, &marked_before[..])
398                 }
399                 IdentTT(ref expander, tt_span, allow_internal_unstable) => {
400                     if ident.name == parse::token::special_idents::invalid.name {
401                         fld.cx.span_err(path_span,
402                                         &format!("macro {}! expects an ident argument",
403                                                 extname));
404                         return SmallVector::zero();
405                     }
406                     fld.cx.bt_push(ExpnInfo {
407                         call_site: span,
408                         callee: NameAndSpan {
409                             format: MacroBang(extname),
410                             span: tt_span,
411                             allow_internal_unstable: allow_internal_unstable,
412                         }
413                     });
414                     // mark before expansion:
415                     let marked_tts = mark_tts(&tts[..], fm);
416                     expander.expand(fld.cx, span, ident, marked_tts)
417                 }
418                 MacroRulesTT => {
419                     if ident.name == parse::token::special_idents::invalid.name {
420                         fld.cx.span_err(path_span, "macro_rules! expects an ident argument");
421                         return SmallVector::zero();
422                     }
423
424                     fld.cx.bt_push(ExpnInfo {
425                         call_site: span,
426                         callee: NameAndSpan {
427                             format: MacroBang(extname),
428                             span: None,
429                             // `macro_rules!` doesn't directly allow
430                             // unstable (this is orthogonal to whether
431                             // the macro it creates allows it)
432                             allow_internal_unstable: false,
433                         }
434                     });
435                     // DON'T mark before expansion.
436
437                     let allow_internal_unstable = attr::contains_name(&attrs,
438                                                                       "allow_internal_unstable");
439
440                     // ensure any #[allow_internal_unstable]s are
441                     // detected (including nested macro definitions
442                     // etc.)
443                     if allow_internal_unstable && !fld.cx.ecfg.enable_allow_internal_unstable() {
444                         feature_gate::emit_feature_err(
445                             &fld.cx.parse_sess.span_diagnostic,
446                             "allow_internal_unstable",
447                             span,
448                             feature_gate::GateIssue::Language,
449                             feature_gate::EXPLAIN_ALLOW_INTERNAL_UNSTABLE)
450                     }
451
452                     let export = attr::contains_name(&attrs, "macro_export");
453                     let def = ast::MacroDef {
454                         ident: ident,
455                         attrs: attrs,
456                         id: ast::DUMMY_NODE_ID,
457                         span: span,
458                         imported_from: None,
459                         export: export,
460                         use_locally: true,
461                         allow_internal_unstable: allow_internal_unstable,
462                         body: tts,
463                     };
464                     fld.cx.insert_macro(def);
465
466                     // macro_rules! has a side effect but expands to nothing.
467                     fld.cx.bt_pop();
468                     return SmallVector::zero();
469                 }
470                 _ => {
471                     fld.cx.span_err(span,
472                                     &format!("{}! is not legal in item position",
473                                             extname));
474                     return SmallVector::zero();
475                 }
476             }
477         };
478
479         expanded.make_items()
480     };
481
482     let items = match items {
483         Some(items) => {
484             items.into_iter()
485                 .map(|i| mark_item(i, fm))
486                 .flat_map(|i| fld.fold_item(i).into_iter())
487                 .collect()
488         }
489         None => {
490             fld.cx.span_err(path_span,
491                             &format!("non-item macro in item position: {}",
492                                     extname));
493             return SmallVector::zero();
494         }
495     };
496
497     fld.cx.bt_pop();
498     items
499 }
500
501 /// Expand a stmt
502 fn expand_stmt(stmt: P<Stmt>, fld: &mut MacroExpander) -> SmallVector<P<Stmt>> {
503     let stmt = stmt.and_then(|stmt| stmt);
504     let (mac, style, attrs) = match stmt.node {
505         StmtMac(mac, style, attrs) => (mac, style, attrs),
506         _ => return expand_non_macro_stmt(stmt, fld)
507     };
508
509     // Assert that we drop any macro attributes on the floor here
510     drop(attrs);
511
512     let maybe_new_items =
513         expand_mac_invoc(mac.and_then(|m| m), stmt.span,
514                          |r| r.make_stmts(),
515                          |stmts, mark| stmts.move_map(|m| mark_stmt(m, mark)),
516                          fld);
517
518     let mut fully_expanded = match maybe_new_items {
519         Some(stmts) => {
520             // Keep going, outside-in.
521             let new_items = stmts.into_iter().flat_map(|s| {
522                 fld.fold_stmt(s).into_iter()
523             }).collect();
524             fld.cx.bt_pop();
525             new_items
526         }
527         None => SmallVector::zero()
528     };
529
530     // If this is a macro invocation with a semicolon, then apply that
531     // semicolon to the final statement produced by expansion.
532     if style == MacStmtWithSemicolon {
533         if let Some(stmt) = fully_expanded.pop() {
534             let new_stmt = stmt.map(|Spanned {node, span}| {
535                 Spanned {
536                     node: match node {
537                         StmtExpr(e, stmt_id) => StmtSemi(e, stmt_id),
538                         _ => node /* might already have a semi */
539                     },
540                     span: span
541                 }
542             });
543             fully_expanded.push(new_stmt);
544         }
545     }
546
547     fully_expanded
548 }
549
550 // expand a non-macro stmt. this is essentially the fallthrough for
551 // expand_stmt, above.
552 fn expand_non_macro_stmt(Spanned {node, span: stmt_span}: Stmt, fld: &mut MacroExpander)
553                          -> SmallVector<P<Stmt>> {
554     // is it a let?
555     match node {
556         StmtDecl(decl, node_id) => decl.and_then(|Spanned {node: decl, span}| match decl {
557             DeclLocal(local) => {
558                 // take it apart:
559                 let rewritten_local = local.map(|Local {id, pat, ty, init, span, attrs}| {
560                     // expand the ty since TyFixedLengthVec contains an Expr
561                     // and thus may have a macro use
562                     let expanded_ty = ty.map(|t| fld.fold_ty(t));
563                     // expand the pat (it might contain macro uses):
564                     let expanded_pat = fld.fold_pat(pat);
565                     // find the PatIdents in the pattern:
566                     // oh dear heaven... this is going to include the enum
567                     // names, as well... but that should be okay, as long as
568                     // the new names are gensyms for the old ones.
569                     // generate fresh names, push them to a new pending list
570                     let idents = pattern_bindings(&expanded_pat);
571                     let mut new_pending_renames =
572                         idents.iter().map(|ident| (*ident, fresh_name(*ident))).collect();
573                     // rewrite the pattern using the new names (the old
574                     // ones have already been applied):
575                     let rewritten_pat = {
576                         // nested binding to allow borrow to expire:
577                         let mut rename_fld = IdentRenamer{renames: &mut new_pending_renames};
578                         rename_fld.fold_pat(expanded_pat)
579                     };
580                     // add them to the existing pending renames:
581                     fld.cx.syntax_env.info().pending_renames
582                           .extend(new_pending_renames);
583                     Local {
584                         id: id,
585                         ty: expanded_ty,
586                         pat: rewritten_pat,
587                         // also, don't forget to expand the init:
588                         init: init.map(|e| fld.fold_expr(e)),
589                         span: span,
590                         attrs: fold::fold_thin_attrs(attrs, fld),
591                     }
592                 });
593                 SmallVector::one(P(Spanned {
594                     node: StmtDecl(P(Spanned {
595                             node: DeclLocal(rewritten_local),
596                             span: span
597                         }),
598                         node_id),
599                     span: stmt_span
600                 }))
601             }
602             _ => {
603                 noop_fold_stmt(Spanned {
604                     node: StmtDecl(P(Spanned {
605                             node: decl,
606                             span: span
607                         }),
608                         node_id),
609                     span: stmt_span
610                 }, fld)
611             }
612         }),
613         _ => {
614             noop_fold_stmt(Spanned {
615                 node: node,
616                 span: stmt_span
617             }, fld)
618         }
619     }
620 }
621
622 // expand the arm of a 'match', renaming for macro hygiene
623 fn expand_arm(arm: ast::Arm, fld: &mut MacroExpander) -> ast::Arm {
624     // expand pats... they might contain macro uses:
625     let expanded_pats = arm.pats.move_map(|pat| fld.fold_pat(pat));
626     if expanded_pats.is_empty() {
627         panic!("encountered match arm with 0 patterns");
628     }
629
630     // apply renaming and then expansion to the guard and the body:
631     let ((rewritten_guard, rewritten_body), rewritten_pats) =
632         rename_in_scope(expanded_pats,
633                         fld,
634                         (arm.guard, arm.body),
635                         |rename_fld, fld, (ag, ab)|{
636         let rewritten_guard = ag.map(|g| fld.fold_expr(rename_fld.fold_expr(g)));
637         let rewritten_body = fld.fold_expr(rename_fld.fold_expr(ab));
638         (rewritten_guard, rewritten_body)
639     });
640
641     ast::Arm {
642         attrs: fold::fold_attrs(arm.attrs, fld),
643         pats: rewritten_pats,
644         guard: rewritten_guard,
645         body: rewritten_body,
646     }
647 }
648
649 fn rename_in_scope<X, F>(pats: Vec<P<ast::Pat>>,
650                          fld: &mut MacroExpander,
651                          x: X,
652                          f: F)
653                          -> (X, Vec<P<ast::Pat>>)
654     where F: Fn(&mut IdentRenamer, &mut MacroExpander, X) -> X
655 {
656     // all of the pats must have the same set of bindings, so use the
657     // first one to extract them and generate new names:
658     let idents = pattern_bindings(&pats[0]);
659     let new_renames = idents.into_iter().map(|id| (id, fresh_name(id))).collect();
660     // apply the renaming, but only to the PatIdents:
661     let mut rename_pats_fld = PatIdentRenamer{renames:&new_renames};
662     let rewritten_pats = pats.move_map(|pat| rename_pats_fld.fold_pat(pat));
663
664     let mut rename_fld = IdentRenamer{ renames:&new_renames };
665     (f(&mut rename_fld, fld, x), rewritten_pats)
666 }
667
668 /// A visitor that extracts the PatIdent (binding) paths
669 /// from a given thingy and puts them in a mutable
670 /// array
671 #[derive(Clone)]
672 struct PatIdentFinder {
673     ident_accumulator: Vec<ast::Ident>
674 }
675
676 impl<'v> Visitor<'v> for PatIdentFinder {
677     fn visit_pat(&mut self, pattern: &ast::Pat) {
678         match *pattern {
679             ast::Pat { id: _, node: ast::PatIdent(_, ref path1, ref inner), span: _ } => {
680                 self.ident_accumulator.push(path1.node);
681                 // visit optional subpattern of PatIdent:
682                 if let Some(ref subpat) = *inner {
683                     self.visit_pat(subpat)
684                 }
685             }
686             // use the default traversal for non-PatIdents
687             _ => visit::walk_pat(self, pattern)
688         }
689     }
690 }
691
692 /// find the PatIdent paths in a pattern
693 fn pattern_bindings(pat: &ast::Pat) -> Vec<ast::Ident> {
694     let mut name_finder = PatIdentFinder{ident_accumulator:Vec::new()};
695     name_finder.visit_pat(pat);
696     name_finder.ident_accumulator
697 }
698
699 /// find the PatIdent paths in a
700 fn fn_decl_arg_bindings(fn_decl: &ast::FnDecl) -> Vec<ast::Ident> {
701     let mut pat_idents = PatIdentFinder{ident_accumulator:Vec::new()};
702     for arg in &fn_decl.inputs {
703         pat_idents.visit_pat(&arg.pat);
704     }
705     pat_idents.ident_accumulator
706 }
707
708 // expand a block. pushes a new exts_frame, then calls expand_block_elts
709 pub fn expand_block(blk: P<Block>, fld: &mut MacroExpander) -> P<Block> {
710     // see note below about treatment of exts table
711     with_exts_frame!(fld.cx.syntax_env,false,
712                      expand_block_elts(blk, fld))
713 }
714
715 // expand the elements of a block.
716 pub fn expand_block_elts(b: P<Block>, fld: &mut MacroExpander) -> P<Block> {
717     b.map(|Block {id, stmts, expr, rules, span}| {
718         let new_stmts = stmts.into_iter().flat_map(|x| {
719             // perform all pending renames
720             let renamed_stmt = {
721                 let pending_renames = &mut fld.cx.syntax_env.info().pending_renames;
722                 let mut rename_fld = IdentRenamer{renames:pending_renames};
723                 rename_fld.fold_stmt(x).expect_one("rename_fold didn't return one value")
724             };
725             // expand macros in the statement
726             fld.fold_stmt(renamed_stmt).into_iter()
727         }).collect();
728         let new_expr = expr.map(|x| {
729             let expr = {
730                 let pending_renames = &mut fld.cx.syntax_env.info().pending_renames;
731                 let mut rename_fld = IdentRenamer{renames:pending_renames};
732                 rename_fld.fold_expr(x)
733             };
734             fld.fold_expr(expr)
735         });
736         Block {
737             id: fld.new_id(id),
738             stmts: new_stmts,
739             expr: new_expr,
740             rules: rules,
741             span: span
742         }
743     })
744 }
745
746 fn expand_pat(p: P<ast::Pat>, fld: &mut MacroExpander) -> P<ast::Pat> {
747     match p.node {
748         PatMac(_) => {}
749         _ => return noop_fold_pat(p, fld)
750     }
751     p.map(|ast::Pat {node, span, ..}| {
752         let (pth, tts) = match node {
753             PatMac(mac) => (mac.node.path, mac.node.tts),
754             _ => unreachable!()
755         };
756         if pth.segments.len() > 1 {
757             fld.cx.span_err(pth.span, "expected macro name without module separators");
758             return DummyResult::raw_pat(span);
759         }
760         let extname = pth.segments[0].identifier.name;
761         let marked_after = match fld.cx.syntax_env.find(extname) {
762             None => {
763                 fld.cx.span_err(pth.span,
764                                 &format!("macro undefined: '{}!'",
765                                         extname));
766                 // let compilation continue
767                 return DummyResult::raw_pat(span);
768             }
769
770             Some(rc) => match *rc {
771                 NormalTT(ref expander, tt_span, allow_internal_unstable) => {
772                     fld.cx.bt_push(ExpnInfo {
773                         call_site: span,
774                         callee: NameAndSpan {
775                             format: MacroBang(extname),
776                             span: tt_span,
777                             allow_internal_unstable: allow_internal_unstable,
778                         }
779                     });
780
781                     let fm = fresh_mark();
782                     let marked_before = mark_tts(&tts[..], fm);
783                     let mac_span = fld.cx.original_span();
784                     let pat = expander.expand(fld.cx,
785                                               mac_span,
786                                               &marked_before[..]).make_pat();
787                     let expanded = match pat {
788                         Some(e) => e,
789                         None => {
790                             fld.cx.span_err(
791                                 pth.span,
792                                 &format!(
793                                     "non-pattern macro in pattern position: {}",
794                                     extname
795                                     )
796                             );
797                             return DummyResult::raw_pat(span);
798                         }
799                     };
800
801                     // mark after:
802                     mark_pat(expanded,fm)
803                 }
804                 _ => {
805                     fld.cx.span_err(span,
806                                     &format!("{}! is not legal in pattern position",
807                                             extname));
808                     return DummyResult::raw_pat(span);
809                 }
810             }
811         };
812
813         let fully_expanded =
814             fld.fold_pat(marked_after).node.clone();
815         fld.cx.bt_pop();
816
817         ast::Pat {
818             id: ast::DUMMY_NODE_ID,
819             node: fully_expanded,
820             span: span
821         }
822     })
823 }
824
825 /// A tree-folder that applies every rename in its (mutable) list
826 /// to every identifier, including both bindings and varrefs
827 /// (and lots of things that will turn out to be neither)
828 pub struct IdentRenamer<'a> {
829     renames: &'a mtwt::RenameList,
830 }
831
832 impl<'a> Folder for IdentRenamer<'a> {
833     fn fold_ident(&mut self, id: Ident) -> Ident {
834         Ident::new(id.name, mtwt::apply_renames(self.renames, id.ctxt))
835     }
836     fn fold_mac(&mut self, mac: ast::Mac) -> ast::Mac {
837         fold::noop_fold_mac(mac, self)
838     }
839 }
840
841 /// A tree-folder that applies every rename in its list to
842 /// the idents that are in PatIdent patterns. This is more narrowly
843 /// focused than IdentRenamer, and is needed for FnDecl,
844 /// where we want to rename the args but not the fn name or the generics etc.
845 pub struct PatIdentRenamer<'a> {
846     renames: &'a mtwt::RenameList,
847 }
848
849 impl<'a> Folder for PatIdentRenamer<'a> {
850     fn fold_pat(&mut self, pat: P<ast::Pat>) -> P<ast::Pat> {
851         match pat.node {
852             ast::PatIdent(..) => {},
853             _ => return noop_fold_pat(pat, self)
854         }
855
856         pat.map(|ast::Pat {id, node, span}| match node {
857             ast::PatIdent(binding_mode, Spanned{span: sp, node: ident}, sub) => {
858                 let new_ident = Ident::new(ident.name,
859                                            mtwt::apply_renames(self.renames, ident.ctxt));
860                 let new_node =
861                     ast::PatIdent(binding_mode,
862                                   Spanned{span: self.new_span(sp), node: new_ident},
863                                   sub.map(|p| self.fold_pat(p)));
864                 ast::Pat {
865                     id: id,
866                     node: new_node,
867                     span: self.new_span(span)
868                 }
869             },
870             _ => unreachable!()
871         })
872     }
873     fn fold_mac(&mut self, mac: ast::Mac) -> ast::Mac {
874         fold::noop_fold_mac(mac, self)
875     }
876 }
877
878 fn expand_annotatable(a: Annotatable,
879                       fld: &mut MacroExpander)
880                       -> SmallVector<Annotatable> {
881     let a = expand_item_multi_modifier(a, fld);
882
883     let mut decorator_items = SmallVector::zero();
884     let mut new_attrs = Vec::new();
885     expand_decorators(a.clone(), fld, &mut decorator_items, &mut new_attrs);
886
887     let mut new_items: SmallVector<Annotatable> = match a {
888         Annotatable::Item(it) => match it.node {
889             ast::ItemMac(..) => {
890                 expand_item_mac(it, fld).into_iter().map(|i| Annotatable::Item(i)).collect()
891             }
892             ast::ItemMod(_) | ast::ItemForeignMod(_) => {
893                 let valid_ident =
894                     it.ident.name != parse::token::special_idents::invalid.name;
895
896                 if valid_ident {
897                     fld.cx.mod_push(it.ident);
898                 }
899                 let macro_use = contains_macro_use(fld, &new_attrs[..]);
900                 let result = with_exts_frame!(fld.cx.syntax_env,
901                                               macro_use,
902                                               noop_fold_item(it, fld));
903                 if valid_ident {
904                     fld.cx.mod_pop();
905                 }
906                 result.into_iter().map(|i| Annotatable::Item(i)).collect()
907             },
908             _ => {
909                 let it = P(ast::Item {
910                     attrs: new_attrs,
911                     ..(*it).clone()
912                 });
913                 noop_fold_item(it, fld).into_iter().map(|i| Annotatable::Item(i)).collect()
914             }
915         },
916
917         Annotatable::TraitItem(it) => match it.node {
918             ast::MethodTraitItem(_, Some(_)) => SmallVector::one(it.map(|ti| ast::TraitItem {
919                 id: ti.id,
920                 ident: ti.ident,
921                 attrs: ti.attrs,
922                 node: match ti.node  {
923                     ast::MethodTraitItem(sig, Some(body)) => {
924                         let (sig, body) = expand_and_rename_method(sig, body, fld);
925                         ast::MethodTraitItem(sig, Some(body))
926                     }
927                     _ => unreachable!()
928                 },
929                 span: fld.new_span(ti.span)
930             })),
931             _ => fold::noop_fold_trait_item(it, fld)
932         }.into_iter().map(Annotatable::TraitItem).collect(),
933
934         Annotatable::ImplItem(ii) => {
935             expand_impl_item(ii, fld).into_iter().map(Annotatable::ImplItem).collect()
936         }
937     };
938
939     new_items.push_all(decorator_items);
940     new_items
941 }
942
943 // Partition a set of attributes into one kind of attribute, and other kinds.
944 macro_rules! partition {
945     ($fn_name: ident, $variant: ident) => {
946         #[allow(deprecated)] // The `allow` is needed because the `Modifier` variant might be used.
947         fn $fn_name(attrs: &[ast::Attribute],
948                     fld: &MacroExpander)
949                      -> (Vec<ast::Attribute>, Vec<ast::Attribute>) {
950             attrs.iter().cloned().partition(|attr| {
951                 match fld.cx.syntax_env.find(intern(&attr.name())) {
952                     Some(rc) => match *rc {
953                         $variant(..) => true,
954                         _ => false
955                     },
956                     _ => false
957                 }
958             })
959         }
960     }
961 }
962
963 partition!(multi_modifiers, MultiModifier);
964
965
966 fn expand_decorators(a: Annotatable,
967                      fld: &mut MacroExpander,
968                      decorator_items: &mut SmallVector<Annotatable>,
969                      new_attrs: &mut Vec<ast::Attribute>)
970 {
971     for attr in a.attrs() {
972         let mname = intern(&attr.name());
973         match fld.cx.syntax_env.find(mname) {
974             Some(rc) => match *rc {
975                 MultiDecorator(ref dec) => {
976                     attr::mark_used(&attr);
977
978                     fld.cx.bt_push(ExpnInfo {
979                         call_site: attr.span,
980                         callee: NameAndSpan {
981                             format: MacroAttribute(mname),
982                             span: Some(attr.span),
983                             // attributes can do whatever they like,
984                             // for now.
985                             allow_internal_unstable: true,
986                         }
987                     });
988
989                     // we'd ideally decorator_items.push_all(expand_annotatable(ann, fld)),
990                     // but that double-mut-borrows fld
991                     let mut items: SmallVector<Annotatable> = SmallVector::zero();
992                     dec.expand(fld.cx,
993                                attr.span,
994                                &attr.node.value,
995                                &a,
996                                &mut |ann| items.push(ann));
997                     decorator_items.extend(items.into_iter()
998                         .flat_map(|ann| expand_annotatable(ann, fld).into_iter()));
999
1000                     fld.cx.bt_pop();
1001                 }
1002                 _ => new_attrs.push((*attr).clone()),
1003             },
1004             _ => new_attrs.push((*attr).clone()),
1005         }
1006     }
1007 }
1008
1009 fn expand_item_multi_modifier(mut it: Annotatable,
1010                               fld: &mut MacroExpander)
1011                               -> Annotatable {
1012     let (modifiers, other_attrs) = multi_modifiers(it.attrs(), fld);
1013
1014     // Update the attrs, leave everything else alone. Is this mutation really a good idea?
1015     it = it.fold_attrs(other_attrs);
1016
1017     if modifiers.is_empty() {
1018         return it
1019     }
1020
1021     for attr in &modifiers {
1022         let mname = intern(&attr.name());
1023
1024         match fld.cx.syntax_env.find(mname) {
1025             Some(rc) => match *rc {
1026                 MultiModifier(ref mac) => {
1027                     attr::mark_used(attr);
1028                     fld.cx.bt_push(ExpnInfo {
1029                         call_site: attr.span,
1030                         callee: NameAndSpan {
1031                             format: MacroAttribute(mname),
1032                             span: Some(attr.span),
1033                             // attributes can do whatever they like,
1034                             // for now
1035                             allow_internal_unstable: true,
1036                         }
1037                     });
1038                     it = mac.expand(fld.cx, attr.span, &*attr.node.value, it);
1039                     fld.cx.bt_pop();
1040                 }
1041                 _ => unreachable!()
1042             },
1043             _ => unreachable!()
1044         }
1045     }
1046
1047     // Expansion may have added new ItemModifiers.
1048     expand_item_multi_modifier(it, fld)
1049 }
1050
1051 fn expand_impl_item(ii: P<ast::ImplItem>, fld: &mut MacroExpander)
1052                  -> SmallVector<P<ast::ImplItem>> {
1053     match ii.node {
1054         ast::ImplItemKind::Method(..) => SmallVector::one(ii.map(|ii| ast::ImplItem {
1055             id: ii.id,
1056             ident: ii.ident,
1057             attrs: ii.attrs,
1058             vis: ii.vis,
1059             node: match ii.node  {
1060                 ast::ImplItemKind::Method(sig, body) => {
1061                     let (sig, body) = expand_and_rename_method(sig, body, fld);
1062                     ast::ImplItemKind::Method(sig, body)
1063                 }
1064                 _ => unreachable!()
1065             },
1066             span: fld.new_span(ii.span)
1067         })),
1068         ast::ImplItemKind::Macro(_) => {
1069             let (span, mac) = ii.and_then(|ii| match ii.node {
1070                 ast::ImplItemKind::Macro(mac) => (ii.span, mac),
1071                 _ => unreachable!()
1072             });
1073             let maybe_new_items =
1074                 expand_mac_invoc(mac, span,
1075                                  |r| r.make_impl_items(),
1076                                  |meths, mark| meths.move_map(|m| mark_impl_item(m, mark)),
1077                                  fld);
1078
1079             match maybe_new_items {
1080                 Some(impl_items) => {
1081                     // expand again if necessary
1082                     let new_items = impl_items.into_iter().flat_map(|ii| {
1083                         expand_impl_item(ii, fld).into_iter()
1084                     }).collect();
1085                     fld.cx.bt_pop();
1086                     new_items
1087                 }
1088                 None => SmallVector::zero()
1089             }
1090         }
1091         _ => fold::noop_fold_impl_item(ii, fld)
1092     }
1093 }
1094
1095 /// Given a fn_decl and a block and a MacroExpander, expand the fn_decl, then use the
1096 /// PatIdents in its arguments to perform renaming in the FnDecl and
1097 /// the block, returning both the new FnDecl and the new Block.
1098 fn expand_and_rename_fn_decl_and_block(fn_decl: P<ast::FnDecl>, block: P<ast::Block>,
1099                                        fld: &mut MacroExpander)
1100                                        -> (P<ast::FnDecl>, P<ast::Block>) {
1101     let expanded_decl = fld.fold_fn_decl(fn_decl);
1102     let idents = fn_decl_arg_bindings(&expanded_decl);
1103     let renames =
1104         idents.iter().map(|id| (*id,fresh_name(*id))).collect();
1105     // first, a renamer for the PatIdents, for the fn_decl:
1106     let mut rename_pat_fld = PatIdentRenamer{renames: &renames};
1107     let rewritten_fn_decl = rename_pat_fld.fold_fn_decl(expanded_decl);
1108     // now, a renamer for *all* idents, for the body:
1109     let mut rename_fld = IdentRenamer{renames: &renames};
1110     let rewritten_body = fld.fold_block(rename_fld.fold_block(block));
1111     (rewritten_fn_decl,rewritten_body)
1112 }
1113
1114 fn expand_and_rename_method(sig: ast::MethodSig, body: P<ast::Block>,
1115                             fld: &mut MacroExpander)
1116                             -> (ast::MethodSig, P<ast::Block>) {
1117     let (rewritten_fn_decl, rewritten_body)
1118         = expand_and_rename_fn_decl_and_block(sig.decl, body, fld);
1119     (ast::MethodSig {
1120         generics: fld.fold_generics(sig.generics),
1121         abi: sig.abi,
1122         explicit_self: fld.fold_explicit_self(sig.explicit_self),
1123         unsafety: sig.unsafety,
1124         constness: sig.constness,
1125         decl: rewritten_fn_decl
1126     }, rewritten_body)
1127 }
1128
1129 pub fn expand_type(t: P<ast::Ty>, fld: &mut MacroExpander) -> P<ast::Ty> {
1130     let t = match t.node.clone() {
1131         ast::Ty_::TyMac(mac) => {
1132             if fld.cx.ecfg.features.unwrap().type_macros {
1133                 let expanded_ty = match expand_mac_invoc(mac, t.span,
1134                                                          |r| r.make_ty(),
1135                                                          mark_ty,
1136                                                          fld) {
1137                     Some(ty) => ty,
1138                     None => {
1139                         return DummyResult::raw_ty(t.span);
1140                     }
1141                 };
1142
1143                 // Keep going, outside-in.
1144                 let fully_expanded = fld.fold_ty(expanded_ty);
1145                 fld.cx.bt_pop();
1146
1147                 fully_expanded.map(|t| ast::Ty {
1148                     id: ast::DUMMY_NODE_ID,
1149                     node: t.node,
1150                     span: t.span,
1151                     })
1152             } else {
1153                 feature_gate::emit_feature_err(
1154                     &fld.cx.parse_sess.span_diagnostic,
1155                     "type_macros",
1156                     t.span,
1157                     feature_gate::GateIssue::Language,
1158                     "type macros are experimental");
1159
1160                 DummyResult::raw_ty(t.span)
1161             }
1162         }
1163         _ => t
1164     };
1165
1166     fold::noop_fold_ty(t, fld)
1167 }
1168
1169 /// A tree-folder that performs macro expansion
1170 pub struct MacroExpander<'a, 'b:'a> {
1171     pub cx: &'a mut ExtCtxt<'b>,
1172 }
1173
1174 impl<'a, 'b> MacroExpander<'a, 'b> {
1175     pub fn new(cx: &'a mut ExtCtxt<'b>) -> MacroExpander<'a, 'b> {
1176         MacroExpander { cx: cx }
1177     }
1178 }
1179
1180 impl<'a, 'b> Folder for MacroExpander<'a, 'b> {
1181     fn fold_expr(&mut self, expr: P<ast::Expr>) -> P<ast::Expr> {
1182         expand_expr(expr, self)
1183     }
1184
1185     fn fold_pat(&mut self, pat: P<ast::Pat>) -> P<ast::Pat> {
1186         expand_pat(pat, self)
1187     }
1188
1189     fn fold_item(&mut self, item: P<ast::Item>) -> SmallVector<P<ast::Item>> {
1190         expand_item(item, self)
1191     }
1192
1193     fn fold_item_underscore(&mut self, item: ast::Item_) -> ast::Item_ {
1194         expand_item_underscore(item, self)
1195     }
1196
1197     fn fold_stmt(&mut self, stmt: P<ast::Stmt>) -> SmallVector<P<ast::Stmt>> {
1198         expand_stmt(stmt, self)
1199     }
1200
1201     fn fold_block(&mut self, block: P<Block>) -> P<Block> {
1202         expand_block(block, self)
1203     }
1204
1205     fn fold_arm(&mut self, arm: ast::Arm) -> ast::Arm {
1206         expand_arm(arm, self)
1207     }
1208
1209     fn fold_trait_item(&mut self, i: P<ast::TraitItem>) -> SmallVector<P<ast::TraitItem>> {
1210         expand_annotatable(Annotatable::TraitItem(i), self)
1211             .into_iter().map(|i| i.expect_trait_item()).collect()
1212     }
1213
1214     fn fold_impl_item(&mut self, i: P<ast::ImplItem>) -> SmallVector<P<ast::ImplItem>> {
1215         expand_annotatable(Annotatable::ImplItem(i), self)
1216             .into_iter().map(|i| i.expect_impl_item()).collect()
1217     }
1218
1219     fn fold_ty(&mut self, ty: P<ast::Ty>) -> P<ast::Ty> {
1220         expand_type(ty, self)
1221     }
1222
1223     fn new_span(&mut self, span: Span) -> Span {
1224         new_span(self.cx, span)
1225     }
1226 }
1227
1228 fn new_span(cx: &ExtCtxt, sp: Span) -> Span {
1229     /* this discards information in the case of macro-defining macros */
1230     Span {
1231         lo: sp.lo,
1232         hi: sp.hi,
1233         expn_id: cx.backtrace(),
1234     }
1235 }
1236
1237 pub struct ExpansionConfig<'feat> {
1238     pub crate_name: String,
1239     pub features: Option<&'feat Features>,
1240     pub recursion_limit: usize,
1241     pub trace_mac: bool,
1242 }
1243
1244 macro_rules! feature_tests {
1245     ($( fn $getter:ident = $field:ident, )*) => {
1246         $(
1247             pub fn $getter(&self) -> bool {
1248                 match self.features {
1249                     Some(&Features { $field: true, .. }) => true,
1250                     _ => false,
1251                 }
1252             }
1253         )*
1254     }
1255 }
1256
1257 impl<'feat> ExpansionConfig<'feat> {
1258     pub fn default(crate_name: String) -> ExpansionConfig<'static> {
1259         ExpansionConfig {
1260             crate_name: crate_name,
1261             features: None,
1262             recursion_limit: 64,
1263             trace_mac: false,
1264         }
1265     }
1266
1267     feature_tests! {
1268         fn enable_quotes = allow_quote,
1269         fn enable_asm = allow_asm,
1270         fn enable_log_syntax = allow_log_syntax,
1271         fn enable_concat_idents = allow_concat_idents,
1272         fn enable_trace_macros = allow_trace_macros,
1273         fn enable_allow_internal_unstable = allow_internal_unstable,
1274         fn enable_custom_derive = allow_custom_derive,
1275         fn enable_pushpop_unsafe = allow_pushpop_unsafe,
1276     }
1277 }
1278
1279 pub fn expand_crate(mut cx: ExtCtxt,
1280                     // these are the macros being imported to this crate:
1281                     imported_macros: Vec<ast::MacroDef>,
1282                     user_exts: Vec<NamedSyntaxExtension>,
1283                     c: Crate) -> (Crate, HashSet<Name>) {
1284     if std_inject::no_core(&c) {
1285         cx.crate_root = None;
1286     } else if std_inject::no_std(&c) {
1287         cx.crate_root = Some("core");
1288     } else {
1289         cx.crate_root = Some("std");
1290     }
1291     let ret = {
1292         let mut expander = MacroExpander::new(&mut cx);
1293
1294         for def in imported_macros {
1295             expander.cx.insert_macro(def);
1296         }
1297
1298         for (name, extension) in user_exts {
1299             expander.cx.syntax_env.insert(name, extension);
1300         }
1301
1302         let mut ret = expander.fold_crate(c);
1303         ret.exported_macros = expander.cx.exported_macros.clone();
1304         cx.parse_sess.span_diagnostic.abort_if_errors();
1305         ret
1306     };
1307     return (ret, cx.syntax_env.names);
1308 }
1309
1310 // HYGIENIC CONTEXT EXTENSION:
1311 // all of these functions are for walking over
1312 // ASTs and making some change to the context of every
1313 // element that has one. a CtxtFn is a trait-ified
1314 // version of a closure in (SyntaxContext -> SyntaxContext).
1315 // the ones defined here include:
1316 // Marker - add a mark to a context
1317
1318 // A Marker adds the given mark to the syntax context
1319 struct Marker { mark: Mrk }
1320
1321 impl Folder for Marker {
1322     fn fold_ident(&mut self, id: Ident) -> Ident {
1323         ast::Ident::new(id.name, mtwt::apply_mark(self.mark, id.ctxt))
1324     }
1325     fn fold_mac(&mut self, Spanned {node, span}: ast::Mac) -> ast::Mac {
1326         Spanned {
1327             node: Mac_ {
1328                 path: self.fold_path(node.path),
1329                 tts: self.fold_tts(&node.tts),
1330                 ctxt: mtwt::apply_mark(self.mark, node.ctxt),
1331             },
1332             span: span,
1333         }
1334     }
1335 }
1336
1337 // apply a given mark to the given token trees. Used prior to expansion of a macro.
1338 fn mark_tts(tts: &[TokenTree], m: Mrk) -> Vec<TokenTree> {
1339     noop_fold_tts(tts, &mut Marker{mark:m})
1340 }
1341
1342 // apply a given mark to the given expr. Used following the expansion of a macro.
1343 fn mark_expr(expr: P<ast::Expr>, m: Mrk) -> P<ast::Expr> {
1344     Marker{mark:m}.fold_expr(expr)
1345 }
1346
1347 // apply a given mark to the given pattern. Used following the expansion of a macro.
1348 fn mark_pat(pat: P<ast::Pat>, m: Mrk) -> P<ast::Pat> {
1349     Marker{mark:m}.fold_pat(pat)
1350 }
1351
1352 // apply a given mark to the given stmt. Used following the expansion of a macro.
1353 fn mark_stmt(stmt: P<ast::Stmt>, m: Mrk) -> P<ast::Stmt> {
1354     Marker{mark:m}.fold_stmt(stmt)
1355         .expect_one("marking a stmt didn't return exactly one stmt")
1356 }
1357
1358 // apply a given mark to the given item. Used following the expansion of a macro.
1359 fn mark_item(expr: P<ast::Item>, m: Mrk) -> P<ast::Item> {
1360     Marker{mark:m}.fold_item(expr)
1361         .expect_one("marking an item didn't return exactly one item")
1362 }
1363
1364 // apply a given mark to the given item. Used following the expansion of a macro.
1365 fn mark_impl_item(ii: P<ast::ImplItem>, m: Mrk) -> P<ast::ImplItem> {
1366     Marker{mark:m}.fold_impl_item(ii)
1367         .expect_one("marking an impl item didn't return exactly one impl item")
1368 }
1369
1370 fn mark_ty(ty: P<ast::Ty>, m: Mrk) -> P<ast::Ty> {
1371     Marker { mark: m }.fold_ty(ty)
1372 }
1373
1374 /// Check that there are no macro invocations left in the AST:
1375 pub fn check_for_macros(sess: &parse::ParseSess, krate: &ast::Crate) {
1376     visit::walk_crate(&mut MacroExterminator{sess:sess}, krate);
1377 }
1378
1379 /// A visitor that ensures that no macro invocations remain in an AST.
1380 struct MacroExterminator<'a>{
1381     sess: &'a parse::ParseSess
1382 }
1383
1384 impl<'a, 'v> Visitor<'v> for MacroExterminator<'a> {
1385     fn visit_mac(&mut self, mac: &ast::Mac) {
1386         self.sess.span_diagnostic.span_bug(mac.span,
1387                                            "macro exterminator: expected AST \
1388                                            with no macro invocations");
1389     }
1390 }
1391
1392
1393 #[cfg(test)]
1394 mod tests {
1395     use super::{pattern_bindings, expand_crate};
1396     use super::{PatIdentFinder, IdentRenamer, PatIdentRenamer, ExpansionConfig};
1397     use ast;
1398     use ast::Name;
1399     use codemap;
1400     use ext::base::ExtCtxt;
1401     use ext::mtwt;
1402     use fold::Folder;
1403     use parse;
1404     use parse::token;
1405     use util::parser_testing::{string_to_parser};
1406     use util::parser_testing::{string_to_pat, string_to_crate, strs_to_idents};
1407     use visit;
1408     use visit::Visitor;
1409
1410     // a visitor that extracts the paths
1411     // from a given thingy and puts them in a mutable
1412     // array (passed in to the traversal)
1413     #[derive(Clone)]
1414     struct PathExprFinderContext {
1415         path_accumulator: Vec<ast::Path> ,
1416     }
1417
1418     impl<'v> Visitor<'v> for PathExprFinderContext {
1419         fn visit_expr(&mut self, expr: &ast::Expr) {
1420             if let ast::ExprPath(None, ref p) = expr.node {
1421                 self.path_accumulator.push(p.clone());
1422             }
1423             visit::walk_expr(self, expr);
1424         }
1425     }
1426
1427     // find the variable references in a crate
1428     fn crate_varrefs(the_crate : &ast::Crate) -> Vec<ast::Path> {
1429         let mut path_finder = PathExprFinderContext{path_accumulator:Vec::new()};
1430         visit::walk_crate(&mut path_finder, the_crate);
1431         path_finder.path_accumulator
1432     }
1433
1434     /// A Visitor that extracts the identifiers from a thingy.
1435     // as a side note, I'm starting to want to abstract over these....
1436     struct IdentFinder {
1437         ident_accumulator: Vec<ast::Ident>
1438     }
1439
1440     impl<'v> Visitor<'v> for IdentFinder {
1441         fn visit_ident(&mut self, _: codemap::Span, id: ast::Ident){
1442             self.ident_accumulator.push(id);
1443         }
1444     }
1445
1446     /// Find the idents in a crate
1447     fn crate_idents(the_crate: &ast::Crate) -> Vec<ast::Ident> {
1448         let mut ident_finder = IdentFinder{ident_accumulator: Vec::new()};
1449         visit::walk_crate(&mut ident_finder, the_crate);
1450         ident_finder.ident_accumulator
1451     }
1452
1453     // these following tests are quite fragile, in that they don't test what
1454     // *kind* of failure occurs.
1455
1456     fn test_ecfg() -> ExpansionConfig<'static> {
1457         ExpansionConfig::default("test".to_string())
1458     }
1459
1460     // make sure that macros can't escape fns
1461     #[should_panic]
1462     #[test] fn macros_cant_escape_fns_test () {
1463         let src = "fn bogus() {macro_rules! z (() => (3+4));}\
1464                    fn inty() -> i32 { z!() }".to_string();
1465         let sess = parse::ParseSess::new();
1466         let crate_ast = parse::parse_crate_from_source_str(
1467             "<test>".to_string(),
1468             src,
1469             Vec::new(), &sess);
1470         // should fail:
1471         let mut gated_cfgs = vec![];
1472         let ecx = ExtCtxt::new(&sess, vec![], test_ecfg(), &mut gated_cfgs);
1473         expand_crate(ecx, vec![], vec![], crate_ast);
1474     }
1475
1476     // make sure that macros can't escape modules
1477     #[should_panic]
1478     #[test] fn macros_cant_escape_mods_test () {
1479         let src = "mod foo {macro_rules! z (() => (3+4));}\
1480                    fn inty() -> i32 { z!() }".to_string();
1481         let sess = parse::ParseSess::new();
1482         let crate_ast = parse::parse_crate_from_source_str(
1483             "<test>".to_string(),
1484             src,
1485             Vec::new(), &sess);
1486         let mut gated_cfgs = vec![];
1487         let ecx = ExtCtxt::new(&sess, vec![], test_ecfg(), &mut gated_cfgs);
1488         expand_crate(ecx, vec![], vec![], crate_ast);
1489     }
1490
1491     // macro_use modules should allow macros to escape
1492     #[test] fn macros_can_escape_flattened_mods_test () {
1493         let src = "#[macro_use] mod foo {macro_rules! z (() => (3+4));}\
1494                    fn inty() -> i32 { z!() }".to_string();
1495         let sess = parse::ParseSess::new();
1496         let crate_ast = parse::parse_crate_from_source_str(
1497             "<test>".to_string(),
1498             src,
1499             Vec::new(), &sess);
1500         let mut gated_cfgs = vec![];
1501         let ecx = ExtCtxt::new(&sess, vec![], test_ecfg(), &mut gated_cfgs);
1502         expand_crate(ecx, vec![], vec![], crate_ast);
1503     }
1504
1505     fn expand_crate_str(crate_str: String) -> ast::Crate {
1506         let ps = parse::ParseSess::new();
1507         let crate_ast = panictry!(string_to_parser(&ps, crate_str).parse_crate_mod());
1508         // the cfg argument actually does matter, here...
1509         let mut gated_cfgs = vec![];
1510         let ecx = ExtCtxt::new(&ps, vec![], test_ecfg(), &mut gated_cfgs);
1511         expand_crate(ecx, vec![], vec![], crate_ast).0
1512     }
1513
1514     // find the pat_ident paths in a crate
1515     fn crate_bindings(the_crate : &ast::Crate) -> Vec<ast::Ident> {
1516         let mut name_finder = PatIdentFinder{ident_accumulator:Vec::new()};
1517         visit::walk_crate(&mut name_finder, the_crate);
1518         name_finder.ident_accumulator
1519     }
1520
1521     #[test] fn macro_tokens_should_match(){
1522         expand_crate_str(
1523             "macro_rules! m((a)=>(13)) ;fn main(){m!(a);}".to_string());
1524     }
1525
1526     // should be able to use a bound identifier as a literal in a macro definition:
1527     #[test] fn self_macro_parsing(){
1528         expand_crate_str(
1529             "macro_rules! foo ((zz) => (287;));
1530             fn f(zz: i32) {foo!(zz);}".to_string()
1531             );
1532     }
1533
1534     // renaming tests expand a crate and then check that the bindings match
1535     // the right varrefs. The specification of the test case includes the
1536     // text of the crate, and also an array of arrays.  Each element in the
1537     // outer array corresponds to a binding in the traversal of the AST
1538     // induced by visit.  Each of these arrays contains a list of indexes,
1539     // interpreted as the varrefs in the varref traversal that this binding
1540     // should match.  So, for instance, in a program with two bindings and
1541     // three varrefs, the array [[1, 2], [0]] would indicate that the first
1542     // binding should match the second two varrefs, and the second binding
1543     // should match the first varref.
1544     //
1545     // Put differently; this is a sparse representation of a boolean matrix
1546     // indicating which bindings capture which identifiers.
1547     //
1548     // Note also that this matrix is dependent on the implicit ordering of
1549     // the bindings and the varrefs discovered by the name-finder and the path-finder.
1550     //
1551     // The comparisons are done post-mtwt-resolve, so we're comparing renamed
1552     // names; differences in marks don't matter any more.
1553     //
1554     // oog... I also want tests that check "bound-identifier-=?". That is,
1555     // not just "do these have the same name", but "do they have the same
1556     // name *and* the same marks"? Understanding this is really pretty painful.
1557     // in principle, you might want to control this boolean on a per-varref basis,
1558     // but that would make things even harder to understand, and might not be
1559     // necessary for thorough testing.
1560     type RenamingTest = (&'static str, Vec<Vec<usize>>, bool);
1561
1562     #[test]
1563     fn automatic_renaming () {
1564         let tests: Vec<RenamingTest> =
1565             vec!(// b & c should get new names throughout, in the expr too:
1566                 ("fn a() -> i32 { let b = 13; let c = b; b+c }",
1567                  vec!(vec!(0,1),vec!(2)), false),
1568                 // both x's should be renamed (how is this causing a bug?)
1569                 ("fn main () {let x: i32 = 13;x;}",
1570                  vec!(vec!(0)), false),
1571                 // the use of b after the + should be renamed, the other one not:
1572                 ("macro_rules! f (($x:ident) => (b + $x)); fn a() -> i32 { let b = 13; f!(b)}",
1573                  vec!(vec!(1)), false),
1574                 // the b before the plus should not be renamed (requires marks)
1575                 ("macro_rules! f (($x:ident) => ({let b=9; ($x + b)})); fn a() -> i32 { f!(b)}",
1576                  vec!(vec!(1)), false),
1577                 // the marks going in and out of letty should cancel, allowing that $x to
1578                 // capture the one following the semicolon.
1579                 // this was an awesome test case, and caught a *lot* of bugs.
1580                 ("macro_rules! letty(($x:ident) => (let $x = 15;));
1581                   macro_rules! user(($x:ident) => ({letty!($x); $x}));
1582                   fn main() -> i32 {user!(z)}",
1583                  vec!(vec!(0)), false)
1584                 );
1585         for (idx,s) in tests.iter().enumerate() {
1586             run_renaming_test(s,idx);
1587         }
1588     }
1589
1590     // no longer a fixme #8062: this test exposes a *potential* bug; our system does
1591     // not behave exactly like MTWT, but a conversation with Matthew Flatt
1592     // suggests that this can only occur in the presence of local-expand, which
1593     // we have no plans to support. ... unless it's needed for item hygiene....
1594     #[ignore]
1595     #[test]
1596     fn issue_8062(){
1597         run_renaming_test(
1598             &("fn main() {let hrcoo = 19; macro_rules! getx(()=>(hrcoo)); getx!();}",
1599               vec!(vec!(0)), true), 0)
1600     }
1601
1602     // FIXME #6994:
1603     // the z flows into and out of two macros (g & f) along one path, and one
1604     // (just g) along the other, so the result of the whole thing should
1605     // be "let z_123 = 3; z_123"
1606     #[ignore]
1607     #[test]
1608     fn issue_6994(){
1609         run_renaming_test(
1610             &("macro_rules! g (($x:ident) =>
1611               ({macro_rules! f(($y:ident)=>({let $y=3;$x}));f!($x)}));
1612               fn a(){g!(z)}",
1613               vec!(vec!(0)),false),
1614             0)
1615     }
1616
1617     // match variable hygiene. Should expand into
1618     // fn z() {match 8 {x_1 => {match 9 {x_2 | x_2 if x_2 == x_1 => x_2 + x_1}}}}
1619     #[test]
1620     fn issue_9384(){
1621         run_renaming_test(
1622             &("macro_rules! bad_macro (($ex:expr) => ({match 9 {x | x if x == $ex => x + $ex}}));
1623               fn z() {match 8 {x => bad_macro!(x)}}",
1624               // NB: the third "binding" is the repeat of the second one.
1625               vec!(vec!(1,3),vec!(0,2),vec!(0,2)),
1626               true),
1627             0)
1628     }
1629
1630     // interpolated nodes weren't getting labeled.
1631     // should expand into
1632     // fn main(){let g1_1 = 13; g1_1}}
1633     #[test]
1634     fn pat_expand_issue_15221(){
1635         run_renaming_test(
1636             &("macro_rules! inner ( ($e:pat ) => ($e));
1637               macro_rules! outer ( ($e:pat ) => (inner!($e)));
1638               fn main() { let outer!(g) = 13; g;}",
1639               vec!(vec!(0)),
1640               true),
1641             0)
1642     }
1643
1644     // create a really evil test case where a $x appears inside a binding of $x
1645     // but *shouldn't* bind because it was inserted by a different macro....
1646     // can't write this test case until we have macro-generating macros.
1647
1648     // method arg hygiene
1649     // method expands to fn get_x(&self_0, x_1: i32) {self_0 + self_2 + x_3 + x_1}
1650     #[test]
1651     fn method_arg_hygiene(){
1652         run_renaming_test(
1653             &("macro_rules! inject_x (()=>(x));
1654               macro_rules! inject_self (()=>(self));
1655               struct A;
1656               impl A{fn get_x(&self, x: i32) {self + inject_self!() + inject_x!() + x;} }",
1657               vec!(vec!(0),vec!(3)),
1658               true),
1659             0)
1660     }
1661
1662     // ooh, got another bite?
1663     // expands to struct A; impl A {fn thingy(&self_1) {self_1;}}
1664     #[test]
1665     fn method_arg_hygiene_2(){
1666         run_renaming_test(
1667             &("struct A;
1668               macro_rules! add_method (($T:ty) =>
1669               (impl $T {  fn thingy(&self) {self;} }));
1670               add_method!(A);",
1671               vec!(vec!(0)),
1672               true),
1673             0)
1674     }
1675
1676     // item fn hygiene
1677     // expands to fn q(x_1: i32){fn g(x_2: i32){x_2 + x_1};}
1678     #[test]
1679     fn issue_9383(){
1680         run_renaming_test(
1681             &("macro_rules! bad_macro (($ex:expr) => (fn g(x: i32){ x + $ex }));
1682               fn q(x: i32) { bad_macro!(x); }",
1683               vec!(vec!(1),vec!(0)),true),
1684             0)
1685     }
1686
1687     // closure arg hygiene (ExprClosure)
1688     // expands to fn f(){(|x_1 : i32| {(x_2 + x_1)})(3);}
1689     #[test]
1690     fn closure_arg_hygiene(){
1691         run_renaming_test(
1692             &("macro_rules! inject_x (()=>(x));
1693             fn f(){(|x : i32| {(inject_x!() + x)})(3);}",
1694               vec!(vec!(1)),
1695               true),
1696             0)
1697     }
1698
1699     // macro_rules in method position. Sadly, unimplemented.
1700     #[test]
1701     fn macro_in_method_posn(){
1702         expand_crate_str(
1703             "macro_rules! my_method (() => (fn thirteen(&self) -> i32 {13}));
1704             struct A;
1705             impl A{ my_method!(); }
1706             fn f(){A.thirteen;}".to_string());
1707     }
1708
1709     // another nested macro
1710     // expands to impl Entries {fn size_hint(&self_1) {self_1;}
1711     #[test]
1712     fn item_macro_workaround(){
1713         run_renaming_test(
1714             &("macro_rules! item { ($i:item) => {$i}}
1715               struct Entries;
1716               macro_rules! iterator_impl {
1717               () => { item!( impl Entries { fn size_hint(&self) { self;}});}}
1718               iterator_impl! { }",
1719               vec!(vec!(0)), true),
1720             0)
1721     }
1722
1723     // run one of the renaming tests
1724     fn run_renaming_test(t: &RenamingTest, test_idx: usize) {
1725         let invalid_name = token::special_idents::invalid.name;
1726         let (teststr, bound_connections, bound_ident_check) = match *t {
1727             (ref str,ref conns, bic) => (str.to_string(), conns.clone(), bic)
1728         };
1729         let cr = expand_crate_str(teststr.to_string());
1730         let bindings = crate_bindings(&cr);
1731         let varrefs = crate_varrefs(&cr);
1732
1733         // must be one check clause for each binding:
1734         assert_eq!(bindings.len(),bound_connections.len());
1735         for (binding_idx,shouldmatch) in bound_connections.iter().enumerate() {
1736             let binding_name = mtwt::resolve(bindings[binding_idx]);
1737             let binding_marks = mtwt::marksof(bindings[binding_idx].ctxt, invalid_name);
1738             // shouldmatch can't name varrefs that don't exist:
1739             assert!((shouldmatch.is_empty()) ||
1740                     (varrefs.len() > *shouldmatch.iter().max().unwrap()));
1741             for (idx,varref) in varrefs.iter().enumerate() {
1742                 let print_hygiene_debug_info = || {
1743                     // good lord, you can't make a path with 0 segments, can you?
1744                     let final_varref_ident = match varref.segments.last() {
1745                         Some(pathsegment) => pathsegment.identifier,
1746                         None => panic!("varref with 0 path segments?")
1747                     };
1748                     let varref_name = mtwt::resolve(final_varref_ident);
1749                     let varref_idents : Vec<ast::Ident>
1750                         = varref.segments.iter().map(|s| s.identifier)
1751                         .collect();
1752                     println!("varref #{}: {:?}, resolves to {}",idx, varref_idents, varref_name);
1753                     println!("varref's first segment's string: \"{}\"", final_varref_ident);
1754                     println!("binding #{}: {}, resolves to {}",
1755                              binding_idx, bindings[binding_idx], binding_name);
1756                     mtwt::with_sctable(|x| mtwt::display_sctable(x));
1757                 };
1758                 if shouldmatch.contains(&idx) {
1759                     // it should be a path of length 1, and it should
1760                     // be free-identifier=? or bound-identifier=? to the given binding
1761                     assert_eq!(varref.segments.len(),1);
1762                     let varref_name = mtwt::resolve(varref.segments[0].identifier);
1763                     let varref_marks = mtwt::marksof(varref.segments[0]
1764                                                            .identifier
1765                                                            .ctxt,
1766                                                      invalid_name);
1767                     if !(varref_name==binding_name) {
1768                         println!("uh oh, should match but doesn't:");
1769                         print_hygiene_debug_info();
1770                     }
1771                     assert_eq!(varref_name,binding_name);
1772                     if bound_ident_check {
1773                         // we're checking bound-identifier=?, and the marks
1774                         // should be the same, too:
1775                         assert_eq!(varref_marks,binding_marks.clone());
1776                     }
1777                 } else {
1778                     let varref_name = mtwt::resolve(varref.segments[0].identifier);
1779                     let fail = (varref.segments.len() == 1)
1780                         && (varref_name == binding_name);
1781                     // temp debugging:
1782                     if fail {
1783                         println!("failure on test {}",test_idx);
1784                         println!("text of test case: \"{}\"", teststr);
1785                         println!("");
1786                         println!("uh oh, matches but shouldn't:");
1787                         print_hygiene_debug_info();
1788                     }
1789                     assert!(!fail);
1790                 }
1791             }
1792         }
1793     }
1794
1795     #[test]
1796     fn fmt_in_macro_used_inside_module_macro() {
1797         let crate_str = "macro_rules! fmt_wrap(($b:expr)=>($b.to_string()));
1798 macro_rules! foo_module (() => (mod generated { fn a() { let xx = 147; fmt_wrap!(xx);}}));
1799 foo_module!();
1800 ".to_string();
1801         let cr = expand_crate_str(crate_str);
1802         // find the xx binding
1803         let bindings = crate_bindings(&cr);
1804         let cxbinds: Vec<&ast::Ident> =
1805             bindings.iter().filter(|b| b.name.as_str() == "xx").collect();
1806         let cxbinds: &[&ast::Ident] = &cxbinds[..];
1807         let cxbind = match (cxbinds.len(), cxbinds.get(0)) {
1808             (1, Some(b)) => *b,
1809             _ => panic!("expected just one binding for ext_cx")
1810         };
1811         let resolved_binding = mtwt::resolve(*cxbind);
1812         let varrefs = crate_varrefs(&cr);
1813
1814         // the xx binding should bind all of the xx varrefs:
1815         for (idx,v) in varrefs.iter().filter(|p| {
1816             p.segments.len() == 1
1817             && p.segments[0].identifier.name.as_str() == "xx"
1818         }).enumerate() {
1819             if mtwt::resolve(v.segments[0].identifier) != resolved_binding {
1820                 println!("uh oh, xx binding didn't match xx varref:");
1821                 println!("this is xx varref \\# {}", idx);
1822                 println!("binding: {}", cxbind);
1823                 println!("resolves to: {}", resolved_binding);
1824                 println!("varref: {}", v.segments[0].identifier);
1825                 println!("resolves to: {}",
1826                          mtwt::resolve(v.segments[0].identifier));
1827                 mtwt::with_sctable(|x| mtwt::display_sctable(x));
1828             }
1829             assert_eq!(mtwt::resolve(v.segments[0].identifier),
1830                        resolved_binding);
1831         };
1832     }
1833
1834     #[test]
1835     fn pat_idents(){
1836         let pat = string_to_pat(
1837             "(a,Foo{x:c @ (b,9),y:Bar(4,d)})".to_string());
1838         let idents = pattern_bindings(&pat);
1839         assert_eq!(idents, strs_to_idents(vec!("a","c","b","d")));
1840     }
1841
1842     // test the list of identifier patterns gathered by the visitor. Note that
1843     // 'None' is listed as an identifier pattern because we don't yet know that
1844     // it's the name of a 0-ary variant, and that 'i' appears twice in succession.
1845     #[test]
1846     fn crate_bindings_test(){
1847         let the_crate = string_to_crate("fn main (a: i32) -> i32 {|b| {
1848         match 34 {None => 3, Some(i) | i => j, Foo{k:z,l:y} => \"banana\"}} }".to_string());
1849         let idents = crate_bindings(&the_crate);
1850         assert_eq!(idents, strs_to_idents(vec!("a","b","None","i","i","z","y")));
1851     }
1852
1853     // test the IdentRenamer directly
1854     #[test]
1855     fn ident_renamer_test () {
1856         let the_crate = string_to_crate("fn f(x: i32){let x = x; x}".to_string());
1857         let f_ident = token::str_to_ident("f");
1858         let x_ident = token::str_to_ident("x");
1859         let int_ident = token::str_to_ident("i32");
1860         let renames = vec!((x_ident,Name(16)));
1861         let mut renamer = IdentRenamer{renames: &renames};
1862         let renamed_crate = renamer.fold_crate(the_crate);
1863         let idents = crate_idents(&renamed_crate);
1864         let resolved : Vec<ast::Name> = idents.iter().map(|id| mtwt::resolve(*id)).collect();
1865         assert_eq!(resolved, [f_ident.name,Name(16),int_ident.name,Name(16),Name(16),Name(16)]);
1866     }
1867
1868     // test the PatIdentRenamer; only PatIdents get renamed
1869     #[test]
1870     fn pat_ident_renamer_test () {
1871         let the_crate = string_to_crate("fn f(x: i32){let x = x; x}".to_string());
1872         let f_ident = token::str_to_ident("f");
1873         let x_ident = token::str_to_ident("x");
1874         let int_ident = token::str_to_ident("i32");
1875         let renames = vec!((x_ident,Name(16)));
1876         let mut renamer = PatIdentRenamer{renames: &renames};
1877         let renamed_crate = renamer.fold_crate(the_crate);
1878         let idents = crate_idents(&renamed_crate);
1879         let resolved : Vec<ast::Name> = idents.iter().map(|id| mtwt::resolve(*id)).collect();
1880         let x_name = x_ident.name;
1881         assert_eq!(resolved, [f_ident.name,Name(16),int_ident.name,Name(16),x_name,x_name]);
1882     }
1883 }