From caeba655b78a0107c1988e5377cdd11fa91c5ea2 Mon Sep 17 00:00:00 2001 From: Hugo Herbelin Date: Sat, 7 Nov 2015 22:48:15 +0100 Subject: Experimenting removing strong normalization of the mid-statement in tactic cut. --- theories/Program/Wf.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Program') diff --git a/theories/Program/Wf.v b/theories/Program/Wf.v index d89919b0a..6e5919b34 100644 --- a/theories/Program/Wf.v +++ b/theories/Program/Wf.v @@ -89,7 +89,7 @@ Section Measure_well_founded. Lemma measure_wf: well_founded MR. Proof with auto. unfold well_founded. - cut (forall a: M, (fun mm: M => forall a0: T, m a0 = mm -> Acc MR a0) a). + cut (forall (a: M) (a0: T), m a0 = a -> Acc MR a0). intros. apply (H (m a))... apply (@well_founded_ind M R wf (fun mm => forall a, m a = mm -> Acc MR a)). -- cgit v1.2.3