File tree Expand file tree Collapse file tree 4 files changed +10
-10
lines changed Expand file tree Collapse file tree 4 files changed +10
-10
lines changed Original file line number Diff line number Diff line change @@ -3216,7 +3216,7 @@ Lemma firstn_ge_all : forall n (A : Set) (ls : list A),
3216
3216
n >= length ls ->
3217
3217
firstn n ls = ls.
3218
3218
3219
- induction n; intuition; simpl in *.
3219
+ induction n; intuition idtac ; simpl in *.
3220
3220
destruct ls; simpl in *.
3221
3221
trivial.
3222
3222
lia.
@@ -3904,7 +3904,7 @@ Theorem app_cons_eq :
3904
3904
forall (A : Type) ls2 ls1 (a : A),
3905
3905
ls2 ++ (a :: ls1) = (ls2 ++ (a :: nil)) ++ ls1.
3906
3906
3907
- induction ls2; intuition; simpl in *.
3907
+ induction ls2; intuition idtac ; simpl in *.
3908
3908
f_equal.
3909
3909
eauto .
3910
3910
Original file line number Diff line number Diff line change @@ -559,7 +559,7 @@ Section OracleMapHybrid.
559
559
rewrite firstn_skipn.
560
560
fcf_skip.
561
561
eapply (compFold_spec' (fun a b c d => a = b /\ snd c = snd d /\ l0++ (fst d) = (fst c)));
562
- intuition.
562
+ intuition idtac .
563
563
simpl.
564
564
eapply app_nil_r.
565
565
simpl in *.
Original file line number Diff line number Diff line change @@ -273,7 +273,7 @@ Theorem comp_spec_seq :
273
273
rewrite ratMult_1_r.
274
274
eapply ratMult_eqRat_compat; intuition.
275
275
specialize (H2 a).
276
- intuition.
276
+ intuition idtac .
277
277
rewrite H2.
278
278
279
279
unfold marginal_l.
@@ -320,7 +320,7 @@ Theorem comp_spec_seq :
320
320
rewrite H5.
321
321
rewrite ratMult_1_r.
322
322
eapply ratMult_eqRat_compat; intuition.
323
- specialize (H2 a); intuition.
323
+ specialize (H2 a); intuition idtac .
324
324
rewrite H6.
325
325
unfold marginal_r; intuition.
326
326
@@ -1719,13 +1719,13 @@ Theorem comp_spec_irr_r :
1719
1719
unfold marginal_l.
1720
1720
dist_inline_first.
1721
1721
dist_irr_r.
1722
- specialize (H0 x0); intuition.
1722
+ specialize (H0 x0); intuition idtac .
1723
1723
eapply H0.
1724
1724
1725
1725
unfold marginal_r.
1726
1726
dist_inline_first.
1727
1727
dist_skip.
1728
- specialize (H0 x0); intuition.
1728
+ specialize (H0 x0); intuition idtac .
1729
1729
apply H2.
1730
1730
repeat simp_in_support.
1731
1731
specialize (H0 x0); intuition.
@@ -1748,13 +1748,13 @@ Theorem comp_spec_irr_l :
1748
1748
unfold marginal_l.
1749
1749
dist_inline_first.
1750
1750
dist_skip.
1751
- specialize (H0 x0); intuition.
1751
+ specialize (H0 x0); intuition idtac .
1752
1752
eapply H0.
1753
1753
1754
1754
unfold marginal_r.
1755
1755
dist_inline_first.
1756
1756
dist_irr_r.
1757
- specialize (H0 x0); intuition.
1757
+ specialize (H0 x0); intuition idtac .
1758
1758
apply H2.
1759
1759
repeat simp_in_support.
1760
1760
specialize (H0 x0); intuition.
Original file line number Diff line number Diff line change @@ -32,7 +32,7 @@ Lemma well_formed_RndNat : forall n,
32
32
unfold RndNat.
33
33
eapply (well_formed_Repeat).
34
34
unfold eq_dec.
35
- intuition.
35
+ intuition idtac .
36
36
eapply eq_nat_dec.
37
37
unfold RndNat_unchecked.
38
38
eapply well_formed_Bind.
You can’t perform that action at this time.
0 commit comments