aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--plugins/funind/Recdef.v2
-rw-r--r--plugins/funind/recdef.ml3
2 files changed, 4 insertions, 1 deletions
diff --git a/plugins/funind/Recdef.v b/plugins/funind/Recdef.v
index b2955e902..e28c845cc 100644
--- a/plugins/funind/Recdef.v
+++ b/plugins/funind/Recdef.v
@@ -46,3 +46,5 @@ intros m n; case (Compare_dec.le_gt_dec m n).
intros h; exists n; [exact h | apply le_n].
intros h; exists m; [apply le_n | apply Lt.lt_le_weak; exact h].
Defined.
+
+Definition Acc_intro_generator_function := fun A R => @Acc_intro_generator A R 100. \ No newline at end of file
diff --git a/plugins/funind/recdef.ml b/plugins/funind/recdef.ml
index 64bf71ec6..68ac62838 100644
--- a/plugins/funind/recdef.ml
+++ b/plugins/funind/recdef.ml
@@ -139,6 +139,7 @@ let iter_ref () =
let iter = function () -> (constr_of_global (delayed_force iter_ref))
let eq = function () -> (coq_base_constant "eq")
let le_lt_SS = function () -> (constant ["Recdef"] "le_lt_SS")
+let acc_intro_generator_function = function () -> (constant ["Recdef"] "Acc_intro_generator_function")
let le_lt_n_Sm = function () -> (coq_base_constant "le_lt_n_Sm")
let le_trans = function () -> (coq_base_constant "le_trans")
let le_lt_trans = function () -> (coq_base_constant "le_lt_trans")
@@ -276,7 +277,7 @@ let tclUSER tac is_mes l g =
let tclUSER_if_not_mes concl_tac is_mes names_to_suppress =
if is_mes
then tclCOMPLETE (h_simplest_apply (delayed_force well_founded_ltof))
- else tclUSER concl_tac is_mes names_to_suppress
+ else tclTHEN (h_simplest_apply (delayed_force acc_intro_generator_function) ) (tclUSER concl_tac is_mes names_to_suppress)