summaryrefslogtreecommitdiff
path: root/test-suite/interactive/Back.v
blob: 22364254dc0fa7a44cd0f835bef3e0b9b07b66f1 (plain)
1
2
3
4
5
6
7
8
(* Check that reset remains synchronised with the compilation unit cache *)
(* See BZ#1030 *)

Section multiset_defs.
  Require Import Plus.
End multiset_defs.
Unset Implicit Arguments.
Back 1.