src/Pure/Syntax/syntax_phases.ML
changeset 42284 326f57825e1a
parent 42282 4fa41e068ff0
child 42288 2074b31650e6
--- a/src/Pure/Syntax/syntax_phases.ML	Fri Apr 08 11:39:45 2011 +0200
+++ b/src/Pure/Syntax/syntax_phases.ML	Fri Apr 08 13:31:16 2011 +0200
@@ -532,7 +532,7 @@
 
     fun ast_of tm =
       (case strip_comb tm of
-        (t as Abs _, ts) => Ast.mk_appl (ast_of (Syn_Trans.abs_tr' ctxt t)) (map ast_of ts)
+        (t as Abs _, ts) => Ast.mk_appl (ast_of (Syntax_Trans.abs_tr' ctxt t)) (map ast_of ts)
       | ((c as Const ("_free", _)), Free (x, T) :: ts) =>
           Ast.mk_appl (constrain (c $ Lexicon.free x) T) (map ast_of ts)
       | ((c as Const ("_var", _)), Var (xi, T) :: ts) =>
@@ -557,7 +557,7 @@
       else simple_ast_of ctxt t;
   in
     tm
-    |> Syn_Trans.prop_tr'
+    |> Syntax_Trans.prop_tr'
     |> show_types ? (#1 o prune_typs o rpair [])
     |> mark_atoms
     |> ast_of