Skip to content

Commit

Permalink
rollback pclearbot tactic to 74b6b1c
Browse files Browse the repository at this point in the history
  • Loading branch information
minkiminki committed Feb 7, 2019
1 parent a254ff3 commit f772ccf
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 12 deletions.
8 changes: 2 additions & 6 deletions metasrc/pacotacuser.v
Original file line number Diff line number Diff line change
Expand Up @@ -79,14 +79,11 @@ Tactic Notation "pcofix" ident(CIH) := pcofix CIH with r.
(** ** [pclearbot] simplifies all hypotheses of the form [upaco{n} gf bot{n}] to [paco{n} gf bot{n}].
*)

Lemma paco_clear_bot: forall P:Prop, P \/ False <-> P.
Proof. tauto. Qed.

Ltac pclearbot :=
let X := fresh "_X" in
repeat match goal with
| [H: context[pacoid] |- _] => try red in H; setoid_rewrite paco_clear_bot in H
end.
| [H: context[pacoid] |- _] => red in H; destruct H as [H|X]; [|contradiction X]
end.

(** ** [pdestruct H] and [pinversion H]
*)
Expand All @@ -101,4 +98,3 @@ Ltac pinversion H := punfold H; inversion H; pclearbot.

Ltac pmonauto :=
let IN := fresh "IN" in try (repeat intro; destruct IN; eauto; fail).

8 changes: 2 additions & 6 deletions src/pacotacuser.v
Original file line number Diff line number Diff line change
Expand Up @@ -79,14 +79,11 @@ Tactic Notation "pcofix" ident(CIH) := pcofix CIH with r.
(** ** [pclearbot] simplifies all hypotheses of the form [upaco{n} gf bot{n}] to [paco{n} gf bot{n}].
*)

Lemma paco_clear_bot: forall P:Prop, P \/ False <-> P.
Proof. tauto. Qed.

Ltac pclearbot :=
let X := fresh "_X" in
repeat match goal with
| [H: context[pacoid] |- _] => try red in H; setoid_rewrite paco_clear_bot in H
end.
| [H: context[pacoid] |- _] => red in H; destruct H as [H|X]; [|contradiction X]
end.

(** ** [pdestruct H] and [pinversion H]
*)
Expand All @@ -101,4 +98,3 @@ Ltac pinversion H := punfold H; inversion H; pclearbot.

Ltac pmonauto :=
let IN := fresh "IN" in try (repeat intro; destruct IN; eauto; fail).

0 comments on commit f772ccf

Please sign in to comment.