Skip to content

Commit 257619f

Browse files
authored
2 parents e2b94c3 + e786457 commit 257619f

File tree

14 files changed

+47
-47
lines changed

14 files changed

+47
-47
lines changed

implementations/field_of_fractions.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -116,7 +116,7 @@ Proof.
116116
rewrite 2!mult_1_r.
117117
apply (is_ne_0 1).
118118
unfold dec_recip, Frac_dec_recip.
119-
case (decide_rel); simpl; intuition.
119+
case (decide_rel); simpl; intuition; auto with *.
120120
intros [xn xs] Ex.
121121
unfold dec_recip, Frac_dec_recip.
122122
simpl. case (decide_rel); simpl.

implementations/list.v

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -23,7 +23,7 @@ Section equivlistA_misc.
2323
Proof.
2424
split; intros E.
2525
inversion_clear E; auto. now destruct (proj1 (InA_nil eqA x)).
26-
rewrite E. intuition.
26+
rewrite E. intuition; auto with *.
2727
Qed.
2828

2929
Lemma equivlistA_cons_nil x l : ¬equivlistA eqA (x :: l) [].
@@ -81,8 +81,8 @@ Section equivlistA_misc.
8181
Global Instance: Equivalence PermutationA.
8282
Proof.
8383
split.
84-
intros l. induction l; intuition.
85-
intros l₁ l₂. induction 1; eauto. apply permA_skip; intuition.
84+
intros l. induction l; intuition; auto with *.
85+
intros l₁ l₂. induction 1; eauto. apply permA_skip; intuition; auto with *.
8686
intros ???. now apply permA_trans.
8787
Qed.
8888

@@ -92,7 +92,7 @@ Section equivlistA_misc.
9292

9393
Lemma PermutationA_app_head l₁ l₂ k :
9494
PermutationA l₁ l₂ → PermutationA (k ++ l₁) (k ++ l₂).
95-
Proof. intros. induction k. easy. apply permA_skip; intuition. Qed.
95+
Proof. intros. induction k. easy. apply permA_skip; intuition; auto with *. Qed.
9696

9797
Global Instance PermutationA_app :
9898
Proper (PermutationA ==> PermutationA ==> PermutationA) (@app A).
@@ -153,8 +153,8 @@ Section equivlistA_misc.
153153
intros. now rewrite equivlistA_nil_eq by now symmetry.
154154
intros l₂ Pl₂ E2.
155155
destruct (@InA_split _ eqA l₂ x) as [l₂h [y [l₂t [E3 ?]]]].
156-
rewrite <-E2. intuition.
157-
subst. transitivity (y :: l₁); [intuition |].
156+
rewrite <-E2. intuition; auto with *.
157+
subst. transitivity (y :: l₁); [intuition; auto with * |].
158158
apply PermutationA_cons_app, IHPl₁.
159159
now apply NoDupA_split with y.
160160
apply equivlistA_NoDupA_split with x y; intuition.

implementations/ne_list.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -95,10 +95,10 @@ Section contents.
9595
Definition Permutation (x y: L): Prop := ListPermutation x y.
9696

9797
Global Instance: Equivalence Permutation.
98-
Proof with intuition.
98+
Proof.
9999
unfold Permutation.
100-
split; repeat intro...
101-
transitivity y...
100+
split; repeat intro; auto with *.
101+
transitivity y; auto with *.
102102
Qed.
103103

104104
Global Instance: Proper (Permutation ==> ListPermutation) to_list.

implementations/polynomials.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -59,7 +59,7 @@ Section contents.
5959
Proof. now destruct p. Qed.
6060

6161
Instance: Reflexive poly_eq.
62-
Proof with intuition. repeat intro. induction x... split... Qed.
62+
Proof with intuition. repeat intro. induction x; auto with *. split; auto with *. Qed.
6363

6464
Lemma poly_eq_cons :
6565
∀ (a b : R) (p q : poly), (a = b /\ poly_eq p q) <-> poly_eq (a :: p) (b :: q).

orders/minmax.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -30,7 +30,7 @@ Section contents.
3030
Instance: LeftDistribute max min.
3131
Proof.
3232
intros x y z. unfold min, max, sort.
33-
repeat case (decide_rel _); simpl; try solve [intuition].
33+
repeat case (decide_rel _); simpl; try solve [intuition; auto with *].
3434
intros. apply (antisymmetry (≤)); [|easy]. now transitivity y; apply le_flip.
3535
intros. now apply (antisymmetry (≤)).
3636
Qed.

theory/ua_congruence.v

Lines changed: 11 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -38,17 +38,17 @@ Section contents.
3838
Let lifted_normal := @op_type_equiv (sorts σ) v ve.
3939

4040
Instance lifted_e_proper o: Proper ((=) ==> (=) ==> iff) (lifted_e o).
41-
Proof with intuition.
41+
Proof.
4242
induction o; simpl. intuition.
4343
repeat intro.
4444
unfold respectful.
4545
split; intros.
46-
assert (x x1 = y x1). apply H0...
47-
assert (x0 y1 = y0 y1). apply H1...
48-
apply (IHo (x x1) (y x1) H4 (x0 y1) (y0 y1) H5)...
49-
assert (x x1 = y x1). apply H0...
50-
assert (x0 y1 = y0 y1). apply H1...
51-
apply (IHo (x x1) (y x1) H4 (x0 y1) (y0 y1) H5)...
46+
assert (x x1 = y x1). apply H0; auto with *.
47+
assert (x0 y1 = y0 y1). apply H1; auto with *.
48+
apply (IHo (x x1) (y x1) H4 (x0 y1) (y0 y1) H5); auto with *.
49+
assert (x x1 = y x1). apply H0; auto with *.
50+
assert (x0 y1 = y0 y1). apply H1; auto with *.
51+
apply (IHo (x x1) (y x1) H4 (x0 y1) (y0 y1) H5); auto with *.
5252
Qed. (* todo: clean up *)
5353

5454
(* With that out of the way, we show that there are two equivalent ways of stating compatibility with the
@@ -85,8 +85,8 @@ Section contents.
8585
clearbody f.
8686
induction (σ o)...
8787
simpl in *...
88-
apply IHo0...
89-
apply H1...
88+
apply IHo0; intuition; auto with *.
89+
apply H1; auto with *.
9090
Qed. (* todo: clean up *)
9191

9292
Lemma eSub_eAlgebra: eSub → eAlgebra.
@@ -110,7 +110,7 @@ Section contents.
110110
simpl in *.
111111
repeat intro.
112112
unfold respectful in H0.
113-
apply (IHo0 (λ b, f b (if b then x else y)))...
113+
apply (IHo0 (λ b, f b (if b then x else y))); auto with *.
114114
Qed. (* todo: clean up *)
115115

116116
Lemma back_and_forth: iffT eSub eAlgebra.
@@ -231,7 +231,7 @@ Section first_iso.
231231
exists o1...
232232
destruct X.
233233
apply (@op_closed_proper σ B _ _ _ image image_proper _ (o1 z) (o1 (f _ x))).
234-
apply H3...
234+
apply H3; auto with *.
235235
apply IHo0 with (o2 x)...
236236
apply _.
237237
Qed.

theory/ua_products.v

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -198,18 +198,18 @@ Section categorical.
198198

199199
Global Program Instance: IntroProduct c (product c) := λ H h a X i, h i a X.
200200

201-
Next Obligation. Proof with intuition.
201+
Next Obligation. Proof.
202202
repeat constructor; try apply _.
203-
intros ?? E ?. destruct h. simpl. rewrite E...
203+
intros ?? E ?. destruct h. simpl. rewrite E; auto with *.
204204
intro o.
205205
pose proof (λ i, @preserves _ _ _ _ _ _ _ _ (proj2_sig (h i)) o) as H0.
206206
unfold product_ops, algebra_op.
207207
set (o0 := λ i, varieties.variety_ops et (c i) o).
208208
set (o1 := varieties.variety_ops et H o) in *.
209209
change (∀i : I, Preservation et H (c i) (` (h i)) o1 (o0 i)) in H0.
210210
clearbody o0 o1. revert o0 o1 H0.
211-
induction (et o); simpl...
212-
apply (@product_algebra et I c)...
211+
induction (et o); simpl; auto with *.
212+
apply (@product_algebra et I c); auto with *.
213213
Qed.
214214

215215
Global Instance: Product c (product c).

theory/ua_subalgebra.v

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -16,12 +16,12 @@ Section subalgebras.
1616
end.
1717

1818
Global Instance op_closed_proper: ∀ `{∀ s, Proper ((=) ==> iff) (P s)} o, Proper ((=) ==> iff) (@op_closed o).
19-
Proof with intuition.
19+
Proof.
2020
induction o; simpl; intros x y E.
21-
rewrite E...
21+
rewrite E; auto with *.
2222
split; intros.
23-
apply (IHo (x z))... apply E...
24-
apply (IHo _ (y z))... apply E...
23+
apply (IHo (x z)); auto with *. apply E; auto with *.
24+
apply (IHo _ (y z)); auto with *. apply E; auto with *.
2525
Qed.
2626

2727
Class ClosedSubset: Prop :=

theory/ua_subalgebraT.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -28,10 +28,10 @@ Section subalgebras.
2828
intuition.
2929
split; intros...
3030
apply (IHo (x z))...
31-
apply E...
32-
apply (IHo (y z))...
31+
apply E; auto with *.
32+
apply (IHo (y z)); auto with *.
3333
symmetry.
34-
apply E...
34+
apply E; auto with *.
3535
Qed.
3636

3737
Class ClosedSubset: Type :=

theory/ua_subvariety.v

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -33,23 +33,23 @@ Section contents.
3333
transitivity x0...
3434
transitivity x1...
3535
transitivity y0...
36-
assert (∀ u, x u = y u). intros. apply U...
36+
assert (∀ u, x u = y u). intros. apply U; auto with *.
3737
split; repeat intro.
3838
apply -> (IHo (x u) (y u) (H1 u) (x0 (proj1_sig u)))...
39-
apply K...
39+
apply K; auto with *.
4040
apply <- (IHo (x u) (y u) (H1 u) (x0 (proj1_sig u)))...
41-
apply K...
41+
apply K; auto with *.
4242
Qed.
4343

4444
Lemma heq_eval vars {o} (t: T et o): heq (eval et vars t) (eval et (Pvars vars) t).
4545
Proof with intuition.
4646
induction t; simpl...
47-
unfold Pvars...
47+
unfold Pvars; auto with *.
4848
simpl in IHt1.
4949
generalize (IHt1 (eval et vars t3)). clear IHt1.
5050
apply heq_proper.
5151
pose proof (@eval_proper et (carrier P) _ _ _ nat (ne_list.cons y t1)).
52-
apply H1; try intro...
52+
apply H1; try intro; auto with *.
5353
pose proof (@eval_proper et A _ _ _ nat (ne_list.cons y t1)).
5454
apply H1...
5555
unfold heq in IHt2. (* todo: this wasn't needed in a previous Coq version *)

0 commit comments

Comments
 (0)