ProgTutorial/Base.thy
changeset 394 0019ebf76e10
parent 346 0fea8b7a14a1
child 396 a2e49e0771b3
equal deleted inserted replaced
393:d8b6d5003823 394:0019ebf76e10
     2 imports Main LaTeXsugar
     2 imports Main LaTeXsugar
     3 uses
     3 uses
     4   ("output_tutorial.ML")
     4   ("output_tutorial.ML")
     5   ("antiquote_setup.ML")
     5   ("antiquote_setup.ML")
     6 begin
     6 begin
       
     7 
       
     8 notation (latex output)
       
     9   Cons ("_ # _" [66,65] 65)
       
    10 
     7 
    11 
     8 (* rebinding of writeln and tracing so that it can *)
    12 (* rebinding of writeln and tracing so that it can *)
     9 (* be compared in intiquotations                   *)
    13 (* be compared in intiquotations                   *)
    10 ML {* 
    14 ML {* 
    11 fun writeln s = (Output.writeln s; s)
    15 fun writeln s = (Output.writeln s; s)
    84 end
    88 end
    85 *}
    89 *}
    86 
    90 
    87 ML {*
    91 ML {*
    88 fun propagate_env (context as Context.Proof lthy) =
    92 fun propagate_env (context as Context.Proof lthy) =
    89       Context.Proof (LocalTheory.map_contexts (ML_Env.inherit context) lthy)
    93       Context.Proof (Local_Theory.map_contexts (ML_Env.inherit context) lthy)
    90   | propagate_env context = context
    94   | propagate_env context = context
    91 
    95 
    92 fun propagate_env_prf prf = Proof.map_contexts
    96 fun propagate_env_prf prf = Proof.map_contexts
    93   (Context.proof_map (ML_Env.inherit (Context.Proof (Proof.context_of prf)))) prf
    97   (Context.proof_map (ML_Env.inherit (Context.Proof (Proof.context_of prf)))) prf
    94 *}
    98 *}