src/Pure/Isar/element.ML
changeset 63352 4eaf35781b23
parent 62681 45b8dd2d3827
child 63395 734723445a8c
--- a/src/Pure/Isar/element.ML	Wed Jun 22 16:04:03 2016 +0200
+++ b/src/Pure/Isar/element.ML	Thu Jun 23 11:01:14 2016 +0200
@@ -239,8 +239,8 @@
         then insert (op =) (Variable.revert_fixed ctxt' x, T) else I | _ => I) prop []);
   in
     pretty_ctxt ctxt' (Fixes (map (fn (x, T) => (Binding.name x, SOME T, NoSyn)) fixes)) @
-    pretty_ctxt ctxt' (Assumes (map (fn t => (Attrib.empty_binding, [(t, [])])) assumes)) @
-     (if null cases then pretty_stmt ctxt' (Shows [(Attrib.empty_binding, [(concl, [])])])
+    pretty_ctxt ctxt' (Assumes (map (fn t => (Binding.empty_atts, [(t, [])])) assumes)) @
+     (if null cases then pretty_stmt ctxt' (Shows [(Binding.empty_atts, [(concl, [])])])
       else
         let val (clauses, ctxt'') = fold_map obtain cases ctxt'
         in pretty_stmt ctxt'' (Obtains clauses) end)
@@ -293,7 +293,7 @@
   in
     Proof.map_context (K goal_ctxt) #>
     Proof.internal_goal (K (K ())) (Proof_Context.get_mode goal_ctxt) true cmd
-      NONE after_qed' [] [] (map (pair Thm.empty_binding) propp) #> snd
+      NONE after_qed' [] [] (map (pair Binding.empty_atts) propp) #> snd
   end;
 
 in