aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Program
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-26 16:42:56 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-26 16:42:56 +0000
commit9a9aada110be18fc88a7559b9dce05d66edf156a (patch)
tree11355778b8b2abb44f6331160c9e33f6bde064e9 /theories/Program
parent99826cb11dc8478b1c9bf7c0f7116e621e8618cb (diff)
Add [Next Obligation with tactic] support (wish #1953).
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12691 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Program')
-rw-r--r--theories/Program/Tactics.v7
1 files changed, 6 insertions, 1 deletions
diff --git a/theories/Program/Tactics.v b/theories/Program/Tactics.v
index b3b08e067..75aa5eb7c 100644
--- a/theories/Program/Tactics.v
+++ b/theories/Program/Tactics.v
@@ -308,6 +308,11 @@ Ltac program_simplify :=
subst*; autoinjections ; try discriminates ;
try (solve [ red ; intros ; destruct_conjs ; autoinjections ; discriminates ]).
-Ltac program_simpl := program_simplify ; auto.
+Ltac program_solve_wf :=
+ match goal with
+ |- well_founded _ => auto with *
+ end.
+
+Ltac program_simpl := program_simplify ; auto; try program_solve_wf.
Obligation Tactic := program_simpl.