src/Pure/Isar/proof_context.ML
changeset 42360 da8817d01e7c
parent 42359 6ca5407863ed
child 42363 e52e3f697510
equal deleted inserted replaced
42359:6ca5407863ed 42360:da8817d01e7c
   159   val verbose: bool Unsynchronized.ref
   159   val verbose: bool Unsynchronized.ref
   160   val pretty_ctxt: Proof.context -> Pretty.T list
   160   val pretty_ctxt: Proof.context -> Pretty.T list
   161   val pretty_context: Proof.context -> Pretty.T list
   161   val pretty_context: Proof.context -> Pretty.T list
   162 end;
   162 end;
   163 
   163 
   164 structure ProofContext: PROOF_CONTEXT =
   164 structure Proof_Context: PROOF_CONTEXT =
   165 struct
   165 struct
   166 
   166 
   167 open ProofContext;
   167 open Proof_Context;
   168 
   168 
   169 
   169 
   170 (** inner syntax mode **)
   170 (** inner syntax mode **)
   171 
   171 
   172 datatype mode =
   172 datatype mode =
   595   in T end;
   595   in T end;
   596 
   596 
   597 
   597 
   598 local
   598 local
   599 
   599 
   600 val dummies = Config.bool (Config.declare "ProofContext.dummies" (K (Config.Bool false)));
   600 val dummies = Config.bool (Config.declare "Proof_Context.dummies" (K (Config.Bool false)));
   601 
   601 
   602 fun check_dummies ctxt t =
   602 fun check_dummies ctxt t =
   603   if Config.get ctxt dummies then t
   603   if Config.get ctxt dummies then t
   604   else Term.no_dummy_patterns t handle TERM _ => error "Illegal dummy pattern(s) in term";
   604   else Term.no_dummy_patterns t handle TERM _ => error "Illegal dummy pattern(s) in term";
   605 
   605 
  1343     verb single (fn () => Pretty.big_list "default sorts:" (map prt_defS (Vartab.dest sorts)))
  1343     verb single (fn () => Pretty.big_list "default sorts:" (map prt_defS (Vartab.dest sorts)))
  1344   end;
  1344   end;
  1345 
  1345 
  1346 end;
  1346 end;
  1347 
  1347 
  1348 val show_abbrevs = ProofContext.show_abbrevs;
  1348 val show_abbrevs = Proof_Context.show_abbrevs;
  1349 
  1349