From 5eda8fb59597c7a39335d2eb99f44cd07b25433d Mon Sep 17 00:00:00 2001 From: Julien Forest Date: Thu, 21 Nov 2013 09:46:40 +0100 Subject: Add Acc_intro_generator on top of all wf function proof (much much faster execution) --- plugins/funind/Recdef.v | 2 ++ 1 file changed, 2 insertions(+) (limited to 'plugins/funind/Recdef.v') 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 -- cgit v1.2.3