aboutsummaryrefslogtreecommitdiff
path: root/ci/compile-tests/007-slow-require/a2.v.orig
blob: 60ac1279ceab2dbd407dfc485c7da9bec73f3881 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
(* This file is part of Proof General.
 *
 * © Copyright 2021  Hendrik Tews
 *
 * Authors: Hendrik Tews
 * Maintainer: Hendrik Tews <hendrik@askra.de>
 *
 * License:     GPL (GNU GENERAL PUBLIC LICENSE)
 *
 *
 * This file is part of an automatic test case for parallel background
 * compilation in coq-par-compile.el. See test.el in this directory.
 *)

(* The test script relies on absolute line numbers. 
 * DO NOT INSERT ANY LINE UNLESS YOU KNOW WHAT YOU ARE DOING.
 *)

(* The delay for coqdep is specified in comments with key coqdep-delay,
 * see compile-test-start-delayed.
 *)


(* This is line 24 *)
Require Export b2.
Require Export c2.
(* This is line 27 *)


(* This is line 30 *)
Definition sum : nat := 9.


(* This is line 34 *)
Lemma x : b + c + d = sum.
Proof using.
  unfold b, c, d, sum in *.
  simpl.
  trivial.
Qed.
(* This is line 41 *)