summaryrefslogtreecommitdiff
path: root/tests/coq/demo
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--tests/coq/demo/Demo.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/tests/coq/demo/Demo.v b/tests/coq/demo/Demo.v
index 22a0a131..ec7ca29d 100644
--- a/tests/coq/demo/Demo.v
+++ b/tests/coq/demo/Demo.v
@@ -160,8 +160,8 @@ Definition CounterUsize : Counter_t usize := {|
(** [demo::use_counter]:
Source: 'src/demo.rs', lines 95:0-95:59 *)
Definition use_counter
- (T : Type) (counterTInst : Counter_t T) (cnt : T) : result (usize * T) :=
- counterTInst.(Counter_t_incr) cnt
+ (T : Type) (counterInst : Counter_t T) (cnt : T) : result (usize * T) :=
+ counterInst.(Counter_t_incr) cnt
.
End Demo.