mk_core m e as_simp, m is used to decide which definitions will be unfolded in patterns.
  If as_simp is tt, then this tactic will try to use the left-hand-side of the conclusion
  as a pattern.
    
def
to_hinst_lemmas_core
    (m : tactic.transparency)
    (a : bool)
    (a_1 : list name)
    (a_2 : hinst_lemmas) :
    
def
merge_hinst_lemma_attrs
    (m : tactic.transparency)
    (as_simp : bool)
    (a : list name)
    (a_1 : hinst_lemmas) :
Create a new "cached" attribute (attr_name : user_attribute hinst_lemmas). It also creates "cached" attributes for each attr_names and simp_attr_names if they have not been defined yet. Moreover, the hinst_lemmas for attr_name will be the union of the lemmas tagged with attr_name, attrs_name, and simp_attr_names. For the ones in simp_attr_names, we use the left-hand-side of the conclusion as the pattern.
    
constant
tactic.ematch_core
    (a : tactic.transparency)
    (a_1 : cc_state)
    (a_2 : ematch_state)
    (a_3 : hinst_lemma)
    (a_4 : expr) :
    
constant
tactic.ematch_all_core
    (a : tactic.transparency)
    (a_1 : cc_state)
    (a_2 : ematch_state)
    (a_3 : hinst_lemma)
    (a_4 : bool) :