Library hydras.Prelude.MoreLibHyps

From LibHyps Require Import LibHyps.

Tactic Notation (at level 4) tactic4(Tac) "/" "dr" :=
  Tac ; {< fun htry generalize dependent h }.

Tactic Notation (at level 4) tactic4(Tac) "/" "r?" :=
  Tac ; {< fun htry revert h }.

From Coq Require Import List.
Import ListNotations.
#[local] Open Scope autonaming_scope.


Ltac old_rename := rename_hyp_default.

Ltac rename_short n th :=
  match th with
  | (?f ?x ?y) ⇒ name ((f # 1) ++ (x # 1))
  | (?f ?x) ⇒ name ((f # 1))
  | _old_rename n th
  end.