src/Pure/Isar/proof_context.ML
changeset 52156 576aceb343dc
parent 51686 532e0ac5a66d
child 52223 5bb6ae8acb87
equal deleted inserted replaced
52155:761c325a65d4 52156:576aceb343dc
    26   val syn_of: Proof.context -> Syntax.syntax
    26   val syn_of: Proof.context -> Syntax.syntax
    27   val tsig_of: Proof.context -> Type.tsig
    27   val tsig_of: Proof.context -> Type.tsig
    28   val set_defsort: sort -> Proof.context -> Proof.context
    28   val set_defsort: sort -> Proof.context -> Proof.context
    29   val default_sort: Proof.context -> indexname -> sort
    29   val default_sort: Proof.context -> indexname -> sort
    30   val consts_of: Proof.context -> Consts.T
    30   val consts_of: Proof.context -> Consts.T
    31   val the_const_constraint: Proof.context -> string -> typ
       
    32   val set_syntax_mode: Syntax.mode -> Proof.context -> Proof.context
    31   val set_syntax_mode: Syntax.mode -> Proof.context -> Proof.context
    33   val restore_syntax_mode: Proof.context -> Proof.context -> Proof.context
    32   val restore_syntax_mode: Proof.context -> Proof.context -> Proof.context
    34   val facts_of: Proof.context -> Facts.T
    33   val facts_of: Proof.context -> Facts.T
    35   val cases_of: Proof.context -> (string * (Rule_Cases.T * bool)) list
    34   val cases_of: Proof.context -> (string * (Rule_Cases.T * bool)) list
    36   val map_naming: (Name_Space.naming -> Name_Space.naming) -> Proof.context -> Proof.context
    35   val map_naming: (Name_Space.naming -> Name_Space.naming) -> Proof.context -> Proof.context
   262 val tsig_of = #1 o #tsig o rep_data;
   261 val tsig_of = #1 o #tsig o rep_data;
   263 val set_defsort = map_tsig o apfst o Type.set_defsort;
   262 val set_defsort = map_tsig o apfst o Type.set_defsort;
   264 fun default_sort ctxt = the_default (Type.defaultS (tsig_of ctxt)) o Variable.def_sort ctxt;
   263 fun default_sort ctxt = the_default (Type.defaultS (tsig_of ctxt)) o Variable.def_sort ctxt;
   265 
   264 
   266 val consts_of = #1 o #consts o rep_data;
   265 val consts_of = #1 o #consts o rep_data;
   267 val the_const_constraint = Consts.the_constraint o consts_of;
       
   268 
       
   269 val facts_of = #facts o rep_data;
   266 val facts_of = #facts o rep_data;
   270 val cases_of = #cases o rep_data;
   267 val cases_of = #cases o rep_data;
   271 
   268 
   272 
   269 
   273 (* naming *)
   270 (* naming *)