diff options
Diffstat (limited to 'mathcomp/ssrtest/set_pattern.v')
| -rw-r--r-- | mathcomp/ssrtest/set_pattern.v | 2 |
1 files changed, 2 insertions, 0 deletions
diff --git a/mathcomp/ssrtest/set_pattern.v b/mathcomp/ssrtest/set_pattern.v index 50dc262..86de57c 100644 --- a/mathcomp/ssrtest/set_pattern.v +++ b/mathcomp/ssrtest/set_pattern.v @@ -1,3 +1,5 @@ +(* (c) Copyright 2006-2015 Microsoft Corporation and Inria. *) +(* Distributed under the terms of CeCILL-B. *) Require Import mathcomp.ssreflect.ssreflect. Axiom daemon : False. Ltac myadmit := case: daemon. |
