aboutsummaryrefslogtreecommitdiffstats
path: root/examples/Example.v
diff options
context:
space:
mode:
authorChantal Keller <Chantal.Keller@lri.fr>2020-07-06 12:40:48 +0200
committerChantal Keller <Chantal.Keller@lri.fr>2020-07-06 12:40:48 +0200
commit52621f58edcabc36e7d1cd10d9b4da8be1a08649 (patch)
treede5831e7b1b0fb79fe459a819bbe2590e14a1682 /examples/Example.v
parentea73755e6e1b7efea8db79b9fc0cf456ed5c640f (diff)
parentd7a33ad9b479317701eba7c787744599de134f78 (diff)
downloadsmtcoq-52621f58edcabc36e7d1cd10d9b4da8be1a08649.tar.gz
smtcoq-52621f58edcabc36e7d1cd10d9b4da8be1a08649.zip
Merge branch 'coq-8.10' of github.com:smtcoq/smtcoq into coq-8.10
Diffstat (limited to 'examples/Example.v')
-rw-r--r--examples/Example.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/examples/Example.v b/examples/Example.v
index 2d48776..7beed4a 100644
--- a/examples/Example.v
+++ b/examples/Example.v
@@ -11,7 +11,7 @@
(* [Require Import SMTCoq.SMTCoq.] loads the SMTCoq library.
- If you are using native-coq instead of Coq 8.9, replace it with:
+ If you are using native-coq instead of Coq 8.10, replace it with:
Require Import SMTCoq.
*)