src/Pure/raw_simplifier.ML
changeset 70586 57df8a85317a
parent 70528 9b3610fe74d6
child 71177 71467e35fc3c
equal deleted inserted replaced
70583:17909568216e 70586:57df8a85317a
    80      {mk: Proof.context -> thm -> thm list,
    80      {mk: Proof.context -> thm -> thm list,
    81       mk_cong: Proof.context -> thm -> thm,
    81       mk_cong: Proof.context -> thm -> thm,
    82       mk_sym: Proof.context -> thm -> thm option,
    82       mk_sym: Proof.context -> thm -> thm option,
    83       mk_eq_True: Proof.context -> thm -> thm option,
    83       mk_eq_True: Proof.context -> thm -> thm option,
    84       reorient: Proof.context -> term list -> term -> term -> bool},
    84       reorient: Proof.context -> term list -> term -> term -> bool},
    85     term_ord: term * term -> order,
    85     term_ord: term ord,
    86     subgoal_tac: Proof.context -> int -> tactic,
    86     subgoal_tac: Proof.context -> int -> tactic,
    87     loop_tacs: (string * (Proof.context -> int -> tactic)) list,
    87     loop_tacs: (string * (Proof.context -> int -> tactic)) list,
    88     solvers: solver list * solver list}
    88     solvers: solver list * solver list}
    89   val map_ss: (Proof.context -> Proof.context) -> Context.generic -> Context.generic
    89   val map_ss: (Proof.context -> Proof.context) -> Context.generic -> Context.generic
    90   val prems_of: Proof.context -> thm list
    90   val prems_of: Proof.context -> thm list
    99   val mksimps: Proof.context -> thm -> thm list
    99   val mksimps: Proof.context -> thm -> thm list
   100   val set_mksimps: (Proof.context -> thm -> thm list) -> Proof.context -> Proof.context
   100   val set_mksimps: (Proof.context -> thm -> thm list) -> Proof.context -> Proof.context
   101   val set_mkcong: (Proof.context -> thm -> thm) -> Proof.context -> Proof.context
   101   val set_mkcong: (Proof.context -> thm -> thm) -> Proof.context -> Proof.context
   102   val set_mksym: (Proof.context -> thm -> thm option) -> Proof.context -> Proof.context
   102   val set_mksym: (Proof.context -> thm -> thm option) -> Proof.context -> Proof.context
   103   val set_mkeqTrue: (Proof.context -> thm -> thm option) -> Proof.context -> Proof.context
   103   val set_mkeqTrue: (Proof.context -> thm -> thm option) -> Proof.context -> Proof.context
   104   val set_term_ord: (term * term -> order) -> Proof.context -> Proof.context
   104   val set_term_ord: term ord -> Proof.context -> Proof.context
   105   val set_subgoaler: (Proof.context -> int -> tactic) -> Proof.context -> Proof.context
   105   val set_subgoaler: (Proof.context -> int -> tactic) -> Proof.context -> Proof.context
   106   val solver: Proof.context -> solver -> int -> tactic
   106   val solver: Proof.context -> solver -> int -> tactic
   107   val default_mk_sym: Proof.context -> thm -> thm option
   107   val default_mk_sym: Proof.context -> thm -> thm option
   108   val add_prems: thm list -> Proof.context -> Proof.context
   108   val add_prems: thm list -> Proof.context -> Proof.context
   109   val set_reorient: (Proof.context -> term list -> term -> term -> bool) ->
   109   val set_reorient: (Proof.context -> term list -> term -> term -> bool) ->
   266      {mk: Proof.context -> thm -> thm list,
   266      {mk: Proof.context -> thm -> thm list,
   267       mk_cong: Proof.context -> thm -> thm,
   267       mk_cong: Proof.context -> thm -> thm,
   268       mk_sym: Proof.context -> thm -> thm option,
   268       mk_sym: Proof.context -> thm -> thm option,
   269       mk_eq_True: Proof.context -> thm -> thm option,
   269       mk_eq_True: Proof.context -> thm -> thm option,
   270       reorient: Proof.context -> term list -> term -> term -> bool},
   270       reorient: Proof.context -> term list -> term -> term -> bool},
   271     term_ord: term * term -> order,
   271     term_ord: term ord,
   272     subgoal_tac: Proof.context -> int -> tactic,
   272     subgoal_tac: Proof.context -> int -> tactic,
   273     loop_tacs: (string * (Proof.context -> int -> tactic)) list,
   273     loop_tacs: (string * (Proof.context -> int -> tactic)) list,
   274     solvers: solver list * solver list};
   274     solvers: solver list * solver list};
   275 
   275 
   276 fun internal_ss (Simpset (_, ss2)) = ss2;
   276 fun internal_ss (Simpset (_, ss2)) = ss2;