From c22a1828063756fdc11876993e6f1e2ca3bba04d Mon Sep 17 00:00:00 2001 From: Cyril SIX Date: Mon, 4 May 2020 16:35:45 +0200 Subject: Adding copyrights --- backend/ProfilingExploit.v | 12 ++++++++++++ 1 file changed, 12 insertions(+) (limited to 'backend/ProfilingExploit.v') diff --git a/backend/ProfilingExploit.v b/backend/ProfilingExploit.v index cfca1a12..2325f582 100644 --- a/backend/ProfilingExploit.v +++ b/backend/ProfilingExploit.v @@ -1,3 +1,15 @@ +(* *************************************************************) +(* *) +(* The Compcert verified compiler *) +(* *) +(* David Monniaux CNRS, VERIMAG *) +(* *) +(* Copyright VERIMAG. All rights reserved. *) +(* This file is distributed under the terms of the INRIA *) +(* Non-Commercial License Agreement. *) +(* *) +(* *************************************************************) + Require Import Coqlib Maps Errors Integers Floats Lattice Kildall. Require Import AST Linking. Require Import Memory Registers Op RTL. -- cgit