This file is indexed.

/usr/lib/coq/user-contrib/AAC_tactics/print.mli is in libaac-tactics-ocaml-dev 8.6.1-1.

This file is owned by root:root, with mode 0o644.

The actual contents of the file can be viewed below.

 1
 2
 3
 4
 5
 6
 7
 8
 9
10
11
12
13
14
15
16
17
18
19
20
21
22
(***************************************************************************)
(*  This is part of aac_tactics, it is distributed under the terms of the  *)
(*         GNU Lesser General Public License version 3                     *)
(*              (see file LICENSE for more details)                        *)
(*                                                                         *)
(*       Copyright 2009-2010: Thomas Braibant, Damien Pous.                *)
(***************************************************************************)

(** Pretty printing functions we use for the aac_instances
    tactic. *)


(** The main printing function. {!print} uses the rel-context
    to rename the variables, and rebuilds raw Coq terms (for the given
    context, and the terms in the environment). In order to do so, it
    requires the information gathered by the {!Theory.Trans} module.*)
val print :
  Coq.Relation.t ->
  Theory.Trans.ir ->
  (int * Matcher.Terms.t * Matcher.Subst.t Search_monad.m) Search_monad.m ->
  Context.Rel.t  ->
  Proof_type.tactic