src/Pure/Isar/calculation.ML
changeset 42360 da8817d01e7c
parent 39557 fe5722fce758
child 45375 7fe19930dfc9
equal deleted inserted replaced
42359:6ca5407863ed 42360:da8817d01e7c
   114     val state' = put_calculation (SOME calc) state;
   114     val state' = put_calculation (SOME calc) state;
   115     val ctxt' = Proof.context_of state';
   115     val ctxt' = Proof.context_of state';
   116     val _ =
   116     val _ =
   117       if int then
   117       if int then
   118         Pretty.writeln
   118         Pretty.writeln
   119           (ProofContext.pretty_fact ctxt'
   119           (Proof_Context.pretty_fact ctxt'
   120             (ProofContext.full_name ctxt' (Binding.name calculationN), calc))
   120             (Proof_Context.full_name ctxt' (Binding.name calculationN), calc))
   121       else ();
   121       else ();
   122   in state' |> final ? (put_calculation NONE #> Proof.chain_facts calc) end;
   122   in state' |> final ? (put_calculation NONE #> Proof.chain_facts calc) end;
   123 
   123 
   124 
   124 
   125 (* also and finally *)
   125 (* also and finally *)