aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-12-22 16:26:24 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2018-06-04 11:17:34 +0200
commit0daae2bd1ab518d8fcb6d59a5616786ade94d1e5 (patch)
tree7b3b9845e42cc1b9632e6136f867f52921dce4be /theories
parent01128a2ff774f0ef249ee54a67e88d49ae254a4d (diff)
Deprecate implicit tactic solving.
Diffstat (limited to 'theories')
-rw-r--r--theories/Logic/Diaconescu.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/theories/Logic/Diaconescu.v b/theories/Logic/Diaconescu.v
index 3317766c9..66e82ddbf 100644
--- a/theories/Logic/Diaconescu.v
+++ b/theories/Logic/Diaconescu.v
@@ -234,8 +234,6 @@ Qed.
(** An alternative more concise proof can be done by directly using
the guarded relational choice *)
-Declare Implicit Tactic auto.
-
Lemma proof_irrel_rel_choice_imp_eq_dec' : a1=a2 \/ ~a1=a2.
Proof.
assert (decide: forall x:A, x=a1 \/ x=a2 ->