Skip to content

Commit 53ecd2e

Browse files
authored
improved auto goal selection (see coq/#16293) (#39)
1 parent 97071c5 commit 53ecd2e

File tree

4 files changed

+10
-10
lines changed

4 files changed

+10
-10
lines changed

src/FCF/Fold.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -3216,7 +3216,7 @@ Lemma firstn_ge_all : forall n (A : Set) (ls : list A),
32163216
n >= length ls ->
32173217
firstn n ls = ls.
32183218

3219-
induction n; intuition; simpl in *.
3219+
induction n; intuition idtac; simpl in *.
32203220
destruct ls; simpl in *.
32213221
trivial.
32223222
lia.
@@ -3904,7 +3904,7 @@ Theorem app_cons_eq :
39043904
forall (A : Type) ls2 ls1 (a : A),
39053905
ls2 ++ (a :: ls1) = (ls2 ++ (a :: nil)) ++ ls1.
39063906

3907-
induction ls2; intuition; simpl in *.
3907+
induction ls2; intuition idtac; simpl in *.
39083908
f_equal.
39093909
eauto.
39103910

src/FCF/OracleHybrid.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -559,7 +559,7 @@ Section OracleMapHybrid.
559559
rewrite firstn_skipn.
560560
fcf_skip.
561561
eapply (compFold_spec' (fun a b c d => a = b /\ snd c = snd d /\ l0++ (fst d) = (fst c)));
562-
intuition.
562+
intuition idtac.
563563
simpl.
564564
eapply app_nil_r.
565565
simpl in *.

src/FCF/ProgramLogic.v

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -273,7 +273,7 @@ Theorem comp_spec_seq :
273273
rewrite ratMult_1_r.
274274
eapply ratMult_eqRat_compat; intuition.
275275
specialize (H2 a).
276-
intuition.
276+
intuition idtac.
277277
rewrite H2.
278278

279279
unfold marginal_l.
@@ -320,7 +320,7 @@ Theorem comp_spec_seq :
320320
rewrite H5.
321321
rewrite ratMult_1_r.
322322
eapply ratMult_eqRat_compat; intuition.
323-
specialize (H2 a); intuition.
323+
specialize (H2 a); intuition idtac.
324324
rewrite H6.
325325
unfold marginal_r; intuition.
326326

@@ -1719,13 +1719,13 @@ Theorem comp_spec_irr_r :
17191719
unfold marginal_l.
17201720
dist_inline_first.
17211721
dist_irr_r.
1722-
specialize (H0 x0); intuition.
1722+
specialize (H0 x0); intuition idtac.
17231723
eapply H0.
17241724

17251725
unfold marginal_r.
17261726
dist_inline_first.
17271727
dist_skip.
1728-
specialize (H0 x0); intuition.
1728+
specialize (H0 x0); intuition idtac.
17291729
apply H2.
17301730
repeat simp_in_support.
17311731
specialize (H0 x0); intuition.
@@ -1748,13 +1748,13 @@ Theorem comp_spec_irr_l :
17481748
unfold marginal_l.
17491749
dist_inline_first.
17501750
dist_skip.
1751-
specialize (H0 x0); intuition.
1751+
specialize (H0 x0); intuition idtac.
17521752
eapply H0.
17531753

17541754
unfold marginal_r.
17551755
dist_inline_first.
17561756
dist_irr_r.
1757-
specialize (H0 x0); intuition.
1757+
specialize (H0 x0); intuition idtac.
17581758
apply H2.
17591759
repeat simp_in_support.
17601760
specialize (H0 x0); intuition.

src/FCF/RndNat.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -32,7 +32,7 @@ Lemma well_formed_RndNat : forall n,
3232
unfold RndNat.
3333
eapply (well_formed_Repeat).
3434
unfold eq_dec.
35-
intuition.
35+
intuition idtac.
3636
eapply eq_nat_dec.
3737
unfold RndNat_unchecked.
3838
eapply well_formed_Bind.

0 commit comments

Comments
 (0)