aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Program
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-11-07 22:48:15 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-12-05 09:34:02 +0100
commitcaeba655b78a0107c1988e5377cdd11fa91c5ea2 (patch)
treeee6860df02174ae3836a18c331858a655f2bfc12 /theories/Program
parent2e3ee15b03cf4b7428e1a7453385d79f434ec4a7 (diff)
Experimenting removing strong normalization of the mid-statement in tactic cut.
Diffstat (limited to 'theories/Program')
-rw-r--r--theories/Program/Wf.v2
1 files changed, 1 insertions, 1 deletions
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)).