diff options
Diffstat (limited to 'test-suite/complexity/ring2.v')
| -rw-r--r-- | test-suite/complexity/ring2.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/complexity/ring2.v b/test-suite/complexity/ring2.v index af678a2e1f..ab57afdbba 100644 --- a/test-suite/complexity/ring2.v +++ b/test-suite/complexity/ring2.v @@ -1,4 +1,4 @@ -(* This example, checks the efficiency of the abstract machine used by ring *) +(* This example checks the efficiency of the abstract machine used by ring *) (* Expected time < 1.00s *) Require Import BinInt Zbool. |
